diff --git a/.github/workflows/nix-ci.yml b/.github/workflows/nix-ci.yml index 17b0c8c0b773..fdd0ecab6bb2 100644 --- a/.github/workflows/nix-ci.yml +++ b/.github/workflows/nix-ci.yml @@ -78,8 +78,7 @@ jobs: - name: Build run: | # .o files are not a runtime dependency on macOS because of lack of thin archives - # leanc_src is required for building Leanc-deps - nix build $NIX_BUILD_ARGS .#stage0 .#stage1.lean-all .#lean-bin-tools-unwrapped.leanc_src .#Lean.oTree .#iTree .#modDepsFiles -o push-build + nix build $NIX_BUILD_ARGS .#stage0 .#stage1.lean-all .#Lean.oTree .#iTree .#modDepsFiles -o push-build - name: Test run: | nix build $NIX_BUILD_ARGS .#test -o push-test diff --git a/doc/declarations.md b/doc/declarations.md index d117161a841d..5306bcbbb70f 100644 --- a/doc/declarations.md +++ b/doc/declarations.md @@ -74,7 +74,7 @@ Lean provides ways of adding new objects to the environment. The following provi * ``axiom c : α`` : declare a constant named ``c`` of type ``α``, it is postulating that `α` is not an empty type. * ``def c : α := v`` : defines ``c`` to denote ``v``, which should have type ``α``. * ``theorem c : p := v`` : similar to ``def``, but intended to be used when ``p`` is a proposition. -* ``constant c : α (:= v)?`` : declares a opaque constant named ``c`` of type ``α``, the optional value `v` is must have type `α` +* ``opaque c : α (:= v)?`` : declares a opaque constant named ``c`` of type ``α``, the optional value `v` is must have type `α` and can be viewed as a certificate that ``α`` is not an empty type. If the value is not provided, Lean tries to find one using a proceture based on type class resolution. The value `v` is hidden from the type checker. You can assume that Lean "forgets" `v` after type checking this kind of declaration. @@ -89,8 +89,8 @@ Any of ``def``, ``theorem``, ``axiom``, or ``example`` can take a list of argume is interpreted as ``def foo : (a : α) → β := fun a : α => t``. Similarly, a theorem ``theorem foo (a : α) : p := t`` is interpreted as ``theorem foo : ∀ a : α, p := fun a : α => t``. ```lean -constant c : Nat -constant d : Nat +opaque c : Nat +opaque d : Nat axiom cd_eq : c = d def foo : Nat := 5 diff --git a/doc/dev/ffi.md b/doc/dev/ffi.md index f04d0cab2419..0b55f5c4b2dd 100644 --- a/doc/dev/ffi.md +++ b/doc/dev/ffi.md @@ -43,6 +43,7 @@ In the case of `@[extern]` all *irrelevant* types are removed first; see next se * it is none of the types described above * it is not marked `unsafe` * it has a single constructor with a single parameter of *relevant* type + is represented by the representation of that parameter's type. For example, `{ x : α // p }`, the `Subtype` structure of a value of type `α` and an irrelevant proof, is represented by the representation of `α`. diff --git a/doc/examples/ICERM2022/ctor.lean b/doc/examples/ICERM2022/ctor.lean new file mode 100644 index 000000000000..fa7fdd8b8df3 --- /dev/null +++ b/doc/examples/ICERM2022/ctor.lean @@ -0,0 +1,46 @@ +import Lean + +open Lean Meta + +def ctor (mvarId : MVarId) (idx : Nat) : MetaM (List MVarId) := do + /- Set `MetaM` context using `mvarId` -/ + withMVarContext mvarId do + /- Fail if the metavariable is already assigned. -/ + checkNotAssigned mvarId `ctor + /- Retrieve the target type, instantiateMVars, and use `whnf`. -/ + let target ← getMVarType' mvarId + let .const declName us := target.getAppFn + | throwTacticEx `ctor mvarId "target is not an inductive datatype" + let .inductInfo { ctors, .. } ← getConstInfo declName + | throwTacticEx `ctor mvarId "target is not an inductive datatype" + if idx = 0 then + throwTacticEx `ctor mvarId "invalid index, it must be > 0" + else if h : idx - 1 < ctors.length then + apply mvarId (.const ctors[idx - 1] us) + else + throwTacticEx `ctor mvarId "invalid index, inductive datatype has only {ctors.length} contructors" + +open Elab Tactic + +elab "ctor" idx:num : tactic => + liftMetaTactic (ctor · idx.getNat) + +example (p : Prop) : p := by + ctor 1 -- Error + +example (h : q) : p ∨ q := by + ctor 0 -- Error + exact h + +example (h : q) : p ∨ q := by + ctor 3 -- Error + exact h + +example (h : q) : p ∨ q := by + ctor 2 + exact h + +example (h : q) : p ∨ q := by + ctor 1 + exact h -- Error + diff --git a/doc/examples/ICERM2022/meta.lean b/doc/examples/ICERM2022/meta.lean new file mode 100644 index 000000000000..b7082614fac3 --- /dev/null +++ b/doc/examples/ICERM2022/meta.lean @@ -0,0 +1,80 @@ +import Lean + +open Lean Meta + +def ex1 (declName : Name) : MetaM Unit := do + let info ← getConstInfo declName + IO.println s!"{declName} : {← ppExpr info.type}" + if let some val := info.value? then + IO.println s!"{declName} : {← ppExpr val}" + +#eval ex1 ``Nat + +def ex2 (declName : Name) : MetaM Unit := do + let info ← getConstInfo declName + trace[Meta.debug] "{declName} : {info.type}" + if let some val := info.value? then + trace[Meta.debug] "{declName} : {val}" + +#eval ex2 ``Add.add + +set_option trace.Meta.debug true in +#eval ex2 ``Add.add + +def ex3 (declName : Name) : MetaM Unit := do + let info ← getConstInfo declName + forallTelescope info.type fun xs type => do + trace[Meta.debug] "hypotheses : {xs}" + trace[Meta.debug] "resultType : {type}" + for x in xs do + trace[Meta.debug] "{x} : {← inferType x}" + +def myMin [LT α] [DecidableRel (α := α) (·<·)] (a b : α) : α := + if a < b then + a + else + b + +set_option trace.Meta.debug true in +#eval ex3 ``myMin + +def ex4 : MetaM Unit := do + let nat := mkConst ``Nat + withLocalDeclD `a nat fun a => + withLocalDeclD `b nat fun b => do + let e ← mkAppM ``HAdd.hAdd #[a, b] + trace[Meta.debug] "{e} : {← inferType e}" + let e ← mkAdd a (mkNatLit 5) + trace[Meta.debug] "added 5: {e}" + let e ← whnf e + trace[Meta.debug] "whnf: {e}" + let e ← reduce e + trace[Meta.debug] "reduced: {e}" + let a_plus_1 ← mkAdd a (mkNatLit 1) + let succ_a := mkApp (mkConst ``Nat.succ) a + trace[Meta.debug] "({a_plus_1} =?= {succ_a}) == {← isDefEq a_plus_1 succ_a}" + let m ← mkFreshExprMVar nat + let m_plus_1 ← mkAdd m (mkNatLit 1) + trace[Meta.debug] "m_plus_1: {m_plus_1}" + unless (← isDefEq m_plus_1 succ_a) do throwError "isDefEq failed" + trace[Meta.debug] "m_plus_1: {m_plus_1}" + +set_option trace.Meta.debug true in +#eval ex4 + +open Elab Term + +def ex5 : TermElabM Unit := do + let nat := Lean.mkConst ``Nat + withLocalDeclD `a nat fun a => do + withLocalDeclD `b nat fun b => do + let ab ← mkAppM ``HAdd.hAdd #[a, b] + let stx ← `(fun x => if x < 10 then $(← exprToSyntax ab) + x else x + $(← exprToSyntax a)) + let e ← elabTerm stx none + trace[Meta.debug] "{e} : {← inferType e}" + let e := mkApp e (mkNatLit 5) + let e ← whnf e + trace[Meta.debug] "{e}" + +set_option trace.Meta.debug true in +#eval ex5 diff --git a/doc/examples/ICERM2022/notation.lean b/doc/examples/ICERM2022/notation.lean new file mode 100644 index 000000000000..a8b9562d8b0c --- /dev/null +++ b/doc/examples/ICERM2022/notation.lean @@ -0,0 +1,49 @@ +import Lean + +def f (x y : Nat) := x * y + 1 + +infixl:65 " *' " => f + +#check 2 *' 3 + +notation "unitTest " x => Prod.mk x () + +#check unitTest 42 + +notation "parenthesisTest " x => Nat.sub (x) +#check parenthesisTest 12 + +def Set (α : Type u) := α → Prop +def setOf {α : Type} (p : α → Prop) : Set α := p +notation "{ " x " | " p " }" => setOf (fun x => p) + +#check { x | x ≤ 1 } + +notation "cdotTest " "(" x ", " y ")" => Prod.map (· + 1) (1 + ·) (x, y) + +#check cdotTest (13, 12) + +notation "tupleFunctionTest " "(" x ", " y ")"=> Prod.map (Nat.add 1) (Nat.add 2) (x, y) + +#check tupleFunctionTest (15, 12) + +notation "diag " x => Prod.mk x x + +#check diag 12 + +open Lean Meta PrettyPrinter Delaborator SubExpr in +@[delab app.Prod.mk] def delabDoubleRhsTest : Delab := do + let e ← getExpr + let #[_, _, x, y] := e.getAppArgs | failure + guard (← isDefEq x y) + let stx ← withAppArg delab + `(diag $stx) + +#check diag 3 +#check (3, 3) +#check (3, 4) +#check (2+1, 3) +#check (true, true) + + + diff --git a/doc/examples/palindromes.lean b/doc/examples/palindromes.lean index 1aa6004706e7..4d319d93951d 100644 --- a/doc/examples/palindromes.lean +++ b/doc/examples/palindromes.lean @@ -48,7 +48,7 @@ Note that we use `(by simp)` to prove that `a₂ :: as ≠ []` in the recursive -/ def List.last : (as : List α) → as ≠ [] → α | [a], _ => a - | a₁::a₂:: as, _ => (a₂::as).last (by simp) + | _::a₂:: as, _ => (a₂::as).last (by simp) /-! We use the function `List.last` to prove the following theorem that says that if a list `as` is not empty, diff --git a/doc/flake.nix b/doc/flake.nix index 88dd52ada7f5..bcaac39babb5 100644 --- a/doc/flake.nix +++ b/doc/flake.nix @@ -40,7 +40,7 @@ # necessary for `additional-css`...? cp -r --no-preserve=mode $src/doc/* . # overwrite stub .lean.md files - cp -r ${examples}/* . + cp -r ${examples}/* examples/ mdbook build -d $out ''; }; @@ -78,16 +78,17 @@ (with python3Packages; [ pygments dominate beautifulsoup4 docutils ]); doCheck = false; }; - examples = let - renderLean = name: file: runCommandNoCC "${name}.md" { buildInputs = [ alectryon ]; } '' - mkdir -p $out/examples - alectryon --frontend lean4+markup ${file} --backend webpage -o $out/examples/${name}.md - ''; - ents = builtins.readDir ./examples; + renderLean = name: file: runCommandNoCC "${name}.md" { buildInputs = [ alectryon ]; } '' + mkdir -p $out/examples + alectryon --frontend lean4+markup ${file} --backend webpage -o $out/${name}.md + ''; + renderDir = name: dir: let + ents = builtins.readDir dir; inputs = lib.filterAttrs (n: t: builtins.match ".*\.lean" n != null && t == "regular") ents; - outputs = lib.mapAttrs (n: _: renderLean n ./examples/${n}) inputs; + outputs = lib.mapAttrs (n: _: renderLean n "${dir}/${n}") inputs; in - outputs // symlinkJoin { name = "examples"; paths = lib.attrValues outputs; }; + outputs // symlinkJoin { inherit name; paths = lib.attrValues outputs; }; + examples = renderDir "examples" ./examples; doc = book; }; defaultPackage = self.packages.${system}.doc; diff --git a/doc/metaprogramming-arith.lean b/doc/metaprogramming-arith.lean index eb0c093d782a..92763d78f66d 100644 --- a/doc/metaprogramming-arith.lean +++ b/doc/metaprogramming-arith.lean @@ -8,7 +8,7 @@ declare_syntax_cat arith syntax num : arith -- int for Arith.int syntax str : arith -- strings for Arith.symbol -syntax:60 arith:60 "+" arith:61 : arith -- Arith.add +syntax:60 arith:60 "+" arith:61 : arith -- Arith.add syntax:70 arith:70 "*" arith:71 : arith -- Arith.mul syntax "(" arith ")" : arith -- parenthesized expressions diff --git a/nix/bootstrap.nix b/nix/bootstrap.nix index dd891acdedd5..759bc22cf99c 100644 --- a/nix/bootstrap.nix +++ b/nix/bootstrap.nix @@ -104,7 +104,7 @@ rec { Std = attachSharedLib leanshared Std' // { allExternalDeps = [ Init ]; }; Lean = attachSharedLib leanshared Lean' // { allExternalDeps = [ Init Std ]; }; stdlib = [ Init Std Lean ]; - modDepsFiles = symlinkJoin { name = "modDepsFiles"; paths = map (l: l.modDepsFile) stdlib; }; + modDepsFiles = symlinkJoin { name = "modDepsFiles"; paths = map (l: l.modDepsFile) (stdlib ++ [ Leanc ]); }; iTree = symlinkJoin { name = "ileans"; paths = map (l: l.iTree) stdlib; }; extlib = stdlib; # TODO: add Lake Leanc = build { name = "Leanc"; src = lean-bin-tools-unwrapped.leanc_src; deps = stdlib; }; diff --git a/src/Init/Classical.lean b/src/Init/Classical.lean index be8d65f609aa..83e72ce853c7 100644 --- a/src/Init/Classical.lean +++ b/src/Init/Classical.lean @@ -9,7 +9,7 @@ import Init.NotationExtra universe u v -/- Classical reasoning support -/ +/-! # Classical reasoning support -/ namespace Classical @@ -65,7 +65,7 @@ noncomputable def inhabited_of_nonempty {α : Sort u} (h : Nonempty α) : Inhabi noncomputable def inhabited_of_exists {α : Sort u} {p : α → Prop} (h : ∃ x, p x) : Inhabited α := inhabited_of_nonempty (Exists.elim h (fun w _ => ⟨w⟩)) -/- all propositions are Decidable -/ +/-- All propositions are `Decidable`. -/ noncomputable scoped instance (priority := low) propDecidable (a : Prop) : Decidable a := choice <| match em a with | Or.inl h => ⟨isTrue h⟩ diff --git a/src/Init/Coe.lean b/src/Init/Coe.lean index 4bfcc0fe8583..19599db9c7db 100644 --- a/src/Init/Coe.lean +++ b/src/Init/Coe.lean @@ -15,11 +15,11 @@ class Coe (α : Sort u) (β : Sort v) where class CoeTC (α : Sort u) (β : Sort v) where coe : α → β -/- Expensive coercion that can only appear at the beginning of a sequence of coercions. -/ +/-- Expensive coercion that can only appear at the beginning of a sequence of coercions. -/ class CoeHead (α : Sort u) (β : Sort v) where coe : α → β -/- Expensive coercion that can only appear at the end of a sequence of coercions. -/ +/-- Expensive coercion that can only appear at the end of a sequence of coercions. -/ class CoeTail (α : Sort u) (β : Sort v) where coe : α → β @@ -30,7 +30,7 @@ class CoeHTCT (α : Sort u) (β : Sort v) where class CoeDep (α : Sort u) (_ : α) (β : Sort v) where coe : β -/- Combines CoeHead, CoeTC, CoeTail, CoeDep -/ +/-- Combines CoeHead, CoeTC, CoeTail, CoeDep -/ class CoeT (α : Sort u) (_ : α) (β : Sort v) where coe : β @@ -81,7 +81,7 @@ instance coeId {α : Sort u} (a : α) : CoeT α a α where instance coeSortToCoeTail [inst : CoeSort α β] : CoeTail α β where coe := inst.coe -/- Basic instances -/ +/-! # Basic instances -/ @[inline] instance boolToProp : Coe Bool Prop where coe b := Eq b true @@ -98,7 +98,7 @@ instance optionCoe {α : Type u} : CoeTail α (Option α) where instance subtypeCoe {α : Sort u} {p : α → Prop} : CoeHead (Subtype p) α where coe v := v.val -/- Coe bridge -/ +/-! # Coe bridge -/ -- Helper definition used by the elaborator. It is not meant to be used directly by users @[inline] def Lean.Internal.liftCoeM {m : Type u → Type v} {n : Type u → Type w} {α β : Type u} [MonadLiftT m n] [∀ a, CoeT α a β] [Monad n] (x : m α) : n β := do diff --git a/src/Init/Control/Basic.lean b/src/Init/Control/Basic.lean index 23394c7b7601..84db5c300ba2 100644 --- a/src/Init/Control/Basic.lean +++ b/src/Init/Control/Basic.lean @@ -217,7 +217,7 @@ def control {m : Type u → Type v} {n : Type u → Type w} [MonadControlT m n] (f : ({β : Type u} → n β → m (stM m n β)) → m (stM m n α)) : n α := controlAt m f -/- +/-- Typeclass for the polymorphic `forM` operation described in the "do unchained" paper. Remark: - `γ` is a "container" type of elements of type `α`. diff --git a/src/Init/Control/ExceptCps.lean b/src/Init/Control/ExceptCps.lean index 7c2a859d0363..a8ed4413df07 100644 --- a/src/Init/Control/ExceptCps.lean +++ b/src/Init/Control/ExceptCps.lean @@ -6,7 +6,7 @@ Authors: Leonardo de Moura prelude import Init.Control.Lawful -/- +/-! The Exception monad transformer using CPS style. -/ diff --git a/src/Init/Control/Lawful.lean b/src/Init/Control/Lawful.lean index ccca5831016f..caced776b63f 100644 --- a/src/Init/Control/Lawful.lean +++ b/src/Init/Control/Lawful.lean @@ -90,7 +90,7 @@ theorem seqRight_eq_bind [Monad m] [LawfulMonad m] (x : m α) (y : m β) : x *> theorem seqLeft_eq_bind [Monad m] [LawfulMonad m] (x : m α) (y : m β) : x <* y = x >>= fun a => y >>= fun _ => pure a := by rw [seqLeft_eq]; simp [map_eq_pure_bind, seq_eq_bind_map] -/- Id -/ +/-! # Id -/ namespace Id @@ -103,7 +103,7 @@ instance : LawfulMonad Id := by end Id -/- ExceptT -/ +/-! # ExceptT -/ namespace ExceptT @@ -179,7 +179,7 @@ instance [Monad m] [LawfulMonad m] : LawfulMonad (ExceptT ε m) where end ExceptT -/- ReaderT -/ +/-! # ReaderT -/ namespace ReaderT @@ -225,12 +225,12 @@ instance [Monad m] [LawfulMonad m] : LawfulMonad (ReaderT ρ m) where end ReaderT -/- StateRefT -/ +/-! # StateRefT -/ instance [Monad m] [LawfulMonad m] : LawfulMonad (StateRefT' ω σ m) := inferInstanceAs (LawfulMonad (ReaderT (ST.Ref ω σ) m)) -/- StateT -/ +/-! # StateT -/ namespace StateT diff --git a/src/Init/Control/StateCps.lean b/src/Init/Control/StateCps.lean index ca5f9e50f914..2747b258e8a9 100644 --- a/src/Init/Control/StateCps.lean +++ b/src/Init/Control/StateCps.lean @@ -6,7 +6,7 @@ Authors: Leonardo de Moura prelude import Init.Control.Lawful -/- +/-! The State monad transformer using CPS style. -/ diff --git a/src/Init/Control/StateRef.lean b/src/Init/Control/StateRef.lean index 7c4e92f3bc3e..fd05a47bd451 100644 --- a/src/Init/Control/StateRef.lean +++ b/src/Init/Control/StateRef.lean @@ -11,7 +11,7 @@ import Init.Control.State def StateRefT' (ω : Type) (σ : Type) (m : Type → Type) (α : Type) : Type := ReaderT (ST.Ref ω σ) m α -/- Recall that `StateRefT` is a macro that infers `ω` from the `m`. -/ +/-! Recall that `StateRefT` is a macro that infers `ω` from the `m`. -/ @[inline] def StateRefT'.run {ω σ : Type} {m : Type → Type} [Monad m] [MonadLiftT (ST ω) m] {α : Type} (x : StateRefT' ω σ m α) (s : σ) : m (α × σ) := do let ref ← ST.mkRef s diff --git a/src/Init/Core.lean b/src/Init/Core.lean index e927945b1966..28031221f6ac 100644 --- a/src/Init/Core.lean +++ b/src/Init/Core.lean @@ -79,7 +79,7 @@ structure PSigma {α : Sort u} (β : α → Sort v) where inductive Exists {α : Sort u} (p : α → Prop) : Prop where | intro (w : α) (h : p w) : Exists p -/- Auxiliary type used to compile `for x in xs` notation. -/ +/-- Auxiliary type used to compile `for x in xs` notation. -/ inductive ForInStep (α : Type u) where | done : α → ForInStep α | yield : α → ForInStep α @@ -95,24 +95,24 @@ class ForIn' (m : Type u₁ → Type u₂) (ρ : Type u) (α : outParam (Type v) export ForIn' (forIn') -/- Auxiliary type used to compile `do` notation. -/ +/-- Auxiliary type used to compile `do` notation. -/ inductive DoResultPRBC (α β σ : Type u) where | «pure» : α → σ → DoResultPRBC α β σ | «return» : β → σ → DoResultPRBC α β σ | «break» : σ → DoResultPRBC α β σ | «continue» : σ → DoResultPRBC α β σ -/- Auxiliary type used to compile `do` notation. -/ +/-- Auxiliary type used to compile `do` notation. -/ inductive DoResultPR (α β σ : Type u) where | «pure» : α → σ → DoResultPR α β σ | «return» : β → σ → DoResultPR α β σ -/- Auxiliary type used to compile `do` notation. -/ +/-- Auxiliary type used to compile `do` notation. -/ inductive DoResultBC (σ : Type u) where | «break» : σ → DoResultBC σ | «continue» : σ → DoResultBC σ -/- Auxiliary type used to compile `do` notation. -/ +/-- Auxiliary type used to compile `do` notation. -/ inductive DoResultSBC (α σ : Type u) where | «pureReturn» : α → σ → DoResultSBC α σ | «break» : σ → DoResultSBC α σ @@ -129,7 +129,7 @@ class EmptyCollection (α : Type u) where notation "{" "}" => EmptyCollection.emptyCollection notation "∅" => EmptyCollection.emptyCollection -/- Remark: tasks have an efficient implementation in the runtime. -/ +/-- Remark: tasks have an efficient implementation in the runtime. -/ structure Task (α : Type u) : Type u where pure :: (get : α) deriving Inhabited @@ -166,11 +166,11 @@ protected def bind {α : Type u} {β : Type v} (x : Task α) (f : α → Task β end Task -/- Some type that is not a scalar value in our runtime. -/ +/-- Some type that is not a scalar value in our runtime. -/ structure NonScalar where val : Nat -/- Some type that is not a scalar value in our runtime and is universe polymorphic. -/ +/-- Some type that is not a scalar value in our runtime and is universe polymorphic. -/ inductive PNonScalar : Type u where | mk (v : Nat) : PNonScalar @@ -178,7 +178,7 @@ inductive PNonScalar : Type u where theorem optParam_eq (α : Sort u) (default : α) : optParam α default = α := rfl -/- Boolean operators -/ +/-! # Boolean operators -/ @[extern c inline "#1 || #2"] def strictOr (b₁ b₂ : Bool) := b₁ || b₂ @[extern c inline "#1 && #2"] def strictAnd (b₁ b₂ : Bool) := b₁ && b₂ @@ -205,7 +205,7 @@ instance : LawfulBEq Char := inferInstance instance : LawfulBEq String := inferInstance -/- Logical connectives an equality -/ +/-! # Logical connectives and equality -/ def implies (a b : Prop) := a → b @@ -359,14 +359,14 @@ theorem Iff.comm : (a ↔ b) ↔ (b ↔ a) := theorem And.comm : a ∧ b ↔ b ∧ a := by constructor <;> intro ⟨h₁, h₂⟩ <;> exact ⟨h₂, h₁⟩ -/- Exists -/ +/-! # Exists -/ theorem Exists.elim {α : Sort u} {p : α → Prop} {b : Prop} (h₁ : Exists (fun x => p x)) (h₂ : ∀ (a : α), p a → b) : b := match h₁ with | intro a h => h₂ a h -/- Decidable -/ +/-! # Decidable -/ theorem decide_true_eq_true (h : Decidable True) : @decide True h = true := match h with @@ -457,7 +457,7 @@ instance {p q} [Decidable p] [Decidable q] : Decidable (p ↔ q) := else isTrue ⟨fun h => absurd h hp, fun h => absurd h hq⟩ -/- if-then-else expression theorems -/ +/-! # if-then-else expression theorems -/ theorem if_pos {c : Prop} {h : Decidable c} (hc : c) {α : Sort u} {t e : α} : (ite c t e) = t := match h with @@ -495,7 +495,7 @@ instance {c : Prop} {t : c → Prop} {e : ¬c → Prop} [dC : Decidable c] [dT : | isTrue hc => dT hc | isFalse hc => dE hc -/- Auxiliary definitions for generating compact `noConfusion` for enumeration types -/ +/-- Auxiliary definitions for generating compact `noConfusion` for enumeration types -/ abbrev noConfusionTypeEnum {α : Sort u} {β : Sort v} [inst : DecidableEq β] (f : α → β) (P : Sort w) (x y : α) : Sort w := Decidable.casesOn (motive := fun _ => Sort w) (inst (f x) (f y)) (fun _ => P) @@ -508,7 +508,7 @@ abbrev noConfusionEnum {α : Sort u} {β : Sort v} [inst : DecidableEq β] (f : (fun h' => False.elim (h' (congrArg f h))) (fun _ => fun x => x) -/- Inhabited -/ +/-! # Inhabited -/ instance : Inhabited Prop where default := True @@ -518,7 +518,7 @@ deriving instance Inhabited for NonScalar, PNonScalar, True, ForInStep theorem nonempty_of_exists {α : Sort u} {p : α → Prop} : Exists (fun x => p x) → Nonempty α | ⟨w, _⟩ => ⟨w⟩ -/- Subsingleton -/ +/-! # Subsingleton -/ class Subsingleton (α : Sort u) : Prop where intro :: allEq : (a b : α) → a = b @@ -572,7 +572,7 @@ inductive TC {α : Sort u} (r : α → α → Prop) : α → α → Prop where | base : ∀ a b, r a b → TC r a b | trans : ∀ a b c, TC r a b → TC r b c → TC r a c -/- Subtype -/ +/-! # Subtype -/ namespace Subtype def existsOfSubtype {α : Type u} {p : α → Prop} : { x // p x } → Exists (fun x => p x) @@ -597,7 +597,7 @@ instance {α : Type u} {p : α → Prop} [DecidableEq α] : DecidableEq {x : α end Subtype -/- Sum -/ +/-! # Sum -/ section variable {α : Type u} {β : Type v} @@ -621,7 +621,7 @@ instance {α : Type u} {β : Type v} [DecidableEq α] [DecidableEq β] : Decidab end -/- Product -/ +/-! # Product -/ instance [Inhabited α] [Inhabited β] : Inhabited (α × β) where default := (default, default) @@ -657,7 +657,7 @@ def Prod.map {α₁ : Type u₁} {α₂ : Type u₂} {β₁ : Type v₁} {β₂ (f : α₁ → α₂) (g : β₁ → β₂) : α₁ × β₁ → α₂ × β₂ | (a, b) => (f a, g b) -/- Dependent products -/ +/-! # Dependent products -/ theorem ex_of_PSigma {α : Type u} {p : α → Prop} : (PSigma (fun x => p x)) → Exists (fun x => p x) | ⟨x, hx⟩ => ⟨x, hx⟩ @@ -668,7 +668,7 @@ protected theorem PSigma.eta {α : Sort u} {β : α → Sort v} {a₁ a₂ : α} subst h₂ exact rfl -/- Universe polymorphic unit -/ +/-! # Universe polymorphic unit -/ theorem PUnit.subsingleton (a b : PUnit) : a = b := by cases a; cases b; exact rfl @@ -685,7 +685,7 @@ instance : Inhabited PUnit where instance : DecidableEq PUnit := fun a b => isTrue (PUnit.subsingleton a b) -/- Setoid -/ +/-! # Setoid -/ class Setoid (α : Sort u) where r : α → α → Prop @@ -710,7 +710,7 @@ theorem trans {a b c : α} (hab : a ≈ b) (hbc : b ≈ c) : a ≈ c := end Setoid -/- Propositional extensionality -/ +/-! # Propositional extensionality -/ axiom propext {a b : Prop} : (a ↔ b) → a = b @@ -742,9 +742,9 @@ gen_injective_theorems% Lean.Syntax @[simp] theorem beq_iff_eq [BEq α] [LawfulBEq α] (a b : α) : a == b ↔ a = b := ⟨eq_of_beq, by intro h; subst h; exact LawfulBEq.rfl⟩ -/- Quotients -/ +/-! # Quotients -/ --- Iff can now be used to do substitutions in a calculation +/-- Iff can now be used to do substitutions in a calculation -/ theorem Iff.subst {a b : Prop} {p : Prop → Prop} (h₁ : a ↔ b) (h₂ : p a) : p b := Eq.subst (propext h₁) h₂ @@ -1018,7 +1018,7 @@ instance {α : Sort u} {s : Setoid α} [d : ∀ (a b : α), Decidable (a ≈ b)] | isTrue h₁ => isTrue (Quotient.sound h₁) | isFalse h₂ => isFalse fun h => absurd (Quotient.exact h) h₂ -/- Function extensionality -/ +/-! # Function extensionality -/ namespace Function variable {α : Sort u} {β : α → Sort v} @@ -1067,7 +1067,7 @@ instance {α : Sort u} {β : α → Sort v} [∀ a, Subsingleton (β a)] : Subsi allEq f₁ f₂ := funext (fun a => Subsingleton.elim (f₁ a) (f₂ a)) -/- Squash -/ +/-! # Squash -/ def Squash (α : Type u) := Quot (fun (_ _ : α) => True) @@ -1086,13 +1086,13 @@ instance : Subsingleton (Squash α) where apply Quot.sound trivial -/- Relations -/ +/-! # Relations -/ class Antisymm {α : Sort u} (r : α → α → Prop) where antisymm {a b : α} : r a b → r b a → a = b namespace Lean -/- Kernel reduction hints -/ +/-! # Kernel reduction hints -/ /-- When the kernel tries to reduce a term `Lean.reduceBool c`, it will invoke the Lean interpreter to evaluate `c`. diff --git a/src/Init/Data/Array/Basic.lean b/src/Init/Data/Array/Basic.lean index 16732966b6f0..b41dab9d4887 100644 --- a/src/Init/Data/Array/Basic.lean +++ b/src/Init/Data/Array/Basic.lean @@ -34,7 +34,7 @@ def isEmpty (a : Array α) : Bool := def singleton (v : α) : Array α := mkArray 1 v -/- Low-level version of `fget` which is as fast as a C array read. +/-- Low-level version of `fget` which is as fast as a C array read. `Fin` values are represented as tag pointers in the Lean runtime. Thus, `fget` may be slightly slower than `uget`. -/ @[extern "lean_array_uget"] @@ -64,7 +64,7 @@ abbrev getLit {α : Type u} {n : Nat} (a : Array α) (i : Nat) (h₁ : a.size = @[simp] theorem size_push (a : Array α) (v : α) : (push a v).size = a.size + 1 := List.length_concat .. -/- Low-level version of `fset` which is as fast as a C array fset. +/-- Low-level version of `fset` which is as fast as a C array fset. `Fin` values are represented as tag pointers in the Lean runtime. Thus, `fset` may be slightly slower than `uset`. -/ @[extern "lean_array_uset"] @@ -141,7 +141,7 @@ def modify (a : Array α) (i : Nat) (f : α → α) : Array α := def modifyOp (self : Array α) (idx : Nat) (f : α → α) : Array α := self.modify idx f -/- +/-- We claim this unsafe implementation is correct because an array cannot have more than `usizeSz` elements in our runtime. This kind of low level trick can be removed with a little bit of compiler support. For example, if the compiler simplifies `as.size < usizeSz` to true. -/ @@ -157,7 +157,7 @@ def modifyOp (self : Array α) (idx : Nat) (f : α → α) : Array α := pure b loop 0 b -/- Reference implementation for `forIn` -/ +/-- Reference implementation for `forIn` -/ @[implementedBy Array.forInUnsafe] protected def forIn {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (as : Array α) (b : β) (f : α → β → m (ForInStep β)) : m β := let rec loop (i : Nat) (h : i ≤ as.size) (b : β) : m β := do @@ -175,7 +175,7 @@ protected def forIn {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m instance : ForIn m (Array α) α where forIn := Array.forIn -/- See comment at forInUnsafe -/ +/-- See comment at `forInUnsafe` -/ @[inline] unsafe def foldlMUnsafe {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : β → α → m β) (init : β) (as : Array α) (start := 0) (stop := as.size) : m β := let rec @[specialize] fold (i : USize) (stop : USize) (b : β) : m β := do @@ -191,7 +191,7 @@ unsafe def foldlMUnsafe {α : Type u} {β : Type v} {m : Type v → Type w} [Mon else pure init -/- Reference implementation for `foldlM` -/ +/-- Reference implementation for `foldlM` -/ @[implementedBy foldlMUnsafe] def foldlM {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : β → α → m β) (init : β) (as : Array α) (start := 0) (stop := as.size) : m β := let fold (stop : Nat) (h : stop ≤ as.size) := @@ -210,7 +210,7 @@ def foldlM {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : β else fold as.size (Nat.le_refl _) -/- See comment at forInUnsafe -/ +/-- See comment at `forInUnsafe` -/ @[inline] unsafe def foldrMUnsafe {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : α → β → m β) (init : β) (as : Array α) (start := as.size) (stop := 0) : m β := let rec @[specialize] fold (i : USize) (stop : USize) (b : β) : m β := do @@ -228,7 +228,7 @@ unsafe def foldrMUnsafe {α : Type u} {β : Type v} {m : Type v → Type w} [Mon else pure init -/- Reference implementation for `foldrM` -/ +/-- Reference implementation for `foldrM` -/ @[implementedBy foldrMUnsafe] def foldrM {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : α → β → m β) (init : β) (as : Array α) (start := as.size) (stop := 0) : m β := let rec fold (i : Nat) (h : i ≤ as.size) (b : β) : m β := do @@ -249,7 +249,7 @@ def foldrM {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : α else pure init -/- See comment at forInUnsafe -/ +/-- See comment at `forInUnsafe` -/ @[inline] unsafe def mapMUnsafe {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : α → m β) (as : Array α) : m (Array β) := let sz := USize.ofNat as.size @@ -266,7 +266,7 @@ unsafe def mapMUnsafe {α : Type u} {β : Type v} {m : Type v → Type w} [Monad pure (unsafeCast r) unsafeCast <| map 0 (unsafeCast as) -/- Reference implementation for `mapM` -/ +/-- Reference implementation for `mapM` -/ @[implementedBy mapMUnsafe] def mapM {α : Type u} {β : Type v} {m : Type v → Type w} [Monad m] (f : α → m β) (as : Array α) : m (Array β) := as.foldlM (fun bs a => do let b ← f a; pure (bs.push b)) (mkEmpty as.size) diff --git a/src/Init/Data/ByteArray/Basic.lean b/src/Init/Data/ByteArray/Basic.lean index 4c7f861c68bd..52b22c535f62 100644 --- a/src/Init/Data/ByteArray/Basic.lean +++ b/src/Init/Data/ByteArray/Basic.lean @@ -102,7 +102,7 @@ partial def toList (bs : ByteArray) : List UInt8 := none loop start -/- +/-- We claim this unsafe implementation is correct because an array cannot have more than `usizeSz` elements in our runtime. This is similar to the `Array` version. @@ -120,7 +120,7 @@ partial def toList (bs : ByteArray) : List UInt8 := pure b loop 0 b -/- Reference implementation for `forIn` -/ +/-- Reference implementation for `forIn` -/ @[implementedBy ByteArray.forInUnsafe] protected def forIn {β : Type v} {m : Type v → Type w} [Monad m] (as : ByteArray) (b : β) (f : UInt8 → β → m (ForInStep β)) : m β := let rec loop (i : Nat) (h : i ≤ as.size) (b : β) : m β := do @@ -138,10 +138,8 @@ protected def forIn {β : Type v} {m : Type v → Type w} [Monad m] (as : ByteAr instance : ForIn m ByteArray UInt8 where forIn := ByteArray.forIn -/- - See comment at forInUnsafe - TODO: avoid code duplication. --/ +/-- See comment at `forInUnsafe` -/ +-- TODO: avoid code duplication. @[inline] unsafe def foldlMUnsafe {β : Type v} {m : Type v → Type w} [Monad m] (f : β → UInt8 → m β) (init : β) (as : ByteArray) (start := 0) (stop := as.size) : m β := let rec @[specialize] fold (i : USize) (stop : USize) (b : β) : m β := do @@ -157,7 +155,7 @@ unsafe def foldlMUnsafe {β : Type v} {m : Type v → Type w} [Monad m] (f : β else pure init -/- Reference implementation for `foldlM` -/ +/-- Reference implementation for `foldlM` -/ @[implementedBy foldlMUnsafe] def foldlM {β : Type v} {m : Type v → Type w} [Monad m] (f : β → UInt8 → m β) (init : β) (as : ByteArray) (start := 0) (stop := as.size) : m β := let fold (stop : Nat) (h : stop ≤ as.size) := diff --git a/src/Init/Data/Fin/Basic.lean b/src/Init/Data/Fin/Basic.lean index 5c4827521d0e..69c70b926ce5 100644 --- a/src/Init/Data/Fin/Basic.lean +++ b/src/Init/Data/Fin/Basic.lean @@ -44,7 +44,7 @@ protected def mul : Fin n → Fin n → Fin n protected def sub : Fin n → Fin n → Fin n | ⟨a, h⟩, ⟨b, _⟩ => ⟨(a + (n - b)) % n, mlt h⟩ -/- +/-! Remark: mod/div/modn/land/lor can be defined without using (% n), but we are trying to minimize the number of Nat theorems needed to boostrap Lean. diff --git a/src/Init/Data/FloatArray/Basic.lean b/src/Init/Data/FloatArray/Basic.lean index b35f2a38ee74..eef9c53b49a1 100644 --- a/src/Init/Data/FloatArray/Basic.lean +++ b/src/Init/Data/FloatArray/Basic.lean @@ -84,12 +84,11 @@ partial def toList (ds : FloatArray) : List Float := r.reverse loop 0 [] -/- +/-- We claim this unsafe implementation is correct because an array cannot have more than `usizeSz` elements in our runtime. This is similar to the `Array` version. - - TODO: avoid code duplication in the future after we improve the compiler. -/ +-- TODO: avoid code duplication in the future after we improve the compiler. @[inline] unsafe def forInUnsafe {β : Type v} {m : Type v → Type w} [Monad m] (as : FloatArray) (b : β) (f : Float → β → m (ForInStep β)) : m β := let sz := USize.ofNat as.size let rec @[specialize] loop (i : USize) (b : β) : m β := do @@ -102,7 +101,7 @@ partial def toList (ds : FloatArray) : List Float := pure b loop 0 b -/- Reference implementation for `forIn` -/ +/-- Reference implementation for `forIn` -/ @[implementedBy FloatArray.forInUnsafe] protected def forIn {β : Type v} {m : Type v → Type w} [Monad m] (as : FloatArray) (b : β) (f : Float → β → m (ForInStep β)) : m β := let rec loop (i : Nat) (h : i ≤ as.size) (b : β) : m β := do @@ -120,10 +119,8 @@ protected def forIn {β : Type v} {m : Type v → Type w} [Monad m] (as : FloatA instance : ForIn m FloatArray Float where forIn := FloatArray.forIn -/- - See comment at forInUnsafe - TODO: avoid code duplication. --/ +/-- See comment at `forInUnsafe` -/ +-- TODO: avoid code duplication. @[inline] unsafe def foldlMUnsafe {β : Type v} {m : Type v → Type w} [Monad m] (f : β → Float → m β) (init : β) (as : FloatArray) (start := 0) (stop := as.size) : m β := let rec @[specialize] fold (i : USize) (stop : USize) (b : β) : m β := do @@ -139,7 +136,7 @@ unsafe def foldlMUnsafe {β : Type v} {m : Type v → Type w} [Monad m] (f : β else pure init -/- Reference implementation for `foldlM` -/ +/-- Reference implementation for `foldlM` -/ @[implementedBy foldlMUnsafe] def foldlM {β : Type v} {m : Type v → Type w} [Monad m] (f : β → Float → m β) (init : β) (as : FloatArray) (start := 0) (stop := as.size) : m β := let fold (stop : Nat) (h : stop ≤ as.size) := diff --git a/src/Init/Data/Format/Basic.lean b/src/Init/Data/Format/Basic.lean index 480d33092467..b84a453bfdfe 100644 --- a/src/Init/Data/Format/Basic.lean +++ b/src/Init/Data/Format/Basic.lean @@ -23,8 +23,8 @@ inductive Format where | nest (indent : Int) : Format → Format | append : Format → Format → Format | group : Format → (behavior : FlattenBehavior := FlattenBehavior.allOrNone) → Format - /- Used for associating auxiliary information (e.g. `Expr`s) with `Format` objects. -/ - | tag : Nat → Format → Format + | /-- Used for associating auxiliary information (e.g. `Expr`s) with `Format` objects. -/ + tag : Nat → Format → Format deriving Inhabited namespace Format diff --git a/src/Init/Data/Int/Basic.lean b/src/Init/Data/Int/Basic.lean index 763d196d00a0..d073f1bc839f 100644 --- a/src/Init/Data/Int/Basic.lean +++ b/src/Init/Data/Int/Basic.lean @@ -11,7 +11,7 @@ import Init.Data.Nat.Div import Init.Data.List.Basic open Nat -/- the Type, coercions, and notation -/ +/-! # the Type, coercions, and notation -/ inductive Int : Type where | ofNat : Nat → Int @@ -62,7 +62,7 @@ protected def mul (m n : @& Int) : Int := | negSucc m, ofNat n => negOfNat (succ m * n) | negSucc m, negSucc n => ofNat (succ m * succ n) -/- +/-- The `Neg Int` default instance must have priority higher than `low` since the default instance `OfNat Nat n` has `low` priority. ``` diff --git a/src/Init/Data/List/BasicAux.lean b/src/Init/Data/List/BasicAux.lean index 942dd1bbcb89..3cbffb0a709f 100644 --- a/src/Init/Data/List/BasicAux.lean +++ b/src/Init/Data/List/BasicAux.lean @@ -11,7 +11,7 @@ import Init.Util universe u namespace List -/- The following functions can't be defined at `Init.Data.List.Basic`, because they depend on `Init.Util`, +/-! The following functions can't be defined at `Init.Data.List.Basic`, because they depend on `Init.Util`, and `Init.Util` depends on `Init.Data.List.Basic`. -/ def get! [Inhabited α] : List α → Nat → α diff --git a/src/Init/Data/List/Control.lean b/src/Init/Data/List/Control.lean index 3e58b27ff5fa..2c4727029153 100644 --- a/src/Init/Data/List/Control.lean +++ b/src/Init/Data/List/Control.lean @@ -10,7 +10,7 @@ import Init.Data.List.Basic namespace List universe u v w u₁ u₂ -/- +/-! Remark: we can define `mapM`, `mapM₂` and `forM` using `Applicative` instead of `Monad`. Example: ``` @@ -193,4 +193,7 @@ instance : ForM m (List α) α where @[simp] theorem forM_cons [Monad m] (f : α → m PUnit) (a : α) (as : List α) : forM (a::as) f = f a >>= fun _ => forM as f := rfl +instance : Functor List where + map := List.map + end List diff --git a/src/Init/Data/Nat/Basic.lean b/src/Init/Data/Nat/Basic.lean index 271aa24329b5..eb6d9aa6d64f 100644 --- a/src/Init/Data/Nat/Basic.lean +++ b/src/Init/Data/Nat/Basic.lean @@ -26,7 +26,7 @@ namespace Nat | 0 => false | succ n => f (s - (succ n)) || anyAux f s n -/- `any f n = true` iff there is `i in [0, n-1]` s.t. `f i = true` -/ +/-- `any f n = true` iff there is `i in [0, n-1]` s.t. `f i = true` -/ @[inline] def any (f : Nat → Bool) (n : Nat) : Bool := anyAux f n n @@ -44,7 +44,7 @@ def blt (a b : Nat) : Bool := attribute [simp] Nat.zero_le -/- Helper "packing" theorems -/ +/-! # Helper "packing" theorems -/ @[simp] theorem zero_eq : Nat.zero = 0 := rfl @[simp] theorem add_eq : Nat.add x y = x + y := rfl @@ -53,7 +53,7 @@ attribute [simp] Nat.zero_le @[simp] theorem lt_eq : Nat.lt x y = (x < y) := rfl @[simp] theorem le_eq : Nat.le x y = (x ≤ y) := rfl -/- Helper Bool relation theorems -/ +/-! # Helper Bool relation theorems -/ @[simp] theorem beq_refl (a : Nat) : Nat.beq a a = true := by induction a with simp [Nat.beq] @@ -75,7 +75,7 @@ instance : LawfulBEq Nat where have : ¬ ((a == b) = true) := fun h' => absurd (eq_of_beq h') h by simp [this]) -/- Nat.add theorems -/ +/-! # Nat.add theorems -/ @[simp] protected theorem zero_add : ∀ (n : Nat), 0 + n = n | 0 => rfl @@ -120,7 +120,7 @@ protected theorem add_right_cancel {n m k : Nat} (h : n + m = k + m) : n = k := rw [Nat.add_comm n m, Nat.add_comm k m] at h apply Nat.add_left_cancel h -/- Nat.mul theorems -/ +/-! # Nat.mul theorems -/ @[simp] protected theorem mul_zero (n : Nat) : n * 0 = 0 := rfl @@ -168,7 +168,7 @@ protected theorem mul_assoc : ∀ (n m k : Nat), (n * m) * k = n * (m * k) protected theorem mul_left_comm (n m k : Nat) : n * (m * k) = m * (n * k) := by rw [← Nat.mul_assoc, Nat.mul_comm n m, Nat.mul_assoc] -/- Inequalities -/ +/-! # Inequalities -/ attribute [simp] Nat.le_refl @@ -379,7 +379,7 @@ protected theorem le_of_add_le_add_right {a b c : Nat} : a + b ≤ c + b → a rw [Nat.add_comm _ b, Nat.add_comm _ b] apply Nat.le_of_add_le_add_left -/- Basic theorems for comparing numerals -/ +/-! # Basic theorems for comparing numerals -/ theorem ctor_eq_zero : Nat.zero = 0 := rfl @@ -393,7 +393,7 @@ protected theorem zero_ne_one : 0 ≠ (1 : Nat) := theorem succ_ne_zero (n : Nat) : succ n ≠ 0 := fun h => Nat.noConfusion h -/- mul + order -/ +/-! # mul + order -/ theorem mul_le_mul_left {n m : Nat} (k : Nat) (h : n ≤ m) : k * n ≤ k * m := match le.dest h with @@ -429,7 +429,7 @@ protected theorem eq_of_mul_eq_mul_left {m k n : Nat} (hn : 0 < n) (h : n * m = theorem eq_of_mul_eq_mul_right {n m k : Nat} (hm : 0 < m) (h : n * m = k * m) : n = k := by rw [Nat.mul_comm n m, Nat.mul_comm k m] at h; exact Nat.eq_of_mul_eq_mul_left hm h -/- power -/ +/-! # power -/ theorem pow_succ (n m : Nat) : n^(succ m) = n^m * n := rfl @@ -455,7 +455,7 @@ theorem pow_le_pow_of_le_right {n : Nat} (hx : n > 0) {i : Nat} : ∀ {j}, i ≤ theorem pos_pow_of_pos {n : Nat} (m : Nat) (h : 0 < n) : 0 < n^m := pow_le_pow_of_le_right h (Nat.zero_le _) -/- min/max -/ +/-! # min/max -/ protected def min (n m : Nat) : Nat := if n ≤ m then n else m @@ -463,7 +463,7 @@ protected def min (n m : Nat) : Nat := protected def max (n m : Nat) : Nat := if n ≤ m then m else n -/- Auxiliary theorems for well-founded recursion -/ +/-! # Auxiliary theorems for well-founded recursion -/ theorem not_eq_zero_of_lt (h : b < a) : a ≠ 0 := by cases a @@ -473,7 +473,7 @@ theorem not_eq_zero_of_lt (h : b < a) : a ≠ 0 := by theorem pred_lt' {n m : Nat} (h : m < n) : pred n < n := pred_lt (not_eq_zero_of_lt h) -/- sub/pred theorems -/ +/-! # sub/pred theorems -/ theorem add_sub_self_left (a b : Nat) : (a + b) - a = b := by induction a with @@ -656,7 +656,7 @@ protected theorem mul_sub_right_distrib (n m k : Nat) : (n - m) * k = n * k - m protected theorem mul_sub_left_distrib (n m k : Nat) : n * (m - k) = n * m - n * k := by rw [Nat.mul_comm, Nat.mul_sub_right_distrib, Nat.mul_comm m n, Nat.mul_comm n k] -/- Helper normalization theorems -/ +/-! # Helper normalization theorems -/ theorem not_le_eq (a b : Nat) : (¬ (a ≤ b)) = (b + 1 ≤ a) := propext <| Iff.intro (fun h => Nat.gt_of_not_le h) (fun h => Nat.not_le_of_gt h) diff --git a/src/Init/Data/Nat/Linear.lean b/src/Init/Data/Nat/Linear.lean index b00538b40274..9115fbf39233 100644 --- a/src/Init/Data/Nat/Linear.lean +++ b/src/Init/Data/Nat/Linear.lean @@ -13,7 +13,7 @@ import Init.Data.Prod namespace Nat.Linear -/--! +/-! Helper definitions and theorems for constructing linear arithmetic proofs. -/ diff --git a/src/Init/Data/OfScientific.lean b/src/Init/Data/OfScientific.lean index f1105181075f..584bec1c3c59 100644 --- a/src/Init/Data/OfScientific.lean +++ b/src/Init/Data/OfScientific.lean @@ -8,7 +8,7 @@ import Init.Meta import Init.Data.Float import Init.Data.Nat -/- For decimal and scientific numbers (e.g., `1.23`, `3.12e10`). +/-- For decimal and scientific numbers (e.g., `1.23`, `3.12e10`). Examples: - `OfScientific.ofScientific 123 true 2` represents `1.23` - `OfScientific.ofScientific 121 false 100` represents `121e100` @@ -31,8 +31,8 @@ protected opaque Float.ofScientific (m : Nat) (s : Bool) (e : Nat) : Float := else Float.ofBinaryScientific (m * 5^e) e -/- - The `OfScientifi Float` must have priority higher than `mid` since +/-- + The `OfScientific Float` must have priority higher than `mid` since the default instance `Neg Int` has `mid` priority. ``` #check -42.0 -- must be Float diff --git a/src/Init/Data/Random.lean b/src/Init/Data/Random.lean index b00e37516359..dba66d541a94 100644 --- a/src/Init/Data/Random.lean +++ b/src/Init/Data/Random.lean @@ -8,27 +8,27 @@ import Init.System.IO import Init.Data.Int universe u -/- +/-! Basic random number generator support based on the one available on the Haskell library -/ -/- Interface for random number generators. -/ +/-- Interface for random number generators. -/ class RandomGen (g : Type u) where - /- `range` returns the range of values returned by + /-- `range` returns the range of values returned by the generator. -/ range : g → Nat × Nat - /- `next` operation returns a natural number that is uniformly distributed + /-- `next` operation returns a natural number that is uniformly distributed the range returned by `range` (including both end points), and a new generator. -/ next : g → Nat × g - /- + /-- The 'split' operation allows one to obtain two distinct random number generators. This is very useful in functional programs (for example, when passing a random number generator down to recursive calls). -/ split : g → g × g -/- "Standard" random number generator. -/ +/-- "Standard" random number generator. -/ structure StdGen where s1 : Nat s2 : Nat @@ -76,7 +76,7 @@ def mkStdGen (s : Nat := 0) : StdGen := let s2 := q % 2147483398 ⟨s1 + 1, s2 + 1⟩ -/- +/-- Auxiliary function for randomNatVal. Generate random values until we exceed the target magnitude. `genLo` and `genMag` are the generator lower bound and magnitude. diff --git a/src/Init/Data/Repr.lean b/src/Init/Data/Repr.lean index db7b519797b9..8e10b7499cb8 100644 --- a/src/Init/Data/Repr.lean +++ b/src/Init/Data/Repr.lean @@ -27,7 +27,7 @@ abbrev reprStr [Repr α] (a : α) : String := abbrev reprArg [Repr α] (a : α) : Format := reprPrec a max_prec -/- Auxiliary class for marking types that should be considered atomic by `Repr` methods. +/-- Auxiliary class for marking types that should be considered atomic by `Repr` methods. We use it at `Repr (List α)` to decide whether `bracketFill` should be used or not. -/ class ReprAtom (α : Type u) diff --git a/src/Init/Data/Stream.lean b/src/Init/Data/Stream.lean index 7a68b62a5351..2eb2fb5143c7 100644 --- a/src/Init/Data/Stream.lean +++ b/src/Init/Data/Stream.lean @@ -7,7 +7,7 @@ prelude import Init.Data.Array.Subarray import Init.Data.Range -/- +/-! Remark: we considered using the following alternative design ``` structure Stream (α : Type u) where @@ -22,7 +22,7 @@ The key problem is that the type `Stream α` "lives" in a universe higher than ` This is a problem because we want to use `Stream`s in monadic code. -/ -/- +/-- Streams are used to implement parallel `for` statements. Example: ``` diff --git a/src/Init/Data/String/Extra.lean b/src/Init/Data/String/Extra.lean index 18709a010a42..d8a19e7a58b0 100644 --- a/src/Init/Data/String/Extra.lean +++ b/src/Init/Data/String/Extra.lean @@ -66,4 +66,21 @@ theorem Iterator.sizeOf_next_lt_of_atEnd (i : String.Iterator) (h : ¬ i.atEnd = macro_rules | `(tactic| decreasing_trivial) => `(tactic| apply String.Iterator.sizeOf_next_lt_of_atEnd; assumption) +namespace Iterator + +@[specialize] def find (it : Iterator) (p : Char → Bool) : Iterator := + if it.atEnd then it + else if p it.curr then it + else find it.next p + +@[specialize] def foldUntil (it : Iterator) (init : α) (f : α → Char → Option α) : α × Iterator := + if it.atEnd then + (init, it) + else if let some a := f init it.curr then + foldUntil it.next a f + else + (init, it) + +end Iterator + end String diff --git a/src/Init/Meta.lean b/src/Init/Meta.lean index b73abdae484f..154ed3a6b8b7 100644 --- a/src/Init/Meta.lean +++ b/src/Init/Meta.lean @@ -64,7 +64,7 @@ def toolchain := @[extern c inline "LEAN_IS_STAGE0"] opaque Internal.isStage0 (u : Unit) : Bool -/- Valid identifier names -/ +/-- Valid identifier names -/ def isGreek (c : Char) : Bool := 0x391 ≤ c.val && c.val ≤ 0x3dd @@ -448,7 +448,7 @@ end Syntax @[inline] def mkNode (k : SyntaxNodeKind) (args : Array Syntax) : TSyntax k := ⟨Syntax.node SourceInfo.none k args⟩ -/- Syntax objects for a Lean module. -/ +/-- Syntax objects for a Lean module. -/ structure Module where header : Syntax commands : Array Syntax @@ -491,7 +491,7 @@ partial def expandMacros (stx : Syntax) (p : SyntaxNodeKind → Bool := fun k => return stx | stx => return stx -/- Helper functions for processing Syntax programmatically -/ +/-! # Helper functions for processing Syntax programmatically -/ /-- Create an identifier copying the position from `src`. @@ -588,7 +588,7 @@ def mkScientificLit (val : String) (info := SourceInfo.none) : TSyntax scientifi def mkNameLit (val : String) (info := SourceInfo.none) : NameLit := mkLit nameLitKind val info -/- Recall that we don't have special Syntax constructors for storing numeric and string atoms. +/-! Recall that we don't have special Syntax constructors for storing numeric and string atoms. The idea is to have an extensible approach where embedded DSLs may have new kind of atoms and/or different ways of representing them. So, our atoms contain just the parsed string. The main Lean parser uses the kind `numLitKind` for storing natural numbers that can be encoded @@ -966,7 +966,7 @@ instance Option.hasQuote {α : Type} [Quote α `term] : Quote (Option α) `term | (some x) => Syntax.mkCApp ``some #[quote x] -/- Evaluator for `prec` DSL -/ +/-- Evaluator for `prec` DSL -/ def evalPrec (stx : Syntax) : MacroM Nat := Macro.withIncRecDepth stx do let stx ← expandMacros stx @@ -982,7 +982,7 @@ macro_rules macro "eval_prec " p:prec:max : term => return quote (k := `term) (← evalPrec p) -/- Evaluator for `prio` DSL -/ +/-- Evaluator for `prio` DSL -/ def evalPrio (stx : Syntax) : MacroM Nat := Macro.withIncRecDepth stx do let stx ← expandMacros stx @@ -1061,6 +1061,18 @@ def SepArray.getElems (sa : SepArray sep) : Array Syntax := def TSepArray.getElems (sa : TSepArray k sep) : TSyntaxArray k := .mk sa.elemsAndSeps.getSepElems +def TSepArray.push (sa : TSepArray k sep) (e : TSyntax k) : TSepArray k sep := + if sa.elemsAndSeps.isEmpty then + { elemsAndSeps := #[e] } + else + { elemsAndSeps := sa.elemsAndSeps.push (mkAtom sep) |>.push e } + +instance : EmptyCollection (SepArray sep) where + emptyCollection := ⟨∅⟩ + +instance : EmptyCollection (TSepArray sep k) where + emptyCollection := ⟨∅⟩ + /- We use `CoeTail` here instead of `Coe` to avoid a "loop" when computing `CoeTC`. The "loop" is interrupted using the maximum instance size threshold, but it is a performance bottleneck. @@ -1094,7 +1106,8 @@ set_option linter.unusedVariables.funArgs false in For example, the tactic will *not* be invoked during type class resolution. -/ abbrev autoParam.{u} (α : Sort u) (tactic : Lean.Syntax) : Sort u := α -/- Helper functions for manipulating interpolated strings -/ +/-! # Helper functions for manipulating interpolated strings -/ + namespace Lean.Syntax private def decodeInterpStrQuotedChar (s : String) (i : String.Pos) : Option (Char × String.Pos) := do diff --git a/src/Init/Notation.lean b/src/Init/Notation.lean index ab33e4967b4f..d212fea88a2a 100644 --- a/src/Init/Notation.lean +++ b/src/Init/Notation.lean @@ -37,7 +37,7 @@ macro "lead" : prec => `(1022) -- precedence used for terms not supposed to be u macro "(" p:prec ")" : prec => return p macro "min" : prec => `(10) -- minimum precedence used in term parsers macro "min1" : prec => `(11) -- `(min+1) we can only `min+1` after `Meta.lean` -/- +/-- `max:prec` as a term. It is equivalent to `eval_prec max` for `eval_prec` defined at `Meta.lean`. We use `max_prec` to workaround bootstrapping issues. -/ macro "max_prec" : term => `(1024) @@ -61,10 +61,10 @@ macro_rules | `(stx| $p ?) => `(stx| optional($p)) | `(stx| $p₁ <|> $p₂) => `(stx| orelse($p₁, $p₂)) -/- Comma-separated sequence. -/ +/-- Comma-separated sequence. -/ macro:arg x:stx:max ",*" : stx => `(stx| sepBy($x, ",", ", ")) macro:arg x:stx:max ",+" : stx => `(stx| sepBy1($x, ",", ", ")) -/- Comma-separated sequence with optional trailing comma. -/ +/-- Comma-separated sequence with optional trailing comma. -/ macro:arg x:stx:max ",*,?" : stx => `(stx| sepBy($x, ",", ", ", allowTrailingSep)) macro:arg x:stx:max ",+,?" : stx => `(stx| sepBy1($x, ",", ", ", allowTrailingSep)) @@ -89,7 +89,7 @@ infixr:80 " ^ " => HPow.hPow infixl:65 " ++ " => HAppend.hAppend prefix:100 "-" => Neg.neg prefix:100 "~~~" => Complement.complement -/- +/-! Remark: the infix commands above ensure a delaborator is generated for each relations. We redefine the macros below to be able to use the auxiliary `binop%` elaboration helper for binary operators. It addresses issue #382. -/ @@ -101,6 +101,7 @@ macro_rules | `($x - $y) => `(binop% HSub.hSub $x $y) macro_rules | `($x * $y) => `(binop% HMul.hMul $x $y) macro_rules | `($x / $y) => `(binop% HDiv.hDiv $x $y) macro_rules | `($x % $y) => `(binop% HMod.hMod $x $y) +macro_rules | `($x ^ $y) => `(binop% HPow.hPow $x $y) macro_rules | `($x ++ $y) => `(binop% HAppend.hAppend $x $y) -- declare ASCII alternatives first so that the latter Unicode unexpander wins @@ -112,7 +113,7 @@ infix:50 " ≥ " => GE.ge infix:50 " > " => GT.gt infix:50 " = " => Eq infix:50 " == " => BEq.beq -/- +/-! Remark: the infix commands above ensure a delaborator is generated for each relations. We redefine the macros below to be able to use the auxiliary `binrel%` elaboration helper for binary relations. It has better support for applying coercions. For example, suppose we have `binrel% Eq n i` where `n : Nat` and @@ -188,7 +189,7 @@ macro_rules | `($a |> $f $args*) => `($f $args* $a) | `($a |> $f) => `($f $a) --- Haskell-like pipe <| +/-- Haskell-like pipe `<|` -/ -- Note that we have a whitespace after `$` to avoid an ambiguity with the antiquotations. syntax:min term atomic(" $" ws) term:min : term @@ -202,7 +203,7 @@ macro_rules | `({ $x : $type // $p }) => ``(Subtype (fun ($x:ident : $type) => $p)) | `({ $x // $p }) => ``(Subtype (fun ($x:ident : _) => $p)) -/- +/-- `without_expected_type t` instructs Lean to elaborate `t` without an expected type. Recall that terms such as `match ... with ...` and `⟨...⟩` will postpone elaboration until expected type is known. So, `without_expected_type` is not effective in this case. -/ diff --git a/src/Init/NotationExtra.lean b/src/Init/NotationExtra.lean index 2cf1faebf6bb..b9cc5e0e6c14 100644 --- a/src/Init/NotationExtra.lean +++ b/src/Init/NotationExtra.lean @@ -64,15 +64,15 @@ def expandBrackedBinders (combinatorDeclName : Name) (bracketedExplicitBinders : syntax unifConstraint := term (" =?= " <|> " ≟ ") term syntax unifConstraintElem := colGe unifConstraint ", "? -syntax attrKind "unif_hint " (ident)? bracketedBinder* " where " withPosition(unifConstraintElem*) ("|-" <|> "⊢ ") unifConstraint : command +syntax (docComment)? attrKind "unif_hint " (ident)? bracketedBinder* " where " withPosition(unifConstraintElem*) ("|-" <|> "⊢ ") unifConstraint : command macro_rules - | `($kind:attrKind unif_hint $(n)? $bs:bracketedBinder* where $[$cs₁:term ≟ $cs₂]* |- $t₁:term ≟ $t₂) => do + | `($[$doc?:docComment]? $kind:attrKind unif_hint $(n)? $bs* where $[$cs₁:term ≟ $cs₂]* |- $t₁:term ≟ $t₂) => do let mut body ← `($t₁ = $t₂) for (c₁, c₂) in cs₁.zip cs₂ |>.reverse do body ← `($c₁ = $c₂ → $body) let hint : Ident ← `(hint) - `(@[$kind:attrKind unificationHint] def $(n.getD hint):ident $bs:bracketedBinder* : Sort _ := $body) + `($[$doc?:docComment]? @[$kind:attrKind unificationHint] def $(n.getD hint) $bs:bracketedBinder* : Sort _ := $body) end Lean open Lean @@ -207,7 +207,7 @@ macro_rules `(let y := %[ $[$y],* | $k ] %[ $[$z],* | y ]) -/- +/-- Expands ``` class abbrev C := D_1, ..., D_n @@ -241,7 +241,7 @@ macro_rules | `(tactic| solve $[| $ts]* ) => `(tactic| focus first $[| ($ts); done]*) namespace Lean -/- `repeat` and `while` notation -/ +/-! # `repeat` and `while` notation -/ inductive Loop where | mk @@ -262,6 +262,11 @@ syntax "repeat " doSeq : doElem macro_rules | `(doElem| repeat $seq) => `(doElem| for _ in Loop.mk do $seq) +syntax "while " ident " : " termBeforeDo " do " doSeq : doElem + +macro_rules + | `(doElem| while $h : $cond do $seq) => `(doElem| repeat if $h : $cond then $seq else break) + syntax "while " termBeforeDo " do " doSeq : doElem macro_rules diff --git a/src/Init/Prelude.lean b/src/Init/Prelude.lean index 01c00a93d81e..507fca5fc4ab 100644 --- a/src/Init/Prelude.lean +++ b/src/Init/Prelude.lean @@ -86,9 +86,9 @@ theorem congr {α : Sort u} {β : Sort v} {f₁ f₂ : α → β} {a₁ a₂ : theorem congrFun {α : Sort u} {β : α → Sort v} {f g : (x : α) → β x} (h : Eq f g) (a : α) : Eq (f a) (g a) := h ▸ rfl -/- +/-! Initialize the Quotient Module, which effectively adds the following definitions: - +``` opaque Quot {α : Sort u} (r : α → α → Prop) : Sort u opaque Quot.mk {α : Sort u} (r : α → α → Prop) (a : α) : Quot r @@ -98,6 +98,7 @@ opaque Quot.lift {α : Sort u} {r : α → α → Prop} {β : Sort v} (f : α opaque Quot.ind {α : Sort u} {r : α → α → Prop} {β : Quot r → Prop} : (∀ a : α, β (Quot.mk r a)) → ∀ q : Quot r, β q +``` -/ init_quot @@ -156,7 +157,7 @@ inductive Bool : Type where export Bool (false true) -/- Remark: Subtype must take a Sort instead of Type because of the axiom strongIndefiniteDescription. -/ +/-- Remark: Subtype must take a Sort instead of Type because of the axiom strongIndefiniteDescription. -/ structure Subtype {α : Sort u} (p : α → Prop) where val : α property : p val @@ -175,7 +176,7 @@ set_option linter.unusedVariables.funArgs false in /-- Auxiliary Declaration used to implement the named patterns `x@h:p` -/ @[reducible] def namedPattern {α : Sort u} (x a : α) (h : Eq x a) : α := a -/- Auxiliary axiom used to implement `sorry`. -/ +/-- Auxiliary axiom used to implement `sorry`. -/ @[extern "lean_sorry", neverExtract] axiom sorryAx (α : Sort u) (synthetic := false) : α @@ -236,14 +237,14 @@ deriving instance Inhabited for Bool structure PLift (α : Sort u) : Type u where up :: (down : α) -/- Bijection between α and PLift α -/ +/-- Bijection between α and PLift α -/ theorem PLift.up_down {α : Sort u} : ∀ (b : PLift α), Eq (up (down b)) b | up _ => rfl theorem PLift.down_up {α : Sort u} (a : α) : Eq (down (up a)) a := rfl -/- Pointed types -/ +/-- Pointed types -/ def NonemptyType := Subtype fun α : Type u => Nonempty α abbrev NonemptyType.type (type : NonemptyType.{u}) : Type u := @@ -256,7 +257,7 @@ instance : Inhabited NonemptyType.{u} where structure ULift.{r, s} (α : Type s) : Type (max s r) where up :: (down : α) -/- Bijection between α and ULift.{v} α -/ +/-- Bijection between α and ULift.{v} α -/ theorem ULift.up_down {α : Type u} : ∀ (b : ULift.{v} α), Eq (up (down b)) b | up _ => rfl @@ -316,6 +317,7 @@ theorem of_decide_eq_self_eq_true [inst : DecidableEq α] (a : α) : Eq (decide | true, true => isTrue rfl class BEq (α : Type u) where + /-- Boolean equality. -/ beq : α → α → Bool open BEq (beq) @@ -328,7 +330,7 @@ instance [DecidableEq α] : BEq α where @[macroInline] def dite {α : Sort u} (c : Prop) [h : Decidable c] (t : c → α) (e : Not c → α) : α := Decidable.casesOn (motive := fun _ => α) h e t -/- if-then-else -/ +/-! # if-then-else -/ @[macroInline] def ite {α : Sort u} (c : Prop) [h : Decidable c] (t e : α) : α := Decidable.casesOn (motive := fun _ => α) h (fun _ => e) (fun _ => t) @@ -358,7 +360,7 @@ instance [dp : Decidable p] : Decidable (Not p) := | isTrue hp => isFalse (absurd hp) | isFalse hp => isTrue hp -/- Boolean operators -/ +/-! # Boolean operators -/ @[macroInline] def cond {α : Type u} (c : Bool) (x y : α) : α := match c with @@ -379,6 +381,7 @@ instance [dp : Decidable p] : Decidable (Not p) := | true => false | false => true +/-- The type of natural numbers. `0`, `1`, `2`, ...-/ inductive Nat where | zero : Nat | succ (n : Nat) : Nat @@ -386,7 +389,7 @@ inductive Nat where instance : Inhabited Nat where default := Nat.zero -/- For numeric literals notation -/ +/-- For numeric literals notation -/ class OfNat (α : Type u) (_ : Nat) where ofNat : α @@ -799,12 +802,15 @@ instance : Sub Nat where @[extern "lean_system_platform_nbits"] opaque System.Platform.getNumBits : Unit → Subtype fun (n : Nat) => Or (Eq n 32) (Eq n 64) := fun _ => ⟨64, Or.inr rfl⟩ -- inhabitant +/-- Gets the word size of the platform. +That is, whether the platform is 64 or 32 bits. -/ def System.Platform.numBits : Nat := (getNumBits ()).val theorem System.Platform.numBits_eq : Or (Eq numBits 32) (Eq numBits 64) := (getNumBits ()).property +/-- `Fin n` is a natural number `i` with the constraint that `0 ≤ i < n`. -/ structure Fin (n : Nat) where val : Nat isLt : LT.lt val n @@ -834,6 +840,7 @@ instance Fin.decLt {n} (a b : Fin n) : Decidable (LT.lt a b) := Nat.decLt .. instance Fin.decLe {n} (a b : Fin n) : Decidable (LE.le a b) := Nat.decLe .. def UInt8.size : Nat := 256 +/-- Unsigned 8-bit integer. -/ structure UInt8 where val : Fin UInt8.size @@ -858,6 +865,7 @@ instance : Inhabited UInt8 where default := UInt8.ofNatCore 0 (by decide) def UInt16.size : Nat := 65536 +/-- Unsigned 16-bit integer. -/ structure UInt16 where val : Fin UInt16.size @@ -882,6 +890,7 @@ instance : Inhabited UInt16 where default := UInt16.ofNatCore 0 (by decide) def UInt32.size : Nat := 4294967296 +/-- Unsigned, 32-bit integer. -/ structure UInt32 where val : Fin UInt32.size @@ -930,6 +939,7 @@ instance (a b : UInt32) : Decidable (LT.lt a b) := UInt32.decLt a b instance (a b : UInt32) : Decidable (LE.le a b) := UInt32.decLe a b def UInt64.size : Nat := 18446744073709551616 +/-- Unsigned, 64-bit integer. -/ structure UInt64 where val : Fin UInt64.size @@ -961,6 +971,12 @@ theorem usize_size_eq : Or (Eq USize.size 4294967296) (Eq USize.size 18446744073 | _, Or.inl rfl => Or.inl (by decide) | _, Or.inr rfl => Or.inr (by decide) +/-- A USize is an unsigned integer with the size of a word +for the platform's architecture. + +For example, if running on a 32-bit machine, USize is equivalent to UInt32. +Or on a 64-bit machine, UInt64. +-/ structure USize where val : Fin USize.size @@ -1214,7 +1230,7 @@ unsafe def unsafeCast {α : Sort u} {β : Sort v} (a : α) : β := @[neverExtract, extern "lean_panic_fn"] opaque panicCore {α : Type u} [Inhabited α] (msg : String) : α -/- +/-- This is workaround for `panic` occurring in monadic code. See issue #695. The `panicCore` definition cannot be specialized since it is an extern. When `panic` occurs in monadic code, the `Inhabited α` parameter depends on a `[inst : Monad m]` instance. @@ -1234,7 +1250,7 @@ class GetElem (Cont : Type u) (Idx : Type v) (Elem : outParam (Type w)) (Dom : o export GetElem (getElem) -/- +/-- The Compiler has special support for arrays. They are implemented using dynamic arrays: https://en.wikipedia.org/wiki/Dynamic_array -/ @@ -1244,7 +1260,7 @@ structure Array (α : Type u) where attribute [extern "lean_array_data"] Array.data attribute [extern "lean_array_mk"] Array.mk -/- The parameter `c` is the initial capacity -/ +/-- The parameter `c` is the initial capacity -/ @[extern "lean_mk_empty_array_with_capacity"] def Array.mkEmpty {α : Type u} (c : @& Nat) : Array α := { data := List.nil @@ -1264,7 +1280,7 @@ def Array.get {α : Type u} (a : @& Array α) (i : @& Fin a.size) : α := @[inline] abbrev Array.getD (a : Array α) (i : Nat) (v₀ : α) : α := dite (LT.lt i a.size) (fun h => a.get ⟨i, h⟩) (fun _ => v₀) -/- "Comfortable" version of `fget`. It performs a bound check at runtime. -/ +/-- "Comfortable" version of `fget`. It performs a bound check at runtime. -/ @[extern "lean_array_get"] def Array.get! {α : Type u} [Inhabited α] (a : @& Array α) (i : @& Nat) : α := Array.getD a i default @@ -1562,14 +1578,14 @@ instance {ρ : Type u} {m : Type u → Type v} [Monad m] : MonadWithReaderOf ρ In contrast to the Haskell implementation, we use overlapping instances to derive instances automatically from `monadLift`. -/ class MonadStateOf (σ : Type u) (m : Type u → Type v) where - /- Obtain the top-most State of a Monad stack. -/ + /-- Obtain the top-most State of a Monad stack. -/ get : m σ - /- Set the top-most State of a Monad stack. -/ + /-- Set the top-most State of a Monad stack. -/ set : σ → m PUnit - /- Map the top-most State of a Monad stack. + /-- Map the top-most State of a Monad stack. - Note: `modifyGet f` may be preferable to `do s <- get; let (a, s) := f s; put s; pure a` - because the latter does not use the State linearly (without sufficient inlining). -/ + Note: `modifyGet f` may be preferable to `do s <- get; let (a, s) := f s; put s; pure a` + because the latter does not use the State linearly (without sufficient inlining). -/ modifyGet {α : Type u} : (σ → Prod α σ) → m α export MonadStateOf (set) @@ -1715,7 +1731,7 @@ instance {δ} [Backtrackable δ σ] : MonadExceptOf ε (EStateM ε σ) where @[inline] def dummyRestore : σ → PUnit → σ := fun s _ => s -/- Dummy default instance -/ +/-- Dummy default instance -/ instance nonBacktrackable : Backtrackable PUnit σ where save := dummySave restore := dummyRestore @@ -1744,11 +1760,40 @@ instance : Hashable String where namespace Lean -/- Hierarchical names -/ +/-- +Hierarchical names. We use hierarchical names to name declarations and +for creating unique identifiers for free variables and metavariables. + +You can create hierarchical names using the following quotation notation. +``` +`Lean.Meta.whnf +``` +It is short for `.str (.str (.str .anonymous "Lean") "Meta") "whnf"` +You can use double quotes to request Lean to statically check whether the name +corresponds to a Lean declaration in scope. +``` +``Lean.Meta.whnf +``` +If the name is not in scope, Lean will report an error. +-/ inductive Name where - | anonymous : Name - | str : Name → String → Name - | num : Name → Nat → Name + | /-- The "anonymous" name. -/ + anonymous : Name + | /-- +A string name. The name `Lean.Meta.run` is represented at +```lean +.str (.str (.str .anonymous "Lean") "Meta") "run" +``` +-/ + str (pre : Name) (str : String) + | /-- +A numerical name. This kind of name is used, for example, to create hierarchical names for +free variables and metavariables. The identifier `_uniq.231` is represented as +```lean +.num (.str .anonymous "_uniq") 231 +``` +-/ + num (pre : Name) (i : Nat) with @[computedField] hash : Name → UInt64 | .anonymous => .ofNatCore 1723 (by decide) @@ -1763,14 +1808,23 @@ instance : Hashable Name where namespace Name +/-- +`.str p s` is now the preferred form. +-/ @[export lean_name_mk_string] abbrev mkStr (p : Name) (s : String) : Name := Name.str p s +/-- +`.num p v` is now the preferred form. +-/ @[export lean_name_mk_numeral] abbrev mkNum (p : Name) (v : Nat) : Name := Name.num p v +/-- +Short for `.str .anonymous s`. +-/ abbrev mkSimple (s : String) : Name := mkStr Name.anonymous s @@ -1784,6 +1838,13 @@ protected def beq : (@& Name) → (@& Name) → Bool instance : BEq Name where beq := Name.beq +/-- +Append two hierarchical names. Example: +```lean +`Lean.Meta ++ `Tactic.simp +``` +return `Lean.Meta.Tactic.simp` +-/ protected def append : Name → Name → Name | n, anonymous => n | n, str p s => Name.mkStr (Name.append n p) s @@ -1794,22 +1855,26 @@ instance : Append Name where end Name -/- Syntax -/ +/-! # Syntax -/ /-- Source information of tokens. -/ inductive SourceInfo where - /- + | /-- Token from original input with whitespace and position information. `leading` will be inferred after parsing by `Syntax.updateLeading`. During parsing, - it is not at all clear what the preceding token was, especially with backtracking. -/ - | original (leading : Substring) (pos : String.Pos) (trailing : Substring) (endPos : String.Pos) - /- + it is not at all clear what the preceding token was, especially with backtracking. + -/ + original (leading : Substring) (pos : String.Pos) (trailing : Substring) (endPos : String.Pos) + | /-- Synthesized token (e.g. from a quotation) annotated with a span from the original source. In the delaborator, we "misuse" this constructor to store synthetic positions identifying - subterms. -/ - | synthetic (pos : String.Pos) (endPos : String.Pos) - /- Synthesized token without position information. -/ - | protected none + subterms. + -/ + synthetic (pos : String.Pos) (endPos : String.Pos) + | /-- + Synthesized token without position information. + -/ + protected none instance : Inhabited SourceInfo := ⟨SourceInfo.none⟩ @@ -1825,7 +1890,7 @@ end SourceInfo abbrev SyntaxNodeKind := Name -/- Syntax AST -/ +/-! # Syntax AST -/ /-- Syntax objects used by the parser, macro expander, delaborator, etc. @@ -1833,36 +1898,37 @@ Syntax objects used by the parser, macro expander, delaborator, etc. inductive Syntax where | missing : Syntax | /-- - Node in the syntax tree. - - The `info` field is used by the delaborator - to store the position of the subexpression - corresponding to this node. - The parser sets the `info` field to `none`. - - (Remark: the `node` constructor - did not have an `info` field in previous versions. - This caused a bug in the interactive widgets, - where the popup for `a + b` was the same as for `a`. - The delaborator used to associate subexpressions - with pretty-printed syntax by setting - the (string) position of the first atom/identifier - to the (expression) position of the subexpression. - For example, both `a` and `a + b` - have the same first identifier, - and so their infos got mixed up.) - -/ node (info : SourceInfo) (kind : SyntaxNodeKind) (args : Array Syntax) : Syntax + Node in the syntax tree. + + The `info` field is used by the delaborator + to store the position of the subexpression + corresponding to this node. + The parser sets the `info` field to `none`. + + (Remark: the `node` constructor + did not have an `info` field in previous versions. + This caused a bug in the interactive widgets, + where the popup for `a + b` was the same as for `a`. + The delaborator used to associate subexpressions + with pretty-printed syntax by setting + the (string) position of the first atom/identifier + to the (expression) position of the subexpression. + For example, both `a` and `a + b` + have the same first identifier, + and so their infos got mixed up.) + -/ + node (info : SourceInfo) (kind : SyntaxNodeKind) (args : Array Syntax) : Syntax | atom (info : SourceInfo) (val : String) : Syntax | ident (info : SourceInfo) (rawVal : Substring) (val : Name) (preresolved : List (Prod Name (List String))) : Syntax def SyntaxNodeKinds := List SyntaxNodeKind /-- - A `Syntax` value of one of the given syntax kinds. - Note that while syntax quotations produce/expect `TSyntax` values of the correct kinds, - this is not otherwise enforced and can easily be circumvented by direct use of the constructor. - The namespace `TSyntax.Compat` can be opened to expose a general coercion from `Syntax` to any - `TSyntax ks` for porting older code. -/ +A `Syntax` value of one of the given syntax kinds. +Note that while syntax quotations produce/expect `TSyntax` values of the correct kinds, +this is not otherwise enforced and can easily be circumvented by direct use of the constructor. +The namespace `TSyntax.Compat` can be opened to expose a general coercion from `Syntax` to any +`TSyntax ks` for porting older code. -/ structure TSyntax (ks : SyntaxNodeKinds) where raw : Syntax @@ -1872,7 +1938,7 @@ instance : Inhabited Syntax where instance : Inhabited (TSyntax ks) where default := ⟨default⟩ -/- Builtin kinds -/ +/-! Builtin kinds -/ abbrev choiceKind : SyntaxNodeKind := `choice abbrev nullKind : SyntaxNodeKind := `null abbrev groupKind : SyntaxNodeKind := `group @@ -2033,7 +2099,7 @@ def mkAtom (val : String) : Syntax := def mkAtomFrom (src : Syntax) (val : String) : Syntax := Syntax.atom (SourceInfo.fromRef src) val -/- Parser descriptions -/ +/-! # Parser descriptions -/ inductive ParserDescr where | const (name : Name) @@ -2054,7 +2120,7 @@ instance : Inhabited ParserDescr where abbrev TrailingParserDescr := ParserDescr -/- +/-! Runtime support for making quotation terms auto-hygienic, by mangling identifiers introduced by them with a "macro scope" supplied by the context. Details to appear in a paper soon. @@ -2095,10 +2161,11 @@ def replaceRef (ref : Syntax) (oldRef : Syntax) : Syntax := introduced symbol, which results in better error positions than not applying any position. -/ class MonadQuotation (m : Type → Type) extends MonadRef m where - -- Get the fresh scope of the current macro invocation + /-- Get the fresh scope of the current macro invocation -/ getCurrMacroScope : m MacroScope getMainModule : m Name - /- Execute action in a new macro invocation context. This transformer should be + /-- + Execute action in a new macro invocation context. This transformer should be used at all places that morally qualify as the beginning of a "macro call", e.g. `elabCommand` and `elabTerm` in the case of the elaborator. However, it can also be used internally inside a "macro" if identifiers introduced by @@ -2121,7 +2188,7 @@ instance {m n : Type → Type} [MonadFunctor m n] [MonadLift m n] [MonadQuotatio getMainModule := liftM (m := m) getMainModule withFreshMacroScope := monadMap (m := m) withFreshMacroScope -/- +/-! We represent a name with macro scopes as ``` ._@.(.)*.._hyg. @@ -2164,7 +2231,7 @@ private def simpMacroScopesAux : Name → Name | .num p i => Name.mkNum (simpMacroScopesAux p) i | n => eraseMacroScopesAux n -/- Helper function we use to create binder names that do not need to be unique. -/ +/-- Helper function we use to create binder names that do not need to be unique. -/ @[export lean_simp_macro_scopes] def Name.simpMacroScopes (n : Name) : Name := match n.hasMacroScopes with @@ -2275,7 +2342,7 @@ end Syntax namespace Macro -/- References -/ +/-- References -/ private opaque MethodsRefPointed : NonemptyType.{0} private def MethodsRef : Type := MethodsRefPointed.type diff --git a/src/Init/SizeOf.lean b/src/Init/SizeOf.lean index 17682469ec85..2aaf0e889123 100644 --- a/src/Init/SizeOf.lean +++ b/src/Init/SizeOf.lean @@ -6,19 +6,19 @@ Authors: Leonardo de Moura prelude import Init.Tactics -/- SizeOf -/ +/-! # SizeOf -/ class SizeOf (α : Sort u) where sizeOf : α → Nat export SizeOf (sizeOf) -/- +/-! Declare sizeOf instances and theorems for types declared before SizeOf. From now on, the inductive Compiler will automatically generate sizeOf instances and theorems. -/ -/- Every Type `α` has a default SizeOf instance that just returns 0 for every element of `α` -/ +/-- Every Type `α` has a default SizeOf instance that just returns 0 for every element of `α` -/ protected def default.sizeOf (α : Sort u) : α → Nat | _ => 0 @@ -62,7 +62,7 @@ deriving instance SizeOf for EStateM.Result namespace Lean -/- We manually define `Lean.Name` instance because we use +/-- We manually define `Lean.Name` instance because we use an opaque function for computing the hashcode field. -/ protected noncomputable def Name.sizeOf : Name → Nat | anonymous => 1 diff --git a/src/Init/System/IO.lean b/src/Init/System/IO.lean index 1e62b8e42d5b..1919b54d671e 100644 --- a/src/Init/System/IO.lean +++ b/src/Init/System/IO.lean @@ -91,7 +91,7 @@ set_option compiler.extract_closed false in @[extern "lean_io_timeit"] opaque timeit (msg : @& String) (fn : IO α) : IO α @[extern "lean_io_allocprof"] opaque allocprof (msg : @& String) (fn : IO α) : IO α -/- Programs can execute IO actions during initialization that occurs before +/-- Programs can execute IO actions during initialization that occurs before the `main` function is executed. The attribute `[init ]` specifies which IO action is executed to set the value of an opaque constant. @@ -511,21 +511,21 @@ def Stdio.toHandleType : Stdio → Type | Stdio.null => Unit structure StdioConfig where - /- Configuration for the process' stdin handle. -/ + /-- Configuration for the process' stdin handle. -/ stdin := Stdio.inherit - /- Configuration for the process' stdout handle. -/ + /-- Configuration for the process' stdout handle. -/ stdout := Stdio.inherit - /- Configuration for the process' stderr handle. -/ + /-- Configuration for the process' stderr handle. -/ stderr := Stdio.inherit structure SpawnArgs extends StdioConfig where - /- Command name. -/ + /-- Command name. -/ cmd : String - /- Arguments for the process -/ + /-- Arguments for the process -/ args : Array String := #[] - /- Working directory for the process. Inherit from current process if `none`. -/ + /-- Working directory for the process. Inherit from current process if `none`. -/ cwd : Option FilePath := none - /- Add or remove environment variables for the process. -/ + /-- Add or remove environment variables for the process. -/ env : Array (String × Option String) := #[] -- TODO(Sebastian): constructor must be private @@ -599,7 +599,7 @@ def FileRight.flags (acc : FileRight) : UInt32 := def setAccessRights (filename : FilePath) (mode : FileRight) : IO Unit := Prim.setAccessRights filename mode.flags -/- References -/ +/-- References -/ abbrev Ref (α : Type) := ST.Ref IO.RealWorld α instance : MonadLift (ST IO.RealWorld) BaseIO := ⟨id⟩ diff --git a/src/Init/System/IOError.lean b/src/Init/System/IOError.lean index 91229e0702c3..63ad083a02c1 100644 --- a/src/Init/System/IOError.lean +++ b/src/Init/System/IOError.lean @@ -10,7 +10,7 @@ import Init.Data.UInt import Init.Data.ToString.Basic import Init.Data.String.Basic -/- +/-- Imitate the structure of IOErrorType in Haskell: https://hackage.haskell.org/package/base-4.12.0.0/docs/System-IO-Error.html#t:IOErrorType -/ diff --git a/src/Init/System/ST.lean b/src/Init/System/ST.lean index f5550bcb5667..106dd06704cd 100644 --- a/src/Init/System/ST.lean +++ b/src/Init/System/ST.lean @@ -41,7 +41,7 @@ instance {ε σ} : MonadLift (ST σ) (EST ε σ) := ⟨fun x s => namespace ST -/- References -/ +/-- References -/ opaque RefPointed : NonemptyType.{0} structure Ref (σ : Type) (α : Type) : Type where @@ -53,7 +53,7 @@ instance {σ α} [s : Nonempty α] : Nonempty (Ref σ α) := namespace Prim -/- Auxiliary definition for showing that `ST σ α` is inhabited when we have a `Ref σ α` -/ +/-- Auxiliary definition for showing that `ST σ α` is inhabited when we have a `Ref σ α` -/ private noncomputable def inhabitedFromRef {σ α} (r : Ref σ α) : ST σ α := let _ : Inhabited α := Classical.inhabited_of_nonempty r.h pure default diff --git a/src/Init/Util.lean b/src/Init/Util.lean index 2902ce958628..d023c2c784b2 100644 --- a/src/Init/Util.lean +++ b/src/Init/Util.lean @@ -10,14 +10,15 @@ import Init.Data.ToString.Basic universe u v set_option linter.unusedVariables.funArgs false -/- debugging helper functions -/ +/-! # Debugging helper functions -/ + @[neverExtract, extern "lean_dbg_trace"] def dbgTrace {α : Type u} (s : String) (f : Unit → α) : α := f () def dbgTraceVal {α : Type u} [ToString α] (a : α) : α := dbgTrace (toString a) (fun _ => a) -/- Display the given message if `a` is shared, that is, RC(a) > 1 -/ +/-- Display the given message if `a` is shared, that is, RC(a) > 1 -/ @[neverExtract, extern "lean_dbg_trace_if_shared"] def dbgTraceIfShared {α : Type u} (s : String) (a : α) : α := a @@ -42,8 +43,15 @@ unsafe def ptrAddrUnsafe {α : Type u} (a : @& α) : USize := 0 @[inline] unsafe def withPtrAddrUnsafe {α : Type u} {β : Type v} (a : α) (k : USize → β) (h : ∀ u₁ u₂, k u₁ = k u₂) : β := k (ptrAddrUnsafe a) +@[inline] unsafe def ptrEq (a b : α) : Bool := ptrAddrUnsafe a == ptrAddrUnsafe b + +unsafe def ptrEqList : (as bs : List α) → Bool + | [], [] => true + | a::as, b::bs => if ptrEq a b then ptrEqList as bs else false + | _, _ => false + @[inline] unsafe def withPtrEqUnsafe {α : Type u} (a b : α) (k : Unit → Bool) (h : a = b → k () = true) : Bool := - if ptrAddrUnsafe a == ptrAddrUnsafe b then true else k () + if ptrEq a b then true else k () @[implementedBy withPtrEqUnsafe] def withPtrEq {α : Type u} (a b : α) (k : Unit → Bool) (h : a = b → k () = true) : Bool := k () diff --git a/src/Lean/Attributes.lean b/src/Lean/Attributes.lean index 946f0e53c0e2..6bdb1875cfe1 100644 --- a/src/Lean/Attributes.lean +++ b/src/Lean/Attributes.lean @@ -24,6 +24,17 @@ structure AttributeImplCore where applicationTime := AttributeApplicationTime.afterTypeChecking deriving Inhabited +/-- You can tag attributes with the 'local' or 'scoped' kind. +For example: `attribute [local myattr, scoped yourattr, theirattr]`. + +This is used to indicate how an attribute should be scoped. +- local means that the attribute should only be applied in the current scope and forgotten once the current section, namespace, or file is closed. +- scoped means that the attribute should only be applied while the namespace is open. +- global means that the attribute should always be applied. + +Note that the attribute handler (`AttributeImpl.add`) is responsible for interpreting the kind and +making sure that these kinds are respected. +-/ inductive AttributeKind | «global» | «local» | «scoped» deriving BEq, Inhabited @@ -44,7 +55,7 @@ open Std (PersistentHashMap) builtin_initialize attributeMapRef : IO.Ref (PersistentHashMap Name AttributeImpl) ← IO.mkRef {} -/- Low level attribute registration function. -/ +/-- Low level attribute registration function. -/ def registerBuiltinAttribute (attr : AttributeImpl) : IO Unit := do let m ← attributeMapRef.get if m.contains attr.name then throw (IO.userError ("invalid builtin attribute declaration, '" ++ toString attr.name ++ "' has already been used")) @@ -52,7 +63,7 @@ def registerBuiltinAttribute (attr : AttributeImpl) : IO Unit := do throw (IO.userError "failed to register attribute, attributes can only be registered during initialization") attributeMapRef.modify fun m => m.insert attr.name attr -/- +/-! Helper methods for decoding the parameters of builtin attributes that are defined before `Lean.Parser`. We have the following ones: ``` @@ -224,7 +235,7 @@ def setParam {α : Type} (attr : ParametricAttribute α) (env : Environment) (de end ParametricAttribute -/- +/-- Given a list `[a₁, ..., a_n]` of elements of type `α`, `EnumAttributes` provides an attribute `Attr_i` for associating a value `a_i` with an declaration. `α` is usually an enumeration type. Note that whenever we register an `EnumAttributes`, we create `n` attributes, but only one environment extension. -/ @@ -283,7 +294,7 @@ def setValue {α : Type} (attrs : EnumAttributes α) (env : Environment) (decl : end EnumAttributes -/- +/-! Attribute extension and builders. We use builders to implement attribute factories for parser categories. -/ @@ -360,12 +371,12 @@ builtin_initialize attributeExtension : AttributeExtension ← statsFn := fun s => format "number of local entries: " ++ format s.newEntries.length } -/- Return true iff `n` is the name of a registered attribute. -/ +/-- Return true iff `n` is the name of a registered attribute. -/ @[export lean_is_attribute] def isBuiltinAttribute (n : Name) : IO Bool := do let m ← attributeMapRef.get; pure (m.contains n) -/- Return the name of all registered attributes. -/ +/-- Return the name of all registered attributes. -/ def getBuiltinAttributeNames : IO (List Name) := return (← attributeMapRef.get).foldl (init := []) fun r n _ => n::r diff --git a/src/Lean/Class.lean b/src/Lean/Class.lean index e63eca064271..eb1642ac1823 100644 --- a/src/Lean/Class.lean +++ b/src/Lean/Class.lean @@ -8,8 +8,16 @@ import Lean.Attributes namespace Lean structure ClassEntry where - name : Name - hasOutParam : Bool + name : Name + /-- + Position of the class `outParams`. + For example, for class + ``` + class GetElem (Cont : Type u) (Idx : Type v) (Elem : outParam (Type w)) (Dom : outParam (Cont → Idx → Prop)) where + ``` + `outParams := #[2, 3]` + -/ + outParams : Array Nat namespace ClassEntry @@ -19,16 +27,16 @@ def lt (a b : ClassEntry) : Bool := end ClassEntry structure ClassState where - hasOutParam : SMap Name Bool := SMap.empty + outParamMap : SMap Name (Array Nat) := SMap.empty deriving Inhabited namespace ClassState def addEntry (s : ClassState) (entry : ClassEntry) : ClassState := - { s with hasOutParam := s.hasOutParam.insert entry.name entry.hasOutParam } + { s with outParamMap := s.outParamMap.insert entry.name entry.outParams } def switch (s : ClassState) : ClassState := - { s with hasOutParam := s.hasOutParam.switch } + { s with outParamMap := s.outParamMap.switch } end ClassState @@ -42,17 +50,23 @@ builtin_initialize classExtension : SimplePersistentEnvExtension ClassEntry Clas @[export lean_is_class] def isClass (env : Environment) (n : Name) : Bool := - (classExtension.getState env).hasOutParam.contains n + (classExtension.getState env).outParamMap.contains n + +/-- + If `declName` is a class, return the position of its `outParams`. +-/ +def getOutParamPositions? (env : Environment) (declName : Name) : Option (Array Nat) := + (classExtension.getState env).outParamMap.find? declName @[export lean_has_out_params] -def hasOutParams (env : Environment) (n : Name) : Bool := - match (classExtension.getState env).hasOutParam.find? n with - | some b => b - | none => false +def hasOutParams (env : Environment) (declName : Name) : Bool := + match getOutParamPositions? env declName with + | some outParams => !outParams.isEmpty + | none => false /-- - Auxiliary function for checking whether a class has `outParam`, and - whether they are being correctly used. + Auxiliary function for collection the position class `outParams`, and + checking whether they are being correctly used. A regular (i.e., non `outParam`) must not depend on an `outParam`. Reason for this restriction: When performing type class resolution, we replace arguments that @@ -62,19 +76,19 @@ def hasOutParams (env : Environment) (n : Name) : Bool := incorrect. This transformation would be counterintuitive to users since we would implicitly treat these regular parameters as `outParam`s. -/ -private partial def checkOutParam : Nat → Array FVarId → Expr → Except String Bool - | i, outParams, Expr.forallE _ d b _ => +private partial def checkOutParam (i : Nat) (outParamFVarIds : Array FVarId) (outParams : Array Nat) (type : Expr) : Except String (Array Nat) := + match type with + | .forallE _ d b _ => if d.isOutParam then - let fvarId := { name := Name.mkNum `_fvar outParams.size } - let outParams := outParams.push fvarId + let fvarId := { name := Name.mkNum `_fvar outParamFVarIds.size } let fvar := mkFVar fvarId let b := b.instantiate1 fvar - checkOutParam (i+1) outParams b - else if d.hasAnyFVar fun fvarId => outParams.contains fvarId then - Except.error s!"invalid class, parameter #{i} depends on `outParam`, but it is not an `outParam`" + checkOutParam (i+1) (outParamFVarIds.push fvarId) (outParams.push i) b + else if d.hasAnyFVar fun fvarId => outParamFVarIds.contains fvarId then + Except.error s!"invalid class, parameter #{i+1} depends on `outParam`, but it is not an `outParam`" else - checkOutParam (i+1) outParams b - | _, outParams, _ => pure (outParams.size > 0) + checkOutParam (i+1) outParamFVarIds outParams b + | _ => return outParams def addClass (env : Environment) (clsName : Name) : Except String Environment := do if isClass env clsName then @@ -83,17 +97,17 @@ def addClass (env : Environment) (clsName : Name) : Except String Environment := | throw s!"unknown declaration '{clsName}'" unless decl matches .inductInfo .. | .axiomInfo .. do throw s!"invalid 'class', declaration '{clsName}' must be inductive datatype, structure, or constant" - let b ← checkOutParam 1 #[] decl.type - return classExtension.addEntry env { name := clsName, hasOutParam := b } + let outParams ← checkOutParam 0 #[] #[] decl.type + return classExtension.addEntry env { name := clsName, outParams } private def consumeNLambdas : Nat → Expr → Option Expr - | 0, e => some e - | i+1, Expr.lam _ _ b _ => consumeNLambdas i b - | _, _ => none + | 0, e => some e + | i+1, .lam _ _ b _ => consumeNLambdas i b + | _, _ => none partial def getClassName (env : Environment) : Expr → Option Name - | Expr.forallE _ _ b _ => getClassName env b - | e => do + | .forallE _ _ b _ => getClassName env b + | e => do let Expr.const c _ ← pure e.getAppFn | none let info ← env.find? c match info.value? with @@ -106,8 +120,8 @@ partial def getClassName (env : Environment) : Expr → Option Name builtin_initialize registerBuiltinAttribute { - name := `class, - descr := "type class", + name := `class + descr := "type class" add := fun decl stx kind => do let env ← getEnv Attribute.Builtin.ensureNoArgs stx diff --git a/src/Lean/Compiler/ConstFolding.lean b/src/Lean/Compiler/ConstFolding.lean index f249789bc17d..350663d9a0e6 100644 --- a/src/Lean/Compiler/ConstFolding.lean +++ b/src/Lean/Compiler/ConstFolding.lean @@ -6,7 +6,7 @@ Authors: Leonardo de Moura import Lean.Expr import Lean.Compiler.Util -/- Constant folding for primitives that have special runtime support. -/ +/-! Constant folding for primitives that have special runtime support. -/ namespace Lean.Compiler diff --git a/src/Lean/Compiler/ExternAttr.lean b/src/Lean/Compiler/ExternAttr.lean index 3095d13e538a..8e456e088738 100644 --- a/src/Lean/Compiler/ExternAttr.lean +++ b/src/Lean/Compiler/ExternAttr.lean @@ -17,7 +17,7 @@ inductive ExternEntry where | standard (backend : Name) (fn : String) | foreign (backend : Name) (fn : String) -/- +/-- - `@[extern]` encoding: ```.entries = [adhoc `all]``` - `@[extern "level_hash"]` @@ -123,7 +123,7 @@ def getExternEntryFor (d : ExternAttrData) (backend : Name) : Option ExternEntry def isExtern (env : Environment) (fn : Name) : Bool := getExternAttrData env fn |>.isSome -/- We say a Lean function marked as `[extern ""]` is for all backends, and it is implemented using `extern "C"`. +/-- We say a Lean function marked as `[extern ""]` is for all backends, and it is implemented using `extern "C"`. Thus, there is no name mangling. -/ def isExternC (env : Environment) (fn : Name) : Bool := match getExternAttrData env fn with diff --git a/src/Lean/Compiler/IR/Basic.lean b/src/Lean/Compiler/IR/Basic.lean index 16199b9730b9..2702889daa8e 100644 --- a/src/Lean/Compiler/IR/Basic.lean +++ b/src/Lean/Compiler/IR/Basic.lean @@ -7,7 +7,7 @@ import Lean.Data.KVMap import Lean.Data.Name import Lean.Data.Format import Lean.Compiler.ExternAttr -/- +/-! Implements (extended) λPure and λRc proposed in the article "Counting Immutable Beans", Sebastian Ullrich and Leonardo de Moura. @@ -17,15 +17,15 @@ above are implemented in Lean. -/ namespace Lean.IR -/- Function identifier -/ +/-- Function identifier -/ abbrev FunId := Name abbrev Index := Nat -/- Variable identifier -/ +/-- Variable identifier -/ structure VarId where idx : Index deriving Inhabited -/- Join point identifier -/ +/-- Join point identifier -/ structure JoinPointId where idx : Index deriving Inhabited @@ -45,7 +45,7 @@ instance : Hashable JoinPointId := ⟨fun a => hash a.idx⟩ abbrev MData := KVMap abbrev MData.empty : MData := {} -/- Low Level IR types. Most are self explanatory. +/-- Low Level IR types. Most are self explanatory. - `usize` represents the C++ `size_t` Type. We have it here because it is 32-bit in 32-bit machines, and 64-bit in 64-bit machines, @@ -130,7 +130,7 @@ def isUnion : IRType → Bool end IRType -/- Arguments to applications, constructors, etc. +/-- Arguments to applications, constructors, etc. We use `irrelevant` for Lean types, propositions and proofs that have been erased. Recall that for a Function `f`, we also generate `f._rarg` which does not take `irrelevant` arguments. However, `f._rarg` is only safe to be used in full applications. -/ @@ -159,7 +159,7 @@ def LitVal.beq : LitVal → LitVal → Bool instance : BEq LitVal := ⟨LitVal.beq⟩ -/- Constructor information. +/-- Constructor information. - `name` is the Name of the Constructor in Lean. - `cidx` is the Constructor index (aka tag). @@ -191,36 +191,36 @@ def CtorInfo.isScalar (info : CtorInfo) : Bool := !info.isRef inductive Expr where - /- We use `ctor` mainly for constructing Lean object/tobject values `lean_ctor_object` in the runtime. - This instruction is also used to creat `struct` and `union` return values. - For `union`, only `i.cidx` is relevant. For `struct`, `i` is irrelevant. -/ - | ctor (i : CtorInfo) (ys : Array Arg) + | /-- We use `ctor` mainly for constructing Lean object/tobject values `lean_ctor_object` in the runtime. + This instruction is also used to creat `struct` and `union` return values. + For `union`, only `i.cidx` is relevant. For `struct`, `i` is irrelevant. -/ + ctor (i : CtorInfo) (ys : Array Arg) | reset (n : Nat) (x : VarId) - /- `reuse x in ctor_i ys` instruction in the paper. -/ - | reuse (x : VarId) (i : CtorInfo) (updtHeader : Bool) (ys : Array Arg) - /- Extract the `tobject` value at Position `sizeof(void*)*i` from `x`. - We also use `proj` for extracting fields from `struct` return values, and casting `union` return values. -/ - | proj (i : Nat) (x : VarId) - /- Extract the `Usize` value at Position `sizeof(void*)*i` from `x`. -/ - | uproj (i : Nat) (x : VarId) - /- Extract the scalar value at Position `sizeof(void*)*n + offset` from `x`. -/ - | sproj (n : Nat) (offset : Nat) (x : VarId) - /- Full application. -/ - | fap (c : FunId) (ys : Array Arg) - /- Partial application that creates a `pap` value (aka closure in our nonstandard terminology). -/ - | pap (c : FunId) (ys : Array Arg) - /- Application. `x` must be a `pap` value. -/ - | ap (x : VarId) (ys : Array Arg) - /- Given `x : ty` where `ty` is a scalar type, this operation returns a value of Type `tobject`. + | /-- `reuse x in ctor_i ys` instruction in the paper. -/ + reuse (x : VarId) (i : CtorInfo) (updtHeader : Bool) (ys : Array Arg) + | /-- Extract the `tobject` value at Position `sizeof(void*)*i` from `x`. + We also use `proj` for extracting fields from `struct` return values, and casting `union` return values. -/ + proj (i : Nat) (x : VarId) + | /-- Extract the `Usize` value at Position `sizeof(void*)*i` from `x`. -/ + uproj (i : Nat) (x : VarId) + | /-- Extract the scalar value at Position `sizeof(void*)*n + offset` from `x`. -/ + sproj (n : Nat) (offset : Nat) (x : VarId) + | /-- Full application. -/ + fap (c : FunId) (ys : Array Arg) + | /-- Partial application that creates a `pap` value (aka closure in our nonstandard terminology). -/ + pap (c : FunId) (ys : Array Arg) + | /-- Application. `x` must be a `pap` value. -/ + ap (x : VarId) (ys : Array Arg) + | /-- Given `x : ty` where `ty` is a scalar type, this operation returns a value of Type `tobject`. For small scalar values, the Result is a tagged pointer, and no memory allocation is performed. -/ - | box (ty : IRType) (x : VarId) - /- Given `x : [t]object`, obtain the scalar value. -/ - | unbox (x : VarId) + box (ty : IRType) (x : VarId) + | /-- Given `x : [t]object`, obtain the scalar value. -/ + unbox (x : VarId) | lit (v : LitVal) - /- Return `1 : uint8` Iff `RC(x) > 1` -/ - | isShared (x : VarId) - /- Return `1 : uint8` Iff `x : tobject` is a tagged pointer (storing a scalar value). -/ - | isTaggedPtr (x : VarId) + | /-- Return `1 : uint8` Iff `RC(x) > 1` -/ + isShared (x : VarId) + | /-- Return `1 : uint8` Iff `x : tobject` is a tagged pointer (storing a scalar value). -/ + isTaggedPtr (x : VarId) @[export lean_ir_mk_ctor_expr] def mkCtorExpr (n : Name) (cidx : Nat) (size : Nat) (usize : Nat) (ssize : Nat) (ys : Array Arg) : Expr := Expr.ctor ⟨n, cidx, size, usize, ssize⟩ ys @@ -247,31 +247,31 @@ inductive AltCore (FnBody : Type) : Type where | default (b : FnBody) : AltCore FnBody inductive FnBody where - /- `let x : ty := e; b` -/ - | vdecl (x : VarId) (ty : IRType) (e : Expr) (b : FnBody) - /- Join point Declaration `block_j (xs) := e; b` -/ - | jdecl (j : JoinPointId) (xs : Array Param) (v : FnBody) (b : FnBody) - /- Store `y` at Position `sizeof(void*)*i` in `x`. `x` must be a Constructor object and `RC(x)` must be 1. - This operation is not part of λPure is only used during optimization. -/ - | set (x : VarId) (i : Nat) (y : Arg) (b : FnBody) + | /-- `let x : ty := e; b` -/ + vdecl (x : VarId) (ty : IRType) (e : Expr) (b : FnBody) + | /-- Join point Declaration `block_j (xs) := e; b` -/ + jdecl (j : JoinPointId) (xs : Array Param) (v : FnBody) (b : FnBody) + | /-- Store `y` at Position `sizeof(void*)*i` in `x`. `x` must be a Constructor object and `RC(x)` must be 1. + This operation is not part of λPure is only used during optimization. -/ + set (x : VarId) (i : Nat) (y : Arg) (b : FnBody) | setTag (x : VarId) (cidx : Nat) (b : FnBody) - /- Store `y : Usize` at Position `sizeof(void*)*i` in `x`. `x` must be a Constructor object and `RC(x)` must be 1. -/ - | uset (x : VarId) (i : Nat) (y : VarId) (b : FnBody) - /- Store `y : ty` at Position `sizeof(void*)*i + offset` in `x`. `x` must be a Constructor object and `RC(x)` must be 1. + | /-- Store `y : Usize` at Position `sizeof(void*)*i` in `x`. `x` must be a Constructor object and `RC(x)` must be 1. -/ + uset (x : VarId) (i : Nat) (y : VarId) (b : FnBody) + | /-- Store `y : ty` at Position `sizeof(void*)*i + offset` in `x`. `x` must be a Constructor object and `RC(x)` must be 1. `ty` must not be `object`, `tobject`, `irrelevant` nor `Usize`. -/ - | sset (x : VarId) (i : Nat) (offset : Nat) (y : VarId) (ty : IRType) (b : FnBody) - /- RC increment for `object`. If c == `true`, then `inc` must check whether `x` is a tagged pointer or not. + sset (x : VarId) (i : Nat) (offset : Nat) (y : VarId) (ty : IRType) (b : FnBody) + | /-- RC increment for `object`. If c == `true`, then `inc` must check whether `x` is a tagged pointer or not. If `persistent == true` then `x` is statically known to be a persistent object. -/ - | inc (x : VarId) (n : Nat) (c : Bool) (persistent : Bool) (b : FnBody) - /- RC decrement for `object`. If c == `true`, then `inc` must check whether `x` is a tagged pointer or not. + inc (x : VarId) (n : Nat) (c : Bool) (persistent : Bool) (b : FnBody) + | /-- RC decrement for `object`. If c == `true`, then `inc` must check whether `x` is a tagged pointer or not. If `persistent == true` then `x` is statically known to be a persistent object. -/ - | dec (x : VarId) (n : Nat) (c : Bool) (persistent : Bool) (b : FnBody) + dec (x : VarId) (n : Nat) (c : Bool) (persistent : Bool) (b : FnBody) | del (x : VarId) (b : FnBody) | mdata (d : MData) (b : FnBody) | case (tid : Name) (x : VarId) (xType : IRType) (cs : Array (AltCore FnBody)) | ret (x : Arg) - /- Jump to join point `j` -/ - | jmp (j : JoinPointId) (ys : Array Arg) + | /-- Jump to join point `j` -/ + jmp (j : JoinPointId) (ys : Array Arg) | unreachable instance : Inhabited FnBody := ⟨FnBody.unreachable⟩ @@ -331,7 +331,7 @@ def FnBody.setBody : FnBody → FnBody → FnBody @[inline] def FnBody.resetBody (b : FnBody) : FnBody := b.setBody FnBody.nil -/- If b is a non terminal, then return a pair `(c, b')` s.t. `b == c <;> b'`, +/-- If b is a non terminal, then return a pair `(c, b')` s.t. `b == c <;> b'`, and c.body == FnBody.nil -/ @[inline] def FnBody.split (b : FnBody) : FnBody × FnBody := let b' := b.body diff --git a/src/Lean/Compiler/IR/Borrow.lean b/src/Lean/Compiler/IR/Borrow.lean index 56988b9d7928..591a4eb9f328 100644 --- a/src/Lean/Compiler/IR/Borrow.lean +++ b/src/Lean/Compiler/IR/Borrow.lean @@ -29,7 +29,7 @@ abbrev OwnedSet := Std.HashMap Key Unit def OwnedSet.insert (s : OwnedSet) (k : OwnedSet.Key) : OwnedSet := Std.HashMap.insert s k () def OwnedSet.contains (s : OwnedSet) (k : OwnedSet.Key) : Bool := Std.HashMap.contains s k -/- We perform borrow inference in a block of mutually recursive functions. +/-! We perform borrow inference in a block of mutually recursive functions. Join points are viewed as local functions, and are identified using their local id + the name of the surrounding function. We keep a mapping from function and joint points to parameters (`Array Param`). @@ -63,11 +63,11 @@ instance : ToFormat ParamMap := ⟨ParamMap.fmt⟩ instance : ToString ParamMap := ⟨fun m => Format.pretty (format m)⟩ namespace InitParamMap -/- Mark parameters that take a reference as borrow -/ +/-- Mark parameters that take a reference as borrow -/ def initBorrow (ps : Array Param) : Array Param := ps.map fun p => { p with borrow := p.ty.isObj } -/- We do perform borrow inference for constants marked as `export`. +/-- We do perform borrow inference for constants marked as `export`. Reason: we current write wrappers in C++ for using exported functions. These wrappers use smart pointers such as `object_ref`. When writing a new wrapper we need to know whether an argument is a borrow @@ -100,7 +100,7 @@ end InitParamMap def mkInitParamMap (env : Environment) (decls : Array Decl) : ParamMap := (InitParamMap.visitDecls env decls *> get).run' {} -/- Apply the inferred borrow annotations stored at `ParamMap` to a block of mutually +/-! Apply the inferred borrow annotations stored at `ParamMap` to a block of mutually recursive functions. -/ namespace ApplyParamMap @@ -141,7 +141,7 @@ structure BorrowInfCtx where paramSet : IndexSet := {} -- Set of all function parameters in scope. This is used to implement the heuristic at `ownArgsUsingParams` structure BorrowInfState where - /- Set of variables that must be `owned`. -/ + /-- Set of variables that must be `owned`. -/ owned : OwnedSet := {} modified : Bool := false paramMap : ParamMap @@ -174,7 +174,7 @@ def isOwned (x : VarId) : M Bool := do let s ← get return s.owned.contains (currFn, x.idx) -/- Updates `map[k]` using the current set of `owned` variables. -/ +/-- Updates `map[k]` using the current set of `owned` variables. -/ def updateParamMap (k : ParamMap.Key) : M Unit := do let s ← get match s.paramMap.find? k with @@ -202,14 +202,14 @@ def getParamInfo (k : ParamMap.Key) : M (Array Param) := do | none => unreachable! | _ => unreachable! -/- For each ps[i], if ps[i] is owned, then mark xs[i] as owned. -/ +/-- For each ps[i], if ps[i] is owned, then mark xs[i] as owned. -/ def ownArgsUsingParams (xs : Array Arg) (ps : Array Param) : M Unit := xs.size.forM fun i => do let x := xs[i]! let p := ps[i]! unless p.borrow do ownArg x -/- For each xs[i], if xs[i] is owned, then mark ps[i] as owned. +/-- For each xs[i], if xs[i] is owned, then mark ps[i] as owned. We use this action to preserve tail calls. That is, if we have a tail call `f xs`, if the i-th parameter is borrowed, but `xs[i]` is owned we would have to insert a `dec xs[i]` after `f xs` and consequently @@ -222,7 +222,7 @@ def ownParamsUsingArgs (xs : Array Arg) (ps : Array Param) : M Unit := | Arg.var x => if (← isOwned x) then ownVar p.x | _ => pure () -/- Mark `xs[i]` as owned if it is one of the parameters `ps`. +/-- Mark `xs[i]` as owned if it is one of the parameters `ps`. We use this action to mark function parameters that are being "packed" inside constructors. This is a heuristic, and is not related with the effectiveness of the reset/reuse optimization. It is useful for code such as @@ -287,7 +287,7 @@ partial def collectDecl : Decl → M Unit updateParamMap (ParamMap.Key.decl f) | _ => pure () -/- Keep executing `x` until it reaches a fixpoint -/ +/-- Keep executing `x` until it reaches a fixpoint -/ @[inline] partial def whileModifing (x : M Unit) : M Unit := do modify fun s => { s with modified := false } x diff --git a/src/Lean/Compiler/IR/Boxing.lean b/src/Lean/Compiler/IR/Boxing.lean index 8fae3896e33e..ddddb66e79da 100644 --- a/src/Lean/Compiler/IR/Boxing.lean +++ b/src/Lean/Compiler/IR/Boxing.lean @@ -12,7 +12,7 @@ import Lean.Compiler.IR.FreeVars import Lean.Compiler.IR.ElimDeadVars namespace Lean.IR.ExplicitBoxing -/- +/-! Add explicit boxing and unboxing instructions. Recall that the Lean to λ_pure compiler produces code without these instructions. @@ -74,7 +74,7 @@ def addBoxedVersions (env : Environment) (decls : Array Decl) : Array Decl := if requiresBoxedVersion env decl then newDecls.push (mkBoxedVersion decl) else newDecls decls ++ boxedDecls -/- Infer scrutinee type using `case` alternatives. +/-- Infer scrutinee type using `case` alternatives. This can be done whenever `alts` does not contain an `Alt.default _` value. -/ def getScrutineeType (alts : Array Alt) : IRType := let isScalar := @@ -103,7 +103,7 @@ structure BoxingContext where structure BoxingState where nextIdx : Index - /- We create auxiliary declarations when boxing constant and literals. + /-- We create auxiliary declarations when boxing constant and literals. The idea is to avoid code such as ``` let x1 := Uint64.inhabited; @@ -155,7 +155,7 @@ def getDecl (fid : FunId) : M Decl := do @[inline] def withJDecl {α : Type} (j : JoinPointId) (xs : Array Param) (v : FnBody) (k : M α) : M α := withReader (fun ctx => { ctx with localCtx := ctx.localCtx.addJP j xs v }) k -/- If `x` declaration is of the form `x := Expr.lit _` or `x := Expr.fap c #[]`, +/-- If `x` declaration is of the form `x := Expr.lit _` or `x := Expr.fap c #[]`, and `x`'s type is not cheap to box (e.g., it is `UInt64), then return its value. -/ private def isExpensiveConstantValueBoxing (x : VarId) (xType : IRType) : M (Option Expr) := if !xType.isScalar then @@ -173,7 +173,7 @@ private def isExpensiveConstantValueBoxing (x : VarId) (xType : IRType) : M (Opt | _ => return none | _ => return none -/- Auxiliary function used by castVarIfNeeded. +/-- Auxiliary function used by castVarIfNeeded. It is used when the expected type does not match `xType`. If `xType` is scalar, then we need to "box" it. Otherwise, we need to "unbox" it. -/ def mkCast (x : VarId) (xType : IRType) (expectedType : IRType) : M Expr := do diff --git a/src/Lean/Compiler/IR/CompilerM.lean b/src/Lean/Compiler/IR/CompilerM.lean index 0c0d39af9070..e4cecf98f687 100644 --- a/src/Lean/Compiler/IR/CompilerM.lean +++ b/src/Lean/Compiler/IR/CompilerM.lean @@ -73,7 +73,7 @@ open Std (HashMap) abbrev DeclMap := SMap Name Decl -/- Create an array of decls to be saved on .olean file. +/-- Create an array of decls to be saved on .olean file. `decls` may contain duplicate entries, but we assume the one that occurs last is the most recent one. -/ private def mkEntryArray (decls : List Decl) : Array Decl := /- Remove duplicates by adding decls into a map -/ diff --git a/src/Lean/Compiler/IR/EmitC.lean b/src/Lean/Compiler/IR/EmitC.lean index b680be6a44d6..874e9f96f5a5 100644 --- a/src/Lean/Compiler/IR/EmitC.lean +++ b/src/Lean/Compiler/IR/EmitC.lean @@ -530,7 +530,7 @@ def paramEqArg (p : Param) (x : Arg) : Bool := | Arg.var x => p.x == x | _ => false -/- +/-- Given `[p_0, ..., p_{n-1}]`, `[y_0, ..., y_{n-1}]`, representing the assignments ``` p_0 := y_0, diff --git a/src/Lean/Compiler/IR/EmitUtil.lean b/src/Lean/Compiler/IR/EmitUtil.lean index 86b1922ae095..bcce85879ddd 100644 --- a/src/Lean/Compiler/IR/EmitUtil.lean +++ b/src/Lean/Compiler/IR/EmitUtil.lean @@ -6,10 +6,10 @@ Authors: Leonardo de Moura import Lean.Compiler.InitAttr import Lean.Compiler.IR.CompilerM -/- Helper functions for backend code generators -/ +/-! # Helper functions for backend code generators -/ namespace Lean.IR -/- Return true iff `b` is of the form `let x := g ys; ret x` -/ +/-- Return true iff `b` is of the form `let x := g ys; ret x` -/ def isTailCallTo (g : Name) (b : FnBody) : Bool := match b with | FnBody.vdecl x _ (Expr.fap f _) (FnBody.ret (Arg.var y)) => x == y && f == g @@ -62,7 +62,7 @@ def collectParams (ps : Array Param) : Collector := @[inline] def collectJP (j : JoinPointId) (xs : Array Param) : Collector | (vs, js) => (vs, js.insert j xs) -/- `collectFnBody` assumes the variables in -/ +/-- `collectFnBody` assumes the variables in -/ partial def collectFnBody : FnBody → Collector | FnBody.vdecl x t _ b => collectVar x t ∘ collectFnBody b | FnBody.jdecl j xs v b => collectJP j xs ∘ collectParams xs ∘ collectFnBody v ∘ collectFnBody b @@ -75,7 +75,7 @@ def collectDecl : Decl → Collector end CollectMaps -/- Return a pair `(v, j)`, where `v` is a mapping from variable/parameter to type, +/-- Return a pair `(v, j)`, where `v` is a mapping from variable/parameter to type, and `j` is a mapping from join point to parameters. This function assumes `d` has normalized indexes (see `normids.lean`). -/ def mkVarJPMaps (d : Decl) : VarTypeMap × JPParamsMap := diff --git a/src/Lean/Compiler/IR/ExpandResetReuse.lean b/src/Lean/Compiler/IR/ExpandResetReuse.lean index feb2201b11ff..9d7363e2f848 100644 --- a/src/Lean/Compiler/IR/ExpandResetReuse.lean +++ b/src/Lean/Compiler/IR/ExpandResetReuse.lean @@ -8,7 +8,7 @@ import Lean.Compiler.IR.NormIds import Lean.Compiler.IR.FreeVars namespace Lean.IR.ExpandResetReuse -/- Mapping from variable to projections -/ +/-- Mapping from variable to projections -/ abbrev ProjMap := Std.HashMap VarId Expr namespace CollectProjMap abbrev Collector := ProjMap → ProjMap @@ -26,7 +26,7 @@ partial def collectFnBody : FnBody → Collector | e => if e.isTerminal then id else collectFnBody e.body end CollectProjMap -/- Create a mapping from variables to projections. +/-- Create a mapping from variables to projections. This function assumes variable ids have been normalized -/ def mkProjMap (d : Decl) : ProjMap := match d with @@ -36,7 +36,7 @@ def mkProjMap (d : Decl) : ProjMap := structure Context where projMap : ProjMap -/- Return true iff `x` is consumed in all branches of the current block. +/-- Return true iff `x` is consumed in all branches of the current block. Here consumption means the block contains a `dec x` or `reuse x ...`. -/ partial def consumed (x : VarId) : FnBody → Bool | FnBody.vdecl _ _ v b => @@ -49,7 +49,7 @@ partial def consumed (x : VarId) : FnBody → Bool abbrev Mask := Array (Option VarId) -/- Auxiliary function for eraseProjIncFor -/ +/-- Auxiliary function for eraseProjIncFor -/ partial def eraseProjIncForAux (y : VarId) (bs : Array FnBody) (mask : Mask) (keep : Array FnBody) : Array FnBody × Mask := let done (_ : Unit) := (bs ++ keep.reverse, mask) let keepInstr (b : FnBody) := eraseProjIncForAux y bs.pop mask (keep.push b) @@ -81,12 +81,12 @@ partial def eraseProjIncForAux (y : VarId) (bs : Array FnBody) (mask : Mask) (ke | _ => done () | _ => done () -/- Try to erase `inc` instructions on projections of `y` occurring in the tail of `bs`. +/-- Try to erase `inc` instructions on projections of `y` occurring in the tail of `bs`. Return the updated `bs` and a bit mask specifying which `inc`s have been removed. -/ def eraseProjIncFor (n : Nat) (y : VarId) (bs : Array FnBody) : Array FnBody × Mask := eraseProjIncForAux y bs (mkArray n none) #[] -/- Replace `reuse x ctor ...` with `ctor ...`, and remoce `dec x` -/ +/-- Replace `reuse x ctor ...` with `ctor ...`, and remoce `dec x` -/ partial def reuseToCtor (x : VarId) : FnBody → FnBody | FnBody.dec y n c p b => if x == y then b -- n must be 1 since `x := reset ...` @@ -109,7 +109,7 @@ partial def reuseToCtor (x : VarId) : FnBody → FnBody let b := reuseToCtor x b instr.setBody b -/- +/-- replace ``` x := reset y; b @@ -143,7 +143,7 @@ def releaseUnreadFields (y : VarId) (mask : Mask) (b : FnBody) : M FnBody := def setFields (y : VarId) (zs : Array Arg) (b : FnBody) : FnBody := zs.size.fold (init := b) fun i b => FnBody.set y i (zs.get! i) b -/- Given `set x[i] := y`, return true iff `y := proj[i] x` -/ +/-- Given `set x[i] := y`, return true iff `y := proj[i] x` -/ def isSelfSet (ctx : Context) (x : VarId) (i : Nat) (y : Arg) : Bool := match y with | Arg.var y => @@ -152,19 +152,19 @@ def isSelfSet (ctx : Context) (x : VarId) (i : Nat) (y : Arg) : Bool := | _ => false | _ => false -/- Given `uset x[i] := y`, return true iff `y := uproj[i] x` -/ +/-- Given `uset x[i] := y`, return true iff `y := uproj[i] x` -/ def isSelfUSet (ctx : Context) (x : VarId) (i : Nat) (y : VarId) : Bool := match ctx.projMap.find? y with | some (Expr.uproj j w) => j == i && w == x | _ => false -/- Given `sset x[n, i] := y`, return true iff `y := sproj[n, i] x` -/ +/-- Given `sset x[n, i] := y`, return true iff `y := sproj[n, i] x` -/ def isSelfSSet (ctx : Context) (x : VarId) (n : Nat) (i : Nat) (y : VarId) : Bool := match ctx.projMap.find? y with | some (Expr.sproj m j w) => n == m && j == i && w == x | _ => false -/- Remove unnecessary `set/uset/sset` operations -/ +/-- Remove unnecessary `set/uset/sset` operations -/ partial def removeSelfSet (ctx : Context) : FnBody → FnBody | FnBody.set x i y b => if isSelfSet ctx x i y then removeSelfSet ctx b @@ -208,7 +208,7 @@ partial def reuseToSet (ctx : Context) (x y : VarId) : FnBody → FnBody let b := reuseToSet ctx x y b instr.setBody b -/- +/-- replace ``` x := reset y; b diff --git a/src/Lean/Compiler/IR/FreeVars.lean b/src/Lean/Compiler/IR/FreeVars.lean index 4b5c4a395adc..848fce030935 100644 --- a/src/Lean/Compiler/IR/FreeVars.lean +++ b/src/Lean/Compiler/IR/FreeVars.lean @@ -8,7 +8,7 @@ import Lean.Compiler.IR.Basic namespace Lean.IR namespace MaxIndex -/- Compute the maximum index `M` used in a declaration. +/-! Compute the maximum index `M` used in a declaration. We `M` to initialize the fresh index generator used to create fresh variable and join point names. @@ -85,7 +85,7 @@ def Decl.maxIndex (d : Decl) : Index := MaxIndex.collectDecl d 0 namespace FreeIndices -/- We say a variable (join point) index (aka name) is free in a function body +/-! We say a variable (join point) index (aka name) is free in a function body if there isn't a `FnBody.vdecl` (`Fnbody.jdecl`) binding it. -/ abbrev Collector := IndexSet → IndexSet → IndexSet @@ -177,7 +177,7 @@ def FnBody.freeIndices (b : FnBody) : IndexSet := b.collectFreeIndices {} namespace HasIndex -/- In principle, we can check whether a function body `b` contains an index `i` using +/-! In principle, we can check whether a function body `b` contains an index `i` using `b.freeIndices.contains i`, but it is more efficient to avoid the construction of the set of freeIndices and just search whether `i` occurs in `b` or not. -/ diff --git a/src/Lean/Compiler/IR/LiveVars.lean b/src/Lean/Compiler/IR/LiveVars.lean index d83ff8576576..bbdaa02d0b1e 100644 --- a/src/Lean/Compiler/IR/LiveVars.lean +++ b/src/Lean/Compiler/IR/LiveVars.lean @@ -8,7 +8,7 @@ import Lean.Compiler.IR.FreeVars namespace Lean.IR -/- Remark: in the paper "Counting Immutable Beans" the concepts of +/-! Remark: in the paper "Counting Immutable Beans" the concepts of free and live variables coincide because the paper does *not* consider join points. For example, consider the function body `B` ``` @@ -20,13 +20,13 @@ namespace Lean.IR block_1 (x : obj) : obj := let z := ctor_0 x y; ret z - `` + ``` The variable `y` is live in the function body `B` since it occurs in `block_1` which is "invoked" by `B`. -/ namespace IsLive -/- +/-- We use `State Context` instead of `ReaderT Context Id` because we remove non local joint points from `Context` whenever we visit them instead of maintaining a set of visited non local join points. @@ -69,7 +69,7 @@ partial def visitFnBody (w : Index) : FnBody → M Bool end IsLive -/- Return true if `x` is live in the function body `b` in the context `ctx`. +/-- Return true if `x` is live in the function body `b` in the context `ctx`. Remark: the context only needs to contain all (free) join point declarations. diff --git a/src/Lean/Compiler/IR/NormIds.lean b/src/Lean/Compiler/IR/NormIds.lean index b71d9613850d..02ee71405d20 100644 --- a/src/Lean/Compiler/IR/NormIds.lean +++ b/src/Lean/Compiler/IR/NormIds.lean @@ -29,7 +29,7 @@ partial def checkDecl : Decl → M Bool end UniqueIds -/- Return true if variable, parameter and join point ids are unique -/ +/-- Return true if variable, parameter and join point ids are unique -/ def Decl.uniqueIds (d : Decl) : Bool := (UniqueIds.checkDecl d).run' {} @@ -119,11 +119,11 @@ def normDecl (d : Decl) : N Decl := end NormalizeIds -/- Create a declaration equivalent to `d` s.t. `d.normalizeIds.uniqueIds == true` -/ +/-- Create a declaration equivalent to `d` s.t. `d.normalizeIds.uniqueIds == true` -/ def Decl.normalizeIds (d : Decl) : Decl := (NormalizeIds.normDecl d {}).run' 1 -/- Apply a function `f : VarId → VarId` to variable occurrences. +/-! Apply a function `f : VarId → VarId` to variable occurrences. The following functions assume the IR code does not have variable shadowing. -/ namespace MapVars @@ -171,7 +171,7 @@ end MapVars @[inline] def FnBody.mapVars (f : VarId → VarId) (b : FnBody) : FnBody := MapVars.mapFnBody f b -/- Replace `x` with `y` in `b`. This function assumes `b` does not shadow `x` -/ +/-- Replace `x` with `y` in `b`. This function assumes `b` does not shadow `x` -/ def FnBody.replaceVar (x y : VarId) (b : FnBody) : FnBody := b.mapVars fun z => if x == z then y else z diff --git a/src/Lean/Compiler/IR/RC.lean b/src/Lean/Compiler/IR/RC.lean index 7b4a7b05150d..c45b640251f0 100644 --- a/src/Lean/Compiler/IR/RC.lean +++ b/src/Lean/Compiler/IR/RC.lean @@ -8,7 +8,7 @@ import Lean.Compiler.IR.CompilerM import Lean.Compiler.IR.LiveVars namespace Lean.IR.ExplicitRC -/- Insert explicit RC instructions. So, it assumes the input code does not contain `inc` nor `dec` instructions. +/-! Insert explicit RC instructions. So, it assumes the input code does not contain `inc` nor `dec` instructions. This transformation is applied before lower level optimizations that introduce the instructions `release` and `set` -/ @@ -74,12 +74,12 @@ private def addDecForAlt (ctx : Context) (caseLiveVars altLiveVars : LiveVarSet) caseLiveVars.fold (init := b) fun b x => if !altLiveVars.contains x && mustConsume ctx x then addDec ctx x b else b -/- `isFirstOcc xs x i = true` if `xs[i]` is the first occurrence of `xs[i]` in `xs` -/ +/-- `isFirstOcc xs x i = true` if `xs[i]` is the first occurrence of `xs[i]` in `xs` -/ private def isFirstOcc (xs : Array Arg) (i : Nat) : Bool := let x := xs[i]! i.all fun j => xs[j]! != x -/- Return true if `x` also occurs in `ys` in a position that is not consumed. +/-- Return true if `x` also occurs in `ys` in a position that is not consumed. That is, it is also passed as a borrow reference. -/ private def isBorrowParamAux (x : VarId) (ys : Array Arg) (consumeParamPred : Nat → Bool) : Bool := ys.size.any fun i => @@ -91,7 +91,7 @@ private def isBorrowParamAux (x : VarId) (ys : Array Arg) (consumeParamPred : Na private def isBorrowParam (x : VarId) (ys : Array Arg) (ps : Array Param) : Bool := isBorrowParamAux x ys fun i => not ps[i]!.borrow -/- +/-- Return `n`, the number of times `x` is consumed. - `ys` is a sequence of instruction parameters where we search for `x`. - `consumeParamPred i = true` if parameter `i` is consumed. @@ -124,7 +124,7 @@ private def addIncBeforeAux (ctx : Context) (xs : Array Arg) (consumeParamPred : private def addIncBefore (ctx : Context) (xs : Array Arg) (ps : Array Param) (b : FnBody) (liveVarsAfter : LiveVarSet) : FnBody := addIncBeforeAux ctx xs (fun i => not ps[i]!.borrow) b liveVarsAfter -/- See `addIncBeforeAux`/`addIncBefore` for the procedure that inserts `inc` operations before an application. -/ +/-- See `addIncBeforeAux`/`addIncBefore` for the procedure that inserts `inc` operations before an application. -/ private def addDecAfterFullApp (ctx : Context) (xs : Array Arg) (ps : Array Param) (b : FnBody) (bLiveVars : LiveVarSet) : FnBody := xs.size.fold (init := b) fun i b => match xs[i]! with @@ -141,7 +141,7 @@ xs.size.fold (init := b) fun i b => private def addIncBeforeConsumeAll (ctx : Context) (xs : Array Arg) (b : FnBody) (liveVarsAfter : LiveVarSet) : FnBody := addIncBeforeAux ctx xs (fun _ => true) b liveVarsAfter -/- Add `dec` instructions for parameters that are references, are not alive in `b`, and are not borrow. +/-- Add `dec` instructions for parameters that are references, are not alive in `b`, and are not borrow. That is, we must make sure these parameters are consumed. -/ private def addDecForDeadParams (ctx : Context) (ps : Array Param) (b : FnBody) (bLiveVars : LiveVarSet) : FnBody := ps.foldl (init := b) fun b p => @@ -151,14 +151,14 @@ private def isPersistent : Expr → Bool | Expr.fap _ xs => xs.isEmpty -- all global constants are persistent objects | _ => false -/- We do not need to consume the projection of a variable that is not consumed -/ +/-- We do not need to consume the projection of a variable that is not consumed -/ private def consumeExpr (m : VarMap) : Expr → Bool | Expr.proj _ x => match m.find? x with | some info => info.consume | none => true | _ => true -/- Return true iff `v` at runtime is a scalar value stored in a tagged pointer. +/-- Return true iff `v` at runtime is a scalar value stored in a tagged pointer. We do not need RC operations for this kind of value. -/ private def isScalarBoxedInTaggedPtr (v : Expr) : Bool := match v with diff --git a/src/Lean/Compiler/IR/ResetReuse.lean b/src/Lean/Compiler/IR/ResetReuse.lean index 0e519ef4153a..2793c7e40266 100644 --- a/src/Lean/Compiler/IR/ResetReuse.lean +++ b/src/Lean/Compiler/IR/ResetReuse.lean @@ -8,11 +8,11 @@ import Lean.Compiler.IR.LiveVars import Lean.Compiler.IR.Format namespace Lean.IR.ResetReuse -/- Remark: the insertResetReuse transformation is applied before we have +/-! Remark: the insertResetReuse transformation is applied before we have inserted `inc/dec` instructions, and perfomed lower level optimizations that introduce the instructions `release` and `set`. -/ -/- Remark: the functions `S`, `D` and `R` defined here implement the +/-! Remark: the functions `S`, `D` and `R` defined here implement the corresponding functions in the paper "Counting Immutable Beans" Here are the main differences: @@ -50,7 +50,7 @@ private partial def S (w : VarId) (c : CtorInfo) : FnBody → FnBody (instr, b) := b.split instr.setBody (S w c b) -/- We use `Context` to track join points in scope. -/ +/-- We use `Context` to track join points in scope. -/ abbrev M := ReaderT LocalContext (StateT Index Id) private def mkFresh : M VarId := do @@ -77,7 +77,7 @@ private def isCtorUsing (b : FnBody) (x : VarId) : Bool := | (FnBody.vdecl _ _ (Expr.ctor _ ys) _) => argsContainsVar ys x | _ => false -/- Given `Dmain b`, the resulting pair `(new_b, flag)` contains the new body `new_b`, +/-- Given `Dmain b`, the resulting pair `(new_b, flag)` contains the new body `new_b`, and `flag == true` if `x` is live in `b`. Note that, in the function `D` defined in the paper, for each `let x := e; F`, diff --git a/src/Lean/Compiler/Util.lean b/src/Lean/Compiler/Util.lean index 9f825302d2a6..421733fac7de 100644 --- a/src/Lean/Compiler/Util.lean +++ b/src/Lean/Compiler/Util.lean @@ -57,7 +57,7 @@ def atMostOnce (e : Expr) (x : FVarId) : Bool := let {result := result, ..} := visit x e {found := false, result := true} result -/- Helper functions for creating auxiliary names used in compiler passes. -/ +/-! Helper functions for creating auxiliary names used in compiler passes. -/ @[export lean_mk_eager_lambda_lifting_name] def mkEagerLambdaLiftingName (n : Name) (idx : Nat) : Name := @@ -104,14 +104,14 @@ end Compiler namespace Environment -/- +/-- Compile the given block of mutual declarations. Assumes the declarations have already been added to the environment using `addDecl`. -/ @[extern "lean_compile_decls"] opaque compileDecls (env : Environment) (opt : @& Options) (decls : @& List Name) : Except KernelException Environment -/- Compile the given declaration, it assumes the declaration has already been added to the environment using `addDecl`. -/ +/-- Compile the given declaration, it assumes the declaration has already been added to the environment using `addDecl`. -/ def compileDecl (env : Environment) (opt : @& Options) (decl : @& Declaration) : Except KernelException Environment := compileDecls env opt (Compiler.getDeclNamesForCodeGen decl) diff --git a/src/Lean/CoreM.lean b/src/Lean/CoreM.lean index ea9542a2a184..5290b9a4f15f 100644 --- a/src/Lean/CoreM.lean +++ b/src/Lean/CoreM.lean @@ -228,15 +228,15 @@ export Core (CoreM mkFreshUserName checkMaxHeartbeats withCurrHeartbeats) try x catch ex => match ex with - | Exception.error _ _ => throw ex - | Exception.internal id' _ => if id == id' then h ex else throw ex + | .error .. => throw ex + | .internal id' _ => if id == id' then h ex else throw ex @[inline] def catchInternalIds [Monad m] [MonadExcept Exception m] (ids : List InternalExceptionId) (x : m α) (h : Exception → m α) : m α := do try x catch ex => match ex with - | Exception.error _ _ => throw ex - | Exception.internal id _ => if ids.contains id then h ex else throw ex + | .error .. => throw ex + | .internal id _ => if ids.contains id then h ex else throw ex /-- Return true if `ex` was generated by `throwMaxHeartbeat`. diff --git a/src/Lean/Data/FuzzyMatching.lean b/src/Lean/Data/FuzzyMatching.lean index 8915f0f88121..d9878ead3123 100644 --- a/src/Lean/Data/FuzzyMatching.lean +++ b/src/Lean/Data/FuzzyMatching.lean @@ -42,7 +42,7 @@ private def containsInOrderLower (a b : String) : Bool := Id.run do end Utils -/- Represents the type of a single character. -/ +/-- Represents the type of a single character. -/ inductive CharType where | lower | upper | separator @@ -55,7 +55,7 @@ def charType (c : Char) : CharType := CharType.separator -/- Represents the role of a character inside a word. -/ +/-- Represents the role of a character inside a word. -/ inductive CharRole where | head | tail | separator deriving Inhabited @@ -72,7 +72,7 @@ inductive CharRole where else CharRole.head -/- Add additional information to each character in a string. -/ +/-- Add additional information to each character in a string. -/ private def stringInfo (s : String) : Array CharRole := iterateLookaround (string := s) fun (prev?, curr, next?) => charRole (prev?.map charType) (charType curr) (next?.map charType) @@ -85,7 +85,7 @@ private def selectBest (missScore? matchScore? : Option Int) : Option Int := | (some missScore, some matchScore) => some <| max missScore matchScore -/- Match the given pattern with the given word. The algorithm uses dynamic +/-- Match the given pattern with the given word. The algorithm uses dynamic programming to find the best scores. In addition to the current characters in the pattern and the word, the @@ -145,7 +145,7 @@ private def fuzzyMatchCore (pattern word : String) (patternRoles wordRoles : Arr let idx := patternIdx * (word.length + 1) * 2 + wordIdx * 2 result |>.set! idx missValue |>.set! (idx + 1) matchValue - /- Heuristic to penalize skipping characters in the word. -/ + /-- Heuristic to penalize skipping characters in the word. -/ skipPenalty (wordRole : CharRole) (patternComplete : Bool) (wordStart : Bool) : Int := Id.run do /- Skipping characters if the match is already completed is free. -/ if patternComplete then @@ -159,7 +159,7 @@ private def fuzzyMatchCore (pattern word : String) (patternRoles wordRoles : Arr return 0 - /- Whether characters from the pattern and the word match. -/ + /-- Whether characters from the pattern and the word match. -/ allowMatch (patternChar wordChar : Char) (patternRole wordRole : CharRole) : Bool := Id.run do /- Different characters do not match. -/ if patternChar.toLower != wordChar.toLower then @@ -170,7 +170,7 @@ private def fuzzyMatchCore (pattern word : String) (patternRoles wordRoles : Arr return true - /- Heuristic to rate a match. -/ + /-- Heuristic to rate a match. -/ matchResult (patternChar wordChar : Char) (patternRole wordRole : CharRole) (consecutive : Bool) (wordStart : Bool) : Int := Id.run do let mut score := 1 /- Case-sensitive equality or beginning of a segment in pattern and word. -/ @@ -185,7 +185,7 @@ private def fuzzyMatchCore (pattern word : String) (patternRoles wordRoles : Arr return score -/- Match the given pattern with the given word using a fuzzy matching +/-- Match the given pattern with the given word using a fuzzy matching algorithm. The resulting scores are in the interval `[0, 1]` or `none` if no match was found. -/ def fuzzyMatchScore? (pattern word : String) : Option Float := Id.run do @@ -214,7 +214,7 @@ def fuzzyMatchScore? (pattern word : String) : Option Float := Id.run do def fuzzyMatchScoreWithThreshold? (pattern word : String) (threshold := 0.2) : Option Float := fuzzyMatchScore? pattern word |>.filter (· > threshold) -/- Match the given pattern with the given word using a fuzzy matching +/-- Match the given pattern with the given word using a fuzzy matching algorithm. Return `false` if no match was found or the found match received a score below the given threshold. -/ def fuzzyMatch (pattern word : String) (threshold := 0.2) : Bool := diff --git a/src/Lean/Data/Json/FromToJson.lean b/src/Lean/Data/Json/FromToJson.lean index accf79ebfab0..34dc91118be7 100644 --- a/src/Lean/Data/Json/FromToJson.lean +++ b/src/Lean/Data/Json/FromToJson.lean @@ -88,7 +88,7 @@ instance : FromJson Name where instance : ToJson Name where toJson n := toString n -/- Note that `USize`s and `UInt64`s are stored as strings because JavaScript +/-- Note that `USize`s and `UInt64`s are stored as strings because JavaScript cannot represent 64-bit numbers. -/ def bignumFromJson? (j : Json) : Except String Nat := do let s ← j.getStr? diff --git a/src/Lean/Data/JsonRpc.lean b/src/Lean/Data/JsonRpc.lean index a72d739c8209..dc42ce3611a6 100644 --- a/src/Lean/Data/JsonRpc.lean +++ b/src/Lean/Data/JsonRpc.lean @@ -78,7 +78,7 @@ instance : ToJson ErrorCode := ⟨fun | ErrorCode.workerExited => (-32901 : Int) | ErrorCode.workerCrashed => (-32902 : Int)⟩ -/- Uses separate constructors for notifications and errors because client and server +/-- Uses separate constructors for notifications and errors because client and server behavior is expected to be wildly different for both. -/ inductive Message where | request (id : RequestID) (method : String) (params? : Option Structured) diff --git a/src/Lean/Data/KVMap.lean b/src/Lean/Data/KVMap.lean index 6a674566d59c..4908974b8e36 100644 --- a/src/Lean/Data/KVMap.lean +++ b/src/Lean/Data/KVMap.lean @@ -53,7 +53,7 @@ instance : Coe Int DataValue := ⟨DataValue.ofInt⟩ instance : Coe Syntax DataValue := ⟨DataValue.ofSyntax⟩ -/- Remark: we do not use RBMap here because we need to manipulate KVMap objects in +/-- Remark: we do not use RBMap here because we need to manipulate KVMap objects in C++ and RBMap is implemented in Lean. So, we use just a List until we can generate C++ code from Lean code. -/ structure KVMap where diff --git a/src/Lean/Data/Lsp/Basic.lean b/src/Lean/Data/Lsp/Basic.lean index 41a4bcf03c2a..0e44f4b3f03c 100644 --- a/src/Lean/Data/Lsp/Basic.lean +++ b/src/Lean/Data/Lsp/Basic.lean @@ -61,7 +61,7 @@ structure LocationLink where -- NOTE: Diagnostic defined in Diagnostics.lean -/- NOTE: No specific commands are specified by LSP, hence +/-- NOTE: No specific commands are specified by LSP, hence possible commands need to be announced as capabilities. -/ structure Command where title : String diff --git a/src/Lean/Data/Lsp/InitShutdown.lean b/src/Lean/Data/Lsp/InitShutdown.lean index eff005e2a3b5..732f9854a181 100644 --- a/src/Lean/Data/Lsp/InitShutdown.lean +++ b/src/Lean/Data/Lsp/InitShutdown.lean @@ -58,7 +58,7 @@ structure InitializeParams where rootUri? : Option String := none initializationOptions? : Option InitializationOptions := none capabilities : ClientCapabilities - /- If omitted, we default to off. -/ + /-- If omitted, we default to off. -/ trace : Trace := Trace.off workspaceFolders? : Option (Array WorkspaceFolder) := none deriving ToJson diff --git a/src/Lean/Data/Lsp/Internal.lean b/src/Lean/Data/Lsp/Internal.lean index a69a2cc6862d..d82a9dae579c 100644 --- a/src/Lean/Data/Lsp/Internal.lean +++ b/src/Lean/Data/Lsp/Internal.lean @@ -15,7 +15,7 @@ workers. These messages are not visible externally to users of the LSP server. namespace Lean.Lsp open Std -/- Most reference-related types have custom FromJson/ToJson implementations to +/-! Most reference-related types have custom FromJson/ToJson implementations to reduce the size of the resulting JSON. -/ inductive RefIdent where diff --git a/src/Lean/Data/Lsp/LanguageFeatures.lean b/src/Lean/Data/Lsp/LanguageFeatures.lean index 58c4f91eac42..dde13e1b2575 100644 --- a/src/Lean/Data/Lsp/LanguageFeatures.lean +++ b/src/Lean/Data/Lsp/LanguageFeatures.lean @@ -226,11 +226,13 @@ structure SymbolInformation where deriving ToJson inductive SemanticTokenType where + -- Used by Lean | keyword | «variable» | property | function - /- + /- Other types included by default in the LSP specification. + Not used by the Lean core, but useful to users extending the Lean server. -/ | «namespace» | type | «class» @@ -249,19 +251,29 @@ inductive SemanticTokenType where | number | regexp | operator - -/ + | decorator + deriving ToJson, FromJson +-- must be in the same order as the constructors def SemanticTokenType.names : Array String := - #["keyword", "variable", "property", "function"] - --- must be the correct index in `names` -def SemanticTokenType.toNat : SemanticTokenType → Nat - | keyword => 0 - | «variable» => 1 - | property => 2 - | function => 3 - -/- + #["keyword", "variable", "property", "function", "namespace", "type", "class", + "enum", "interface", "struct", "typeParameter", "parameter", "enumMember", + "event", "method", "macro", "modifier", "comment", "string", "number", + "regexp", "operator", "decorator"] + +def SemanticTokenType.toNat (type : SemanticTokenType) : Nat := + type.toCtorIdx + +-- sanity check +example {v : SemanticTokenType} : open SemanticTokenType in + names[v.toNat]?.map (toString <| toJson ·) = some (toString <| toJson v) := by + cases v <;> native_decide + +/-- +The semantic token modifiers included by default in the LSP specification. +Not used by the Lean core, but implementing them here allows them to be +utilized by users extending the Lean server. +-/ inductive SemanticTokenModifier where | declaration | definition @@ -273,7 +285,20 @@ inductive SemanticTokenModifier where | modification | documentation | defaultLibrary --/ + deriving ToJson, FromJson + +-- must be in the same order as the constructors +def SemanticTokenModifier.names : Array String := + #["declaration", "definition", "readonly", "static", "deprecated", "abstract", + "async", "modification", "documentation", "defaultLibrary"] + +def SemanticTokenModifier.toNat (modifier : SemanticTokenModifier) : Nat := + modifier.toCtorIdx + +-- sanity check +example {v : SemanticTokenModifier} : open SemanticTokenModifier in + names[v.toNat]?.map (toString <| toJson ·) = some (toString <| toJson v) := by + cases v <;> native_decide structure SemanticTokensLegend where tokenTypes : Array String @@ -298,7 +323,7 @@ structure SemanticTokensRangeParams where deriving FromJson, ToJson structure SemanticTokens where - -- resultId?: string; + resultId? : Option String := none data : Array Nat deriving FromJson, ToJson diff --git a/src/Lean/Data/Lsp/TextSync.lean b/src/Lean/Data/Lsp/TextSync.lean index 99d61ead3379..96b796d8b7f6 100644 --- a/src/Lean/Data/Lsp/TextSync.lean +++ b/src/Lean/Data/Lsp/TextSync.lean @@ -78,7 +78,7 @@ structure DidCloseTextDocumentParams where -- TODO: TextDocumentSyncClientCapabilities -/- NOTE: This is defined twice in the spec. The latter version has more fields. -/ +/-- NOTE: This is defined twice in the spec. The latter version has more fields. -/ structure TextDocumentSyncOptions where openClose : Bool change : TextDocumentSyncKind diff --git a/src/Lean/Data/Name.lean b/src/Lean/Data/Name.lean index dcc554cd1b99..a60c037cce33 100644 --- a/src/Lean/Data/Name.lean +++ b/src/Lean/Data/Name.lean @@ -100,14 +100,14 @@ def quickCmp (n₁ n₂ : Name) : Ordering := def quickLt (n₁ n₂ : Name) : Bool := quickCmp n₁ n₂ == Ordering.lt -/- Alternative HasLt instance. -/ +/-- Alternative HasLt instance. -/ @[inline] protected def hasLtQuick : LT Name := ⟨fun a b => Name.quickLt a b = true⟩ @[inline] instance : DecidableRel (@LT.lt Name Name.hasLtQuick) := inferInstanceAs (DecidableRel (fun a b => Name.quickLt a b = true)) -/- The frontend does not allow user declarations to start with `_` in any of its parts. +/-- The frontend does not allow user declarations to start with `_` in any of its parts. We use name parts starting with `_` internally to create auxiliary names (e.g., `_private`). -/ def isInternal : Name → Bool | str p s => s.get 0 == '_' || isInternal p diff --git a/src/Lean/Data/Options.lean b/src/Lean/Data/Options.lean index 3a65a921e837..e2ba13b3fd4a 100644 --- a/src/Lean/Data/Options.lean +++ b/src/Lean/Data/Options.lean @@ -107,7 +107,7 @@ export MonadWithOptions (withOptions) instance [MonadFunctor m n] [MonadWithOptions m] : MonadWithOptions n where withOptions f x := monadMap (m := m) (withOptions f) x -/- Remark: `_inPattern` is an internal option for communicating to the delaborator that +/-! Remark: `_inPattern` is an internal option for communicating to the delaborator that the term being delaborated should be treated as a pattern. -/ def withInPattern [MonadWithOptions m] (x : m α) : m α := diff --git a/src/Lean/Data/SMap.lean b/src/Lean/Data/SMap.lean index 966fc8acf4c1..38d9e1a4d300 100644 --- a/src/Lean/Data/SMap.lean +++ b/src/Lean/Data/SMap.lean @@ -11,7 +11,7 @@ namespace Lean open Std (HashMap PHashMap) -/- Staged map for implementing the Environment. The idea is to store +/-- Staged map for implementing the Environment. The idea is to store imported entries into a hashtable and local entries into a persistent hashtable. Hypotheses: @@ -65,7 +65,7 @@ def empty : SMap α β := {} | ⟨true, m₁, _⟩, k => m₁.contains k | ⟨false, m₁, m₂⟩, k => m₁.contains k || m₂.contains k -/- Similar to `find?`, but searches for result in the hashmap first. +/-- Similar to `find?`, but searches for result in the hashmap first. So, the result is correct only if we never "overwrite" `map₁` entries using `map₂`. -/ @[specialize] def find?' : SMap α β → α → Option β | ⟨true, m₁, _⟩, k => m₁.find? k @@ -75,7 +75,7 @@ def forM [Monad m] (s : SMap α β) (f : α → β → m PUnit) : m PUnit := do s.map₁.forM f s.map₂.forM f -/- Move from stage 1 into stage 2. -/ +/-- Move from stage 1 into stage 2. -/ def switch (m : SMap α β) : SMap α β := if m.stage₁ then { m with stage₁ := false } else m diff --git a/src/Lean/Data/SSet.lean b/src/Lean/Data/SSet.lean index de5ff9540fd5..578340f86402 100644 --- a/src/Lean/Data/SSet.lean +++ b/src/Lean/Data/SSet.lean @@ -7,8 +7,7 @@ import Lean.Data.SMap namespace Lean -/- Staged set. It is just a simple wrapper on top of Staged maps. -/ - +/-- Staged set. It is just a simple wrapper on top of Staged maps. -/ def SSet (α : Type u) [BEq α] [Hashable α] := SMap α Unit namespace SSet @@ -27,7 +26,7 @@ abbrev contains (s : SSet α) (a : α) : Bool := abbrev forM [Monad m] (s : SSet α) (f : α → m PUnit) : m PUnit := SMap.forM s fun a _ => f a -/- Move from stage 1 into stage 2. -/ +/-- Move from stage 1 into stage 2. -/ abbrev switch (s : SSet α) : SSet α := SMap.switch s diff --git a/src/Lean/Declaration.lean b/src/Lean/Declaration.lean index 29747fc285d6..06411490d862 100644 --- a/src/Lean/Declaration.lean +++ b/src/Lean/Declaration.lean @@ -121,7 +121,7 @@ structure TheoremVal extends ConstantVal where all : List Name := [name] deriving Inhabited -/- Value for an opaque constant declaration `constant x : t := e` -/ +/-- Value for an opaque constant declaration `opaque x : t := e` -/ structure OpaqueVal extends ConstantVal where value : Expr isUnsafe : Bool diff --git a/src/Lean/DocString.lean b/src/Lean/DocString.lean index 8b2fdf97b922..9b233b2da193 100644 --- a/src/Lean/DocString.lean +++ b/src/Lean/DocString.lean @@ -11,11 +11,48 @@ namespace Lean private builtin_initialize builtinDocStrings : IO.Ref (NameMap String) ← IO.mkRef {} private builtin_initialize docStringExt : MapDeclarationExtension String ← mkMapDeclarationExtension `docstring +private def findLeadingSpacesSize (s : String) : Nat := + let it := s.iter + let it := it.find (· == '\n') |>.next + let (min, it) := it.foldUntil 0 fun num c => if c == ' ' || c == '\t' then some (num + 1) else none + findNextLine it min +where + consumeSpaces (it : String.Iterator) (curr min : Nat) : Nat := + if it.atEnd then min + else if it.curr == ' ' || it.curr == '\t' then consumeSpaces it.next (curr + 1) min + else findNextLine it.next (Nat.min curr min) + findNextLine (it : String.Iterator) (min : Nat) : Nat := + if it.atEnd then min + else if it.curr == '\n' then consumeSpaces it.next 0 min + else findNextLine it.next min + +private def removeNumLeadingSpaces (n : Nat) (s : String) : String := + consumeSpaces n s.iter "" +where + consumeSpaces (n : Nat) (it : String.Iterator) (r : String) : String := + match n with + | 0 => saveLine it r + | n+1 => + if it.atEnd then r + else if it.curr == ' ' || it.curr == '\t' then consumeSpaces n it.next r + else saveLine it r + saveLine (it : String.Iterator) (r : String) : String := + if it.atEnd then r + else if it.curr == '\n' then consumeSpaces n it.next (r.push '\n') + else saveLine it.next (r.push it.curr) +termination_by + consumeSpaces n it r => (it, 1) + saveLine it r => (it, 0) + +private def removeLeadingSpaces (s : String) : String := + let n := findLeadingSpacesSize s + if n == 0 then s else removeNumLeadingSpaces n s + def addBuiltinDocString (declName : Name) (docString : String) : IO Unit := - builtinDocStrings.modify (·.insert declName docString) + builtinDocStrings.modify (·.insert declName (removeLeadingSpaces docString)) def addDocString [MonadEnv m] (declName : Name) (docString : String) : m Unit := - modifyEnv fun env => docStringExt.insert env declName docString + modifyEnv fun env => docStringExt.insert env declName (removeLeadingSpaces docString) def addDocString' [Monad m] [MonadEnv m] (declName : Name) (docString? : Option String) : m Unit := match docString? with diff --git a/src/Lean/Elab/App.lean b/src/Lean/Elab/App.lean index c26931f12c57..38ca824bcbee 100644 --- a/src/Lean/Elab/App.lean +++ b/src/Lean/Elab/App.lean @@ -37,7 +37,7 @@ private def ensureArgType (f : Expr) (arg : Expr) (expectedType : Expr) : TermEl try ensureHasTypeAux expectedType argType arg f catch - | ex@(Exception.error ..) => + | ex@(.error ..) => if (← read).errToSorry then exceptionToSorry ex expectedType else @@ -53,7 +53,7 @@ private def mkProjAndCheck (structName : Name) (idx : Nat) (e : Expr) : MetaM Ex throwError "invalid projection, the expression{indentExpr e}\nis a proposition and has type{indentExpr eType}\nbut the projected value is not, it has type{indentExpr rType}" return r -/- +/-- Relevant definitions: ``` class CoeFun (α : Sort u) (γ : α → outParam (Sort v)) @@ -125,7 +125,7 @@ structure Context where -/ resultIsOutParamSupport : Bool -/- Auxiliary structure for elaborating the application `f args namedArgs`. -/ +/-- Auxiliary structure for elaborating the application `f args namedArgs`. -/ structure State where f : Expr fType : Expr @@ -249,7 +249,7 @@ private def fTypeHasOptAutoParams : M Bool := do See `propagateExpectedType`. Remark: `(explicit : Bool) == true` when `@` modifier is used. -/ private partial def getForallBody (explicit : Bool) : Nat → List NamedArg → Expr → Option Expr - | i, namedArgs, type@(Expr.forallE n d b bi) => + | i, namedArgs, type@(.forallE n d b bi) => match namedArgs.find? fun (namedArg : NamedArg) => namedArg.name == n with | some _ => getForallBody explicit i (eraseNamedArgCore namedArgs n) b | none => @@ -465,7 +465,7 @@ where | .bvar idx => idx == i | _ => false - /- (quick filter) Return true if `type` constains a binder `[C ...]` where `C` is a class containing outparams. -/ + /-- (quick filter) Return true if `type` constains a binder `[C ...]` where `C` is a class containing outparams. -/ hasLocalInstaceWithOutParams (type : Expr) : CoreM Bool := do let .forallE _ d b bi := type | return false if bi.isInstImplicit then @@ -497,7 +497,7 @@ where return false mutual - /- + /-- Create a fresh local variable with the current binder name and argument type, add it to `etaArgs` and `f`, and then execute the main loop.-/ private partial def addEtaArg (argName : Name) : M Expr := do @@ -524,7 +524,7 @@ mutual addNewArg argName arg main - /- + /-- Process a `fType` of the form `(x : A) → B x`. This method assume `fType` is a function type -/ private partial def processExplictArg (argName : Name) : M Expr := do @@ -538,7 +538,7 @@ mutual let argType ← getArgExpectedType match (← read).explicit, argType.getOptParamDefault?, argType.getAutoParamTactic? with | false, some defVal, _ => addNewArg argName defVal; main - | false, _, some (Expr.const tacticDecl _) => + | false, _, some (.const tacticDecl _) => let env ← getEnv let opts ← getOptions match evalSyntaxConstant env opts tacticDecl with @@ -568,7 +568,7 @@ mutual else finalize - /- + /-- Process a `fType` of the form `{x : A} → B x`. This method assume `fType` is a function type -/ private partial def processImplicitArg (argName : Name) : M Expr := do @@ -577,7 +577,7 @@ mutual else addImplicitArg argName - /- + /-- Process a `fType` of the form `{{x : A}} → B x`. This method assume `fType` is a function type -/ private partial def processStrictImplicitArg (argName : Name) : M Expr := do @@ -588,7 +588,7 @@ mutual else finalize - /- + /-- Process a `fType` of the form `[x : A] → B x`. This method assume `fType` is a function type -/ private partial def processInstImplicitArg (argName : Name) : M Expr := do @@ -608,7 +608,7 @@ mutual addNewArg argName arg main - /- Elaborate function application arguments. -/ + /-- Elaborate function application arguments. -/ partial def main : M Expr := do let fType ← normalizeFunType if fType.isForall then @@ -768,7 +768,7 @@ private def resolveLValAux (e : Expr) (eType : Expr) (lval : LVal) : TermElabM L throwInvalidFieldNotation e eType | _, _ => throwInvalidFieldNotation e eType -/- whnfCore + implicit consumption. +/-- whnfCore + implicit consumption. Example: given `e` with `eType := {α : Type} → (fun β => List β) α `, it produces `(e ?m, List ?m)` where `?m` is fresh metavariable. -/ private partial def consumeImplicits (stx : Syntax) (e eType : Expr) (hasArgs : Bool) : TermElabM (Expr × Expr) := do let eType ← whnfCore eType @@ -832,7 +832,7 @@ private def typeMatchesBaseName (type : Expr) (baseName : Name) : MetaM Bool := else return (← whnfR type).isAppOf baseName -/- Auxiliary method for field notation. It tries to add `e` as a new argument to `args` or `namedArgs`. +/-- Auxiliary method for field notation. It tries to add `e` as a new argument to `args` or `namedArgs`. This method first finds the parameter with a type of the form `(baseName ...)`. When the parameter is found, if it an explicit one and `args` is big enough, we add `e` to `args`. Otherwise, if there isn't another parameter with the same name, we add `e` to `namedArgs`. @@ -932,8 +932,8 @@ private def elabAppLVals (f : Expr) (lvals : List LVal) (namedArgs : Array Named def elabExplicitUnivs (lvls : Array Syntax) : TermElabM (List Level) := do lvls.foldrM (init := []) fun stx lvls => return (← elabLevel stx)::lvls -/- -Interaction between `errToSorry` and `observing`. +/-! +# Interaction between `errToSorry` and `observing`. - The method `elabTerm` catches exceptions, log them, and returns a synthetic sorry (IF `ctx.errToSorry` == true). @@ -988,17 +988,17 @@ private partial def resolveDotName (id : Syntax) (expectedType? : Option Expr) : go resultType expectedType #[] where go (resultType : Expr) (expectedType : Expr) (previousExceptions : Array Exception) : TermElabM Name := do - let resultTypeFn := (← instantiateMVars resultType).consumeMDataAndTypeAnnotations.getAppFn + let resultTypeFn := (← instantiateMVars resultType).cleanupAnnotations.getAppFn try tryPostponeIfMVar resultTypeFn - let .const declName .. := resultTypeFn.consumeMDataAndTypeAnnotations + let .const declName .. := resultTypeFn.cleanupAnnotations | throwError "invalid dotted identifier notation, expected type is not of the form (... → C ...) where C is a constant{indentExpr expectedType}" let idNew := declName ++ id.getId.eraseMacroScopes unless (← getEnv).contains idNew do throwError "invalid dotted identifier notation, unknown identifier `{idNew}` from expected type{indentExpr expectedType}" return idNew catch - | ex@(.error _ _) => + | ex@(.error ..) => match (← unfoldDefinition? resultType) with | some resultType => go (← whnfCore resultType) expectedType (previousExceptions.push ex) | none => @@ -1107,8 +1107,8 @@ private def elabAppAux (f : Syntax) (namedArgs : Array NamedArg) (args : Array A else if successes.size > 1 then let msgs : Array MessageData ← successes.mapM fun success => do match success with - | EStateM.Result.ok e s => withMCtx s.meta.meta.mctx <| withEnv s.meta.core.env do addMessageContext m!"{e} : {← inferType e}" - | _ => unreachable! + | .ok e s => withMCtx s.meta.meta.mctx <| withEnv s.meta.core.env do addMessageContext m!"{e} : {← inferType e}" + | _ => unreachable! throwErrorAt f "ambiguous, possible interpretations {toMessageList msgs}" else withRef f <| mergeFailures candidates diff --git a/src/Lean/Elab/Attributes.lean b/src/Lean/Elab/Attributes.lean index 053dc8175110..1045f027aaf2 100644 --- a/src/Lean/Elab/Attributes.lean +++ b/src/Lean/Elab/Attributes.lean @@ -23,7 +23,7 @@ instance : ToFormat Attribute where | AttributeKind.scoped => "scoped " Format.bracket "@[" f!"{kindStr}{attr.name}{toString attr.stx}" "]" -/- +/-- ``` attrKind := leading_parser optional («scoped» <|> «local») ``` @@ -57,14 +57,17 @@ def elabAttr [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMa So, we expand them before here before we invoke the attributer handlers implemented using `AttrM`. -/ pure { kind := attrKind, name := attrName, stx := attr } -def elabAttrs [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] (attrInstances : Array Syntax) : m (Array Attribute) := do +def elabAttrs [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] [MonadLog m] [MonadLiftT IO m] (attrInstances : Array Syntax) : m (Array Attribute) := do let mut attrs := #[] for attr in attrInstances do - attrs := attrs.push (← elabAttr attr) + try + attrs := attrs.push (← withRef attr do elabAttr attr) + catch ex => + logException ex return attrs -- leading_parser "@[" >> sepBy1 attrInstance ", " >> "]" -def elabDeclAttrs [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] (stx : Syntax) : m (Array Attribute) := +def elabDeclAttrs [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] [MonadLog m] [MonadLiftT IO m] (stx : Syntax) : m (Array Attribute) := elabAttrs stx[1].getSepArgs end Lean.Elab diff --git a/src/Lean/Elab/AutoBound.lean b/src/Lean/Elab/AutoBound.lean index 132680d439fe..7887d73f2549 100644 --- a/src/Lean/Elab/AutoBound.lean +++ b/src/Lean/Elab/AutoBound.lean @@ -5,7 +5,7 @@ Authors: Leonardo de Moura -/ import Lean.Data.Options -/- Basic support for auto bound implicit local names -/ +/-! # Basic support for auto bound implicit local names -/ namespace Lean.Elab @@ -23,7 +23,7 @@ register_builtin_option relaxedAutoImplicit : Bool := { private def isValidAutoBoundSuffix (s : String) : Bool := s.toSubstring.drop 1 |>.all fun c => c.isDigit || isSubScriptAlnum c || c == '_' || c == '\'' -/- +/-! Remark: Issue #255 exposed a nasty interaction between macro scopes and auto-bound-implicit names. ``` local notation "A" => id x diff --git a/src/Lean/Elab/Binders.lean b/src/Lean/Elab/Binders.lean index 199c5c6bf8a5..d696daf64365 100644 --- a/src/Lean/Elab/Binders.lean +++ b/src/Lean/Elab/Binders.lean @@ -45,8 +45,8 @@ structure BinderView where bi : BinderInfo partial def quoteAutoTactic : Syntax → TermElabM Syntax - | stx@(Syntax.ident _ _ _ _) => throwErrorAt stx "invalid auto tactic, identifier is not allowed" - | stx@(Syntax.node _ k args) => do + | stx@(.ident ..) => throwErrorAt stx "invalid auto tactic, identifier is not allowed" + | stx@(.node _ k args) => do if stx.isAntiquot then throwErrorAt stx "invalid auto tactic, antiquotation is not allowed" else @@ -58,8 +58,8 @@ partial def quoteAutoTactic : Syntax → TermElabM Syntax let quotedArg ← quoteAutoTactic arg quotedArgs ← `(Array.push $quotedArgs $quotedArg) `(Syntax.node SourceInfo.none $(quote k) $quotedArgs) - | Syntax.atom _ val => `(mkAtom $(quote val)) - | Syntax.missing => throwError "invalid auto tactic, tactic is missing" + | .atom _ val => `(mkAtom $(quote val)) + | .missing => throwError "invalid auto tactic, tactic is missing" def declareTacticSyntax (tactic : Syntax) : TermElabM Name := withFreshMacroScope do @@ -75,7 +75,7 @@ def declareTacticSyntax (tactic : Syntax) : TermElabM Name := compileDecl decl return name -/- +/-- Expand `optional (binderTactic <|> binderDefault)` def binderTactic := leading_parser " := " >> " by " >> tacticParser def binderDefault := leading_parser " := " >> termParser @@ -108,28 +108,28 @@ private def matchBinder (stx : Syntax) : TermElabM (Array BinderView) := do let k := stx.getKind if stx.isIdent || k == ``hole then -- binderIdent - pure #[{ id := (← expandBinderIdent stx), type := mkHole stx, bi := BinderInfo.default }] + return #[{ id := (← expandBinderIdent stx), type := mkHole stx, bi := .default }] else if k == ``Lean.Parser.Term.explicitBinder then -- `(` binderIdent+ binderType (binderDefault <|> binderTactic)? `)` let ids ← getBinderIds stx[1] let type := stx[2] let optModifier := stx[3] - ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := (← expandBinderModifier (expandBinderType id type) optModifier), bi := BinderInfo.default } + ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := (← expandBinderModifier (expandBinderType id type) optModifier), bi := .default } else if k == ``Lean.Parser.Term.implicitBinder then -- `{` binderIdent+ binderType `}` let ids ← getBinderIds stx[1] let type := stx[2] - ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := expandBinderType id type, bi := BinderInfo.implicit } + ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := expandBinderType id type, bi := .implicit } else if k == ``Lean.Parser.Term.strictImplicitBinder then -- `⦃` binderIdent+ binderType `⦄` let ids ← getBinderIds stx[1] let type := stx[2] - ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := expandBinderType id type, bi := BinderInfo.strictImplicit } + ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := expandBinderType id type, bi := .strictImplicit } else if k == ``Lean.Parser.Term.instBinder then -- `[` optIdent type `]` let id ← expandOptIdent stx[1] let type := stx[2] - pure #[ { id := id, type := type, bi := BinderInfo.instImplicit } ] + return #[ { id := id, type := type, bi := .instImplicit } ] else throwUnsupportedSyntax @@ -149,11 +149,11 @@ register_builtin_option checkBinderAnnotations : Bool := { descr := "check whether type is a class instance whenever the binder annotation `[...]` is used" } -private partial def elabBinderViews {α} (binderViews : Array BinderView) (fvars : Array (Syntax × Expr)) (k : Array (Syntax × Expr) → TermElabM α) +private partial def elabBinderViews (binderViews : Array BinderView) (fvars : Array (Syntax × Expr)) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := let rec loop (i : Nat) (fvars : Array (Syntax × Expr)) : TermElabM α := do if h : i < binderViews.size then - let binderView := binderViews.get ⟨i, h⟩ + let binderView := binderViews[i] ensureAtomicBinderName binderView let type ← elabType binderView.type registerFailedToInferBinderTypeInfo type binderView.type @@ -167,10 +167,10 @@ private partial def elabBinderViews {α} (binderViews : Array BinderView) (fvars k fvars loop 0 fvars -private partial def elabBindersAux {α} (binders : Array Syntax) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := +private partial def elabBindersAux (binders : Array Syntax) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := let rec loop (i : Nat) (fvars : Array (Syntax × Expr)) : TermElabM α := do if h : i < binders.size then - let binderViews ← matchBinder (binders.get ⟨i, h⟩) + let binderViews ← matchBinder binders[i] elabBinderViews binderViews fvars <| loop (i+1) else k fvars @@ -181,7 +181,7 @@ private partial def elabBindersAux {α} (binders : Array Syntax) (k : Array (Syn `elabBinders(Ex)` automatically adds binder info nodes for the produced fvars, but storing the syntax nodes might be necessary when later adding the same binders back to the local context so that info nodes can manually be added for the new fvars; see `MutualDef` for an example. -/ -def elabBindersEx {α} (binders : Array Syntax) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := +def elabBindersEx (binders : Array Syntax) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := universeConstraintsCheckpoint do if binders.isEmpty then k #[] @@ -201,7 +201,7 @@ def elabBinders (binders : Array Syntax) (k : Array Expr → TermElabM α) : Ter elabBindersEx binders (fun fvars => k (fvars.map (·.2))) /-- Same as `elabBinder` with a single binder.-/ -def elabBinder {α} (binder : Syntax) (x : Expr → TermElabM α) : TermElabM α := +def elabBinder (binder : Syntax) (x : Expr → TermElabM α) : TermElabM α := elabBinders #[binder] fun fvars => x fvars[0]! def expandSimpleBinderWithType (type : Term) (binder : Syntax) : MacroM Syntax := @@ -289,7 +289,7 @@ private partial def getFunBinderIds? (stx : Syntax) : OptionT MacroM (Array Synt partial def expandFunBinders (binders : Array Syntax) (body : Syntax) : MacroM (Array Syntax × Syntax × Bool) := let rec loop (body : Syntax) (i : Nat) (newBinders : Array Syntax) := do if h : i < binders.size then - let binder := binders.get ⟨i, h⟩ + let binder := binders[i] let processAsPattern : Unit → MacroM (Array Syntax × Syntax × Bool) := fun _ => do let pattern := binder let major ← mkFreshIdent binder @@ -352,19 +352,19 @@ private def propagateExpectedType (fvar : Expr) (fvarType : Expr) (s : State) : | some expectedType => let expectedType ← whnfForall expectedType match expectedType with - | Expr.forallE _ d b _ => + | .forallE _ d b _ => discard <| isDefEq fvarType d let b := b.instantiate1 fvar - pure { s with expectedType? := some b } + return { s with expectedType? := some b } | _ => - pure { s with expectedType? := none } + return { s with expectedType? := none } private partial def elabFunBinderViews (binderViews : Array BinderView) (i : Nat) (s : State) : TermElabM State := do if h : i < binderViews.size then - let binderView := binderViews.get ⟨i, h⟩ + let binderView := binderViews[i] ensureAtomicBinderName binderView withRef binderView.type <| withLCtx s.lctx s.localInsts do - let type ← elabType binderView.type + let type ← elabType binderView.type registerFailedToInferBinderTypeInfo type binderView.type let fvarId ← mkFreshFVarId let fvar := mkFVar fvarId @@ -378,19 +378,19 @@ private partial def elabFunBinderViews (binderViews : Array BinderView) (i : Nat let lctx := s.lctx.mkLocalDecl fvarId binderView.id.getId type binderView.bi addTermInfo' (lctx? := some lctx) (isBinder := true) binderView.id fvar let s ← withRef binderView.id <| propagateExpectedType fvar type s - let s := { s with lctx := lctx } + let s := { s with lctx } match (← isClass? type) with | none => elabFunBinderViews binderViews (i+1) s | some className => resettingSynthInstanceCache do - let localInsts := s.localInsts.push { className := className, fvar := mkFVar fvarId } - elabFunBinderViews binderViews (i+1) { s with localInsts := localInsts } + let localInsts := s.localInsts.push { className, fvar := mkFVar fvarId } + elabFunBinderViews binderViews (i+1) { s with localInsts } else pure s partial def elabFunBindersAux (binders : Array Syntax) (i : Nat) (s : State) : TermElabM State := do if h : i < binders.size then - let binderViews ← matchBinder (binders.get ⟨i, h⟩) + let binderViews ← matchBinder binders[i] let s ← elabFunBinderViews binderViews 0 s elabFunBindersAux binders (i+1) s else @@ -398,13 +398,13 @@ partial def elabFunBindersAux (binders : Array Syntax) (i : Nat) (s : State) : T end FunBinders -def elabFunBinders {α} (binders : Array Syntax) (expectedType? : Option Expr) (x : Array Expr → Option Expr → TermElabM α) : TermElabM α := +def elabFunBinders (binders : Array Syntax) (expectedType? : Option Expr) (x : Array Expr → Option Expr → TermElabM α) : TermElabM α := if binders.isEmpty then x #[] expectedType? else do let lctx ← getLCtx let localInsts ← getLocalInstances - let s ← FunBinders.elabFunBindersAux binders 0 { lctx := lctx, localInsts := localInsts, expectedType? := expectedType? } + let s ← FunBinders.elabFunBindersAux binders 0 { lctx, localInsts, expectedType? } resettingSynthInstanceCacheWhen (s.localInsts.size > localInsts.size) <| withLCtx s.lctx s.localInsts <| x s.fvars s.expectedType? @@ -419,7 +419,7 @@ def expandWhereDeclsOpt (whereDeclsOpt : Syntax) (body : Syntax) : MacroM Syntax else expandWhereDecls whereDeclsOpt[0] body -/- Helper function for `expandMatchAltsIntoMatch` -/ +/-- Helper function for `expandMatchAltsIntoMatch` -/ private def expandMatchAltsIntoMatchAux (matchAlts : Syntax) (matchTactic : Bool) : Nat → Array Syntax → MacroM Syntax | 0, discrs => do if matchTactic then @@ -583,7 +583,7 @@ open Lean.Elab.Term.Quotation in mkLambdaFVars xs e | _ => throwUnsupportedSyntax -/- If `useLetExpr` is true, then a kernel let-expression `let x : type := val; body` is created. +/-- If `useLetExpr` is true, then a kernel let-expression `let x : type := val; body` is created. Otherwise, we create a term of the form `(fun (x : type) => body) val` The default elaboration order is `binders`, `typeStx`, `valStx`, and `body`. @@ -650,7 +650,7 @@ def mkLetIdDeclView (letIdDecl : Syntax) : LetIdDeclView := let optType := letIdDecl[2] let type := expandOptType id optType let value := letIdDecl[4] - { id := id, binders := binders, type := type, value := value } + { id, binders, type, value } def expandLetEqnsDecl (letDecl : Syntax) : MacroM Syntax := do let ref := letDecl @@ -662,8 +662,8 @@ def elabLetDeclCore (stx : Syntax) (expectedType? : Option Expr) (useLetExpr : B let letDecl := stx[1][0] let body := stx[3] if letDecl.getKind == ``Lean.Parser.Term.letIdDecl then - let { id := id, binders := binders, type := type, value := val } := mkLetIdDeclView letDecl - elabLetDeclAux id binders type val body expectedType? useLetExpr elabBodyFirst usedLetOnly + let { id, binders, type, value } := mkLetIdDeclView letDecl + elabLetDeclAux id binders type value body expectedType? useLetExpr elabBodyFirst usedLetOnly else if letDecl.getKind == ``Lean.Parser.Term.letPatDecl then -- node `Lean.Parser.Term.letPatDecl $ try (termParser >> pushNone >> optType >> " := ") >> termParser if elabBodyFirst then diff --git a/src/Lean/Elab/BindersUtil.lean b/src/Lean/Elab/BindersUtil.lean index 2c08ecac7a88..b6dc925fdeed 100644 --- a/src/Lean/Elab/BindersUtil.lean +++ b/src/Lean/Elab/BindersUtil.lean @@ -6,7 +6,7 @@ Authors: Leonardo de Moura import Lean.Parser.Term namespace Lean.Elab.Term -/- +/-- Recall that ``` def typeSpec := leading_parser " : " >> termParser @@ -21,7 +21,7 @@ def expandOptType (ref : Syntax) (optType : Syntax) : Syntax := open Lean.Parser.Term -/- Helper function for `expandEqnsIntoMatch` -/ +/-- Helper function for `expandEqnsIntoMatch` -/ def getMatchAltsNumPatterns (matchAlts : Syntax) : Nat := let alt0 := matchAlts[0][0] let pats := alt0[1][0].getSepArgs diff --git a/src/Lean/Elab/BuiltinNotation.lean b/src/Lean/Elab/BuiltinNotation.lean index bff865e8ee4e..cae20f5348d4 100644 --- a/src/Lean/Elab/BuiltinNotation.lean +++ b/src/Lean/Elab/BuiltinNotation.lean @@ -242,7 +242,7 @@ where | _ => Term.expandCDot? stx -/- +/-- Try to expand `·` notation. Recall that in Lean the `·` notation must be surrounded by parentheses. We may change this is the future, but right now, here are valid examples diff --git a/src/Lean/Elab/BuiltinTerm.lean b/src/Lean/Elab/BuiltinTerm.lean index 037deca1c6a6..8aaa29509224 100644 --- a/src/Lean/Elab/BuiltinTerm.lean +++ b/src/Lean/Elab/BuiltinTerm.lean @@ -26,7 +26,7 @@ private def elabOptLevel (stx : Syntax) : TermElabM Level := @[builtinTermElab «type»] def elabTypeStx : TermElab := fun stx _ => return mkSort (mkLevelSucc (← elabOptLevel stx[1])) -/- +/-! the method `resolveName` adds a completion point for it using the given expected type. Thus, we propagate the expected type if `stx[0]` is an identifier. It doesn't "hurt" if the identifier can be resolved because the expected type is not used in this case. @@ -205,7 +205,7 @@ def elabScientificLit : TermElab := fun stx expectedType? => do | some val => return mkApp (Lean.mkConst ``Char.ofNat) (mkRawNatLit val.toNat) | none => throwIllFormedSyntax -/- A literal of type `Name`. -/ +/-- A literal of type `Name`. -/ @[builtinTermElab quotedName] def elabQuotedName : TermElab := fun stx _ => match stx[0].isNameLit? with | some val => pure $ toExpr val diff --git a/src/Lean/Elab/Command.lean b/src/Lean/Elab/Command.lean index f3c29074d192..2254b7f50efd 100644 --- a/src/Lean/Elab/Command.lean +++ b/src/Lean/Elab/Command.lean @@ -239,7 +239,7 @@ private def elabCommandUsing (s : State) (stx : Syntax) : List (KeyedDeclsAttrib (withInfoTreeContext (mkInfoTree := mkInfoTree elabFn.declName stx) <| elabFn.value stx) (fun _ => do set s; elabCommandUsing s stx elabFns) -/- Elaborate `x` with `stx` on the macro stack -/ +/-- Elaborate `x` with `stx` on the macro stack -/ def withMacroExpansion {α} (beforeStx afterStx : Syntax) (x : CommandElabM α) : CommandElabM α := withInfoContext (mkInfo := pure <| .ofMacroExpansionInfo { stx := beforeStx, output := afterStx, lctx := .empty }) do withReader (fun ctx => { ctx with macroStack := { before := beforeStx, after := afterStx } :: ctx.macroStack }) x @@ -259,18 +259,6 @@ register_builtin_option showPartialSyntaxErrors : Bool := { descr := "show elaboration errors from partial syntax trees (i.e. after parser recovery)" } -def withLogging (x : CommandElabM Unit) : CommandElabM Unit := do - try - x - catch ex => match ex with - | Exception.error _ _ => logException ex - | Exception.internal id _ => - if isAbortExceptionId id then - pure () - else - let idName ← liftIO <| id.getName; - logError m!"internal exception {idName}" - builtin_initialize registerTraceClass `Elab.command partial def elabCommand (stx : Syntax) : CommandElabM Unit := do diff --git a/src/Lean/Elab/Config.lean b/src/Lean/Elab/Config.lean index 2f497c7b642a..f7ad2d85ca56 100644 --- a/src/Lean/Elab/Config.lean +++ b/src/Lean/Elab/Config.lean @@ -7,7 +7,7 @@ import Lean.Meta.Basic namespace Lean.Elab.Term -/- +/-- Set `isDefEq` configuration for the elaborator. Note that we enable all approximations but `quasiPatternApprox` diff --git a/src/Lean/Elab/DeclModifiers.lean b/src/Lean/Elab/DeclModifiers.lean index 45d454907360..ae9899a942fc 100644 --- a/src/Lean/Elab/DeclModifiers.lean +++ b/src/Lean/Elab/DeclModifiers.lean @@ -96,7 +96,7 @@ def expandOptDocComment? [Monad m] [MonadError m] (optDocComment : Syntax) : m ( section Methods -variable [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] +variable [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] [MonadLog m] [MonadLiftT IO m] def elabModifiers (stx : Syntax) : m Modifiers := do let docCommentStx := stx[0] @@ -183,7 +183,7 @@ def mkDeclName (currNamespace : Name) (modifiers : Modifiers) (shortName : Name) | _ => throwError "protected declarations must be in a namespace" | _ => pure (declName, shortName) -/- +/-- `declId` is of the form ``` leading_parser ident >> optional (".{" >> sepBy1 ident ", " >> "}") diff --git a/src/Lean/Elab/Declaration.lean b/src/Lean/Elab/Declaration.lean index ee14792a9084..4952d0a005ea 100644 --- a/src/Lean/Elab/Declaration.lean +++ b/src/Lean/Elab/Declaration.lean @@ -13,7 +13,6 @@ import Lean.Elab.DeclarationRange namespace Lean.Elab.Command open Meta -open TSyntax.Compat private def ensureValidNamespace (name : Name) : MacroM Unit := do match name with @@ -143,7 +142,7 @@ private def inductiveSyntaxToView (modifiers : Modifiers) (decl : Syntax) : Comm classes ← getOptDerivingClasses decl[5] else computedFields ← (decl[5].getOptional?.map (·[1].getArgs) |>.getD #[]).mapM fun cf => withRef cf do - return { ref := cf, modifiers := cf[0], fieldId := cf[1].getId, type := cf[3], matchAlts := cf[4] } + return { ref := cf, modifiers := cf[0], fieldId := cf[1].getId, type := ⟨cf[3]⟩, matchAlts := ⟨cf[4]⟩ } classes ← getOptDerivingClasses decl[6] return { ref := decl @@ -180,26 +179,29 @@ def elabDeclaration : CommandElab := fun stx => do match (← liftMacroM <| expandDeclNamespace? stx) with | some (ns, newStx) => do let ns := mkIdentFrom stx ns - let newStx ← `(namespace $ns:ident $newStx end $ns:ident) + let newStx ← `(namespace $ns:ident $(⟨newStx⟩) end $ns:ident) withMacroExpansion stx newStx <| elabCommand newStx | none => do - let modifiers ← elabModifiers stx[0] let decl := stx[1] let declKind := decl.getKind if declKind == ``Lean.Parser.Command.«axiom» then + let modifiers ← elabModifiers stx[0] elabAxiom modifiers decl else if declKind == ``Lean.Parser.Command.«inductive» then + let modifiers ← elabModifiers stx[0] elabInductive modifiers decl else if declKind == ``Lean.Parser.Command.classInductive then + let modifiers ← elabModifiers stx[0] elabClassInductive modifiers decl else if declKind == ``Lean.Parser.Command.«structure» then + let modifiers ← elabModifiers stx[0] elabStructure modifiers decl else if isDefLike decl then elabMutualDef #[stx] (getTerminationHints stx) else throwError "unexpected declaration" -/- Return true if all elements of the mutual-block are inductive declarations. -/ +/-- Return true if all elements of the mutual-block are inductive declarations. -/ private def isMutualInductive (stx : Syntax) : Bool := stx[1].getArgs.all fun elem => let decl := elem[1] @@ -212,7 +214,7 @@ private def elabMutualInductive (elems : Array Syntax) : CommandElabM Unit := do inductiveSyntaxToView modifiers stx[1] elabInductiveViews views -/- Return true if all elements of the mutual-block are definitions/theorems/abbrevs. -/ +/-- Return true if all elements of the mutual-block are definitions/theorems/abbrevs. -/ private def isMutualDef (stx : Syntax) : Bool := stx[1].getArgs.all fun elem => let decl := elem[1] @@ -257,7 +259,7 @@ def expandMutualNamespace : Macro := fun stx => do | some ns => let ns := mkIdentFrom stx ns let stxNew := stx.setArg 1 (mkNullNode elemsNew) - `(namespace $ns:ident $stxNew end $ns:ident) + `(namespace $ns:ident $(⟨stxNew⟩) end $ns:ident) | none => Macro.throwUnsupported @[builtinMacro Lean.Parser.Command.mutual] @@ -310,9 +312,10 @@ def elabMutual : CommandElab := fun stx => do for attrKindStx in stx[2].getSepArgs do if attrKindStx.getKind == ``Lean.Parser.Command.eraseAttr then let attrName := attrKindStx[1].getId.eraseMacroScopes - unless isAttribute (← getEnv) attrName do - throwError "unknown attribute [{attrName}]" - toErase := toErase.push attrName + if isAttribute (← getEnv) attrName then + toErase := toErase.push attrName + else + logErrorAt attrKindStx "unknown attribute [{attrName}]" else attrInsts := attrInsts.push attrKindStx let attrs ← elabAttrs attrInsts @@ -323,35 +326,19 @@ def elabMutual : CommandElab := fun stx => do for attrName in toErase do Attribute.erase declName attrName -def expandInitCmd (builtin : Bool) : Macro := fun stx => do - let optVisibility := stx[0] - let optHeader := stx[2] - let doSeq := stx[3] - let attrId := mkIdentFrom stx <| if builtin then `builtinInit else `init - if optHeader.isNone then - unless optVisibility.isNone do - Macro.throwError "invalid initialization command, 'visibility' modifer is not allowed" - `(@[$attrId:ident]def initFn : IO Unit := do $doSeq) - else - let id := optHeader[0] - let type := optHeader[1][1] - if optVisibility.isNone then - `(def initFn : IO $type := do $doSeq - @[$attrId:ident initFn] opaque $id : $type) - else if optVisibility[0].getKind == ``Parser.Command.private then - `(def initFn : IO $type := do $doSeq - @[$attrId:ident initFn] private opaque $id : $type) - else if optVisibility[0].getKind == ``Parser.Command.protected then - `(def initFn : IO $type := do $doSeq - @[$attrId:ident initFn] protected opaque $id : $type) +@[builtinMacro Lean.Parser.Command.«initialize»] def expandInitialize : Macro + | stx@`($declModifiers:declModifiers $kw:initializeKeyword $[$id? : $type? ←]? $doSeq) => do + let attrId := mkIdentFrom stx <| if kw.raw[0].isToken "initialize" then `init else `builtinInit + if let (some id, some type) := (id?, type?) then + let `(Parser.Command.declModifiersT| $[$doc?:docComment]? $[@[$attrs?,*]]? $(vis?)? $[unsafe%$unsafe?]?) := stx[0] + | Macro.throwErrorAt declModifiers "invalid initialization command, unexpected modifiers" + `($[unsafe%$unsafe?]? def initFn : IO $type := do $doSeq + $[$doc?:docComment]? @[$attrId:ident initFn, $(attrs?.getD ∅),*] $(vis?)? opaque $id : $type) else - Macro.throwError "unexpected visibility annotation" - -@[builtinMacro Lean.Parser.Command.«initialize»] def expandInitialize : Macro := - expandInitCmd (builtin := false) - -@[builtinMacro Lean.Parser.Command.«builtin_initialize»] def expandBuiltinInitialize : Macro := - expandInitCmd (builtin := true) + let `(Parser.Command.declModifiersT| ) := declModifiers + | Macro.throwErrorAt declModifiers "invalid initialization command, unexpected modifiers" + `(@[$attrId:ident] def initFn : IO Unit := do $doSeq) + | _ => Macro.throwUnsupported builtin_initialize registerTraceClass `Elab.axiom diff --git a/src/Lean/Elab/Deriving/FromToJson.lean b/src/Lean/Elab/Deriving/FromToJson.lean index 32872a120701..a0c1f61b49d6 100644 --- a/src/Lean/Elab/Deriving/FromToJson.lean +++ b/src/Lean/Elab/Deriving/FromToJson.lean @@ -30,7 +30,7 @@ def mkToJsonInstanceHandler (declNames : Array Name) : CommandElabM Bool := do let (isOptField, nm) := mkJsonField field if isOptField then ``(opt $nm $(mkIdent <| header.targetNames[0]! ++ field)) else ``([($nm, toJson $(mkIdent <| header.targetNames[0]! ++ field))]) - let cmd ← `(private def $(mkIdent ctx.auxFunNames[0]!):ident $header.binders:bracketedBinder* := + let cmd ← `(private def $(mkIdent ctx.auxFunNames[0]!):ident $header.binders:bracketedBinder* : Json := mkObj <| List.join [$fields,*]) return #[cmd] ++ (← mkInstanceCmds ctx ``ToJson declNames) cmds.forM elabCommand @@ -63,9 +63,9 @@ def mkToJsonInstanceHandler (declNames : Array Name) : CommandElabM Bool := do if ctx.usePartial then let letDecls ← mkLocalInstanceLetDecls ctx ``ToJson header.argNames let auxTerm ← mkLet letDecls auxTerm - `(private partial def $toJsonFuncId:ident $header.binders:bracketedBinder* := $auxTerm) + `(private partial def $toJsonFuncId:ident $header.binders:bracketedBinder* : Json := $auxTerm) else - `(private def $toJsonFuncId:ident $header.binders:bracketedBinder* := $auxTerm) + `(private def $toJsonFuncId:ident $header.binders:bracketedBinder* : Json := $auxTerm) return #[auxCmd] ++ (← mkInstanceCmds ctx ``ToJson declNames) cmds.forM elabCommand return true diff --git a/src/Lean/Elab/Deriving/Inhabited.lean b/src/Lean/Elab/Deriving/Inhabited.lean index b4677459df4d..e85736038fba 100644 --- a/src/Lean/Elab/Deriving/Inhabited.lean +++ b/src/Lean/Elab/Deriving/Inhabited.lean @@ -56,7 +56,7 @@ where | _ => pure () runST (fun _ => visit |>.run usedInstIdxs) |>.2 - /- Create an `instance` command using the constructor `ctorName` with a hypothesis `Inhabited α` when `α` is one of the inductive type parameters + /-- Create an `instance` command using the constructor `ctorName` with a hypothesis `Inhabited α` when `α` is one of the inductive type parameters at position `i` and `i ∈ assumingParamIdxs`. -/ mkInstanceCmdWith (assumingParamIdxs : IndexSet) : TermElabM Syntax := do let indVal ← getConstInfoInduct inductiveTypeName diff --git a/src/Lean/Elab/Deriving/SizeOf.lean b/src/Lean/Elab/Deriving/SizeOf.lean index c681a3da81da..f57f360f1ad9 100644 --- a/src/Lean/Elab/Deriving/SizeOf.lean +++ b/src/Lean/Elab/Deriving/SizeOf.lean @@ -6,7 +6,7 @@ Authors: Leonardo de Moura import Lean.Meta.SizeOf import Lean.Elab.Deriving.Basic -/- +/-! Remark: `SizeOf` instances are automatically generated. We add support for `deriving instance` for `SizeOf` just to be able to use them to define instances for types defined at `Prelude.lean` -/ diff --git a/src/Lean/Elab/Do.lean b/src/Lean/Elab/Do.lean index bbb25ade1dde..7ae5e7cddd7a 100644 --- a/src/Lean/Elab/Do.lean +++ b/src/Lean/Elab/Do.lean @@ -128,7 +128,7 @@ namespace Do abbrev Var := Syntax -- TODO: should be `Ident` -/- A `doMatch` alternative. `vars` is the array of variables declared by `patterns`. -/ +/-- A `doMatch` alternative. `vars` is the array of variables declared by `patterns`. -/ structure Alt (σ : Type) where ref : Syntax vars : Array Var @@ -136,7 +136,7 @@ structure Alt (σ : Type) where rhs : σ deriving Inhabited -/- +/-- Auxiliary datastructure for representing a `do` code block, and compiling "reassignments" (e.g., `x := x + 1`). We convert `Code` into a `Syntax` term representing the: - `do`-block, or @@ -187,22 +187,22 @@ structure Alt (σ : Type) where inductive Code where | decl (xs : Array Var) (doElem : Syntax) (k : Code) | reassign (xs : Array Var) (doElem : Syntax) (k : Code) - /- The Boolean value in `params` indicates whether we should use `(x : typeof! x)` when generating term Syntax or not -/ - | joinpoint (name : Name) (params : Array (Var × Bool)) (body : Code) (k : Code) + | /-- The Boolean value in `params` indicates whether we should use `(x : typeof! x)` when generating term Syntax or not -/ + joinpoint (name : Name) (params : Array (Var × Bool)) (body : Code) (k : Code) | seq (action : Syntax) (k : Code) | action (action : Syntax) | «break» (ref : Syntax) | «continue» (ref : Syntax) | «return» (ref : Syntax) (val : Syntax) - /- Recall that an if-then-else may declare a variable using `optIdent` for the branches `thenBranch` and `elseBranch`. We store the variable name at `var?`. -/ - | ite (ref : Syntax) (h? : Option Var) (optIdent : Syntax) (cond : Syntax) (thenBranch : Code) (elseBranch : Code) + | /-- Recall that an if-then-else may declare a variable using `optIdent` for the branches `thenBranch` and `elseBranch`. We store the variable name at `var?`. -/ + ite (ref : Syntax) (h? : Option Var) (optIdent : Syntax) (cond : Syntax) (thenBranch : Code) (elseBranch : Code) | «match» (ref : Syntax) (gen : Syntax) (discrs : Syntax) (optMotive : Syntax) (alts : Array (Alt Code)) | jmp (ref : Syntax) (jpName : Name) (args : Array Syntax) deriving Inhabited abbrev VarSet := Std.RBMap Name Syntax Name.cmp -/- A code block, and the collection of variables updated by it. -/ +/-- A code block, and the collection of variables updated by it. -/ structure CodeBlock where code : Code uvars : VarSet := {} -- set of variables updated by `code` @@ -231,7 +231,7 @@ partial def CodeBlocl.toMessageData (codeBlock : CodeBlock) : MessageData := ++ alts.foldl (init := m!"") fun acc alt => acc ++ m!"\n| {alt.patterns} => {loop alt.rhs}" loop codeBlock.code -/- Return true if the give code contains an exit point that satisfies `p` -/ +/-- Return true if the give code contains an exit point that satisfies `p` -/ partial def hasExitPointPred (c : Code) (p : Code → Bool) : Bool := let rec loop : Code → Bool | Code.decl _ _ k => loop k @@ -278,7 +278,7 @@ def mkAuxDeclFor {m} [Monad m] [MonadQuotation m] (e : Syntax) (mkCont : Syntax let k ← mkCont y return Code.decl #[y] doElem k -/- Convert `action _ e` instructions in `c` into `let y ← e; jmp _ jp (xs y)`. -/ +/-- Convert `action _ e` instructions in `c` into `let y ← e; jmp _ jp (xs y)`. -/ partial def convertTerminalActionIntoJmp (code : Code) (jp : Name) (xs : Array Var) : MacroM Code := let rec loop : Code → MacroM Code | Code.decl xs stx k => return Code.decl xs stx (← loop k) @@ -334,7 +334,7 @@ def eraseOptVar (rs : VarSet) (x? : Option Var) : VarSet := | none => rs | some x => rs.insert x.getId x -/- Create a new jointpoint for `c`, and jump to it with the variables `rs` -/ +/-- Create a new jointpoint for `c`, and jump to it with the variables `rs` -/ def mkSimpleJmp (ref : Syntax) (rs : VarSet) (c : Code) : StateRefT (Array JPDecl) TermElabM Code := do let xs := varSetToArray rs let jp ← addFreshJP (xs.map fun x => (x, true)) c @@ -344,7 +344,7 @@ def mkSimpleJmp (ref : Syntax) (rs : VarSet) (c : Code) : StateRefT (Array JPDec else return Code.jmp ref jp xs -/- Create a new joinpoint that takes `rs` and `val` as arguments. `val` must be syntax representing a pure value. +/-- Create a new joinpoint that takes `rs` and `val` as arguments. `val` must be syntax representing a pure value. The body of the joinpoint is created using `mkJPBody yFresh`, where `yFresh` is a fresh variable created by this method. -/ def mkJmp (ref : Syntax) (rs : VarSet) (val : Syntax) (mkJPBody : Syntax → MacroM Code) : StateRefT (Array JPDecl) TermElabM Code := do @@ -357,7 +357,7 @@ def mkJmp (ref : Syntax) (rs : VarSet) (val : Syntax) (mkJPBody : Syntax → Mac let jp ← addFreshJP ps jpBody return Code.jmp ref jp args -/- `pullExitPointsAux rs c` auxiliary method for `pullExitPoints`, `rs` is the set of update variable in the current path. -/ +/-- `pullExitPointsAux rs c` auxiliary method for `pullExitPoints`, `rs` is the set of update variable in the current path. -/ partial def pullExitPointsAux : VarSet → Code → StateRefT (Array JPDecl) TermElabM Code | rs, Code.decl xs stx k => return Code.decl xs stx (← pullExitPointsAux (eraseVars rs xs) k) | rs, Code.reassign xs stx k => return Code.reassign xs stx (← pullExitPointsAux (insertVars rs xs) k) @@ -375,7 +375,7 @@ partial def pullExitPointsAux : VarSet → Code → StateRefT (Array JPDecl) Ter let ref := e mkJmp ref rs y (fun yFresh => return Code.action (← ``(Pure.pure $yFresh))) -/- +/-- Auxiliary operation for adding new variables to the collection of updated variables in a CodeBlock. When a new variable is not already in the collection, but is shadowed by some declaration in `c`, we create auxiliary join points to make sure we preserve the semantics of the code block. @@ -458,7 +458,7 @@ partial def extendUpdatedVarsAux (c : Code) (ws : VarSet) : TermElabM Code := | c => return c update c -/- +/-- Extend the set of updated variables. It assumes `ws` is a super set of `c.uvars`. We **cannot** simply update the field `c.uvars`, because `c` may have shadowed some variable in `ws`. See discussion at `pullExitPoints`. @@ -473,7 +473,7 @@ partial def extendUpdatedVars (c : CodeBlock) (ws : VarSet) : TermElabM CodeBloc private def union (s₁ s₂ : VarSet) : VarSet := s₁.fold (·.insert ·) s₂ -/- +/-- Given two code blocks `c₁` and `c₂`, make sure they have the same set of updated variables. Let `ws` the union of the updated variables in `c₁‵ and ‵c₂`. We use `extendUpdatedVars c₁ ws` and `extendUpdatedVars c₂ ws` @@ -484,7 +484,7 @@ def homogenize (c₁ c₂ : CodeBlock) : TermElabM (CodeBlock × CodeBlock) := d let c₂ ← extendUpdatedVars c₂ ws pure (c₁, c₂) -/- +/-- Extending code blocks with variable declarations: `let x : t := v` and `let x : t ← v`. We remove `x` from the collection of updated varibles. Remark: `stx` is the syntax for the declaration (e.g., `letDecl`), and `xs` are the variables @@ -496,7 +496,7 @@ def mkVarDeclCore (xs : Array Var) (stx : Syntax) (c : CodeBlock) : CodeBlock := uvars := eraseVars c.uvars xs } -/- +/-- Extending code blocks with reassignments: `x : t := v` and `x : t ← v`. Remark: `stx` is the syntax for the declaration (e.g., `letDecl`), and `xs` are the variables declared by it. It is an array because we have let-declarations that declare multiple variables. @@ -554,7 +554,7 @@ def mkMatch (ref : Syntax) (genParam : Syntax) (discrs : Syntax) (optMotive : Sy return { ref := alt.ref, vars := alt.vars, patterns := alt.patterns, rhs := rhs.code : Alt Code } return { code := Code.«match» ref genParam discrs optMotive alts, uvars := ws } -/- Return a code block that executes `terminal` and then `k` with the value produced by `terminal`. +/-- Return a code block that executes `terminal` and then `k` with the value produced by `terminal`. This method assumes `terminal` is a terminal -/ def concat (terminal : CodeBlock) (kRef : Syntax) (y? : Option Var) (k : CodeBlock) : TermElabM CodeBlock := do unless hasTerminalAction terminal.code do @@ -669,7 +669,7 @@ def mkDoSeq (doElems : Array Syntax) : Syntax := def mkSingletonDoSeq (doElem : Syntax) : Syntax := mkDoSeq #[doElem] -/- +/-- If the given syntax is a `doIf`, return an equivalente `doIf` that has an `else` but no `else if`s or `if let`s. -/ private def expandDoIf? (stx : Syntax) : MacroM (Option Syntax) := match stx with | `(doElem|if $_:doIfProp then $_ else $_) => pure none @@ -694,7 +694,7 @@ structure DoIfView where thenBranch : Syntax elseBranch : Syntax -/- This method assumes `expandDoIf?` is not applicable. -/ +/-- This method assumes `expandDoIf?` is not applicable. -/ private def mkDoIfView (doIf : Syntax) : MacroM DoIfView := do pure { ref := doIf, @@ -704,7 +704,7 @@ private def mkDoIfView (doIf : Syntax) : MacroM DoIfView := do elseBranch := doIf[5][1] } -/- +/-- We use `MProd` instead of `Prod` to group values when expanding the `do` notation. `MProd` is a universe monomorphic product. The motivation is to generate simpler universe constraints in code @@ -722,7 +722,7 @@ private def mkTuple (elems : Array Syntax) : MacroM Syntax := do elems.extract 0 (elems.size - 1) |>.foldrM (init := elems.back) fun elem tuple => ``(MProd.mk $elem $tuple) -/- Return `some action` if `doElem` is a `doExpr `-/ +/-- Return `some action` if `doElem` is a `doExpr `-/ def isDoExpr? (doElem : Syntax) : Option Syntax := if doElem.getKind == ``Lean.Parser.Term.doExpr then some doElem[0] @@ -764,7 +764,7 @@ where `(let $a:ident := $x.1; let x := $x.2; $rest) | _ => unreachable! -/- +/-! The procedure `ToTerm.run` converts a `CodeBlock` into a `Syntax` term. We use this method to convert 1- The `CodeBlock` for a root `do ...` term into a `Syntax` term. This kind of @@ -1037,7 +1037,7 @@ partial def toTerm (c : Code) : M Syntax := do def run (code : Code) (m : Syntax) (returnType : Syntax) (uvars : Array Var := #[]) (kind := Kind.regular) : MacroM Syntax := toTerm code { m, returnType, kind, uvars } -/- Given +/-- Given - `a` is true if the code block has a `Code.action _` exit point - `r` is true if the code block has a `Code.return _ _` exit point - `bc` is true if the code block has a `Code.break _` or `Code.continue _` exit point @@ -1057,7 +1057,7 @@ def mkNestedKind (a r bc : Bool) : Kind := def mkNestedTerm (code : Code) (m : Syntax) (returnType : Syntax) (uvars : Array Var) (a r bc : Bool) : MacroM Syntax := do ToTerm.run code m returnType uvars (mkNestedKind a r bc) -/- Given a term `term` produced by `ToTerm.run`, pattern match on its result. +/-- Given a term `term` produced by `ToTerm.run`, pattern match on its result. See comment at the beginning of the `ToTerm` namespace. - `a` is true if the code block has a `Code.action _` exit point @@ -1208,7 +1208,7 @@ def checkLetArrowRHS (doElem : Syntax) : M Unit := do kind == ``Lean.Parser.Term.doReassignArrow then throwErrorAt doElem "invalid kind of value '{kind}' in an assignment" -/- Generate `CodeBlock` for `doReturn` which is of the form +/-- Generate `CodeBlock` for `doReturn` which is of the form ``` "return " >> optional termParser ``` @@ -1240,7 +1240,7 @@ def tryCatchPred (tryCode : CodeBlock) (catches : Array Catch) (finallyCode? : O | some finallyCode => p finallyCode.code mutual - /- "Concatenate" `c` with `doSeqToCode doElems` -/ + /-- "Concatenate" `c` with `doSeqToCode doElems` -/ partial def concatWith (c : CodeBlock) (doElems : List Syntax) : M CodeBlock := match doElems with | [] => pure c @@ -1249,7 +1249,7 @@ mutual let ref := nextDoElem concat c ref none k - /- Generate `CodeBlock` for `doLetArrow; doElems` + /-- Generate `CodeBlock` for `doLetArrow; doElems` `doLetArrow` is of the form ``` "let " >> optional "mut " >> (doIdDecl <|> doPatDecl) @@ -1304,7 +1304,7 @@ mutual let auxDo ← `(do let discr := $val; match discr with | $pattern:term => $contSeq | _ => $elseSeq) doSeqToCode <| getDoSeqElems (getDoSeq auxDo) - /- Generate `CodeBlock` for `doReassignArrow; doElems` + /-- Generate `CodeBlock` for `doReassignArrow; doElems` `doReassignArrow` is of the form ``` (doIdDecl <|> doPatDecl) @@ -1329,7 +1329,7 @@ mutual else throwError "unexpected kind of 'do' reassignment" - /- Generate `CodeBlock` for `doIf; doElems` + /-- Generate `CodeBlock` for `doIf; doElems` `doIf` is of the form ``` "if " >> optIdent >> termParser >> " then " >> doSeq @@ -1343,7 +1343,7 @@ mutual let ite ← mkIte view.ref view.optIdent view.cond thenBranch elseBranch concatWith ite doElems - /- Generate `CodeBlock` for `doUnless; doElems` + /-- Generate `CodeBlock` for `doUnless; doElems` `doUnless` is of the form ``` "unless " >> termParser >> "do " >> doSeq @@ -1355,7 +1355,7 @@ mutual let unlessCode ← liftMacroM <| mkUnless cond body concatWith unlessCode doElems - /- Generate `CodeBlock` for `doFor; doElems` + /-- Generate `CodeBlock` for `doFor; doElems` `doFor` is of the form ``` def doForDecl := leading_parser termParser >> " in " >> withForbidden "do" termParser diff --git a/src/Lean/Elab/Extra.lean b/src/Lean/Elab/Extra.lean index d092458f061c..644f1e52bd6f 100644 --- a/src/Lean/Elab/Extra.lean +++ b/src/Lean/Elab/Extra.lean @@ -5,9 +5,7 @@ Authors: Leonardo de Moura -/ import Lean.Elab.App -/- -Auxiliary elaboration functions: AKA custom elaborators --/ +/-! # Auxiliary elaboration functions: AKA custom elaborators -/ namespace Lean.Elab.Term open Meta @@ -38,15 +36,15 @@ private def throwForInFailure (forInInstance : Expr) : TermElabM Expr := catch _ => tryPostpone; throwError "failed to construct 'ForIn' instance for collection{indentExpr colType}\nand monad{indentExpr m}" match (← trySynthInstance forInInstance) with - | LOption.some inst => + | .some inst => let forInFn ← mkConst ``forIn elabAppArgs forInFn (namedArgs := #[{ name := `m, val := Arg.expr m}, { name := `α, val := Arg.expr elemType }, { name := `self, val := Arg.expr inst }]) (args := #[Arg.stx col, Arg.stx init, Arg.stx body]) (expectedType? := expectedType?) (explicit := false) (ellipsis := false) (resultIsOutParamSupport := false) - | LOption.undef => tryPostpone; throwForInFailure forInInstance - | LOption.none => throwForInFailure forInInstance + | .undef => tryPostpone; throwForInFailure forInInstance + | .none => throwForInFailure forInInstance | _ => throwUnsupportedSyntax @[builtinTermElab forInMacro'] def elabForIn' : TermElab := fun stx expectedType? => do @@ -66,19 +64,19 @@ private def throwForInFailure (forInInstance : Expr) : TermElabM Expr := catch _ => tryPostpone; throwError "failed to construct `ForIn'` instance for collection{indentExpr colType}\nand monad{indentExpr m}" match (← trySynthInstance forInInstance) with - | LOption.some inst => + | .some inst => let forInFn ← mkConst ``forIn' elabAppArgs forInFn (namedArgs := #[{ name := `m, val := Arg.expr m}, { name := `α, val := Arg.expr elemType}, { name := `self, val := Arg.expr inst }]) (args := #[Arg.expr colFVar, Arg.stx init, Arg.stx body]) (expectedType? := expectedType?) (explicit := false) (ellipsis := false) (resultIsOutParamSupport := false) - | LOption.undef => tryPostpone; throwForInFailure forInInstance - | LOption.none => throwForInFailure forInInstance + | .undef => tryPostpone; throwForInFailure forInInstance + | .none => throwForInFailure forInInstance | _ => throwUnsupportedSyntax namespace BinOp -/- +/-! The elaborator for `binop%` terms works as follows: @@ -157,9 +155,9 @@ private def hasCoe (fromType toType : Expr) : TermElabM Bool := do let v ← getLevel toType let coeInstType := mkAppN (Lean.mkConst ``CoeHTCT [u, v]) #[fromType, toType] match ← trySynthInstance coeInstType (some (maxCoeSize.get (← getOptions))) with - | LOption.some _ => return true - | LOption.none => return false - | LOption.undef => return false -- TODO: should we do something smarter here? + | .some _ => return true + | .none => return false + | .undef => return false -- TODO: should we do something smarter here? else return false @@ -168,10 +166,10 @@ private structure AnalyzeResult where hasUncomparable : Bool := false -- `true` if there are two types `α` and `β` where we don't have coercions in any direction. private def isUnknow : Expr → Bool - | Expr.mvar .. => true - | Expr.app f .. => isUnknow f - | Expr.letE _ _ _ b _ => isUnknow b - | Expr.mdata _ b => isUnknow b + | .mvar .. => true + | .app f _ => isUnknow f + | .letE _ _ _ b _ => isUnknow b + | .mdata _ b => isUnknow b | _ => false private def analyze (t : Tree) (expectedType? : Option Expr) : TermElabM AnalyzeResult := do @@ -205,15 +203,11 @@ where private def mkOp (f : Expr) (lhs rhs : Expr) : TermElabM Expr := elabAppArgs f #[] #[Arg.expr lhs, Arg.expr rhs] (expectedType? := none) (explicit := false) (ellipsis := false) (resultIsOutParamSupport := false) -private def toExpr (t : Tree) : TermElabM Expr := do +private def toExprCore (t : Tree) : TermElabM Expr := do match t with - | Tree.term _ e => return e - | Tree.op ref true f lhs rhs => withRef ref <| mkOp f (← toExpr lhs) (← mkFunUnit (← toExpr rhs)) - | Tree.op ref false f lhs rhs => withRef ref <| mkOp f (← toExpr lhs) (← toExpr rhs) - -private def getResultingType : Expr → Expr - | .forallE _ _ b _ => getResultingType b - | e => e + | .term _ e => return e + | .op ref true f lhs rhs => withRef ref <| mkOp f (← toExprCore lhs) (← mkFunUnit (← toExprCore rhs)) + | .op ref false f lhs rhs => withRef ref <| mkOp f (← toExprCore lhs) (← toExprCore rhs) /-- Auxiliary function to decide whether we should coerce `f`'s argument to `maxType` or not. @@ -245,66 +239,96 @@ private def hasHeterogeneousDefaultInstances (f : Expr) (maxType : Expr) (lhs : let className := fName.getPrefix let defInstances ← getDefaultInstances className if defInstances.length ≤ 1 then return false - for (instName, _) in (← getDefaultInstances className) do - let instInfo ← getConstInfo instName - let type := getResultingType instInfo.type - if type.getAppNumArgs >= 3 then - if lhs then - return type.appFn!.appArg!.isAppOf typeName - else - return type.appFn!.appArg!.appArg!.isAppOf typeName + for (instName, _) in defInstances do + if let .app (.app (.app _heteroClass lhsType) rhsType) _resultType := + (← getConstInfo instName).type.getForallBody then + if lhs && rhsType.isAppOf typeName then return true + if !lhs && lhsType.isAppOf typeName then return true return false /-- - Try to coerce elements in the `t` to `maxType` when needed. - If the type of an element in `t` is unknown we only coerce it to `maxType` if `maxType` does not have heterogeneous - default instances. This extra check is approximated by `hasHeterogeneousDefaultInstances`. + Return `true` if polymorphic function `f` has a homogenous instance of `maxType`. + The coercions to `maxType` only makes sense if such instance exists. - Remark: If `maxType` does not implement heterogeneous default instances, we do want to assign unknown types `?m` to - `maxType` because it produces better type information propagation. Our test suite has many tests that would break if - we don't do this. For example, consider the term - ``` - eq_of_isEqvAux a b hsz (i+1) (Nat.succ_le_of_lt h) heqv.2 - ``` - `Nat.succ_le_of_lt h` type depends on `i+1`, but `i+1` only reduces to `Nat.succ i` if we know that `1` is a `Nat`. - There are several other examples like that in our test suite, and one can find them by just replacing the - `← hasHeterogeneousDefaultInstances f maxType lhs` test with `true` + For example, suppose `maxType` is `Int`, and `f` is `HPow.hPow`. Then, + adding coercions to `maxType` only make sense if we have an instance `HPow Int Int Int`. +-/ +private def hasHomogeneousInstance (f : Expr) (maxType : Expr) : MetaM Bool := do + let .const fName .. := f | return false + let className := fName.getPrefix + try + let inst ← mkAppM className #[maxType, maxType, maxType] + return (← trySynthInstance inst) matches .some _ + catch _ => + return false +mutual + /-- + Try to coerce elements in the `t` to `maxType` when needed. + If the type of an element in `t` is unknown we only coerce it to `maxType` if `maxType` does not have heterogeneous + default instances. This extra check is approximated by `hasHeterogeneousDefaultInstances`. + + Remark: If `maxType` does not implement heterogeneous default instances, we do want to assign unknown types `?m` to + `maxType` because it produces better type information propagation. Our test suite has many tests that would break if + we don't do this. For example, consider the term + ``` + eq_of_isEqvAux a b hsz (i+1) (Nat.succ_le_of_lt h) heqv.2 + ``` + `Nat.succ_le_of_lt h` type depends on `i+1`, but `i+1` only reduces to `Nat.succ i` if we know that `1` is a `Nat`. + There are several other examples like that in our test suite, and one can find them by just replacing the + `← hasHeterogeneousDefaultInstances f maxType lhs` test with `true` + + + Remark: if `hasHeterogeneousDefaultInstances` implementation is not good enough we should refine it in the future. + -/ + private partial def applyCoe (t : Tree) (maxType : Expr) (isPred : Bool) : TermElabM Tree := do + go t none false isPred + where + go (t : Tree) (f? : Option Expr) (lhs : Bool) (isPred : Bool) : TermElabM Tree := do + match t with + | .op ref lazy f lhs rhs => + /- + We only keep applying coercions to `maxType` if `f` is predicate or + `f` has a homogenous instance with `maxType`. See `hasHomogeneousInstance` for additional details. + + Remark: We assume `binrel%` elaborator is only used with homogenous predicates. + -/ + if (← pure isPred <||> hasHomogeneousInstance f maxType) then + return Tree.op ref lazy f (← go lhs f true false) (← go rhs f false false) + else + let lhs ← toExpr lhs none + let rhs ← toExpr rhs none + return Tree.term ref (← mkOp f lhs rhs) + | .term ref e => + let type ← instantiateMVars (← inferType e) + trace[Elab.binop] "visiting {e} : {type} =?= {maxType}" + if isUnknow type then + if let some f := f? then + if (← hasHeterogeneousDefaultInstances f maxType lhs) then + -- See comment at `hasHeterogeneousDefaultInstances` + return t + if (← isDefEqGuarded maxType type) then + return t + else + trace[Elab.binop] "added coercion: {e} : {type} => {maxType}" + withRef ref <| return Tree.term ref (← mkCoe maxType type e) + + private partial def toExpr (tree : Tree) (expectedType? : Option Expr) : TermElabM Expr := do + let r ← analyze tree expectedType? + trace[Elab.binop] "hasUncomparable: {r.hasUncomparable}, maxType: {r.max?}" + if r.hasUncomparable || r.max?.isNone then + let result ← toExprCore tree + ensureHasType expectedType? result + else + let result ← toExprCore (← applyCoe tree r.max?.get! (isPred := false)) + trace[Elab.binop] "result: {result}" + ensureHasType expectedType? result - Remark: if `hasHeterogeneousDefaultInstances` implementation is not good enough we should refine it in the future. --/ -private def applyCoe (t : Tree) (maxType : Expr) : TermElabM Tree := do - go t none false -where - go (t : Tree) (f? : Option Expr) (lhs : Bool) : TermElabM Tree := do - match t with - | Tree.op ref lazy f lhs rhs => return Tree.op ref lazy f (← go lhs f true) (← go rhs f false) - | Tree.term ref e => - let type ← instantiateMVars (← inferType e) - trace[Elab.binop] "visiting {e} : {type} =?= {maxType}" - if isUnknow type then - if let some f := f? then - if (← hasHeterogeneousDefaultInstances f maxType lhs) then - -- See comment at `hasHeterogeneousDefaultInstances` - return t - if (← isDefEqGuarded maxType type) then - return t - else - trace[Elab.binop] "added coercion: {e} : {type} => {maxType}" - withRef ref <| return Tree.term ref (← mkCoe maxType type e) +end @[builtinTermElab binop] def elabBinOp : TermElab := fun stx expectedType? => do - let tree ← toTree stx - let r ← analyze tree expectedType? - trace[Elab.binop] "hasUncomparable: {r.hasUncomparable}, maxType: {r.max?}" - if r.hasUncomparable || r.max?.isNone then - let result ← toExpr tree - ensureHasType expectedType? result - else - let result ← toExpr (← applyCoe tree r.max?.get!) - trace[Elab.binop] "result: {result}" - ensureHasType expectedType? result + toExpr (← toTree stx) expectedType? @[builtinTermElab binop_lazy] def elabBinOpLazy : TermElab := elabBinOp @@ -327,8 +351,8 @@ def elabBinRelCore (noProp : Bool) (stx : Syntax) (expectedType? : Option Expr) trace[Elab.binrel] "hasUncomparable: {r.hasUncomparable}, maxType: {r.max?}" if r.hasUncomparable || r.max?.isNone then -- Use default elaboration strategy + `toBoolIfNecessary` - let lhs ← toExpr lhs - let rhs ← toExpr rhs + let lhs ← toExprCore lhs + let rhs ← toExprCore rhs let lhs ← toBoolIfNecessary lhs let rhs ← toBoolIfNecessary rhs let lhsType ← inferType lhs @@ -340,7 +364,7 @@ def elabBinRelCore (noProp : Bool) (stx : Syntax) (expectedType? : Option Expr) if noProp then if (← withNewMCtxDepth <| isDefEq maxType (mkSort levelZero)) then maxType := Lean.mkConst ``Bool - let result ← toExpr (← applyCoe tree maxType) + let result ← toExprCore (← applyCoe tree maxType (isPred := true)) trace[Elab.binrel] "result: {result}" return result | none => throwUnknownConstant stx[1].getId diff --git a/src/Lean/Elab/Inductive.lean b/src/Lean/Elab/Inductive.lean index 65bed617de74..7221dd33775c 100644 --- a/src/Lean/Elab/Inductive.lean +++ b/src/Lean/Elab/Inductive.lean @@ -173,7 +173,7 @@ private def elabHeader (views : Array InductiveView) : TermElabM (Array ElabHead checkHeaders rs numParams 0 none return rs -/- Create a local declaration for each inductive type in `rs`, and execute `x params indFVars`, where `params` are the inductive type parameters and +/-- Create a local declaration for each inductive type in `rs`, and execute `x params indFVars`, where `params` are the inductive type parameters and `indFVars` are the new local declarations. We use the local context/instances and parameters of rs[0]. Note that this method is executed after we executed `checkHeaders` and established all @@ -295,7 +295,7 @@ private def withExplicitToImplicit (xs : Array Expr) (k : TermElabM α) : TermEl toImplicit := toImplicit.push (x.fvarId!, BinderInfo.implicit) withNewBinderInfos toImplicit k -/- +/-- Elaborate constructor types. Remark: we check whether the resulting type is correct, and the parameter occurrences are consistent, but @@ -615,7 +615,7 @@ private def mkIndFVar2Const (views : Array InductiveView) (indFVars : Array Expr m := m.insert indFVar (mkConst view.declName levelParams) return m -/- Remark: `numVars <= numParams`. `numVars` is the number of context `variables` used in the inductive declaration, +/-- Remark: `numVars <= numParams`. `numVars` is the number of context `variables` used in the inductive declaration, and `numParams` is `numVars` + number of explicit parameters provided in the declaration. -/ private def replaceIndFVarsWithConsts (views : Array InductiveView) (indFVars : Array Expr) (levelNames : List Name) (numVars : Nat) (numParams : Nat) (indTypes : List InductiveType) : TermElabM (List InductiveType) := diff --git a/src/Lean/Elab/MacroArgUtil.lean b/src/Lean/Elab/MacroArgUtil.lean index 4f605981a2a8..16e84d9dbc81 100644 --- a/src/Lean/Elab/MacroArgUtil.lean +++ b/src/Lean/Elab/MacroArgUtil.lean @@ -10,7 +10,7 @@ open Lean.Syntax open Lean.Parser.Term hiding macroArg open Lean.Parser.Command -/- Convert `macro` arg into a `syntax` command item and a pattern element -/ +/-- Convert `macro` arg into a `syntax` command item and a pattern element -/ partial def expandMacroArg (stx : TSyntax ``macroArg) : CommandElabM (TSyntax `stx × Term) := do let (id?, id, stx) ← match (← liftMacroM <| expandMacros stx) with | `(macroArg| $id:ident:$stx) => pure (some id, (id : Term), stx) diff --git a/src/Lean/Elab/MacroRules.lean b/src/Lean/Elab/MacroRules.lean index f3e964809ca3..57c0f5e5249f 100644 --- a/src/Lean/Elab/MacroRules.lean +++ b/src/Lean/Elab/MacroRules.lean @@ -11,7 +11,7 @@ open Lean.Syntax open Lean.Parser.Term hiding macroArg open Lean.Parser.Command -/- +/-- Remark: `k` is the user provided kind with the current namespace included. Recall that syntax node kinds contain the current namespace. -/ diff --git a/src/Lean/Elab/Match.lean b/src/Lean/Elab/Match.lean index 5228c0c44ff6..dc239f1441bd 100644 --- a/src/Lean/Elab/Match.lean +++ b/src/Lean/Elab/Match.lean @@ -76,7 +76,7 @@ structure Discr where structure ElabMatchTypeAndDiscrsResult where discrs : Array Discr matchType : Expr - /- `true` when performing dependent elimination. We use this to decide whether we optimize the "match unit" case. + /-- `true` when performing dependent elimination. We use this to decide whether we optimize the "match unit" case. See `isMatchUnit?`. -/ isDep : Bool alts : Array MatchAltView @@ -92,7 +92,7 @@ private partial def elabMatchTypeAndDiscrs (discrStxs : Array Syntax) (matchOptM let (discrs, isDep) ← elabDiscrsWitMatchType matchType return { discrs := discrs, matchType := matchType, isDep := isDep, alts := matchAltViews } where - /- Easy case: elaborate discriminant when the match-type has been explicitly provided by the user. -/ + /-- Easy case: elaborate discriminant when the match-type has been explicitly provided by the user. -/ elabDiscrsWitMatchType (matchType : Expr) : TermElabM (Array Discr × Bool) := do let mut discrs := #[] let mut i := 0 @@ -116,7 +116,7 @@ where markIsDep (r : ElabMatchTypeAndDiscrsResult) := { r with isDep := true } - /- Elaborate discriminants inferring the match-type -/ + /-- Elaborate discriminants inferring the match-type -/ elabDiscrs (i : Nat) (discrs : Array Discr) : TermElabM ElabMatchTypeAndDiscrsResult := do if h : i < discrStxs.size then let discrStx := discrStxs.get ⟨i, h⟩ @@ -153,7 +153,7 @@ private def getMatchGeneralizing? : Syntax → Option Bool | `(match (generalizing := false) $[$motive]? $_discrs,* with $_alts:matchAlt*) => some false | _ => none -/- Given `stx` a match-expression, return its alternatives. -/ +/-- Given `stx` a match-expression, return its alternatives. -/ private def getMatchAlts : Syntax → Array MatchAltView | `(match $[$gen]? $[$motive]? $_discrs,* with $alts:matchAlt*) => alts.filterMap fun alt => match alt with @@ -180,7 +180,7 @@ open Lean.Elab.Term.Quotation in Quotation.withNewLocals (getPatternVarNames vars) <| precheck rhs | _ => throwUnsupportedSyntax -/- We convert the collected `PatternVar`s intro `PatternVarDecl` -/ +/-- We convert the collected `PatternVar`s intro `PatternVarDecl` -/ structure PatternVarDecl where fvarId : FVarId @@ -195,7 +195,7 @@ private partial def withPatternVars {α} (pVars : Array PatternVar) (k : Array P k decls loop 0 #[] #[] -/- +/-! Remark: when performing dependent pattern matching, we often had to write code such as ```lean @@ -217,7 +217,7 @@ try to "sort" the new discriminants. If the refinement process fails, we report the original error message. -/ -/- Auxiliary structure for storing an type mismatch exception when processing the +/-- Auxiliary structure for storing an type mismatch exception when processing the pattern #`idx` of some alternative. -/ structure PatternElabException where ex : Exception @@ -646,11 +646,11 @@ where partial def savePatternInfo (p : Expr) : TermElabM Expr := go p |>.run false where - /- The `Bool` context is true iff we are inside of an "inaccessible" pattern. -/ + /-- The `Bool` context is true iff we are inside of an "inaccessible" pattern. -/ go (p : Expr) : ReaderT Bool TermElabM Expr := do match p with - | .forallE n d b _ => withLocalDecl n b.binderInfo (← go d) fun x => do mkForallFVars #[x] (← go (b.instantiate1 x)) - | .lam n d b _ => withLocalDecl n b.binderInfo (← go d) fun x => do mkLambdaFVars #[x] (← go (b.instantiate1 x)) + | .forallE n d b bi => withLocalDecl n bi (← go d) fun x => do mkForallFVars #[x] (← go (b.instantiate1 x)) + | .lam n d b bi => withLocalDecl n bi (← go d) fun x => do mkLambdaFVars #[x] (← go (b.instantiate1 x)) | .letE n t v b .. => withLetDecl n (← go t) (← go v) fun x => do mkLetFVars #[x] (← go (b.instantiate1 x)) | .app f a => return mkApp (← go f) (← go a) | .proj _ _ b => return p.updateProj! (← go b) @@ -896,7 +896,7 @@ private def generalize (discrs : Array Discr) (matchType : Expr) (altViews : Arr private partial def elabMatchAltViews (generalizing? : Option Bool) (discrs : Array Discr) (matchType : Expr) (altViews : Array MatchAltView) : TermElabM (Array Discr × Expr × Array (AltLHS × Expr) × Bool) := do loop discrs #[] matchType altViews none where - /- + /-- "Discriminant refinement" main loop. `first?` contains the first error message we found before updated the `discrs`. -/ loop (discrs : Array Discr) (toClear : Array FVarId) (matchType : Expr) (altViews : Array MatchAltView) (first? : Option (SavedState × Exception)) @@ -953,7 +953,7 @@ where containsFVar (es : Array Expr) (fvarId : FVarId) : Bool := es.any fun e => e.isFVar && e.fvarId! == fvarId - /- Update `indices` by including any free variable `x` s.t. + /-- Update `indices` by including any free variable `x` s.t. - Type of some `discr` depends on `x`. - Type of `x` depends on some free variable in `indices`. @@ -1086,14 +1086,16 @@ private def elabMatchAux (generalizing? : Option Bool) (discrStxs : Array Syntax -/ withRef altLHS.ref do for d in altLHS.fvarDecls do - if d.hasExprMVar then + if d.hasExprMVar then + tryPostpone withExistingLocalDecls altLHS.fvarDecls do - tryPostpone - throwMVarError m!"invalid match-expression, type of pattern variable '{d.toExpr}' contains metavariables{indentExpr d.type}" + runPendingTacticsAt d.type + if (← instantiateMVars d.type).hasExprMVar then + throwMVarError m!"invalid match-expression, type of pattern variable '{d.toExpr}' contains metavariables{indentExpr d.type}" for p in altLHS.patterns do - if p.hasExprMVar then + if (← Match.instantiatePatternMVars p).hasExprMVar then + tryPostpone withExistingLocalDecls altLHS.fvarDecls do - tryPostpone throwMVarError m!"invalid match-expression, pattern contains metavariables{indentExpr (← p.toExpr)}" pure altLHS return (discrs, matchType, altLHSS, isDep, rhss) @@ -1174,7 +1176,7 @@ private def tryPostponeIfDiscrTypeIsMVar (matchStx : Syntax) : TermElabM Unit := trace[Elab.match] "discr {d} : {dType}" tryPostponeIfMVar dType -/- +/-- We (try to) elaborate a `match` only when the expected type is available. If the `matchType` has not been provided by the user, we also try to postpone elaboration if the type of a discriminant is not available. That is, it is of the form `(?m ...)`. @@ -1211,7 +1213,7 @@ private def waitExpectedTypeAndDiscrs (matchStx : Syntax) (expectedType? : Optio | some expectedType => return expectedType | none => mkFreshTypeMVar -/- +/-- ``` leading_parser "match " >> optional generalizingParam >> optional motive >> sepBy1 matchDiscr ", " >> " with " >> ppDedent matchAlts ``` diff --git a/src/Lean/Elab/MatchAltView.lean b/src/Lean/Elab/MatchAltView.lean index 40c47578c98b..30ae0b676617 100644 --- a/src/Lean/Elab/MatchAltView.lean +++ b/src/Lean/Elab/MatchAltView.lean @@ -7,7 +7,7 @@ import Lean.Elab.Term namespace Lean.Elab.Term -/- This modules assumes "match"-expressions use the following syntax. +/-! This module assumes `match`-expressions use the following syntax. ```lean def matchDiscr := leading_parser optional (try (ident >> checkNoWsBefore "no space before ':'" >> ":")) >> termParser diff --git a/src/Lean/Elab/MutualDef.lean b/src/Lean/Elab/MutualDef.lean index ca704343cf7e..b3671dd93ef1 100644 --- a/src/Lean/Elab/MutualDef.lean +++ b/src/Lean/Elab/MutualDef.lean @@ -16,7 +16,7 @@ import Lean.Elab.DeclarationRange namespace Lean.Elab open Lean.Parser.Term -/- DefView after elaborating the header. -/ +/-- `DefView` after elaborating the header. -/ structure DefViewElabHeader where ref : Syntax modifiers : Modifiers @@ -263,7 +263,7 @@ private def getFunName (fvarId : FVarId) (letRecsToLift : List LetRecToLift) : T | none => throwError "unknown function" | some n => pure n -/- +/-- Ensures that the of let-rec definition types do not contain functions being defined. In principle, this test can be improved. We could perform it after we separate the set of functions is strongly connected components. However, this extra complication doesn't seem worth it. @@ -278,10 +278,10 @@ private def checkLetRecsToLiftTypes (funVars : Array Expr) (letRecsToLift : List namespace MutualClosure -/- A mapping from FVarId to Set of FVarIds. -/ +/-- A mapping from FVarId to Set of FVarIds. -/ abbrev UsedFVarsMap := FVarIdMap FVarIdSet -/- +/-- Create the `UsedFVarsMap` mapping that takes the variable id for the mutually recursive functions being defined to the set of free variables in its definition. @@ -348,7 +348,7 @@ private def mkInitialUsedFVarsMap [Monad m] [MonadMCtx m] (sectionVars : Array E usedFVarMap := usedFVarMap.insert toLift.fvarId set return usedFVarMap -/- +/-! The let-recs may invoke each other. Example: ``` let rec @@ -456,7 +456,7 @@ private def preprocess (e : Expr) : TermElabM Expr := do Meta.check e pure e -/- Push free variables in `s` to `toProcess` if they are not already there. -/ +/-- Push free variables in `s` to `toProcess` if they are not already there. -/ private def pushNewVars (toProcess : Array FVarId) (s : CollectFVars.State) : Array FVarId := s.fvarSet.fold (init := toProcess) fun toProcess fvarId => if toProcess.contains fvarId then toProcess else toProcess.push fvarId @@ -551,7 +551,7 @@ private def mkLetRecClosures (sectionVars : Array Expr) (mainFVarIds : Array FVa result := result.push (← mkLetRecClosureFor toLift (freeVarMap.find? toLift.fvarId).get!) return result.toList -/- Mapping from FVarId of mutually recursive functions being defined to "closure" expression. -/ +/-- Mapping from FVarId of mutually recursive functions being defined to "closure" expression. -/ abbrev Replacement := FVarIdMap Expr def insertReplacementForMainFns (r : Replacement) (sectionVars : Array Expr) (mainHeaders : Array DefViewElabHeader) (mainFVars : Array Expr) : Replacement := @@ -610,7 +610,7 @@ def getModifiersForLetRecs (mainHeaders : Array DefViewElabHeader) : Modifiers : isUnsafe := mainHeaders.any fun h => h.modifiers.isUnsafe } -/- +/-- - `sectionVars`: The section variables used in the `mutual` block. - `mainHeaders`: The elaborated header of the top-level definitions being defined by the mutual block. - `mainFVars`: The auxiliary variables used to represent the top-level definitions being defined by the mutual block. @@ -777,9 +777,14 @@ where withFunLocalDecls headers fun funFVars => do for view in views, funFVar in funFVars do addLocalVarInfo view.declId funFVar - let values ← elabFunValues headers - Term.synthesizeSyntheticMVarsNoPostponing - let values ← values.mapM (instantiateMVars ·) + let values ← + try + let values ← elabFunValues headers + Term.synthesizeSyntheticMVarsNoPostponing + values.mapM (instantiateMVars ·) + catch ex => + logException ex + headers.mapM fun header => mkSorry header.type (synthetic := true) let headers ← headers.mapM instantiateMVarsAtHeader let letRecsToLift ← getLetRecsToLift let letRecsToLift ← letRecsToLift.mapM instantiateMVarsAtLetRecToLift diff --git a/src/Lean/Elab/Notation.lean b/src/Lean/Elab/Notation.lean index 68f9f03281a0..be2205c7c2fd 100644 --- a/src/Lean/Elab/Notation.lean +++ b/src/Lean/Elab/Notation.lean @@ -12,7 +12,7 @@ open Lean.Syntax open Lean.Parser.Term hiding macroArg open Lean.Parser.Command -/- Wrap all occurrences of the given `ident` nodes in antiquotations -/ +/-- Wrap all occurrences of the given `ident` nodes in antiquotations -/ private partial def antiquote (vars : Array Syntax) : Syntax → Syntax | stx => match stx with | `($id:ident) => @@ -24,13 +24,13 @@ private partial def antiquote (vars : Array Syntax) : Syntax → Syntax | Syntax.node i k args => Syntax.node i k (args.map (antiquote vars)) | stx => stx -/- Convert `notation` command lhs item into a `syntax` command item -/ +/-- Convert `notation` command lhs item into a `syntax` command item -/ def expandNotationItemIntoSyntaxItem : TSyntax ``notationItem → MacroM (TSyntax `stx) | `(notationItem| $_:ident$[:$prec?]?) => `(stx| term $[:$prec?]?) | `(notationItem| $s:str) => `(stx| $s:str) | _ => Macro.throwUnsupported -/- Convert `notation` command lhs item into a pattern element -/ +/-- Convert `notation` command lhs item into a pattern element -/ def expandNotationItemIntoPattern (stx : Syntax) : MacroM Syntax := let k := stx.getKind if k == `Lean.Parser.Command.identPrec then diff --git a/src/Lean/Elab/PatternVar.lean b/src/Lean/Elab/PatternVar.lean index 78807b63a707..db85be576016 100644 --- a/src/Lean/Elab/PatternVar.lean +++ b/src/Lean/Elab/PatternVar.lean @@ -13,7 +13,7 @@ open Meta abbrev PatternVar := Syntax -- TODO: should be `Ident` -/- +/-! Patterns define new local variables. This module collect them and preprocess `_` occurring in patterns. Recall that an `_` may represent anonymous variables or inaccessible terms @@ -49,7 +49,7 @@ private def throwCtorExpected {α} : M α := private def throwInvalidPattern {α} : M α := throwError "invalid pattern" -/- +/-! An application in a pattern can be 1- A constructor application @@ -231,7 +231,7 @@ where processCtor (stx : Syntax) : M Syntax := do processCtorAppCore stx #[] #[] false - /- Check whether `stx` is a pattern variable or constructor-like (i.e., constructor or constant tagged with `[matchPattern]` attribute) -/ + /-- Check whether `stx` is a pattern variable or constructor-like (i.e., constructor or constant tagged with `[matchPattern]` attribute) -/ processId (stx : Syntax) : M Syntax := do match (← resolveId? stx "pattern") with | none => processVar stx @@ -324,7 +324,7 @@ def collectPatternVars (alt : MatchAltView) : TermElabM (Array PatternVar × Mat let (alt, s) ← (CollectPatternVars.main alt).run {} return (s.vars, alt) -/- Return the pattern variables in the given pattern. +/-- Return the pattern variables in the given pattern. Remark: this method is not used by the main `match` elaborator, but in the precheck hook and other macros (e.g., at `Do.lean`). -/ def getPatternVars (patternStx : Syntax) : TermElabM (Array PatternVar) := do let patternStx ← liftMacroM <| expandMacros patternStx diff --git a/src/Lean/Elab/PreDefinition/Basic.lean b/src/Lean/Elab/PreDefinition/Basic.lean index cdc955f3a3f3..bc75208e54ba 100644 --- a/src/Lean/Elab/PreDefinition/Basic.lean +++ b/src/Lean/Elab/PreDefinition/Basic.lean @@ -74,7 +74,7 @@ def abstractNestedProofs (preDef : PreDefinition) : MetaM PreDefinition := let value ← Meta.abstractNestedProofs preDef.declName preDef.value pure { preDef with value := value } -/- Auxiliary method for (temporarily) adding pre definition as an axiom -/ +/-- Auxiliary method for (temporarily) adding pre definition as an axiom -/ def addAsAxiom (preDef : PreDefinition) : MetaM Unit := do withRef preDef.ref do addDecl <| Declaration.axiomDecl { name := preDef.declName, levelParams := preDef.levelParams, type := preDef.type, isUnsafe := preDef.modifiers.isUnsafe } diff --git a/src/Lean/Elab/PreDefinition/MkInhabitant.lean b/src/Lean/Elab/PreDefinition/MkInhabitant.lean index 5050baa096cd..1ed531927f18 100644 --- a/src/Lean/Elab/PreDefinition/MkInhabitant.lean +++ b/src/Lean/Elab/PreDefinition/MkInhabitant.lean @@ -31,7 +31,6 @@ private def mkFnInhabitant? (xs : Array Expr) (type : Expr) (useOfNonempty : Boo loop xs.size type /- TODO: add a global IO.Ref to let users customize/extend this procedure -/ - def mkInhabitantFor (declName : Name) (xs : Array Expr) (type : Expr) : MetaM Expr := do let go? (useOfNonempty : Bool) : MetaM (Option Expr) := do match (← mkInhabitant? type useOfNonempty) with diff --git a/src/Lean/Elab/PreDefinition/Structural/BRecOn.lean b/src/Lean/Elab/PreDefinition/Structural/BRecOn.lean index 92659fa21457..2fc755fd4f42 100644 --- a/src/Lean/Elab/PreDefinition/Structural/BRecOn.lean +++ b/src/Lean/Elab/PreDefinition/Structural/BRecOn.lean @@ -16,7 +16,7 @@ open Meta private def throwToBelowFailed : MetaM α := throwError "toBelow failed" -/- See toBelow -/ +/-- See `toBelow` -/ private partial def toBelowAux (C : Expr) (belowDict : Expr) (arg : Expr) (F : Expr) : MetaM Expr := do let belowDict ← whnf belowDict trace[Elab.definition.structural] "belowDict: {belowDict}, arg: {arg}" @@ -43,7 +43,7 @@ private partial def toBelowAux (C : Expr) (belowDict : Expr) (arg : Expr) (F : E pure (mkAppN F argTailArgs) | _ => throwToBelowFailed -/- See toBelow -/ +/-- See `toBelow` -/ private def withBelowDict (below : Expr) (numIndParams : Nat) (k : Expr → Expr → MetaM α) : MetaM α := do let belowType ← inferType below trace[Elab.definition.structural] "belowType: {belowType}" @@ -59,7 +59,7 @@ private def withBelowDict (below : Expr) (numIndParams : Nat) (k : Expr → Expr let belowDict := mkAppN belowDict (args.extract (numIndParams + 1) args.size) k C belowDict -/- +/-- `below` is a free variable with type of the form `I.below indParams motive indices major`, where `I` is the name of an inductive datatype. @@ -148,7 +148,7 @@ private partial def replaceRecApps (recFnName : Name) (recArgInfo : RecArgInfo) if !recArgHasLooseBVarsAt recFnName recArgInfo.recArgPos e then processApp e else - /- Here is an example we currently not handle + /- Here is an example we currently do not handle ``` def g (xs : List Nat) : Nat := match xs with diff --git a/src/Lean/Elab/PreDefinition/Structural/Basic.lean b/src/Lean/Elab/PreDefinition/Structural/Basic.lean index ff7f265b0efc..c3f392129ecb 100644 --- a/src/Lean/Elab/PreDefinition/Structural/Basic.lean +++ b/src/Lean/Elab/PreDefinition/Structural/Basic.lean @@ -9,23 +9,32 @@ import Lean.Meta.ForEachExpr namespace Lean.Elab.Structural structure RecArgInfo where - /- `fixedParams ++ ys` are the arguments of the function we are trying to justify termination using structural recursion. -/ + /-- `fixedParams ++ ys` are the arguments of the function we are trying to justify termination using structural recursion. -/ fixedParams : Array Expr - ys : Array Expr -- recursion arguments - pos : Nat -- position in `ys` of the argument we are recursing on - indicesPos : Array Nat -- position in `ys` of the inductive datatype indices we are recursing on - indName : Name -- inductive datatype name of the argument we are recursing on - indLevels : List Level -- inductice datatype universe levels of the argument we are recursing on - indParams : Array Expr -- inductive datatype parameters of the argument we are recursing on - indIndices : Array Expr -- inductive datatype indices of the argument we are recursing on, it is equal to `indicesPos.map fun i => ys.get! i` - reflexive : Bool -- true if we are recursing over a reflexive inductive datatype - indPred : Bool -- true if the type is an inductive predicate + /-- recursion arguments -/ + ys : Array Expr + /-- position in `ys` of the argument we are recursing on -/ + pos : Nat + /-- position in `ys` of the inductive datatype indices we are recursing on -/ + indicesPos : Array Nat + /-- inductive datatype name of the argument we are recursing on -/ + indName : Name + /-- inductive datatype universe levels of the argument we are recursing on -/ + indLevels : List Level + /-- inductive datatype parameters of the argument we are recursing on -/ + indParams : Array Expr + /-- inductive datatype indices of the argument we are recursing on, it is equal to `indicesPos.map fun i => ys.get! i` -/ + indIndices : Array Expr + /-- true if we are recursing over a reflexive inductive datatype -/ + reflexive : Bool + /-- true if the type is an inductive predicate -/ + indPred : Bool def RecArgInfo.recArgPos (info : RecArgInfo) : Nat := info.fixedParams.size + info.pos structure State where - /- As part of the inductive predicates case, we keep adding more and more discriminants from the + /-- As part of the inductive predicates case, we keep adding more and more discriminants from the local context and build up a bigger matcher application until we reach a fixed point. As a side-effect, this creates matchers. Here we capture all these side-effects, because the construction rolls back any changes done to the environment and the side-effects diff --git a/src/Lean/Elab/PreDefinition/WF/TerminationHint.lean b/src/Lean/Elab/PreDefinition/WF/TerminationHint.lean index 9b17b636e6c2..ec13ac67c506 100644 --- a/src/Lean/Elab/PreDefinition/WF/TerminationHint.lean +++ b/src/Lean/Elab/PreDefinition/WF/TerminationHint.lean @@ -7,7 +7,7 @@ import Lean.Parser.Command namespace Lean.Elab.WF -/- Support for `decreasing_by` and `termination_by'` notations -/ +/-! # Support for `decreasing_by` and `termination_by'` notations -/ structure TerminationHintValue where ref : Syntax @@ -73,7 +73,7 @@ def TerminationHint.ensureAllUsed (t : TerminationHint) : MacroM Unit := do | TerminationHint.many m => m.forM fun _ v => Macro.throwErrorAt v.ref "unused termination hint element" | _ => pure () -/- Support for `termination_by` notation -/ +/-! # Support for `termination_by` notation -/ structure TerminationByElement where ref : Syntax diff --git a/src/Lean/Elab/Quotation.lean b/src/Lean/Elab/Quotation.lean index 971555aa0a44..0cf443a916d9 100644 --- a/src/Lean/Elab/Quotation.lean +++ b/src/Lean/Elab/Quotation.lean @@ -234,9 +234,9 @@ elab_stx_quot Parser.Term.doElem.quot elab_stx_quot Parser.Term.dynamicQuot elab_stx_quot Parser.Command.quot -/- match -/ +/-! # match -/ --- an "alternative" of patterns plus right-hand side +/-- an "alternative" of patterns plus right-hand side -/ private abbrev Alt := List Term × Term /-- @@ -244,45 +244,45 @@ private abbrev Alt := List Term × Term alternative. This datatype describes what kind of check this involves, which helps other patterns decide if they are covered by the same check and don't have to be checked again (see also `MatchResult`). -/ inductive HeadCheck where - -- match step that always succeeds: _, x, `($x), ... - | unconditional - -- match step based on kind and, optionally, arity of discriminant - -- If `arity` is given, that number of new discriminants is introduced. `covered` patterns should then introduce the - -- same number of new patterns. - -- We actually check the arity at run time only in the case of `null` nodes since it should otherwise by implied by - -- the node kind. - -- without arity: `($x:k) - -- with arity: any quotation without an antiquotation head pattern - | shape (k : List SyntaxNodeKind) (arity : Option Nat) - -- Match step that succeeds on `null` nodes of arity at least `numPrefix + numSuffix`, introducing discriminants - -- for the first `numPrefix` children, one `null` node for those in between, and for the `numSuffix` last children. - -- example: `([$x, $xs,*, $y]) is `slice 2 2` - | slice (numPrefix numSuffix : Nat) - -- other, complicated match step that will probably only cover identical patterns - -- example: antiquotation splices `($[...]*) - | other (pat : Syntax) + | /-- match step that always succeeds: _, x, `($x), ... -/ + unconditional + | /-- match step based on kind and, optionally, arity of discriminant + If `arity` is given, that number of new discriminants is introduced. `covered` patterns should then introduce the + same number of new patterns. + We actually check the arity at run time only in the case of `null` nodes since it should otherwise by implied by + the node kind. + without arity: `($x:k) + with arity: any quotation without an antiquotation head pattern -/ + shape (k : List SyntaxNodeKind) (arity : Option Nat) + | /-- Match step that succeeds on `null` nodes of arity at least `numPrefix + numSuffix`, introducing discriminants + for the first `numPrefix` children, one `null` node for those in between, and for the `numSuffix` last children. + example: `([$x, $xs,*, $y]) is `slice 2 2` -/ + slice (numPrefix numSuffix : Nat) + | /-- other, complicated match step that will probably only cover identical patterns + example: antiquotation splices `($[...]*) -/ + other (pat : Syntax) open HeadCheck /-- Describe whether a pattern is covered by a head check (induced by the pattern itself or a different pattern). -/ inductive MatchResult where - -- Pattern agrees with head check, remove and transform remaining alternative. - -- If `exhaustive` is `false`, *also* include unchanged alternative in the "no" branch. - | covered (f : Alt → TermElabM Alt) (exhaustive : Bool) - -- Pattern disagrees with head check, include in "no" branch only - | uncovered - -- Pattern is not quite sure yet; include unchanged in both branches - | undecided + | /-- Pattern agrees with head check, remove and transform remaining alternative. + If `exhaustive` is `false`, *also* include unchanged alternative in the "no" branch. -/ + covered (f : Alt → TermElabM Alt) (exhaustive : Bool) + | /-- Pattern disagrees with head check, include in "no" branch only -/ + uncovered + | /-- Pattern is not quite sure yet; include unchanged in both branches -/ + undecided open MatchResult /-- All necessary information on a pattern head. -/ structure HeadInfo where - -- check induced by the pattern + /-- check induced by the pattern -/ check : HeadCheck - -- compute compatibility of pattern with given head check + /-- compute compatibility of pattern with given head check -/ onMatch (taken : HeadCheck) : MatchResult - -- actually run the specified head check, with the discriminant bound to `discr` + /-- actually run the specified head check, with the discriminant bound to `discr` -/ doMatch (yes : (newDiscrs : List Term) → TermElabM Term) (no : TermElabM Term) : TermElabM Term /-- Adapt alternatives that do not introduce new discriminants in `doMatch`, but are covered by those that do so. -/ @@ -475,7 +475,7 @@ private partial def getHeadInfo (alt : Alt) : TermElabM HeadInfo := | r => r } | _ => throwErrorAt pat "match (syntax) : unexpected pattern kind {pat}" --- Bind right-hand side to new `let_delayed` decl in order to prevent code duplication +/-- Bind right-hand side to new `let_delayed` decl in order to prevent code duplication -/ private def deduplicate (floatedLetDecls : Array Syntax) : Alt → TermElabM (Array Syntax × Alt) -- NOTE: new macro scope so that introduced bindings do not collide | (pats, rhs) => do diff --git a/src/Lean/Elab/StructInst.lean b/src/Lean/Elab/StructInst.lean index 1e3dabb88fe9..7747b9498f3f 100644 --- a/src/Lean/Elab/StructInst.lean +++ b/src/Lean/Elab/StructInst.lean @@ -254,8 +254,8 @@ def Field.isSimple {σ} : Field σ → Bool | _ => false inductive Struct where - /- Remark: the field `params` is use for default value propagation. It is initially empty, and then set at `elabStruct`. -/ - | mk (ref : Syntax) (structName : Name) (params : Array (Name × Expr)) (fields : List (Field Struct)) (source : Source) + | /-- Remark: the field `params` is use for default value propagation. It is initially empty, and then set at `elabStruct`. -/ + mk (ref : Syntax) (structName : Name) (params : Array (Name × Expr)) (fields : List (Field Struct)) (source : Source) deriving Inhabited abbrev Fields := List (Field Struct) @@ -393,7 +393,7 @@ private def expandNumLitFields (s : Struct) : TermElabM Struct := else return { field with lhs := .fieldName ref fieldNames[idx - 1]! :: rest } | _ => return field -/- For example, consider the following structures: +/-- For example, consider the following structures: ``` structure A where x : Nat diff --git a/src/Lean/Elab/Structure.lean b/src/Lean/Elab/Structure.lean index 9a1976b96042..e2750400c112 100644 --- a/src/Lean/Elab/Structure.lean +++ b/src/Lean/Elab/Structure.lean @@ -21,7 +21,7 @@ namespace Lean.Elab.Command open Meta open TSyntax.Compat -/- Recall that the `structure command syntax is +/-! Recall that the `structure command syntax is ``` leading_parser (structureTk <|> classTk) >> declId >> many Term.bracketedBinder >> optional «extends» >> Term.optType >> optional (" := " >> optional structCtor >> structFields) ``` @@ -500,7 +500,7 @@ private def elabFieldTypeValue (view : StructFieldView) : TermElabM (Option Expr Term.synthesizeSyntheticMVarsNoPostponing -- TODO: add forbidden predicate using `shortDeclName` from `view` let params ← Term.addAutoBoundImplicits params - let value ← Term.elabTerm valStx none + let value ← Term.withoutAutoBoundImplicit <| Term.elabTerm valStx none let value ← mkLambdaFVars params value return (none, value) | some typeStx => @@ -512,7 +512,7 @@ private def elabFieldTypeValue (view : StructFieldView) : TermElabM (Option Expr let type ← mkForallFVars params type return (type, none) | some valStx => - let value ← Term.elabTermEnsuringType valStx type + let value ← Term.withoutAutoBoundImplicit <| Term.elabTermEnsuringType valStx type Term.synthesizeSyntheticMVarsNoPostponing let type ← mkForallFVars params type let value ← mkLambdaFVars params value diff --git a/src/Lean/Elab/Syntax.lean b/src/Lean/Elab/Syntax.lean index 65eaaaa4f5f1..b2d4349b2762 100644 --- a/src/Lean/Elab/Syntax.lean +++ b/src/Lean/Elab/Syntax.lean @@ -8,7 +8,7 @@ import Lean.Parser.Syntax import Lean.Elab.Util namespace Lean.Elab.Term -/- +/-- Expand `optional «precedence»` where «precedence» := leading_parser " : " >> precedenceParser -/ def expandOptPrecedence (stx : Syntax) : MacroM (Option Nat) := @@ -33,7 +33,7 @@ structure ToParserDescrContext where catName : Name first : Bool leftRec : Bool -- true iff left recursion is allowed - /- See comment at `Parser.ParserCategory`. -/ + /-- See comment at `Parser.ParserCategory`. -/ behavior : Parser.LeadingIdentBehavior abbrev ToParserDescrM := ReaderT ToParserDescrContext (StateRefT (Option Nat) TermElabM) @@ -126,7 +126,7 @@ where | some stxNew => process stxNew | none => throwErrorAt stx "unexpected syntax kind of category `syntax`: {kind}" - /- Sequence (aka NullNode) -/ + /-- Sequence (aka NullNode) -/ processSeq (stx : Syntax) := do let args := stx.getArgs if (← checkLeftRec stx[0]) then @@ -300,7 +300,7 @@ where | .str _ s => s ++ str | _ => str -/- We assume a new syntax can be treated as an atom when it starts and ends with a token. +/-- We assume a new syntax can be treated as an atom when it starts and ends with a token. Here are examples of atom-like syntax. ``` syntax "(" term ")" : term @@ -325,7 +325,7 @@ def resolveSyntaxKind (k : Name) : CommandElabM Name := do throwError "invalid syntax node kind '{k}'" @[builtinCommandElab «syntax»] def elabSyntax : CommandElab := fun stx => do - let `($[$doc?:docComment]? $attrKind:attrKind syntax $[: $prec? ]? $[(name := $name?)]? $[(priority := $prio?)]? $[$ps:stx]* : $catStx) ← pure stx + let `($[$doc?:docComment]? $[ @[ $attrInstances:attrInstance,* ] ]? $attrKind:attrKind syntax $[: $prec? ]? $[(name := $name?)]? $[(priority := $prio?)]? $[$ps:stx]* : $catStx) ← pure stx | throwUnsupportedSyntax let cat := catStx.getId.eraseMacroScopes unless (Parser.isParserCategory (← getEnv) cat) do @@ -344,11 +344,14 @@ def resolveSyntaxKind (k : Name) : CommandElabM Name := do let catParserId := mkIdentFrom stx (cat.appendAfter "Parser") let (val, lhsPrec?) ← runTermElabM none fun _ => Term.toParserDescr syntaxParser cat let declName := mkIdentFrom stx name + let attrInstance ← `(attrInstance| $attrKind:attrKind $catParserId:ident $(quote prio):num) + let attrInstances := attrInstances.getD { elemsAndSeps := #[] } + let attrInstances := attrInstances.push attrInstance let d ← if let some lhsPrec := lhsPrec? then - `($[$doc?:docComment]? @[$attrKind:attrKind $catParserId:ident $(quote prio):num] def $declName:ident : Lean.TrailingParserDescr := + `($[$doc?:docComment]? @[$attrInstances,*] def $declName:ident : Lean.TrailingParserDescr := ParserDescr.trailingNode $(quote stxNodeKind) $(quote prec) $(quote lhsPrec) $val) else - `($[$doc?:docComment]? @[$attrKind:attrKind $catParserId:ident $(quote prio):num] def $declName:ident : Lean.ParserDescr := + `($[$doc?:docComment]? @[$attrInstances,*] def $declName:ident : Lean.ParserDescr := ParserDescr.node $(quote stxNodeKind) $(quote prec) $val) trace `Elab fun _ => d withMacroExpansion stx d <| elabCommand d diff --git a/src/Lean/Elab/SyntheticMVars.lean b/src/Lean/Elab/SyntheticMVars.lean index 7d34da61635b..bd8adccaa351 100644 --- a/src/Lean/Elab/SyntheticMVars.lean +++ b/src/Lean/Elab/SyntheticMVars.lean @@ -23,7 +23,7 @@ private def resumeElabTerm (stx : Syntax) (expectedType? : Option Expr) (errToSo It is used to implement `synthesizeSyntheticMVars`. -/ private def resumePostponed (savedContext : SavedContext) (stx : Syntax) (mvarId : MVarId) (postponeOnError : Bool) : TermElabM Bool := withRef stx <| withMVarContext mvarId do - let s ← get + let s ← saveState try withSavedContext savedContext do let mvarDecl ← getMVarDecl mvarId @@ -40,15 +40,15 @@ private def resumePostponed (savedContext : SavedContext) (stx : Syntax) (mvarId else return false catch - | ex@(Exception.internal id _) => + | ex@(.internal id _) => if id == postponeExceptionId then - set s + s.restore (restoreInfo := true) return false else throw ex - | ex@(Exception.error _ _) => + | ex@(.error ..) => if postponeOnError then - set s + s.restore (restoreInfo := true) return false else logException ex @@ -62,8 +62,8 @@ private def synthesizePendingInstMVar (instMVar : MVarId) : TermElabM Bool := try synthesizeInstMVarCore instMVar catch - | ex@(Exception.error _ _) => logException ex; return true - | _ => unreachable! + | ex@(.error ..) => logException ex; return true + | _ => unreachable! /-- Similar to `synthesizePendingInstMVar`, but generates type mismatch error message. @@ -95,8 +95,8 @@ private def synthesizePendingCoeInstMVar return true return false catch - | Exception.error _ msg => throwTypeMismatchError errorMsgHeader? expectedType eType e f? msg - | _ => unreachable! + | .error _ msg => throwTypeMismatchError errorMsgHeader? expectedType eType e f? msg + | _ => unreachable! /-- Try to synthesize `mvarId` by starting using a default instance with the give privority. @@ -203,25 +203,25 @@ where let some mvarIds ← synthesizeSomeUsingDefault? mvarIds | return false synthesizePending mvarIds -/- Used to implement `synthesizeUsingDefault`. This method only consider default instances with the given priority. -/ +/-- Used to implement `synthesizeUsingDefault`. This method only consider default instances with the given priority. -/ private def synthesizeSomeUsingDefaultPrio (prio : Nat) : TermElabM Bool := do - let rec visit (syntheticMVars : List SyntheticMVarDecl) (syntheticMVarsNew : List SyntheticMVarDecl) : TermElabM Bool := do - match syntheticMVars with + let rec visit (pendingMVars : List MVarId) (pendingMVarsNew : List MVarId) : TermElabM Bool := do + match pendingMVars with | [] => return false - | mvarDecl :: mvarDecls => + | mvarId :: pendingMVars => + let some mvarDecl ← getSyntheticMVarDecl? mvarId | visit pendingMVars (mvarId :: pendingMVarsNew) match mvarDecl.kind with - | SyntheticMVarKind.typeClass => - if (← withRef mvarDecl.stx <| synthesizeUsingDefaultPrio mvarDecl.mvarId prio) then - let syntheticMVarsNew := mvarDecls.reverse ++ syntheticMVarsNew - modify fun s => { s with syntheticMVars := syntheticMVarsNew } + | .typeClass => + if (← withRef mvarDecl.stx <| synthesizeUsingDefaultPrio mvarId prio) then + modify fun s => { s with pendingMVars := pendingMVars.reverse ++ pendingMVarsNew } return true else - visit mvarDecls (mvarDecl :: syntheticMVarsNew) - | _ => visit mvarDecls (mvarDecl :: syntheticMVarsNew) - /- Recall that s.syntheticMVars is essentially a stack. The first metavariable was the last one created. + visit pendingMVars (mvarId :: pendingMVarsNew) + | _ => visit pendingMVars (mvarId :: pendingMVarsNew) + /- Recall that s.pendingMVars is essentially a stack. The first metavariable was the last one created. We want to apply the default instance in reverse creation order. Otherwise, `toString 0` will produce a `OfNat String _` cannot be synthesized error. -/ - visit (← get).syntheticMVars.reverse [] + visit (← get).pendingMVars.reverse [] /-- Apply default value to any pending synthetic metavariable of kind `SyntheticMVarKind.withDefault` @@ -234,16 +234,17 @@ private def synthesizeUsingDefault : TermElabM Bool := do return true return false -def reportStuckSyntheticMVar (mvarSyntheticDecl : SyntheticMVarDecl) (ignoreStuckTC := false) : TermElabM Unit := +def reportStuckSyntheticMVar (mvarId : MVarId) (ignoreStuckTC := false) : TermElabM Unit := do + let some mvarSyntheticDecl ← getSyntheticMVarDecl? mvarId | return () withRef mvarSyntheticDecl.stx do match mvarSyntheticDecl.kind with - | SyntheticMVarKind.typeClass => + | .typeClass => unless ignoreStuckTC do - withMVarContext mvarSyntheticDecl.mvarId do - let mvarDecl ← getMVarDecl mvarSyntheticDecl.mvarId + withMVarContext mvarId do + let mvarDecl ← getMVarDecl mvarId unless (← MonadLog.hasErrors) do throwError "typeclass instance problem is stuck, it is often due to metavariables{indentExpr mvarDecl.type}" - | SyntheticMVarKind.coe header eNew expectedType eType e f? => + | .coe header eNew expectedType eType e f? => let mvarId := eNew.appArg!.mvarId! withMVarContext mvarId do let mvarDecl ← getMVarDecl mvarId @@ -255,15 +256,16 @@ def reportStuckSyntheticMVar (mvarSyntheticDecl : SyntheticMVarDecl) (ignoreStuc Remark: we set `ignoreStuckTC := true` when elaborating `simp` arguments. -/ private def reportStuckSyntheticMVars (ignoreStuckTC := false) : TermElabM Unit := do - let syntheticMVars ← modifyGet fun s => (s.syntheticMVars, { s with syntheticMVars := [] }) - for mvarSyntheticDecl in syntheticMVars do - reportStuckSyntheticMVar mvarSyntheticDecl ignoreStuckTC + let pendingMVars ← modifyGet fun s => (s.pendingMVars, { s with pendingMVars := [] }) + for mvarId in pendingMVars do + reportStuckSyntheticMVar mvarId ignoreStuckTC private def getSomeSynthethicMVarsRef : TermElabM Syntax := do - let s ← get - match s.syntheticMVars.find? fun (mvarDecl : SyntheticMVarDecl) => !mvarDecl.stx.getPos?.isNone with - | some mvarDecl => return mvarDecl.stx - | none => return Syntax.missing + for mvarId in (← get).pendingMVars do + if let some decl ← getSyntheticMVarDecl? mvarId then + if decl.stx.getPos?.isSome then + return decl.stx + return .missing /-- Generate an nicer error message for stuck universe constraints. @@ -307,6 +309,13 @@ private def processPostponedUniverseContraints : TermElabM Unit := do unless (← processPostponed (mayPostpone := false) (exceptionOnFailure := true)) do throwStuckAtUniverseCnstr +/-- + Remove `mvarId` from the `syntheticMVars` table. We use this method after + the metavariable has been synthesized. +-/ +private def markAsResolved (mvarId : MVarId) : TermElabM Unit := + modify fun s => { s with syntheticMVars := s.syntheticMVars.erase mvarId } + mutual partial def runTactic (mvarId : MVarId) (tacticCode : Syntax) : TermElabM Unit := do @@ -320,17 +329,18 @@ mutual reportUnsolvedGoals remainingGoals /-- Try to synthesize the given pending synthetic metavariable. -/ - private partial def synthesizeSyntheticMVar (mvarSyntheticDecl : SyntheticMVarDecl) (postponeOnError : Bool) (runTactics : Bool) : TermElabM Bool := + private partial def synthesizeSyntheticMVar (mvarId : MVarId) (postponeOnError : Bool) (runTactics : Bool) : TermElabM Bool := do + let some mvarSyntheticDecl ← getSyntheticMVarDecl? mvarId | return true -- The metavariable has already been synthesized withRef mvarSyntheticDecl.stx do match mvarSyntheticDecl.kind with - | SyntheticMVarKind.typeClass => synthesizePendingInstMVar mvarSyntheticDecl.mvarId - | SyntheticMVarKind.coe header? eNew expectedType eType e f? => synthesizePendingCoeInstMVar mvarSyntheticDecl.mvarId header? eNew expectedType eType e f? + | .typeClass => synthesizePendingInstMVar mvarId + | .coe header? eNew expectedType eType e f? => synthesizePendingCoeInstMVar mvarId header? eNew expectedType eType e f? -- NOTE: actual processing at `synthesizeSyntheticMVarsAux` - | SyntheticMVarKind.postponed savedContext => resumePostponed savedContext mvarSyntheticDecl.stx mvarSyntheticDecl.mvarId postponeOnError - | SyntheticMVarKind.tactic tacticCode savedContext => + | .postponed savedContext => resumePostponed savedContext mvarSyntheticDecl.stx mvarId postponeOnError + | .tactic tacticCode savedContext => withSavedContext savedContext do if runTactics then - runTactic mvarSyntheticDecl.mvarId tacticCode + runTactic mvarId tacticCode return true else return false @@ -341,26 +351,27 @@ mutual let ctx ← read traceAtCmdPos `Elab.resuming fun _ => m!"resuming synthetic metavariables, mayPostpone: {ctx.mayPostpone}, postponeOnError: {postponeOnError}" - let syntheticMVars := (← get).syntheticMVars - let numSyntheticMVars := syntheticMVars.length - -- We reset `syntheticMVars` because new synthetic metavariables may be created by `synthesizeSyntheticMVar`. - modify fun s => { s with syntheticMVars := [] } - -- Recall that `syntheticMVars` is a list where head is the most recent pending synthetic metavariable. + let pendingMVars := (← get).pendingMVars + let numSyntheticMVars := pendingMVars.length + -- We reset `pendingMVars` because new synthetic metavariables may be created by `synthesizeSyntheticMVar`. + modify fun s => { s with pendingMVars := [] } + -- Recall that `pendingMVars` is a list where head is the most recent pending synthetic metavariable. -- We use `filterRevM` instead of `filterM` to make sure we process the synthetic metavariables using the order they were created. -- It would not be incorrect to use `filterM`. - let remainingSyntheticMVars ← syntheticMVars.filterRevM fun mvarDecl => do + let remainingPendingMVars ← pendingMVars.filterRevM fun mvarId => do -- We use `traceM` because we want to make sure the metavar local context is used to trace the message - traceM `Elab.postpone (withMVarContext mvarDecl.mvarId do addMessageContext m!"resuming {mkMVar mvarDecl.mvarId}") - let succeeded ← synthesizeSyntheticMVar mvarDecl postponeOnError runTactics + traceM `Elab.postpone (withMVarContext mvarId do addMessageContext m!"resuming {mkMVar mvarId}") + let succeeded ← synthesizeSyntheticMVar mvarId postponeOnError runTactics + if succeeded then markAsResolved mvarId trace[Elab.postpone] if succeeded then format "succeeded" else format "not ready yet" pure !succeeded - -- Merge new synthetic metavariables with `remainingSyntheticMVars`, i.e., metavariables that still couldn't be synthesized - modify fun s => { s with syntheticMVars := s.syntheticMVars ++ remainingSyntheticMVars } - return numSyntheticMVars != remainingSyntheticMVars.length + -- Merge new synthetic metavariables with `remainingPendingMVars`, i.e., metavariables that still couldn't be synthesized + modify fun s => { s with pendingMVars := s.pendingMVars ++ remainingPendingMVars } + return numSyntheticMVars != remainingPendingMVars.length /-- Try to process pending synthetic metavariables. If `mayPostpone == false`, - then `syntheticMVars` is `[]` after executing this method. + then `pendingMVars` is `[]` after executing this method. It keeps executing `synthesizeSyntheticMVarsStep` while progress is being made. If `mayPostpone == false`, then it applies default instances to `SyntheticMVarKind.typeClass` (if available) @@ -374,7 +385,7 @@ mutual partial def synthesizeSyntheticMVars (mayPostpone := true) (ignoreStuckTC := false) : TermElabM Unit := do let rec loop (_ : Unit) : TermElabM Unit := do withRef (← getSomeSynthethicMVarsRef) <| withIncRecDepth do - unless (← get).syntheticMVars.isEmpty do + unless (← get).pendingMVars.isEmpty do if ← synthesizeSyntheticMVarsStep (postponeOnError := false) (runTactics := false) then loop () else if !mayPostpone then @@ -412,7 +423,7 @@ end def synthesizeSyntheticMVarsNoPostponing (ignoreStuckTC := false) : TermElabM Unit := synthesizeSyntheticMVars (mayPostpone := false) (ignoreStuckTC := ignoreStuckTC) -/- Keep invoking `synthesizeUsingDefault` until it returns false. -/ +/-- Keep invoking `synthesizeUsingDefault` until it returns false. -/ private partial def synthesizeUsingDefaultLoop : TermElabM Unit := do if (← synthesizeUsingDefault) then synthesizeSyntheticMVars (mayPostpone := true) @@ -423,8 +434,8 @@ def synthesizeSyntheticMVarsUsingDefault : TermElabM Unit := do synthesizeUsingDefaultLoop private partial def withSynthesizeImp {α} (k : TermElabM α) (mayPostpone : Bool) (synthesizeDefault : Bool) : TermElabM α := do - let syntheticMVarsSaved := (← get).syntheticMVars - modify fun s => { s with syntheticMVars := [] } + let pendingMVarsSaved := (← get).pendingMVars + modify fun s => { s with pendingMVars := [] } try let a ← k synthesizeSyntheticMVars mayPostpone @@ -432,7 +443,7 @@ private partial def withSynthesizeImp {α} (k : TermElabM α) (mayPostpone : Boo synthesizeUsingDefaultLoop return a finally - modify fun s => { s with syntheticMVars := s.syntheticMVars ++ syntheticMVarsSaved } + modify fun s => { s with pendingMVars := s.pendingMVars ++ pendingMVarsSaved } /-- Execute `k`, and synthesize pending synthetic metavariables created while executing `k` are solved. @@ -450,6 +461,14 @@ def elabTermAndSynthesize (stx : Syntax) (expectedType? : Option Expr) : TermEla withRef stx do instantiateMVars (← withSynthesize <| elabTerm stx expectedType?) +def runPendingTacticsAt (e : Expr) : TermElabM Unit := do + for mvarId in (← getMVars e) do + let mvarId ← getDelayedMVarRoot mvarId + if let some { kind := .tactic tacticCode savedContext, .. } ← getSyntheticMVarDecl? mvarId then + withSavedContext savedContext do + runTactic mvarId tacticCode + markAsResolved mvarId + builtin_initialize registerTraceClass `Elab.resume diff --git a/src/Lean/Elab/Tactic/Basic.lean b/src/Lean/Elab/Tactic/Basic.lean index 8a53d25144a4..6415fdb772c8 100644 --- a/src/Lean/Elab/Tactic/Basic.lean +++ b/src/Lean/Elab/Tactic/Basic.lean @@ -19,7 +19,7 @@ import Lean.Elab.Binders namespace Lean.Elab open Meta -/- Assign `mvarId := sorry` -/ +/-- Assign `mvarId := sorry` -/ def admitGoal (mvarId : MVarId) : MetaM Unit := withMVarContext mvarId do let mvarType ← inferType (mkMVar mvarId) @@ -48,7 +48,7 @@ structure Context where structure SavedState where term : Term.SavedState tactic : State - + abbrev TacticM := ReaderT Context $ StateRefT State TermElabM abbrev Tactic := Syntax → TacticM Unit @@ -79,8 +79,8 @@ def getUnsolvedGoals : TacticM (List MVarId) := do def run (mvarId : MVarId) (x : TacticM Unit) : TermElabM (List MVarId) := withMVarContext mvarId do - let savedSyntheticMVars := (← get).syntheticMVars - modify fun s => { s with syntheticMVars := [] } + let pendingMVarsSaved := (← get).pendingMVars + modify fun s => { s with pendingMVars := [] } let aux : TacticM (List MVarId) := /- Important: the following `try` does not backtrack the state. This is intentional because we don't want to backtrack the error messages when we catch the "abort internal exception" @@ -93,15 +93,15 @@ def run (mvarId : MVarId) (x : TacticM Unit) : TermElabM (List MVarId) := else throw ex try - aux.runCore' { elaborator := Name.anonymous } { goals := [mvarId] } + aux.runCore' { elaborator := .anonymous } { goals := [mvarId] } finally - modify fun s => { s with syntheticMVars := savedSyntheticMVars } + modify fun s => { s with pendingMVars := pendingMVarsSaved } protected def saveState : TacticM SavedState := return { term := (← Term.saveState), tactic := (← get) } -def SavedState.restore (b : SavedState) : TacticM Unit := do - b.term.restore +def SavedState.restore (b : SavedState) (restoreInfo := false) : TacticM Unit := do + b.term.restore restoreInfo set b.tactic protected def getCurrMacroScope : TacticM MacroScope := do pure (← readThe Core.Context).currMacroScope @@ -130,69 +130,81 @@ def mkInitialTacticInfo (stx : Syntax) : TacticM (TacticM Info) := do @[inline] def withTacticInfoContext (stx : Syntax) (x : TacticM α) : TacticM α := do withInfoContext x (← mkInitialTacticInfo stx) -/- -Important: we must define `evalTacticUsing` and `expandTacticMacroFns` before we define +/-! +Important: we must define `evalTactic` before we define the instance `MonadExcept` for `TacticM` since it backtracks the state including error messages, and this is bad when rethrowing the exception at the `catch` block in these methods. We marked these places with a `(*)` in these methods. -/ -private def evalTacticUsing (s : SavedState) (stx : Syntax) (tactics : List (KeyedDeclsAttribute.AttributeEntry Tactic)) : TacticM Unit := do - let rec loop - | [] => throwErrorAt stx "unexpected syntax {indentD stx}" - | evalFn::evalFns => do - try - withReader ({ · with elaborator := evalFn.declName }) <| withTacticInfoContext stx <| evalFn.value stx - catch - | ex@(Exception.error _ _) => - match evalFns with - | [] => throw ex -- (*) - | evalFns => s.restore; loop evalFns - | ex@(Exception.internal id _) => +/-- + Auxiliary datastructure for capturing exceptions at `evalTactic`. +-/ +structure EvalTacticFailure where + exception : Exception + state : SavedState + +partial def evalTactic (stx : Syntax) : TacticM Unit := + withRef stx <| withIncRecDepth <| withFreshMacroScope <| match stx with + | .node _ k _ => + if k == nullKind then + -- Macro writers create a sequence of tactics `t₁ ... tₙ` using `mkNullNode #[t₁, ..., tₙ]` + stx.getArgs.forM evalTactic + else do + trace[Elab.step] "{stx}" + let evalFns := tacticElabAttribute.getEntries (← getEnv) stx.getKind + let macros := macroAttribute.getEntries (← getEnv) stx.getKind + if evalFns.isEmpty && macros.isEmpty then + throwErrorAt stx "tactic '{stx.getKind}' has not been implemented" + let s ← Tactic.saveState + expandEval s macros evalFns #[] + | .missing => pure () + | _ => throwError m!"unexpected tactic{indentD stx}" +where + throwExs (failures : Array EvalTacticFailure) : TacticM Unit := do + if let some fail := failures[0]? then + -- Recall that `failures[0]` is the highest priority evalFn/macro + fail.state.restore (restoreInfo := true) + throw fail.exception -- (*) + else + throwErrorAt stx "unexpected syntax {indentD stx}" + + @[inline] handleEx (s : SavedState) (failures : Array EvalTacticFailure) (ex : Exception) (k : Array EvalTacticFailure → TacticM Unit) := do + match ex with + | .error .. => + trace[Elab.tactic.backtrack] ex.toMessageData + let failures := failures.push ⟨ex, ← Tactic.saveState⟩ + s.restore (restoreInfo := true); k failures + | .internal id _ => if id == unsupportedSyntaxExceptionId then - s.restore; loop evalFns + -- We do not store `unsupportedSyntaxExceptionId`, see throwExs + s.restore (restoreInfo := true); k failures + else if id == abortTacticExceptionId then + for msg in (← Core.getMessageLog).toList do + trace[Elab.tactic.backtrack] msg.data + let failures := failures.push ⟨ex, ← Tactic.saveState⟩ + s.restore (restoreInfo := true); k failures else - throw ex - loop tactics + throw ex -- (*) -mutual - - partial def expandTacticMacroFns (s : SavedState) (stx : Syntax) (macros : List (KeyedDeclsAttribute.AttributeEntry Macro)) : TacticM Unit := - let rec loop - | [] => throwErrorAt stx "tactic '{stx.getKind}' has not been implemented" - | m::ms => do + expandEval (s : SavedState) (macros : List _) (evalFns : List _) (failures : Array EvalTacticFailure) : TacticM Unit := + match macros with + | [] => eval s evalFns failures + | m :: ms => try withReader ({ · with elaborator := m.declName }) do withTacticInfoContext stx do let stx' ← adaptMacro m.value stx evalTactic stx' - catch ex => - if ms.isEmpty then throw ex -- (*) - s.restore; loop ms - loop macros - - partial def expandTacticMacro (s : SavedState) (stx : Syntax) : TacticM Unit := do - expandTacticMacroFns s stx (macroAttribute.getEntries (← getEnv) stx.getKind) - - partial def evalTacticAux (stx : Syntax) : TacticM Unit := - withRef stx <| withIncRecDepth <| withFreshMacroScope <| match stx with - | Syntax.node _ k _ => - if k == nullKind then - -- Macro writers create a sequence of tactics `t₁ ... tₙ` using `mkNullNode #[t₁, ..., tₙ]` - stx.getArgs.forM evalTactic - else do - trace[Elab.step] "{stx}" - let s ← Tactic.saveState - match tacticElabAttribute.getEntries (← getEnv) stx.getKind with - | [] => expandTacticMacro s stx - | evalFns => evalTacticUsing s stx evalFns - | Syntax.missing => pure () - | _ => throwError m!"unexpected tactic{indentD stx}" - - partial def evalTactic (stx : Syntax) : TacticM Unit := - evalTacticAux stx - -end + catch ex => handleEx s failures ex (expandEval s ms evalFns) + + eval (s : SavedState) (evalFns : List _) (failures : Array EvalTacticFailure) : TacticM Unit := do + match evalFns with + | [] => throwExs failures + | evalFn::evalFns => do + try + withReader ({ · with elaborator := evalFn.declName }) <| withTacticInfoContext stx <| evalFn.value stx + catch ex => handleEx s failures ex (eval s evalFns) def throwNoGoalsToBeSolved : TacticM α := throwError "no goals to be solved" @@ -217,7 +229,7 @@ def focusAndDone (tactic : TacticM α) : TacticM α := done pure a -/- Close the main goal using the given tactic. If it fails, log the error and `admit` -/ +/-- Close the main goal using the given tactic. If it fails, log the error and `admit` -/ def closeUsingOrAdmit (tac : TacticM Unit) : TacticM Unit := do /- Important: we must define `closeUsingOrAdmit` before we define the instance `MonadExcept` for `TacticM` since it backtracks the state including error messages. -/ @@ -248,17 +260,17 @@ instance : MonadExcept Exception TacticM where def withoutRecover (x : TacticM α) : TacticM α := withReader (fun ctx => { ctx with recover := false }) x -@[inline] protected def orElse {α} (x : TacticM α) (y : Unit → TacticM α) : TacticM α := do +@[inline] protected def orElse (x : TacticM α) (y : Unit → TacticM α) : TacticM α := do try withoutRecover x catch _ => y () -instance {α} : OrElse (TacticM α) where +instance : OrElse (TacticM α) where orElse := Tactic.orElse instance : Alternative TacticM where failure := fun {_} => throwError "failed" orElse := Tactic.orElse -/- +/-- Save the current tactic state for a token `stx`. This method is a no-op if `stx` has no position information. We use this method to save the tactic state at punctuation such as `;` @@ -267,9 +279,9 @@ def saveTacticInfoForToken (stx : Syntax) : TacticM Unit := do unless stx.getPos?.isNone do withTacticInfoContext stx (pure ()) -/- Elaborate `x` with `stx` on the macro stack -/ +/-- Elaborate `x` with `stx` on the macro stack -/ @[inline] -def withMacroExpansion {α} (beforeStx afterStx : Syntax) (x : TacticM α) : TacticM α := +def withMacroExpansion (beforeStx afterStx : Syntax) (x : TacticM α) : TacticM α := withMacroExpansionInfo beforeStx afterStx do withTheReader Term.Context (fun ctx => { ctx with macroStack := { before := beforeStx, after := afterStx } :: ctx.macroStack }) x @@ -348,6 +360,8 @@ def closeMainGoal (val : Expr) (checkUnassigned := true): TacticM Unit := do replaceMainGoal mvarIds pure a +/-- Get the mvarid of the main goal, run the given `tactic`, +then set the new goals to be the resulting goal list.-/ @[inline] def liftMetaTactic (tactic : MVarId → MetaM (List MVarId)) : TacticM Unit := liftMetaTacticAux fun mvarId => do let gs ← tactic mvarId @@ -406,5 +420,6 @@ def withCaseRef [Monad m] [MonadRef m] (arrow body : Syntax) (x : m α) : m α : withRef (mkNullNode #[arrow, body]) x builtin_initialize registerTraceClass `Elab.tactic +builtin_initialize registerTraceClass `Elab.tactic.backtrack end Lean.Elab.Tactic diff --git a/src/Lean/Elab/Tactic/BuiltinTactic.lean b/src/Lean/Elab/Tactic/BuiltinTactic.lean index ae2d4c4a0cfa..78de6362e135 100644 --- a/src/Lean/Elab/Tactic/BuiltinTactic.lean +++ b/src/Lean/Elab/Tactic/BuiltinTactic.lean @@ -64,7 +64,7 @@ where else return result ++ acc -/- Evaluate `many (group (tactic >> optional ";")) -/ +/-- Evaluate `many (group (tactic >> optional ";")) -/ def evalManyTacticOptSemi (stx : Syntax) : TacticM Unit := do for seqElem in (← addCheckpoints stx.getArgs) do evalTactic seqElem[0] diff --git a/src/Lean/Elab/Tactic/Conv/Basic.lean b/src/Lean/Elab/Tactic/Conv/Basic.lean index e5b90e228a5c..2e8783220c66 100644 --- a/src/Lean/Elab/Tactic/Conv/Basic.lean +++ b/src/Lean/Elab/Tactic/Conv/Basic.lean @@ -12,6 +12,8 @@ import Lean.Elab.Tactic.BuiltinTactic namespace Lean.Elab.Tactic.Conv open Meta +/-- Given `lhs`, returns a pair of metavariables `(?rhs, ?newGoal)` +where `?newGoal : lhs = ?rhs`.-/ def mkConvGoalFor (lhs : Expr) : MetaM (Expr × Expr) := do let lhsType ← inferType lhs let rhs ← mkFreshExprMVar lhsType @@ -25,6 +27,9 @@ def markAsConvGoal (mvarId : MVarId) : MetaM MVarId := do return mvarId -- it is already tagged as LHS goal replaceTargetDefEq mvarId (mkLHSGoal (← getMVarType mvarId)) +/-- Given `lhs`, runs the `conv` tactic with the goal `⊢ lhs = ?rhs`. +`conv` should produce no remaining goals that are not solvable with refl. +Returns a pair of instantiated expressions `(?rhs, ?p)` where `?p : lhs = ?rhs`. -/ def convert (lhs : Expr) (conv : TacticM Unit) : TacticM (Expr × Expr) := do let (rhs, newGoal) ← mkConvGoalFor lhs let savedGoals ← getGoals diff --git a/src/Lean/Elab/Tactic/ElabTerm.lean b/src/Lean/Elab/Tactic/ElabTerm.lean index 3f5d6ae0ad16..a656a2478e20 100644 --- a/src/Lean/Elab/Tactic/ElabTerm.lean +++ b/src/Lean/Elab/Tactic/ElabTerm.lean @@ -14,7 +14,7 @@ import Lean.Elab.SyntheticMVars namespace Lean.Elab.Tactic open Meta -/- `elabTerm` for Tactics and basic tactics that use it. -/ +/-! # `elabTerm` for Tactics and basic tactics that use it. -/ def elabTerm (stx : Syntax) (expectedType? : Option Expr) (mayPostpone := false) : TacticM Expr := do /- If error recovery is disabled, we disable `Term.withoutErrToSorry` -/ @@ -42,7 +42,7 @@ def elabTermEnsuringType (stx : Syntax) (expectedType? : Option Expr) (mayPostpo Term.throwTypeMismatchError none expectedType eType e return e -/- Try to close main goal using `x target`, where `target` is the type of the main goal. -/ +/-- Try to close main goal using `x target`, where `target` is the type of the main goal. -/ def closeMainGoalUsing (x : Expr → TacticM Expr) (checkUnassigned := true) : TacticM Unit := withMainContext do closeMainGoal (checkUnassigned := checkUnassigned) (← x (← getMainTarget)) @@ -81,7 +81,7 @@ def elabTermWithHoles (stx : Syntax) (expectedType? : Option Expr) (tagSuffix : tagUntaggedGoals (← getMainTag) tagSuffix newMVarIds pure (val, newMVarIds) -/- If `allowNaturalHoles == true`, then we allow the resultant expression to contain unassigned "natural" metavariables. +/-- If `allowNaturalHoles == true`, then we allow the resultant expression to contain unassigned "natural" metavariables. Recall that "natutal" metavariables are created for explicit holes `_` and implicit arguments. They are meant to be filled by typing constraints. "Synthetic" metavariables are meant to be filled by tactics and are usually created using the synthetic hole notation `?`. -/ @@ -224,7 +224,7 @@ def elabAsFVar (stx : Syntax) (userName? : Option Name := none) : TacticM FVarId withMainContext do let e ← elabTerm stx none match e with - | Expr.fvar fvarId => pure fvarId + | .fvar fvarId => pure fvarId | _ => let type ← inferType e let intro (userName : Name) (preserveBinderNames : Bool) : TacticM FVarId := do @@ -242,14 +242,10 @@ def elabAsFVar (stx : Syntax) (userName? : Option Name := none) : TacticM FVarId match stx with | `(tactic| rename $typeStx:term => $h:ident) => do withMainContext do - /- Remark: we must not use `withoutModifyingState` because we may miss errors message. - For example, suppose the following `elabTerm` logs an error during elaboration. - In this scenario, the term `type` contains a synthetic `sorry`, and the error - message `"failed to find ..."` is not logged by the outer loop. - By using `withoutModifyingStateWithInfoAndMessages`, we ensure that - the messages and the info trees are preserved while the rest of the - state is backtracked. -/ - let fvarId ← withoutModifyingStateWithInfoAndMessages <| withNewMCtxDepth do + /- Remark: we also use `withoutRecover` to make sure `elabTerm` does not succeed + using `sorryAx`, and we get `"failed to find ..."` which will not be logged because + it contains synthetic sorry's -/ + let fvarId ← withoutModifyingState <| withNewMCtxDepth <| withoutRecover do let type ← elabTerm typeStx none (mayPostpone := true) let fvarId? ← (← getLCtx).findDeclRevM? fun localDecl => do if (← isDefEq type localDecl.type) then return localDecl.fvarId else return none diff --git a/src/Lean/Elab/Tactic/Induction.lean b/src/Lean/Elab/Tactic/Induction.lean index 94e7c0f6ac7c..1acf41703a7f 100644 --- a/src/Lean/Elab/Tactic/Induction.lean +++ b/src/Lean/Elab/Tactic/Induction.lean @@ -68,7 +68,7 @@ def evalAlt (mvarId : MVarId) (alt : Syntax) (remainingGoals : Array MVarId) : T closeUsingOrAdmit (withTacticInfoContext alt (evalTactic rhs)) return remainingGoals -/- +/-! Helper method for creating an user-defined eliminator/recursor application. -/ namespace ElimApp @@ -90,9 +90,9 @@ abbrev M := ReaderT Context $ StateRefT State TermElabM private def addNewArg (arg : Expr) : M Unit := modify fun s => { s with argPos := s.argPos+1, f := mkApp s.f arg, fType := s.fType.bindingBody!.instantiate1 arg } -/- Return the binder name at `fType`. This method assumes `fType` is a function type. -/ +/-- Return the binder name at `fType`. This method assumes `fType` is a function type. -/ private def getBindingName : M Name := return (← get).fType.bindingName! -/- Return the next argument expected type. This method assumes `fType` is a function type. -/ +/-- Return the next argument expected type. This method assumes `fType` is a function type. -/ private def getArgExpectedType : M Expr := return (← get).fType.bindingDomain! private def getFType : M Expr := do @@ -114,7 +114,7 @@ structure Result where partial def mkElimApp (elimInfo : ElimInfo) (targets : Array Expr) (tag : Name) : TermElabM Result := do let rec loop : M Unit := do match (← getFType) with - | Expr.forallE binderName _ _ c => + | .forallE binderName _ _ c => let ctx ← read let argPos := (← get).argPos if ctx.elimInfo.motivePos == argPos then @@ -131,13 +131,13 @@ partial def mkElimApp (elimInfo : ElimInfo) (targets : Array Expr) (tag : Name) modify fun s => { s with targetPos := s.targetPos + 1 } addNewArg target else match c with - | BinderInfo.implicit => + | .implicit => let arg ← mkFreshExprMVar (← getArgExpectedType) addNewArg arg - | BinderInfo.strictImplicit => + | .strictImplicit => let arg ← mkFreshExprMVar (← getArgExpectedType) addNewArg arg - | BinderInfo.instImplicit => + | .instImplicit => let arg ← mkFreshExprMVar (← getArgExpectedType) (kind := MetavarKind.synthetic) (userName := appendTag tag binderName) modify fun s => { s with insts := s.insts.push arg.mvarId! } addNewArg arg @@ -164,7 +164,7 @@ partial def mkElimApp (elimInfo : ElimInfo) (targets : Array Expr) (tag : Name) let alts ← s.alts.filterM fun alt => return !(← isExprMVarAssigned alt.2) return { elimApp := (← instantiateMVars s.f), alts, others := others } -/- Given a goal `... targets ... |- C[targets]` associated with `mvarId`, assign +/-- Given a goal `... targets ... |- C[targets]` associated with `mvarId`, assign `motiveArg := fun targets => C[targets]` -/ def setMotiveArg (mvarId : MVarId) (motiveArg : MVarId) (targets : Array FVarId) : MetaM Unit := do let type ← inferType (mkMVar mvarId) @@ -441,7 +441,7 @@ private def expandCases? (induction : Syntax) : Option Syntax := do let inductionAlts' ← expandInductionAlts? optInductionAlts[0] return induction.setArg 3 (mkNullNode #[inductionAlts']) -/- +/-- We may have at most one `| _ => ...` (wildcard alternative), and it must not set variable names. The idea is to make sure users do not write unstructured tactics. -/ private def checkAltsOfOptInductionAlts (optInductionAlts : Syntax) : TacticM Unit := diff --git a/src/Lean/Elab/Tactic/Location.lean b/src/Lean/Elab/Tactic/Location.lean index 84979e858489..6ae34f3678a7 100644 --- a/src/Lean/Elab/Tactic/Location.lean +++ b/src/Lean/Elab/Tactic/Location.lean @@ -8,9 +8,13 @@ import Lean.Elab.Tactic.ElabTerm namespace Lean.Elab.Tactic +/-- Denotes a set of locations where a tactic should be applied for the main goal. See also `withLocation`. -/ inductive Location where - | wildcard - | targets (hypotheses : Array Syntax) (type : Bool) + | /-- Apply the tactic everywhere. -/ + wildcard + | /-- `hypotheses` are hypothesis names in the main goal that the tactic should be applied to. + If `type` is true, then the tactic should also be applied to the target type. -/ + targets (hypotheses : Array Syntax) (type : Bool) /- Recall that @@ -35,6 +39,9 @@ def expandOptLocation (stx : Syntax) : Location := open Meta +/-- Runs the given `atLocal` and `atTarget` methods on each of the locations selected by the given `loc`. +If any of the selected tactic applications fail, it will call `failed` with the main goal mvar. + -/ def withLocation (loc : Location) (atLocal : FVarId → TacticM Unit) (atTarget : TacticM Unit) (failed : MVarId → TacticM Unit) : TacticM Unit := do match loc with | Location.targets hyps type => diff --git a/src/Lean/Elab/Tactic/Simp.lean b/src/Lean/Elab/Tactic/Simp.lean index c8e1f56ad965..9145e2e9a609 100644 --- a/src/Lean/Elab/Tactic/Simp.lean +++ b/src/Lean/Elab/Tactic/Simp.lean @@ -126,11 +126,11 @@ inductive ResolveSimpIdResult where | ext (ext : SimpExtension) /-- - Elaborate extra simp theorems provided to `simp`. `stx` is of the `simpTheorem,*` + Elaborate extra simp theorems provided to `simp`. `stx` is of the form `"[" simpTheorem,* "]"` If `eraseLocal == true`, then we consider local declarations when resolving names for erased theorems (`- id`), this option only makes sense for `simp_all`. -/ -private def elabSimpArgs (stx : Syntax) (ctx : Simp.Context) (eraseLocal : Bool) (kind : SimpKind) : TacticM ElabSimpArgsResult := do +def elabSimpArgs (stx : Syntax) (ctx : Simp.Context) (eraseLocal : Bool) (kind : SimpKind) : TacticM ElabSimpArgsResult := do if stx.isNone then return { ctx } else diff --git a/src/Lean/Elab/Term.lean b/src/Lean/Elab/Term.lean index bb0245b94e13..56757f91419f 100644 --- a/src/Lean/Elab/Term.lean +++ b/src/Lean/Elab/Term.lean @@ -50,18 +50,19 @@ inductive SyntheticMVarKind where tactic (tacticCode : Syntax) (ctx : SavedContext) | /-- Metavariable represents a hole whose elaboration has been postponed. -/ postponed (ctx : SavedContext) + deriving Inhabited instance : ToString SyntheticMVarKind where toString - | SyntheticMVarKind.typeClass => "typeclass" - | SyntheticMVarKind.coe .. => "coe" - | SyntheticMVarKind.tactic .. => "tactic" - | SyntheticMVarKind.postponed .. => "postponed" + | .typeClass => "typeclass" + | .coe .. => "coe" + | .tactic .. => "tactic" + | .postponed .. => "postponed" structure SyntheticMVarDecl where - mvarId : MVarId stx : Syntax kind : SyntheticMVarKind + deriving Inhabited /-- We can optionally associate an error context with a metavariable (see `MVarErrorInfo`). @@ -78,9 +79,9 @@ inductive MVarErrorKind where instance : ToString MVarErrorKind where toString - | MVarErrorKind.implicitArg _ => "implicitArg" - | MVarErrorKind.hole => "hole" - | MVarErrorKind.custom _ => "custom" + | .implicitArg _ => "implicitArg" + | .hole => "hole" + | .custom _ => "custom" /-- We can optionally associate an error context with metavariables. @@ -114,7 +115,8 @@ structure LetRecToLift where -/ structure State where levelNames : List Name := [] - syntheticMVars : List SyntheticMVarDecl := [] + syntheticMVars : MVarIdMap SyntheticMVarDecl := {} + pendingMVars : List MVarId := {} mvarErrorInfos : MVarIdMap MVarErrorInfo := {} letRecsToLift : List LetRecToLift := [] infoState : InfoState := {} @@ -252,7 +254,7 @@ def SavedState.restore (s : SavedState) (restoreInfo : Bool := false) : TermElab set s.elab setTraceState traceState unless restoreInfo do - modify fun s => { s with infoState := infoState } + modify fun s => { s with infoState } instance : MonadBacktrack SavedState TermElabM where saveState := Term.saveState @@ -278,11 +280,11 @@ def observing (x : TermElabM α) : TermElabM (TermElabResult α) := do s.restore (restoreInfo := true) return EStateM.Result.ok e sNew catch - | ex@(Exception.error _ _) => + | ex@(.error ..) => let sNew ← saveState s.restore (restoreInfo := true) - return EStateM.Result.error ex sNew - | ex@(Exception.internal id _) => + return .error ex sNew + | ex@(.internal id _) => if id == postponeExceptionId then s.restore (restoreInfo := true) throw ex @@ -292,8 +294,8 @@ def observing (x : TermElabM α) : TermElabM (TermElabResult α) := do We use this method to implement overloaded notation and symbols. -/ def applyResult (result : TermElabResult α) : TermElabM α := do match result with - | EStateM.Result.ok a r => r.restore (restoreInfo := true); return a - | EStateM.Result.error ex r => r.restore (restoreInfo := true); throw ex + | .ok a r => r.restore (restoreInfo := true); return a + | .error ex r => r.restore (restoreInfo := true); throw ex /-- Execute `x`, but keep state modifications only if `x` did not postpone. @@ -342,7 +344,7 @@ def withoutModifyingElabMetaStateWithInfo (x : TermElabM α) : TermElabM α := d let s ← get let sMeta ← getThe Meta.State try - withSaveInfoContext x + withSaveInfoContext x finally modify ({ s with infoState := ·.infoState }) set sMeta @@ -380,22 +382,22 @@ builtin_initialize termElabAttribute : KeyedDeclsAttribute TermElab ← mkTermEl -/ inductive LVal where | fieldIdx (ref : Syntax) (i : Nat) - /- Field `suffix?` is for producing better error messages because `x.y` may be a field access or a hierachical/composite name. + | /-- Field `suffix?` is for producing better error messages because `x.y` may be a field access or a hierachical/composite name. `ref` is the syntax object representing the field. `targetStx` is the target object being accessed. -/ - | fieldName (ref : Syntax) (name : String) (suffix? : Option Name) (targetStx : Syntax) + fieldName (ref : Syntax) (name : String) (suffix? : Option Name) (targetStx : Syntax) def LVal.getRef : LVal → Syntax - | LVal.fieldIdx ref _ => ref - | LVal.fieldName ref .. => ref + | .fieldIdx ref _ => ref + | .fieldName ref .. => ref def LVal.isFieldName : LVal → Bool - | LVal.fieldName .. => true + | .fieldName .. => true | _ => false instance : ToString LVal where toString - | LVal.fieldIdx _ i => toString i - | LVal.fieldName _ n .. => n + | .fieldIdx _ i => toString i + | .fieldName _ n .. => n /-- Return the name of the declaration being elaborated if available. -/ def getDeclName? : TermElabM (Option Name) := return (← read).declName? @@ -453,22 +455,22 @@ def liftLevelM (x : LevelElabM α) : TermElabM α := do let ngen ← getNGen let lvlCtx : Level.Context := { options := (← getOptions), ref := (← getRef), autoBoundImplicit := ctx.autoBoundImplicit } match (x lvlCtx).run { ngen := ngen, mctx := mctx, levelNames := (← getLevelNames) } with - | EStateM.Result.ok a newS => setMCtx newS.mctx; setNGen newS.ngen; setLevelNames newS.levelNames; pure a - | EStateM.Result.error ex _ => throw ex + | .ok a newS => setMCtx newS.mctx; setNGen newS.ngen; setLevelNames newS.levelNames; pure a + | .error ex _ => throw ex def elabLevel (stx : Syntax) : TermElabM Level := liftLevelM <| Level.elabLevel stx -/- Elaborate `x` with `stx` on the macro stack -/ +/-- Elaborate `x` with `stx` on the macro stack -/ def withMacroExpansion (beforeStx afterStx : Syntax) (x : TermElabM α) : TermElabM α := withMacroExpansionInfo beforeStx afterStx do withReader (fun ctx => { ctx with macroStack := { before := beforeStx, after := afterStx } :: ctx.macroStack }) x -/- +/-- Add the given metavariable to the list of pending synthetic metavariables. The method `synthesizeSyntheticMVars` is used to process the metavariables on this list. -/ def registerSyntheticMVar (stx : Syntax) (mvarId : MVarId) (kind : SyntheticMVarKind) : TermElabM Unit := do - modify fun s => { s with syntheticMVars := { mvarId := mvarId, stx := stx, kind := kind } :: s.syntheticMVars } + modify fun s => { s with syntheticMVars := s.syntheticMVars.insert mvarId { stx, kind }, pendingMVars := mvarId :: s.pendingMVars } def registerSyntheticMVarWithCurrRef (mvarId : MVarId) (kind : SyntheticMVarKind) : TermElabM Unit := do registerSyntheticMVar (← getRef) mvarId kind @@ -477,13 +479,13 @@ def registerMVarErrorInfo (mvarErrorInfo : MVarErrorInfo) : TermElabM Unit := modify fun s => { s with mvarErrorInfos := s.mvarErrorInfos.insert mvarErrorInfo.mvarId mvarErrorInfo } def registerMVarErrorHoleInfo (mvarId : MVarId) (ref : Syntax) : TermElabM Unit := - registerMVarErrorInfo { mvarId := mvarId, ref := ref, kind := MVarErrorKind.hole } + registerMVarErrorInfo { mvarId, ref, kind := .hole } def registerMVarErrorImplicitArgInfo (mvarId : MVarId) (ref : Syntax) (app : Expr) : TermElabM Unit := do - registerMVarErrorInfo { mvarId := mvarId, ref := ref, kind := MVarErrorKind.implicitArg app } + registerMVarErrorInfo { mvarId, ref, kind := .implicitArg app } def registerMVarErrorCustomInfo (mvarId : MVarId) (ref : Syntax) (msgData : MessageData) : TermElabM Unit := do - registerMVarErrorInfo { mvarId := mvarId, ref := ref, kind := MVarErrorKind.custom msgData } + registerMVarErrorInfo { mvarId, ref, kind := .custom msgData } def getMVarErrorInfo? (mvarId : MVarId) : TermElabM (Option MVarErrorInfo) := do return (← get).mvarErrorInfos.find? mvarId @@ -493,7 +495,7 @@ def registerCustomErrorIfMVar (e : Expr) (ref : Syntax) (msgData : MessageData) | Expr.mvar mvarId => registerMVarErrorCustomInfo mvarId ref msgData | _ => pure () -/- +/-- Auxiliary method for reporting errors of the form "... contains metavariables ...". This kind of error is thrown, for example, at `Match.lean` where elaboration cannot continue if there are metavariables in patterns. @@ -569,7 +571,7 @@ def ensureNoUnassignedMVars (decl : Declaration) : TermElabM Unit := do if (← logUnassignedUsingErrorInfos pendingMVarIds) then throwAbortCommand -/- +/-- Execute `x` without allowing it to postpone elaboration tasks. That is, `tryPostpone` is a noop. -/ def withoutPostponing (x : TermElabM α) : TermElabM α := @@ -615,6 +617,7 @@ private def applyAttributesCore (declName : Name) (attrs : Array Attribute) (applicationTime? : Option AttributeApplicationTime) : TermElabM Unit := for attr in attrs do + withRef attr.stx do withLogging do let env ← getEnv match getAttributeImpl env attr.name with | Except.error errMsg => throwError errMsg @@ -670,17 +673,17 @@ abbrev M := MonadCacheT Expr Unit (OptionT TermElabM) partial def visit (e : Expr) : M Unit := do checkCache e fun _ => do match e with - | Expr.forallE _ d b _ => visit d; visit b - | Expr.lam _ d b _ => visit d; visit b - | Expr.letE _ t v b _ => visit t; visit v; visit b - | Expr.app f a => visit f; visit a - | Expr.mdata _ b => visit b - | Expr.proj _ _ b => visit b - | Expr.fvar fvarId .. => + | .forallE _ d b _ => visit d; visit b + | .lam _ d b _ => visit d; visit b + | .letE _ t v b _ => visit t; visit v; visit b + | .app f a => visit f; visit a + | .mdata _ b => visit b + | .proj _ _ b => visit b + | .fvar fvarId .. => match (← getLocalDecl fvarId) with - | LocalDecl.cdecl .. => return () + | .cdecl .. => return () | LocalDecl.ldecl (value := v) .. => visit v - | Expr.mvar mvarId .. => + | .mvar mvarId .. => let e' ← instantiateMVars e if e' != e then visit e' @@ -745,8 +748,8 @@ def synthesizeInstMVarCore (instMVar : MVarId) (maxResultSize? : Option Nat := n unless (← isDefEq (mkMVar instMVar) val) do throwError "failed to assign synthesized type class instance{indentExpr val}" return true - | LOption.undef => return false -- we will try later - | LOption.none => + | .undef => return false -- we will try later + | .none => if (← read).ignoreTCFailures then return false else @@ -771,7 +774,7 @@ def synthesizeCoeInstMVarCore (instMVar : MVarId) : TermElabM Bool := do -/ def tryCoeThunk? (expectedType : Expr) (eType : Expr) (e : Expr) : TermElabM (Option Expr) := do match expectedType with - | Expr.app (Expr.const ``Thunk u) arg => + | .app (.const ``Thunk u) arg => if (← isDefEq eType arg) then return some (mkApp2 (mkConst ``Thunk.mk u) arg (mkSimpleThunk e)) else @@ -797,8 +800,8 @@ def mkCoe (expectedType : Expr) (eType : Expr) (e : Expr) (f? : Option Expr := n registerSyntheticMVarWithCurrRef mvarAux.mvarId! (SyntheticMVarKind.coe errorMsgHeader? eNew expectedType eType e f?) return mvarAux catch - | Exception.error _ msg => throwTypeMismatchError errorMsgHeader? expectedType eType e f? msg - | _ => throwTypeMismatchError errorMsgHeader? expectedType eType e f? + | .error _ msg => throwTypeMismatchError errorMsgHeader? expectedType eType e f? msg + | _ => throwTypeMismatchError errorMsgHeader? expectedType eType e f? /-- Try to apply coercion to make sure `e` has type `expectedType`. @@ -819,17 +822,17 @@ private def tryCoe (errorMsgHeader? : Option String) (expectedType : Expr) (eTyp def isTypeApp? (type : Expr) : TermElabM (Option (Expr × Expr)) := do let type ← withReducible <| whnf type match type with - | Expr.app m α => return some ((← instantiateMVars m), (← instantiateMVars α)) - | _ => return none + | .app m α => return some ((← instantiateMVars m), (← instantiateMVars α)) + | _ => return none /-- Helper method used to implement auto-lift and coercions -/ private def synthesizeInst (type : Expr) : TermElabM Expr := do let type ← instantiateMVars type match (← trySynthInstance type) with - | LOption.some val => return val + | .some val => return val -- Note that `ignoreTCFailures` is not checked here since it must return a result. - | LOption.undef => throwError "failed to synthesize instance{indentExpr type}" - | LOption.none => throwError "failed to synthesize instance{indentExpr type}" + | .undef => throwError "failed to synthesize instance{indentExpr type}" + | .none => throwError "failed to synthesize instance{indentExpr type}" /-- Return `true` if `type` is of the form `m α` where `m` is a `Monad`. @@ -847,13 +850,13 @@ Otherwise, we just use the basic `tryCoe`. Extensions for monads. -1- Try to unify `n` and `m`. If it succeeds, then we use - ``` - coeM {m : Type u → Type v} {α β : Type u} [∀ a, CoeT α a β] [Monad m] (x : m α) : m β - ``` - `n` must be a `Monad` to use this one. +1. Try to unify `n` and `m`. If it succeeds, then we use + ``` + coeM {m : Type u → Type v} {α β : Type u} [∀ a, CoeT α a β] [Monad m] (x : m α) : m β + ``` + `n` must be a `Monad` to use this one. -2- If there is monad lift from `m` to `n` and we can unify `α` and `β`, we use +2. If there is monad lift from `m` to `n` and we can unify `α` and `β`, we use ``` liftM : ∀ {m : Type u_1 → Type u_2} {n : Type u_1 → Type u_3} [self : MonadLiftT m n] {α : Type u_1}, m α → n α ``` @@ -868,7 +871,7 @@ Extensions for monads. ``` -3- If there is a monad lif from `m` to `n` and a coercion from `α` to `β`, we use +3. If there is a monad lif from `m` to `n` and a coercion from `α` to `β`, we use ``` liftCoeM {m : Type u → Type v} {n : Type u → Type w} {α β : Type u} [MonadLiftT m n] [∀ a, CoeT α a β] [Monad n] (x : m α) : n β ``` @@ -1052,7 +1055,7 @@ private def postponeElabTerm (stx : Syntax) (expectedType? : Option Expr) : Term return mvar def getSyntheticMVarDecl? (mvarId : MVarId) : TermElabM (Option SyntheticMVarDecl) := - return (← get).syntheticMVars.find? fun d => d.mvarId == mvarId + return (← get).syntheticMVars.find? mvarId /-- Create an auxiliary annotation to make sure we create a `Info` even if `e` is a metavariable. @@ -1094,9 +1097,9 @@ def isTacticOrPostponedHole? (e : Expr) : TermElabM (Option MVarId) := do match e with | Expr.mvar mvarId => match (← getSyntheticMVarDecl? mvarId) with - | some { kind := SyntheticMVarKind.tactic .., .. } => return mvarId - | some { kind := SyntheticMVarKind.postponed .., .. } => return mvarId - | _ => return none + | some { kind := .tactic .., .. } => return mvarId + | some { kind := .postponed .., .. } => return mvarId + | _ => return none | _ => pure none def mkTermInfo (elaborator : Name) (stx : Syntax) (e : Expr) (expectedType? : Option Expr := none) (lctx? : Option LocalContext := none) (isBinder := false) : TermElabM (Sum Info MVarId) := do @@ -1123,7 +1126,7 @@ def withInfoContext' (stx : Syntax) (x : TermElabM Expr) (mkInfo : Expr → Term else Elab.withInfoContext' x mkInfo -/- +/-- Helper function for `elabTerm` is tries the registered elaboration functions for `stxNode` kind until it finds one that supports the syntax or an error is found. -/ private def elabUsingElabFnsAux (s : SavedState) (stx : Syntax) (expectedType? : Option Expr) (catchExPostpone : Bool) @@ -1136,12 +1139,12 @@ private def elabUsingElabFnsAux (s : SavedState) (stx : Syntax) (expectedType? : (try elabFn.value stx expectedType? catch ex => match ex with - | Exception.error _ _ => + | .error .. => if (← read).errToSorry then exceptionToSorry ex expectedType? else throw ex - | Exception.internal id _ => + | .internal id _ => if (← read).errToSorry && id == abortTermExceptionId then exceptionToSorry ex expectedType? else if id == unsupportedSyntaxExceptionId then @@ -1166,7 +1169,7 @@ private def elabUsingElabFnsAux (s : SavedState) (stx : Syntax) (expectedType? : else throw ex) catch ex => match ex with - | Exception.internal id _ => + | .internal id _ => if id == unsupportedSyntaxExceptionId then s.restore -- also removes the info tree created above elabUsingElabFnsAux s stx expectedType? catchExPostpone elabFns @@ -1261,7 +1264,7 @@ private def useImplicitLambda? (stx : Syntax) (expectedType? : Option Expr) : Te else let expectedType ← whnfForall expectedType match expectedType with - | Expr.forallE _ _ _ c => + | .forallE _ _ _ c => if c.isImplicit || c.isInstImplicit then return some expectedType else @@ -1271,7 +1274,7 @@ private def useImplicitLambda? (stx : Syntax) (expectedType? : Option Expr) : Te private def decorateErrorMessageWithLambdaImplicitVars (ex : Exception) (impFVars : Array Expr) : TermElabM Exception := do match ex with - | Exception.error ref msg => + | .error ref msg => if impFVars.isEmpty then return Exception.error ref msg else @@ -1298,7 +1301,7 @@ private partial def elabImplicitLambda (stx : Syntax) (catchExPostpone : Bool) ( loop type #[] where loop - | type@(Expr.forallE n d b c), fvars => + | type@(.forallE n d b c), fvars => if c.isExplicit then elabImplicitLambdaAux stx catchExPostpone type fvars else withFreshMacroScope do @@ -1309,9 +1312,9 @@ where | type, fvars => elabImplicitLambdaAux stx catchExPostpone type fvars -/- Main loop for `elabTerm` -/ +/-- Main loop for `elabTerm` -/ private partial def elabTermAux (expectedType? : Option Expr) (catchExPostpone : Bool) (implicitLambda : Bool) : Syntax → TermElabM Expr - | Syntax.missing => mkSyntheticSorryFor expectedType? + | .missing => mkSyntheticSorryFor expectedType? | stx => withFreshMacroScope <| withIncRecDepth do trace[Elab.step] "expected type: {expectedType?}, term\n{stx}" checkMaxHeartbeats "elaborator" @@ -1332,7 +1335,7 @@ private partial def elabTermAux (expectedType? : Option Expr) (catchExPostpone : /-- Store in the `InfoTree` that `e` is a "dot"-completion target. -/ def addDotCompletionInfo (stx : Syntax) (e : Expr) (expectedType? : Option Expr) (field? : Option Syntax := none) : TermElabM Unit := do - addCompletionInfo <| CompletionInfo.dot { expr := e, stx, lctx := (← getLCtx), elaborator := Name.anonymous, expectedType? } (field? := field?) (expectedType? := expectedType?) + addCompletionInfo <| CompletionInfo.dot { expr := e, stx, lctx := (← getLCtx), elaborator := .anonymous, expectedType? } (field? := field?) (expectedType? := expectedType?) /-- Main function for elaborating terms. @@ -1358,17 +1361,6 @@ def elabTermEnsuringType (stx : Syntax) (expectedType? : Option Expr) (catchExPo let e ← elabTerm stx expectedType? catchExPostpone implicitLambda withRef stx <| ensureHasType expectedType? e errorMsgHeader? -/-- - Execute `x` and then restore `syntheticMVars`, `levelNames`, `mvarErrorInfos`, and `letRecsToLift`. - We use this combinator when we don't want the pending problems created by `x` to persist after its execution. -/ -def withoutPending (x : TermElabM α) : TermElabM α := do - let saved ← get - try - x - finally - modify fun s => { s with syntheticMVars := saved.syntheticMVars, levelNames := saved.levelNames, - letRecsToLift := saved.letRecsToLift, mvarErrorInfos := saved.mvarErrorInfos } - /-- Execute `x` and return `some` if no new errors were recorded or exceptions was thrown. Otherwise, return `none` -/ def commitIfNoErrors? (x : TermElabM α) : TermElabM (Option α) := do let saved ← saveState @@ -1413,7 +1405,7 @@ private def tryCoeSort (α : Expr) (a : Expr) : TermElabM Expr := do let u ← getLevel α let v ← getLevel β let coeSortInstType := mkAppN (Lean.mkConst ``CoeSort [u, v]) #[α, β] - let mvar ← mkFreshExprMVar coeSortInstType MetavarKind.synthetic + let mvar ← mkFreshExprMVar coeSortInstType .synthetic let mvarId := mvar.mvarId! try withoutMacroStackAtErr do @@ -1425,8 +1417,8 @@ private def tryCoeSort (α : Expr) (a : Expr) : TermElabM Expr := do else throwError "type expected" catch - | Exception.error _ msg => throwError "type expected\n{msg}" - | _ => throwError "type expected" + | .error _ msg => throwError "type expected\n{msg}" + | _ => throwError "type expected" /-- Make sure `e` is a type by inferring its type and making sure it is a `Expr.sort` @@ -1463,7 +1455,7 @@ partial def withAutoBoundImplicit (k : TermElabM α) : TermElabM α := do | some n => -- Restore state, declare `n`, and try again s.restore - withLocalDecl n BinderInfo.implicit (← mkFreshTypeMVar) fun x => + withLocalDecl n .implicit (← mkFreshTypeMVar) fun x => withReader (fun ctx => { ctx with autoBoundImplicits := ctx.autoBoundImplicits.push x } ) do loop (← saveState) | none => throw ex @@ -1552,7 +1544,7 @@ def mkAuxName (suffix : Name) : TermElabM Name := do builtin_initialize registerTraceClass `Elab.letrec -/- Return true if mvarId is an auxiliary metavariable created for compiling `let rec` or it +/-- Return true if mvarId is an auxiliary metavariable created for compiling `let rec` or it is delayed assigned to one. -/ def isLetRecAuxMVar (mvarId : MVarId) : TermElabM Bool := do trace[Elab.letrec] "mvarId: {mkMVar mvarId} letrecMVars: {(← get).letRecsToLift.map (mkMVar $ ·.mvarId)}" diff --git a/src/Lean/Elab/Util.lean b/src/Lean/Elab/Util.lean index 883232d2d5fd..96fa3b626b41 100644 --- a/src/Lean/Elab/Util.lean +++ b/src/Lean/Elab/Util.lean @@ -8,6 +8,7 @@ import Lean.Parser.Syntax import Lean.Parser.Extension import Lean.KeyedDeclsAttribute import Lean.Elab.Exception +import Lean.Elab.InfoTree import Lean.DocString import Lean.DeclarationRange import Lean.Compiler.InitAttr @@ -44,7 +45,7 @@ structure MacroStackElem where abbrev MacroStack := List MacroStackElem -/- If `ref` does not have position information, then try to use macroStack -/ +/-- If `ref` does not have position information, then try to use macroStack -/ def getBetterRef (ref : Syntax) (macroStack : MacroStack) : Syntax := match ref.getPos? with | some _ => ref @@ -204,6 +205,10 @@ def logException [Monad m] [MonadLog m] [AddMessageContext m] [MonadLiftT IO m] let name ← id.getName logError m!"internal exception: {name}" +def withLogging [Monad m] [MonadLog m] [MonadExcept Exception m] [AddMessageContext m] [MonadLiftT IO m] + (x : m Unit) : m Unit := do + try x catch ex => logException ex + @[inline] def trace [Monad m] [MonadLog m] [AddMessageContext m] [MonadOptions m] (cls : Name) (msg : Unit → MessageData) : m Unit := do if checkTraceOption (← getOptions) cls then logTrace cls (msg ()) diff --git a/src/Lean/Environment.lean b/src/Lean/Environment.lean index 048fe30174c4..388890eb1773 100644 --- a/src/Lean/Environment.lean +++ b/src/Lean/Environment.lean @@ -13,7 +13,7 @@ import Lean.Util.FindExpr import Lean.Util.Profile namespace Lean -/- Opaque environment extension state. -/ +/-- Opaque environment extension state. -/ opaque EnvExtensionStateSpec : (α : Type) × Inhabited α := ⟨Unit, ⟨()⟩⟩ def EnvExtensionState : Type := EnvExtensionStateSpec.fst instance : Inhabited EnvExtensionState := EnvExtensionStateSpec.snd @@ -44,12 +44,12 @@ opaque CompactedRegion.isMemoryMapped : CompactedRegion → Bool @[extern "lean_compacted_region_free"] unsafe opaque CompactedRegion.free : CompactedRegion → IO Unit -/- Opaque persistent environment extension entry. -/ +/-- Opaque persistent environment extension entry. -/ opaque EnvExtensionEntrySpec : NonemptyType.{0} def EnvExtensionEntry : Type := EnvExtensionEntrySpec.type instance : Nonempty EnvExtensionEntry := EnvExtensionEntrySpec.property -/- Content of a .olean file. +/-- Content of a .olean file. We use `compact.cpp` to generate the image of this object in disk. -/ structure ModuleData where imports : Array Import @@ -57,7 +57,7 @@ structure ModuleData where entries : Array (Name × Array EnvExtensionEntry) deriving Inhabited -/- Environment fields that are not used often. -/ +/-- Environment fields that are not used often. -/ structure EnvironmentHeader where trustLevel : UInt32 := 0 quotInit : Bool := false @@ -145,13 +145,13 @@ inductive KernelException where namespace Environment -/- Type check given declaration and add it to the environment -/ +/-- Type check given declaration and add it to the environment -/ @[extern "lean_add_decl"] opaque addDecl (env : Environment) (decl : @& Declaration) : Except KernelException Environment end Environment -/- Interface for managing environment extensions. -/ +/-- Interface for managing environment extensions. -/ structure EnvExtensionInterface where ext : Type → Type inhabitedExt {σ} : Inhabited σ → Inhabited (ext σ) @@ -174,7 +174,7 @@ instance : Inhabited EnvExtensionInterface where mkInitialExtStates := pure #[] } -/- Unsafe implementation of `EnvExtensionInterface` -/ +/-! # Unsafe implementation of `EnvExtensionInterface` -/ namespace EnvExtensionInterfaceUnsafe structure Ext (σ : Type) where @@ -272,7 +272,7 @@ def modifyState {σ : Type} (ext : EnvExtension σ) (env : Environment) (f : σ def getState {σ : Type} [Inhabited σ] (ext : EnvExtension σ) (env : Environment) : σ := EnvExtensionInterfaceImp.getState ext env end EnvExtension -/- Environment extensions can only be registered during initialization. +/-- Environment extensions can only be registered during initialization. Reasons: 1- Our implementation assumes the number of extensions does not change after an environment object is created. 2- We do not use any synchronization primitive to access `envExtensionsRef`. @@ -304,7 +304,7 @@ structure ImportM.Context where abbrev ImportM := ReaderT Lean.ImportM.Context IO -/- An environment extension with support for storing/retrieving entries from a .olean file. +/-- An environment extension with support for storing/retrieving entries from a .olean file. - α is the type of the entries that are stored in .olean files. - β is the type of values used to update the state. - σ is the actual state. @@ -396,8 +396,7 @@ unsafe def registerPersistentEnvExtensionUnsafe {α β σ : Type} [Inhabited σ] @[implementedBy registerPersistentEnvExtensionUnsafe] opaque registerPersistentEnvExtension {α β σ : Type} [Inhabited σ] (descr : PersistentEnvExtensionDescr α β σ) : IO (PersistentEnvExtension α β σ) -/- Simple PersistentEnvExtension that implements exportEntriesFn using a list of entries. -/ - +/-- Simple `PersistentEnvExtension` that implements `exportEntriesFn` using a list of entries. -/ def SimplePersistentEnvExtension (α σ : Type) := PersistentEnvExtension α α (List α × σ) @[specialize] def mkStateFromImportedEntries {α σ : Type} (addEntryFn : σ → α → σ) (initState : σ) (as : Array (Array α)) : σ := @@ -761,7 +760,7 @@ def hasUnsafe (env : Environment) (e : Expr) : Bool := end Environment namespace Kernel -/- Kernel API -/ +/-! # Kernel API -/ /-- Kernel isDefEq predicate. We use it mainly for debugging purposes. diff --git a/src/Lean/Exception.lean b/src/Lean/Exception.lean index bd9839db9c33..a15ef5992cae 100644 --- a/src/Lean/Exception.lean +++ b/src/Lean/Exception.lean @@ -10,7 +10,7 @@ import Lean.Util.MonadCache namespace Lean -/- Exception type used in most Lean monads -/ +/-- Exception type used in most Lean monads -/ inductive Exception where | error (ref : Syntax) (msg : MessageData) | internal (id : InternalExceptionId) (extra : KVMap := {}) @@ -25,7 +25,7 @@ def Exception.getRef : Exception → Syntax instance : Inhabited Exception := ⟨Exception.error default default⟩ -/- Similar to `AddMessageContext`, but for error messages. +/-- Similar to `AddMessageContext`, but for error messages. The default instance just uses `AddMessageContext`. In error messages, we may want to provide additional information (e.g., macro expansion stack), and refine the `(ref : Syntax)`. -/ diff --git a/src/Lean/Expr.lean b/src/Lean/Expr.lean index 7d00d292b32f..82f09a7c326f 100644 --- a/src/Lean/Expr.lean +++ b/src/Lean/Expr.lean @@ -8,22 +8,29 @@ import Lean.Level namespace Lean +/-- Literal values for `Expr`. -/ inductive Literal where - | natVal (val : Nat) - | strVal (val : String) + | /-- Natural number literal -/ + natVal (val : Nat) + | /-- String literal -/ + strVal (val : String) deriving Inhabited, BEq, Repr protected def Literal.hash : Literal → UInt64 - | Literal.natVal v => hash v - | Literal.strVal v => hash v + | .natVal v => hash v + | .strVal v => hash v instance : Hashable Literal := ⟨Literal.hash⟩ +/-- +Total order on `Expr` literal values. +Natural number values are smaller than string literal values. +-/ def Literal.lt : Literal → Literal → Bool - | Literal.natVal _, Literal.strVal _ => true - | Literal.natVal v₁, Literal.natVal v₂ => v₁ < v₂ - | Literal.strVal v₁, Literal.strVal v₂ => v₁ < v₂ - | _, _ => false + | .natVal _, .strVal _ => true + | .natVal v₁, .natVal v₂ => v₁ < v₂ + | .strVal v₁, .strVal v₂ => v₁ < v₂ + | _, _ => false instance : LT Literal := ⟨fun a b => a.lt b⟩ @@ -46,7 +53,7 @@ This can be set to The difference between implicit `{}` and strict-implicit `⦃⦄` is how implicit arguments are treated that are *not* followed by explicit arguments. `{}` arguments are applied eagerly, while `⦃⦄` arguments are left partially applied: -```lean +```lean4 def foo {x : Nat} : Nat := x def bar ⦃x : Nat⦄ : Nat := x #check foo -- foo : Nat @@ -56,32 +63,59 @@ def bar ⦃x : Nat⦄ : Nat := x See also the Lean manual: https://leanprover.github.io/lean4/doc/expressions.html#implicit-arguments -/ inductive BinderInfo where - | default | implicit | strictImplicit | instImplicit | auxDecl + | /-- Default binder annotation, e.g. `(x : α)` -/ + default + | /-- Implicit binder annotation, e.g., `{x : α}` -/ + implicit + | /-- Strict implict binder annotation, e.g., `{{ x : α }}` -/ + strictImplicit + | /-- Local instance binder annotataion, e.g., `[Decidable α]` -/ + instImplicit + | /-- + Auxiliary declarations used by Lean when elaborating recursive declarations. + When defining a function such as + ``` + def f : Nat → Nat + | 0 => 1 + | x+1 => (x+1)*f x + ``` + Lean adds a local declaration `f : Nat → Nat` to the local context (`LocalContext`) + with `BinderInfo` set to `auxDecl`. + This local declaration is later removed by the termination checker. + -/ + auxDecl deriving Inhabited, BEq, Repr def BinderInfo.hash : BinderInfo → UInt64 - | BinderInfo.default => 947 - | BinderInfo.implicit => 1019 - | BinderInfo.strictImplicit => 1087 - | BinderInfo.instImplicit => 1153 - | BinderInfo.auxDecl => 1229 + | .default => 947 + | .implicit => 1019 + | .strictImplicit => 1087 + | .instImplicit => 1153 + | .auxDecl => 1229 +/-- +Return `true` if the given `BinderInfo` does not correspond to an implicit binder annotation +(i.e., `implicit`, `strictImplicit`, or `instImplicit`). +-/ def BinderInfo.isExplicit : BinderInfo → Bool - | BinderInfo.implicit => false - | BinderInfo.strictImplicit => false - | BinderInfo.instImplicit => false - | _ => true + | .implicit => false + | .strictImplicit => false + | .instImplicit => false + | _ => true instance : Hashable BinderInfo := ⟨BinderInfo.hash⟩ +/-- Return `true` if the given `BinderInfo` is an instance implicit annotation (e.g., `[Decidable α]`) -/ def BinderInfo.isInstImplicit : BinderInfo → Bool | BinderInfo.instImplicit => true | _ => false +/-- Return `true` if the given `BinderInfo` is a regular implicit annotation (e.g., `{α : Type u}`) -/ def BinderInfo.isImplicit : BinderInfo → Bool | BinderInfo.implicit => true | _ => false +/-- Return `true` if the given `BinderInfo` is a strict implicit annotation (e.g., `{{α : Type u}}`) -/ def BinderInfo.isStrictImplicit : BinderInfo → Bool | BinderInfo.strictImplicit => true | _ => false @@ -95,16 +129,19 @@ abbrev MData := KVMap abbrev MData.empty : MData := {} /-- - Cached hash code, cached results, and other data for `Expr`. - hash : 32-bits - hasFVar : 1-bit -- does it contain free variables? - hasExprMVar : 1-bit -- does it contain metavariables? - hasLevelMVar : 1-bit -- does it contain level metavariables? - hasLevelParam : 1-bit -- does it contain level parameters? - nonDepLet : 1-bit -- internal flag, for tracking whether let x := v; b is equivalent to (fun x => b) v - binderInfo : 3-bits -- encoding of BinderInfo - approxDepth : 8-bits -- the approximate depth is used to minimize the number of hash collisions - looseBVarRange : 16-bits +Cached hash code, cached results, and other data for `Expr`. +- hash : 32-bits +- hasFVar : 1-bit -- does it contain free variables? +- hasExprMVar : 1-bit -- does it contain metavariables? +- hasLevelMVar : 1-bit -- does it contain level metavariables? +- hasLevelParam : 1-bit -- does it contain level parameters? +- nonDepLet : 1-bit -- internal flag, for tracking whether let x := v; b is equivalent to (fun x => b) v +- binderInfo : 3-bits -- encoding of BinderInfo -- TODO remove +- approxDepth : 8-bits -- the approximate depth is used to minimize the number of hash collisions +- looseBVarRange : 16-bits + +Remark: this is mostly an internal datastructure used to implement `Expr`, +most will never have to use it. -/ def Expr.Data := UInt64 @@ -211,6 +248,14 @@ instance : Repr Expr.Data where open Expr +/-- +The unique free variable identifier. It is just a hierarchical name, +but we wrap it in `FVarId` to make sure they don't get mixed up with `MVarId`. + +This is not the user-facing name for a free variable. This information is stored +in the local context (`LocalContext`). The unique identifiers are generated using +a `NameGenerator`. +-/ structure FVarId where name : Name deriving Inhabited, BEq, Hashable @@ -218,14 +263,24 @@ structure FVarId where instance : Repr FVarId where reprPrec n p := reprPrec n.name p +/-- +A set of unique free variable identifiers. +This is a persistent data structure implemented using red-black trees. -/ def FVarIdSet := Std.RBTree FVarId (Name.quickCmp ·.name ·.name) deriving Inhabited, EmptyCollection instance : ForIn m FVarIdSet FVarId := inferInstanceAs (ForIn _ (Std.RBTree ..) ..) +/-- +A set of unique free variable identifiers implemented using hashtables. +Hashtables are faster than red-black trees if they are used linearly. +They are not persistent data-structures. -/ def FVarIdHashSet := Std.HashSet FVarId deriving Inhabited, EmptyCollection +/-- +A mapping from free variable identifiers to values of type `α`. +This is a persistent data structure implemented using red-black trees. -/ def FVarIdMap (α : Type) := Std.RBMap FVarId α (Name.quickCmp ·.name ·.name) instance : EmptyCollection (FVarIdMap α) := inferInstanceAs (EmptyCollection (Std.RBMap ..)) @@ -233,21 +288,137 @@ instance : EmptyCollection (FVarIdMap α) := inferInstanceAs (EmptyCollection (S instance : Inhabited (FVarIdMap α) where default := {} -/- We use the `E` suffix (short for `Expr`) to avoid collision with keywords. - We considered using «...», but it is too inconvenient to use. -/ +/-- +Lean expressions. This datastructure is used in the kernel and +elaborator. Howewer, expressions sent to the kernel should not +contain metavariables. + +Remark: we use the `E` suffix (short for `Expr`) to avoid collision with keywords. +We considered using «...», but it is too inconvenient to use. -/ inductive Expr where - | bvar : Nat → Expr -- bound variables - | fvar : FVarId → Expr -- free variables - | mvar : MVarId → Expr -- meta variables - | sort : Level → Expr -- Sort - | const : Name → List Level → Expr -- constants - | app : Expr → Expr → Expr -- application - | lam : Name → Expr → Expr → BinderInfo → Expr -- lambda abstraction - | forallE : Name → Expr → Expr → BinderInfo → Expr -- (dependent) arrow - | letE : Name → Expr → Expr → Expr → Bool → Expr -- let expressions - | lit : Literal → Expr -- literals - | mdata : MData → Expr → Expr -- metadata - | proj : Name → Nat → Expr → Expr -- projection + | /-- + Bound variables. The natural number is the "de Bruijn" index + for the bound variable. See https://en.wikipedia.org/wiki/De_Bruijn_index for additional information. + Example, the expression `fun x : Nat => forall y : Nat, x = y` + ```lean + .lam `x (.const `Nat []) + (.forall `y (.const `Nat []) + (.app (.app (.app (.const `Eq [.succ .zero]) + (.const `Nat [])) (.bvar 1)) + (.bvar 0)) + .default) + .default + ``` + -/ + bvar (deBruijnIndex : Nat) + | /-- + Free variable. Lean uses the locally nameless approach. + See https://citeseerx.ist.psu.edu/viewdoc/download?doi=10.1.1.365.2479&rep=rep1&type=pdf for additional details. + When "visiting" the body of a binding expression (`lam`, `forallE`, or `letE`), bound variables + are converted into free variables using a unique identifier, and their user-facing name, type, + value (for `LetE`), and binder annotation are stored in the `LocalContext`. + -/ + fvar (fvarId : FVarId) + | /-- + Metavariables are used to represent "holes" in expressions, and goals in the + tactic framework. Metavariable declarations are stored in the `MetavarContext`. + Metavariables are used during elaboration, and are not allowed in the kernel, + or in the code generator. + -/ + mvar (mvarId : MVarId) + | /-- + `Type u`, `Sort u`, `Prop`. - + - `Prop` is represented as `.sort .zero`, + - `Sort u` as ``.sort (.param `u)``, and + - `Type u` as ``.sort (.succ (.param `u))`` + -/ + sort (u : Level) + | /-- + A (universe polymorphic) constant. For example, + `@Eq.{1}` is represented as ``.const `Eq [.succ .zero]``, and + `@Array.map.{0, 0}` is represented as ``.cons `Array.map [.zero, .zero]``. + -/ + const (declName : Name) (us : List Level) + | /-- + Function application. `Nat.succ Nat.zero` is represented as + ```lean4 + .app (.const `Nat.succ []) (.const .zero []) + ``` + -/ + app (fn : Expr) (arg : Expr) + | /-- + Lambda abstraction (aka anonymous functions). + - `fun x : Nat => x` is represented as + ```lean4 + .lam `x (.const `Nat []) (.bvar 0) .default + ``` + -/ + lam (binderName : Name) (binderType : Expr) (body : Expr) (binderInfo : BinderInfo) + | /-- + A dependent arrow (aka forall-expression). It is also used to represent non-dependent arrows. + Examples: + + - `forall x : Prop, x ∧ x` is represented as + ```lean4 + .forallE `x + (.sort .zero) + (.app (.app (.const `And []) (.bvar 0)) (.bvar 0)) + .default + ``` + - `Nat → Bool` as + ```lean4 + .forallE `a (.const `Nat []) (.const `Bool []) .default + ``` + -/ + forallE (binderName : Name) (binderType : Expr) (body : Expr) (binderInfo : BinderInfo) + | /-- + Let-expressions. The field `nonDep` is not currently used, but will be used in the future + by the code generator (and possibly `simp`) to track whether a let-expression is non-dependent + or not. Given an environment, metavariable context, and local context, we say a let-expression + `let x : t := v; e` is non-dependent when it is equivalent to `(fun x : t => e) v`. + Here is an example of a dependent let-expression + `let n : Nat := 2; fun (a : Array Nat n) (b : Array Nat 2) => a = b` is type correct, but + `(fun (n : Nat) (a : Array Nat n) (b : Array Nat 2) => a = b) 2` is not. + The let-expression `let x : Nat := 2; Nat.succ x` is represented as + ``` + .letE `x (.const `Nat []) (.lit (.natVal 2)) (.bvar 0) true + ``` + -/ + letE (declName : Name) (type : Expr) (value : Expr) (body : Expr) (nonDep : Bool) + | /-- + Natural number and string literal values. They are not really needed, but provide a more + compact representation in memory for these two kinds of literals, and are used to implement + efficient reduction in the elaborator and kernel. + The "raw" natural number `2` can be represented as `.lit (.natVal 2)`. Note that, it is + definitionally equal to + ```lean4 + .app (.const `Nat.succ []) (.app (.const `Nat.succ []) (.const `Nat.zero [])) + ``` + -/ + lit : Literal → Expr + | /-- + Metadata (aka annotations). We use annotations to provide hints to the pretty-printer, + store references to `Syntax` nodes, position information, and save information for + elaboration procedures (e.g., we use the `inaccessible` annotation during elaboration to + mark `Expr`s that correspond to inaccessible patterns). + Note that `.mdata data e` is definitionally equal to `e`. + -/ + mdata (data : MData) (expr : Expr) + | /-- + Projection-expressions. They are redundant, but are used to create more compact + terms, speedup reduction, and implement eta for structures. + The type of `struct` must be an structure-like inductive type. That is, it has only one + constructor, is not recursive, and it is not an inductive predicate. The kernel and elaborators + check whether the `typeName` matches the type of `struct`, and whether the (zero-based) index + is valid (i.e., it is smaller than the numbef of constructor fields). + When exporting Lean developments to other systems, `proj` can be replaced with `typeName`.`rec` + applications. + Example, given `a : Nat x Bool`, `a.1` is represented as + ```lean4 + .proj `Prod 0 a + ``` + -/ + proj (typeName : Name) (idx : Nat) (struct : Expr) with @[computedField, extern c inline "lean_ctor_get_uint64(#1, lean_ctor_num_objs(#1)*sizeof(void*))"] data : @& Expr → Data @@ -299,6 +470,7 @@ deriving Inhabited, Repr namespace Expr +/-- The constructor name for the given expression. This is used for debugging purposes. -/ def ctorName : Expr → String | bvar .. => "bvar" | fvar .. => "fvar" @@ -318,27 +490,52 @@ protected def hash (e : Expr) : UInt64 := instance : Hashable Expr := ⟨Expr.hash⟩ +/-- +Return `true` if `e` contains free variables. +This is a constant time operation. +-/ def hasFVar (e : Expr) : Bool := e.data.hasFVar +/-- +Return `true` if `e` contains expression metavariables. +This is a constant time operation. +-/ def hasExprMVar (e : Expr) : Bool := e.data.hasExprMVar +/-- +Return `true` if `e` contains universe (aka `Level`) metavariables. +This is a constant time operation. +-/ def hasLevelMVar (e : Expr) : Bool := e.data.hasLevelMVar -/-- Does the expression contain level or expression metavariables?-/ +/-- +Does the expression contain level (aka universe) or expression metavariables? +This is a constant time operation. +-/ def hasMVar (e : Expr) : Bool := let d := e.data d.hasExprMVar || d.hasLevelMVar +/-- +Return true if `e` contains universe level parameters. +This is a constant time operation. +-/ def hasLevelParam (e : Expr) : Bool := e.data.hasLevelParam +/-- +Return the approximated depth of an expression. This information is used to compute +the expression hash code, and speedup comparisons. +This is a constant time operation. We say it is approximate because it maxes out at `255`. +-/ def approxDepth (e : Expr) : UInt32 := e.data.approxDepth.toUInt32 -/-- The range of de-Bruijn variables that are loose. +/-- +The range of de-Bruijn variables that are loose. That is, bvars that are not bound by a binder. For example, `bvar i` has range `i + 1` and an expression with no loose bvars has range `0`. @@ -346,9 +543,15 @@ an expression with no loose bvars has range `0`. def looseBVarRange (e : Expr) : Nat := e.data.looseBVarRange.toNat +/-- +Return the binder information if `e` is a lambda or forall expression, and `.default` otherwise. +-/ def binderInfo (e : Expr) : BinderInfo := e.data.binderInfo +/-! +Export functions. +-/ @[export lean_expr_hash] def hashEx : Expr → UInt64 := hash @[export lean_expr_has_fvar] def hasFVarEx : Expr → Bool := hasFVar @[export lean_expr_has_expr_mvar] def hasExprMVarEx : Expr → Bool := hasExprMVar @@ -360,53 +563,85 @@ def binderInfo (e : Expr) : BinderInfo := end Expr -def mkConst (n : Name) (lvls : List Level := []) : Expr := - Expr.const n lvls +/-- `mkConst declName us` return `.const declName us`. -/ +def mkConst (declName : Name) (us : List Level := []) : Expr := + .const declName us +/-- Return the type of a literal value. -/ def Literal.type : Literal → Expr - | Literal.natVal _ => mkConst `Nat - | Literal.strVal _ => mkConst `String + | .natVal _ => mkConst `Nat + | .strVal _ => mkConst `String @[export lean_lit_type] def Literal.typeEx : Literal → Expr := Literal.type +/-- `.bvar idx` is now the preferred form. -/ def mkBVar (idx : Nat) : Expr := - Expr.bvar idx + .bvar idx -def mkSort (lvl : Level) : Expr := - Expr.sort lvl +/-- `.sort u` is now the preferred form. -/ +def mkSort (u : Level) : Expr := + .sort u +/-- +`.fvar fvarId` is now the preferred form. +This function is seldom used, free variables are often automatically created using the +telescope functions (e.g., `forallTelescope` and `lambdaTelescope`) at `MetaM`. +-/ def mkFVar (fvarId : FVarId) : Expr := - Expr.fvar fvarId + .fvar fvarId -def mkMVar (fvarId : MVarId) : Expr := - Expr.mvar fvarId +/-- +`.mvar mvarId` is now the preferred form. +This function is seldom used, metavariables are often created using functions such +as `mkFresheExprMVar` at `MetaM`. +-/ +def mkMVar (mvarId : MVarId) : Expr := + .mvar mvarId +/-- +`.mdata m e` is now the preferred form. +-/ def mkMData (m : MData) (e : Expr) : Expr := - Expr.mdata m e + .mdata m e -def mkProj (s : Name) (i : Nat) (e : Expr) : Expr := - Expr.proj s i e +/-- +`.proj structName idx struct` is now the preferred form. +-/ +def mkProj (structName : Name) (idx : Nat) (struct : Expr) : Expr := + .proj structName idx struct +/-- +`.app f a` is now the preferred form. +-/ def mkApp (f a : Expr) : Expr := - Expr.app f a + .app f a +/-- +`.lam x t b bi` is now the preferred form. +-/ def mkLambda (x : Name) (bi : BinderInfo) (t : Expr) (b : Expr) : Expr := - Expr.lam x t b bi + .lam x t b bi +/-- +`.forallE x t b bi` is now the preferred form. +-/ def mkForall (x : Name) (bi : BinderInfo) (t : Expr) (b : Expr) : Expr := - Expr.forallE x t b bi + .forallE x t b bi /-- Return `Unit -> type`. Do not confuse with `Thunk type` -/ def mkSimpleThunkType (type : Expr) : Expr := - mkForall Name.anonymous BinderInfo.default (Lean.mkConst `Unit) type + mkForall Name.anonymous .default (mkConst `Unit) type /-- Return `fun (_ : Unit), e` -/ def mkSimpleThunk (type : Expr) : Expr := - mkLambda `_ BinderInfo.default (Lean.mkConst `Unit) type + mkLambda `_ BinderInfo.default (mkConst `Unit) type +/-- +`.letE x t v b nonDep` is now the preferred form. +-/ def mkLet (x : Name) (t : Expr) (v : Expr) (b : Expr) (nonDep : Bool := false) : Expr := - Expr.letE x t v b nonDep + .letE x t v b nonDep def mkAppB (f a b : Expr) := mkApp (mkApp f a) b def mkApp2 (f a b : Expr) := mkAppB f a b @@ -419,18 +654,32 @@ def mkApp8 (f a b c d e₁ e₂ e₃ e₄ : Expr) := mkApp4 (mkApp4 f a b c d) e def mkApp9 (f a b c d e₁ e₂ e₃ e₄ e₅ : Expr) := mkApp5 (mkApp4 f a b c d) e₁ e₂ e₃ e₄ e₅ def mkApp10 (f a b c d e₁ e₂ e₃ e₄ e₅ e₆ : Expr) := mkApp6 (mkApp4 f a b c d) e₁ e₂ e₃ e₄ e₅ e₆ +/-- +`.lit l` is now the preferred form. +-/ def mkLit (l : Literal) : Expr := - Expr.lit l + .lit l +/-- +Return the "raw" natural number `.lit (.natVal n)`. +This is not the default representation used by the Lean frontend. +See `mkNatLit`. +-/ def mkRawNatLit (n : Nat) : Expr := - mkLit (Literal.natVal n) + mkLit (.natVal n) +/-- +Return a natural number literal used in the frontend. It is a `OfNat.ofNat` application. +Recall that all theorems and definitions containing numeric literals are encoded using +`OfNat.ofNat` applications in the frontend. +-/ def mkNatLit (n : Nat) : Expr := let r := mkRawNatLit n mkApp3 (mkConst ``OfNat.ofNat [levelZero]) (mkConst ``Nat) r (mkApp (mkConst ``instOfNatNat) r) +/-- Return the string literal `.lit (.strVal s)` -/ def mkStrLit (s : String) : Expr := - mkLit (Literal.strVal s) + mkLit (.strVal s) @[export lean_expr_mk_bvar] def mkBVarEx : Nat → Expr := mkBVar @[export lean_expr_mk_fvar] def mkFVarEx : FVarId → Expr := mkFVar @@ -465,105 +714,136 @@ namespace Expr @[extern "lean_expr_dbg_to_string"] opaque dbgToString (e : @& Expr) : String +/-- A total order for expressions. We say it is quick because it first compares the hashcodes. -/ @[extern "lean_expr_quick_lt"] opaque quickLt (a : @& Expr) (b : @& Expr) : Bool +/-- A total order for expressions that takes the structure into account (e.g., variable names). -/ @[extern "lean_expr_lt"] opaque lt (a : @& Expr) (b : @& Expr) : Bool -/-- Return true iff `a` and `b` are alpha equivalent. - Binder annotations are ignored. -/ +/-- +Return true iff `a` and `b` are alpha equivalent. +Binder annotations are ignored. +-/ @[extern "lean_expr_eqv"] opaque eqv (a : @& Expr) (b : @& Expr) : Bool instance : BEq Expr where beq := Expr.eqv -protected unsafe def ptrEq (a b : Expr) : Bool := - ptrAddrUnsafe a == ptrAddrUnsafe b - -/- Return true iff `a` and `b` are equal. - Binder names and annotations are taking into account. -/ +/-- +Return true iff `a` and `b` are equal. +Binder names and annotations are taking into account. +-/ @[extern "lean_expr_equal"] opaque equal (a : @& Expr) (b : @& Expr) : Bool +/-- Return `true` if the given expression is a `.sort ..` -/ def isSort : Expr → Bool | sort .. => true | _ => false +/-- Return `true` if the given expression is of the form `.sort (.succ ..)`. -/ def isType : Expr → Bool - | sort (Level.succ ..) => true + | sort (.succ ..) => true | _ => false +/-- Return `true` if the given expression is a `.sort .zero` -/ def isProp : Expr → Bool - | sort (Level.zero ..) => true + | sort (.zero ..) => true | _ => false +/-- Return `true` if the given expression is a bound variable. -/ def isBVar : Expr → Bool | bvar .. => true | _ => false +/-- Return `true` if the given expression is a metavariable. -/ def isMVar : Expr → Bool | mvar .. => true | _ => false +/-- Return `true` if the given expression is a free variable. -/ def isFVar : Expr → Bool | fvar .. => true | _ => false +/-- Return `true` if the given expression is an application. -/ def isApp : Expr → Bool | app .. => true | _ => false +/-- Return `true` if the given expression is a projection `.proj ..` -/ def isProj : Expr → Bool | proj .. => true | _ => false +/-- Return `true` if the given expression is a constant. -/ def isConst : Expr → Bool | const .. => true | _ => false +/-- +Return `true` if the given expression is a constant of the give name. +Examples: +- `` (.const `Nat []).isConstOf `Nat `` is `true` +- `` (.const `Nat []).isConstOf `False `` is `false` +-/ def isConstOf : Expr → Name → Bool | const n .., m => n == m | _, _ => false +/-- Return `true` if the given expression is a forall-expression aka (dependent) arrow. -/ def isForall : Expr → Bool | forallE .. => true | _ => false +/-- Return `true` if the given expression is a lambda abstraction aka anonymous function. -/ def isLambda : Expr → Bool | lam .. => true | _ => false +/-- Return `true` if the given expression is a forall or lambda expression. -/ def isBinding : Expr → Bool | lam .. => true | forallE .. => true | _ => false +/-- Return `true` if the given expression is a let-expression. -/ def isLet : Expr → Bool | letE .. => true | _ => false +/-- Return `true` if the given expression is a metadata. -/ def isMData : Expr → Bool | mdata .. => true | _ => false +/-- Return `true` if the given expression is a literal value. -/ def isLit : Expr → Bool | lit .. => true | _ => false +/-- +Return the "body" of a forall expression. +Example: let `e` be the representation for `forall (p : Prop) (q : Prop), p ∧ q`, then +`getForallBody e` returns ``.app (.app (.const `And []) (.bvar 1)) (.bvar 0)`` +-/ def getForallBody : Expr → Expr | forallE _ _ b .. => getForallBody b | e => e -/-- If the given expression is a sequence of +/-- +If the given expression is a sequence of function applications `f a₁ .. aₙ`, return `f`. -Otherwise return the input expression. -/ +Otherwise return the input expression. +-/ def getAppFn : Expr → Expr | app f _ => getAppFn f | e => e -def getAppNumArgsAux : Expr → Nat → Nat +private def getAppNumArgsAux : Expr → Nat → Nat | app f _, n => getAppNumArgsAux f (n+1) | _, n => n @@ -637,8 +917,10 @@ def isAppOf (e : Expr) (n : Name) : Bool := | const c _ => c == n | _ => false -/-- Given `f a₁ ... aᵢ`, returns true if `f` is a constant -with name `n` and has the correct number of arguments. -/ +/-- +Given `f a₁ ... aᵢ`, returns true if `f` is a constant +with name `n` and has the correct number of arguments. +-/ def isAppOfArity : Expr → Name → Nat → Bool | const c _, n, 0 => c == n | app f _, n, a+1 => isAppOfArity f n a @@ -771,7 +1053,10 @@ def projIdx! : Expr → Nat def hasLooseBVars (e : Expr) : Bool := e.looseBVarRange > 0 -/- Remark: the following function assumes `e` does not have loose bound variables. -/ +/-- +Return `true` if `e` is a non-dependent arrow. +Remark: the following function assumes `e` does not have loose bound variables. +-/ def isArrow (e : Expr) : Bool := match e with | forallE _ _ b _ => !b.hasLooseBVars @@ -787,11 +1072,12 @@ def hasLooseBVarInExplicitDomain : Expr → Nat → Bool → Bool | e, bvarIdx, tryRange => tryRange && hasLooseBVar e bvarIdx /-- - Lower the loose bound variables `>= s` in `e` by `d`. - That is, a loose bound variable `bvar i`. - `i >= s` is mapped into `bvar (i-d)`. +Lower the loose bound variables `>= s` in `e` by `d`. +That is, a loose bound variable `bvar i`. +`i >= s` is mapped into `bvar (i-d)`. - Remark: if `s < d`, then result is `e` -/ +Remark: if `s < d`, then result is `e` +-/ @[extern "lean_expr_lower_loose_bvars"] opaque lowerLooseBVars (e : @& Expr) (s d : @& Nat) : Expr @@ -801,12 +1087,12 @@ opaque lowerLooseBVars (e : @& Expr) (s d : @& Nat) : Expr opaque liftLooseBVars (e : @& Expr) (s d : @& Nat) : Expr /-- - `inferImplicit e numParams considerRange` updates the first `numParams` parameter binder annotations of the `e` forall type. - It marks any parameter with an explicit binder annotation if there is another explicit arguments that depends on it or - the resulting type if `considerRange == true`. +`inferImplicit e numParams considerRange` updates the first `numParams` parameter binder annotations of the `e` forall type. +It marks any parameter with an explicit binder annotation if there is another explicit arguments that depends on it or +the resulting type if `considerRange == true`. - Remark: we use this function to infer the bind annotations of inductive datatype constructors, and structure projections. - When the `{}` annotation is used in these commands, we set `considerRange == false`. +Remark: we use this function to infer the bind annotations of inductive datatype constructors, and structure projections. +When the `{}` annotation is used in these commands, we set `considerRange == false`. -/ def inferImplicit : Expr → Nat → Bool → Expr | Expr.forallE n d b bi, i+1, considerRange => @@ -816,8 +1102,10 @@ def inferImplicit : Expr → Nat → Bool → Expr | e, 0, _ => e | e, _, _ => e -/-- Instantiate the loose bound variables in `e` using `subst`. - That is, a loose `Expr.bvar i` is replaced with `subst[i]`. -/ +/-- +Instantiate the loose bound variables in `e` using `subst`. +That is, a loose `Expr.bvar i` is replaced with `subst[i]`. +-/ @[extern "lean_expr_instantiate"] opaque instantiate (e : @& Expr) (subst : @& Array Expr) : Expr @@ -828,13 +1116,17 @@ opaque instantiate1 (e : @& Expr) (subst : @& Expr) : Expr @[extern "lean_expr_instantiate_rev"] opaque instantiateRev (e : @& Expr) (subst : @& Array Expr) : Expr -/-- Similar to `instantiate`, but consider only the variables `xs` in the range `[beginIdx, endIdx)`. - Function panics if `beginIdx <= endIdx <= xs.size` does not hold. -/ +/-- +Similar to `instantiate`, but consider only the variables `xs` in the range `[beginIdx, endIdx)`. +Function panics if `beginIdx <= endIdx <= xs.size` does not hold. +-/ @[extern "lean_expr_instantiate_range"] opaque instantiateRange (e : @& Expr) (beginIdx endIdx : @& Nat) (xs : @& Array Expr) : Expr -/-- Similar to `instantiateRev`, but consider only the variables `xs` in the range `[beginIdx, endIdx)`. - Function panics if `beginIdx <= endIdx <= xs.size` does not hold. -/ +/-- +Similar to `instantiateRev`, but consider only the variables `xs` in the range `[beginIdx, endIdx)`. +Function panics if `beginIdx <= endIdx <= xs.size` does not hold. +-/ @[extern "lean_expr_instantiate_rev_range"] opaque instantiateRevRange (e : @& Expr) (beginIdx endIdx : @& Nat) (xs : @& Array Expr) : Expr @@ -887,7 +1179,7 @@ abbrev ExprSet := HashSet Expr abbrev PersistentExprSet := PHashSet Expr abbrev PExprSet := PersistentExprSet -/- Auxiliary type for forcing `==` to be structural equality for `Expr` -/ +/-- Auxiliary type for forcing `==` to be structural equality for `Expr` -/ structure ExprStructEq where val : Expr deriving Inhabited @@ -924,19 +1216,19 @@ def mkAppRevRange (f : Expr) (beginIdx endIdx : Nat) (revArgs : Array Expr) : Ex mkAppRevRangeAux revArgs beginIdx f endIdx /-- - If `f` is a lambda expression, than "beta-reduce" it using `revArgs`. - This function is often used with `getAppRev` or `withAppRev`. - Examples: - - `betaRev (fun x y => t x y) #[]` ==> `fun x y => t x y` - - `betaRev (fun x y => t x y) #[a]` ==> `fun y => t a y` - - `betaRev (fun x y => t x y) #[a, b]` ==> `t b a` - - `betaRev (fun x y => t x y) #[a, b, c, d]` ==> `t d c b a` - Suppose `t` is `(fun x y => t x y) a b c d`, then - `args := t.getAppRev` is `#[d, c, b, a]`, - and `betaRev (fun x y => t x y) #[d, c, b, a]` is `t a b c d`. - - If `useZeta` is true, the function also performs zeta-reduction (reduction of let binders) to create further - opportunities for beta reduction. +If `f` is a lambda expression, than "beta-reduce" it using `revArgs`. +This function is often used with `getAppRev` or `withAppRev`. +Examples: +- `betaRev (fun x y => t x y) #[]` ==> `fun x y => t x y` +- `betaRev (fun x y => t x y) #[a]` ==> `fun y => t a y` +- `betaRev (fun x y => t x y) #[a, b]` ==> `t b a` +- `betaRev (fun x y => t x y) #[a, b, c, d]` ==> `t d c b a` +Suppose `t` is `(fun x y => t x y) a b c d`, then +`args := t.getAppRev` is `#[d, c, b, a]`, +and `betaRev (fun x y => t x y) #[d, c, b, a]` is `t a b c d`. + +If `useZeta` is true, the function also performs zeta-reduction (reduction of let binders) to create further +opportunities for beta reduction. -/ partial def betaRev (f : Expr) (revArgs : Array Expr) (useZeta := false) (preserveMData := false) : Expr := if revArgs.size == 0 then f @@ -967,11 +1259,20 @@ partial def betaRev (f : Expr) (revArgs : Array Expr) (useZeta := false) (preser mkAppRevRange (b.instantiateRange n sz revArgs) 0 n revArgs go f 0 -/-- Apply the given arguments to `f`, beta-reducing if `f` is a -lambda expression. See docstring for `betaRev` for examples. -/ +/-- +Apply the given arguments to `f`, beta-reducing if `f` is a +lambda expression. See docstring for `betaRev` for examples. +-/ def beta (f : Expr) (args : Array Expr) : Expr := betaRev f args.reverse +/-- +Return true if the given expression is the function of an expression that is target for (head) beta reduction. +If `useZeta = true`, then `let`-expressions are visited. That is, it assumes +that zeta-reduction (aka let-expansion) is going to be used. + +See `isHeadBetaTarget`. +-/ def isHeadBetaTargetFn (useZeta : Bool) : Expr → Bool | Expr.lam .. => true | Expr.letE _ _ _ b _ => useZeta && isHeadBetaTargetFn useZeta b @@ -983,6 +1284,11 @@ def headBeta (e : Expr) : Expr := let f := e.getAppFn if f.isHeadBetaTargetFn false then betaRev f e.getAppRevArgs else e +/-- +Return true if the given expression is a target for (head) beta reduction. +If `useZeta = true`, then `let`-expressions are visited. That is, it assumes +that zeta-reduction (aka let-expansion) is going to be used. +-/ def isHeadBetaTarget (e : Expr) (useZeta := false) : Bool := e.getAppFn.isHeadBetaTargetFn useZeta @@ -996,12 +1302,13 @@ private def etaExpandedAux : Expr → Nat → Option Expr | e, n => etaExpandedBody e n 0 /-- - If `e` is of the form `(fun x₁ ... xₙ => f x₁ ... xₙ)` and `f` does not contain `x₁`, ..., `xₙ`, - then return `some f`. Otherwise, return `none`. +If `e` is of the form `(fun x₁ ... xₙ => f x₁ ... xₙ)` and `f` does not contain `x₁`, ..., `xₙ`, +then return `some f`. Otherwise, return `none`. - It assumes `e` does not have loose bound variables. +It assumes `e` does not have loose bound variables. - Remark: `ₙ` may be 0 -/ +Remark: `ₙ` may be 0 +-/ def etaExpanded? (e : Expr) : Option Expr := etaExpandedAux e 0 @@ -1010,28 +1317,40 @@ def etaExpandedStrict? : Expr → Option Expr | lam _ _ b _ => etaExpandedAux b 1 | _ => none +/-- Return `some e'` if `e` is of the form `optParam _ e'` -/ def getOptParamDefault? (e : Expr) : Option Expr := if e.isAppOfArity ``optParam 2 then some e.appArg! else none +/-- Return `some e'` if `e` is of the form `autoParam _ e'` -/ def getAutoParamTactic? (e : Expr) : Option Expr := if e.isAppOfArity ``autoParam 2 then some e.appArg! else none +/-- Return `true` if `e` is of the form `outParam _` -/ @[export lean_is_out_param] def isOutParam (e : Expr) : Bool := e.isAppOfArity ``outParam 1 +/-- Return `true` if `e` is of the form `optParam _ _` -/ def isOptParam (e : Expr) : Bool := e.isAppOfArity ``optParam 2 +/-- Return `true` if `e` is of the form `autoParam _ _` -/ def isAutoParam (e : Expr) : Bool := e.isAppOfArity ``autoParam 2 +/-- +Remove `outParam`, `optParam`, and `autoParam` applications/annotations from `e`. +Note that it does not remove nested annotations. +Examples: +- Given `e` of the form `outParam (optParam Nat b)`, `consumeTypeAnnotations e = b`. +- Given `e` of the form `Nat → outParam (optParam Nat b)`, `consumeTypeAnnotations e = e`. +-/ @[export lean_expr_consume_type_annotations] partial def consumeTypeAnnotations (e : Expr) : Expr := if e.isOptParam || e.isAutoParam then @@ -1041,9 +1360,16 @@ partial def consumeTypeAnnotations (e : Expr) : Expr := else e -partial def consumeMDataAndTypeAnnotations (e : Expr) : Expr := +/-- +Remove metadata annotations and `outParam`, `optParam`, and `autoParam` applications/annotations from `e`. +Note that it does not remove nested annotations. +Examples: +- Given `e` of the form `outParam (optParam Nat b)`, `cleanupAnnotations e = b`. +- Given `e` of the form `Nat → outParam (optParam Nat b)`, `cleanupAnnotations e = e`. +-/ +partial def cleanupAnnotations (e : Expr) : Expr := let e' := e.consumeMData.consumeTypeAnnotations - if e' == e then e else consumeMDataAndTypeAnnotations e' + if e' == e then e else cleanupAnnotations e' /-- Return true iff `e` contains a free variable which statisfies `p`. -/ @[inline] def hasAnyFVar (e : Expr) (p : FVarId → Bool) : Bool := @@ -1059,108 +1385,133 @@ partial def consumeMDataAndTypeAnnotations (e : Expr) : Expr := | _ => false visit e +/-- Return `true` if `e` contains the given free variable. -/ def containsFVar (e : Expr) (fvarId : FVarId) : Bool := e.hasAnyFVar (· == fvarId) -/- The update functions here are defined using C code. They will try to avoid - allocating new values using pointer equality. - The hypotheses `(h : e.is...)` are used to ensure Lean will not crash - at runtime. - The `update*!` functions are inlined and provide a convenient way of using the - update proofs without providing proofs. - Note that if they are used under a match-expression, the compiler will eliminate - the double-match. -/ - -@[extern "lean_expr_update_app"] -def updateApp (e : Expr) (newFn : Expr) (newArg : Expr) (h : e.isApp) : Expr := - mkApp newFn newArg - -@[inline] def updateApp! (e : Expr) (newFn : Expr) (newArg : Expr) : Expr := - match h : e with - | app .. => updateApp e newFn newArg (h ▸ rfl) - | _ => panic! "application expected" - -@[extern "lean_expr_update_const"] -def updateConst (e : Expr) (newLevels : List Level) (h : e.isConst) : Expr := - mkConst e.constName! newLevels - -@[inline] def updateConst! (e : Expr) (newLevels : List Level) : Expr := - match h : e with - | const .. => updateConst e newLevels (h ▸ rfl) - | _ => panic! "constant expected" - -@[extern "lean_expr_update_sort"] -def updateSort (e : Expr) (newLevel : Level) (h : e.isSort) : Expr := - mkSort newLevel - -@[inline] def updateSort! (e : Expr) (newLevel : Level) : Expr := - match h : e with - | sort .. => updateSort e newLevel (h ▸ rfl) - | _ => panic! "level expected" - -@[extern "lean_expr_update_proj"] -def updateProj (e : Expr) (newExpr : Expr) (h : e.isProj) : Expr := +/-! +The update functions try to avoid allocating new values using pointer equality. +Note that if the `update*!` functions are used under a match-expression, +the compiler will eliminate the double-match. +-/ + +@[inline] private unsafe def updateApp!Impl (e : Expr) (newFn : Expr) (newArg : Expr) : Expr := + match e with + | app fn arg => if ptrEq fn newFn && ptrEq arg newArg then e else mkApp newFn newArg + | _ => panic! "application expected" + +@[implementedBy updateApp!Impl] +def updateApp! (e : Expr) (newFn : Expr) (newArg : Expr) : Expr := match e with - | proj s i .. => mkProj s i newExpr - | _ => e -- unreachable because of `h` + | app _ _ => mkApp newFn newArg + | _ => panic! "application expected" -@[extern "lean_expr_update_mdata"] -def updateMData (e : Expr) (newExpr : Expr) (h : e.isMData) : Expr := +@[inline] private unsafe def updateConst!Impl (e : Expr) (newLevels : List Level) : Expr := match e with - | mdata d .. => mkMData d newExpr - | _ => e -- unreachable because of `h` + | const n ls => if ptrEqList ls newLevels then e else mkConst n newLevels + | _ => panic! "constant expected" -@[inline] def updateMData! (e : Expr) (newExpr : Expr) : Expr := - match h : e with - | mdata .. => updateMData e newExpr (h ▸ rfl) - | _ => panic! "mdata expected" +@[implementedBy updateConst!Impl] +def updateConst! (e : Expr) (newLevels : List Level) : Expr := + match e with + | const n _ => mkConst n newLevels + | _ => panic! "constant expected" -@[inline] def updateProj! (e : Expr) (newExpr : Expr) : Expr := - match h : e with - | proj .. => updateProj e newExpr (h ▸ rfl) - | _ => panic! "proj expected" +@[inline] private unsafe def updateSort!Impl (e : Expr) (u' : Level) : Expr := + match e with + | sort u => if ptrEq u u' then e else mkSort u' + | _ => panic! "level expected" -@[extern "lean_expr_update_forall"] -def updateForall (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) (h : e.isForall) : Expr := - mkForall e.bindingName! newBinfo newDomain newBody +@[implementedBy updateSort!Impl] +def updateSort! (e : Expr) (newLevel : Level) : Expr := + match e with + | sort _ => mkSort newLevel + | _ => panic! "level expected" -@[inline] def updateForall! (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := - match h : e with - | forallE .. => updateForall e newBinfo newDomain newBody (h ▸ rfl) - | _ => panic! "forall expected" +@[inline] private unsafe def updateMData!Impl (e : Expr) (newExpr : Expr) : Expr := + match e with + | mdata d a => if ptrEq a newExpr then e else mkMData d newExpr + | _ => panic! "mdata expected" -@[inline] def updateForallE! (e : Expr) (newDomain : Expr) (newBody : Expr) : Expr := - match h : e with - | forallE _ _ _ c => updateForall e c newDomain newBody (h ▸ rfl) +@[implementedBy updateMData!Impl] +def updateMData! (e : Expr) (newExpr : Expr) : Expr := + match e with + | mdata d _ => mkMData d newExpr + | _ => panic! "mdata expected" + +@[inline] private unsafe def updateProj!Impl (e : Expr) (newExpr : Expr) : Expr := + match e with + | proj s i a => if ptrEq a newExpr then e else mkProj s i newExpr + | _ => panic! "proj expected" + +@[implementedBy updateProj!Impl] +def updateProj! (e : Expr) (newExpr : Expr) : Expr := + match e with + | proj s i _ => mkProj s i newExpr + | _ => panic! "proj expected" + +@[inline] private unsafe def updateForall!Impl (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | forallE n d b bi => + if ptrEq d newDomain && ptrEq b newBody && bi == newBinfo then + e + else + mkForall n newBinfo newDomain newBody | _ => panic! "forall expected" -@[extern "lean_expr_update_lambda"] -def updateLambda (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) (h : e.isLambda) : Expr := - mkLambda e.bindingName! newBinfo newDomain newBody +@[implementedBy updateForall!Impl] +def updateForall! (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | forallE n _ _ _ => mkForall n newBinfo newDomain newBody + | _ => panic! "forall expected" -@[inline] def updateLambda! (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := - match h : e with - | lam .. => updateLambda e newBinfo newDomain newBody (h ▸ rfl) - | _ => panic! "lambda expected" +@[inline] def updateForallE! (e : Expr) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | forallE n d b bi => updateForall! (forallE n d b bi) bi newDomain newBody + | _ => panic! "forall expected" -@[inline] def updateLambdaE! (e : Expr) (newDomain : Expr) (newBody : Expr) : Expr := - match h : e with - | lam _ _ _ c => updateLambda e c newDomain newBody (h ▸ rfl) +@[inline] private unsafe def updateLambda!Impl (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | lam n d b bi => + if ptrEq d newDomain && ptrEq b newBody && bi == newBinfo then + e + else + mkLambda n newBinfo newDomain newBody | _ => panic! "lambda expected" -@[extern "lean_expr_update_let"] -def updateLet (e : Expr) (newType : Expr) (newVal : Expr) (newBody : Expr) (h : e.isLet) : Expr := - mkLet e.letName! newType newVal newBody +@[implementedBy updateLambda!Impl] +def updateLambda! (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | lam n _ _ _ => mkLambda n newBinfo newDomain newBody + | _ => panic! "lambda expected" -@[inline] def updateLet! (e : Expr) (newType : Expr) (newVal : Expr) (newBody : Expr) : Expr := - match h : e with - | letE .. => updateLet e newType newVal newBody (h ▸ rfl) - | _ => panic! "let expression expected" +@[inline] def updateLambdaE! (e : Expr) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | lam n d b bi => updateLambda! (lam n d b bi) bi newDomain newBody + | _ => panic! "lambda expected" + +@[inline] private unsafe def updateLet!Impl (e : Expr) (newType : Expr) (newVal : Expr) (newBody : Expr) : Expr := + match e with + | letE n t v b nonDep => + if ptrEq t newType && ptrEq v newVal && ptrEq b newBody then + e + else + letE n newType newVal newBody nonDep + | _ => panic! "let expression expected" + +@[implementedBy updateLet!Impl] +def updateLet! (e : Expr) (newType : Expr) (newVal : Expr) (newBody : Expr) : Expr := + match e with + | letE n _ _ _ c => letE n newType newVal newBody c + | _ => panic! "let expression expected" def updateFn : Expr → Expr → Expr | e@(app f a), g => e.updateApp! (updateFn f g) a | _, g => g +/-- +Eta reduction. If `e` is of the form `(fun x => f x)`, then return `f`. +-/ partial def eta (e : Expr) : Expr := match e with | Expr.lam _ d b _ => @@ -1174,8 +1525,9 @@ partial def eta (e : Expr) : Expr := | _ => e.updateLambdaE! d b' | _ => e -/- Instantiate level parameters -/ - +/-- +Instantiate level parameters +-/ @[inline] def instantiateLevelParamsCore (s : Name → Option Level) (e : Expr) : Expr := let rec @[specialize] visit (e : Expr) : Expr := if !e.hasLevelParam then e @@ -1195,6 +1547,10 @@ private def getParamSubst : List Name → List Level → Name → Option Level | p::ps, u::us, p' => if p == p' then some u else getParamSubst ps us p' | _, _, _ => none +/-- +Instantiate univeres level parameters names `paramNames` with `lvls` in `e`. +If the two lists have different length, the smallest one is used. +-/ def instantiateLevelParams (e : Expr) (paramNames : List Name) (lvls : List Level) : Expr := instantiateLevelParamsCore (getParamSubst paramNames lvls) e @@ -1207,23 +1563,38 @@ private partial def getParamSubstArray (ps : Array Name) (us : Array Level) (p' else none else none +/-- +Instantiate univeres level parameters names `paramNames` with `lvls` in `e`. +If the two arrays have different length, the smallest one is used. +-/ def instantiateLevelParamsArray (e : Expr) (paramNames : Array Name) (lvls : Array Level) : Expr := instantiateLevelParamsCore (fun p => getParamSubstArray paramNames lvls p 0) e -/-- Annotate `e` with the given option. -/ +/-- +Annotate `e` with the given option. +The information is stored using metadata around `e`. +-/ def setOption (e : Expr) (optionName : Name) [KVMap.Value α] (val : α) : Expr := mkMData (MData.empty.set optionName val) e -/-- Annotate `e` with `pp.explicit := true` - The delaborator uses `pp` options. -/ +/-- +Annotate `e` with `pp.explicit := flag` +The delaborator uses `pp` options. +-/ def setPPExplicit (e : Expr) (flag : Bool) := e.setOption `pp.explicit flag +/-- +Annotate `e` with `pp.universes := flag` +The delaborator uses `pp` options. +-/ def setPPUniverses (e : Expr) (flag : Bool) := e.setOption `pp.universes flag -/-- If `e` is an application `f a_1 ... a_n` annotate `f`, `a_1` ... `a_n` with `pp.explicit := false`, - and annotate `e` with `pp.explicit := true`. -/ +/-- +If `e` is an application `f a_1 ... a_n` annotate `f`, `a_1` ... `a_n` with `pp.explicit := false`, +and annotate `e` with `pp.explicit := true`. +-/ def setAppPPExplicit (e : Expr) : Expr := match e with | app .. => @@ -1232,8 +1603,10 @@ def setAppPPExplicit (e : Expr) : Expr := mkAppN f args |>.setPPExplicit true | _ => e -/-- Similar for `setAppPPExplicit`, but only annotate children with `pp.explicit := false` if - `e` does not contain metavariables. -/ +/-- +Similar for `setAppPPExplicit`, but only annotate children with `pp.explicit := false` if +`e` does not contain metavariables. +-/ def setAppPPExplicitForExposingMVars (e : Expr) : Expr := match e with | app .. => @@ -1244,40 +1617,60 @@ def setAppPPExplicitForExposingMVars (e : Expr) : Expr := end Expr +/-- +Annotate `e` with the given annotation name `kind`. +It uses metadata to store the annotation. +-/ def mkAnnotation (kind : Name) (e : Expr) : Expr := mkMData (KVMap.empty.insert kind (DataValue.ofBool true)) e +/-- +Return `some e'` if `e = mkAnnotation kind e'` +-/ def annotation? (kind : Name) (e : Expr) : Option Expr := match e with | .mdata d b => if d.size == 1 && d.getBool kind false then some b else none | _ => none +/-- +Annotate `e` with the `let_fun` annotation. This annotation is used as hint for the delaborator. +If `e` is of the form `(fun x : t => b) v`, then `mkLetFunAnnotation e` is delaborated at +`let_fun x : t := v; b` +-/ def mkLetFunAnnotation (e : Expr) : Expr := mkAnnotation `let_fun e +/-- +Return `some e'` if `e = mkLetFunAnnotation e'` +-/ def letFunAnnotation? (e : Expr) : Option Expr := annotation? `let_fun e +/-- +Return true if `e = mkLetFunAnnotation e'`, and `e'` is of the form `(fun x : t => b) v` +-/ def isLetFun (e : Expr) : Bool := match letFunAnnotation? e with | none => false | some e => e.isApp && e.appFn!.isLambda /-- - Auxiliary annotation used to mark terms marked with the "inaccessible" annotation `.(t)` and - `_` in patterns. -/ +Auxiliary annotation used to mark terms marked with the "inaccessible" annotation `.(t)` and +`_` in patterns. +-/ def mkInaccessible (e : Expr) : Expr := mkAnnotation `_inaccessible e +/-- Return `some e'` if `e = mkInaccessible e'`. -/ def inaccessible? (e : Expr) : Option Expr := annotation? `_inaccessible e private def patternRefAnnotationKey := `_patWithRef /-- - During elaboration expressions corresponding to pattern matching terms - are annotated with `Syntax` objects. This function returns `some (stx, p')` if - `p` is the pattern `p'` annotated with `stx` +During elaboration expressions corresponding to pattern matching terms +are annotated with `Syntax` objects. This function returns `some (stx, p')` if +`p` is the pattern `p'` annotated with `stx` -/ def patternWithRef? (p : Expr) : Option (Syntax × Expr) := match p with @@ -1288,8 +1681,8 @@ def patternWithRef? (p : Expr) : Option (Syntax × Expr) := | _ => none /-- - Annotate the pattern `p` with `stx`. This is an auxiliary annotation - for producing better hover information. +Annotate the pattern `p` with `stx`. This is an auxiliary annotation +for producing better hover information. -/ def mkPatternWithRef (p : Expr) (stx : Syntax) : Expr := if patternWithRef? p |>.isSome then @@ -1307,12 +1700,14 @@ def patternAnnotation? (e : Expr) : Option Expr := none /-- - Annotate `e` with the LHS annotation. The delaborator displays - expressions of the form `lhs = rhs` as `lhs` when they have this annotation. +Annotate `e` with the LHS annotation. The delaborator displays +expressions of the form `lhs = rhs` as `lhs` when they have this annotation. +This is used to implement the infoview for the `conv` mode. -/ def mkLHSGoal (e : Expr) : Expr := mkAnnotation `_lhsGoal e +/-- Return `some lhs` if `e = mkLHGoal e'`, where `e'` is of the form `lhs = rhs`. -/ def isLHSGoal? (e : Expr) : Option Expr := match annotation? `_lhsGoal e with | none => none @@ -1322,15 +1717,27 @@ def isLHSGoal? (e : Expr) : Option Expr := else none -def mkFreshFVarId {m : Type → Type} [Monad m] [MonadNameGenerator m] : m FVarId := +/-- +Polymorphic operation for generating unique/fresh free variable identifiers. +It is available in any monad `m` that implements the inferface `MonadNameGenerator`. +-/ +def mkFreshFVarId [Monad m] [MonadNameGenerator m] : m FVarId := return { name := (← mkFreshId) } -def mkFreshMVarId {m : Type → Type} [Monad m] [MonadNameGenerator m] : m MVarId := +/-- +Polymorphic operation for generating unique/fresh metavariable identifiers. +It is available in any monad `m` that implements the inferface `MonadNameGenerator`. +-/ +def mkFreshMVarId [Monad m] [MonadNameGenerator m] : m MVarId := return { name := (← mkFreshId) } +/-- Return `Not p` -/ def mkNot (p : Expr) : Expr := mkApp (mkConst ``Not) p +/-- Return `p ∨ q` -/ def mkOr (p q : Expr) : Expr := mkApp2 (mkConst ``Or) p q +/-- Return `p ∧ q` -/ def mkAnd (p q : Expr) : Expr := mkApp2 (mkConst ``And) p q +/-- Return `Classical.em p` -/ def mkEM (p : Expr) : Expr := mkApp (mkConst ``Classical.em) p end Lean diff --git a/src/Lean/HeadIndex.lean b/src/Lean/HeadIndex.lean index 57f1c51e7ea2..ebea4bf733d8 100644 --- a/src/Lean/HeadIndex.lean +++ b/src/Lean/HeadIndex.lean @@ -51,7 +51,7 @@ private def headNumArgsAux : Expr → Nat → Nat def headNumArgs (e : Expr) : Nat := headNumArgsAux e 0 -/- +/-- Quick version that may fail if it "hits" a loose bound variable. This can happen, for example, if the input expression is of the form. ``` @@ -73,7 +73,7 @@ private def toHeadIndexQuick? : Expr → Option HeadIndex | mdata _ e => toHeadIndexQuick? e | _ => none -/- +/-- Slower version of `toHeadIndexQuick?` that "expands" let-declarations to make sure we never hit a loose bound variable. The performance of the `letE` alternative can be improved, but this function should not be in the hotpath diff --git a/src/Lean/Hygiene.lean b/src/Lean/Hygiene.lean index cda2e1a11283..efa8f2eb562e 100644 --- a/src/Lean/Hygiene.lean +++ b/src/Lean/Hygiene.lean @@ -8,7 +8,7 @@ import Lean.Data.Options import Lean.Data.Format namespace Lean -/- Remark: `MonadQuotation` class is part of the `Init` package and loaded by default since it is used in the builtin command `macro`. -/ +/-! Remark: `MonadQuotation` class is part of the `Init` package and loaded by default since it is used in the builtin command `macro`. -/ structure Unhygienic.Context where ref : Syntax diff --git a/src/Lean/ImportingFlag.lean b/src/Lean/ImportingFlag.lean index 3fc36632fac8..9107ffd27c6c 100644 --- a/src/Lean/ImportingFlag.lean +++ b/src/Lean/ImportingFlag.lean @@ -27,7 +27,7 @@ unsafe def enableInitializersExecution : IO Unit := def isInitializerExecutionEnabled : IO Bool := runInitializersRef.get -/- We say Lean is "initializing" when it is executing `builtin_initialize` declarations or importing modules. +/-- We say Lean is "initializing" when it is executing `builtin_initialize` declarations or importing modules. Recall that Lean excutes `initialize` declarations while importing modules. -/ def initializing : IO Bool := IO.initializing <||> importingRef.get diff --git a/src/Lean/KeyedDeclsAttribute.lean b/src/Lean/KeyedDeclsAttribute.lean index be9855988ae9..29dd7360ff4a 100644 --- a/src/Lean/KeyedDeclsAttribute.lean +++ b/src/Lean/KeyedDeclsAttribute.lean @@ -44,7 +44,7 @@ structure OLeanEntry where deriving Inhabited structure AttributeEntry (γ : Type) extends OLeanEntry where - /- Recall that we cannot store `γ` into .olean files because it is a closure. + /-- Recall that we cannot store `γ` into .olean files because it is a closure. Given `OLeanEntry.declName`, we convert it into a `γ` by using the unsafe function `evalConstCheck`. -/ value : γ diff --git a/src/Lean/Level.lean b/src/Lean/Level.lean index c5efb8df8e67..4e93c0b56fc5 100644 --- a/src/Lean/Level.lean +++ b/src/Lean/Level.lean @@ -493,11 +493,9 @@ end Level elseK () /- Similar to `mkLevelMax`, but applies cheap simplifications -/ -@[export lean_level_mk_max_simp] def mkLevelMax' (u v : Level) : Level := mkLevelMaxCore u v fun _ => mkLevelMax u v -@[export lean_level_simp_max] def simpLevelMax' (u v : Level) (d : Level) : Level := mkLevelMaxCore u v fun _ => d @@ -509,51 +507,52 @@ def simpLevelMax' (u v : Level) (d : Level) : Level := else elseK () /- Similar to `mkLevelIMax`, but applies cheap simplifications -/ -@[export lean_level_mk_imax_simp] def mkLevelIMax' (u v : Level) : Level := mkLevelIMaxCore u v fun _ => mkLevelIMax u v -@[export lean_level_simp_imax] def simpLevelIMax' (u v : Level) (d : Level) := mkLevelIMaxCore u v fun _ => d namespace Level -/- The update functions here are defined using C code. They will try to avoid - allocating new values using pointer equality. - The hypotheses `(h : e.is...)` are used to ensure Lean will not crash - at runtime. - The `update*!` functions are inlined and provide a convenient way of using the - update proofs without providing proofs. - Note that if they are used under a match-expression, the compiler will eliminate - the double-match. -/ - -@[extern "lean_level_update_succ"] -def updateSucc (lvl : Level) (newLvl : Level) (h : lvl.isSucc) : Level := - mkLevelSucc newLvl - -@[inline] def updateSucc! (lvl : Level) (newLvl : Level) : Level := -match h : lvl with - | succ .. => updateSucc lvl newLvl (h ▸ rfl) - | _ => panic! "succ level expected" - -@[extern "lean_level_update_max"] -def updateMax (lvl : Level) (newLhs : Level) (newRhs : Level) (h : lvl.isMax) : Level := - mkLevelMax' newLhs newRhs - -@[inline] def updateMax! (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := - match h : lvl with - | max .. => updateMax lvl newLhs newRhs (h ▸ rfl) - | _ => panic! "max level expected" - -@[extern "lean_level_update_imax"] -def updateIMax (lvl : Level) (newLhs : Level) (newRhs : Level) (h : lvl.isIMax) : Level := - mkLevelIMax' newLhs newRhs - -@[inline] def updateIMax! (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := - match h : lvl with - | imax .. => updateIMax lvl newLhs newRhs (h ▸ rfl) - | _ => panic! "imax level expected" +/-! +The update functions try to avoid allocating new values using pointer equality. +Note that if the `update*!` functions are used under a match-expression, +the compiler will eliminate the double-match. +-/ + +@[inline] private unsafe def updateSucc!Impl (lvl : Level) (newLvl : Level) : Level := + match lvl with + | succ l => if ptrEq l newLvl then lvl else mkLevelSucc newLvl + | _ => panic! "succ level expected" + +@[implementedBy updateSucc!Impl] +def updateSucc! (lvl : Level) (newLvl : Level) : Level := + match lvl with + | succ _ => mkLevelSucc newLvl + | _ => panic! "succ level expected" + +@[inline] private unsafe def updateMax!Impl (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := + match lvl with + | max lhs rhs => if ptrEq lhs newLhs && ptrEq rhs newRhs then simpLevelMax' newLhs newRhs lvl else mkLevelMax' newLhs newRhs + | _ => panic! "max level expected" + +@[implementedBy updateMax!Impl] +def updateMax! (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := + match lvl with + | max _ _ => mkLevelMax' newLhs newRhs + | _ => panic! "max level expected" + +@[inline] private unsafe def updateIMax!Impl (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := + match lvl with + | imax lhs rhs => if ptrEq lhs newLhs && ptrEq rhs newRhs then simpLevelIMax' newLhs newRhs lvl else mkLevelIMax' newLhs newRhs + | _ => panic! "imax level expected" + +@[implementedBy updateIMax!Impl] +def updateIMax! (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := + match lvl with + | imax _ _ => mkLevelIMax' newLhs newRhs + | _ => panic! "imax level expected" def mkNaryMax : List Level → Level | [] => levelZero diff --git a/src/Lean/Linter/Basic.lean b/src/Lean/Linter/Basic.lean index dc627c584d40..c2f28b5abc76 100644 --- a/src/Lean/Linter/Basic.lean +++ b/src/Lean/Linter/Basic.lean @@ -25,12 +25,12 @@ def getLinterUnusedVariables (o : Options) : Bool := o.get linter.unusedVariable def getLinterUnusedVariablesFunArgs (o : Options) : Bool := o.get linter.unusedVariables.funArgs.name (getLinterUnusedVariables o) def getLinterUnusedVariablesPatternVars (o : Options) : Bool := o.get linter.unusedVariables.patternVars.name (getLinterUnusedVariables o) -def unusedVariables : Linter := fun stx => do +def unusedVariables : Linter := fun cmdStx => do -- NOTE: `messages` is local to the current command if (← get).messages.hasErrors then return - let some stxRange := stx.getRange? + let some cmdStxRange := cmdStx.getRange? | pure () let infoTrees := (← get).infoState.trees.toArray @@ -40,7 +40,7 @@ def unusedVariables : Linter := fun stx => do return -- collect references - let refs := findModuleRefs fileMap infoTrees + let refs := findModuleRefs fileMap infoTrees (allowSimultaneousBinderUse := true) let mut vars : HashMap FVarId RefInfo := .empty let mut constDecls : HashSet String.Range := .empty @@ -76,6 +76,7 @@ def unusedVariables : Linter := fun stx => do -- determine unused variables for (id, ⟨decl?, uses⟩) in vars.toList do + -- process declaration let some decl := decl? | continue let declStx := skipDeclIdIfPresent decl.stx @@ -83,43 +84,63 @@ def unusedVariables : Linter := fun stx => do | continue let some localDecl := decl.info.lctx.find? id | continue - if !stxRange.contains range.start || localDecl.userName.hasMacroScopes then + if !cmdStxRange.contains range.start || localDecl.userName.hasMacroScopes then continue + -- check if variable is used + if !uses.isEmpty || tacticFVarUses.contains id || decl.aliases.any (match · with | .fvar id => tacticFVarUses.contains id | _ => false) then + continue + + -- check linter options let opts := decl.ci.options if !getLinterUnusedVariables opts then continue - let mut ignoredPatternFns := #[ + -- collect ignore functions + let mut ignoreFns := #[ isTopLevelDecl constDecls, matchesUnusedPattern, isVariable, isInStructure, isInInductive, isInCtorOrStructBinder, - isInConstantOrAxiom, + isInOpaqueOrAxiom, isInDefWithForeignDefinition, isInDepArrow ] if !getLinterUnusedVariablesFunArgs opts then - ignoredPatternFns := ignoredPatternFns.append #[ + ignoreFns := ignoreFns.append #[ isInLetDeclaration, isInDeclarationSignature, isInFun ] if !getLinterUnusedVariablesPatternVars opts then - ignoredPatternFns := ignoredPatternFns.append #[ + ignoreFns := ignoreFns.append #[ isPatternVar ] - let some stack := findSyntaxStack? stx declStx - | continue - if ignoredPatternFns.any (· declStx stack) then + -- evaluate ignore functions on original syntax + if let some stack := findSyntaxStack? cmdStx declStx then + if ignoreFns.any (· declStx stack) then + continue + else + continue + + -- evaluate ignore functions on macro expansion outputs + if ← infoTrees.anyM fun tree => do + if let some macroExpansions ← collectMacroExpansions? range tree then + return macroExpansions.any fun expansion => + if let some stack := findSyntaxStack? expansion.output declStx then + ignoreFns.any (· declStx stack) + else + false + else + return false + then continue - if uses.isEmpty && !tacticFVarUses.contains id && - decl.aliases.all (match · with | .fvar id => !tacticFVarUses.contains id | _ => false) then - publishMessage s!"unused variable `{localDecl.userName}`" range + -- publish warning if variable is unused and not ignored + publishMessage s!"unused variable `{localDecl.userName}`" range return () where @@ -149,7 +170,7 @@ where stackMatches stack [`null, none, `null, ``Lean.Parser.Command.optDeclSig, none] && (stack.get? 4 |>.any fun (stx, _) => [``Lean.Parser.Command.ctor, ``Lean.Parser.Command.structSimpleBinder].any (stx.isOfKind ·)) - isInConstantOrAxiom (_ : Syntax) (stack : SyntaxStack) := + isInOpaqueOrAxiom (_ : Syntax) (stack : SyntaxStack) := stackMatches stack [`null, none, `null, ``Lean.Parser.Command.declSig, none] && (stack.get? 4 |>.any fun (stx, _) => [``Lean.Parser.Command.opaque, ``Lean.Parser.Command.axiom].any (stx.isOfKind ·)) diff --git a/src/Lean/Linter/Util.lean b/src/Lean/Linter/Util.lean index 9203e86bf05b..90f4ee0fd4bd 100644 --- a/src/Lean/Linter/Util.lean +++ b/src/Lean/Linter/Util.lean @@ -20,8 +20,45 @@ do let messages := (← get).messages |>.add (mkMessageCore ctx.fileName ctx.fileMap content severity range.start range.stop) modify ({ · with messages := messages }) +/-- Go upwards through the given `tree` starting from the smallest node that +contains the given `range` and collect all `MacroExpansionInfo`s on the way up. +The result is `some []` if no `MacroExpansionInfo` was found on the way and +`none` if no `InfoTree` node was found that covers the given `range`. + +Return the result reversed, s.t. the macro expansion that would be applied to +the original syntax first is the first element of the returned list. -/ +def collectMacroExpansions? {m} [Monad m] (range : String.Range) (tree : Elab.InfoTree) : m <| Option <| List Elab.MacroExpansionInfo := do + if let .some <| .some result ← go then + return some result.reverse + else + return none +where + go : m <| Option <| Option <| List Elab.MacroExpansionInfo := tree.visitM (postNode := fun _ i _ results => do + let results := results |>.filterMap id |>.filterMap id + + -- we expect that at most one InfoTree child returns a result + if let results :: _ := results then + if let .ofMacroExpansionInfo i := i then + return some <| i :: results + else + return some results + else if i.contains range.start && i.contains (includeStop := true) range.stop then + if let .ofMacroExpansionInfo i := i then + return some [i] + else + return some [] + else + return none) + +/-- List of `Syntax` nodes in which each succeeding element is the parent of +the current. The associated index is the index of the preceding element in the +list of children of the current element. -/ abbrev SyntaxStack := List (Syntax × Nat) +/-- Go upwards through the given `root` syntax starting from `child` and +collect all `Syntax` nodes on the way up. + +Return `none` if the `child` is not found in `root`. -/ partial def findSyntaxStack? (root child : Syntax) : Option SyntaxStack := Id.run <| do let some childRange := child.getRange? | none @@ -40,6 +77,8 @@ partial def findSyntaxStack? (root child : Syntax) : Option SyntaxStack := Id.ru return none go [] root +/-- Compare the `SyntaxNodeKind`s in `pattern` to those of the `Syntax` +elements in `stack`. Return `false` if `stack` is shorter than `pattern`. -/ def stackMatches (stack : SyntaxStack) (pattern : List $ Option SyntaxNodeKind) : Bool := stack.length >= pattern.length && (stack diff --git a/src/Lean/LocalContext.lean b/src/Lean/LocalContext.lean index a3290c47df31..8bc8898d5cd9 100644 --- a/src/Lean/LocalContext.lean +++ b/src/Lean/LocalContext.lean @@ -318,6 +318,9 @@ instance : ForIn m LocalContext LocalDecl where @[inline] def foldr (lctx : LocalContext) (f : LocalDecl → β → β) (init : β) : β := Id.run <| lctx.foldrM f init +def size (lctx : LocalContext) : Nat := + lctx.foldl (fun n _ => n+1) 0 + @[inline] def findDecl? (lctx : LocalContext) (f : LocalDecl → Option β) : Option β := Id.run <| lctx.findDeclM? f @@ -338,7 +341,7 @@ partial def isSubPrefixOfAux (a₁ a₂ : PArray (Option LocalDecl)) (exceptFVar else false else true -/- Given `lctx₁ - exceptFVars` of the form `(x_1 : A_1) ... (x_n : A_n)`, then return true +/-- Given `lctx₁ - exceptFVars` of the form `(x_1 : A_1) ... (x_n : A_n)`, then return true iff there is a local context `B_1* (x_1 : A_1) ... B_n* (x_n : A_n)` which is a prefix of `lctx₂` where `B_i`'s are (possibly empty) sequences of local declarations. -/ def isSubPrefixOf (lctx₁ lctx₂ : LocalContext) (exceptFVars : Array Expr := #[]) : Bool := diff --git a/src/Lean/Meta/AppBuilder.lean b/src/Lean/Meta/AppBuilder.lean index 2a1f646027f9..450108cab796 100644 --- a/src/Lean/Meta/AppBuilder.lean +++ b/src/Lean/Meta/AppBuilder.lean @@ -24,11 +24,13 @@ def mkExpectedTypeHint (e : Expr) (expectedType : Expr) : MetaM Expr := do let u ← getLevel expectedType return mkApp2 (mkConst ``id [u]) expectedType e +/-- Return `a = b`. -/ def mkEq (a b : Expr) : MetaM Expr := do let aType ← inferType a let u ← getLevel aType return mkApp3 (mkConst ``Eq [u]) aType a b +/-- Return `HEq a b`. -/ def mkHEq (a b : Expr) : MetaM Expr := do let aType ← inferType a let bType ← inferType b @@ -47,21 +49,25 @@ def mkEqHEq (a b : Expr) : MetaM Expr := do else return mkApp4 (mkConst ``HEq [u]) aType a bType b +/-- Return a proof of `a = a`. -/ def mkEqRefl (a : Expr) : MetaM Expr := do let aType ← inferType a let u ← getLevel aType return mkApp2 (mkConst ``Eq.refl [u]) aType a +/-- Return a proof of `HEq a a`. -/ def mkHEqRefl (a : Expr) : MetaM Expr := do let aType ← inferType a let u ← getLevel aType return mkApp2 (mkConst ``HEq.refl [u]) aType a +/-- Given `hp : P` and `nhp : Not P` returns an instance of type `e`. -/ def mkAbsurd (e : Expr) (hp hnp : Expr) : MetaM Expr := do let p ← inferType hp let u ← getLevel e return mkApp4 (mkConst ``absurd [u]) p e hp hnp +/-- Given `h : False`, return an instance of type `e`. -/ def mkFalseElim (e : Expr) (h : Expr) : MetaM Expr := do let u ← getLevel e return mkApp2 (mkConst ``False.elim [u]) e h @@ -76,6 +82,7 @@ private def hasTypeMsg (e type : Expr) : MessageData := private def throwAppBuilderException {α} (op : Name) (msg : MessageData) : MetaM α := throwError "AppBuilder for '{op}', {msg}" +/-- Given `h : a = b`, returns a proof of `b = a`. -/ def mkEqSymm (h : Expr) : MetaM Expr := do if h.isAppOf ``Eq.refl then return h @@ -87,6 +94,7 @@ def mkEqSymm (h : Expr) : MetaM Expr := do return mkApp4 (mkConst ``Eq.symm [u]) α a b h | none => throwAppBuilderException ``Eq.symm ("equality proof expected" ++ hasTypeMsg h hType) +/-- Given `h₁ : a = b` and `h₂ : b = c` returns a proof of `a = c`. -/ def mkEqTrans (h₁ h₂ : Expr) : MetaM Expr := do if h₁.isAppOf ``Eq.refl then return h₂ @@ -102,6 +110,7 @@ def mkEqTrans (h₁ h₂ : Expr) : MetaM Expr := do | none, _ => throwAppBuilderException ``Eq.trans ("equality proof expected" ++ hasTypeMsg h₁ hType₁) | _, none => throwAppBuilderException ``Eq.trans ("equality proof expected" ++ hasTypeMsg h₂ hType₂) +/-- Given `h : HEq a b`, returns a proof of `HEq b a`. -/ def mkHEqSymm (h : Expr) : MetaM Expr := do if h.isAppOf ``HEq.refl then return h @@ -114,6 +123,7 @@ def mkHEqSymm (h : Expr) : MetaM Expr := do | none => throwAppBuilderException ``HEq.symm ("heterogeneous equality proof expected" ++ hasTypeMsg h hType) +/-- Given `h₁ : HEq a b`, `h₂ : HEq b c`, returns a proof of `HEq a c`. -/ def mkHEqTrans (h₁ h₂ : Expr) : MetaM Expr := do if h₁.isAppOf ``HEq.refl then return h₂ @@ -129,6 +139,7 @@ def mkHEqTrans (h₁ h₂ : Expr) : MetaM Expr := do | none, _ => throwAppBuilderException ``HEq.trans ("heterogeneous equality proof expected" ++ hasTypeMsg h₁ hType₁) | _, none => throwAppBuilderException ``HEq.trans ("heterogeneous equality proof expected" ++ hasTypeMsg h₂ hType₂) +/-- Given `h : Eq a b`, returns a proof of `HEq a b`. -/ def mkEqOfHEq (h : Expr) : MetaM Expr := do let hType ← infer h match hType.heq? with @@ -140,6 +151,7 @@ def mkEqOfHEq (h : Expr) : MetaM Expr := do | _ => throwAppBuilderException ``HEq.trans m!"heterogeneous equality proof expected{indentExpr h}" +/-- Given `f : α → β` and `h : a = b`, returns a proof of `f a = f b`.-/ def mkCongrArg (f h : Expr) : MetaM Expr := do if h.isAppOf ``Eq.refl then mkEqRefl (mkApp f h.appArg!) @@ -154,6 +166,7 @@ def mkCongrArg (f h : Expr) : MetaM Expr := do | none, _ => throwAppBuilderException ``congrArg ("non-dependent function expected" ++ hasTypeMsg f fType) | _, none => throwAppBuilderException ``congrArg ("equality proof expected" ++ hasTypeMsg h hType) +/-- Given `h : f = g` and `a : α`, returns a proof of `f a = g a`.-/ def mkCongrFun (h a : Expr) : MetaM Expr := do if h.isAppOf ``Eq.refl then mkEqRefl (mkApp h.appArg! a) @@ -171,6 +184,7 @@ def mkCongrFun (h a : Expr) : MetaM Expr := do | _ => throwAppBuilderException ``congrFun ("equality proof between functions expected" ++ hasTypeMsg h hType) | _ => throwAppBuilderException ``congrFun ("equality proof expected" ++ hasTypeMsg h hType) +/-- Given `h₁ : f = g` and `h₂ : a = b`, returns a proof of `f a = g b`. -/ def mkCongr (h₁ h₂ : Expr) : MetaM Expr := do if h₁.isAppOf ``Eq.refl then mkCongrArg h₁.appArg! h₂ @@ -369,6 +383,7 @@ def mkNoConfusion (target : Expr) (h : Expr) : MetaM Expr := do let u ← getLevel target return mkAppN (mkConst (Name.mkStr v.name "noConfusion") (u :: us)) (α.getAppArgs ++ #[target, a, b, h]) +/-- Given a `monad` and `e : α`, makes `pure e`.-/ def mkPure (monad : Expr) (e : Expr) : MetaM Expr := mkAppOptM ``Pure.pure #[monad, none, none, e] diff --git a/src/Lean/Meta/Basic.lean b/src/Lean/Meta/Basic.lean index 65f195760507..cf80353b6db1 100644 --- a/src/Lean/Meta/Basic.lean +++ b/src/Lean/Meta/Basic.lean @@ -19,7 +19,7 @@ import Lean.Meta.DiscrTreeTypes import Lean.Eval import Lean.CoreM -/- +/-! This module provides four (mutually dependent) goodies that are needed for building the elaborator and tactic frameworks. 1- Weak head normal form computation with support for metavariables and transparency modes. 2- Definitionally equality checking with support for metavariables (aka unification modulo definitional equality). @@ -34,31 +34,31 @@ namespace Lean.Meta builtin_initialize isDefEqStuckExceptionId : InternalExceptionId ← registerInternalExceptionId `isDefEqStuck /-- - Configuration flags for the `MetaM` monad. - Many of them are used to control the `isDefEq` function that checks whether two terms are definitionally equal or not. - Recall that when `isDefEq` is trying to check whether - `?m@C a₁ ... aₙ` and `t` are definitionally equal (`?m@C a₁ ... aₙ =?= t`), where - `?m@C` as a shorthand for `C |- ?m : t` where `t` is the type of `?m`. - We solve it using the assignment `?m := fun a₁ ... aₙ => t` if - 1) `a₁ ... aₙ` are pairwise distinct free variables that are ​*not*​ let-variables. - 2) `a₁ ... aₙ` are not in `C` - 3) `t` only contains free variables in `C` and/or `{a₁, ..., aₙ}` - 4) For every metavariable `?m'@C'` occurring in `t`, `C'` is a subprefix of `C` - 5) `?m` does not occur in `t` +Configuration flags for the `MetaM` monad. +Many of them are used to control the `isDefEq` function that checks whether two terms are definitionally equal or not. +Recall that when `isDefEq` is trying to check whether +`?m@C a₁ ... aₙ` and `t` are definitionally equal (`?m@C a₁ ... aₙ =?= t`), where +`?m@C` as a shorthand for `C |- ?m : t` where `t` is the type of `?m`. +We solve it using the assignment `?m := fun a₁ ... aₙ => t` if +1) `a₁ ... aₙ` are pairwise distinct free variables that are ​*not*​ let-variables. +2) `a₁ ... aₙ` are not in `C` +3) `t` only contains free variables in `C` and/or `{a₁, ..., aₙ}` +4) For every metavariable `?m'@C'` occurring in `t`, `C'` is a subprefix of `C` +5) `?m` does not occur in `t` -/ structure Config where /-- If `foApprox` is set to true, and some `aᵢ` is not a free variable, - then we use first-order unification - ``` - ?m a_1 ... a_i a_{i+1} ... a_{i+k} =?= f b_1 ... b_k - ``` - reduces to - ``` - ?m a_1 ... a_i =?= f - a_{i+1} =?= b_1 - ... - a_{i+k} =?= b_k + then we use first-order unification + ``` + ?m a_1 ... a_i a_{i+1} ... a_{i+k} =?= f b_1 ... b_k + ``` + reduces to + ``` + ?m a_1 ... a_i =?= f + a_{i+1} =?= b_1 + ... + a_{i+k} =?= b_k ``` -/ foApprox : Bool := false @@ -136,6 +136,34 @@ structure ParamInfo where This information affects the generation of congruence theorems. -/ isDecInst : Bool := false + /-- + `higherOrderOutParam` is true if this parameter is a higher-order output parameter + of local instance. + Example: + ``` + getElem : + {Cont : Type u_1} → {Idx : Type u_2} → {Elem : Type u_3} → + {Dom : Cont → Idx → Prop} → [self : GetElem Cont Idx Elem Dom] → + (xs : Cont) → (i : Idx) → Dom xs i → Elem + ``` + This flag is true for the parameter `Dom` because it is output parameter of + `[self : GetElem Cont Idx Elem Dom]` + -/ + higherOrderOutParam : Bool := false + /-- + `dependsOnHigherOrderOutParam` is true if the type of this parameter depends on + the higher-order output parameter of a previous local instance. + Example: + ``` + getElem : + {Cont : Type u_1} → {Idx : Type u_2} → {Elem : Type u_3} → + {Dom : Cont → Idx → Prop} → [self : GetElem Cont Idx Elem Dom] → + (xs : Cont) → (i : Idx) → Dom xs i → Elem + ``` + This flag is true for the parameter with type `Dom xs i` since `Dom` is an output parameter + of the instance `[self : GetElem Cont Idx Elem Dom]` + -/ + dependsOnHigherOrderOutParam : Bool := false deriving Inhabited def ParamInfo.isImplicit (p : ParamInfo) : Bool := @@ -396,7 +424,7 @@ def useEtaStruct (inductName : Name) : MetaM Bool := do | .all => return true | .notClasses => return !isClass (← getEnv) inductName -/- WARNING: The following 4 constants are a hack for simulating forward declarations. +/-! WARNING: The following 4 constants are a hack for simulating forward declarations. They are defined later using the `export` attribute. This is hackish because we have to hard-code the true arity of these definitions here, and make sure the C names match. We have used another hack based on `IO.Ref`s in the past, it was safer but less efficient. -/ @@ -453,7 +481,7 @@ def mkFreshTypeMVar (kind := MetavarKind.natural) (userName := Name.anonymous) : let u ← mkFreshLevelMVar mkFreshExprMVar (mkSort u) kind userName -/- Low-level version of `MkFreshExprMVar` which allows users to create/reserve a `mvarId` using `mkFreshId`, and then later create +/-- Low-level version of `MkFreshExprMVar` which allows users to create/reserve a `mvarId` using `mkFreshId`, and then later create the metavar using this method. -/ private def mkFreshExprMVarWithIdCore (mvarId : MVarId) (type : Expr) (kind : MetavarKind := MetavarKind.natural) (userName : Name := Name.anonymous) (numScopeArgs : Nat := 0) @@ -509,7 +537,7 @@ def isSyntheticMVar (e : Expr) : MetaM Bool := do def setMVarKind (mvarId : MVarId) (kind : MetavarKind) : MetaM Unit := modifyMCtx fun mctx => mctx.setMVarKind mvarId kind -/- Update the type of the given metavariable. This function assumes the new type is +/-- Update the type of the given metavariable. This function assumes the new type is definitionally equal to the current one -/ def setMVarType (mvarId : MVarId) (type : Expr) : MetaM Unit := do modifyMCtx fun mctx => mctx.setMVarType mvarId type @@ -662,7 +690,7 @@ private def getDefInfoTemp (info : ConstantInfo) : MetaM (Option ConstantInfo) : else return none -/- Remark: we later define `getConst?` at `GetConst.lean` after we define `Instances.lean`. +/-- Remark: we later define `getConst?` at `GetConst.lean` after we define `Instances.lean`. This method is only used to implement `isClassQuickConst?`. It is very similar to `getConst?`, but it returns none when `TransparencyMode.instances` and `constName` is an instance. This difference should be irrelevant for `isClassQuickConst?`. -/ @@ -1237,7 +1265,7 @@ private partial def instantiateForallAux (ps : Array Expr) (i : Nat) (e : Expr) else pure e -/- Given `e` of the form `forall (a_1 : A_1) ... (a_n : A_n), B[a_1, ..., a_n]` and `p_1 : A_1, ... p_n : A_n`, return `B[p_1, ..., p_n]`. -/ +/-- Given `e` of the form `forall (a_1 : A_1) ... (a_n : A_n), B[a_1, ..., a_n]` and `p_1 : A_1, ... p_n : A_n`, return `B[p_1, ..., p_n]`. -/ def instantiateForall (e : Expr) (ps : Array Expr) : MetaM Expr := instantiateForallAux ps 0 e @@ -1250,7 +1278,7 @@ private partial def instantiateLambdaAux (ps : Array Expr) (i : Nat) (e : Expr) else pure e -/- Given `e` of the form `fun (a_1 : A_1) ... (a_n : A_n) => t[a_1, ..., a_n]` and `p_1 : A_1, ... p_n : A_n`, return `t[p_1, ..., p_n]`. +/-- Given `e` of the form `fun (a_1 : A_1) ... (a_n : A_n) => t[a_1, ..., a_n]` and `p_1 : A_1, ... p_n : A_n`, return `t[p_1, ..., p_n]`. It uses `whnf` to reduce `e` if it is not a lambda -/ def instantiateLambda (e : Expr) (ps : Array Expr) : MetaM Expr := instantiateLambdaAux ps 0 e diff --git a/src/Lean/Meta/Check.lean b/src/Lean/Meta/Check.lean index 241e79d0a282..e4b99a578a3c 100644 --- a/src/Lean/Meta/Check.lean +++ b/src/Lean/Meta/Check.lean @@ -5,7 +5,7 @@ Authors: Leonardo de Moura -/ import Lean.Meta.InferType -/- +/-! This is not the Kernel type checker, but an auxiliary method for checking whether terms produced by tactics and `isDefEq` are type correct. -/ @@ -35,8 +35,8 @@ private def getFunctionDomain (f : Expr) : MetaM (Expr × BinderInfo) := do | Expr.forallE _ d _ c => return (d, c) | _ => throwFunctionExpected f -/- -Given to expressions `a` and `b`, this method tries to annotate terms with `pp.explicit := true` to +/-- +Given two expressions `a` and `b`, this method tries to annotate terms with `pp.explicit := true` to expose "implicit" differences. For example, suppose `a` and `b` are of the form ```lean @HashMap Nat Nat eqInst hasInst1 @@ -111,7 +111,7 @@ where return some (as.set! i ai, bs.set! i bi) return none -/- +/-- Return error message "has type{givenType}\nbut is expected to have type{expectedType}" -/ def mkHasTypeButIsExpectedMsg (givenType expectedType : Expr) : MetaM MessageData := do diff --git a/src/Lean/Meta/Closure.lean b/src/Lean/Meta/Closure.lean index d8e52610c8cb..3a9a52a71688 100644 --- a/src/Lean/Meta/Closure.lean +++ b/src/Lean/Meta/Closure.lean @@ -10,7 +10,7 @@ import Lean.Util.FoldConsts import Lean.Meta.Basic import Lean.Meta.Check -/- +/-! This module provides functions for "closing" open terms and creating auxiliary definitions. Here, we say a term is "open" if diff --git a/src/Lean/Meta/DecLevel.lean b/src/Lean/Meta/DecLevel.lean index c535289d52b0..565147f10e26 100644 --- a/src/Lean/Meta/DecLevel.lean +++ b/src/Lean/Meta/DecLevel.lean @@ -63,7 +63,7 @@ def decLevel (u : Level) : MetaM Level := do | some u => return u | none => throwError "invalid universe level, {u} is not greater than 0" -/- This method is useful for inferring universe level parameters for function that take arguments such as `{α : Type u}`. +/-- This method is useful for inferring universe level parameters for function that take arguments such as `{α : Type u}`. Recall that `Type u` is `Sort (u+1)` in Lean. Thus, given `α`, we must infer its universe level, and then decrement 1 to obtain `u`. -/ def getDecLevel (type : Expr) : MetaM Level := do diff --git a/src/Lean/Meta/DiscrTree.lean b/src/Lean/Meta/DiscrTree.lean index 379de6739226..b068fe00a6c5 100644 --- a/src/Lean/Meta/DiscrTree.lean +++ b/src/Lean/Meta/DiscrTree.lean @@ -10,7 +10,7 @@ import Lean.Meta.WHNF import Lean.Meta.Match.MatcherInfo namespace Lean.Meta.DiscrTree -/- +/-! (Imperfect) discrimination trees. We use a hybrid representation. - A `PersistentHashMap` for the root node which usually contains many children. @@ -108,7 +108,7 @@ partial def format [ToFormat α] (d : DiscrTree α) : Format := instance [ToFormat α] : ToFormat (DiscrTree α) := ⟨format⟩ -/- The discrimination tree ignores implicit arguments and proofs. +/-- The discrimination tree ignores implicit arguments and proofs. We use the following auxiliary id as a "mark". -/ private def tmpMVarId : MVarId := { name := `_discr_tree_tmp } private def tmpStar := mkMVar tmpMVarId @@ -205,7 +205,7 @@ private def isOffset (fName : Name) (e : Expr) : MetaM Bool := do else return fName == ``Nat.succ && e.getAppNumArgs == 1 -/- +/-- TODO: add hook for users adding their own functions for controlling `shouldAddAsStar` Different `DiscrTree` users may populate this set using, for example, attributes. diff --git a/src/Lean/Meta/DiscrTreeTypes.lean b/src/Lean/Meta/DiscrTreeTypes.lean index 07a6ceff7fd6..5300aa4d7750 100644 --- a/src/Lean/Meta/DiscrTreeTypes.lean +++ b/src/Lean/Meta/DiscrTreeTypes.lean @@ -7,7 +7,7 @@ import Lean.Expr namespace Lean.Meta -/- See file `DiscrTree.lean` for the actual implementation and documentation. -/ +/-! See file `DiscrTree.lean` for the actual implementation and documentation. -/ namespace DiscrTree diff --git a/src/Lean/Meta/ExprDefEq.lean b/src/Lean/Meta/ExprDefEq.lean index eb4c2c71955a..154cf2ff2e7d 100644 --- a/src/Lean/Meta/ExprDefEq.lean +++ b/src/Lean/Meta/ExprDefEq.lean @@ -133,7 +133,51 @@ def isEtaUnassignedMVar (e : Expr) : MetaM Bool := do pure true | _ => pure false -/- +private def trySynthPending (e : Expr) : MetaM Bool := do + let mvarId? ← getStuckMVar? e + match mvarId? with + | some mvarId => Meta.synthPending mvarId + | none => pure false + +/-- + Result type for `isDefEqArgsFirstPass`. +-/ +inductive DefEqArgsFirstPassResult where + | /-- + Failed to establish that explicit arguments are def-eq. + Remark: higher output parameters, and parameters that depend on them + are postponed. + -/ + failed + | /-- + Succeeded. The array `postponedImplicit` contains the position + of the implicit arguments for which def-eq has been postponed. + `postponedHO` contains the higher order output parameters, and parameters + that depend on them. They should be processed after the implict ones. + `postponedHO` is used to handle applications involving functions that + contain higher order output parameters. Example: + ```lean + getElem : + {Cont : Type u_1} → {Idx : Type u_2} → {Elem : Type u_3} → + {Dom : Cont → Idx → Prop} → [self : GetElem Cont Idx Elem Dom] → + (xs : Cont) → (i : Idx) → (h : Dom xs i) → Elem + ``` + The argumengs `Dom` and `h` must be processed after all implicit arguments + otherwise higher-order unification problems are generated. See issue #1299, + when trying to solve + ``` + getElem ?a ?i ?h =?= getElem a i (Fin.val_lt_of_le i ...) + ``` + we have to solve the constraint + ``` + ?Dom a i.val =?= LT.lt i.val (Array.size a) + ``` + by solving after the instance has been synthesized, we reduce this constraint to + a simple check. + -/ + ok (postponedImplicit : Array Nat) (postponedHO : Array Nat) + +/-- First pass for `isDefEqArgs`. We unify explicit arguments, *and* easy cases Here, we say a case is easy if it is of the form @@ -161,66 +205,61 @@ def isEtaUnassignedMVar (e : Expr) : MetaM Bool := do introduce counter intuitive behavior. Pre: `paramInfo.size <= args₁.size = args₂.size` + + See `DefEqArgsFirstPassResult` for additional information. -/ -private partial def isDefEqArgsFirstPass - (paramInfo : Array ParamInfo) (args₁ args₂ : Array Expr) : MetaM (Option (Array Nat)) := do - let rec loop (i : Nat) (postponed : Array Nat) := do - if h : i < paramInfo.size then - let info := paramInfo.get ⟨i, h⟩ - let a₁ := args₁[i]! - let a₂ := args₂[i]! - if !info.isExplicit then - if (← isEtaUnassignedMVar a₁ <||> isEtaUnassignedMVar a₂) then - if (← Meta.isExprDefEqAux a₁ a₂) then - loop (i+1) postponed - else - pure none - else - loop (i+1) (postponed.push i) - else if (← Meta.isExprDefEqAux a₁ a₂) then - loop (i+1) postponed - else - pure none +private def isDefEqArgsFirstPass + (paramInfo : Array ParamInfo) (args₁ args₂ : Array Expr) : MetaM DefEqArgsFirstPassResult := do + let mut postponedImplicit := #[] + let mut postponedHO := #[] + for i in [:paramInfo.size] do + let info := paramInfo[i]! + let a₁ := args₁[i]! + let a₂ := args₂[i]! + if info.dependsOnHigherOrderOutParam || info.higherOrderOutParam then + trace[Meta.isDefEq] "found messy {a₁} =?= {a₂}" + postponedHO := postponedHO.push i + else if info.isExplicit then + unless (← Meta.isExprDefEqAux a₁ a₂) do + return .failed + else if (← isEtaUnassignedMVar a₁ <||> isEtaUnassignedMVar a₂) then + unless (← Meta.isExprDefEqAux a₁ a₂) do + return .failed else - pure (some postponed) - loop 0 #[] - -private def trySynthPending (e : Expr) : MetaM Bool := do - let mvarId? ← getStuckMVar? e - match mvarId? with - | some mvarId => Meta.synthPending mvarId - | none => pure false - -private partial def isDefEqArgs (f : Expr) (args₁ args₂ : Array Expr) : MetaM Bool := - if h : args₁.size = args₂.size then do - let finfo ← getFunInfoNArgs f args₁.size - let (some postponed) ← isDefEqArgsFirstPass finfo.paramInfo args₁ args₂ | pure false - let rec processOtherArgs (i : Nat) : MetaM Bool := do - if h₁ : i < args₁.size then - let a₁ := args₁.get ⟨i, h₁⟩ - let a₂ := args₂.get ⟨i, Eq.subst h h₁⟩ - if (← Meta.isExprDefEqAux a₁ a₂) then - processOtherArgs (i+1) - else - pure false - else - pure true - if (← processOtherArgs finfo.paramInfo.size) then - postponed.allM fun i => do - /- Second pass: unify implicit arguments. - In the second pass, we make sure we are unfolding at - least non reducible definitions (default setting). -/ - let a₁ := args₁[i]! - let a₂ := args₂[i]! - let info := finfo.paramInfo[i]! - if info.isInstImplicit then - discard <| trySynthPending a₁ - discard <| trySynthPending a₂ - withAtLeastTransparency TransparencyMode.default <| Meta.isExprDefEqAux a₁ a₂ + postponedImplicit := postponedImplicit.push i + return .ok postponedImplicit postponedHO + +private partial def isDefEqArgs (f : Expr) (args₁ args₂ : Array Expr) : MetaM Bool := do + unless args₁.size == args₂.size do return false + let finfo ← getFunInfoNArgs f args₁.size + let .ok postponedImplicit postponedHO ← isDefEqArgsFirstPass finfo.paramInfo args₁ args₂ | pure false + -- finfo.paramInfo.size may be smaller than args₁.size + for i in [finfo.paramInfo.size:args₁.size] do + unless (← Meta.isExprDefEqAux args₁[i]! args₂[i]!) do + return false + for i in postponedImplicit do + /- Second pass: unify implicit arguments. + In the second pass, we make sure we are unfolding at + least non reducible definitions (default setting). -/ + let a₁ := args₁[i]! + let a₂ := args₂[i]! + let info := finfo.paramInfo[i]! + if info.isInstImplicit then + discard <| trySynthPending a₁ + discard <| trySynthPending a₂ + unless (← withAtLeastTransparency TransparencyMode.default <| Meta.isExprDefEqAux a₁ a₂) do + return false + for i in postponedHO do + let a₁ := args₁[i]! + let a₂ := args₂[i]! + let info := finfo.paramInfo[i]! + if info.isInstImplicit then + unless (← withAtLeastTransparency TransparencyMode.default <| Meta.isExprDefEqAux a₁ a₂) do + return false else - pure false - else - pure false + unless (← Meta.isExprDefEqAux a₁ a₂) do + return false + return true /-- Check whether the types of the free variables at `fvars` are @@ -250,7 +289,7 @@ private partial def isDefEqArgs (f : Expr) (args₁ args₂ : Array Expr) : Meta k loop 0 -/- Auxiliary function for `isDefEqBinding` for handling binders `forall/fun`. +/-- Auxiliary function for `isDefEqBinding` for handling binders `forall/fun`. It accumulates the new free variables in `fvars`, and declare them at `lctx`. We use the domain types of `e₁` to create the new free variables. We store the domain types of `e₂` at `ds₂`. -/ @@ -329,7 +368,7 @@ private partial def mkLambdaFVarsWithLetDeps (xs : Array Expr) (v : Expr) : Meta mkLambdaFVars ys v where - /- Return true if there are let-declarions between `xs[0]` and `xs[xs.size-1]`. + /-- Return true if there are let-declarions between `xs[0]` and `xs[xs.size-1]`. We use it a quick-check to avoid the more expensive collection procedure. -/ hasLetDeclsInBetween : MetaM Bool := do let check (lctx : LocalContext) : Bool := Id.run do @@ -347,7 +386,7 @@ where else return check (← getLCtx) - /- Traverse `e` and stores in the state `NameHashSet` any let-declaration with index greater than `(← read)`. + /-- Traverse `e` and stores in the state `NameHashSet` any let-declaration with index greater than `(← read)`. The context `Nat` is the position of `xs[0]` in the local context. -/ collectLetDeclsFrom (e : Expr) : ReaderT Nat (StateRefT FVarIdHashSet MetaM) Unit := do let rec visit (e : Expr) : MonadCacheT Expr Unit (ReaderT Nat (StateRefT FVarIdHashSet MetaM)) Unit := @@ -366,7 +405,7 @@ where | _ => pure () visit (← instantiateMVars e) |>.run - /- + /-- Auxiliary definition for traversing all declarations between `xs[0]` ... `xs.back` backwards. The `Nat` argument is the current position in the local context being visited, and it is less than or equal to the position of `xs.back` in the local context. @@ -388,7 +427,7 @@ where | _ => pure () collectLetDepsAux i - /- Computes the set `ys`. It is a set of `FVarId`s, -/ + /-- Computes the set `ys`. It is a set of `FVarId`s, -/ collectLetDeps : MetaM FVarIdHashSet := do let lctx ← getLCtx let start := lctx.getFVar! xs[0]! |>.index @@ -397,7 +436,7 @@ where let (_, s) ← collectLetDepsAux stop |>.run start |>.run s return s - /- Computes the array `ys` containing let-decls between `xs[0]` and `xs.back` that + /-- Computes the array `ys` containing let-decls between `xs[0]` and `xs.back` that some `x` in `xs` depends on. -/ addLetDeps : MetaM (Array Expr) := do let lctx ← getLCtx @@ -414,7 +453,7 @@ where ys := ys.push localDecl.toExpr return ys -/- +/-! Each metavariable is declared in a particular local context. We use the notation `C |- ?m : t` to denote a metavariable `?m` that was declared at the local context `C` with type `t` (see `MetavarDecl`). @@ -700,7 +739,7 @@ mutual traceM `Meta.isDefEq.assign.readOnlyMVarWithBiggerLCtx <| addAssignmentInfo (mkMVar mvarId) throwCheckAssignmentFailure - /- + /-- Auxiliary function used to "fix" subterms of the form `?m x_1 ... x_n` where `x_i`s are free variables, and one of them is out-of-scope. See `Expr.app` case at `check`. @@ -851,14 +890,15 @@ def checkAssignment (mvarId : MVarId) (fvars : Array Expr) (v : Expr) : MetaM (O private def processAssignmentFOApproxAux (mvar : Expr) (args : Array Expr) (v : Expr) : MetaM Bool := match v with + | .mdata _ e => processAssignmentFOApproxAux mvar args e | Expr.app f a => if args.isEmpty then pure false else Meta.isExprDefEqAux args.back a <&&> Meta.isExprDefEqAux (mkAppRange mvar 0 (args.size - 1) args) f - | _ => pure false + | _ => pure false -/- +/-- Auxiliary method for applying first-order unification. It is an approximation. Remark: this method is trying to solve the unification constraint: @@ -899,14 +939,14 @@ private partial def simpAssignmentArgAux : Expr → MetaM Expr | _ => pure e | e => pure e -/- Auxiliary procedure for processing `?m a₁ ... aₙ =?= v`. +/-- Auxiliary procedure for processing `?m a₁ ... aₙ =?= v`. We apply it to each `aᵢ`. It instantiates assigned metavariables if `aᵢ` is of the form `f[?n] b₁ ... bₘ`, and then removes metadata, and zeta-expand let-decls. -/ private def simpAssignmentArg (arg : Expr) : MetaM Expr := do let arg ← if arg.getAppFn.hasExprMVar then instantiateMVars arg else pure arg simpAssignmentArgAux arg -/- Assign `mvar := fun a_1 ... a_{numArgs} => v`. +/-- Assign `mvar := fun a_1 ... a_{numArgs} => v`. We use it at `processConstApprox` and `isDefEqMVarSelf` -/ private def assignConst (mvar : Expr) (numArgs : Nat) (v : Expr) : MetaM Bool := do let mvarDecl ← getMVarDecl mvar.mvarId! @@ -1294,15 +1334,6 @@ private def expandDelayedAssigned? (t : Expr) : MetaM (Option Expr) := do if tArgs.size < fvars.size then return none return some (mkAppRange (mkMVar mvarIdPending) fvars.size tArgs.size tArgs) -private def isSynthetic : Expr → MetaM Bool - | Expr.mvar mvarId => do - let mvarDecl ← getMVarDecl mvarId - match mvarDecl.kind with - | MetavarKind.synthetic => pure true - | MetavarKind.syntheticOpaque => pure true - | MetavarKind.natural => pure false - | _ => pure false - private def isAssignable : Expr → MetaM Bool | Expr.mvar mvarId => do let b ← isReadOnlyOrSyntheticOpaqueExprMVar mvarId; pure (!b) | _ => pure false @@ -1358,7 +1389,7 @@ private def isDefEqProofIrrel (t s : Expr) : MetaM LBool := do else pure LBool.undef -/- Try to solve constraint of the form `?m args₁ =?= ?m args₂`. +/-- Try to solve constraint of the form `?m args₁ =?= ?m args₂`. - First try to unify `args₁` and `args₂`, and return true if successful - Otherwise, try to assign `?m` to a constant function of the form `fun x_1 ... x_n => ?n` where `?n` is a fresh metavariable. See `assignConst`. -/ @@ -1380,7 +1411,7 @@ private def isDefEqMVarSelf (mvar : Expr) (args₁ args₂ : Array Expr) : MetaM else pure false -/- Remove unnecessary let-decls -/ +/-- Remove unnecessary let-decls -/ private def consumeLet : Expr → Expr | e@(Expr.letE _ _ _ b _) => if b.hasLooseBVars then e else consumeLet b | e => e @@ -1530,7 +1561,7 @@ private partial def isDefEqQuickOther (t s : Expr) : MetaM LBool := do else isDefEqQuickMVarMVar t s --- Both `t` and `s` are terms of the form `?m ...` +/-- Both `t` and `s` are terms of the form `?m ...` -/ private partial def isDefEqQuickMVarMVar (t s : Expr) : MetaM LBool := do if s.isMVar && !t.isMVar then /- Solve `?m t =?= ?n` by trying first `?n := ?m t`. @@ -1577,7 +1608,7 @@ private def isDefEqProj : Expr → Expr → MetaM Bool | v, Expr.proj structName 0 s => isDefEqSingleton structName s v | _, _ => pure false where - /- If `structName` is a structure with a single field and `(?m ...).1 =?= v`, then solve contraint as `?m ... =?= ⟨v⟩` -/ + /-- If `structName` is a structure with a single field and `(?m ...).1 =?= v`, then solve contraint as `?m ... =?= ⟨v⟩` -/ isDefEqSingleton (structName : Name) (s : Expr) (v : Expr) : MetaM Bool := do let ctorVal := getStructureCtor (← getEnv) structName if ctorVal.numFields != 1 then @@ -1596,7 +1627,7 @@ where else return false -/- +/-- Given applications `t` and `s` that are in WHNF (modulo the current transparency setting), check whether they are definitionally equal or not. -/ @@ -1625,7 +1656,7 @@ private def isDefEqUnitLike (t : Expr) (s : Expr) : MetaM Bool := do else return false -/- +/-- The `whnf` procedure has support for unfolding class projections when the transparency mode is set to `.instances`. This method ensures the behavior of `whnf` and `isDefEq` is consistent in this transparency mode. diff --git a/src/Lean/Meta/FunInfo.lean b/src/Lean/Meta/FunInfo.lean index e1a37d3b5405..9194fa7bd53f 100644 --- a/src/Lean/Meta/FunInfo.lean +++ b/src/Lean/Meta/FunInfo.lean @@ -9,9 +9,8 @@ import Lean.Meta.InferType namespace Lean.Meta @[inline] private def checkFunInfoCache (fn : Expr) (maxArgs? : Option Nat) (k : MetaM FunInfo) : MetaM FunInfo := do - let s ← get let t ← getTransparency - match s.cache.funInfo.find? ⟨t, fn, maxArgs?⟩ with + match (← get).cache.funInfo.find? ⟨t, fn, maxArgs?⟩ with | some finfo => pure finfo | none => do let finfo ← k @@ -57,21 +56,38 @@ private def getFunInfoAux (fn : Expr) (maxArgs? : Option Nat) : MetaM FunInfo := let fnType ← inferType fn withTransparency TransparencyMode.default do forallBoundedTelescope fnType maxArgs? fun fvars type => do - let mut pinfo := #[] + let mut paramInfo := #[] + let mut higherOrderOutParams : FVarIdSet := {} for i in [:fvars.size] do let fvar := fvars[i]! let decl ← getFVarLocalDecl fvar let backDeps := collectDeps fvars decl.type - pinfo := updateHasFwdDeps pinfo backDeps - pinfo := pinfo.push { - backDeps := backDeps - binderInfo := decl.binderInfo - isProp := (← isProp decl.type) - isDecInst := (← forallTelescopeReducing decl.type fun _ type => return type.isAppOf ``Decidable) + let dependsOnHigherOrderOutParam := + !higherOrderOutParams.isEmpty + && Option.isSome (decl.type.find? fun e => e.isFVar && higherOrderOutParams.contains e.fvarId!) + paramInfo := updateHasFwdDeps paramInfo backDeps + paramInfo := paramInfo.push { + backDeps, dependsOnHigherOrderOutParam + binderInfo := decl.binderInfo + isProp := (← isProp decl.type) + isDecInst := (← forallTelescopeReducing decl.type fun _ type => return type.isAppOf ``Decidable) } + if decl.binderInfo == .instImplicit then + /- Collect higher order output parameters of this class -/ + if let some className ← isClass? decl.type then + if let some outParamPositions := getOutParamPositions? (← getEnv) className then + unless outParamPositions.isEmpty do + let args := decl.type.getAppArgs + for i in [:args.size] do + if outParamPositions.contains i then + let arg := args[i]! + if let some idx := fvars.indexOf? arg then + if (← whnf (← inferType arg)).isForall then + paramInfo := paramInfo.modify idx fun info => { info with higherOrderOutParam := true } + higherOrderOutParams := higherOrderOutParams.insert arg.fvarId! let resultDeps := collectDeps fvars type - pinfo := updateHasFwdDeps pinfo resultDeps - pure { resultDeps := resultDeps, paramInfo := pinfo } + paramInfo := updateHasFwdDeps paramInfo resultDeps + return { resultDeps, paramInfo } def getFunInfo (fn : Expr) : MetaM FunInfo := getFunInfoAux fn none diff --git a/src/Lean/Meta/Inductive.lean b/src/Lean/Meta/Inductive.lean index 84e5a2c865db..25ba641af1e1 100644 --- a/src/Lean/Meta/Inductive.lean +++ b/src/Lean/Meta/Inductive.lean @@ -5,11 +5,11 @@ Authors: Leonardo de Moura -/ import Lean.Meta.Basic -/- Helper methods for inductive datatypes -/ +/-! # Helper methods for inductive datatypes -/ namespace Lean.Meta -/- Return true if the types of the given constructors are compatible. -/ +/-- Return true if the types of the given constructors are compatible. -/ def compatibleCtors (ctorName₁ ctorName₂ : Name) : MetaM Bool := do let ctorInfo₁ ← getConstInfoCtor ctorName₁ let ctorInfo₂ ← getConstInfoCtor ctorName₂ diff --git a/src/Lean/Meta/InferType.lean b/src/Lean/Meta/InferType.lean index 69b8f7db2cd4..d4336e7648ba 100644 --- a/src/Lean/Meta/InferType.lean +++ b/src/Lean/Meta/InferType.lean @@ -8,7 +8,7 @@ import Lean.Meta.Basic namespace Lean -/- +/-- Auxiliary function for instantiating the loose bound variables in `e` with `args[start:stop]`. This function is similar to `instantiateRevRange`, but it applies beta-reduction when we instantiate a bound variable with a lambda expression. @@ -145,7 +145,7 @@ private def inferForallType (e : Expr) : MetaM Expr := return mkLevelIMax' xTypeLvl lvl return mkSort lvl.normalize -/- Infer type of lambda and let expressions -/ +/-- Infer type of lambda and let expressions -/ private def inferLambdaType (e : Expr) : MetaM Expr := lambdaLetTelescope e fun xs e => do let type ← inferType e diff --git a/src/Lean/Meta/Instances.lean b/src/Lean/Meta/Instances.lean index 853895d3b7b8..ba760dd3cd23 100644 --- a/src/Lean/Meta/Instances.lean +++ b/src/Lean/Meta/Instances.lean @@ -81,7 +81,7 @@ def getGlobalInstancesIndex : CoreM (DiscrTree InstanceEntry) := def getErasedInstances : CoreM (Std.PHashSet Name) := return Meta.instanceExtension.getState (← getEnv) |>.erased -/- Default instance support -/ +/-! # Default instance support -/ structure DefaultInstanceEntry where className : Name diff --git a/src/Lean/Meta/Match/Basic.lean b/src/Lean/Meta/Match/Basic.lean index ed9fad00d416..c507a34813ca 100644 --- a/src/Lean/Meta/Match/Basic.lean +++ b/src/Lean/Meta/Match/Basic.lean @@ -65,7 +65,7 @@ where let fields ← fields.mapM visit pure $ mkAppN (mkConst ctorName us) (params ++ fields).toArray -/- Apply the free variable substitution `s` to the given pattern -/ +/-- Apply the free variable substitution `s` to the given pattern -/ partial def applyFVarSubst (s : FVarSubst) : Pattern → Pattern | inaccessible e => inaccessible $ s.apply e | ctor n us ps fs => ctor n us (ps.map s.apply) $ fs.map (applyFVarSubst s) @@ -157,7 +157,7 @@ def replaceFVarId (fvarId : FVarId) (v : Expr) (alt : Alt) : Alt := decls.map $ replaceFVarIdAtLocalDecl fvarId v, rhs := alt.rhs.replaceFVarId fvarId v } -/- +/-- Similar to `checkAndReplaceFVarId`, but ensures type of `v` is definitionally equal to type of `fvarId`. This extra check is necessary when performing dependent elimination and inaccessible terms have been used. For example, consider the following code fragment: diff --git a/src/Lean/Meta/Match/MVarRenaming.lean b/src/Lean/Meta/Match/MVarRenaming.lean index 0dc7ee9ca740..366ad65e34c1 100644 --- a/src/Lean/Meta/Match/MVarRenaming.lean +++ b/src/Lean/Meta/Match/MVarRenaming.lean @@ -7,7 +7,7 @@ import Lean.Util.ReplaceExpr namespace Lean.Meta -/- A mapping from MVarId to MVarId -/ +/-- A mapping from MVarId to MVarId -/ structure MVarRenaming where map : MVarIdMap MVarId := {} diff --git a/src/Lean/Meta/Match/Match.lean b/src/Lean/Meta/Match/Match.lean index b2ba02d2c82d..02bdc4c5d1ab 100644 --- a/src/Lean/Meta/Match/Match.lean +++ b/src/Lean/Meta/Match/Match.lean @@ -188,18 +188,18 @@ private def processAsPattern (p : Problem) : MetaM Problem := match alt.patterns with | Pattern.as fvarId p h :: ps => /- We used to use `checkAndReplaceFVarId` here, but `x` and `fvarId` may have different types - when dependent types are beind used. Let's consider the repro for issue #471 - ``` - inductive vec : Nat → Type - | nil : vec 0 - | cons : Int → vec n → vec n.succ - - def vec_len : vec n → Nat - | vec.nil => 0 - | x@(vec.cons h t) => vec_len t + 1 - - ``` - we reach the state + when dependent types are beind used. Let's consider the repro for issue #471 + ``` + inductive vec : Nat → Type + | nil : vec 0 + | cons : Int → vec n → vec n.succ + + def vec_len : vec n → Nat + | vec.nil => 0 + | x@(vec.cons h t) => vec_len t + 1 + + ``` + we reach the state ``` [Meta.Match.match] remaining variables: [x✝:(vec n✝)] alternatives: @@ -297,7 +297,7 @@ def assign (fvarId : FVarId) (v : Expr) : M Bool := do The first step is a variable-transition which replaces `β` with `β✝` in the first and third alternatives. The constraint `β✝ === α` in the second alternative is lost. Note that `α` is not an alternative variable. After applying the variable-transition step twice, we reach the following state - ``lean + ```lean [Meta.Match.match] remaining variables: [f✝:(Arrow β✝ γ✝), g✝:(Arrow α β✝)] alternatives: [g:(Arrow α β✝)] |- [(Arrow.id .(β✝)), g] => h_1 β✝ g @@ -392,7 +392,7 @@ private def hasRecursiveType (x : Expr) : MetaM Bool := do | some val => return val.isRec | _ => return false -/- Given `alt` s.t. the next pattern is an inaccessible pattern `e`, +/-- Given `alt` s.t. the next pattern is an inaccessible pattern `e`, try to normalize `e` into a constructor application. If it is not a constructor, throw an error. Otherwise, if it is a constructor application of `ctorName`, @@ -688,7 +688,7 @@ private def moveToFront (p : Problem) (i : Nat) : Problem := private partial def process (p : Problem) : StateRefT State MetaM Unit := search 0 where - /- If `p.vars` is empty, then we are done. Otherwise, we process `p.vars[0]`. -/ + /-- If `p.vars` is empty, then we are done. Otherwise, we process `p.vars[0]`. -/ tryToProcess (p : Problem) : StateRefT State MetaM Unit := withIncRecDepth do traceState p let isInductive ← isCurrVarInductive p @@ -727,7 +727,7 @@ where checkNextPatternTypes p throwNonSupported p - /- Return `true` if `type` does not depend on the first `i` elements in `xs` -/ + /-- Return `true` if `type` does not depend on the first `i` elements in `xs` -/ checkVarDeps (xs : List Expr) (i : Nat) (type : Expr) : MetaM Bool := do match i, xs with | 0, _ => return true @@ -787,7 +787,7 @@ register_builtin_option bootstrap.genMatcherCode : Bool := { builtin_initialize matcherExt : EnvExtension (Std.PHashMap (Expr × Bool) Name) ← registerEnvExtension (pure {}) -/- Similar to `mkAuxDefinition`, but uses the cache `matcherExt`. +/-- Similar to `mkAuxDefinition`, but uses the cache `matcherExt`. It also returns an Boolean that indicates whether a new matcher function was added to the environment or not. -/ def mkMatcherAuxDefinition (name : Name) (type : Expr) (value : Expr) : MetaM (Expr × Option (MatcherInfo → MetaM Unit)) := do trace[Meta.Match.debug] "{name} : {type} := {value}" @@ -985,7 +985,7 @@ def getMkMatcherInputInContext (matcherApp : MatcherApp) : MetaM MkMatcherInput return { matcherName, matchType, discrInfos := matcherInfo.discrInfos, lhss := lhss.toList } -/- This function is only used for testing purposes -/ +/-- This function is only used for testing purposes -/ def withMkMatcherInput (matcherName : Name) (k : MkMatcherInput → MetaM α) : MetaM α := do let some matcherInfo ← getMatcherInfo? matcherName | throwError "not a matcher: {matcherName}" let matcherConst ← getConstInfo matcherName @@ -998,7 +998,7 @@ def withMkMatcherInput (matcherName : Name) (k : MkMatcherInput → MetaM α) : end Match -/- Auxiliary function for MatcherApp.addArg -/ +/-- Auxiliary function for MatcherApp.addArg -/ private partial def updateAlts (typeNew : Expr) (altNumParams : Array Nat) (alts : Array Expr) (i : Nat) : MetaM (Array Nat × Array Expr) := do if h : i < alts.size then let alt := alts.get ⟨i, h⟩ @@ -1016,7 +1016,7 @@ private partial def updateAlts (typeNew : Expr) (altNumParams : Array Nat) (alts else return (altNumParams, alts) -/- Given +/-- Given - matcherApp `match_i As (fun xs => motive[xs]) discrs (fun ys_1 => (alt_1 : motive (C_1[ys_1])) ... (fun ys_n => (alt_n : motive (C_n[ys_n]) remaining`, and - expression `e : B[discrs]`, Construct the term diff --git a/src/Lean/Meta/Match/MatchEqsExt.lean b/src/Lean/Meta/Match/MatchEqsExt.lean index 6484dbc3b716..0fa05e6c2ce6 100644 --- a/src/Lean/Meta/Match/MatchEqsExt.lean +++ b/src/Lean/Meta/Match/MatchEqsExt.lean @@ -27,7 +27,7 @@ builtin_initialize matchEqnsExt : EnvExtension MatchEqnsExtState ← def registerMatchEqns (matchDeclName : Name) (matchEqns : MatchEqns) : CoreM Unit := modifyEnv fun env => matchEqnsExt.modifyState env fun s => { s with map := s.map.insert matchDeclName matchEqns } -/- +/-- Forward definition. We want to use `getEquationsFor` in the simplifier, `getEquationsFor` depends on `mkEquationsfor` which uses the simplifier. -/ @[extern "lean_get_match_equations_for"] diff --git a/src/Lean/Meta/MatchUtil.lean b/src/Lean/Meta/MatchUtil.lean index e8dcb817fdbb..06d1a924c49e 100644 --- a/src/Lean/Meta/MatchUtil.lean +++ b/src/Lean/Meta/MatchUtil.lean @@ -19,6 +19,7 @@ namespace Lean.Meta | none => p? (← whnf e) | s => return s +/-- Matches `e` with `lhs = (rhs : α)` and returns `(α, lhs, rhs)`. -/ def matchEq? (e : Expr) : MetaM (Option (Expr × Expr × Expr)) := matchHelper? e fun e => return Expr.eq? e diff --git a/src/Lean/Meta/Offset.lean b/src/Lean/Meta/Offset.lean index e3eb148cd243..71ecc0196a11 100644 --- a/src/Lean/Meta/Offset.lean +++ b/src/Lean/Meta/Offset.lean @@ -59,7 +59,7 @@ where failure | _ => failure -/- Quick function for converting `e` into `s + k` s.t. `e` is definitionally equal to `Nat.add s k`. -/ +/-- Quick function for converting `e` into `s + k` s.t. `e` is definitionally equal to `Nat.add s k`. -/ private partial def getOffsetAux : Expr → Bool → OptionT MetaM (Expr × Nat) | e@(Expr.app _ a), top => do let f := e.getAppFn diff --git a/src/Lean/Meta/PPGoal.lean b/src/Lean/Meta/PPGoal.lean index 8addf605b5cb..829255cec010 100644 --- a/src/Lean/Meta/PPGoal.lean +++ b/src/Lean/Meta/PPGoal.lean @@ -43,12 +43,12 @@ structure Context where abbrev M := ReaderT Context $ StateRefT State MetaM -/- Return true if `fvarId` is marked as an hidden inaccessible or inaccessible proposition -/ +/-- Return true if `fvarId` is marked as an hidden inaccessible or inaccessible proposition -/ def isMarked (fvarId : FVarId) : M Bool := do let s ← get return s.hiddenInaccessible.contains fvarId || s.hiddenInaccessibleProp.contains fvarId -/- If `fvarId` isMarked, then unmark it. -/ +/-- If `fvarId` isMarked, then unmark it. -/ def unmark (fvarId : FVarId) : M Unit := do modify fun s => { hiddenInaccessible := s.hiddenInaccessible.erase fvarId @@ -63,7 +63,7 @@ def moveToHiddeProp (fvarId : FVarId) : M Unit := do modified := true } -/- Return true if the given local declaration has a "visible dependency", that is, it contains +/-- Return true if the given local declaration has a "visible dependency", that is, it contains a free variable that is `hiddenInaccessible` Recall that hiddenInaccessibleProps are visible, only their names are hidden -/ @@ -71,14 +71,14 @@ def hasVisibleDep (localDecl : LocalDecl) : M Bool := do let s ← get findLocalDeclDependsOn localDecl (!s.hiddenInaccessible.contains ·) -/- Return true if the given local declaration has a "nonvisible dependency", that is, it contains +/-- Return true if the given local declaration has a "nonvisible dependency", that is, it contains a free variable that is `hiddenInaccessible` or `hiddenInaccessibleProp` -/ def hasInaccessibleNameDep (localDecl : LocalDecl) : M Bool := do let s ← get findLocalDeclDependsOn localDecl fun fvarId => s.hiddenInaccessible.contains fvarId || s.hiddenInaccessibleProp.contains fvarId -/- If `e` is visible, then any inaccessible in `e` marked as hidden should be unmarked. -/ +/-- If `e` is visible, then any inaccessible in `e` marked as hidden should be unmarked. -/ partial def visitVisibleExpr (e : Expr) : M Unit := do visit (← instantiateMVars e) |>.run where @@ -128,7 +128,7 @@ private def getInitialHiddenInaccessible (propOnly : Bool) : MetaM FVarIdSet := return r.insert localDecl.fvarId return r -/- +/-- If pp.inaccessibleNames == false, then collect two sets of `FVarId`s : `hiddenInaccessible` and `hiddenInaccessibleProp` 1- `hiddenInaccessible` contains `FVarId`s of free variables with inaccessible names that a) are not propositions or diff --git a/src/Lean/Meta/RecursorInfo.lean b/src/Lean/Meta/RecursorInfo.lean index bf790bf8993e..8b48ca96e654 100644 --- a/src/Lean/Meta/RecursorInfo.lean +++ b/src/Lean/Meta/RecursorInfo.lean @@ -107,7 +107,7 @@ private def checkMotive (declName : Name) (motive : Expr) (motiveArgs : Array Ex unless motive.isFVar && motiveArgs.all Expr.isFVar do throwError "invalid user defined recursor '{declName}', result type must be of the form (C t), where C is a bound variable, and t is a (possibly empty) sequence of bound variables" -/- Compute number of parameters for (user-defined) recursor. +/-- Compute number of parameters for (user-defined) recursor. We assume a parameter is anything that occurs before the motive -/ private partial def getNumParams (xs : Array Expr) (motive : Expr) (i : Nat) : Nat := if h : i < xs.size then diff --git a/src/Lean/Meta/SizeOf.lean b/src/Lean/Meta/SizeOf.lean index 3cb1d16864bd..fe00dcdb12d6 100644 --- a/src/Lean/Meta/SizeOf.lean +++ b/src/Lean/Meta/SizeOf.lean @@ -190,7 +190,7 @@ def mkSizeOfSpecLemmaInstance (ctorApp : Expr) : MetaM Expr := let lemmaArgMask := lemmaArgMask ++ ctorFields.toArray.map some mkAppOptM lemmaName lemmaArgMask -/- SizeOf spec theorem for nested inductive types -/ +/-! # SizeOf spec theorem for nested inductive types -/ namespace SizeOfSpecNested structure Context where @@ -259,13 +259,14 @@ mutual let sizeOfBaseArgs := lhsArgs[:lhsArgs.size - info.numIndices - 1] let indicesMajor := lhsArgs[lhsArgs.size - info.numIndices - 1:] let sizeOfLevels := lhs.getAppFn.constLevels! - /- Auxiliary function for constructing an `_sizeOf_` for `ys`, - where `ys` are the indices + major. - Recall that if `info.name` is part of a mutually inductive declaration, then the resulting application - is not necessarily a `lhs.getAppFn` application. - The result is an application of one of the `(← read),sizeOfFns` functions. - We use this auxiliary function to builtin the motive of the recursor. -/ - let rec mkSizeOf (ys : Array Expr) : M Expr := do + let rec + /-- Auxiliary function for constructing an `_sizeOf_` for `ys`, + where `ys` are the indices + major. + Recall that if `info.name` is part of a mutually inductive declaration, then the resulting application + is not necessarily a `lhs.getAppFn` application. + The result is an application of one of the `(← read),sizeOfFns` functions. + We use this auxiliary function to builtin the motive of the recursor. -/ + mkSizeOf (ys : Array Expr) : M Expr := do for sizeOfFn in (← read).sizeOfFns do let candidate := mkAppN (mkAppN (mkConst sizeOfFn sizeOfLevels) sizeOfBaseArgs) ys if (← isTypeCorrect candidate) then diff --git a/src/Lean/Meta/SynthInstance.lean b/src/Lean/Meta/SynthInstance.lean index fb49e5c73139..57d39fcdfc98 100644 --- a/src/Lean/Meta/SynthInstance.lean +++ b/src/Lean/Meta/SynthInstance.lean @@ -60,7 +60,7 @@ def Waiter.isRoot : Waiter → Bool | Waiter.consumerNode _ => false | Waiter.root => true -/- +/-! In tabled resolution, we creating a mapping from goals (e.g., `Coe Nat ?x`) to answers and waiters. Waiters are consumer nodes that are waiting for answers for a particular node. @@ -141,7 +141,7 @@ partial def normExpr (e : Expr) : M Expr := do end MkTableKey -/- Remark: `mkTableKey` assumes `e` does not contain assigned metavariables. -/ +/-- Remark: `mkTableKey` assumes `e` does not contain assigned metavariables. -/ def mkTableKey [Monad m] [MonadMCtx m] (e : Expr) : m Expr := do let (r, s) := MkTableKey.normExpr e |>.run { mctx := (← getMCtx) } setMCtx s.mctx @@ -161,7 +161,7 @@ structure Context where maxResultSize : Nat maxHeartbeats : Nat -/- +/-- Remark: the SynthInstance.State is not really an extension of `Meta.State`. The field `postponed` is not needed, and the field `mctx` is misleading since `synthInstance` methods operate over different `MetavarContext`s simultaneously. @@ -259,7 +259,7 @@ def mkTableKeyFor (mctx : MetavarContext) (mvar : Expr) : SynthM Expr := let mvarType ← instantiateMVars mvarType mkTableKey mvarType -/- See `getSubgoals` and `getSubgoalsAux` +/-- See `getSubgoals` and `getSubgoalsAux` We use the parameter `j` to reduce the number of `instantiate*` invocations. It is the same approach we use at `forallTelescope` and `lambdaTelescope`. @@ -597,7 +597,7 @@ def main (type : Expr) (maxResultSize : Nat) : MetaM (Option AbstractMVarsResult end SynthInstance -/- +/-! Type class parameters can be annotated with `outParam` annotations. Given `C a_1 ... a_n`, we replace `a_i` with a fresh metavariable `?m_i` IF @@ -656,7 +656,7 @@ private def preprocessOutParam (type : Expr) : MetaM Expr := | _ => return type -/- +/-! Remark: when `maxResultSize? == none`, the configuration option `synthInstance.maxResultSize` is used. Remark: we use a different option for controlling the maximum result size for coercions. -/ diff --git a/src/Lean/Meta/Tactic/Apply.lean b/src/Lean/Meta/Tactic/Apply.lean index b81c48b0d567..32d8dc69fd3f 100644 --- a/src/Lean/Meta/Tactic/Apply.lean +++ b/src/Lean/Meta/Tactic/Apply.lean @@ -10,7 +10,7 @@ import Lean.Meta.Tactic.Util namespace Lean.Meta -/- +/-- Compute the number of expected arguments and whether the result type is of the form (?m ...) where ?m is an unassigned metavariable. -/ diff --git a/src/Lean/Meta/Tactic/Cases.lean b/src/Lean/Meta/Tactic/Cases.lean index c4f3928078c6..d87d57864af5 100644 --- a/src/Lean/Meta/Tactic/Cases.lean +++ b/src/Lean/Meta/Tactic/Cases.lean @@ -155,7 +155,7 @@ private def mkCasesContext? (majorFVarId : FVarId) : MetaM (Option Context) := d } | _ => pure none -/- +/-- We say the major premise has independent indices IF 1- its type is *not* an indexed inductive family, OR 2- its type is an indexed inductive family, but all indices are distinct free variables, and @@ -187,7 +187,7 @@ private def elimAuxIndices (s₁ : GeneralizeIndicesSubgoal) (s₂ : Array Cases (pure s) | _ => pure s -/- +/-- Convert `s` into an array of `CasesSubgoal`, by attaching the corresponding constructor name, and adding the substitution `majorFVarId -> ctor_i us params fields` into each subgoal. -/ private def toCasesSubgoals (s : Array InductionSubgoal) (ctorNames : Array Name) (majorFVarId : FVarId) (us : List Level) (params : Array Expr) diff --git a/src/Lean/Meta/Tactic/Cleanup.lean b/src/Lean/Meta/Tactic/Cleanup.lean index 1eb8d4347842..4c7dc621ed32 100644 --- a/src/Lean/Meta/Tactic/Cleanup.lean +++ b/src/Lean/Meta/Tactic/Cleanup.lean @@ -44,7 +44,7 @@ where modify fun (_, s) => (true, s.insert fvarId) addDeps fvarId - /- We include `p` in the used-set, if `p` is a proposition that contains a `x` that is in the used-set. -/ + /-- We include `p` in the used-set, if `p` is a proposition that contains a `x` that is in the used-set. -/ collectPropsStep : StateRefT (Bool × FVarIdSet) MetaM Unit := do let usedSet := (← get).2 for localDecl in (← getLCtx) do diff --git a/src/Lean/Meta/Tactic/Constructor.lean b/src/Lean/Meta/Tactic/Constructor.lean index 29b6132866c8..93ab1236602e 100644 --- a/src/Lean/Meta/Tactic/Constructor.lean +++ b/src/Lean/Meta/Tactic/Constructor.lean @@ -9,7 +9,11 @@ import Lean.Meta.Tactic.Apply namespace Lean.Meta -def constructor (mvarId : MVarId) : MetaM (List MVarId) := do +/-- +When the goal `mvarId` is an inductive datatype, +`constructor` calls `apply` with the first matching constructor. +-/ +def constructor (mvarId : MVarId) (cfg : ApplyConfig := {}) : MetaM (List MVarId) := do withMVarContext mvarId do checkNotAssigned mvarId `constructor let target ← getMVarType' mvarId @@ -18,7 +22,7 @@ def constructor (mvarId : MVarId) : MetaM (List MVarId) := do fun ival us => do for ctor in ival.ctors do try - return ← apply mvarId (Lean.mkConst ctor us) + return ← apply mvarId (Lean.mkConst ctor us) cfg catch _ => pure () throwTacticEx `constructor mvarId "no applicable constructor found" diff --git a/src/Lean/Meta/Tactic/Delta.lean b/src/Lean/Meta/Tactic/Delta.lean index c231d88ecf9a..afd7ba82166c 100644 --- a/src/Lean/Meta/Tactic/Delta.lean +++ b/src/Lean/Meta/Tactic/Delta.lean @@ -16,7 +16,7 @@ def delta? (e : Expr) (p : Name → Bool := fun _ => true) : CoreM (Option Expr) else return none -/- Low-level delta expansion. It is used to implement equation lemmas and elimination principles for recursive definitions. -/ +/-- Low-level delta expansion. It is used to implement equation lemmas and elimination principles for recursive definitions. -/ def deltaExpand (e : Expr) (p : Name → Bool) : CoreM Expr := Core.transform e fun e => do match (← delta? e p) with diff --git a/src/Lean/Meta/Tactic/FVarSubst.lean b/src/Lean/Meta/Tactic/FVarSubst.lean index 9293126dd2f9..e502987efcc5 100644 --- a/src/Lean/Meta/Tactic/FVarSubst.lean +++ b/src/Lean/Meta/Tactic/FVarSubst.lean @@ -9,7 +9,7 @@ import Lean.LocalContext import Lean.Util.ReplaceExpr namespace Lean.Meta -/- +/-- Some tactics substitute hypotheses with expressions. We track these substitutions using `FVarSubst`. It is just a mapping from the original FVarId (internal) name @@ -29,7 +29,7 @@ def isEmpty (s : FVarSubst) : Bool := def contains (s : FVarSubst) (fvarId : FVarId) : Bool := s.map.contains fvarId -/- Add entry `fvarId |-> v` to `s` if `s` does not contain an entry for `fvarId`. -/ +/-- Add entry `fvarId |-> v` to `s` if `s` does not contain an entry for `fvarId`. -/ def insert (s : FVarSubst) (fvarId : FVarId) (v : Expr) : FVarSubst := if s.contains fvarId then s else diff --git a/src/Lean/Meta/Tactic/Intro.lean b/src/Lean/Meta/Tactic/Intro.lean index 1ebbee1c9f51..43c9e1cd4f9b 100644 --- a/src/Lean/Meta/Tactic/Intro.lean +++ b/src/Lean/Meta/Tactic/Intro.lean @@ -53,7 +53,7 @@ namespace Lean.Meta `whnf` instantiates metavariables, and consumes `MData`, but it also expands the `let`. -/ - let newType := (← instantiateMVars type).consumeMDataAndTypeAnnotations + let newType := (← instantiateMVars type).cleanupAnnotations if newType.isForall || newType.isLet then loop (i+1) lctx fvars fvars.size s newType else diff --git a/src/Lean/Meta/Tactic/Simp/Rewrite.lean b/src/Lean/Meta/Tactic/Simp/Rewrite.lean index 0384c3663e56..9a2bba2be438 100644 --- a/src/Lean/Meta/Tactic/Simp/Rewrite.lean +++ b/src/Lean/Meta/Tactic/Simp/Rewrite.lean @@ -123,7 +123,7 @@ def tryTheorem? (e : Expr) (thm : SimpTheorem) (discharge? : Expr → SimpM (Opt tryTheoremCore lhs xs bis val type e thm (eNumArgs - lhsNumArgs) discharge? else return none -/- +/-- Remark: the parameter tag is used for creating trace messages. It is irrelevant otherwise. -/ def rewrite? (e : Expr) (s : DiscrTree SimpTheorem) (erased : Std.PHashSet Name) (discharge? : Expr → SimpM (Option Expr)) (tag : String) (rflOnly : Bool) : SimpM (Option Result) := do diff --git a/src/Lean/Meta/Tactic/Simp/SimpTheorems.lean b/src/Lean/Meta/Tactic/Simp/SimpTheorems.lean index a4922676a255..783dc02c5477 100644 --- a/src/Lean/Meta/Tactic/Simp/SimpTheorems.lean +++ b/src/Lean/Meta/Tactic/Simp/SimpTheorems.lean @@ -333,7 +333,7 @@ def getSimpExtension? (attrName : Name) : IO (Option SimpExtension) := def getSimpTheorems : CoreM SimpTheorems := simpExtension.getTheorems -/- Auxiliary method for adding a global declaration to a `SimpTheorems` datastructure. -/ +/-- Auxiliary method for adding a global declaration to a `SimpTheorems` datastructure. -/ def SimpTheorems.addConst (s : SimpTheorems) (declName : Name) (post : Bool := true) (inv : Bool := false) (prio : Nat := eval_prio default) : MetaM SimpTheorems := do let s := { s with erased := s.erased.erase declName } let simpThms ← mkSimpTheoremsFromConst declName post inv prio @@ -356,12 +356,12 @@ private def preprocessProof (val : Expr) (inv : Bool) : MetaM (Array Expr) := do let ps ← preprocess val type inv (isGlobal := false) return ps.toArray.map fun (val, _) => val -/- Auxiliary method for creating simp theorems from a proof term `val`. -/ +/-- Auxiliary method for creating simp theorems from a proof term `val`. -/ def mkSimpTheorems (levelParams : Array Name) (proof : Expr) (post : Bool := true) (inv : Bool := false) (prio : Nat := eval_prio default) (name? : Option Name := none): MetaM (Array SimpTheorem) := withReducible do (← preprocessProof proof inv).mapM fun val => mkSimpTheoremCore val levelParams val post prio name? -/- Auxiliary method for adding a local simp theorem to a `SimpTheorems` datastructure. -/ +/-- Auxiliary method for adding a local simp theorem to a `SimpTheorems` datastructure. -/ def SimpTheorems.add (s : SimpTheorems) (levelParams : Array Name) (proof : Expr) (inv : Bool := false) (post : Bool := true) (prio : Nat := eval_prio default) (name? : Option Name := none): MetaM SimpTheorems := do if proof.isConst then s.addConst proof.constName! post inv prio diff --git a/src/Lean/Meta/Tactic/Split.lean b/src/Lean/Meta/Tactic/Split.lean index 64b5b923e501..3fd3ca6a9c97 100644 --- a/src/Lean/Meta/Tactic/Split.lean +++ b/src/Lean/Meta/Tactic/Split.lean @@ -152,7 +152,7 @@ private partial def generalizeMatchDiscrs (mvarId : MVarId) (matcherDeclName : N let (discrEqs, mvarId') ← introNP mvarId' discrs.size return (discrs', discrEqs, mvarId') where - /- + /-- - `eqs` are free variables `h_eq : discr = discrVar`. `eqs.size == discrs.size` - `altEqs` are free variables of the form `h_altEq : discr = pattern`. `altEqs.size = numDiscrEqs ≤ discrs.size` This method executes `k altEqsNew subst` where diff --git a/src/Lean/Meta/Tactic/UnifyEq.lean b/src/Lean/Meta/Tactic/UnifyEq.lean index 7e6234b29476..0dad193463d9 100644 --- a/src/Lean/Meta/Tactic/UnifyEq.lean +++ b/src/Lean/Meta/Tactic/UnifyEq.lean @@ -7,7 +7,7 @@ import Lean.Meta.Tactic.Injection namespace Lean.Meta -/- Convert heterogeneous equality into a homegeneous one -/ +/-- Convert heterogeneous equality into a homegeneous one -/ private def heqToEq' (mvarId : MVarId) (eqDecl : LocalDecl) : MetaM MVarId := do /- Convert heterogeneous equality into a homegeneous one -/ let prf ← mkEqOfHEq (mkFVar eqDecl.fvarId) diff --git a/src/Lean/Meta/WHNF.lean b/src/Lean/Meta/WHNF.lean index cdeb894d3c4f..db2066943be1 100644 --- a/src/Lean/Meta/WHNF.lean +++ b/src/Lean/Meta/WHNF.lean @@ -15,11 +15,11 @@ import Lean.Meta.Match.MatchPatternAttr namespace Lean.Meta -/- =========================== - Smart unfolding support - =========================== -/ +-- =========================== +/-! # Smart unfolding support -/ +-- =========================== -/- +/-- Forward declaration. It is defined in the module `src/Lean/Elab/PreDefinition/Structural/Eqns.lean`. It is possible to avoid this hack if we move `Structural.EqnInfo` and `Structural.eqnInfoExt` to this module. @@ -54,9 +54,10 @@ def markSmartUnfoldingMatchAlt (e : Expr) : Expr := def smartUnfoldingMatchAlt? (e : Expr) : Option Expr := annotation? `sunfoldMatchAlt e -/- =========================== - Helper methods - =========================== -/ +-- =========================== +/-! # Helper methods -/ +-- =========================== + def isAuxDef (constName : Name) : MetaM Bool := do let env ← getEnv return isAuxRecursor env constName || isNoConfusion env constName @@ -68,9 +69,9 @@ def isAuxDef (constName : Name) : MetaM Bool := do k cinfo lvls | _ => failK () -/- =========================== - Helper functions for reducing recursors - =========================== -/ +-- =========================== +/-! # Helper functions for reducing recursors -/ +-- =========================== private def getFirstCtor (d : Name) : MetaM (Option Name) := do let some (ConstantInfo.inductInfo { ctors := ctor::_, ..}) ← getConstNoEx? d | pure none @@ -195,9 +196,9 @@ private def reduceRec (recVal : RecursorVal) (recLvls : List Level) (recArgs : A else failK () -/- =========================== - Helper functions for reducing Quot.lift and Quot.ind - =========================== -/ +-- =========================== +/-! # Helper functions for reducing Quot.lift and Quot.ind -/ +-- =========================== /-- Auxiliary function for reducing `Quot.lift` and `Quot.ind` applications. -/ private def reduceQuotRec (recVal : QuotVal) (recLvls : List Level) (recArgs : Array Expr) (failK : Unit → MetaM α) (successK : Expr → MetaM α) : MetaM α := @@ -220,9 +221,9 @@ private def reduceQuotRec (recVal : QuotVal) (recLvls : List Level) (recArgs : | QuotKind.ind => process 4 3 | _ => failK () -/- =========================== - Helper function for extracting "stuck term" - =========================== -/ +-- =========================== +/-! # Helper function for extracting "stuck term" -/ +-- =========================== mutual private partial def isRecStuck? (recVal : RecursorVal) (recArgs : Array Expr) : MetaM (Option MVarId) := @@ -254,31 +255,30 @@ mutual /-- Return `some (Expr.mvar mvarId)` if metavariable `mvarId` is blocking reduction. -/ partial def getStuckMVar? (e : Expr) : MetaM (Option MVarId) := do match e with - | Expr.mdata _ e => getStuckMVar? e - | Expr.proj _ _ e => getStuckMVar? (← whnf e) - | Expr.mvar .. => do + | .mdata _ e => getStuckMVar? e + | .proj _ _ e => getStuckMVar? (← whnf e) + | .mvar .. => do let e ← instantiateMVars e match e with | Expr.mvar mvarId => pure (some mvarId) | _ => getStuckMVar? e - | Expr.app f .. => + | .app f .. => let f := f.getAppFn match f with - | Expr.mvar mvarId => return some mvarId - | Expr.const fName _ => - let cinfo? ← getConstNoEx? fName - match cinfo? with - | some $ ConstantInfo.recInfo recVal => isRecStuck? recVal e.getAppArgs - | some $ ConstantInfo.quotInfo recVal => isQuotRecStuck? recVal e.getAppArgs - | _ => return none - | Expr.proj _ _ e => getStuckMVar? (← whnf e) + | .mvar mvarId => return some mvarId + | .const fName _ => + match (← getConstNoEx? fName) with + | some <| .recInfo recVal => isRecStuck? recVal e.getAppArgs + | some <| .quotInfo recVal => isQuotRecStuck? recVal e.getAppArgs + | _ => return none + | .proj _ _ e => getStuckMVar? (← whnf e) | _ => return none | _ => return none end -/- =========================== - Weak Head Normal Form auxiliary combinators - =========================== -/ +-- =========================== +/-! # Weak Head Normal Form auxiliary combinators -/ +-- =========================== /-- Auxiliary combinator for handling easy WHNF cases. It takes a function for handling the "hard" cases as an argument -/ @[specialize] partial def whnfEasyCases (e : Expr) (k : Expr → MetaM Expr) : MetaM Expr := do diff --git a/src/Lean/MetavarContext.lean b/src/Lean/MetavarContext.lean index d32ea9e63310..9299d79c334c 100644 --- a/src/Lean/MetavarContext.lean +++ b/src/Lean/MetavarContext.lean @@ -8,7 +8,7 @@ import Lean.LocalContext namespace Lean -/- +/-! The metavariable context stores metavariable declarations and their assignments. It is used in the elaborator, tactic framework, unifier (aka `isDefEq`), and type class resolution (TC). First, we list all @@ -319,7 +319,7 @@ def getDelayedMVarAssignment? [Monad m] [MonadMCtx m] (mvarId : MVarId) : m (Opt markUsedAssignment return result? -/- Given a sequence of delayed assignments +/-- Given a sequence of delayed assignments ``` mvarId₁ := mvarId₂ ...; ... @@ -420,13 +420,19 @@ def hasAssignableMVar [Monad m] [MonadMCtx m] : Expr → m Bool def assignLevelMVar [MonadMCtx m] (mvarId : MVarId) (val : Level) : m Unit := modifyMCtx fun m => { m with lAssignment := m.lAssignment.insert mvarId val, usedAssignment := true } +/-- +Add `mvarId := x` to the metavariable assignment. +This method does not check whether `mvarId` is already assigned, nor it checks whether +a cycle is being introduced, or whether the expression has the right type. +This is a low-level API, and it is safer to use `isDefEq (mkMVar mvarId) x`. +-/ def assignExprMVar [MonadMCtx m] (mvarId : MVarId) (val : Expr) : m Unit := modifyMCtx fun m => { m with eAssignment := m.eAssignment.insert mvarId val, usedAssignment := true } def assignDelayedMVar [MonadMCtx m] (mvarId : MVarId) (fvars : Array Expr) (mvarIdPending : MVarId) : m Unit := modifyMCtx fun m => { m with dAssignment := m.dAssignment.insert mvarId { fvars, mvarIdPending }, usedAssignment := true } -/- +/-- Notes on artificial eta-expanded terms due to metavariables. We try avoid synthetic terms such as `((fun x y => t) a b)` in the output produced by the elaborator. This kind of term may be generated when instantiating metavariable assignments. @@ -705,7 +711,7 @@ instance : Inhabited MetavarContext := ⟨{}⟩ @[export lean_mk_metavar_ctx] def mkMetavarContext : Unit → MetavarContext := fun _ => {} -/- Low level API for adding/declaring metavariable declarations. +/-- Low level API for adding/declaring metavariable declarations. It is used to implement actions in the monads `MetaM`, `ElabM` and `TacticM`. It should not be used directly since the argument `(mvarId : MVarId)` is assumed to be "unique". -/ def addExprMVarDecl (mctx : MetavarContext) @@ -733,7 +739,7 @@ def addExprMVarDeclExp (mctx : MetavarContext) (mvarId : MVarId) (userName : Nam (type : Expr) (kind : MetavarKind) : MetavarContext := addExprMVarDecl mctx mvarId userName lctx localInstances type kind -/- Low level API for adding/declaring universe level metavariable declarations. +/-- Low level API for adding/declaring universe level metavariable declarations. It is used to implement actions in the monads `MetaM`, `ElabM` and `TacticM`. It should not be used directly since the argument `(mvarId : MVarId)` is assumed to be "unique". -/ def addLevelMVarDecl (mctx : MetavarContext) (mvarId : MVarId) : MetavarContext := @@ -770,7 +776,7 @@ def setMVarUserNameTemporarily (mctx : MetavarContext) (mvarId : MVarId) (userNa let decl := mctx.getDecl mvarId { mctx with decls := mctx.decls.insert mvarId { decl with userName := userName } } -/- Update the type of the given metavariable. This function assumes the new type is +/-- Update the type of the given metavariable. This function assumes the new type is definitionally equal to the current one -/ def setMVarType (mctx : MetavarContext) (mvarId : MVarId) (type : Expr) : MetavarContext := let decl := mctx.getDecl mvarId diff --git a/src/Lean/Modifiers.lean b/src/Lean/Modifiers.lean index 46000614ddab..3048be128021 100644 --- a/src/Lean/Modifiers.lean +++ b/src/Lean/Modifiers.lean @@ -17,7 +17,7 @@ def addProtected (env : Environment) (n : Name) : Environment := def isProtected (env : Environment) (n : Name) : Bool := protectedExt.isTagged env n -/- Private name support. +/-! # Private name support. Suppose the user marks as declaration `n` as private. Then, we create the name: `_private..0 ++ n`. diff --git a/src/Lean/MonadEnv.lean b/src/Lean/MonadEnv.lean index 7837c6ec3435..fce70f927196 100644 --- a/src/Lean/MonadEnv.lean +++ b/src/Lean/MonadEnv.lean @@ -138,7 +138,7 @@ def addDecl [Monad m] [MonadEnv m] [MonadError m] [MonadOptions m] [MonadLog m] private def supportedRecursors := #[``Empty.rec, ``False.rec, ``Eq.ndrec, ``Eq.rec, ``Eq.recOn, ``Eq.casesOn, ``False.casesOn, ``Empty.casesOn, ``And.rec, ``And.casesOn] -/- This is a temporary workaround for generating better error messages for the compiler. It can be deleted after we +/-- This is a temporary workaround for generating better error messages for the compiler. It can be deleted after we rewrite the remaining parts of the compiler in Lean. -/ private def checkUnsupported [Monad m] [MonadEnv m] [MonadError m] (decl : Declaration) : m Unit := do let env ← getEnv diff --git a/src/Lean/Parser/Attr.lean b/src/Lean/Parser/Attr.lean index 69785a09dc71..7d037d3325fa 100644 --- a/src/Lean/Parser/Attr.lean +++ b/src/Lean/Parser/Attr.lean @@ -33,11 +33,11 @@ end Priority namespace Attr @[builtinAttrParser] def simple := leading_parser ident >> optional (priorityParser <|> ident) -/- Remark, We can't use `simple` for `class`, `instance`, `export`, and `macro` because they are keywords. -/ +/- Remark, We can't use `simple` for `class`, `instance`, `export`, and `macro` because they are keywords. -/ @[builtinAttrParser] def «macro» := leading_parser "macro " >> ident @[builtinAttrParser] def «export» := leading_parser "export " >> ident -/- We don't use `simple` for recursor because the argument is not a priority-/ +/- We don't use `simple` for recursor because the argument is not a priority -/ @[builtinAttrParser] def recursor := leading_parser nonReservedSymbol "recursor " >> numLit @[builtinAttrParser] def «class» := leading_parser "class" @[builtinAttrParser] def «instance» := leading_parser "instance" >> optional priorityParser diff --git a/src/Lean/Parser/Basic.lean b/src/Lean/Parser/Basic.lean index d595ee7ed400..26a491ca80e6 100644 --- a/src/Lean/Parser/Basic.lean +++ b/src/Lean/Parser/Basic.lean @@ -74,11 +74,11 @@ abbrev mkAtom (info : SourceInfo) (val : String) : Syntax := abbrev mkIdent (info : SourceInfo) (rawVal : Substring) (val : Name) : Syntax := Syntax.ident info rawVal val [] -/- Return character after position `pos` -/ +/-- Return character after position `pos` -/ def getNext (input : String) (pos : String.Pos) : Char := input.get (input.next pos) -/- Maximal (and function application) precedence. +/-- Maximal (and function application) precedence. In the standard lean language, no parser has precedence higher than `maxPrec`. Note that nothing prevents users from using a higher precedence, but we strongly @@ -109,7 +109,7 @@ abbrev SyntaxNodeKindSet := Std.PersistentHashMap SyntaxNodeKind Unit def SyntaxNodeKindSet.insert (s : SyntaxNodeKindSet) (k : SyntaxNodeKind) : SyntaxNodeKindSet := Std.PersistentHashMap.insert s k () -/- +/-- Input string and related data. Recall that the `FileMap` is a helper structure for mapping `String.Pos` in the input string to line/column information. -/ structure InputContext where @@ -410,14 +410,14 @@ def errorAtSavedPosFn (msg : String) (delta : Bool) : ParserFn := fun c s => match s with | ⟨stack, lhsPrec, _, cache, _⟩ => ⟨stack.push Syntax.missing, lhsPrec, pos, cache, some { unexpected := msg }⟩ -/- Generate an error at the position saved with the `withPosition` combinator. +/-- Generate an error at the position saved with the `withPosition` combinator. If `delta == true`, then it reports at saved position+1. This useful to make sure a parser consumed at least one character. -/ @[inline] def errorAtSavedPos (msg : String) (delta : Bool) : Parser := { fn := errorAtSavedPosFn msg delta } -/- Succeeds if `c.prec <= prec` -/ +/-- Succeeds if `c.prec <= prec` -/ def checkPrecFn (prec : Nat) : ParserFn := fun c s => if c.prec <= prec then s else s.mkUnexpectedError "unexpected token at this precedence level; consider parenthesizing the term" @@ -427,7 +427,7 @@ def checkPrecFn (prec : Nat) : ParserFn := fun c s => fn := checkPrecFn prec } -/- Succeeds if `c.lhsPrec >= prec` -/ +/-- Succeeds if `c.lhsPrec >= prec` -/ def checkLhsPrecFn (prec : Nat) : ParserFn := fun _ s => if s.lhsPrec >= prec then s else s.mkUnexpectedError "unexpected token at this precedence level; consider parenthesizing the term" @@ -680,7 +680,7 @@ def sepBy1Fn (allowTrailingSep : Bool) (p : ParserFn) (sep : ParserFn) : ParserF fn := sepBy1Fn allowTrailingSep p.fn sep.fn } -/- Apply `f` to the syntax object produced by `p` -/ +/-- Apply `f` to the syntax object produced by `p` -/ def withResultOfFn (p : ParserFn) (f : Syntax → Syntax) : ParserFn := fun c s => let s := p c s if s.hasError then s @@ -745,7 +745,7 @@ partial def finishCommentBlock (nesting : Nat) : ParserFn := fun c s => where eoi s := s.mkUnexpectedError "unterminated comment" -/- Consume whitespace and comments -/ +/-- Consume whitespace and comments -/ partial def whitespace : ParserFn := fun c s => let input := c.input let i := s.pos @@ -1107,7 +1107,7 @@ def peekToken (c : ParserContext) (s : ParserState) : ParserState × Except Pars else peekTokenAux c s -/- Treat keywords as identifiers. -/ +/-- Treat keywords as identifiers. -/ def rawIdentFn : ParserFn := fun c s => let input := c.input let i := s.pos @@ -1561,26 +1561,12 @@ structure PrattParsingTables where instance : Inhabited PrattParsingTables := ⟨{}⟩ -/- +/-- The type `leadingIdentBehavior` specifies how the parsing table lookup function behaves for identifiers. The function `prattParser` uses two tables `leadingTable` and `trailingTable`. They map tokens to parsers. - - `LeadingIdentBehavior.default`: if the leading token - is an identifier, then `prattParser` just executes the parsers - associated with the auxiliary token "ident". - - - `LeadingIdentBehavior.symbol`: if the leading token is - an identifier ``, and there are parsers `P` associated with - the toek ``, then it executes `P`. Otherwise, it executes - only the parsers associated with the auxiliary token "ident". - - - `LeadingIdentBehavior.both`: if the leading token - an identifier ``, the it executes the parsers associated - with token `` and parsers associated with the auxiliary - token "ident". - We use `LeadingIdentBehavior.symbol` and `LeadingIdentBehavior.both` and `nonReservedSymbol` parser to implement the `tactic` parsers. The idea is to avoid creating a reserved symbol for each @@ -1588,11 +1574,21 @@ instance : Inhabited PrattParsingTables := ⟨{}⟩ may still use these symbols as identifiers (e.g., naming a function). -/ - inductive LeadingIdentBehavior where - | default - | symbol - | both + | /-- `LeadingIdentBehavior.default`: if the leading token + is an identifier, then `prattParser` just executes the parsers + associated with the auxiliary token "ident". -/ + default + | /-- `LeadingIdentBehavior.symbol`: if the leading token is + an identifier ``, and there are parsers `P` associated with + the toek ``, then it executes `P`. Otherwise, it executes + only the parsers associated with the auxiliary token "ident". -/ + symbol + | /-- `LeadingIdentBehavior.both`: if the leading token + an identifier ``, the it executes the parsers associated + with token `` and parsers associated with the auxiliary + token "ident". -/ + both deriving Inhabited, BEq, Repr /-- @@ -1661,9 +1657,9 @@ def categoryParser (catName : Name) (prec : Nat) : Parser := { @[inline] def termParser (prec : Nat := 0) : Parser := categoryParser `term prec -/- ============== -/ -/- Antiquotations -/ -/- ============== -/ +-- ================== +/-! # Antiquotations -/ +-- ================== /-- Fail if previous token is immediately followed by ':'. -/ def checkNoImmediateColon : Parser := { @@ -1796,9 +1792,9 @@ def withAntiquotSpliceAndSuffix (kind : SyntaxNodeKind) (p suffix : Parser) := def nodeWithAntiquot (name : String) (kind : SyntaxNodeKind) (p : Parser) (anonymous := false) : Parser := withAntiquot (mkAntiquot name kind anonymous) $ node kind p -/- ===================== -/ -/- End of Antiquotations -/ -/- ===================== -/ +-- ========================= +/-! # End of Antiquotations -/ +-- ========================= def sepByElemParser (p : Parser) (sep : String) : Parser := withAntiquotSpliceAndSuffix `sepBy p (symbol (sep.trim ++ "*")) diff --git a/src/Lean/Parser/Command.lean b/src/Lean/Parser/Command.lean index be0f7bcc2fb2..4d41c87f6899 100644 --- a/src/Lean/Parser/Command.lean +++ b/src/Lean/Parser/Command.lean @@ -132,12 +132,12 @@ def openDecl := openHiding <|> openRenaming <|> openOnly <|> openSimple @[builtinCommandParser] def «open» := leading_parser withPosition ("open " >> openDecl) @[builtinCommandParser] def «mutual» := leading_parser "mutual " >> many1 (ppLine >> notSymbol "end" >> commandParser) >> ppDedent (ppLine >> "end") >> terminationSuffix -@[builtinCommandParser] def «initialize» := leading_parser optional visibility >> "initialize " >> optional (atomic (ident >> Term.typeSpec >> Term.leftArrow)) >> Term.doSeq -@[builtinCommandParser] def «builtin_initialize» := leading_parser optional visibility >> "builtin_initialize " >> optional (atomic (ident >> Term.typeSpec >> Term.leftArrow)) >> Term.doSeq +def initializeKeyword := leading_parser "initialize " <|> "builtin_initialize " +@[builtinCommandParser] def «initialize» := leading_parser declModifiers false >> initializeKeyword >> optional (atomic (ident >> Term.typeSpec >> Term.leftArrow)) >> Term.doSeq @[builtinCommandParser] def «in» := trailing_parser withOpen (" in " >> commandParser) -/- +/-- This is an auxiliary command for generation constructor injectivity theorems for inductive types defined at `Prelude.lean`. It is meant for bootstrapping purposes only. -/ @[builtinCommandParser] def genInjectiveTheorems := leading_parser "gen_injective_theorems% " >> ident @@ -153,6 +153,7 @@ builtin_initialize register_parser_alias declVal register_parser_alias optDeclSig register_parser_alias openDecl + register_parser_alias docComment end Command diff --git a/src/Lean/Parser/Do.lean b/src/Lean/Parser/Do.lean index 3975b6b41666..fe662ee6fe42 100644 --- a/src/Lean/Parser/Do.lean +++ b/src/Lean/Parser/Do.lean @@ -50,7 +50,7 @@ def letIdDeclNoBinders := node `Lean.Parser.Term.letIdDecl $ atomic (ident >> pu @[builtinDoElemParser] def doReassign := leading_parser notFollowedByRedefinedTermToken >> (letIdDeclNoBinders <|> letPatDecl) @[builtinDoElemParser] def doReassignArrow := leading_parser notFollowedByRedefinedTermToken >> withPosition (doIdDecl <|> doPatDecl) @[builtinDoElemParser] def doHave := leading_parser "have " >> Term.haveDecl -/- +/-- In `do` blocks, we support `if` without an `else`. Thus, we use indentation to prevent examples such as ``` if c_1 then @@ -108,7 +108,7 @@ def doFinally := leading_parser "finally " >> doSeq @[builtinDoElemParser] def doDbgTrace := leading_parser:leadPrec "dbg_trace " >> ((interpolatedStr termParser) <|> termParser) @[builtinDoElemParser] def doAssert := leading_parser:leadPrec "assert! " >> termParser -/- +/-- We use `notFollowedBy` to avoid counterintuitive behavior. For example, the `if`-term parser diff --git a/src/Lean/Parser/Extension.lean b/src/Lean/Parser/Extension.lean index 9daeccd190d6..5472544f438d 100644 --- a/src/Lean/Parser/Extension.lean +++ b/src/Lean/Parser/Extension.lean @@ -164,7 +164,7 @@ def ParserExtension.addEntryImpl (s : State) (e : Entry) : State := | Except.ok categories => { s with categories := categories } | _ => unreachable! -/- Parser aliases for making `ParserDescr` extensible -/ +/-- Parser aliases for making `ParserDescr` extensible -/ inductive AliasValue (α : Type) where | const (p : α) | unary (p : α → α) @@ -294,7 +294,7 @@ def mkParserOfConstant (categories : ParserCategories) (constName : Name) : Impo mkParserOfConstantAux constName (compileParserDescr categories) structure ParserAttributeHook where - /- Called after a parser attribute is applied to a declaration. -/ + /-- Called after a parser attribute is applied to a declaration. -/ postAdd (catName : Name) (declName : Name) (builtin : Bool) : AttrM Unit builtin_initialize parserAttributeHooks : IO.Ref (List ParserAttributeHook) ← IO.mkRef {} @@ -358,7 +358,10 @@ def leadingIdentBehavior (env : Environment) (catName : Name) : LeadingIdentBeha unsafe def evalParserConstUnsafe (declName : Name) : ParserFn := fun ctx s => unsafeBaseIO do let categories := (parserExtension.getState ctx.env).categories match (← (mkParserOfConstant categories declName { env := ctx.env, opts := ctx.options }).toBaseIO) with - | .ok (_, p) => return p.fn ctx s + | .ok (_, p) => + -- We should manually register `p`'s tokens before invoking it as it might not be part of any syntax category (yet) + let ctx := { ctx with tokens := p.info.collectTokens [] |>.foldl (fun tks tk => tks.insert tk tk) ctx.tokens } + return p.fn ctx s | .error e => return s.mkUnexpectedError e.toString @[implementedBy evalParserConstUnsafe] @@ -448,7 +451,7 @@ def mkParserContext (ictx : InputContext) (pmctx : ParserModuleContext) : Parser def mkParserState (input : String) : ParserState := { cache := initCacheForInput input } -/- convenience function for testing -/ +/-- convenience function for testing -/ def runParserCategory (env : Environment) (catName : Name) (input : String) (fileName := "") : Except String Syntax := let c := mkParserContext (mkInputContext input fileName) { env := env, options := {} } let s := mkParserState input @@ -496,7 +499,7 @@ private def BuiltinParserAttribute.add (attrName : Name) (catName : Name) declareBuiltin (declName ++ `declRange) (mkAppN (mkConst ``addBuiltinDeclarationRanges) #[toExpr declName, toExpr declRanges]) runParserAttributeHooks catName declName (builtin := true) -/- +/-- The parsing tables for builtin parsers are "stored" in the extracted source code. -/ def registerBuiltinParserAttribute (attrName : Name) (catName : Name) (behavior := LeadingIdentBehavior.default) : IO Unit := do @@ -536,7 +539,7 @@ def mkParserAttributeImpl (attrName : Name) (catName : Name) : AttributeImpl whe add declName stx attrKind := ParserAttribute.add attrName catName declName stx attrKind applicationTime := AttributeApplicationTime.afterCompilation -/- A builtin parser attribute that can be extended by users. -/ +/-- A builtin parser attribute that can be extended by users. -/ def registerBuiltinDynamicParserAttribute (attrName : Name) (catName : Name) : IO Unit := do registerBuiltinAttribute (mkParserAttributeImpl attrName catName) diff --git a/src/Lean/Parser/Syntax.lean b/src/Lean/Parser/Syntax.lean index 1c44599a65bc..9eaddf7db810 100644 --- a/src/Lean/Parser/Syntax.lean +++ b/src/Lean/Parser/Syntax.lean @@ -69,7 +69,7 @@ def optKind : Parser := optional ("(" >> nonReservedSymbol "kind" >> ":=" >> ide def notationItem := ppSpace >> withAntiquot (mkAntiquot "notationItem" `Lean.Parser.Command.notationItem) (strLit <|> identPrec) @[builtinCommandParser] def «notation» := leading_parser Term.attrKind >> "notation" >> optPrecedence >> optNamedName >> optNamedPrio >> many notationItem >> darrow >> termParser @[builtinCommandParser] def «macro_rules» := suppressInsideQuot (leading_parser optional docComment >> Term.attrKind >> "macro_rules" >> optKind >> Term.matchAlts) -@[builtinCommandParser] def «syntax» := leading_parser optional docComment >> Term.attrKind >> "syntax " >> optPrecedence >> optNamedName >> optNamedPrio >> many1 (syntaxParser argPrec) >> " : " >> ident +@[builtinCommandParser] def «syntax» := leading_parser optional docComment >> optional (Term.«attributes») >> Term.attrKind >> "syntax " >> optPrecedence >> optNamedName >> optNamedPrio >> many1 (syntaxParser argPrec) >> " : " >> ident @[builtinCommandParser] def syntaxAbbrev := leading_parser optional docComment >> "syntax " >> ident >> " := " >> many1 syntaxParser def catBehaviorBoth := leading_parser nonReservedSymbol "both" def catBehaviorSymbol := leading_parser nonReservedSymbol "symbol" diff --git a/src/Lean/Parser/Term.lean b/src/Lean/Parser/Term.lean index 29ff0373ceaa..3154db96f3c8 100644 --- a/src/Lean/Parser/Term.lean +++ b/src/Lean/Parser/Term.lean @@ -38,7 +38,7 @@ def tacticSeqBracketed : Parser := def tacticSeq := leading_parser tacticSeqBracketed <|> tacticSeq1Indented -/- Raw sequence for quotation and grouping -/ +/-- Raw sequence for quotation and grouping -/ def seq1 := node `Lean.Parser.Tactic.seq1 $ sepBy1 tacticParser ";\n" (allowTrailingSep := true) @@ -49,7 +49,7 @@ def semicolonOrLinebreak := ";" <|> checkLinebreakBefore >> pushNone namespace Term -/- Built-in parsers -/ +/-! # Built-in parsers -/ @[builtinTermParser] def byTactic := leading_parser:leadPrec ppAllowUngrouped >> "by " >> Tactic.tacticSeq @@ -114,7 +114,7 @@ def instBinder := ppGroup $ leading_parser "[" >> optIdent >> termParser >> "]" def bracketedBinder (requireType := false) := withAntiquot (mkAntiquot "bracketedBinder" `Lean.Parser.Term.bracketedBinder (isPseudoKind := true)) <| explicitBinder requireType <|> strictImplicitBinder requireType <|> implicitBinder requireType <|> instBinder -/- +/-- It is feasible to support dependent arrows such as `{α} → α → α` without sacrificing the quality of the error messages for the longer case. `{α} → α → α` would be short for `{α : Type} → α → α` Here is the encoding: @@ -178,11 +178,11 @@ def withAnonymousAntiquot := leading_parser atomic ("(" >> nonReservedSymbol "wi @[builtinTermParser] def doubleQuotedName := leading_parser "`" >> checkNoWsBefore >> rawCh '`' (trailingWs := false) >> ident def letIdBinder := withAntiquot (mkAntiquot "letIdBinder" `Lean.Parser.Term.letIdBinder (isPseudoKind := true)) (binderIdent <|> bracketedBinder) -/- Remark: we use `checkWsBefore` to ensure `let x[i] := e; b` is not parsed as `let x [i] := e; b` where `[i]` is an `instBinder`. -/ +/-- Remark: we use `checkWsBefore` to ensure `let x[i] := e; b` is not parsed as `let x [i] := e; b` where `[i]` is an `instBinder`. -/ def letIdLhs : Parser := ident >> notFollowedBy (checkNoWsBefore "" >> "[") "space is required before instance '[...]' binders to distinguish them from array updates `let x[i] := e; ...`" >> many (ppSpace >> letIdBinder) >> optType def letIdDecl := leading_parser (withAnonymousAntiquot := false) atomic (letIdLhs >> " := ") >> termParser def letPatDecl := leading_parser (withAnonymousAntiquot := false) atomic (termParser >> pushNone >> optType >> " := ") >> termParser -/- +/-- Remark: the following `(" := " <|> matchAlts)` is a hack we use to produce a better error message at `letDecl`. Consider this following example ``` @@ -206,7 +206,7 @@ def letDecl := leading_parser (withAnonymousAntiquot := false) notFollowedBy instance : Coe (TSyntax ``letIdBinder) (TSyntax ``funBinder) where coe stx := ⟨stx⟩ --- like `let_fun` but with optional name +/-- like `let_fun` but with optional name -/ def haveIdLhs := optional (ident >> many (ppSpace >> letIdBinder)) >> optType def haveIdDecl := leading_parser (withAnonymousAntiquot := false) atomic (haveIdLhs >> " := ") >> termParser def haveEqnsDecl := leading_parser (withAnonymousAntiquot := false) haveIdLhs >> matchAlts diff --git a/src/Lean/PrettyPrinter.lean b/src/Lean/PrettyPrinter.lean index 297dc796a8a3..808532b07a92 100644 --- a/src/Lean/PrettyPrinter.lean +++ b/src/Lean/PrettyPrinter.lean @@ -20,10 +20,12 @@ def PPContext.runMetaM {α : Type} (ppCtx : PPContext) (x : MetaM α) : IO α := namespace PrettyPrinter -def ppTerm (stx : Term) : CoreM Format := do +def ppCategory (cat : Name) (stx : Syntax) : CoreM Format := do let opts ← getOptions let stx := (sanitizeSyntax stx).run' { options := opts } - parenthesizeTerm stx >>= formatTerm + parenthesizeCategory cat stx >>= formatCategory cat + +def ppTerm (stx : Term) : CoreM Format := ppCategory `term stx def ppUsing (e : Expr) (delab : Expr → MetaM Term) : MetaM Format := do let lctx := (← getLCtx).sanitizeNames.run' { options := (← getOptions) } @@ -50,11 +52,9 @@ def ppConst (e : Expr) : MetaM Format := do def ppExprLegacy (env : Environment) (mctx : MetavarContext) (lctx : LocalContext) (opts : Options) (e : Expr) : IO Format := Prod.fst <$> ((ppExpr e).run' { lctx := lctx } { mctx := mctx }).toIO { options := opts, fileName := "", fileMap := default } { env := env } -def ppTactic (stx : TSyntax `tactic) : CoreM Format := - parenthesizeTactic stx >>= formatTactic +def ppTactic (stx : TSyntax `tactic) : CoreM Format := ppCategory `tactic stx -def ppCommand (stx : Syntax.Command) : CoreM Format := - parenthesizeCommand stx >>= formatCommand +def ppCommand (stx : Syntax.Command) : CoreM Format := ppCategory `command stx def ppModule (stx : TSyntax ``Parser.Module.module) : CoreM Format := do parenthesize Lean.Parser.Module.module.parenthesizer stx >>= format Lean.Parser.Module.module.formatter diff --git a/src/Lean/PrettyPrinter/Formatter.lean b/src/Lean/PrettyPrinter/Formatter.lean index eaff61d972b6..50c1757f0c7d 100644 --- a/src/Lean/PrettyPrinter/Formatter.lean +++ b/src/Lean/PrettyPrinter/Formatter.lean @@ -530,7 +530,7 @@ def format (formatter : Formatter) (stx : Syntax) : CoreM Format := do pure $ Format.fill $ st.stack.get! 0) (fun _ => throwError "format: uncaught backtrack exception") -def formatCategory (cat : Name) := format $ categoryFormatter cat +def formatCategory (cat : Name) := format <| categoryFormatter cat def formatTerm := formatCategory `term def formatTactic := formatCategory `tactic diff --git a/src/Lean/PrettyPrinter/Parenthesizer.lean b/src/Lean/PrettyPrinter/Parenthesizer.lean index 15066a22056b..f40e94208ed4 100644 --- a/src/Lean/PrettyPrinter/Parenthesizer.lean +++ b/src/Lean/PrettyPrinter/Parenthesizer.lean @@ -533,9 +533,11 @@ def parenthesize (parenthesizer : Parenthesizer) (stx : Syntax) : CoreM Syntax : pure st.stxTrav.cur) (fun _ => throwError "parenthesize: uncaught backtrack exception") -def parenthesizeTerm := parenthesize $ categoryParser.parenthesizer `term 0 -def parenthesizeTactic := parenthesize $ categoryParser.parenthesizer `tactic 0 -def parenthesizeCommand := parenthesize $ categoryParser.parenthesizer `command 0 +def parenthesizeCategory (cat : Name) := parenthesize <| categoryParser.parenthesizer cat 0 + +def parenthesizeTerm := parenthesizeCategory `term +def parenthesizeTactic := parenthesizeCategory `tactic +def parenthesizeCommand := parenthesizeCategory `command builtin_initialize registerTraceClass `PrettyPrinter.parenthesize diff --git a/src/Lean/ProjFns.lean b/src/Lean/ProjFns.lean index 9f2f866ceaf1..0814a01ad877 100644 --- a/src/Lean/ProjFns.lean +++ b/src/Lean/ProjFns.lean @@ -7,7 +7,7 @@ import Lean.Environment namespace Lean -/- Given a structure `S`, Lean automatically creates an auxiliary definition (projection function) +/-- Given a structure `S`, Lean automatically creates an auxiliary definition (projection function) for each field. This structure caches information about these auxiliary definitions. -/ structure ProjectionFunctionInfo where ctorName : Name -- Constructor associated with the auxiliary projection function. diff --git a/src/Lean/ResolveName.lean b/src/Lean/ResolveName.lean index 624eb3ed7df1..abdbe3e026c9 100644 --- a/src/Lean/ResolveName.lean +++ b/src/Lean/ResolveName.lean @@ -29,14 +29,14 @@ builtin_initialize aliasExtension : SimplePersistentEnvExtension AliasEntry Alia addImportedFn := fun es => mkStateFromImportedEntries addAliasEntry {} es |>.switch } -/- Add alias `a` for `e` -/ +/-- Add alias `a` for `e` -/ @[export lean_add_alias] def addAlias (env : Environment) (a : Name) (e : Name) : Environment := aliasExtension.addEntry env (a, e) def getAliasState (env : Environment) : AliasState := aliasExtension.getState env -/- +/-- Retrieve aliases for `a`. If `skipProtected` is `true`, then the resulting list only includes declarations that are not marked as `proctected`. -/ @@ -53,10 +53,10 @@ def getAliases (env : Environment) (a : Name) (skipProtected : Bool) : List Name def getRevAliases (env : Environment) (e : Name) : List Name := (aliasExtension.getState env).fold (fun as a es => if List.contains es e then a :: as else as) [] -/- Global name resolution -/ +/-! # Global name resolution -/ namespace ResolveName -/- Check whether `ns ++ id` is a valid namepace name and/or there are aliases names `ns ++ id`. -/ +/-- Check whether `ns ++ id` is a valid namepace name and/or there are aliases names `ns ++ id`. -/ private def resolveQualifiedName (env : Environment) (ns : Name) (id : Name) : List Name := let resolvedId := ns ++ id -- We ignore protected aliases if `id` is atomic. @@ -69,7 +69,7 @@ private def resolveQualifiedName (env : Environment) (ns : Name) (id : Name) : L if env.contains resolvedIdPrv then resolvedIdPrv :: resolvedIds else resolvedIds -/- Check surrounding namespaces -/ +/-- Check surrounding namespaces -/ private def resolveUsingNamespace (env : Environment) (id : Name) : Name → List Name | ns@(.str p _) => match resolveQualifiedName env ns id with @@ -77,7 +77,7 @@ private def resolveUsingNamespace (env : Environment) (id : Name) : Name → Lis | resolvedIds => resolvedIds | _ => [] -/- Check exact name -/ +/-- Check exact name -/ private def resolveExact (env : Environment) (id : Name) : Option Name := if id.isAtomic then none else @@ -90,7 +90,7 @@ private def resolveExact (env : Environment) (id : Name) : Option Name := if env.contains resolvedIdPrv then some resolvedIdPrv else none -/- Check `OpenDecl`s -/ +/-- Check `OpenDecl`s -/ private def resolveOpenDecls (env : Environment) (id : Name) : List OpenDecl → List Name → List Name | [], resolvedIds => resolvedIds | OpenDecl.simple ns exs :: openDecls, resolvedIds => @@ -138,7 +138,7 @@ def resolveGlobalName (env : Environment) (ns : Name) (openDecls : List OpenDecl | _ => [] loop extractionResult.name [] -/- Namespace resolution -/ +/-! # Namespace resolution -/ def resolveNamespaceUsingScope? (env : Environment) (n : Name) : Name → Option Name | .anonymous => if env.isNamespace n then some n else none diff --git a/src/Lean/Server/Completion.lean b/src/Lean/Server/Completion.lean index 658ea76972dc..58359cd3adb0 100644 --- a/src/Lean/Server/Completion.lean +++ b/src/Lean/Server/Completion.lean @@ -166,7 +166,7 @@ private def matchDecl? (ns : Name) (id : Name) (danglingDot : Bool) (declName : else return none -/- +/-- Truncate the given identifier and make sure it has length `≤ newLength`. This function assumes `id` does not contain `Name.num` constructors. -/ diff --git a/src/Lean/Server/FileWorker.lean b/src/Lean/Server/FileWorker.lean index 4eac3db89fe6..330659e0bfee 100644 --- a/src/Lean/Server/FileWorker.lean +++ b/src/Lean/Server/FileWorker.lean @@ -65,7 +65,8 @@ structure WorkerContext where initParams : InitializeParams clientHasWidgets : Bool -/- Asynchronous snapshot elaboration. -/ +/-! # Asynchronous snapshot elaboration -/ + section Elab structure AsyncElabState where snaps : Array Snapshot diff --git a/src/Lean/Server/FileWorker/RequestHandling.lean b/src/Lean/Server/FileWorker/RequestHandling.lean index 25bbe32573fb..837af70f139f 100644 --- a/src/Lean/Server/FileWorker/RequestHandling.lean +++ b/src/Lean/Server/FileWorker/RequestHandling.lean @@ -259,18 +259,10 @@ open Parser.Command in partial def handleDocumentSymbol (_ : DocumentSymbolParams) : RequestM (RequestTask DocumentSymbolResult) := do let doc ← readDoc - mapTask (← doc.cmdSnaps.waitHead?) fun _ => do - let ⟨cmdSnaps, e?⟩ ← doc.cmdSnaps.getFinishedPrefix - let mut stxs := cmdSnaps.map (·.stx) - match e? with - | some ElabTaskError.aborted => - throw RequestError.fileChanged - | some (ElabTaskError.ioError e) => - throw (e : RequestError) - | _ => pure () - - let lastSnap := cmdSnaps.getLast! -- see `waitHead?` above - stxs := stxs ++ (← parseAhead doc.meta.mkInputContext lastSnap).toList + -- bad: we have to wait on elaboration of the entire file before we can report document symbols + let t ← doc.cmdSnaps.waitAll + mapTask t fun (snaps, _) => do + let mut stxs := snaps.map (·.stx) let (syms, _) := toDocumentSymbols doc.meta.text stxs return { syms := syms.toArray } where @@ -328,7 +320,8 @@ def noHighlightKinds : Array SyntaxNodeKind := #[ ``Lean.Parser.Term.prop, -- not really keywords `antiquotName, - ``Lean.Parser.Command.docComment] + ``Lean.Parser.Command.docComment, + ``Lean.Parser.Command.moduleDoc] structure SemanticTokensContext where beginPos : String.Pos diff --git a/src/Lean/Server/FileWorker/Utils.lean b/src/Lean/Server/FileWorker/Utils.lean index ef5996e91874..e065bd139206 100644 --- a/src/Lean/Server/FileWorker/Utils.lean +++ b/src/Lean/Server/FileWorker/Utils.lean @@ -50,7 +50,7 @@ and parser state after each command so that edits can be applied without recompiling code appearing earlier in the file. -/ structure EditableDocument where meta : DocumentMeta - /- State snapshots after header and each command. -/ + /-- State snapshots after header and each command. -/ cmdSnaps : AsyncList ElabTaskError Snapshot cancelTk : CancelToken diff --git a/src/Lean/Server/InfoUtils.lean b/src/Lean/Server/InfoUtils.lean index 099fe6d1c012..dc24e9318390 100644 --- a/src/Lean/Server/InfoUtils.lean +++ b/src/Lean/Server/InfoUtils.lean @@ -244,7 +244,7 @@ structure GoalsAtResult where -- for overlapping goals, only keep those of the highest reported priority priority : Nat -/- +/-- Try to retrieve `TacticInfo` for `hoverPos`. We retrieve all `TacticInfo` nodes s.t. `hoverPos` is inside the node's range plus trailing whitespace. We usually prefer the innermost such nodes so that for composite tactics such as `induction`, we show the nested proofs' states. diff --git a/src/Lean/Server/References.lean b/src/Lean/Server/References.lean index dc48abf3f669..078f51fee052 100644 --- a/src/Lean/Server/References.lean +++ b/src/Lean/Server/References.lean @@ -13,7 +13,7 @@ import Lean.Server.Utils import Lean.Server.InfoUtils import Lean.Server.Snapshots -/- Representing collected and deduplicated definitions and usages -/ +/-! # Representing collected and deduplicated definitions and usages -/ namespace Lean.Server open Lsp Lean.Elab Std @@ -127,7 +127,7 @@ def load (path : System.FilePath) : IO Ilean := do | Except.error msg => throwServerError s!"Failed to load ilean at {path}: {msg}" end Ilean -/- Collecting and deduplicating definitions and usages -/ +/-! # Collecting and deduplicating definitions and usages -/ def identOf : Info → Option (RefIdent × Bool) | Info.ofTermInfo ti => match ti.expr with @@ -178,13 +178,11 @@ partial def combineFvars (refs : Array Reference) : Array Reference := Id.run do let mut refs' := #[] for ref in refs do match ref with - | { ident := ident@(RefIdent.fvar id), isBinder, .. } => - if isBinder && idMap.contains id then - -- downgrade chained definitions to usages - -- (we shouldn't completely remove them in case they do not have usages) - refs' := refs'.push { ref with ident := applyIdMap idMap ident, isBinder := false, aliases := #[ident] } - else - refs' := refs'.push { ref with ident := applyIdMap idMap ident } + | { ident := ident@(RefIdent.fvar id), .. } => + if idMap.contains id then + refs' := refs'.push { ref with ident := applyIdMap idMap ident, aliases := #[ident] } + else if !idMap.contains id then + refs' := refs'.push ref | _ => refs' := refs'.push ref refs' @@ -198,27 +196,31 @@ where | m, RefIdent.fvar id => RefIdent.fvar <| findCanonicalBinder m id | _, ident => ident -def dedupReferences (refs : Array Reference) : Array Reference := Id.run do - let mut refsByIdAndRange : HashMap (RefIdent × Lsp.Range) Reference := HashMap.empty +def dedupReferences (refs : Array Reference) (allowSimultaneousBinderUse := false) : Array Reference := Id.run do + let mut refsByIdAndRange : HashMap (RefIdent × Option Bool × Lsp.Range) Reference := HashMap.empty for ref in refs do - let key := (ref.ident, ref.range) + let isBinder := if allowSimultaneousBinderUse then some ref.isBinder else none + let key := (ref.ident, isBinder, ref.range) refsByIdAndRange := match refsByIdAndRange[key] with - | some ref' => refsByIdAndRange.insert key { ref' with isBinder := ref'.isBinder || ref.isBinder, aliases := ref'.aliases ++ ref.aliases } + | some ref' => refsByIdAndRange.insert key { ref' with aliases := ref'.aliases ++ ref.aliases } | none => refsByIdAndRange.insert key ref let dedupedRefs := refsByIdAndRange.fold (init := #[]) fun refs _ ref => refs.push ref return dedupedRefs.qsort (·.range < ·.range) def findModuleRefs (text : FileMap) (trees : Array InfoTree) (localVars : Bool := true) - : ModuleRefs := Id.run do - let mut refs := dedupReferences <| combineFvars <| findReferences text trees + (allowSimultaneousBinderUse := false) : ModuleRefs := Id.run do + let mut refs := + dedupReferences (allowSimultaneousBinderUse := allowSimultaneousBinderUse) <| + combineFvars <| + findReferences text trees if !localVars then refs := refs.filter fun | { ident := RefIdent.fvar _, .. } => false | _ => true refs.foldl (init := HashMap.empty) fun m ref => m.addRef ref -/- Collecting and maintaining reference info from different sources -/ +/-! # Collecting and maintaining reference info from different sources -/ structure References where /-- References loaded from ilean files -/ diff --git a/src/Lean/Server/Requests.lean b/src/Lean/Server/Requests.lean index 575cb3223807..b9a84ecf6509 100644 --- a/src/Lean/Server/Requests.lean +++ b/src/Lean/Server/Requests.lean @@ -122,7 +122,7 @@ def bindWaitFindSnap (doc : EditableDocument) (p : Snapshot → Bool) end RequestM -/- The global request handlers table. -/ +/-! # The global request handlers table -/ section HandlerTable open Lsp @@ -133,7 +133,7 @@ structure RequestHandler where builtin_initialize requestHandlers : IO.Ref (Std.PersistentHashMap String RequestHandler) ← IO.mkRef {} -/-- NB: This method may only be called in `builtin_initialize` blocks. +/-- NB: This method may only be called in `initialize` blocks (user or builtin). A registration consists of: - a type of JSON-parsable request data `paramType` @@ -149,7 +149,7 @@ def registerLspRequestHandler (method : String) paramType [FromJson paramType] [FileSource paramType] respType [ToJson respType] (handler : paramType → RequestM (RequestTask respType)) : IO Unit := do - if !(← IO.initializing) then + if !(← Lean.initializing) then throw <| IO.userError s!"Failed to register LSP request handler for '{method}': only possible during initialization" if (← requestHandlers.get).contains method then throw <| IO.userError s!"Failed to register LSP request handler for '{method}': already registered" @@ -165,7 +165,7 @@ def registerLspRequestHandler (method : String) def lookupLspRequestHandler (method : String) : IO (Option RequestHandler) := return (← requestHandlers.get).find? method -/-- NB: This method may only be called in `builtin_initialize` blocks. +/-- NB: This method may only be called in `initialize` blocks (user or builtin). Register another handler to invoke after the last one registered for a method. At least one handler for the method must have already been registered to perform @@ -176,7 +176,7 @@ def chainLspRequestHandler (method : String) paramType [FromJson paramType] respType [FromJson respType] [ToJson respType] (handler : paramType → RequestTask respType → RequestM (RequestTask respType)) : IO Unit := do - if !(← IO.initializing) then + if !(← Lean.initializing) then throw <| IO.userError s!"Failed to chain LSP request handler for '{method}': only possible during initialization" if let some oldHandler ← lookupLspRequestHandler method then let handle := fun j => do diff --git a/src/Lean/Server/Rpc/Basic.lean b/src/Lean/Server/Rpc/Basic.lean index 1d1c5f93c0a5..b0e451048126 100644 --- a/src/Lean/Server/Rpc/Basic.lean +++ b/src/Lean/Server/Rpc/Basic.lean @@ -42,10 +42,13 @@ non-JSON-serializable fields can be auto-encoded in two ways: -- TODO(WN): for Lean.js, have third parameter defining the client-side structure; -- or, compile `WithRpcRef` to "opaque reference" on the client class RpcEncoding (α : Type) (β : outParam Type) where - rpcEncode {m : Type → Type} [Monad m] [MonadRpcSession m] : α → m β + rpcEncode {m : Type → Type} [Monad m] [MonadRpcSession m] : α → ExceptT String m β rpcDecode {m : Type → Type} [Monad m] [MonadRpcSession m] : β → ExceptT String m α export RpcEncoding (rpcEncode rpcDecode) +instance : Nonempty (RpcEncoding α β) := + ⟨{ rpcEncode := fun _ => throw "unreachable", rpcDecode := fun _ => throw "unreachable" }⟩ + instance [FromJson α] [ToJson α] : RpcEncoding α α where rpcEncode := pure rpcDecode := pure diff --git a/src/Lean/Server/Rpc/Deriving.lean b/src/Lean/Server/Rpc/Deriving.lean index c106b84d0747..8ad3231d0797 100644 --- a/src/Lean/Server/Rpc/Deriving.lean +++ b/src/Lean/Server/Rpc/Deriving.lean @@ -20,26 +20,14 @@ private def deriveWithRefInstance (typeNm : Name) : CommandElabM Bool := do -- TODO(WN): check that `typeNm` is not a scalar type let typeId := mkIdent typeNm let cmds ← `( - section - variable {m : Type → Type} - unsafe def encodeUnsafe [Monad m] [MonadRpcSession m] (r : WithRpcRef $typeId:ident) : m Lsp.RpcRef := - WithRpcRef.encodeUnsafe $(quote typeNm) r - - @[implementedBy encodeUnsafe] - opaque encode [Monad m] [MonadRpcSession m] (r : WithRpcRef $typeId:ident) : m Lsp.RpcRef := - pure ⟨0⟩ - - unsafe def decodeUnsafe [Monad m] [MonadRpcSession m] (r : Lsp.RpcRef) : ExceptT String m (WithRpcRef $typeId:ident) := - WithRpcRef.decodeUnsafeAs $typeId:ident $(quote typeNm) r - - @[implementedBy decodeUnsafe] - opaque decode [Monad m] [MonadRpcSession m] (r : Lsp.RpcRef) : ExceptT String m (WithRpcRef $typeId:ident) := - throw "unreachable" - - instance : RpcEncoding (WithRpcRef $typeId:ident) Lsp.RpcRef := - { rpcEncode := encode - rpcDecode := decode } - end + unsafe def unsafeInst : RpcEncoding (WithRpcRef $typeId:ident) Lsp.RpcRef where + rpcEncode := WithRpcRef.encodeUnsafe $(quote typeNm) + rpcDecode := WithRpcRef.decodeUnsafeAs $typeId:ident $(quote typeNm) + + @[implementedBy unsafeInst] + opaque inst : RpcEncoding (WithRpcRef $typeId) Lsp.RpcRef + + instance : RpcEncoding (WithRpcRef $typeId) Lsp.RpcRef := inst ) elabCommand cmds return true @@ -85,45 +73,27 @@ def withFieldsFlattened (indVal : InductiveVal) (params : Array Expr) end -def isOptField (n : Name) : Bool := - n.toString.endsWith "?" +private def getRpcPacketFor (ty : Expr) : MetaM Expr := do + let packetTy ← mkFreshExprMVar (Expr.sort levelOne) + let _ ← synthInstance (mkApp2 (mkConst ``RpcEncoding) ty packetTy) + instantiateMVars packetTy -private def deriveStructureInstance (indVal : InductiveVal) (params : Array Expr) : TermElabM Command := +private def deriveStructureInstance (indVal : InductiveVal) (params : Array Expr) + (paramBinders packetParamBinders encInstBinders : Array (TSyntax ``Parser.Term.bracketedBinder)) : TermElabM Command := do withFields indVal params fun fields => do trace[Elab.Deriving.RpcEncoding] "for structure {indVal.name} with params {params}" - -- Postulate that every field have a rpc encoding, storing the encoding type ident - -- in `fieldEncIds`. When multiple fields have the same type, we reuse the encoding type - -- as otherwise typeclass synthesis fails. let mut binders := #[] let mut fieldIds := #[] - let mut fieldEncIds : Array Term := #[] - let mut uniqFieldEncIds : Array Ident := #[] - let mut fieldEncIds' : DiscrTree Ident := {} + let mut fieldEncTypeStxs := #[] for (fieldName, fieldTp) in fields do let mut fieldTp := fieldTp - if isOptField fieldName then - if !fieldTp.isAppOf ``Option then - throwError "optional field '{fieldName}' has type{indentD m!"{fieldTp}"}\nbut is expected to have type{indentD "Option _"}" --" - fieldTp := fieldTp.getArg! 0 - -- postulate that the field has an encoding and remember the encoding's binder name + let fieldEncTypeStx ← PrettyPrinter.delab (← getRpcPacketFor fieldTp) + let stx ← PrettyPrinter.delab fieldTp fieldIds := fieldIds.push <| mkIdent fieldName - let mut fieldEncId : Ident := ⟨Syntax.missing⟩ - match (← fieldEncIds'.getMatch fieldTp).back? with - | none => - fieldEncId ← mkIdent <$> mkFreshUserName fieldName - binders := binders.push (← `(bracketedBinder| ( $fieldEncId:ident ))) - let stx ← PrettyPrinter.delab fieldTp - binders := binders.push - (← `(bracketedBinder| [ $(mkIdent ``Lean.Server.RpcEncoding) $stx $fieldEncId:ident ])) - fieldEncIds' ← fieldEncIds'.insert fieldTp fieldEncId - uniqFieldEncIds := uniqFieldEncIds.push fieldEncId - | some fid => fieldEncId := fid - - if isOptField fieldName then - fieldEncIds := fieldEncIds.push <| ← ``(Option $fieldEncId:ident) - else - fieldEncIds := fieldEncIds.push fieldEncId + fieldEncTypeStxs := fieldEncTypeStxs.push fieldEncTypeStx + binders := binders.push + (← `(bracketedBinder| [ RpcEncoding $stx $fieldEncTypeStx ])) -- helpers for field initialization syntax let fieldInits (func : Name) := fieldIds.mapM fun fid => @@ -134,115 +104,88 @@ private def deriveStructureInstance (indVal : InductiveVal) (params : Array Expr -- helpers for type name syntax let paramIds ← params.mapM fun p => return mkIdent (← getFVarLocalDecl p).userName let typeId := Syntax.mkApp (← `(@$(mkIdent indVal.name))) paramIds - let packetId ← mkIdent <$> mkFreshUserName `RpcEncodingPacket - let packetAppliedId := Syntax.mkApp packetId uniqFieldEncIds - - `(variable $binders* - - structure $packetId:ident where - $[($fieldIds : $fieldEncIds)]* - deriving $(mkIdent ``FromJson), $(mkIdent ``ToJson) - - instance : $(mkIdent ``RpcEncoding) $typeId $packetAppliedId where - rpcEncode a := return { - $[$encInits],* - } - rpcDecode a := return { - $[$decInits],* - } + let instId := mkIdent (`_root_ ++ indVal.name.appendBefore "instRpcEncoding") + + `(variable $packetParamBinders* in + structure RpcEncodingPacket where + $[($fieldIds : $fieldEncTypeStxs)]* + deriving FromJson, ToJson + + variable $(paramBinders ++ packetParamBinders ++ encInstBinders)* in + @[instance] def $instId := show RpcEncoding $typeId (RpcEncodingPacket ..) from { + rpcEncode := fun a => return { $[$encInits],* } + rpcDecode := fun a => return { $[$decInits],* } + } ) private structure CtorState where - -- names of encoded argument types in the RPC packet - encArgTypes : DiscrTree Name := {} - uniqEncArgTypes : Array Name := #[] - -- binders for `encArgTypes` as well as the relevant `RpcEncoding`s - binders : Array (TSyntax ``Parser.Term.bracketedBinder) := #[] -- the syntax of each constructor in the packet ctors : Array (TSyntax ``Parser.Command.ctor) := #[] -- syntax of each arm of the `rpcEncode` pattern-match encodes : Array (TSyntax ``Parser.Term.matchAlt) := #[] -- syntax of each arm of the `rpcDecode` pattern-match decodes : Array (TSyntax ``Parser.Term.matchAlt) := #[] - deriving Inhabited private def matchF := Lean.Parser.Term.matchAlt (rhsParser := Lean.Parser.termParser) -private def deriveInductiveInstance (indVal : InductiveVal) (params : Array Expr) : TermElabM Command := do +private def deriveInductiveInstance (indVal : InductiveVal) (params : Array Expr) + (paramBinders packetParamBinders encInstBinders : Array (TSyntax ``Parser.Term.bracketedBinder)) : TermElabM Command := do trace[Elab.Deriving.RpcEncoding] "for inductive {indVal.name} with params {params}" - - -- produce all encoding types and binders for them - let st ← foldWithConstructors indVal params (init := { : CtorState}) fun acc ctor argVars tp => do - trace[Elab.Deriving.RpcEncoding] "{ctor} : {argVars} → {tp}" - let mut acc := acc - let argFVars ← argVars.mapM (LocalDecl.fvarId <$> getFVarLocalDecl ·) - for arg in argVars do - let argTp ← inferType arg - if (← findExprDependsOn argTp (pf := fun fv => argFVars.contains fv)) then - throwError "cross-argument dependencies are not supported ({arg} : {argTp})" - - if (← acc.encArgTypes.getMatch argTp).isEmpty then - let tid ← mkFreshUserName `_rpcEnc - let argTpStx ← PrettyPrinter.delab argTp - acc := { acc with encArgTypes := ← acc.encArgTypes.insert argTp tid - uniqEncArgTypes := acc.uniqEncArgTypes.push tid - binders := acc.binders.append #[ - (← `(bracketedBinder| ( $(mkIdent tid):ident ))), - (← `(bracketedBinder| [ $(mkIdent ``Lean.Server.RpcEncoding) $argTpStx $(mkIdent tid):ident ])) - ] } - return acc - - -- introduce encoding types into the local context so that we can use the delaborator to print them - withLocalDecls - (st.uniqEncArgTypes.map fun tid => (tid, BinderInfo.default, fun _ => pure <| mkSort levelOne)) - fun ts => do - trace[Elab.Deriving.RpcEncoding] m!"RpcEncoding type binders : {ts}" - - let packetNm ← mkFreshUserName `RpcEncodingPacket - let st ← foldWithConstructors indVal params (init := st) fun acc ctor argVars _ => do - -- create the constructor - let mut pktCtorTp := Lean.mkConst packetNm - for arg in argVars.reverse do - let argTp ← inferType arg - let encTpNm := (← acc.encArgTypes.getMatch argTp).back - let encTp ← elabTerm (mkIdent encTpNm) none - pktCtorTp := mkForall (← getFVarLocalDecl arg).userName BinderInfo.default encTp pktCtorTp - -- TODO(WN): this relies on delab printing non-macro-scoped user names in non-dependent foralls - -- to generate the expected JSON encoding - let pktCtorTpStx ← PrettyPrinter.delab pktCtorTp - let pktCtor ← `(Lean.Parser.Command.ctor| | $(mkIdent ctor.getString!):ident : $pktCtorTpStx:term) - - -- create encoder and decoder match arms - let nms ← argVars.mapM fun _ => mkIdent <$> mkFreshBinderName - let mkPattern (src : Name) := Syntax.mkApp (mkIdent <| Name.mkStr src ctor.getString!) nms - let mkBody (tgt : Name) (func : Name) : TermElabM Term := do - let items ← nms.mapM fun nm => `(← $(mkIdent func) $nm) - let tm := Syntax.mkApp (mkIdent <| Name.mkStr tgt ctor.getString!) items - `(return $tm:term) - - let encArm ← `(matchF| | $(mkPattern indVal.name):term => $(← mkBody packetNm ``rpcEncode)) - let decArm ← `(matchF| | $(mkPattern packetNm):term => $(← mkBody indVal.name ``rpcDecode)) - - return { acc with ctors := acc.ctors.push pktCtor - encodes := acc.encodes.push ⟨encArm⟩ - decodes := acc.decodes.push ⟨decArm⟩ } - - -- helpers for type name syntax - let paramIds ← params.mapM fun p => return mkIdent (← getFVarLocalDecl p).userName - let typeId := Syntax.mkApp (← `(@$(mkIdent indVal.name))) paramIds - let packetAppliedId := Syntax.mkApp (mkIdent packetNm) (st.uniqEncArgTypes.map (mkIdent ·)) - - `(variable $st.binders* - - inductive $(mkIdent packetNm) where - $[$(st.ctors):ctor]* - deriving $(mkIdent ``FromJson), $(mkIdent ``ToJson) - - instance : $(mkIdent ``RpcEncoding) $typeId $packetAppliedId where - rpcEncode := fun x => match x with - $[$(st.encodes):matchAlt]* - rpcDecode := fun x => match x with - $[$(st.decodes):matchAlt]* - ) + withoutModifyingEnv do + let packetNm := (← `(RpcEncodingPacket)).1.getId + addDecl <| .axiomDecl { + name := packetNm + levelParams := [] + type := mkSort levelOne + isUnsafe := true + } + let pktCtorTp := mkConst packetNm + let recInstTp := mkApp2 (mkConst ``RpcEncoding) (mkAppN (mkConst indVal.name) params) pktCtorTp + withLocalDecl `inst .instImplicit recInstTp fun _ => do + let st ← foldWithConstructors indVal params (init := { : CtorState }) fun acc ctor argVars _ => do + -- create the constructor + let fieldStxs ← argVars.mapM fun arg => do + let packetTp ← getRpcPacketFor (← inferType arg) + let tyStx ← PrettyPrinter.delab packetTp + let name := (← getFVarLocalDecl arg).userName + `(bracketedBinder| ($(mkIdent name) : $tyStx)) + let pktCtor ← `(Parser.Command.ctor| | $(mkIdent ctor.getString!):ident $[$fieldStxs]* : RpcEncodingPacket) + + -- create encoder and decoder match arms + let nms ← argVars.mapM fun _ => mkIdent <$> mkFreshBinderName + let mkPattern (src : Name) := Syntax.mkApp (mkIdent <| Name.mkStr src ctor.getString!) nms + let mkBody (tgt : Name) (func : Name) : TermElabM Term := do + let items ← nms.mapM fun nm => `(← $(mkIdent func) $nm) + let tm := Syntax.mkApp (mkIdent <| Name.mkStr tgt ctor.getString!) items + `(return $tm:term) + + let encArm ← `(matchF| | $(mkPattern indVal.name):term => $(← mkBody packetNm ``rpcEncode)) + let decArm ← `(matchF| | $(mkPattern packetNm):term => $(← mkBody indVal.name ``rpcDecode)) + + return { acc with ctors := acc.ctors.push pktCtor + encodes := acc.encodes.push ⟨encArm⟩ + decodes := acc.decodes.push ⟨decArm⟩ } + + -- helpers for type name syntax + let paramIds ← params.mapM fun p => return mkIdent (← getFVarLocalDecl p).userName + let typeId := Syntax.mkApp (← `(@$(mkIdent indVal.name))) paramIds + let instId := mkIdent (`_root_ ++ indVal.name.appendBefore "instRpcEncoding") + + `(variable $packetParamBinders:bracketedBinder* in + inductive RpcEncodingPacket where + $[$(st.ctors):ctor]* + deriving FromJson, ToJson + + variable $(paramBinders ++ packetParamBinders ++ encInstBinders)* in + @[instance] partial def $instId := show RpcEncoding $typeId (RpcEncodingPacket ..) from + { rpcEncode, rpcDecode } + where + rpcEncode {m} [Monad m] [MonadRpcSession m] (x : $typeId) : ExceptT String m (RpcEncodingPacket ..) := + have inst : RpcEncoding $typeId (RpcEncodingPacket ..) := { rpcEncode, rpcDecode } + match x with $[$(st.encodes):matchAlt]* + rpcDecode {m} [Monad m] [MonadRpcSession m] (x : RpcEncodingPacket ..) : ExceptT String m $typeId := + have inst : RpcEncoding $typeId (RpcEncodingPacket ..) := { rpcEncode, rpcDecode } + match x with $[$(st.decodes):matchAlt]* + ) /-- Creates an `RpcEncodingPacket` for `typeName`. For structures, the packet is a structure with the same field names. For inductives, it mirrors the inductive structure with every field @@ -255,33 +198,35 @@ private def deriveInstance (typeName : Name) : CommandElabM Bool := do if indVal.numIndices ≠ 0 then throwError "indexed inductive families are not supported" - let cmds ← liftTermElabM none <| + let (paramBinders, packetParamBinders, encInstBinders) ← liftTermElabM none do -- introduce fvars for all the parameters forallTelescopeReducing indVal.type fun params _ => do - assert! params.size == indVal.numParams + let mut paramBinders := #[] -- input parameters + let mut packetParamBinders := #[] -- RPC encoding packets for type input parameters + let mut encInstBinders := #[] -- RPC encoding instance binders corresponding to packetParamBinders - -- bind every parameter and *some* (not named) `RpcEncoding` for it - let mut binders := #[] for param in params do - let paramNm := (←getFVarLocalDecl param).userName - binders := binders.push (← `(bracketedBinder| ( $(mkIdent paramNm) ))) + let paramNm := (← getFVarLocalDecl param).userName + let ty ← PrettyPrinter.delab (← inferType param) + paramBinders := paramBinders.push (← `(bracketedBinder| ($(mkIdent paramNm) : $ty))) + let packet := mkIdent (← mkFreshUserName (paramNm.appendAfter "Packet")) -- only look for encodings for `Type` parameters - if !(← inferType param).isType then continue - binders := binders.push - (← `(bracketedBinder| [ $(mkIdent ``Lean.Server.RpcEncoding) $(mkIdent paramNm) _ ])) - - return #[ - ← `(section), - ← `(variable $binders*), - ← if isStructure (← getEnv) typeName then - deriveStructureInstance indVal params + if (← inferType param).isType then + packetParamBinders := packetParamBinders.push (← `(bracketedBinder| ($packet : Type))) + encInstBinders := encInstBinders.push (← `(bracketedBinder| [RpcEncoding $(mkIdent paramNm) $packet])) else - deriveInductiveInstance indVal params, - ← `(end) - ] + packetParamBinders := packetParamBinders.push paramBinders.back + + return (paramBinders, packetParamBinders, encInstBinders) + + elabCommand <| ← liftTermElabM none do + Term.elabBinders (paramBinders ++ packetParamBinders ++ encInstBinders) fun locals => do + let params := locals[:paramBinders.size] + if isStructure (← getEnv) typeName then + deriveStructureInstance indVal params paramBinders packetParamBinders encInstBinders + else + deriveInductiveInstance indVal params paramBinders packetParamBinders encInstBinders - for cmd in cmds do - elabCommand cmd.raw return true private unsafe def dispatchDeriveInstanceUnsafe (declNames : Array Name) (args? : Option (TSyntax ``Parser.Term.structInst)) : CommandElabM Bool := do @@ -289,8 +234,7 @@ private unsafe def dispatchDeriveInstanceUnsafe (declNames : Array Name) (args? return false let args ← if let some args := args? then - let n ← liftCoreM <| mkFreshUserName `_args - liftTermElabM (some n) do + liftTermElabM none do let argsT := mkConst ``DerivingParams let args ← elabTerm args argsT evalExpr' DerivingParams ``DerivingParams args diff --git a/src/Lean/Server/Rpc/RequestHandling.lean b/src/Lean/Server/Rpc/RequestHandling.lean index 1da7da08fd8c..5ad94572cf28 100644 --- a/src/Lean/Server/Rpc/RequestHandling.lean +++ b/src/Lean/Server/Rpc/RequestHandling.lean @@ -82,8 +82,18 @@ def wrapRpcProcedure (method : Name) paramType respType RequestM.mapTask t fun | Except.error e => throw e | Except.ok ret => do - let act := rpcEncode (α := respType) (β := respLspType) (m := StateM FileWorker.RpcSession) ret - return toJson (← seshRef.modifyGet act.run)⟩ + let act : StateM FileWorker.RpcSession (Except String respLspType) := do + let s ← get + match ← rpcEncode (α := respType) (β := respLspType) (m := StateM FileWorker.RpcSession) ret with + | .ok x => return .ok x + | .error e => set s; return .error e + match ← seshRef.modifyGet act.run with + | .ok x => return toJson x + | .error e => + throwThe RequestError { + code := JsonRpc.ErrorCode.invalidParams + message := s!"Cannot encode result of RPC call '{method}'\n{e}" + }⟩ def registerBuiltinRpcProcedure (method : Name) paramType respType {paramLspType} [RpcEncoding paramType paramLspType] [FromJson paramLspType] diff --git a/src/Lean/Server/Snapshots.lean b/src/Lean/Server/Snapshots.lean index 3afe0e8565cb..f3b6d77627cb 100644 --- a/src/Lean/Server/Snapshots.lean +++ b/src/Lean/Server/Snapshots.lean @@ -83,22 +83,6 @@ def parseNextCmd (inputCtx : Parser.InputContext) (snap : Snapshot) : IO Syntax Parser.parseCommand inputCtx pmctx snap.mpState snap.msgLog return cmdStx -/-- - Parse remaining file without elaboration. NOTE that doing so can lead to parse errors or even wrong syntax objects, - so it should only be done for reporting preliminary results! -/ -partial def parseAhead (inputCtx : Parser.InputContext) (snap : Snapshot) : IO (Array Syntax) := do - let cmdState := snap.cmdState - let scope := cmdState.scopes.head! - let pmctx := { env := cmdState.env, options := scope.opts, currNamespace := scope.currNamespace, openDecls := scope.openDecls } - go inputCtx pmctx snap.mpState #[] - where - go inputCtx pmctx cmdParserState stxs := do - let (cmdStx, cmdParserState, _) := Parser.parseCommand inputCtx pmctx cmdParserState snap.msgLog - if Parser.isEOI cmdStx || Parser.isExitCommand cmdStx then - return stxs.push cmdStx - else - go inputCtx pmctx cmdParserState (stxs.push cmdStx) - register_builtin_option server.stderrAsMessages : Bool := { defValue := true group := "server" diff --git a/src/Lean/Server/Watchdog.lean b/src/Lean/Server/Watchdog.lean index 56c8e059f0d4..1b5eb95786c2 100644 --- a/src/Lean/Server/Watchdog.lean +++ b/src/Lean/Server/Watchdog.lean @@ -83,21 +83,21 @@ section Utils /-- Events that worker-specific tasks signal to the main thread. -/ inductive WorkerEvent where - /- A synthetic event signalling that the grouped edits should be processed. -/ - | processGroupedEdits + | /-- A synthetic event signalling that the grouped edits should be processed. -/ + processGroupedEdits | terminated | crashed (e : IO.Error) | ioError (e : IO.Error) inductive WorkerState where - /- The watchdog can detect a crashed file worker in two places: When trying to send a message to the file worker - and when reading a request reply. - In the latter case, the forwarding task terminates and delegates a `crashed` event to the main task. - Then, in both cases, the file worker has its state set to `crashed` and requests that are in-flight are errored. - Upon receiving the next packet for that file worker, the file worker is restarted and the packet is forwarded - to it. If the crash was detected while writing a packet, we queue that packet until the next packet for the file - worker arrives. -/ - | crashed (queuedMsgs : Array JsonRpc.Message) + | /-- The watchdog can detect a crashed file worker in two places: When trying to send a message to the file worker + and when reading a request reply. + In the latter case, the forwarding task terminates and delegates a `crashed` event to the main task. + Then, in both cases, the file worker has its state set to `crashed` and requests that are in-flight are errored. + Upon receiving the next packet for that file worker, the file worker is restarted and the packet is forwarded + to it. If the crash was detected while writing a packet, we queue that packet until the next packet for the file + worker arrives. -/ + crashed (queuedMsgs : Array JsonRpc.Message) | running abbrev PendingRequestMap := RBMap RequestID JsonRpc.Message compare @@ -684,7 +684,7 @@ def mkLeanServerCapabilities : ServerCapabilities := { semanticTokensProvider? := some { legend := { tokenTypes := SemanticTokenType.names - tokenModifiers := #[] + tokenModifiers := SemanticTokenModifier.names } full := true range := true diff --git a/src/Lean/Syntax.lean b/src/Lean/Syntax.lean index 24fc5ba7c267..26ff877bdb50 100644 --- a/src/Lean/Syntax.lean +++ b/src/Lean/Syntax.lean @@ -12,7 +12,7 @@ def SourceInfo.updateTrailing (trailing : Substring) : SourceInfo → SourceInfo | SourceInfo.original leading pos _ endPos => SourceInfo.original leading pos trailing endPos | info => info -/- Syntax AST -/ +/-! # Syntax AST -/ inductive IsNode : Syntax → Prop where | mk (info : SourceInfo) (kind : SyntaxNodeKind) (args : Array Syntax) : IsNode (Syntax.node info kind args) @@ -123,7 +123,7 @@ private def updateInfo : SourceInfo → String.Pos → String.Pos → SourceInfo private def chooseNiceTrailStop (trail : Substring) : String.Pos := trail.startPos + trail.posOf '\n' -/- Remark: the State `String.Pos` is the `SourceInfo.trailing.stopPos` of the previous token, +/-- Remark: the State `String.Pos` is the `SourceInfo.trailing.stopPos` of the previous token, or the beginning of the String. -/ @[inline] private def updateLeadingAux : Syntax → StateM String.Pos (Option Syntax) diff --git a/src/Lean/Util/ForEachExpr.lean b/src/Lean/Util/ForEachExpr.lean index 43ba06805476..d8902efe403b 100644 --- a/src/Lean/Util/ForEachExpr.lean +++ b/src/Lean/Util/ForEachExpr.lean @@ -7,7 +7,7 @@ import Lean.Expr import Lean.Util.MonadCache namespace Lean -/- +/-! Remark: we cannot use the caching trick used at `FindExpr` and `ReplaceExpr` because they may visit the same expression multiple times if they are stored in different memory addresses. Note that the following code is parametric in a monad `m`. diff --git a/src/Lean/Util/HasConstCache.lean b/src/Lean/Util/HasConstCache.lean index a131d7172864..bad4046f9bed 100644 --- a/src/Lean/Util/HasConstCache.lean +++ b/src/Lean/Util/HasConstCache.lean @@ -11,7 +11,7 @@ structure HasConstCache (declName : Name) where cache : Std.HashMapImp Expr Bool := Std.mkHashMapImp unsafe def HasConstCache.containsUnsafe (e : Expr) : StateM (HasConstCache declName) Bool := do - if let some r := (← get).cache.find? (beq := ⟨Expr.ptrEq⟩) e then + if let some r := (← get).cache.find? (beq := ⟨ptrEq⟩) e then return r else match e with @@ -25,7 +25,7 @@ unsafe def HasConstCache.containsUnsafe (e : Expr) : StateM (HasConstCache declN | _ => return false where cache (e : Expr) (r : Bool) : StateM (HasConstCache declName) Bool := do - modify fun ⟨cache⟩ => ⟨cache.insert (beq := ⟨Expr.ptrEq⟩) e r |>.1⟩ + modify fun ⟨cache⟩ => ⟨cache.insert (beq := ⟨ptrEq⟩) e r |>.1⟩ return r /-- diff --git a/src/Lean/Util/SCC.lean b/src/Lean/Util/SCC.lean index b5de260964f9..93884e753475 100644 --- a/src/Lean/Util/SCC.lean +++ b/src/Lean/Util/SCC.lean @@ -5,7 +5,7 @@ Authors: Leonardo de Moura -/ import Std.Data.HashMap namespace Lean.SCC -/- +/-! Very simple implementation of Tarjan's SCC algorithm. Performance is not a goal here since we use this module to compiler mutually recursive definitions, where each function diff --git a/src/Lean/Widget/InteractiveDiagnostic.lean b/src/Lean/Widget/InteractiveDiagnostic.lean index 74265f3b9958..2de55833e207 100644 --- a/src/Lean/Widget/InteractiveDiagnostic.lean +++ b/src/Lean/Widget/InteractiveDiagnostic.lean @@ -53,14 +53,14 @@ private def mkPPContext (nCtx : NamingContext) (ctx : MessageDataContext) : PPCo } private inductive EmbedFmt - /- Tags denote `Info` objects. -/ - | expr (ctx : Elab.ContextInfo) (infos : Std.RBMap Nat Elab.Info compare) + | /-- Tags denote `Info` objects. -/ + expr (ctx : Elab.ContextInfo) (infos : Std.RBMap Nat Elab.Info compare) | goal (ctx : Elab.ContextInfo) (lctx : LocalContext) (g : MVarId) - /- Some messages (in particular, traces) are too costly to print eagerly. Instead, we allow - the user to expand sub-traces interactively. -/ - | lazyTrace (nCtx : NamingContext) (ctx? : Option MessageDataContext) (cls : Name) (m : MessageData) - /- Ignore any tags in this subtree. -/ - | ignoreTags + | /-- Some messages (in particular, traces) are too costly to print eagerly. Instead, we allow + the user to expand sub-traces interactively. -/ + lazyTrace (nCtx : NamingContext) (ctx? : Option MessageDataContext) (cls : Name) (m : MessageData) + | /-- Ignore any tags in this subtree. -/ + ignoreTags deriving Inhabited private abbrev MsgFmtM := StateT (Array EmbedFmt) IO diff --git a/src/Std/Data/AssocList.lean b/src/Std/Data/AssocList.lean index 0a829930e2ce..a0cd18f01e4d 100644 --- a/src/Std/Data/AssocList.lean +++ b/src/Std/Data/AssocList.lean @@ -6,7 +6,7 @@ Author: Leonardo de Moura universe u v w w' namespace Std -/- List-like type to avoid extra level of indirection -/ +/-- List-like type to avoid extra level of indirection -/ inductive AssocList (α : Type u) (β : Type v) where | nil : AssocList α β | cons (key : α) (value : β) (tail : AssocList α β) : AssocList α β diff --git a/src/Std/Data/BinomialHeap.lean b/src/Std/Data/BinomialHeap.lean index 791033adc09c..e062dcd6a57a 100644 --- a/src/Std/Data/BinomialHeap.lean +++ b/src/Std/Data/BinomialHeap.lean @@ -173,65 +173,65 @@ variable {α : Type u} {le : α → α → Bool} @[inline] def isEmpty : BinomialHeap α le → Bool | ⟨b, _⟩ => BinomialHeapImp.isEmpty b -/- O(1) -/ +/-- O(1) -/ @[inline] def singleton (a : α) : BinomialHeap α le := ⟨BinomialHeapImp.singleton a, WellFormed.singleton a⟩ -/- O(log n) -/ +/-- O(log n) -/ @[inline] def merge : BinomialHeap α le → BinomialHeap α le → BinomialHeap α le | ⟨b₁, h₁⟩, ⟨b₂, h₂⟩ => ⟨BinomialHeapImp.merge le b₁ b₂, WellFormed.merge b₁ b₂ h₁ h₂⟩ -/- O(log n) -/ +/-- O(log n) -/ @[inline] def insert (a : α) (h : BinomialHeap α le) : BinomialHeap α le := merge (singleton a) h -/- O(n log n) -/ +/-- O(n log n) -/ def ofList (le : α → α → Bool) (as : List α) : BinomialHeap α le := as.foldl (flip insert) empty -/- O(n log n) -/ +/-- O(n log n) -/ def ofArray (le : α → α → Bool) (as : Array α) : BinomialHeap α le := as.foldl (flip insert) empty -/- O(log n) -/ +/-- O(log n) -/ @[inline] def deleteMin : BinomialHeap α le → Option (α × BinomialHeap α le) | ⟨b, h⟩ => match eq: BinomialHeapImp.deleteMin le b with | none => none | some (a, tl) => some (a, ⟨tl, WellFormed.deleteMin a b tl h eq⟩) -/- O(log n) -/ +/-- O(log n) -/ @[inline] def head [Inhabited α] : BinomialHeap α le → α | ⟨b, _⟩ => BinomialHeapImp.head le b -/- O(log n) -/ +/-- O(log n) -/ @[inline] def head? : BinomialHeap α le → Option α | ⟨b, _⟩ => BinomialHeapImp.head? le b -/- O(log n) -/ +/-- O(log n) -/ @[inline] def tail? : BinomialHeap α le → Option (BinomialHeap α le) | ⟨b, h⟩ => match eq: BinomialHeapImp.tail? le b with | none => none | some tl => some ⟨tl, WellFormed.tail? b tl h eq⟩ -/- O(log n) -/ +/-- O(log n) -/ @[inline] def tail : BinomialHeap α le → BinomialHeap α le | ⟨b, h⟩ => ⟨BinomialHeapImp.tail le b, WellFormed.tail b h⟩ -/- O(n log n) -/ +/-- O(n log n) -/ @[inline] def toList : BinomialHeap α le → List α | ⟨b, _⟩ => BinomialHeapImp.toList le b -/- O(n log n) -/ +/-- O(n log n) -/ @[inline] def toArray : BinomialHeap α le → Array α | ⟨b, _⟩ => BinomialHeapImp.toArray le b -/- O(n) -/ +/-- O(n) -/ @[inline] def toListUnordered : BinomialHeap α le → List α | ⟨b, _⟩ => BinomialHeapImp.toListUnordered b -/- O(n) -/ +/-- O(n) -/ @[inline] def toArrayUnordered : BinomialHeap α le → Array α | ⟨b, _⟩ => BinomialHeapImp.toArrayUnordered b diff --git a/src/Std/ShareCommon.lean b/src/Std/ShareCommon.lean index d10a87179345..de4dec84af05 100644 --- a/src/Std/ShareCommon.lean +++ b/src/Std/ShareCommon.lean @@ -85,7 +85,7 @@ unsafe def ObjectPersistentSet.find? (s : ObjectPersistentSet) (o : Object) : Op unsafe def ObjectPersistentSet.insert (s : ObjectPersistentSet) (o : Object) : ObjectPersistentSet := @PersistentHashSet.insert Object ⟨Object.eq⟩ ⟨Object.hash⟩ s o -/- Internally `State` is implemented as a pair `ObjectMap` and `ObjectSet` -/ +/-- Internally `State` is implemented as a pair `ObjectMap` and `ObjectSet` -/ opaque StatePointed : NonemptyType abbrev State : Type u := StatePointed.type @[extern "lean_sharecommon_mk_state"] @@ -93,7 +93,7 @@ opaque mkState : Unit → State := fun _ => Classical.choice StatePointed.proper def State.empty : State := mkState () instance State.inhabited : Inhabited State := ⟨State.empty⟩ -/- Internally `PersistentState` is implemented as a pair `ObjectPersistentMap` and `ObjectPersistentSet` -/ +/-- Internally `PersistentState` is implemented as a pair `ObjectPersistentMap` and `ObjectPersistentSet` -/ opaque PersistentStatePointed : NonemptyType abbrev PersistentState : Type u := PersistentStatePointed.type @[extern "lean_sharecommon_mk_pstate"] diff --git a/src/kernel/expr.cpp b/src/kernel/expr.cpp index 4904d97f2406..ebce32cbf184 100644 --- a/src/kernel/expr.cpp +++ b/src/kernel/expr.cpp @@ -330,97 +330,6 @@ expr update_let(expr const & e, expr const & new_type, expr const & new_value, e return e; } -extern "C" LEAN_EXPORT object * lean_expr_update_mdata(obj_arg e, obj_arg new_expr) { - if (mdata_expr(TO_REF(expr, e)).raw() != new_expr) { - object * r = lean_expr_mk_mdata(mdata_data(TO_REF(expr, e)).to_obj_arg(), new_expr); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_expr); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_const(obj_arg e, obj_arg new_levels) { - if (const_levels(TO_REF(expr, e)).raw() != new_levels) { - object * r = lean_expr_mk_const(const_name(TO_REF(expr, e)).to_obj_arg(), new_levels); - lean_dec_ref(e); - return r; - } else { - lean_dec(new_levels); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_sort(obj_arg e, obj_arg new_level) { - if (sort_level(TO_REF(expr, e)).raw() != new_level) { - object * r = lean_expr_mk_sort(new_level); - lean_dec_ref(e); - return r; - } else { - lean_dec(new_level); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_proj(obj_arg e, obj_arg new_expr) { - if (proj_expr(TO_REF(expr, e)).raw() != new_expr) { - object * r = lean_expr_mk_proj(proj_sname(TO_REF(expr, e)).to_obj_arg(), proj_idx(TO_REF(expr, e)).to_obj_arg(), new_expr); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_expr); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_app(obj_arg e, obj_arg new_fn, obj_arg new_arg) { - if (app_fn(TO_REF(expr, e)).raw() != new_fn || app_arg(TO_REF(expr, e)).raw() != new_arg) { - object * r = lean_expr_mk_app(new_fn, new_arg); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_fn); lean_dec_ref(new_arg); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_forall(obj_arg e, uint8 new_binfo, obj_arg new_domain, obj_arg new_body) { - if (binding_domain(TO_REF(expr, e)).raw() != new_domain || binding_body(TO_REF(expr, e)).raw() != new_body || - binding_info(TO_REF(expr, e)) != static_cast(new_binfo)) { - object * r = lean_expr_mk_forall(binding_name(TO_REF(expr, e)).to_obj_arg(), new_domain, new_body, new_binfo); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_domain); lean_dec_ref(new_body); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_lambda(obj_arg e, uint8 new_binfo, obj_arg new_domain, obj_arg new_body) { - if (binding_domain(TO_REF(expr, e)).raw() != new_domain || binding_body(TO_REF(expr, e)).raw() != new_body || - binding_info(TO_REF(expr, e)) != static_cast(new_binfo)) { - object * r = lean_expr_mk_lambda(binding_name(TO_REF(expr, e)).to_obj_arg(), new_domain, new_body, new_binfo); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_domain); lean_dec_ref(new_body); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_let(obj_arg e, obj_arg new_type, obj_arg new_val, obj_arg new_body) { - if (let_type(TO_REF(expr, e)).raw() != new_type || let_value(TO_REF(expr, e)).raw() != new_val || - let_body(TO_REF(expr, e)).raw() != new_body) { - object * r = lean_expr_mk_let(let_name(TO_REF(expr, e)).to_obj_arg(), new_type, new_val, new_body); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_type); lean_dec_ref(new_val); lean_dec_ref(new_body); - return e; - } -} - extern "C" object * lean_expr_consume_type_annotations(obj_arg e); expr consume_type_annotations(expr const & e) { return expr(lean_expr_consume_type_annotations(e.to_obj_arg())); } diff --git a/src/kernel/level.cpp b/src/kernel/level.cpp index 9ed8d461d9b5..06652dc8ca67 100644 --- a/src/kernel/level.cpp +++ b/src/kernel/level.cpp @@ -29,10 +29,6 @@ extern "C" object * lean_level_mk_mvar(obj_arg); extern "C" object * lean_level_mk_param(obj_arg); extern "C" object * lean_level_mk_max(obj_arg, obj_arg); extern "C" object * lean_level_mk_imax(obj_arg, obj_arg); -extern "C" object * lean_level_mk_max_simp(obj_arg, obj_arg); -extern "C" object * lean_level_mk_imax_simp(obj_arg, obj_arg); -extern "C" object * lean_level_simp_max(obj_arg, obj_arg, obj_arg); -extern "C" object * lean_level_simp_imax(obj_arg, obj_arg, obj_arg); level mk_succ(level const & l) { return level(lean_level_mk_succ(l.to_obj_arg())); } level mk_max_core(level const & l1, level const & l2) { return level(lean_level_mk_max(l1.to_obj_arg(), l2.to_obj_arg())); } @@ -293,34 +289,6 @@ level update_max(level const & l, level const & new_lhs, level const & new_rhs) return mk_imax(new_lhs, new_rhs); } -extern "C" LEAN_EXPORT object * lean_level_update_succ(obj_arg l, obj_arg new_arg) { - if (succ_of(TO_REF(level, l)).raw() == new_arg) { - lean_dec(new_arg); - return l; - } else { - lean_dec_ref(l); - return lean_level_mk_succ(new_arg); - } -} - -extern "C" LEAN_EXPORT object * lean_level_update_max(obj_arg l, obj_arg new_lhs, obj_arg new_rhs) { - if (max_lhs(TO_REF(level, l)).raw() == new_lhs && max_rhs(TO_REF(level, l)).raw() == new_rhs) { - return lean_level_simp_max(new_lhs, new_rhs, l); - } else { - lean_dec_ref(l); - return lean_level_mk_max_simp(new_lhs, new_rhs); - } -} - -extern "C" LEAN_EXPORT object * lean_level_update_imax(obj_arg l, obj_arg new_lhs, obj_arg new_rhs) { - if (imax_lhs(TO_REF(level, l)).raw() == new_lhs && imax_rhs(TO_REF(level, l)).raw() == new_rhs) { - return lean_level_simp_imax(new_lhs, new_rhs, l); - } else { - lean_dec_ref(l); - return lean_level_mk_imax_simp(new_lhs, new_rhs); - } -} - level instantiate(level const & l, names const & ps, levels const & ls) { lean_assert(length(ps) == length(ls)); return replace(l, [=](level const & l) { diff --git a/stage0/src/Init/Data/List/Control.lean b/stage0/src/Init/Data/List/Control.lean index 3e58b27ff5fa..ab5d3bcb0ac3 100644 --- a/stage0/src/Init/Data/List/Control.lean +++ b/stage0/src/Init/Data/List/Control.lean @@ -193,4 +193,7 @@ instance : ForM m (List α) α where @[simp] theorem forM_cons [Monad m] (f : α → m PUnit) (a : α) (as : List α) : forM (a::as) f = f a >>= fun _ => forM as f := rfl +instance : Functor List where + map := List.map + end List diff --git a/stage0/src/Init/Data/String/Extra.lean b/stage0/src/Init/Data/String/Extra.lean index 18709a010a42..d8a19e7a58b0 100644 --- a/stage0/src/Init/Data/String/Extra.lean +++ b/stage0/src/Init/Data/String/Extra.lean @@ -66,4 +66,21 @@ theorem Iterator.sizeOf_next_lt_of_atEnd (i : String.Iterator) (h : ¬ i.atEnd = macro_rules | `(tactic| decreasing_trivial) => `(tactic| apply String.Iterator.sizeOf_next_lt_of_atEnd; assumption) +namespace Iterator + +@[specialize] def find (it : Iterator) (p : Char → Bool) : Iterator := + if it.atEnd then it + else if p it.curr then it + else find it.next p + +@[specialize] def foldUntil (it : Iterator) (init : α) (f : α → Char → Option α) : α × Iterator := + if it.atEnd then + (init, it) + else if let some a := f init it.curr then + foldUntil it.next a f + else + (init, it) + +end Iterator + end String diff --git a/stage0/src/Init/Meta.lean b/stage0/src/Init/Meta.lean index b73abdae484f..5995ef1c12ad 100644 --- a/stage0/src/Init/Meta.lean +++ b/stage0/src/Init/Meta.lean @@ -1061,6 +1061,18 @@ def SepArray.getElems (sa : SepArray sep) : Array Syntax := def TSepArray.getElems (sa : TSepArray k sep) : TSyntaxArray k := .mk sa.elemsAndSeps.getSepElems +def TSepArray.push (sa : TSepArray k sep) (e : TSyntax k) : TSepArray k sep := + if sa.elemsAndSeps.isEmpty then + { elemsAndSeps := #[e] } + else + { elemsAndSeps := sa.elemsAndSeps.push (mkAtom sep) |>.push e } + +instance : EmptyCollection (SepArray sep) where + emptyCollection := ⟨∅⟩ + +instance : EmptyCollection (TSepArray sep k) where + emptyCollection := ⟨∅⟩ + /- We use `CoeTail` here instead of `Coe` to avoid a "loop" when computing `CoeTC`. The "loop" is interrupted using the maximum instance size threshold, but it is a performance bottleneck. diff --git a/stage0/src/Init/Notation.lean b/stage0/src/Init/Notation.lean index ab33e4967b4f..c704923c1f4c 100644 --- a/stage0/src/Init/Notation.lean +++ b/stage0/src/Init/Notation.lean @@ -101,6 +101,7 @@ macro_rules | `($x - $y) => `(binop% HSub.hSub $x $y) macro_rules | `($x * $y) => `(binop% HMul.hMul $x $y) macro_rules | `($x / $y) => `(binop% HDiv.hDiv $x $y) macro_rules | `($x % $y) => `(binop% HMod.hMod $x $y) +macro_rules | `($x ^ $y) => `(binop% HPow.hPow $x $y) macro_rules | `($x ++ $y) => `(binop% HAppend.hAppend $x $y) -- declare ASCII alternatives first so that the latter Unicode unexpander wins diff --git a/stage0/src/Init/NotationExtra.lean b/stage0/src/Init/NotationExtra.lean index 2cf1faebf6bb..493a86dc2fd8 100644 --- a/stage0/src/Init/NotationExtra.lean +++ b/stage0/src/Init/NotationExtra.lean @@ -262,6 +262,11 @@ syntax "repeat " doSeq : doElem macro_rules | `(doElem| repeat $seq) => `(doElem| for _ in Loop.mk do $seq) +syntax "while " ident " : " termBeforeDo " do " doSeq : doElem + +macro_rules + | `(doElem| while $h : $cond do $seq) => `(doElem| repeat if $h : $cond then $seq else break) + syntax "while " termBeforeDo " do " doSeq : doElem macro_rules diff --git a/stage0/src/Init/Prelude.lean b/stage0/src/Init/Prelude.lean index 01c00a93d81e..8b0dcc06c022 100644 --- a/stage0/src/Init/Prelude.lean +++ b/stage0/src/Init/Prelude.lean @@ -316,6 +316,7 @@ theorem of_decide_eq_self_eq_true [inst : DecidableEq α] (a : α) : Eq (decide | true, true => isTrue rfl class BEq (α : Type u) where + /-- Boolean equality. -/ beq : α → α → Bool open BEq (beq) @@ -379,6 +380,7 @@ instance [dp : Decidable p] : Decidable (Not p) := | true => false | false => true +/-- The type of natural numbers. `0`, `1`, `2`, ...-/ inductive Nat where | zero : Nat | succ (n : Nat) : Nat @@ -799,12 +801,15 @@ instance : Sub Nat where @[extern "lean_system_platform_nbits"] opaque System.Platform.getNumBits : Unit → Subtype fun (n : Nat) => Or (Eq n 32) (Eq n 64) := fun _ => ⟨64, Or.inr rfl⟩ -- inhabitant +/-- Gets the word size of the platform. +That is, whether the platform is 64 or 32 bits. -/ def System.Platform.numBits : Nat := (getNumBits ()).val theorem System.Platform.numBits_eq : Or (Eq numBits 32) (Eq numBits 64) := (getNumBits ()).property +/-- `Fin n` is a natural number `i` with the constraint that `0 ≤ i < n`. -/ structure Fin (n : Nat) where val : Nat isLt : LT.lt val n @@ -834,6 +839,7 @@ instance Fin.decLt {n} (a b : Fin n) : Decidable (LT.lt a b) := Nat.decLt .. instance Fin.decLe {n} (a b : Fin n) : Decidable (LE.le a b) := Nat.decLe .. def UInt8.size : Nat := 256 +/-- Unsigned 8-bit integer. -/ structure UInt8 where val : Fin UInt8.size @@ -858,6 +864,7 @@ instance : Inhabited UInt8 where default := UInt8.ofNatCore 0 (by decide) def UInt16.size : Nat := 65536 +/-- Unsigned 16-bit integer. -/ structure UInt16 where val : Fin UInt16.size @@ -882,6 +889,7 @@ instance : Inhabited UInt16 where default := UInt16.ofNatCore 0 (by decide) def UInt32.size : Nat := 4294967296 +/-- Unsigned, 32-bit integer. -/ structure UInt32 where val : Fin UInt32.size @@ -930,6 +938,7 @@ instance (a b : UInt32) : Decidable (LT.lt a b) := UInt32.decLt a b instance (a b : UInt32) : Decidable (LE.le a b) := UInt32.decLe a b def UInt64.size : Nat := 18446744073709551616 +/-- Unsigned, 64-bit integer. -/ structure UInt64 where val : Fin UInt64.size @@ -961,6 +970,12 @@ theorem usize_size_eq : Or (Eq USize.size 4294967296) (Eq USize.size 18446744073 | _, Or.inl rfl => Or.inl (by decide) | _, Or.inr rfl => Or.inr (by decide) +/-- A USize is an unsigned integer with the size of a word +for the platform's architecture. + +For example, if running on a 32-bit machine, USize is equivalent to UInt32. +Or on a 64-bit machine, UInt64. +-/ structure USize where val : Fin USize.size @@ -1744,11 +1759,40 @@ instance : Hashable String where namespace Lean -/- Hierarchical names -/ +/-- +Hierarchical names. We use hierarchical names to name declarations and +for creating unique identifiers for free variables and metavariables. + +You can create hierarchical names using the following quotation notation. +``` +`Lean.Meta.whnf +``` +It is short for `.str (.str (.str .anonymous "Lean") "Meta") "whnf"` +You can use double quotes to request Lean to statically check whether the name +corresponds to a Lean declaration in scope. +``` +``Lean.Meta.whnf +``` +If the name is not in scope, Lean will report an error. +-/ inductive Name where - | anonymous : Name - | str : Name → String → Name - | num : Name → Nat → Name + | /-- The "anonymous" name. -/ + anonymous : Name + | /-- +A string name. The name `Lean.Meta.run` is represented at +```lean +.str (.str (.str .anonymous "Lean") "Meta") "run" +``` +-/ + str (pre : Name) (str : String) + | /-- +A numerical name. This kind of name is used, for example, to create hierarchical names for +free variables and metavariables. The identifier `_uniq.231` is represented as +```lean +.num (.str .anonymous "_uniq") 231 +``` +-/ + num (pre : Name) (i : Nat) with @[computedField] hash : Name → UInt64 | .anonymous => .ofNatCore 1723 (by decide) @@ -1763,14 +1807,23 @@ instance : Hashable Name where namespace Name +/-- +`.str p s` is now the preferred form. +-/ @[export lean_name_mk_string] abbrev mkStr (p : Name) (s : String) : Name := Name.str p s +/-- +`.num p v` is now the preferred form. +-/ @[export lean_name_mk_numeral] abbrev mkNum (p : Name) (v : Nat) : Name := Name.num p v +/-- +Short for `.str .anonymous s`. +-/ abbrev mkSimple (s : String) : Name := mkStr Name.anonymous s @@ -1784,6 +1837,13 @@ protected def beq : (@& Name) → (@& Name) → Bool instance : BEq Name where beq := Name.beq +/-- +Append two hierarchical names. Example: +```lean +`Lean.Meta ++ `Tactic.simp +``` +return `Lean.Meta.Tactic.simp` +-/ protected def append : Name → Name → Name | n, anonymous => n | n, str p s => Name.mkStr (Name.append n p) s @@ -1798,18 +1858,22 @@ end Name /-- Source information of tokens. -/ inductive SourceInfo where - /- + | /-- Token from original input with whitespace and position information. `leading` will be inferred after parsing by `Syntax.updateLeading`. During parsing, - it is not at all clear what the preceding token was, especially with backtracking. -/ - | original (leading : Substring) (pos : String.Pos) (trailing : Substring) (endPos : String.Pos) - /- + it is not at all clear what the preceding token was, especially with backtracking. + -/ + original (leading : Substring) (pos : String.Pos) (trailing : Substring) (endPos : String.Pos) + | /-- Synthesized token (e.g. from a quotation) annotated with a span from the original source. In the delaborator, we "misuse" this constructor to store synthetic positions identifying - subterms. -/ - | synthetic (pos : String.Pos) (endPos : String.Pos) - /- Synthesized token without position information. -/ - | protected none + subterms. + -/ + synthetic (pos : String.Pos) (endPos : String.Pos) + | /-- + Synthesized token without position information. + -/ + protected none instance : Inhabited SourceInfo := ⟨SourceInfo.none⟩ @@ -1833,36 +1897,37 @@ Syntax objects used by the parser, macro expander, delaborator, etc. inductive Syntax where | missing : Syntax | /-- - Node in the syntax tree. - - The `info` field is used by the delaborator - to store the position of the subexpression - corresponding to this node. - The parser sets the `info` field to `none`. - - (Remark: the `node` constructor - did not have an `info` field in previous versions. - This caused a bug in the interactive widgets, - where the popup for `a + b` was the same as for `a`. - The delaborator used to associate subexpressions - with pretty-printed syntax by setting - the (string) position of the first atom/identifier - to the (expression) position of the subexpression. - For example, both `a` and `a + b` - have the same first identifier, - and so their infos got mixed up.) - -/ node (info : SourceInfo) (kind : SyntaxNodeKind) (args : Array Syntax) : Syntax + Node in the syntax tree. + + The `info` field is used by the delaborator + to store the position of the subexpression + corresponding to this node. + The parser sets the `info` field to `none`. + + (Remark: the `node` constructor + did not have an `info` field in previous versions. + This caused a bug in the interactive widgets, + where the popup for `a + b` was the same as for `a`. + The delaborator used to associate subexpressions + with pretty-printed syntax by setting + the (string) position of the first atom/identifier + to the (expression) position of the subexpression. + For example, both `a` and `a + b` + have the same first identifier, + and so their infos got mixed up.) + -/ + node (info : SourceInfo) (kind : SyntaxNodeKind) (args : Array Syntax) : Syntax | atom (info : SourceInfo) (val : String) : Syntax | ident (info : SourceInfo) (rawVal : Substring) (val : Name) (preresolved : List (Prod Name (List String))) : Syntax def SyntaxNodeKinds := List SyntaxNodeKind /-- - A `Syntax` value of one of the given syntax kinds. - Note that while syntax quotations produce/expect `TSyntax` values of the correct kinds, - this is not otherwise enforced and can easily be circumvented by direct use of the constructor. - The namespace `TSyntax.Compat` can be opened to expose a general coercion from `Syntax` to any - `TSyntax ks` for porting older code. -/ +A `Syntax` value of one of the given syntax kinds. +Note that while syntax quotations produce/expect `TSyntax` values of the correct kinds, +this is not otherwise enforced and can easily be circumvented by direct use of the constructor. +The namespace `TSyntax.Compat` can be opened to expose a general coercion from `Syntax` to any +`TSyntax ks` for porting older code. -/ structure TSyntax (ks : SyntaxNodeKinds) where raw : Syntax @@ -1872,7 +1937,7 @@ instance : Inhabited Syntax where instance : Inhabited (TSyntax ks) where default := ⟨default⟩ -/- Builtin kinds -/ +/-! Builtin kinds -/ abbrev choiceKind : SyntaxNodeKind := `choice abbrev nullKind : SyntaxNodeKind := `null abbrev groupKind : SyntaxNodeKind := `group @@ -2095,10 +2160,11 @@ def replaceRef (ref : Syntax) (oldRef : Syntax) : Syntax := introduced symbol, which results in better error positions than not applying any position. -/ class MonadQuotation (m : Type → Type) extends MonadRef m where - -- Get the fresh scope of the current macro invocation + /-- Get the fresh scope of the current macro invocation -/ getCurrMacroScope : m MacroScope getMainModule : m Name - /- Execute action in a new macro invocation context. This transformer should be + /-- + Execute action in a new macro invocation context. This transformer should be used at all places that morally qualify as the beginning of a "macro call", e.g. `elabCommand` and `elabTerm` in the case of the elaborator. However, it can also be used internally inside a "macro" if identifiers introduced by diff --git a/stage0/src/Init/Util.lean b/stage0/src/Init/Util.lean index 2902ce958628..b092ac9afb9d 100644 --- a/stage0/src/Init/Util.lean +++ b/stage0/src/Init/Util.lean @@ -42,8 +42,15 @@ unsafe def ptrAddrUnsafe {α : Type u} (a : @& α) : USize := 0 @[inline] unsafe def withPtrAddrUnsafe {α : Type u} {β : Type v} (a : α) (k : USize → β) (h : ∀ u₁ u₂, k u₁ = k u₂) : β := k (ptrAddrUnsafe a) +@[inline] unsafe def ptrEq (a b : α) : Bool := ptrAddrUnsafe a == ptrAddrUnsafe b + +unsafe def ptrEqList : (as bs : List α) → Bool + | [], [] => true + | a::as, b::bs => if ptrEq a b then ptrEqList as bs else false + | _, _ => false + @[inline] unsafe def withPtrEqUnsafe {α : Type u} (a b : α) (k : Unit → Bool) (h : a = b → k () = true) : Bool := - if ptrAddrUnsafe a == ptrAddrUnsafe b then true else k () + if ptrEq a b then true else k () @[implementedBy withPtrEqUnsafe] def withPtrEq {α : Type u} (a b : α) (k : Unit → Bool) (h : a = b → k () = true) : Bool := k () diff --git a/stage0/src/Lean/Attributes.lean b/stage0/src/Lean/Attributes.lean index 946f0e53c0e2..51956c26388e 100644 --- a/stage0/src/Lean/Attributes.lean +++ b/stage0/src/Lean/Attributes.lean @@ -24,6 +24,17 @@ structure AttributeImplCore where applicationTime := AttributeApplicationTime.afterTypeChecking deriving Inhabited +/-- You can tag attributes with the 'local' or 'scoped' kind. +For example: `attribute [local myattr, scoped yourattr, theirattr]`. + +This is used to indicate how an attribute should be scoped. +- local means that the attribute should only be applied in the current scope and forgotten once the current section, namespace, or file is closed. +- scoped means that the attribute should only be applied while the namespace is open. +- global means that the attribute should always be applied. + +Note that the attribute handler (`AttributeImpl.add`) is responsible for interpreting the kind and +making sure that these kinds are respected. +-/ inductive AttributeKind | «global» | «local» | «scoped» deriving BEq, Inhabited diff --git a/stage0/src/Lean/Class.lean b/stage0/src/Lean/Class.lean index e63eca064271..eb1642ac1823 100644 --- a/stage0/src/Lean/Class.lean +++ b/stage0/src/Lean/Class.lean @@ -8,8 +8,16 @@ import Lean.Attributes namespace Lean structure ClassEntry where - name : Name - hasOutParam : Bool + name : Name + /-- + Position of the class `outParams`. + For example, for class + ``` + class GetElem (Cont : Type u) (Idx : Type v) (Elem : outParam (Type w)) (Dom : outParam (Cont → Idx → Prop)) where + ``` + `outParams := #[2, 3]` + -/ + outParams : Array Nat namespace ClassEntry @@ -19,16 +27,16 @@ def lt (a b : ClassEntry) : Bool := end ClassEntry structure ClassState where - hasOutParam : SMap Name Bool := SMap.empty + outParamMap : SMap Name (Array Nat) := SMap.empty deriving Inhabited namespace ClassState def addEntry (s : ClassState) (entry : ClassEntry) : ClassState := - { s with hasOutParam := s.hasOutParam.insert entry.name entry.hasOutParam } + { s with outParamMap := s.outParamMap.insert entry.name entry.outParams } def switch (s : ClassState) : ClassState := - { s with hasOutParam := s.hasOutParam.switch } + { s with outParamMap := s.outParamMap.switch } end ClassState @@ -42,17 +50,23 @@ builtin_initialize classExtension : SimplePersistentEnvExtension ClassEntry Clas @[export lean_is_class] def isClass (env : Environment) (n : Name) : Bool := - (classExtension.getState env).hasOutParam.contains n + (classExtension.getState env).outParamMap.contains n + +/-- + If `declName` is a class, return the position of its `outParams`. +-/ +def getOutParamPositions? (env : Environment) (declName : Name) : Option (Array Nat) := + (classExtension.getState env).outParamMap.find? declName @[export lean_has_out_params] -def hasOutParams (env : Environment) (n : Name) : Bool := - match (classExtension.getState env).hasOutParam.find? n with - | some b => b - | none => false +def hasOutParams (env : Environment) (declName : Name) : Bool := + match getOutParamPositions? env declName with + | some outParams => !outParams.isEmpty + | none => false /-- - Auxiliary function for checking whether a class has `outParam`, and - whether they are being correctly used. + Auxiliary function for collection the position class `outParams`, and + checking whether they are being correctly used. A regular (i.e., non `outParam`) must not depend on an `outParam`. Reason for this restriction: When performing type class resolution, we replace arguments that @@ -62,19 +76,19 @@ def hasOutParams (env : Environment) (n : Name) : Bool := incorrect. This transformation would be counterintuitive to users since we would implicitly treat these regular parameters as `outParam`s. -/ -private partial def checkOutParam : Nat → Array FVarId → Expr → Except String Bool - | i, outParams, Expr.forallE _ d b _ => +private partial def checkOutParam (i : Nat) (outParamFVarIds : Array FVarId) (outParams : Array Nat) (type : Expr) : Except String (Array Nat) := + match type with + | .forallE _ d b _ => if d.isOutParam then - let fvarId := { name := Name.mkNum `_fvar outParams.size } - let outParams := outParams.push fvarId + let fvarId := { name := Name.mkNum `_fvar outParamFVarIds.size } let fvar := mkFVar fvarId let b := b.instantiate1 fvar - checkOutParam (i+1) outParams b - else if d.hasAnyFVar fun fvarId => outParams.contains fvarId then - Except.error s!"invalid class, parameter #{i} depends on `outParam`, but it is not an `outParam`" + checkOutParam (i+1) (outParamFVarIds.push fvarId) (outParams.push i) b + else if d.hasAnyFVar fun fvarId => outParamFVarIds.contains fvarId then + Except.error s!"invalid class, parameter #{i+1} depends on `outParam`, but it is not an `outParam`" else - checkOutParam (i+1) outParams b - | _, outParams, _ => pure (outParams.size > 0) + checkOutParam (i+1) outParamFVarIds outParams b + | _ => return outParams def addClass (env : Environment) (clsName : Name) : Except String Environment := do if isClass env clsName then @@ -83,17 +97,17 @@ def addClass (env : Environment) (clsName : Name) : Except String Environment := | throw s!"unknown declaration '{clsName}'" unless decl matches .inductInfo .. | .axiomInfo .. do throw s!"invalid 'class', declaration '{clsName}' must be inductive datatype, structure, or constant" - let b ← checkOutParam 1 #[] decl.type - return classExtension.addEntry env { name := clsName, hasOutParam := b } + let outParams ← checkOutParam 0 #[] #[] decl.type + return classExtension.addEntry env { name := clsName, outParams } private def consumeNLambdas : Nat → Expr → Option Expr - | 0, e => some e - | i+1, Expr.lam _ _ b _ => consumeNLambdas i b - | _, _ => none + | 0, e => some e + | i+1, .lam _ _ b _ => consumeNLambdas i b + | _, _ => none partial def getClassName (env : Environment) : Expr → Option Name - | Expr.forallE _ _ b _ => getClassName env b - | e => do + | .forallE _ _ b _ => getClassName env b + | e => do let Expr.const c _ ← pure e.getAppFn | none let info ← env.find? c match info.value? with @@ -106,8 +120,8 @@ partial def getClassName (env : Environment) : Expr → Option Name builtin_initialize registerBuiltinAttribute { - name := `class, - descr := "type class", + name := `class + descr := "type class" add := fun decl stx kind => do let env ← getEnv Attribute.Builtin.ensureNoArgs stx diff --git a/stage0/src/Lean/CoreM.lean b/stage0/src/Lean/CoreM.lean index ea9542a2a184..5290b9a4f15f 100644 --- a/stage0/src/Lean/CoreM.lean +++ b/stage0/src/Lean/CoreM.lean @@ -228,15 +228,15 @@ export Core (CoreM mkFreshUserName checkMaxHeartbeats withCurrHeartbeats) try x catch ex => match ex with - | Exception.error _ _ => throw ex - | Exception.internal id' _ => if id == id' then h ex else throw ex + | .error .. => throw ex + | .internal id' _ => if id == id' then h ex else throw ex @[inline] def catchInternalIds [Monad m] [MonadExcept Exception m] (ids : List InternalExceptionId) (x : m α) (h : Exception → m α) : m α := do try x catch ex => match ex with - | Exception.error _ _ => throw ex - | Exception.internal id _ => if ids.contains id then h ex else throw ex + | .error .. => throw ex + | .internal id _ => if ids.contains id then h ex else throw ex /-- Return true if `ex` was generated by `throwMaxHeartbeat`. diff --git a/stage0/src/Lean/Data/Lsp/LanguageFeatures.lean b/stage0/src/Lean/Data/Lsp/LanguageFeatures.lean index 58c4f91eac42..dde13e1b2575 100644 --- a/stage0/src/Lean/Data/Lsp/LanguageFeatures.lean +++ b/stage0/src/Lean/Data/Lsp/LanguageFeatures.lean @@ -226,11 +226,13 @@ structure SymbolInformation where deriving ToJson inductive SemanticTokenType where + -- Used by Lean | keyword | «variable» | property | function - /- + /- Other types included by default in the LSP specification. + Not used by the Lean core, but useful to users extending the Lean server. -/ | «namespace» | type | «class» @@ -249,19 +251,29 @@ inductive SemanticTokenType where | number | regexp | operator - -/ + | decorator + deriving ToJson, FromJson +-- must be in the same order as the constructors def SemanticTokenType.names : Array String := - #["keyword", "variable", "property", "function"] - --- must be the correct index in `names` -def SemanticTokenType.toNat : SemanticTokenType → Nat - | keyword => 0 - | «variable» => 1 - | property => 2 - | function => 3 - -/- + #["keyword", "variable", "property", "function", "namespace", "type", "class", + "enum", "interface", "struct", "typeParameter", "parameter", "enumMember", + "event", "method", "macro", "modifier", "comment", "string", "number", + "regexp", "operator", "decorator"] + +def SemanticTokenType.toNat (type : SemanticTokenType) : Nat := + type.toCtorIdx + +-- sanity check +example {v : SemanticTokenType} : open SemanticTokenType in + names[v.toNat]?.map (toString <| toJson ·) = some (toString <| toJson v) := by + cases v <;> native_decide + +/-- +The semantic token modifiers included by default in the LSP specification. +Not used by the Lean core, but implementing them here allows them to be +utilized by users extending the Lean server. +-/ inductive SemanticTokenModifier where | declaration | definition @@ -273,7 +285,20 @@ inductive SemanticTokenModifier where | modification | documentation | defaultLibrary --/ + deriving ToJson, FromJson + +-- must be in the same order as the constructors +def SemanticTokenModifier.names : Array String := + #["declaration", "definition", "readonly", "static", "deprecated", "abstract", + "async", "modification", "documentation", "defaultLibrary"] + +def SemanticTokenModifier.toNat (modifier : SemanticTokenModifier) : Nat := + modifier.toCtorIdx + +-- sanity check +example {v : SemanticTokenModifier} : open SemanticTokenModifier in + names[v.toNat]?.map (toString <| toJson ·) = some (toString <| toJson v) := by + cases v <;> native_decide structure SemanticTokensLegend where tokenTypes : Array String @@ -298,7 +323,7 @@ structure SemanticTokensRangeParams where deriving FromJson, ToJson structure SemanticTokens where - -- resultId?: string; + resultId? : Option String := none data : Array Nat deriving FromJson, ToJson diff --git a/stage0/src/Lean/Declaration.lean b/stage0/src/Lean/Declaration.lean index 29747fc285d6..b54eac4f344c 100644 --- a/stage0/src/Lean/Declaration.lean +++ b/stage0/src/Lean/Declaration.lean @@ -121,7 +121,7 @@ structure TheoremVal extends ConstantVal where all : List Name := [name] deriving Inhabited -/- Value for an opaque constant declaration `constant x : t := e` -/ +/- Value for an opaque constant declaration `opaque x : t := e` -/ structure OpaqueVal extends ConstantVal where value : Expr isUnsafe : Bool diff --git a/stage0/src/Lean/DocString.lean b/stage0/src/Lean/DocString.lean index 8b2fdf97b922..9b233b2da193 100644 --- a/stage0/src/Lean/DocString.lean +++ b/stage0/src/Lean/DocString.lean @@ -11,11 +11,48 @@ namespace Lean private builtin_initialize builtinDocStrings : IO.Ref (NameMap String) ← IO.mkRef {} private builtin_initialize docStringExt : MapDeclarationExtension String ← mkMapDeclarationExtension `docstring +private def findLeadingSpacesSize (s : String) : Nat := + let it := s.iter + let it := it.find (· == '\n') |>.next + let (min, it) := it.foldUntil 0 fun num c => if c == ' ' || c == '\t' then some (num + 1) else none + findNextLine it min +where + consumeSpaces (it : String.Iterator) (curr min : Nat) : Nat := + if it.atEnd then min + else if it.curr == ' ' || it.curr == '\t' then consumeSpaces it.next (curr + 1) min + else findNextLine it.next (Nat.min curr min) + findNextLine (it : String.Iterator) (min : Nat) : Nat := + if it.atEnd then min + else if it.curr == '\n' then consumeSpaces it.next 0 min + else findNextLine it.next min + +private def removeNumLeadingSpaces (n : Nat) (s : String) : String := + consumeSpaces n s.iter "" +where + consumeSpaces (n : Nat) (it : String.Iterator) (r : String) : String := + match n with + | 0 => saveLine it r + | n+1 => + if it.atEnd then r + else if it.curr == ' ' || it.curr == '\t' then consumeSpaces n it.next r + else saveLine it r + saveLine (it : String.Iterator) (r : String) : String := + if it.atEnd then r + else if it.curr == '\n' then consumeSpaces n it.next (r.push '\n') + else saveLine it.next (r.push it.curr) +termination_by + consumeSpaces n it r => (it, 1) + saveLine it r => (it, 0) + +private def removeLeadingSpaces (s : String) : String := + let n := findLeadingSpacesSize s + if n == 0 then s else removeNumLeadingSpaces n s + def addBuiltinDocString (declName : Name) (docString : String) : IO Unit := - builtinDocStrings.modify (·.insert declName docString) + builtinDocStrings.modify (·.insert declName (removeLeadingSpaces docString)) def addDocString [MonadEnv m] (declName : Name) (docString : String) : m Unit := - modifyEnv fun env => docStringExt.insert env declName docString + modifyEnv fun env => docStringExt.insert env declName (removeLeadingSpaces docString) def addDocString' [Monad m] [MonadEnv m] (declName : Name) (docString? : Option String) : m Unit := match docString? with diff --git a/stage0/src/Lean/Elab/App.lean b/stage0/src/Lean/Elab/App.lean index c26931f12c57..6b092d1a0577 100644 --- a/stage0/src/Lean/Elab/App.lean +++ b/stage0/src/Lean/Elab/App.lean @@ -37,7 +37,7 @@ private def ensureArgType (f : Expr) (arg : Expr) (expectedType : Expr) : TermEl try ensureHasTypeAux expectedType argType arg f catch - | ex@(Exception.error ..) => + | ex@(.error ..) => if (← read).errToSorry then exceptionToSorry ex expectedType else @@ -249,7 +249,7 @@ private def fTypeHasOptAutoParams : M Bool := do See `propagateExpectedType`. Remark: `(explicit : Bool) == true` when `@` modifier is used. -/ private partial def getForallBody (explicit : Bool) : Nat → List NamedArg → Expr → Option Expr - | i, namedArgs, type@(Expr.forallE n d b bi) => + | i, namedArgs, type@(.forallE n d b bi) => match namedArgs.find? fun (namedArg : NamedArg) => namedArg.name == n with | some _ => getForallBody explicit i (eraseNamedArgCore namedArgs n) b | none => @@ -538,7 +538,7 @@ mutual let argType ← getArgExpectedType match (← read).explicit, argType.getOptParamDefault?, argType.getAutoParamTactic? with | false, some defVal, _ => addNewArg argName defVal; main - | false, _, some (Expr.const tacticDecl _) => + | false, _, some (.const tacticDecl _) => let env ← getEnv let opts ← getOptions match evalSyntaxConstant env opts tacticDecl with @@ -988,17 +988,17 @@ private partial def resolveDotName (id : Syntax) (expectedType? : Option Expr) : go resultType expectedType #[] where go (resultType : Expr) (expectedType : Expr) (previousExceptions : Array Exception) : TermElabM Name := do - let resultTypeFn := (← instantiateMVars resultType).consumeMDataAndTypeAnnotations.getAppFn + let resultTypeFn := (← instantiateMVars resultType).cleanupAnnotations.getAppFn try tryPostponeIfMVar resultTypeFn - let .const declName .. := resultTypeFn.consumeMDataAndTypeAnnotations + let .const declName .. := resultTypeFn.cleanupAnnotations | throwError "invalid dotted identifier notation, expected type is not of the form (... → C ...) where C is a constant{indentExpr expectedType}" let idNew := declName ++ id.getId.eraseMacroScopes unless (← getEnv).contains idNew do throwError "invalid dotted identifier notation, unknown identifier `{idNew}` from expected type{indentExpr expectedType}" return idNew catch - | ex@(.error _ _) => + | ex@(.error ..) => match (← unfoldDefinition? resultType) with | some resultType => go (← whnfCore resultType) expectedType (previousExceptions.push ex) | none => @@ -1107,8 +1107,8 @@ private def elabAppAux (f : Syntax) (namedArgs : Array NamedArg) (args : Array A else if successes.size > 1 then let msgs : Array MessageData ← successes.mapM fun success => do match success with - | EStateM.Result.ok e s => withMCtx s.meta.meta.mctx <| withEnv s.meta.core.env do addMessageContext m!"{e} : {← inferType e}" - | _ => unreachable! + | .ok e s => withMCtx s.meta.meta.mctx <| withEnv s.meta.core.env do addMessageContext m!"{e} : {← inferType e}" + | _ => unreachable! throwErrorAt f "ambiguous, possible interpretations {toMessageList msgs}" else withRef f <| mergeFailures candidates diff --git a/stage0/src/Lean/Elab/Attributes.lean b/stage0/src/Lean/Elab/Attributes.lean index 053dc8175110..5d2666e85c79 100644 --- a/stage0/src/Lean/Elab/Attributes.lean +++ b/stage0/src/Lean/Elab/Attributes.lean @@ -57,14 +57,17 @@ def elabAttr [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMa So, we expand them before here before we invoke the attributer handlers implemented using `AttrM`. -/ pure { kind := attrKind, name := attrName, stx := attr } -def elabAttrs [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] (attrInstances : Array Syntax) : m (Array Attribute) := do +def elabAttrs [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] [MonadLog m] [MonadLiftT IO m] (attrInstances : Array Syntax) : m (Array Attribute) := do let mut attrs := #[] for attr in attrInstances do - attrs := attrs.push (← elabAttr attr) + try + attrs := attrs.push (← withRef attr do elabAttr attr) + catch ex => + logException ex return attrs -- leading_parser "@[" >> sepBy1 attrInstance ", " >> "]" -def elabDeclAttrs [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] (stx : Syntax) : m (Array Attribute) := +def elabDeclAttrs [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] [MonadLog m] [MonadLiftT IO m] (stx : Syntax) : m (Array Attribute) := elabAttrs stx[1].getSepArgs end Lean.Elab diff --git a/stage0/src/Lean/Elab/Binders.lean b/stage0/src/Lean/Elab/Binders.lean index 199c5c6bf8a5..1f868114e59f 100644 --- a/stage0/src/Lean/Elab/Binders.lean +++ b/stage0/src/Lean/Elab/Binders.lean @@ -45,8 +45,8 @@ structure BinderView where bi : BinderInfo partial def quoteAutoTactic : Syntax → TermElabM Syntax - | stx@(Syntax.ident _ _ _ _) => throwErrorAt stx "invalid auto tactic, identifier is not allowed" - | stx@(Syntax.node _ k args) => do + | stx@(.ident ..) => throwErrorAt stx "invalid auto tactic, identifier is not allowed" + | stx@(.node _ k args) => do if stx.isAntiquot then throwErrorAt stx "invalid auto tactic, antiquotation is not allowed" else @@ -58,8 +58,8 @@ partial def quoteAutoTactic : Syntax → TermElabM Syntax let quotedArg ← quoteAutoTactic arg quotedArgs ← `(Array.push $quotedArgs $quotedArg) `(Syntax.node SourceInfo.none $(quote k) $quotedArgs) - | Syntax.atom _ val => `(mkAtom $(quote val)) - | Syntax.missing => throwError "invalid auto tactic, tactic is missing" + | .atom _ val => `(mkAtom $(quote val)) + | .missing => throwError "invalid auto tactic, tactic is missing" def declareTacticSyntax (tactic : Syntax) : TermElabM Name := withFreshMacroScope do @@ -108,28 +108,28 @@ private def matchBinder (stx : Syntax) : TermElabM (Array BinderView) := do let k := stx.getKind if stx.isIdent || k == ``hole then -- binderIdent - pure #[{ id := (← expandBinderIdent stx), type := mkHole stx, bi := BinderInfo.default }] + return #[{ id := (← expandBinderIdent stx), type := mkHole stx, bi := .default }] else if k == ``Lean.Parser.Term.explicitBinder then -- `(` binderIdent+ binderType (binderDefault <|> binderTactic)? `)` let ids ← getBinderIds stx[1] let type := stx[2] let optModifier := stx[3] - ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := (← expandBinderModifier (expandBinderType id type) optModifier), bi := BinderInfo.default } + ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := (← expandBinderModifier (expandBinderType id type) optModifier), bi := .default } else if k == ``Lean.Parser.Term.implicitBinder then -- `{` binderIdent+ binderType `}` let ids ← getBinderIds stx[1] let type := stx[2] - ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := expandBinderType id type, bi := BinderInfo.implicit } + ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := expandBinderType id type, bi := .implicit } else if k == ``Lean.Parser.Term.strictImplicitBinder then -- `⦃` binderIdent+ binderType `⦄` let ids ← getBinderIds stx[1] let type := stx[2] - ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := expandBinderType id type, bi := BinderInfo.strictImplicit } + ids.mapM fun id => do pure { id := (← expandBinderIdent id), type := expandBinderType id type, bi := .strictImplicit } else if k == ``Lean.Parser.Term.instBinder then -- `[` optIdent type `]` let id ← expandOptIdent stx[1] let type := stx[2] - pure #[ { id := id, type := type, bi := BinderInfo.instImplicit } ] + return #[ { id := id, type := type, bi := .instImplicit } ] else throwUnsupportedSyntax @@ -149,11 +149,11 @@ register_builtin_option checkBinderAnnotations : Bool := { descr := "check whether type is a class instance whenever the binder annotation `[...]` is used" } -private partial def elabBinderViews {α} (binderViews : Array BinderView) (fvars : Array (Syntax × Expr)) (k : Array (Syntax × Expr) → TermElabM α) +private partial def elabBinderViews (binderViews : Array BinderView) (fvars : Array (Syntax × Expr)) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := let rec loop (i : Nat) (fvars : Array (Syntax × Expr)) : TermElabM α := do if h : i < binderViews.size then - let binderView := binderViews.get ⟨i, h⟩ + let binderView := binderViews[i] ensureAtomicBinderName binderView let type ← elabType binderView.type registerFailedToInferBinderTypeInfo type binderView.type @@ -167,10 +167,10 @@ private partial def elabBinderViews {α} (binderViews : Array BinderView) (fvars k fvars loop 0 fvars -private partial def elabBindersAux {α} (binders : Array Syntax) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := +private partial def elabBindersAux (binders : Array Syntax) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := let rec loop (i : Nat) (fvars : Array (Syntax × Expr)) : TermElabM α := do if h : i < binders.size then - let binderViews ← matchBinder (binders.get ⟨i, h⟩) + let binderViews ← matchBinder binders[i] elabBinderViews binderViews fvars <| loop (i+1) else k fvars @@ -181,7 +181,7 @@ private partial def elabBindersAux {α} (binders : Array Syntax) (k : Array (Syn `elabBinders(Ex)` automatically adds binder info nodes for the produced fvars, but storing the syntax nodes might be necessary when later adding the same binders back to the local context so that info nodes can manually be added for the new fvars; see `MutualDef` for an example. -/ -def elabBindersEx {α} (binders : Array Syntax) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := +def elabBindersEx (binders : Array Syntax) (k : Array (Syntax × Expr) → TermElabM α) : TermElabM α := universeConstraintsCheckpoint do if binders.isEmpty then k #[] @@ -201,7 +201,7 @@ def elabBinders (binders : Array Syntax) (k : Array Expr → TermElabM α) : Ter elabBindersEx binders (fun fvars => k (fvars.map (·.2))) /-- Same as `elabBinder` with a single binder.-/ -def elabBinder {α} (binder : Syntax) (x : Expr → TermElabM α) : TermElabM α := +def elabBinder (binder : Syntax) (x : Expr → TermElabM α) : TermElabM α := elabBinders #[binder] fun fvars => x fvars[0]! def expandSimpleBinderWithType (type : Term) (binder : Syntax) : MacroM Syntax := @@ -289,7 +289,7 @@ private partial def getFunBinderIds? (stx : Syntax) : OptionT MacroM (Array Synt partial def expandFunBinders (binders : Array Syntax) (body : Syntax) : MacroM (Array Syntax × Syntax × Bool) := let rec loop (body : Syntax) (i : Nat) (newBinders : Array Syntax) := do if h : i < binders.size then - let binder := binders.get ⟨i, h⟩ + let binder := binders[i] let processAsPattern : Unit → MacroM (Array Syntax × Syntax × Bool) := fun _ => do let pattern := binder let major ← mkFreshIdent binder @@ -352,19 +352,19 @@ private def propagateExpectedType (fvar : Expr) (fvarType : Expr) (s : State) : | some expectedType => let expectedType ← whnfForall expectedType match expectedType with - | Expr.forallE _ d b _ => + | .forallE _ d b _ => discard <| isDefEq fvarType d let b := b.instantiate1 fvar - pure { s with expectedType? := some b } + return { s with expectedType? := some b } | _ => - pure { s with expectedType? := none } + return { s with expectedType? := none } private partial def elabFunBinderViews (binderViews : Array BinderView) (i : Nat) (s : State) : TermElabM State := do if h : i < binderViews.size then - let binderView := binderViews.get ⟨i, h⟩ + let binderView := binderViews[i] ensureAtomicBinderName binderView withRef binderView.type <| withLCtx s.lctx s.localInsts do - let type ← elabType binderView.type + let type ← elabType binderView.type registerFailedToInferBinderTypeInfo type binderView.type let fvarId ← mkFreshFVarId let fvar := mkFVar fvarId @@ -378,19 +378,19 @@ private partial def elabFunBinderViews (binderViews : Array BinderView) (i : Nat let lctx := s.lctx.mkLocalDecl fvarId binderView.id.getId type binderView.bi addTermInfo' (lctx? := some lctx) (isBinder := true) binderView.id fvar let s ← withRef binderView.id <| propagateExpectedType fvar type s - let s := { s with lctx := lctx } + let s := { s with lctx } match (← isClass? type) with | none => elabFunBinderViews binderViews (i+1) s | some className => resettingSynthInstanceCache do - let localInsts := s.localInsts.push { className := className, fvar := mkFVar fvarId } - elabFunBinderViews binderViews (i+1) { s with localInsts := localInsts } + let localInsts := s.localInsts.push { className, fvar := mkFVar fvarId } + elabFunBinderViews binderViews (i+1) { s with localInsts } else pure s partial def elabFunBindersAux (binders : Array Syntax) (i : Nat) (s : State) : TermElabM State := do if h : i < binders.size then - let binderViews ← matchBinder (binders.get ⟨i, h⟩) + let binderViews ← matchBinder binders[i] let s ← elabFunBinderViews binderViews 0 s elabFunBindersAux binders (i+1) s else @@ -398,13 +398,13 @@ partial def elabFunBindersAux (binders : Array Syntax) (i : Nat) (s : State) : T end FunBinders -def elabFunBinders {α} (binders : Array Syntax) (expectedType? : Option Expr) (x : Array Expr → Option Expr → TermElabM α) : TermElabM α := +def elabFunBinders (binders : Array Syntax) (expectedType? : Option Expr) (x : Array Expr → Option Expr → TermElabM α) : TermElabM α := if binders.isEmpty then x #[] expectedType? else do let lctx ← getLCtx let localInsts ← getLocalInstances - let s ← FunBinders.elabFunBindersAux binders 0 { lctx := lctx, localInsts := localInsts, expectedType? := expectedType? } + let s ← FunBinders.elabFunBindersAux binders 0 { lctx, localInsts, expectedType? } resettingSynthInstanceCacheWhen (s.localInsts.size > localInsts.size) <| withLCtx s.lctx s.localInsts <| x s.fvars s.expectedType? @@ -650,7 +650,7 @@ def mkLetIdDeclView (letIdDecl : Syntax) : LetIdDeclView := let optType := letIdDecl[2] let type := expandOptType id optType let value := letIdDecl[4] - { id := id, binders := binders, type := type, value := value } + { id, binders, type, value } def expandLetEqnsDecl (letDecl : Syntax) : MacroM Syntax := do let ref := letDecl @@ -662,8 +662,8 @@ def elabLetDeclCore (stx : Syntax) (expectedType? : Option Expr) (useLetExpr : B let letDecl := stx[1][0] let body := stx[3] if letDecl.getKind == ``Lean.Parser.Term.letIdDecl then - let { id := id, binders := binders, type := type, value := val } := mkLetIdDeclView letDecl - elabLetDeclAux id binders type val body expectedType? useLetExpr elabBodyFirst usedLetOnly + let { id, binders, type, value } := mkLetIdDeclView letDecl + elabLetDeclAux id binders type value body expectedType? useLetExpr elabBodyFirst usedLetOnly else if letDecl.getKind == ``Lean.Parser.Term.letPatDecl then -- node `Lean.Parser.Term.letPatDecl $ try (termParser >> pushNone >> optType >> " := ") >> termParser if elabBodyFirst then diff --git a/stage0/src/Lean/Elab/Command.lean b/stage0/src/Lean/Elab/Command.lean index f3c29074d192..a92f47af9206 100644 --- a/stage0/src/Lean/Elab/Command.lean +++ b/stage0/src/Lean/Elab/Command.lean @@ -259,18 +259,6 @@ register_builtin_option showPartialSyntaxErrors : Bool := { descr := "show elaboration errors from partial syntax trees (i.e. after parser recovery)" } -def withLogging (x : CommandElabM Unit) : CommandElabM Unit := do - try - x - catch ex => match ex with - | Exception.error _ _ => logException ex - | Exception.internal id _ => - if isAbortExceptionId id then - pure () - else - let idName ← liftIO <| id.getName; - logError m!"internal exception {idName}" - builtin_initialize registerTraceClass `Elab.command partial def elabCommand (stx : Syntax) : CommandElabM Unit := do diff --git a/stage0/src/Lean/Elab/DeclModifiers.lean b/stage0/src/Lean/Elab/DeclModifiers.lean index 45d454907360..2ba71001e75b 100644 --- a/stage0/src/Lean/Elab/DeclModifiers.lean +++ b/stage0/src/Lean/Elab/DeclModifiers.lean @@ -96,7 +96,7 @@ def expandOptDocComment? [Monad m] [MonadError m] (optDocComment : Syntax) : m ( section Methods -variable [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] +variable [Monad m] [MonadEnv m] [MonadResolveName m] [MonadError m] [MonadMacroAdapter m] [MonadRecDepth m] [MonadTrace m] [MonadOptions m] [AddMessageContext m] [MonadLog m] [MonadLiftT IO m] def elabModifiers (stx : Syntax) : m Modifiers := do let docCommentStx := stx[0] diff --git a/stage0/src/Lean/Elab/Declaration.lean b/stage0/src/Lean/Elab/Declaration.lean index ee14792a9084..afe1a8795077 100644 --- a/stage0/src/Lean/Elab/Declaration.lean +++ b/stage0/src/Lean/Elab/Declaration.lean @@ -13,7 +13,6 @@ import Lean.Elab.DeclarationRange namespace Lean.Elab.Command open Meta -open TSyntax.Compat private def ensureValidNamespace (name : Name) : MacroM Unit := do match name with @@ -143,7 +142,7 @@ private def inductiveSyntaxToView (modifiers : Modifiers) (decl : Syntax) : Comm classes ← getOptDerivingClasses decl[5] else computedFields ← (decl[5].getOptional?.map (·[1].getArgs) |>.getD #[]).mapM fun cf => withRef cf do - return { ref := cf, modifiers := cf[0], fieldId := cf[1].getId, type := cf[3], matchAlts := cf[4] } + return { ref := cf, modifiers := cf[0], fieldId := cf[1].getId, type := ⟨cf[3]⟩, matchAlts := ⟨cf[4]⟩ } classes ← getOptDerivingClasses decl[6] return { ref := decl @@ -180,19 +179,22 @@ def elabDeclaration : CommandElab := fun stx => do match (← liftMacroM <| expandDeclNamespace? stx) with | some (ns, newStx) => do let ns := mkIdentFrom stx ns - let newStx ← `(namespace $ns:ident $newStx end $ns:ident) + let newStx ← `(namespace $ns:ident $(⟨newStx⟩) end $ns:ident) withMacroExpansion stx newStx <| elabCommand newStx | none => do - let modifiers ← elabModifiers stx[0] let decl := stx[1] let declKind := decl.getKind if declKind == ``Lean.Parser.Command.«axiom» then + let modifiers ← elabModifiers stx[0] elabAxiom modifiers decl else if declKind == ``Lean.Parser.Command.«inductive» then + let modifiers ← elabModifiers stx[0] elabInductive modifiers decl else if declKind == ``Lean.Parser.Command.classInductive then + let modifiers ← elabModifiers stx[0] elabClassInductive modifiers decl else if declKind == ``Lean.Parser.Command.«structure» then + let modifiers ← elabModifiers stx[0] elabStructure modifiers decl else if isDefLike decl then elabMutualDef #[stx] (getTerminationHints stx) @@ -257,7 +259,7 @@ def expandMutualNamespace : Macro := fun stx => do | some ns => let ns := mkIdentFrom stx ns let stxNew := stx.setArg 1 (mkNullNode elemsNew) - `(namespace $ns:ident $stxNew end $ns:ident) + `(namespace $ns:ident $(⟨stxNew⟩) end $ns:ident) | none => Macro.throwUnsupported @[builtinMacro Lean.Parser.Command.mutual] @@ -310,9 +312,10 @@ def elabMutual : CommandElab := fun stx => do for attrKindStx in stx[2].getSepArgs do if attrKindStx.getKind == ``Lean.Parser.Command.eraseAttr then let attrName := attrKindStx[1].getId.eraseMacroScopes - unless isAttribute (← getEnv) attrName do - throwError "unknown attribute [{attrName}]" - toErase := toErase.push attrName + if isAttribute (← getEnv) attrName then + toErase := toErase.push attrName + else + logErrorAt attrKindStx "unknown attribute [{attrName}]" else attrInsts := attrInsts.push attrKindStx let attrs ← elabAttrs attrInsts @@ -323,35 +326,19 @@ def elabMutual : CommandElab := fun stx => do for attrName in toErase do Attribute.erase declName attrName -def expandInitCmd (builtin : Bool) : Macro := fun stx => do - let optVisibility := stx[0] - let optHeader := stx[2] - let doSeq := stx[3] - let attrId := mkIdentFrom stx <| if builtin then `builtinInit else `init - if optHeader.isNone then - unless optVisibility.isNone do - Macro.throwError "invalid initialization command, 'visibility' modifer is not allowed" - `(@[$attrId:ident]def initFn : IO Unit := do $doSeq) - else - let id := optHeader[0] - let type := optHeader[1][1] - if optVisibility.isNone then - `(def initFn : IO $type := do $doSeq - @[$attrId:ident initFn] opaque $id : $type) - else if optVisibility[0].getKind == ``Parser.Command.private then - `(def initFn : IO $type := do $doSeq - @[$attrId:ident initFn] private opaque $id : $type) - else if optVisibility[0].getKind == ``Parser.Command.protected then - `(def initFn : IO $type := do $doSeq - @[$attrId:ident initFn] protected opaque $id : $type) +@[builtinMacro Lean.Parser.Command.«initialize»] def expandInitialize : Macro + | stx@`($declModifiers:declModifiers $kw:initializeKeyword $[$id? : $type? ←]? $doSeq) => do + let attrId := mkIdentFrom stx <| if kw.raw[0].isToken "initialize" then `init else `builtinInit + if let (some id, some type) := (id?, type?) then + let `(Parser.Command.declModifiersT| $[$doc?:docComment]? $[@[$attrs?,*]]? $(vis?)? $[unsafe%$unsafe?]?) := stx[0] + | Macro.throwErrorAt declModifiers "invalid initialization command, unexpected modifiers" + `($[unsafe%$unsafe?]? def initFn : IO $type := do $doSeq + $[$doc?:docComment]? @[$attrId:ident initFn, $(attrs?.getD ∅),*] $(vis?)? opaque $id : $type) else - Macro.throwError "unexpected visibility annotation" - -@[builtinMacro Lean.Parser.Command.«initialize»] def expandInitialize : Macro := - expandInitCmd (builtin := false) - -@[builtinMacro Lean.Parser.Command.«builtin_initialize»] def expandBuiltinInitialize : Macro := - expandInitCmd (builtin := true) + let `(Parser.Command.declModifiersT| ) := declModifiers + | Macro.throwErrorAt declModifiers "invalid initialization command, unexpected modifiers" + `(@[$attrId:ident] def initFn : IO Unit := do $doSeq) + | _ => Macro.throwUnsupported builtin_initialize registerTraceClass `Elab.axiom diff --git a/stage0/src/Lean/Elab/Deriving/FromToJson.lean b/stage0/src/Lean/Elab/Deriving/FromToJson.lean index 32872a120701..a0c1f61b49d6 100644 --- a/stage0/src/Lean/Elab/Deriving/FromToJson.lean +++ b/stage0/src/Lean/Elab/Deriving/FromToJson.lean @@ -30,7 +30,7 @@ def mkToJsonInstanceHandler (declNames : Array Name) : CommandElabM Bool := do let (isOptField, nm) := mkJsonField field if isOptField then ``(opt $nm $(mkIdent <| header.targetNames[0]! ++ field)) else ``([($nm, toJson $(mkIdent <| header.targetNames[0]! ++ field))]) - let cmd ← `(private def $(mkIdent ctx.auxFunNames[0]!):ident $header.binders:bracketedBinder* := + let cmd ← `(private def $(mkIdent ctx.auxFunNames[0]!):ident $header.binders:bracketedBinder* : Json := mkObj <| List.join [$fields,*]) return #[cmd] ++ (← mkInstanceCmds ctx ``ToJson declNames) cmds.forM elabCommand @@ -63,9 +63,9 @@ def mkToJsonInstanceHandler (declNames : Array Name) : CommandElabM Bool := do if ctx.usePartial then let letDecls ← mkLocalInstanceLetDecls ctx ``ToJson header.argNames let auxTerm ← mkLet letDecls auxTerm - `(private partial def $toJsonFuncId:ident $header.binders:bracketedBinder* := $auxTerm) + `(private partial def $toJsonFuncId:ident $header.binders:bracketedBinder* : Json := $auxTerm) else - `(private def $toJsonFuncId:ident $header.binders:bracketedBinder* := $auxTerm) + `(private def $toJsonFuncId:ident $header.binders:bracketedBinder* : Json := $auxTerm) return #[auxCmd] ++ (← mkInstanceCmds ctx ``ToJson declNames) cmds.forM elabCommand return true diff --git a/stage0/src/Lean/Elab/Extra.lean b/stage0/src/Lean/Elab/Extra.lean index d092458f061c..3f78ad6ecc32 100644 --- a/stage0/src/Lean/Elab/Extra.lean +++ b/stage0/src/Lean/Elab/Extra.lean @@ -38,15 +38,15 @@ private def throwForInFailure (forInInstance : Expr) : TermElabM Expr := catch _ => tryPostpone; throwError "failed to construct 'ForIn' instance for collection{indentExpr colType}\nand monad{indentExpr m}" match (← trySynthInstance forInInstance) with - | LOption.some inst => + | .some inst => let forInFn ← mkConst ``forIn elabAppArgs forInFn (namedArgs := #[{ name := `m, val := Arg.expr m}, { name := `α, val := Arg.expr elemType }, { name := `self, val := Arg.expr inst }]) (args := #[Arg.stx col, Arg.stx init, Arg.stx body]) (expectedType? := expectedType?) (explicit := false) (ellipsis := false) (resultIsOutParamSupport := false) - | LOption.undef => tryPostpone; throwForInFailure forInInstance - | LOption.none => throwForInFailure forInInstance + | .undef => tryPostpone; throwForInFailure forInInstance + | .none => throwForInFailure forInInstance | _ => throwUnsupportedSyntax @[builtinTermElab forInMacro'] def elabForIn' : TermElab := fun stx expectedType? => do @@ -66,15 +66,15 @@ private def throwForInFailure (forInInstance : Expr) : TermElabM Expr := catch _ => tryPostpone; throwError "failed to construct `ForIn'` instance for collection{indentExpr colType}\nand monad{indentExpr m}" match (← trySynthInstance forInInstance) with - | LOption.some inst => + | .some inst => let forInFn ← mkConst ``forIn' elabAppArgs forInFn (namedArgs := #[{ name := `m, val := Arg.expr m}, { name := `α, val := Arg.expr elemType}, { name := `self, val := Arg.expr inst }]) (args := #[Arg.expr colFVar, Arg.stx init, Arg.stx body]) (expectedType? := expectedType?) (explicit := false) (ellipsis := false) (resultIsOutParamSupport := false) - | LOption.undef => tryPostpone; throwForInFailure forInInstance - | LOption.none => throwForInFailure forInInstance + | .undef => tryPostpone; throwForInFailure forInInstance + | .none => throwForInFailure forInInstance | _ => throwUnsupportedSyntax namespace BinOp @@ -157,9 +157,9 @@ private def hasCoe (fromType toType : Expr) : TermElabM Bool := do let v ← getLevel toType let coeInstType := mkAppN (Lean.mkConst ``CoeHTCT [u, v]) #[fromType, toType] match ← trySynthInstance coeInstType (some (maxCoeSize.get (← getOptions))) with - | LOption.some _ => return true - | LOption.none => return false - | LOption.undef => return false -- TODO: should we do something smarter here? + | .some _ => return true + | .none => return false + | .undef => return false -- TODO: should we do something smarter here? else return false @@ -168,10 +168,10 @@ private structure AnalyzeResult where hasUncomparable : Bool := false -- `true` if there are two types `α` and `β` where we don't have coercions in any direction. private def isUnknow : Expr → Bool - | Expr.mvar .. => true - | Expr.app f .. => isUnknow f - | Expr.letE _ _ _ b _ => isUnknow b - | Expr.mdata _ b => isUnknow b + | .mvar .. => true + | .app f _ => isUnknow f + | .letE _ _ _ b _ => isUnknow b + | .mdata _ b => isUnknow b | _ => false private def analyze (t : Tree) (expectedType? : Option Expr) : TermElabM AnalyzeResult := do @@ -205,15 +205,11 @@ where private def mkOp (f : Expr) (lhs rhs : Expr) : TermElabM Expr := elabAppArgs f #[] #[Arg.expr lhs, Arg.expr rhs] (expectedType? := none) (explicit := false) (ellipsis := false) (resultIsOutParamSupport := false) -private def toExpr (t : Tree) : TermElabM Expr := do +private def toExprCore (t : Tree) : TermElabM Expr := do match t with - | Tree.term _ e => return e - | Tree.op ref true f lhs rhs => withRef ref <| mkOp f (← toExpr lhs) (← mkFunUnit (← toExpr rhs)) - | Tree.op ref false f lhs rhs => withRef ref <| mkOp f (← toExpr lhs) (← toExpr rhs) - -private def getResultingType : Expr → Expr - | .forallE _ _ b _ => getResultingType b - | e => e + | .term _ e => return e + | .op ref true f lhs rhs => withRef ref <| mkOp f (← toExprCore lhs) (← mkFunUnit (← toExprCore rhs)) + | .op ref false f lhs rhs => withRef ref <| mkOp f (← toExprCore lhs) (← toExprCore rhs) /-- Auxiliary function to decide whether we should coerce `f`'s argument to `maxType` or not. @@ -245,66 +241,96 @@ private def hasHeterogeneousDefaultInstances (f : Expr) (maxType : Expr) (lhs : let className := fName.getPrefix let defInstances ← getDefaultInstances className if defInstances.length ≤ 1 then return false - for (instName, _) in (← getDefaultInstances className) do - let instInfo ← getConstInfo instName - let type := getResultingType instInfo.type - if type.getAppNumArgs >= 3 then - if lhs then - return type.appFn!.appArg!.isAppOf typeName - else - return type.appFn!.appArg!.appArg!.isAppOf typeName + for (instName, _) in defInstances do + if let .app (.app (.app _heteroClass lhsType) rhsType) _resultType := + (← getConstInfo instName).type.getForallBody then + if lhs && rhsType.isAppOf typeName then return true + if !lhs && lhsType.isAppOf typeName then return true return false /-- - Try to coerce elements in the `t` to `maxType` when needed. - If the type of an element in `t` is unknown we only coerce it to `maxType` if `maxType` does not have heterogeneous - default instances. This extra check is approximated by `hasHeterogeneousDefaultInstances`. + Return `true` if polymorphic function `f` has a homogenous instance of `maxType`. + The coercions to `maxType` only makes sense if such instance exists. - Remark: If `maxType` does not implement heterogeneous default instances, we do want to assign unknown types `?m` to - `maxType` because it produces better type information propagation. Our test suite has many tests that would break if - we don't do this. For example, consider the term - ``` - eq_of_isEqvAux a b hsz (i+1) (Nat.succ_le_of_lt h) heqv.2 - ``` - `Nat.succ_le_of_lt h` type depends on `i+1`, but `i+1` only reduces to `Nat.succ i` if we know that `1` is a `Nat`. - There are several other examples like that in our test suite, and one can find them by just replacing the - `← hasHeterogeneousDefaultInstances f maxType lhs` test with `true` + For example, suppose `maxType` is `Int`, and `f` is `HPow.hPow`. Then, + adding coercions to `maxType` only make sense if we have an instance `HPow Int Int Int`. +-/ +private def hasHomogeneousInstance (f : Expr) (maxType : Expr) : MetaM Bool := do + let .const fName .. := f | return false + let className := fName.getPrefix + try + let inst ← mkAppM className #[maxType, maxType, maxType] + return (← trySynthInstance inst) matches .some _ + catch _ => + return false +mutual + /-- + Try to coerce elements in the `t` to `maxType` when needed. + If the type of an element in `t` is unknown we only coerce it to `maxType` if `maxType` does not have heterogeneous + default instances. This extra check is approximated by `hasHeterogeneousDefaultInstances`. + + Remark: If `maxType` does not implement heterogeneous default instances, we do want to assign unknown types `?m` to + `maxType` because it produces better type information propagation. Our test suite has many tests that would break if + we don't do this. For example, consider the term + ``` + eq_of_isEqvAux a b hsz (i+1) (Nat.succ_le_of_lt h) heqv.2 + ``` + `Nat.succ_le_of_lt h` type depends on `i+1`, but `i+1` only reduces to `Nat.succ i` if we know that `1` is a `Nat`. + There are several other examples like that in our test suite, and one can find them by just replacing the + `← hasHeterogeneousDefaultInstances f maxType lhs` test with `true` + + + Remark: if `hasHeterogeneousDefaultInstances` implementation is not good enough we should refine it in the future. + -/ + private partial def applyCoe (t : Tree) (maxType : Expr) (isPred : Bool) : TermElabM Tree := do + go t none false isPred + where + go (t : Tree) (f? : Option Expr) (lhs : Bool) (isPred : Bool) : TermElabM Tree := do + match t with + | .op ref lazy f lhs rhs => + /- + We only keep applying coercions to `maxType` if `f` is predicate or + `f` has a homogenous instance with `maxType`. See `hasHomogeneousInstance` for additional details. + + Remark: We assume `binrel%` elaborator is only used with homogenous predicates. + -/ + if (← pure isPred <||> hasHomogeneousInstance f maxType) then + return Tree.op ref lazy f (← go lhs f true false) (← go rhs f false false) + else + let lhs ← toExpr lhs none + let rhs ← toExpr rhs none + return Tree.term ref (← mkOp f lhs rhs) + | .term ref e => + let type ← instantiateMVars (← inferType e) + trace[Elab.binop] "visiting {e} : {type} =?= {maxType}" + if isUnknow type then + if let some f := f? then + if (← hasHeterogeneousDefaultInstances f maxType lhs) then + -- See comment at `hasHeterogeneousDefaultInstances` + return t + if (← isDefEqGuarded maxType type) then + return t + else + trace[Elab.binop] "added coercion: {e} : {type} => {maxType}" + withRef ref <| return Tree.term ref (← mkCoe maxType type e) + + private partial def toExpr (tree : Tree) (expectedType? : Option Expr) : TermElabM Expr := do + let r ← analyze tree expectedType? + trace[Elab.binop] "hasUncomparable: {r.hasUncomparable}, maxType: {r.max?}" + if r.hasUncomparable || r.max?.isNone then + let result ← toExprCore tree + ensureHasType expectedType? result + else + let result ← toExprCore (← applyCoe tree r.max?.get! (isPred := false)) + trace[Elab.binop] "result: {result}" + ensureHasType expectedType? result - Remark: if `hasHeterogeneousDefaultInstances` implementation is not good enough we should refine it in the future. --/ -private def applyCoe (t : Tree) (maxType : Expr) : TermElabM Tree := do - go t none false -where - go (t : Tree) (f? : Option Expr) (lhs : Bool) : TermElabM Tree := do - match t with - | Tree.op ref lazy f lhs rhs => return Tree.op ref lazy f (← go lhs f true) (← go rhs f false) - | Tree.term ref e => - let type ← instantiateMVars (← inferType e) - trace[Elab.binop] "visiting {e} : {type} =?= {maxType}" - if isUnknow type then - if let some f := f? then - if (← hasHeterogeneousDefaultInstances f maxType lhs) then - -- See comment at `hasHeterogeneousDefaultInstances` - return t - if (← isDefEqGuarded maxType type) then - return t - else - trace[Elab.binop] "added coercion: {e} : {type} => {maxType}" - withRef ref <| return Tree.term ref (← mkCoe maxType type e) +end @[builtinTermElab binop] def elabBinOp : TermElab := fun stx expectedType? => do - let tree ← toTree stx - let r ← analyze tree expectedType? - trace[Elab.binop] "hasUncomparable: {r.hasUncomparable}, maxType: {r.max?}" - if r.hasUncomparable || r.max?.isNone then - let result ← toExpr tree - ensureHasType expectedType? result - else - let result ← toExpr (← applyCoe tree r.max?.get!) - trace[Elab.binop] "result: {result}" - ensureHasType expectedType? result + toExpr (← toTree stx) expectedType? @[builtinTermElab binop_lazy] def elabBinOpLazy : TermElab := elabBinOp @@ -327,8 +353,8 @@ def elabBinRelCore (noProp : Bool) (stx : Syntax) (expectedType? : Option Expr) trace[Elab.binrel] "hasUncomparable: {r.hasUncomparable}, maxType: {r.max?}" if r.hasUncomparable || r.max?.isNone then -- Use default elaboration strategy + `toBoolIfNecessary` - let lhs ← toExpr lhs - let rhs ← toExpr rhs + let lhs ← toExprCore lhs + let rhs ← toExprCore rhs let lhs ← toBoolIfNecessary lhs let rhs ← toBoolIfNecessary rhs let lhsType ← inferType lhs @@ -340,7 +366,7 @@ def elabBinRelCore (noProp : Bool) (stx : Syntax) (expectedType? : Option Expr) if noProp then if (← withNewMCtxDepth <| isDefEq maxType (mkSort levelZero)) then maxType := Lean.mkConst ``Bool - let result ← toExpr (← applyCoe tree maxType) + let result ← toExprCore (← applyCoe tree maxType (isPred := true)) trace[Elab.binrel] "result: {result}" return result | none => throwUnknownConstant stx[1].getId diff --git a/stage0/src/Lean/Elab/Match.lean b/stage0/src/Lean/Elab/Match.lean index 5228c0c44ff6..8c9cbd8b5dae 100644 --- a/stage0/src/Lean/Elab/Match.lean +++ b/stage0/src/Lean/Elab/Match.lean @@ -649,8 +649,8 @@ where /- The `Bool` context is true iff we are inside of an "inaccessible" pattern. -/ go (p : Expr) : ReaderT Bool TermElabM Expr := do match p with - | .forallE n d b _ => withLocalDecl n b.binderInfo (← go d) fun x => do mkForallFVars #[x] (← go (b.instantiate1 x)) - | .lam n d b _ => withLocalDecl n b.binderInfo (← go d) fun x => do mkLambdaFVars #[x] (← go (b.instantiate1 x)) + | .forallE n d b bi => withLocalDecl n bi (← go d) fun x => do mkForallFVars #[x] (← go (b.instantiate1 x)) + | .lam n d b bi => withLocalDecl n bi (← go d) fun x => do mkLambdaFVars #[x] (← go (b.instantiate1 x)) | .letE n t v b .. => withLetDecl n (← go t) (← go v) fun x => do mkLetFVars #[x] (← go (b.instantiate1 x)) | .app f a => return mkApp (← go f) (← go a) | .proj _ _ b => return p.updateProj! (← go b) @@ -1086,14 +1086,16 @@ private def elabMatchAux (generalizing? : Option Bool) (discrStxs : Array Syntax -/ withRef altLHS.ref do for d in altLHS.fvarDecls do - if d.hasExprMVar then + if d.hasExprMVar then + tryPostpone withExistingLocalDecls altLHS.fvarDecls do - tryPostpone - throwMVarError m!"invalid match-expression, type of pattern variable '{d.toExpr}' contains metavariables{indentExpr d.type}" + runPendingTacticsAt d.type + if (← instantiateMVars d.type).hasExprMVar then + throwMVarError m!"invalid match-expression, type of pattern variable '{d.toExpr}' contains metavariables{indentExpr d.type}" for p in altLHS.patterns do - if p.hasExprMVar then + if (← Match.instantiatePatternMVars p).hasExprMVar then + tryPostpone withExistingLocalDecls altLHS.fvarDecls do - tryPostpone throwMVarError m!"invalid match-expression, pattern contains metavariables{indentExpr (← p.toExpr)}" pure altLHS return (discrs, matchType, altLHSS, isDep, rhss) diff --git a/stage0/src/Lean/Elab/MutualDef.lean b/stage0/src/Lean/Elab/MutualDef.lean index ca704343cf7e..7d0eccf1c178 100644 --- a/stage0/src/Lean/Elab/MutualDef.lean +++ b/stage0/src/Lean/Elab/MutualDef.lean @@ -777,9 +777,14 @@ where withFunLocalDecls headers fun funFVars => do for view in views, funFVar in funFVars do addLocalVarInfo view.declId funFVar - let values ← elabFunValues headers - Term.synthesizeSyntheticMVarsNoPostponing - let values ← values.mapM (instantiateMVars ·) + let values ← + try + let values ← elabFunValues headers + Term.synthesizeSyntheticMVarsNoPostponing + values.mapM (instantiateMVars ·) + catch ex => + logException ex + headers.mapM fun header => mkSorry header.type (synthetic := true) let headers ← headers.mapM instantiateMVarsAtHeader let letRecsToLift ← getLetRecsToLift let letRecsToLift ← letRecsToLift.mapM instantiateMVarsAtLetRecToLift diff --git a/stage0/src/Lean/Elab/Structure.lean b/stage0/src/Lean/Elab/Structure.lean index 9a1976b96042..8496c9d5a399 100644 --- a/stage0/src/Lean/Elab/Structure.lean +++ b/stage0/src/Lean/Elab/Structure.lean @@ -500,7 +500,7 @@ private def elabFieldTypeValue (view : StructFieldView) : TermElabM (Option Expr Term.synthesizeSyntheticMVarsNoPostponing -- TODO: add forbidden predicate using `shortDeclName` from `view` let params ← Term.addAutoBoundImplicits params - let value ← Term.elabTerm valStx none + let value ← Term.withoutAutoBoundImplicit <| Term.elabTerm valStx none let value ← mkLambdaFVars params value return (none, value) | some typeStx => @@ -512,7 +512,7 @@ private def elabFieldTypeValue (view : StructFieldView) : TermElabM (Option Expr let type ← mkForallFVars params type return (type, none) | some valStx => - let value ← Term.elabTermEnsuringType valStx type + let value ← Term.withoutAutoBoundImplicit <| Term.elabTermEnsuringType valStx type Term.synthesizeSyntheticMVarsNoPostponing let type ← mkForallFVars params type let value ← mkLambdaFVars params value diff --git a/stage0/src/Lean/Elab/Syntax.lean b/stage0/src/Lean/Elab/Syntax.lean index 65eaaaa4f5f1..56e77d5b9f5e 100644 --- a/stage0/src/Lean/Elab/Syntax.lean +++ b/stage0/src/Lean/Elab/Syntax.lean @@ -325,7 +325,7 @@ def resolveSyntaxKind (k : Name) : CommandElabM Name := do throwError "invalid syntax node kind '{k}'" @[builtinCommandElab «syntax»] def elabSyntax : CommandElab := fun stx => do - let `($[$doc?:docComment]? $attrKind:attrKind syntax $[: $prec? ]? $[(name := $name?)]? $[(priority := $prio?)]? $[$ps:stx]* : $catStx) ← pure stx + let `($[$doc?:docComment]? $[ @[ $attrInstances:attrInstance,* ] ]? $attrKind:attrKind syntax $[: $prec? ]? $[(name := $name?)]? $[(priority := $prio?)]? $[$ps:stx]* : $catStx) ← pure stx | throwUnsupportedSyntax let cat := catStx.getId.eraseMacroScopes unless (Parser.isParserCategory (← getEnv) cat) do @@ -344,11 +344,14 @@ def resolveSyntaxKind (k : Name) : CommandElabM Name := do let catParserId := mkIdentFrom stx (cat.appendAfter "Parser") let (val, lhsPrec?) ← runTermElabM none fun _ => Term.toParserDescr syntaxParser cat let declName := mkIdentFrom stx name + let attrInstance ← `(attrInstance| $attrKind:attrKind $catParserId:ident $(quote prio):num) + let attrInstances := attrInstances.getD { elemsAndSeps := #[] } + let attrInstances := attrInstances.push attrInstance let d ← if let some lhsPrec := lhsPrec? then - `($[$doc?:docComment]? @[$attrKind:attrKind $catParserId:ident $(quote prio):num] def $declName:ident : Lean.TrailingParserDescr := + `($[$doc?:docComment]? @[$attrInstances,*] def $declName:ident : Lean.TrailingParserDescr := ParserDescr.trailingNode $(quote stxNodeKind) $(quote prec) $(quote lhsPrec) $val) else - `($[$doc?:docComment]? @[$attrKind:attrKind $catParserId:ident $(quote prio):num] def $declName:ident : Lean.ParserDescr := + `($[$doc?:docComment]? @[$attrInstances,*] def $declName:ident : Lean.ParserDescr := ParserDescr.node $(quote stxNodeKind) $(quote prec) $val) trace `Elab fun _ => d withMacroExpansion stx d <| elabCommand d diff --git a/stage0/src/Lean/Elab/SyntheticMVars.lean b/stage0/src/Lean/Elab/SyntheticMVars.lean index 7d34da61635b..5ef71672f20e 100644 --- a/stage0/src/Lean/Elab/SyntheticMVars.lean +++ b/stage0/src/Lean/Elab/SyntheticMVars.lean @@ -23,7 +23,7 @@ private def resumeElabTerm (stx : Syntax) (expectedType? : Option Expr) (errToSo It is used to implement `synthesizeSyntheticMVars`. -/ private def resumePostponed (savedContext : SavedContext) (stx : Syntax) (mvarId : MVarId) (postponeOnError : Bool) : TermElabM Bool := withRef stx <| withMVarContext mvarId do - let s ← get + let s ← saveState try withSavedContext savedContext do let mvarDecl ← getMVarDecl mvarId @@ -40,15 +40,15 @@ private def resumePostponed (savedContext : SavedContext) (stx : Syntax) (mvarId else return false catch - | ex@(Exception.internal id _) => + | ex@(.internal id _) => if id == postponeExceptionId then - set s + s.restore (restoreInfo := true) return false else throw ex - | ex@(Exception.error _ _) => + | ex@(.error ..) => if postponeOnError then - set s + s.restore (restoreInfo := true) return false else logException ex @@ -62,8 +62,8 @@ private def synthesizePendingInstMVar (instMVar : MVarId) : TermElabM Bool := try synthesizeInstMVarCore instMVar catch - | ex@(Exception.error _ _) => logException ex; return true - | _ => unreachable! + | ex@(.error ..) => logException ex; return true + | _ => unreachable! /-- Similar to `synthesizePendingInstMVar`, but generates type mismatch error message. @@ -95,8 +95,8 @@ private def synthesizePendingCoeInstMVar return true return false catch - | Exception.error _ msg => throwTypeMismatchError errorMsgHeader? expectedType eType e f? msg - | _ => unreachable! + | .error _ msg => throwTypeMismatchError errorMsgHeader? expectedType eType e f? msg + | _ => unreachable! /-- Try to synthesize `mvarId` by starting using a default instance with the give privority. @@ -205,23 +205,23 @@ where /- Used to implement `synthesizeUsingDefault`. This method only consider default instances with the given priority. -/ private def synthesizeSomeUsingDefaultPrio (prio : Nat) : TermElabM Bool := do - let rec visit (syntheticMVars : List SyntheticMVarDecl) (syntheticMVarsNew : List SyntheticMVarDecl) : TermElabM Bool := do - match syntheticMVars with + let rec visit (pendingMVars : List MVarId) (pendingMVarsNew : List MVarId) : TermElabM Bool := do + match pendingMVars with | [] => return false - | mvarDecl :: mvarDecls => + | mvarId :: pendingMVars => + let some mvarDecl ← getSyntheticMVarDecl? mvarId | visit pendingMVars (mvarId :: pendingMVarsNew) match mvarDecl.kind with - | SyntheticMVarKind.typeClass => - if (← withRef mvarDecl.stx <| synthesizeUsingDefaultPrio mvarDecl.mvarId prio) then - let syntheticMVarsNew := mvarDecls.reverse ++ syntheticMVarsNew - modify fun s => { s with syntheticMVars := syntheticMVarsNew } + | .typeClass => + if (← withRef mvarDecl.stx <| synthesizeUsingDefaultPrio mvarId prio) then + modify fun s => { s with pendingMVars := pendingMVars.reverse ++ pendingMVarsNew } return true else - visit mvarDecls (mvarDecl :: syntheticMVarsNew) - | _ => visit mvarDecls (mvarDecl :: syntheticMVarsNew) - /- Recall that s.syntheticMVars is essentially a stack. The first metavariable was the last one created. + visit pendingMVars (mvarId :: pendingMVarsNew) + | _ => visit pendingMVars (mvarId :: pendingMVarsNew) + /- Recall that s.pendingMVars is essentially a stack. The first metavariable was the last one created. We want to apply the default instance in reverse creation order. Otherwise, `toString 0` will produce a `OfNat String _` cannot be synthesized error. -/ - visit (← get).syntheticMVars.reverse [] + visit (← get).pendingMVars.reverse [] /-- Apply default value to any pending synthetic metavariable of kind `SyntheticMVarKind.withDefault` @@ -234,16 +234,17 @@ private def synthesizeUsingDefault : TermElabM Bool := do return true return false -def reportStuckSyntheticMVar (mvarSyntheticDecl : SyntheticMVarDecl) (ignoreStuckTC := false) : TermElabM Unit := +def reportStuckSyntheticMVar (mvarId : MVarId) (ignoreStuckTC := false) : TermElabM Unit := do + let some mvarSyntheticDecl ← getSyntheticMVarDecl? mvarId | return () withRef mvarSyntheticDecl.stx do match mvarSyntheticDecl.kind with - | SyntheticMVarKind.typeClass => + | .typeClass => unless ignoreStuckTC do - withMVarContext mvarSyntheticDecl.mvarId do - let mvarDecl ← getMVarDecl mvarSyntheticDecl.mvarId + withMVarContext mvarId do + let mvarDecl ← getMVarDecl mvarId unless (← MonadLog.hasErrors) do throwError "typeclass instance problem is stuck, it is often due to metavariables{indentExpr mvarDecl.type}" - | SyntheticMVarKind.coe header eNew expectedType eType e f? => + | .coe header eNew expectedType eType e f? => let mvarId := eNew.appArg!.mvarId! withMVarContext mvarId do let mvarDecl ← getMVarDecl mvarId @@ -255,15 +256,16 @@ def reportStuckSyntheticMVar (mvarSyntheticDecl : SyntheticMVarDecl) (ignoreStuc Remark: we set `ignoreStuckTC := true` when elaborating `simp` arguments. -/ private def reportStuckSyntheticMVars (ignoreStuckTC := false) : TermElabM Unit := do - let syntheticMVars ← modifyGet fun s => (s.syntheticMVars, { s with syntheticMVars := [] }) - for mvarSyntheticDecl in syntheticMVars do - reportStuckSyntheticMVar mvarSyntheticDecl ignoreStuckTC + let pendingMVars ← modifyGet fun s => (s.pendingMVars, { s with pendingMVars := [] }) + for mvarId in pendingMVars do + reportStuckSyntheticMVar mvarId ignoreStuckTC private def getSomeSynthethicMVarsRef : TermElabM Syntax := do - let s ← get - match s.syntheticMVars.find? fun (mvarDecl : SyntheticMVarDecl) => !mvarDecl.stx.getPos?.isNone with - | some mvarDecl => return mvarDecl.stx - | none => return Syntax.missing + for mvarId in (← get).pendingMVars do + if let some decl ← getSyntheticMVarDecl? mvarId then + if decl.stx.getPos?.isSome then + return decl.stx + return .missing /-- Generate an nicer error message for stuck universe constraints. @@ -307,6 +309,13 @@ private def processPostponedUniverseContraints : TermElabM Unit := do unless (← processPostponed (mayPostpone := false) (exceptionOnFailure := true)) do throwStuckAtUniverseCnstr +/-- + Remove `mvarId` from the `syntheticMVars` table. We use this method after + the metavariable has been synthesized. +-/ +private def markAsResolved (mvarId : MVarId) : TermElabM Unit := + modify fun s => { s with syntheticMVars := s.syntheticMVars.erase mvarId } + mutual partial def runTactic (mvarId : MVarId) (tacticCode : Syntax) : TermElabM Unit := do @@ -320,17 +329,18 @@ mutual reportUnsolvedGoals remainingGoals /-- Try to synthesize the given pending synthetic metavariable. -/ - private partial def synthesizeSyntheticMVar (mvarSyntheticDecl : SyntheticMVarDecl) (postponeOnError : Bool) (runTactics : Bool) : TermElabM Bool := + private partial def synthesizeSyntheticMVar (mvarId : MVarId) (postponeOnError : Bool) (runTactics : Bool) : TermElabM Bool := do + let some mvarSyntheticDecl ← getSyntheticMVarDecl? mvarId | return true -- The metavariable has already been synthesized withRef mvarSyntheticDecl.stx do match mvarSyntheticDecl.kind with - | SyntheticMVarKind.typeClass => synthesizePendingInstMVar mvarSyntheticDecl.mvarId - | SyntheticMVarKind.coe header? eNew expectedType eType e f? => synthesizePendingCoeInstMVar mvarSyntheticDecl.mvarId header? eNew expectedType eType e f? + | .typeClass => synthesizePendingInstMVar mvarId + | .coe header? eNew expectedType eType e f? => synthesizePendingCoeInstMVar mvarId header? eNew expectedType eType e f? -- NOTE: actual processing at `synthesizeSyntheticMVarsAux` - | SyntheticMVarKind.postponed savedContext => resumePostponed savedContext mvarSyntheticDecl.stx mvarSyntheticDecl.mvarId postponeOnError - | SyntheticMVarKind.tactic tacticCode savedContext => + | .postponed savedContext => resumePostponed savedContext mvarSyntheticDecl.stx mvarId postponeOnError + | .tactic tacticCode savedContext => withSavedContext savedContext do if runTactics then - runTactic mvarSyntheticDecl.mvarId tacticCode + runTactic mvarId tacticCode return true else return false @@ -341,26 +351,27 @@ mutual let ctx ← read traceAtCmdPos `Elab.resuming fun _ => m!"resuming synthetic metavariables, mayPostpone: {ctx.mayPostpone}, postponeOnError: {postponeOnError}" - let syntheticMVars := (← get).syntheticMVars - let numSyntheticMVars := syntheticMVars.length - -- We reset `syntheticMVars` because new synthetic metavariables may be created by `synthesizeSyntheticMVar`. - modify fun s => { s with syntheticMVars := [] } - -- Recall that `syntheticMVars` is a list where head is the most recent pending synthetic metavariable. + let pendingMVars := (← get).pendingMVars + let numSyntheticMVars := pendingMVars.length + -- We reset `pendingMVars` because new synthetic metavariables may be created by `synthesizeSyntheticMVar`. + modify fun s => { s with pendingMVars := [] } + -- Recall that `pendingMVars` is a list where head is the most recent pending synthetic metavariable. -- We use `filterRevM` instead of `filterM` to make sure we process the synthetic metavariables using the order they were created. -- It would not be incorrect to use `filterM`. - let remainingSyntheticMVars ← syntheticMVars.filterRevM fun mvarDecl => do + let remainingPendingMVars ← pendingMVars.filterRevM fun mvarId => do -- We use `traceM` because we want to make sure the metavar local context is used to trace the message - traceM `Elab.postpone (withMVarContext mvarDecl.mvarId do addMessageContext m!"resuming {mkMVar mvarDecl.mvarId}") - let succeeded ← synthesizeSyntheticMVar mvarDecl postponeOnError runTactics + traceM `Elab.postpone (withMVarContext mvarId do addMessageContext m!"resuming {mkMVar mvarId}") + let succeeded ← synthesizeSyntheticMVar mvarId postponeOnError runTactics + if succeeded then markAsResolved mvarId trace[Elab.postpone] if succeeded then format "succeeded" else format "not ready yet" pure !succeeded - -- Merge new synthetic metavariables with `remainingSyntheticMVars`, i.e., metavariables that still couldn't be synthesized - modify fun s => { s with syntheticMVars := s.syntheticMVars ++ remainingSyntheticMVars } - return numSyntheticMVars != remainingSyntheticMVars.length + -- Merge new synthetic metavariables with `remainingPendingMVars`, i.e., metavariables that still couldn't be synthesized + modify fun s => { s with pendingMVars := s.pendingMVars ++ remainingPendingMVars } + return numSyntheticMVars != remainingPendingMVars.length /-- Try to process pending synthetic metavariables. If `mayPostpone == false`, - then `syntheticMVars` is `[]` after executing this method. + then `pendingMVars` is `[]` after executing this method. It keeps executing `synthesizeSyntheticMVarsStep` while progress is being made. If `mayPostpone == false`, then it applies default instances to `SyntheticMVarKind.typeClass` (if available) @@ -374,7 +385,7 @@ mutual partial def synthesizeSyntheticMVars (mayPostpone := true) (ignoreStuckTC := false) : TermElabM Unit := do let rec loop (_ : Unit) : TermElabM Unit := do withRef (← getSomeSynthethicMVarsRef) <| withIncRecDepth do - unless (← get).syntheticMVars.isEmpty do + unless (← get).pendingMVars.isEmpty do if ← synthesizeSyntheticMVarsStep (postponeOnError := false) (runTactics := false) then loop () else if !mayPostpone then @@ -423,8 +434,8 @@ def synthesizeSyntheticMVarsUsingDefault : TermElabM Unit := do synthesizeUsingDefaultLoop private partial def withSynthesizeImp {α} (k : TermElabM α) (mayPostpone : Bool) (synthesizeDefault : Bool) : TermElabM α := do - let syntheticMVarsSaved := (← get).syntheticMVars - modify fun s => { s with syntheticMVars := [] } + let pendingMVarsSaved := (← get).pendingMVars + modify fun s => { s with pendingMVars := [] } try let a ← k synthesizeSyntheticMVars mayPostpone @@ -432,7 +443,7 @@ private partial def withSynthesizeImp {α} (k : TermElabM α) (mayPostpone : Boo synthesizeUsingDefaultLoop return a finally - modify fun s => { s with syntheticMVars := s.syntheticMVars ++ syntheticMVarsSaved } + modify fun s => { s with pendingMVars := s.pendingMVars ++ pendingMVarsSaved } /-- Execute `k`, and synthesize pending synthetic metavariables created while executing `k` are solved. @@ -450,6 +461,14 @@ def elabTermAndSynthesize (stx : Syntax) (expectedType? : Option Expr) : TermEla withRef stx do instantiateMVars (← withSynthesize <| elabTerm stx expectedType?) +def runPendingTacticsAt (e : Expr) : TermElabM Unit := do + for mvarId in (← getMVars e) do + let mvarId ← getDelayedMVarRoot mvarId + if let some { kind := .tactic tacticCode savedContext, .. } ← getSyntheticMVarDecl? mvarId then + withSavedContext savedContext do + runTactic mvarId tacticCode + markAsResolved mvarId + builtin_initialize registerTraceClass `Elab.resume diff --git a/stage0/src/Lean/Elab/Tactic/Basic.lean b/stage0/src/Lean/Elab/Tactic/Basic.lean index 8a53d25144a4..7021483c5d2e 100644 --- a/stage0/src/Lean/Elab/Tactic/Basic.lean +++ b/stage0/src/Lean/Elab/Tactic/Basic.lean @@ -79,8 +79,8 @@ def getUnsolvedGoals : TacticM (List MVarId) := do def run (mvarId : MVarId) (x : TacticM Unit) : TermElabM (List MVarId) := withMVarContext mvarId do - let savedSyntheticMVars := (← get).syntheticMVars - modify fun s => { s with syntheticMVars := [] } + let pendingMVarsSaved := (← get).pendingMVars + modify fun s => { s with pendingMVars := [] } let aux : TacticM (List MVarId) := /- Important: the following `try` does not backtrack the state. This is intentional because we don't want to backtrack the error messages when we catch the "abort internal exception" @@ -93,15 +93,15 @@ def run (mvarId : MVarId) (x : TacticM Unit) : TermElabM (List MVarId) := else throw ex try - aux.runCore' { elaborator := Name.anonymous } { goals := [mvarId] } + aux.runCore' { elaborator := .anonymous } { goals := [mvarId] } finally - modify fun s => { s with syntheticMVars := savedSyntheticMVars } + modify fun s => { s with pendingMVars := pendingMVarsSaved } protected def saveState : TacticM SavedState := return { term := (← Term.saveState), tactic := (← get) } -def SavedState.restore (b : SavedState) : TacticM Unit := do - b.term.restore +def SavedState.restore (b : SavedState) (restoreInfo := false) : TacticM Unit := do + b.term.restore restoreInfo set b.tactic protected def getCurrMacroScope : TacticM MacroScope := do pure (← readThe Core.Context).currMacroScope @@ -131,68 +131,85 @@ def mkInitialTacticInfo (stx : Syntax) : TacticM (TacticM Info) := do withInfoContext x (← mkInitialTacticInfo stx) /- -Important: we must define `evalTacticUsing` and `expandTacticMacroFns` before we define +Important: we must define `evalTactic` before we define the instance `MonadExcept` for `TacticM` since it backtracks the state including error messages, and this is bad when rethrowing the exception at the `catch` block in these methods. We marked these places with a `(*)` in these methods. -/ -private def evalTacticUsing (s : SavedState) (stx : Syntax) (tactics : List (KeyedDeclsAttribute.AttributeEntry Tactic)) : TacticM Unit := do - let rec loop - | [] => throwErrorAt stx "unexpected syntax {indentD stx}" - | evalFn::evalFns => do - try - withReader ({ · with elaborator := evalFn.declName }) <| withTacticInfoContext stx <| evalFn.value stx - catch - | ex@(Exception.error _ _) => - match evalFns with - | [] => throw ex -- (*) - | evalFns => s.restore; loop evalFns - | ex@(Exception.internal id _) => +/-- + Auxiliary datastructure for capturing exceptions at `evalTactic`. +-/ +inductive EvalTacticFailure where + | /-- Exceptions ≠ AbortException -/ + exception (ex : Exception) + | /-- + `abort` exceptions are used when exceptions have already been logged at the message Log. + Thus, we save the whole state here to make sure we don't lose them. + -/ + abort (s : SavedState) + +partial def evalTactic (stx : Syntax) : TacticM Unit := + withRef stx <| withIncRecDepth <| withFreshMacroScope <| match stx with + | .node _ k _ => + if k == nullKind then + -- Macro writers create a sequence of tactics `t₁ ... tₙ` using `mkNullNode #[t₁, ..., tₙ]` + stx.getArgs.forM evalTactic + else do + trace[Elab.step] "{stx}" + let evalFns := tacticElabAttribute.getEntries (← getEnv) stx.getKind + let macros := macroAttribute.getEntries (← getEnv) stx.getKind + if evalFns.isEmpty && macros.isEmpty then + throwErrorAt stx "tactic '{stx.getKind}' has not been implemented" + let s ← Tactic.saveState + expandEval s macros evalFns #[] + | .missing => pure () + | _ => throwError m!"unexpected tactic{indentD stx}" +where + throwExs (failures : Array EvalTacticFailure) : TacticM Unit := do + let exs := failures.filterMap fun | .abort _ => none | .exception ex => some ex + if exs.isEmpty then + if let some (.abort s) := failures.find? fun | .abort _ => true | _ => false then + s.restore (restoreInfo := true) + throwAbortTactic + else + throwErrorAt stx "unexpected syntax {indentD stx}" + else if h : 0 < exs.size then + throw exs[0] -- (*) + else + withRef stx do throwErrorWithNestedErrors "tactic failed" exs -- (*) + + @[inline] handleEx (s : SavedState) (failures : Array EvalTacticFailure) (ex : Exception) (k : Array EvalTacticFailure → TacticM Unit) := do + match ex with + | .error .. => s.restore (restoreInfo := true); k (failures.push (.exception ex)) + | .internal id _ => if id == unsupportedSyntaxExceptionId then - s.restore; loop evalFns + -- We do not store `unsupportedSyntaxExceptionId`, see throwExs + s.restore (restoreInfo := true); k failures + else if id == abortTacticExceptionId then + let failures := failures.push (.abort (← Tactic.saveState)) + s.restore (restoreInfo := true); k failures else - throw ex - loop tactics + throw ex -- (*) -mutual - - partial def expandTacticMacroFns (s : SavedState) (stx : Syntax) (macros : List (KeyedDeclsAttribute.AttributeEntry Macro)) : TacticM Unit := - let rec loop - | [] => throwErrorAt stx "tactic '{stx.getKind}' has not been implemented" - | m::ms => do + expandEval (s : SavedState) (macros : List _) (evalFns : List _) (failures : Array EvalTacticFailure) : TacticM Unit := + match macros with + | [] => eval s evalFns failures + | m :: ms => try withReader ({ · with elaborator := m.declName }) do withTacticInfoContext stx do let stx' ← adaptMacro m.value stx evalTactic stx' - catch ex => - if ms.isEmpty then throw ex -- (*) - s.restore; loop ms - loop macros - - partial def expandTacticMacro (s : SavedState) (stx : Syntax) : TacticM Unit := do - expandTacticMacroFns s stx (macroAttribute.getEntries (← getEnv) stx.getKind) - - partial def evalTacticAux (stx : Syntax) : TacticM Unit := - withRef stx <| withIncRecDepth <| withFreshMacroScope <| match stx with - | Syntax.node _ k _ => - if k == nullKind then - -- Macro writers create a sequence of tactics `t₁ ... tₙ` using `mkNullNode #[t₁, ..., tₙ]` - stx.getArgs.forM evalTactic - else do - trace[Elab.step] "{stx}" - let s ← Tactic.saveState - match tacticElabAttribute.getEntries (← getEnv) stx.getKind with - | [] => expandTacticMacro s stx - | evalFns => evalTacticUsing s stx evalFns - | Syntax.missing => pure () - | _ => throwError m!"unexpected tactic{indentD stx}" - - partial def evalTactic (stx : Syntax) : TacticM Unit := - evalTacticAux stx - -end + catch ex => handleEx s failures ex (expandEval s ms evalFns) + + eval (s : SavedState) (evalFns : List _) (failures : Array EvalTacticFailure) : TacticM Unit := do + match evalFns with + | [] => throwExs failures + | evalFn::evalFns => do + try + withReader ({ · with elaborator := evalFn.declName }) <| withTacticInfoContext stx <| evalFn.value stx + catch ex => handleEx s failures ex (eval s evalFns) def throwNoGoalsToBeSolved : TacticM α := throwError "no goals to be solved" @@ -248,10 +265,10 @@ instance : MonadExcept Exception TacticM where def withoutRecover (x : TacticM α) : TacticM α := withReader (fun ctx => { ctx with recover := false }) x -@[inline] protected def orElse {α} (x : TacticM α) (y : Unit → TacticM α) : TacticM α := do +@[inline] protected def orElse (x : TacticM α) (y : Unit → TacticM α) : TacticM α := do try withoutRecover x catch _ => y () -instance {α} : OrElse (TacticM α) where +instance : OrElse (TacticM α) where orElse := Tactic.orElse instance : Alternative TacticM where @@ -269,7 +286,7 @@ def saveTacticInfoForToken (stx : Syntax) : TacticM Unit := do /- Elaborate `x` with `stx` on the macro stack -/ @[inline] -def withMacroExpansion {α} (beforeStx afterStx : Syntax) (x : TacticM α) : TacticM α := +def withMacroExpansion (beforeStx afterStx : Syntax) (x : TacticM α) : TacticM α := withMacroExpansionInfo beforeStx afterStx do withTheReader Term.Context (fun ctx => { ctx with macroStack := { before := beforeStx, after := afterStx } :: ctx.macroStack }) x @@ -348,6 +365,8 @@ def closeMainGoal (val : Expr) (checkUnassigned := true): TacticM Unit := do replaceMainGoal mvarIds pure a +/-- Get the mvarid of the main goal, run the given `tactic`, +then set the new goals to be the resulting goal list.-/ @[inline] def liftMetaTactic (tactic : MVarId → MetaM (List MVarId)) : TacticM Unit := liftMetaTacticAux fun mvarId => do let gs ← tactic mvarId diff --git a/stage0/src/Lean/Elab/Tactic/Conv/Basic.lean b/stage0/src/Lean/Elab/Tactic/Conv/Basic.lean index e5b90e228a5c..2e8783220c66 100644 --- a/stage0/src/Lean/Elab/Tactic/Conv/Basic.lean +++ b/stage0/src/Lean/Elab/Tactic/Conv/Basic.lean @@ -12,6 +12,8 @@ import Lean.Elab.Tactic.BuiltinTactic namespace Lean.Elab.Tactic.Conv open Meta +/-- Given `lhs`, returns a pair of metavariables `(?rhs, ?newGoal)` +where `?newGoal : lhs = ?rhs`.-/ def mkConvGoalFor (lhs : Expr) : MetaM (Expr × Expr) := do let lhsType ← inferType lhs let rhs ← mkFreshExprMVar lhsType @@ -25,6 +27,9 @@ def markAsConvGoal (mvarId : MVarId) : MetaM MVarId := do return mvarId -- it is already tagged as LHS goal replaceTargetDefEq mvarId (mkLHSGoal (← getMVarType mvarId)) +/-- Given `lhs`, runs the `conv` tactic with the goal `⊢ lhs = ?rhs`. +`conv` should produce no remaining goals that are not solvable with refl. +Returns a pair of instantiated expressions `(?rhs, ?p)` where `?p : lhs = ?rhs`. -/ def convert (lhs : Expr) (conv : TacticM Unit) : TacticM (Expr × Expr) := do let (rhs, newGoal) ← mkConvGoalFor lhs let savedGoals ← getGoals diff --git a/stage0/src/Lean/Elab/Tactic/ElabTerm.lean b/stage0/src/Lean/Elab/Tactic/ElabTerm.lean index 3f5d6ae0ad16..d105d3b19bf5 100644 --- a/stage0/src/Lean/Elab/Tactic/ElabTerm.lean +++ b/stage0/src/Lean/Elab/Tactic/ElabTerm.lean @@ -224,7 +224,7 @@ def elabAsFVar (stx : Syntax) (userName? : Option Name := none) : TacticM FVarId withMainContext do let e ← elabTerm stx none match e with - | Expr.fvar fvarId => pure fvarId + | .fvar fvarId => pure fvarId | _ => let type ← inferType e let intro (userName : Name) (preserveBinderNames : Bool) : TacticM FVarId := do @@ -242,14 +242,10 @@ def elabAsFVar (stx : Syntax) (userName? : Option Name := none) : TacticM FVarId match stx with | `(tactic| rename $typeStx:term => $h:ident) => do withMainContext do - /- Remark: we must not use `withoutModifyingState` because we may miss errors message. - For example, suppose the following `elabTerm` logs an error during elaboration. - In this scenario, the term `type` contains a synthetic `sorry`, and the error - message `"failed to find ..."` is not logged by the outer loop. - By using `withoutModifyingStateWithInfoAndMessages`, we ensure that - the messages and the info trees are preserved while the rest of the - state is backtracked. -/ - let fvarId ← withoutModifyingStateWithInfoAndMessages <| withNewMCtxDepth do + /- Remark: we also use `withoutRecover` to make sure `elabTerm` does not succeed + using `sorryAx`, and we get `"failed to find ..."` which will not be logged because + it contains synthetic sorry's -/ + let fvarId ← withoutModifyingState <| withNewMCtxDepth <| withoutRecover do let type ← elabTerm typeStx none (mayPostpone := true) let fvarId? ← (← getLCtx).findDeclRevM? fun localDecl => do if (← isDefEq type localDecl.type) then return localDecl.fvarId else return none diff --git a/stage0/src/Lean/Elab/Tactic/Induction.lean b/stage0/src/Lean/Elab/Tactic/Induction.lean index 94e7c0f6ac7c..8a9c2df512a5 100644 --- a/stage0/src/Lean/Elab/Tactic/Induction.lean +++ b/stage0/src/Lean/Elab/Tactic/Induction.lean @@ -114,7 +114,7 @@ structure Result where partial def mkElimApp (elimInfo : ElimInfo) (targets : Array Expr) (tag : Name) : TermElabM Result := do let rec loop : M Unit := do match (← getFType) with - | Expr.forallE binderName _ _ c => + | .forallE binderName _ _ c => let ctx ← read let argPos := (← get).argPos if ctx.elimInfo.motivePos == argPos then @@ -131,13 +131,13 @@ partial def mkElimApp (elimInfo : ElimInfo) (targets : Array Expr) (tag : Name) modify fun s => { s with targetPos := s.targetPos + 1 } addNewArg target else match c with - | BinderInfo.implicit => + | .implicit => let arg ← mkFreshExprMVar (← getArgExpectedType) addNewArg arg - | BinderInfo.strictImplicit => + | .strictImplicit => let arg ← mkFreshExprMVar (← getArgExpectedType) addNewArg arg - | BinderInfo.instImplicit => + | .instImplicit => let arg ← mkFreshExprMVar (← getArgExpectedType) (kind := MetavarKind.synthetic) (userName := appendTag tag binderName) modify fun s => { s with insts := s.insts.push arg.mvarId! } addNewArg arg diff --git a/stage0/src/Lean/Elab/Tactic/Location.lean b/stage0/src/Lean/Elab/Tactic/Location.lean index 84979e858489..6ae34f3678a7 100644 --- a/stage0/src/Lean/Elab/Tactic/Location.lean +++ b/stage0/src/Lean/Elab/Tactic/Location.lean @@ -8,9 +8,13 @@ import Lean.Elab.Tactic.ElabTerm namespace Lean.Elab.Tactic +/-- Denotes a set of locations where a tactic should be applied for the main goal. See also `withLocation`. -/ inductive Location where - | wildcard - | targets (hypotheses : Array Syntax) (type : Bool) + | /-- Apply the tactic everywhere. -/ + wildcard + | /-- `hypotheses` are hypothesis names in the main goal that the tactic should be applied to. + If `type` is true, then the tactic should also be applied to the target type. -/ + targets (hypotheses : Array Syntax) (type : Bool) /- Recall that @@ -35,6 +39,9 @@ def expandOptLocation (stx : Syntax) : Location := open Meta +/-- Runs the given `atLocal` and `atTarget` methods on each of the locations selected by the given `loc`. +If any of the selected tactic applications fail, it will call `failed` with the main goal mvar. + -/ def withLocation (loc : Location) (atLocal : FVarId → TacticM Unit) (atTarget : TacticM Unit) (failed : MVarId → TacticM Unit) : TacticM Unit := do match loc with | Location.targets hyps type => diff --git a/stage0/src/Lean/Elab/Tactic/Simp.lean b/stage0/src/Lean/Elab/Tactic/Simp.lean index c8e1f56ad965..9145e2e9a609 100644 --- a/stage0/src/Lean/Elab/Tactic/Simp.lean +++ b/stage0/src/Lean/Elab/Tactic/Simp.lean @@ -126,11 +126,11 @@ inductive ResolveSimpIdResult where | ext (ext : SimpExtension) /-- - Elaborate extra simp theorems provided to `simp`. `stx` is of the `simpTheorem,*` + Elaborate extra simp theorems provided to `simp`. `stx` is of the form `"[" simpTheorem,* "]"` If `eraseLocal == true`, then we consider local declarations when resolving names for erased theorems (`- id`), this option only makes sense for `simp_all`. -/ -private def elabSimpArgs (stx : Syntax) (ctx : Simp.Context) (eraseLocal : Bool) (kind : SimpKind) : TacticM ElabSimpArgsResult := do +def elabSimpArgs (stx : Syntax) (ctx : Simp.Context) (eraseLocal : Bool) (kind : SimpKind) : TacticM ElabSimpArgsResult := do if stx.isNone then return { ctx } else diff --git a/stage0/src/Lean/Elab/Term.lean b/stage0/src/Lean/Elab/Term.lean index bb0245b94e13..50c6eab7844a 100644 --- a/stage0/src/Lean/Elab/Term.lean +++ b/stage0/src/Lean/Elab/Term.lean @@ -50,18 +50,19 @@ inductive SyntheticMVarKind where tactic (tacticCode : Syntax) (ctx : SavedContext) | /-- Metavariable represents a hole whose elaboration has been postponed. -/ postponed (ctx : SavedContext) + deriving Inhabited instance : ToString SyntheticMVarKind where toString - | SyntheticMVarKind.typeClass => "typeclass" - | SyntheticMVarKind.coe .. => "coe" - | SyntheticMVarKind.tactic .. => "tactic" - | SyntheticMVarKind.postponed .. => "postponed" + | .typeClass => "typeclass" + | .coe .. => "coe" + | .tactic .. => "tactic" + | .postponed .. => "postponed" structure SyntheticMVarDecl where - mvarId : MVarId stx : Syntax kind : SyntheticMVarKind + deriving Inhabited /-- We can optionally associate an error context with a metavariable (see `MVarErrorInfo`). @@ -78,9 +79,9 @@ inductive MVarErrorKind where instance : ToString MVarErrorKind where toString - | MVarErrorKind.implicitArg _ => "implicitArg" - | MVarErrorKind.hole => "hole" - | MVarErrorKind.custom _ => "custom" + | .implicitArg _ => "implicitArg" + | .hole => "hole" + | .custom _ => "custom" /-- We can optionally associate an error context with metavariables. @@ -114,7 +115,8 @@ structure LetRecToLift where -/ structure State where levelNames : List Name := [] - syntheticMVars : List SyntheticMVarDecl := [] + syntheticMVars : MVarIdMap SyntheticMVarDecl := {} + pendingMVars : List MVarId := {} mvarErrorInfos : MVarIdMap MVarErrorInfo := {} letRecsToLift : List LetRecToLift := [] infoState : InfoState := {} @@ -252,7 +254,7 @@ def SavedState.restore (s : SavedState) (restoreInfo : Bool := false) : TermElab set s.elab setTraceState traceState unless restoreInfo do - modify fun s => { s with infoState := infoState } + modify fun s => { s with infoState } instance : MonadBacktrack SavedState TermElabM where saveState := Term.saveState @@ -278,11 +280,11 @@ def observing (x : TermElabM α) : TermElabM (TermElabResult α) := do s.restore (restoreInfo := true) return EStateM.Result.ok e sNew catch - | ex@(Exception.error _ _) => + | ex@(.error ..) => let sNew ← saveState s.restore (restoreInfo := true) - return EStateM.Result.error ex sNew - | ex@(Exception.internal id _) => + return .error ex sNew + | ex@(.internal id _) => if id == postponeExceptionId then s.restore (restoreInfo := true) throw ex @@ -292,8 +294,8 @@ def observing (x : TermElabM α) : TermElabM (TermElabResult α) := do We use this method to implement overloaded notation and symbols. -/ def applyResult (result : TermElabResult α) : TermElabM α := do match result with - | EStateM.Result.ok a r => r.restore (restoreInfo := true); return a - | EStateM.Result.error ex r => r.restore (restoreInfo := true); throw ex + | .ok a r => r.restore (restoreInfo := true); return a + | .error ex r => r.restore (restoreInfo := true); throw ex /-- Execute `x`, but keep state modifications only if `x` did not postpone. @@ -342,7 +344,7 @@ def withoutModifyingElabMetaStateWithInfo (x : TermElabM α) : TermElabM α := d let s ← get let sMeta ← getThe Meta.State try - withSaveInfoContext x + withSaveInfoContext x finally modify ({ s with infoState := ·.infoState }) set sMeta @@ -385,17 +387,17 @@ inductive LVal where | fieldName (ref : Syntax) (name : String) (suffix? : Option Name) (targetStx : Syntax) def LVal.getRef : LVal → Syntax - | LVal.fieldIdx ref _ => ref - | LVal.fieldName ref .. => ref + | .fieldIdx ref _ => ref + | .fieldName ref .. => ref def LVal.isFieldName : LVal → Bool - | LVal.fieldName .. => true + | .fieldName .. => true | _ => false instance : ToString LVal where toString - | LVal.fieldIdx _ i => toString i - | LVal.fieldName _ n .. => n + | .fieldIdx _ i => toString i + | .fieldName _ n .. => n /-- Return the name of the declaration being elaborated if available. -/ def getDeclName? : TermElabM (Option Name) := return (← read).declName? @@ -453,8 +455,8 @@ def liftLevelM (x : LevelElabM α) : TermElabM α := do let ngen ← getNGen let lvlCtx : Level.Context := { options := (← getOptions), ref := (← getRef), autoBoundImplicit := ctx.autoBoundImplicit } match (x lvlCtx).run { ngen := ngen, mctx := mctx, levelNames := (← getLevelNames) } with - | EStateM.Result.ok a newS => setMCtx newS.mctx; setNGen newS.ngen; setLevelNames newS.levelNames; pure a - | EStateM.Result.error ex _ => throw ex + | .ok a newS => setMCtx newS.mctx; setNGen newS.ngen; setLevelNames newS.levelNames; pure a + | .error ex _ => throw ex def elabLevel (stx : Syntax) : TermElabM Level := liftLevelM <| Level.elabLevel stx @@ -468,7 +470,7 @@ def withMacroExpansion (beforeStx afterStx : Syntax) (x : TermElabM α) : TermEl Add the given metavariable to the list of pending synthetic metavariables. The method `synthesizeSyntheticMVars` is used to process the metavariables on this list. -/ def registerSyntheticMVar (stx : Syntax) (mvarId : MVarId) (kind : SyntheticMVarKind) : TermElabM Unit := do - modify fun s => { s with syntheticMVars := { mvarId := mvarId, stx := stx, kind := kind } :: s.syntheticMVars } + modify fun s => { s with syntheticMVars := s.syntheticMVars.insert mvarId { stx, kind }, pendingMVars := mvarId :: s.pendingMVars } def registerSyntheticMVarWithCurrRef (mvarId : MVarId) (kind : SyntheticMVarKind) : TermElabM Unit := do registerSyntheticMVar (← getRef) mvarId kind @@ -477,13 +479,13 @@ def registerMVarErrorInfo (mvarErrorInfo : MVarErrorInfo) : TermElabM Unit := modify fun s => { s with mvarErrorInfos := s.mvarErrorInfos.insert mvarErrorInfo.mvarId mvarErrorInfo } def registerMVarErrorHoleInfo (mvarId : MVarId) (ref : Syntax) : TermElabM Unit := - registerMVarErrorInfo { mvarId := mvarId, ref := ref, kind := MVarErrorKind.hole } + registerMVarErrorInfo { mvarId, ref, kind := .hole } def registerMVarErrorImplicitArgInfo (mvarId : MVarId) (ref : Syntax) (app : Expr) : TermElabM Unit := do - registerMVarErrorInfo { mvarId := mvarId, ref := ref, kind := MVarErrorKind.implicitArg app } + registerMVarErrorInfo { mvarId, ref, kind := .implicitArg app } def registerMVarErrorCustomInfo (mvarId : MVarId) (ref : Syntax) (msgData : MessageData) : TermElabM Unit := do - registerMVarErrorInfo { mvarId := mvarId, ref := ref, kind := MVarErrorKind.custom msgData } + registerMVarErrorInfo { mvarId, ref, kind := .custom msgData } def getMVarErrorInfo? (mvarId : MVarId) : TermElabM (Option MVarErrorInfo) := do return (← get).mvarErrorInfos.find? mvarId @@ -615,6 +617,7 @@ private def applyAttributesCore (declName : Name) (attrs : Array Attribute) (applicationTime? : Option AttributeApplicationTime) : TermElabM Unit := for attr in attrs do + withRef attr.stx do withLogging do let env ← getEnv match getAttributeImpl env attr.name with | Except.error errMsg => throwError errMsg @@ -670,17 +673,17 @@ abbrev M := MonadCacheT Expr Unit (OptionT TermElabM) partial def visit (e : Expr) : M Unit := do checkCache e fun _ => do match e with - | Expr.forallE _ d b _ => visit d; visit b - | Expr.lam _ d b _ => visit d; visit b - | Expr.letE _ t v b _ => visit t; visit v; visit b - | Expr.app f a => visit f; visit a - | Expr.mdata _ b => visit b - | Expr.proj _ _ b => visit b - | Expr.fvar fvarId .. => + | .forallE _ d b _ => visit d; visit b + | .lam _ d b _ => visit d; visit b + | .letE _ t v b _ => visit t; visit v; visit b + | .app f a => visit f; visit a + | .mdata _ b => visit b + | .proj _ _ b => visit b + | .fvar fvarId .. => match (← getLocalDecl fvarId) with - | LocalDecl.cdecl .. => return () + | .cdecl .. => return () | LocalDecl.ldecl (value := v) .. => visit v - | Expr.mvar mvarId .. => + | .mvar mvarId .. => let e' ← instantiateMVars e if e' != e then visit e' @@ -745,8 +748,8 @@ def synthesizeInstMVarCore (instMVar : MVarId) (maxResultSize? : Option Nat := n unless (← isDefEq (mkMVar instMVar) val) do throwError "failed to assign synthesized type class instance{indentExpr val}" return true - | LOption.undef => return false -- we will try later - | LOption.none => + | .undef => return false -- we will try later + | .none => if (← read).ignoreTCFailures then return false else @@ -771,7 +774,7 @@ def synthesizeCoeInstMVarCore (instMVar : MVarId) : TermElabM Bool := do -/ def tryCoeThunk? (expectedType : Expr) (eType : Expr) (e : Expr) : TermElabM (Option Expr) := do match expectedType with - | Expr.app (Expr.const ``Thunk u) arg => + | .app (.const ``Thunk u) arg => if (← isDefEq eType arg) then return some (mkApp2 (mkConst ``Thunk.mk u) arg (mkSimpleThunk e)) else @@ -797,8 +800,8 @@ def mkCoe (expectedType : Expr) (eType : Expr) (e : Expr) (f? : Option Expr := n registerSyntheticMVarWithCurrRef mvarAux.mvarId! (SyntheticMVarKind.coe errorMsgHeader? eNew expectedType eType e f?) return mvarAux catch - | Exception.error _ msg => throwTypeMismatchError errorMsgHeader? expectedType eType e f? msg - | _ => throwTypeMismatchError errorMsgHeader? expectedType eType e f? + | .error _ msg => throwTypeMismatchError errorMsgHeader? expectedType eType e f? msg + | _ => throwTypeMismatchError errorMsgHeader? expectedType eType e f? /-- Try to apply coercion to make sure `e` has type `expectedType`. @@ -819,17 +822,17 @@ private def tryCoe (errorMsgHeader? : Option String) (expectedType : Expr) (eTyp def isTypeApp? (type : Expr) : TermElabM (Option (Expr × Expr)) := do let type ← withReducible <| whnf type match type with - | Expr.app m α => return some ((← instantiateMVars m), (← instantiateMVars α)) - | _ => return none + | .app m α => return some ((← instantiateMVars m), (← instantiateMVars α)) + | _ => return none /-- Helper method used to implement auto-lift and coercions -/ private def synthesizeInst (type : Expr) : TermElabM Expr := do let type ← instantiateMVars type match (← trySynthInstance type) with - | LOption.some val => return val + | .some val => return val -- Note that `ignoreTCFailures` is not checked here since it must return a result. - | LOption.undef => throwError "failed to synthesize instance{indentExpr type}" - | LOption.none => throwError "failed to synthesize instance{indentExpr type}" + | .undef => throwError "failed to synthesize instance{indentExpr type}" + | .none => throwError "failed to synthesize instance{indentExpr type}" /-- Return `true` if `type` is of the form `m α` where `m` is a `Monad`. @@ -847,13 +850,13 @@ Otherwise, we just use the basic `tryCoe`. Extensions for monads. -1- Try to unify `n` and `m`. If it succeeds, then we use - ``` - coeM {m : Type u → Type v} {α β : Type u} [∀ a, CoeT α a β] [Monad m] (x : m α) : m β - ``` - `n` must be a `Monad` to use this one. +1. Try to unify `n` and `m`. If it succeeds, then we use + ``` + coeM {m : Type u → Type v} {α β : Type u} [∀ a, CoeT α a β] [Monad m] (x : m α) : m β + ``` + `n` must be a `Monad` to use this one. -2- If there is monad lift from `m` to `n` and we can unify `α` and `β`, we use +2. If there is monad lift from `m` to `n` and we can unify `α` and `β`, we use ``` liftM : ∀ {m : Type u_1 → Type u_2} {n : Type u_1 → Type u_3} [self : MonadLiftT m n] {α : Type u_1}, m α → n α ``` @@ -868,7 +871,7 @@ Extensions for monads. ``` -3- If there is a monad lif from `m` to `n` and a coercion from `α` to `β`, we use +3. If there is a monad lif from `m` to `n` and a coercion from `α` to `β`, we use ``` liftCoeM {m : Type u → Type v} {n : Type u → Type w} {α β : Type u} [MonadLiftT m n] [∀ a, CoeT α a β] [Monad n] (x : m α) : n β ``` @@ -1052,7 +1055,7 @@ private def postponeElabTerm (stx : Syntax) (expectedType? : Option Expr) : Term return mvar def getSyntheticMVarDecl? (mvarId : MVarId) : TermElabM (Option SyntheticMVarDecl) := - return (← get).syntheticMVars.find? fun d => d.mvarId == mvarId + return (← get).syntheticMVars.find? mvarId /-- Create an auxiliary annotation to make sure we create a `Info` even if `e` is a metavariable. @@ -1094,9 +1097,9 @@ def isTacticOrPostponedHole? (e : Expr) : TermElabM (Option MVarId) := do match e with | Expr.mvar mvarId => match (← getSyntheticMVarDecl? mvarId) with - | some { kind := SyntheticMVarKind.tactic .., .. } => return mvarId - | some { kind := SyntheticMVarKind.postponed .., .. } => return mvarId - | _ => return none + | some { kind := .tactic .., .. } => return mvarId + | some { kind := .postponed .., .. } => return mvarId + | _ => return none | _ => pure none def mkTermInfo (elaborator : Name) (stx : Syntax) (e : Expr) (expectedType? : Option Expr := none) (lctx? : Option LocalContext := none) (isBinder := false) : TermElabM (Sum Info MVarId) := do @@ -1136,12 +1139,12 @@ private def elabUsingElabFnsAux (s : SavedState) (stx : Syntax) (expectedType? : (try elabFn.value stx expectedType? catch ex => match ex with - | Exception.error _ _ => + | .error .. => if (← read).errToSorry then exceptionToSorry ex expectedType? else throw ex - | Exception.internal id _ => + | .internal id _ => if (← read).errToSorry && id == abortTermExceptionId then exceptionToSorry ex expectedType? else if id == unsupportedSyntaxExceptionId then @@ -1166,7 +1169,7 @@ private def elabUsingElabFnsAux (s : SavedState) (stx : Syntax) (expectedType? : else throw ex) catch ex => match ex with - | Exception.internal id _ => + | .internal id _ => if id == unsupportedSyntaxExceptionId then s.restore -- also removes the info tree created above elabUsingElabFnsAux s stx expectedType? catchExPostpone elabFns @@ -1261,7 +1264,7 @@ private def useImplicitLambda? (stx : Syntax) (expectedType? : Option Expr) : Te else let expectedType ← whnfForall expectedType match expectedType with - | Expr.forallE _ _ _ c => + | .forallE _ _ _ c => if c.isImplicit || c.isInstImplicit then return some expectedType else @@ -1271,7 +1274,7 @@ private def useImplicitLambda? (stx : Syntax) (expectedType? : Option Expr) : Te private def decorateErrorMessageWithLambdaImplicitVars (ex : Exception) (impFVars : Array Expr) : TermElabM Exception := do match ex with - | Exception.error ref msg => + | .error ref msg => if impFVars.isEmpty then return Exception.error ref msg else @@ -1298,7 +1301,7 @@ private partial def elabImplicitLambda (stx : Syntax) (catchExPostpone : Bool) ( loop type #[] where loop - | type@(Expr.forallE n d b c), fvars => + | type@(.forallE n d b c), fvars => if c.isExplicit then elabImplicitLambdaAux stx catchExPostpone type fvars else withFreshMacroScope do @@ -1311,7 +1314,7 @@ where /- Main loop for `elabTerm` -/ private partial def elabTermAux (expectedType? : Option Expr) (catchExPostpone : Bool) (implicitLambda : Bool) : Syntax → TermElabM Expr - | Syntax.missing => mkSyntheticSorryFor expectedType? + | .missing => mkSyntheticSorryFor expectedType? | stx => withFreshMacroScope <| withIncRecDepth do trace[Elab.step] "expected type: {expectedType?}, term\n{stx}" checkMaxHeartbeats "elaborator" @@ -1332,7 +1335,7 @@ private partial def elabTermAux (expectedType? : Option Expr) (catchExPostpone : /-- Store in the `InfoTree` that `e` is a "dot"-completion target. -/ def addDotCompletionInfo (stx : Syntax) (e : Expr) (expectedType? : Option Expr) (field? : Option Syntax := none) : TermElabM Unit := do - addCompletionInfo <| CompletionInfo.dot { expr := e, stx, lctx := (← getLCtx), elaborator := Name.anonymous, expectedType? } (field? := field?) (expectedType? := expectedType?) + addCompletionInfo <| CompletionInfo.dot { expr := e, stx, lctx := (← getLCtx), elaborator := .anonymous, expectedType? } (field? := field?) (expectedType? := expectedType?) /-- Main function for elaborating terms. @@ -1358,17 +1361,6 @@ def elabTermEnsuringType (stx : Syntax) (expectedType? : Option Expr) (catchExPo let e ← elabTerm stx expectedType? catchExPostpone implicitLambda withRef stx <| ensureHasType expectedType? e errorMsgHeader? -/-- - Execute `x` and then restore `syntheticMVars`, `levelNames`, `mvarErrorInfos`, and `letRecsToLift`. - We use this combinator when we don't want the pending problems created by `x` to persist after its execution. -/ -def withoutPending (x : TermElabM α) : TermElabM α := do - let saved ← get - try - x - finally - modify fun s => { s with syntheticMVars := saved.syntheticMVars, levelNames := saved.levelNames, - letRecsToLift := saved.letRecsToLift, mvarErrorInfos := saved.mvarErrorInfos } - /-- Execute `x` and return `some` if no new errors were recorded or exceptions was thrown. Otherwise, return `none` -/ def commitIfNoErrors? (x : TermElabM α) : TermElabM (Option α) := do let saved ← saveState @@ -1413,7 +1405,7 @@ private def tryCoeSort (α : Expr) (a : Expr) : TermElabM Expr := do let u ← getLevel α let v ← getLevel β let coeSortInstType := mkAppN (Lean.mkConst ``CoeSort [u, v]) #[α, β] - let mvar ← mkFreshExprMVar coeSortInstType MetavarKind.synthetic + let mvar ← mkFreshExprMVar coeSortInstType .synthetic let mvarId := mvar.mvarId! try withoutMacroStackAtErr do @@ -1425,8 +1417,8 @@ private def tryCoeSort (α : Expr) (a : Expr) : TermElabM Expr := do else throwError "type expected" catch - | Exception.error _ msg => throwError "type expected\n{msg}" - | _ => throwError "type expected" + | .error _ msg => throwError "type expected\n{msg}" + | _ => throwError "type expected" /-- Make sure `e` is a type by inferring its type and making sure it is a `Expr.sort` @@ -1463,7 +1455,7 @@ partial def withAutoBoundImplicit (k : TermElabM α) : TermElabM α := do | some n => -- Restore state, declare `n`, and try again s.restore - withLocalDecl n BinderInfo.implicit (← mkFreshTypeMVar) fun x => + withLocalDecl n .implicit (← mkFreshTypeMVar) fun x => withReader (fun ctx => { ctx with autoBoundImplicits := ctx.autoBoundImplicits.push x } ) do loop (← saveState) | none => throw ex diff --git a/stage0/src/Lean/Elab/Util.lean b/stage0/src/Lean/Elab/Util.lean index 883232d2d5fd..c5517333867d 100644 --- a/stage0/src/Lean/Elab/Util.lean +++ b/stage0/src/Lean/Elab/Util.lean @@ -204,6 +204,10 @@ def logException [Monad m] [MonadLog m] [AddMessageContext m] [MonadLiftT IO m] let name ← id.getName logError m!"internal exception: {name}" +def withLogging [Monad m] [MonadLog m] [MonadExcept Exception m] [AddMessageContext m] [MonadLiftT IO m] + (x : m Unit) : m Unit := do + try x catch ex => logException ex + @[inline] def trace [Monad m] [MonadLog m] [AddMessageContext m] [MonadOptions m] (cls : Name) (msg : Unit → MessageData) : m Unit := do if checkTraceOption (← getOptions) cls then logTrace cls (msg ()) diff --git a/stage0/src/Lean/Expr.lean b/stage0/src/Lean/Expr.lean index 7d00d292b32f..82f09a7c326f 100644 --- a/stage0/src/Lean/Expr.lean +++ b/stage0/src/Lean/Expr.lean @@ -8,22 +8,29 @@ import Lean.Level namespace Lean +/-- Literal values for `Expr`. -/ inductive Literal where - | natVal (val : Nat) - | strVal (val : String) + | /-- Natural number literal -/ + natVal (val : Nat) + | /-- String literal -/ + strVal (val : String) deriving Inhabited, BEq, Repr protected def Literal.hash : Literal → UInt64 - | Literal.natVal v => hash v - | Literal.strVal v => hash v + | .natVal v => hash v + | .strVal v => hash v instance : Hashable Literal := ⟨Literal.hash⟩ +/-- +Total order on `Expr` literal values. +Natural number values are smaller than string literal values. +-/ def Literal.lt : Literal → Literal → Bool - | Literal.natVal _, Literal.strVal _ => true - | Literal.natVal v₁, Literal.natVal v₂ => v₁ < v₂ - | Literal.strVal v₁, Literal.strVal v₂ => v₁ < v₂ - | _, _ => false + | .natVal _, .strVal _ => true + | .natVal v₁, .natVal v₂ => v₁ < v₂ + | .strVal v₁, .strVal v₂ => v₁ < v₂ + | _, _ => false instance : LT Literal := ⟨fun a b => a.lt b⟩ @@ -46,7 +53,7 @@ This can be set to The difference between implicit `{}` and strict-implicit `⦃⦄` is how implicit arguments are treated that are *not* followed by explicit arguments. `{}` arguments are applied eagerly, while `⦃⦄` arguments are left partially applied: -```lean +```lean4 def foo {x : Nat} : Nat := x def bar ⦃x : Nat⦄ : Nat := x #check foo -- foo : Nat @@ -56,32 +63,59 @@ def bar ⦃x : Nat⦄ : Nat := x See also the Lean manual: https://leanprover.github.io/lean4/doc/expressions.html#implicit-arguments -/ inductive BinderInfo where - | default | implicit | strictImplicit | instImplicit | auxDecl + | /-- Default binder annotation, e.g. `(x : α)` -/ + default + | /-- Implicit binder annotation, e.g., `{x : α}` -/ + implicit + | /-- Strict implict binder annotation, e.g., `{{ x : α }}` -/ + strictImplicit + | /-- Local instance binder annotataion, e.g., `[Decidable α]` -/ + instImplicit + | /-- + Auxiliary declarations used by Lean when elaborating recursive declarations. + When defining a function such as + ``` + def f : Nat → Nat + | 0 => 1 + | x+1 => (x+1)*f x + ``` + Lean adds a local declaration `f : Nat → Nat` to the local context (`LocalContext`) + with `BinderInfo` set to `auxDecl`. + This local declaration is later removed by the termination checker. + -/ + auxDecl deriving Inhabited, BEq, Repr def BinderInfo.hash : BinderInfo → UInt64 - | BinderInfo.default => 947 - | BinderInfo.implicit => 1019 - | BinderInfo.strictImplicit => 1087 - | BinderInfo.instImplicit => 1153 - | BinderInfo.auxDecl => 1229 + | .default => 947 + | .implicit => 1019 + | .strictImplicit => 1087 + | .instImplicit => 1153 + | .auxDecl => 1229 +/-- +Return `true` if the given `BinderInfo` does not correspond to an implicit binder annotation +(i.e., `implicit`, `strictImplicit`, or `instImplicit`). +-/ def BinderInfo.isExplicit : BinderInfo → Bool - | BinderInfo.implicit => false - | BinderInfo.strictImplicit => false - | BinderInfo.instImplicit => false - | _ => true + | .implicit => false + | .strictImplicit => false + | .instImplicit => false + | _ => true instance : Hashable BinderInfo := ⟨BinderInfo.hash⟩ +/-- Return `true` if the given `BinderInfo` is an instance implicit annotation (e.g., `[Decidable α]`) -/ def BinderInfo.isInstImplicit : BinderInfo → Bool | BinderInfo.instImplicit => true | _ => false +/-- Return `true` if the given `BinderInfo` is a regular implicit annotation (e.g., `{α : Type u}`) -/ def BinderInfo.isImplicit : BinderInfo → Bool | BinderInfo.implicit => true | _ => false +/-- Return `true` if the given `BinderInfo` is a strict implicit annotation (e.g., `{{α : Type u}}`) -/ def BinderInfo.isStrictImplicit : BinderInfo → Bool | BinderInfo.strictImplicit => true | _ => false @@ -95,16 +129,19 @@ abbrev MData := KVMap abbrev MData.empty : MData := {} /-- - Cached hash code, cached results, and other data for `Expr`. - hash : 32-bits - hasFVar : 1-bit -- does it contain free variables? - hasExprMVar : 1-bit -- does it contain metavariables? - hasLevelMVar : 1-bit -- does it contain level metavariables? - hasLevelParam : 1-bit -- does it contain level parameters? - nonDepLet : 1-bit -- internal flag, for tracking whether let x := v; b is equivalent to (fun x => b) v - binderInfo : 3-bits -- encoding of BinderInfo - approxDepth : 8-bits -- the approximate depth is used to minimize the number of hash collisions - looseBVarRange : 16-bits +Cached hash code, cached results, and other data for `Expr`. +- hash : 32-bits +- hasFVar : 1-bit -- does it contain free variables? +- hasExprMVar : 1-bit -- does it contain metavariables? +- hasLevelMVar : 1-bit -- does it contain level metavariables? +- hasLevelParam : 1-bit -- does it contain level parameters? +- nonDepLet : 1-bit -- internal flag, for tracking whether let x := v; b is equivalent to (fun x => b) v +- binderInfo : 3-bits -- encoding of BinderInfo -- TODO remove +- approxDepth : 8-bits -- the approximate depth is used to minimize the number of hash collisions +- looseBVarRange : 16-bits + +Remark: this is mostly an internal datastructure used to implement `Expr`, +most will never have to use it. -/ def Expr.Data := UInt64 @@ -211,6 +248,14 @@ instance : Repr Expr.Data where open Expr +/-- +The unique free variable identifier. It is just a hierarchical name, +but we wrap it in `FVarId` to make sure they don't get mixed up with `MVarId`. + +This is not the user-facing name for a free variable. This information is stored +in the local context (`LocalContext`). The unique identifiers are generated using +a `NameGenerator`. +-/ structure FVarId where name : Name deriving Inhabited, BEq, Hashable @@ -218,14 +263,24 @@ structure FVarId where instance : Repr FVarId where reprPrec n p := reprPrec n.name p +/-- +A set of unique free variable identifiers. +This is a persistent data structure implemented using red-black trees. -/ def FVarIdSet := Std.RBTree FVarId (Name.quickCmp ·.name ·.name) deriving Inhabited, EmptyCollection instance : ForIn m FVarIdSet FVarId := inferInstanceAs (ForIn _ (Std.RBTree ..) ..) +/-- +A set of unique free variable identifiers implemented using hashtables. +Hashtables are faster than red-black trees if they are used linearly. +They are not persistent data-structures. -/ def FVarIdHashSet := Std.HashSet FVarId deriving Inhabited, EmptyCollection +/-- +A mapping from free variable identifiers to values of type `α`. +This is a persistent data structure implemented using red-black trees. -/ def FVarIdMap (α : Type) := Std.RBMap FVarId α (Name.quickCmp ·.name ·.name) instance : EmptyCollection (FVarIdMap α) := inferInstanceAs (EmptyCollection (Std.RBMap ..)) @@ -233,21 +288,137 @@ instance : EmptyCollection (FVarIdMap α) := inferInstanceAs (EmptyCollection (S instance : Inhabited (FVarIdMap α) where default := {} -/- We use the `E` suffix (short for `Expr`) to avoid collision with keywords. - We considered using «...», but it is too inconvenient to use. -/ +/-- +Lean expressions. This datastructure is used in the kernel and +elaborator. Howewer, expressions sent to the kernel should not +contain metavariables. + +Remark: we use the `E` suffix (short for `Expr`) to avoid collision with keywords. +We considered using «...», but it is too inconvenient to use. -/ inductive Expr where - | bvar : Nat → Expr -- bound variables - | fvar : FVarId → Expr -- free variables - | mvar : MVarId → Expr -- meta variables - | sort : Level → Expr -- Sort - | const : Name → List Level → Expr -- constants - | app : Expr → Expr → Expr -- application - | lam : Name → Expr → Expr → BinderInfo → Expr -- lambda abstraction - | forallE : Name → Expr → Expr → BinderInfo → Expr -- (dependent) arrow - | letE : Name → Expr → Expr → Expr → Bool → Expr -- let expressions - | lit : Literal → Expr -- literals - | mdata : MData → Expr → Expr -- metadata - | proj : Name → Nat → Expr → Expr -- projection + | /-- + Bound variables. The natural number is the "de Bruijn" index + for the bound variable. See https://en.wikipedia.org/wiki/De_Bruijn_index for additional information. + Example, the expression `fun x : Nat => forall y : Nat, x = y` + ```lean + .lam `x (.const `Nat []) + (.forall `y (.const `Nat []) + (.app (.app (.app (.const `Eq [.succ .zero]) + (.const `Nat [])) (.bvar 1)) + (.bvar 0)) + .default) + .default + ``` + -/ + bvar (deBruijnIndex : Nat) + | /-- + Free variable. Lean uses the locally nameless approach. + See https://citeseerx.ist.psu.edu/viewdoc/download?doi=10.1.1.365.2479&rep=rep1&type=pdf for additional details. + When "visiting" the body of a binding expression (`lam`, `forallE`, or `letE`), bound variables + are converted into free variables using a unique identifier, and their user-facing name, type, + value (for `LetE`), and binder annotation are stored in the `LocalContext`. + -/ + fvar (fvarId : FVarId) + | /-- + Metavariables are used to represent "holes" in expressions, and goals in the + tactic framework. Metavariable declarations are stored in the `MetavarContext`. + Metavariables are used during elaboration, and are not allowed in the kernel, + or in the code generator. + -/ + mvar (mvarId : MVarId) + | /-- + `Type u`, `Sort u`, `Prop`. - + - `Prop` is represented as `.sort .zero`, + - `Sort u` as ``.sort (.param `u)``, and + - `Type u` as ``.sort (.succ (.param `u))`` + -/ + sort (u : Level) + | /-- + A (universe polymorphic) constant. For example, + `@Eq.{1}` is represented as ``.const `Eq [.succ .zero]``, and + `@Array.map.{0, 0}` is represented as ``.cons `Array.map [.zero, .zero]``. + -/ + const (declName : Name) (us : List Level) + | /-- + Function application. `Nat.succ Nat.zero` is represented as + ```lean4 + .app (.const `Nat.succ []) (.const .zero []) + ``` + -/ + app (fn : Expr) (arg : Expr) + | /-- + Lambda abstraction (aka anonymous functions). + - `fun x : Nat => x` is represented as + ```lean4 + .lam `x (.const `Nat []) (.bvar 0) .default + ``` + -/ + lam (binderName : Name) (binderType : Expr) (body : Expr) (binderInfo : BinderInfo) + | /-- + A dependent arrow (aka forall-expression). It is also used to represent non-dependent arrows. + Examples: + + - `forall x : Prop, x ∧ x` is represented as + ```lean4 + .forallE `x + (.sort .zero) + (.app (.app (.const `And []) (.bvar 0)) (.bvar 0)) + .default + ``` + - `Nat → Bool` as + ```lean4 + .forallE `a (.const `Nat []) (.const `Bool []) .default + ``` + -/ + forallE (binderName : Name) (binderType : Expr) (body : Expr) (binderInfo : BinderInfo) + | /-- + Let-expressions. The field `nonDep` is not currently used, but will be used in the future + by the code generator (and possibly `simp`) to track whether a let-expression is non-dependent + or not. Given an environment, metavariable context, and local context, we say a let-expression + `let x : t := v; e` is non-dependent when it is equivalent to `(fun x : t => e) v`. + Here is an example of a dependent let-expression + `let n : Nat := 2; fun (a : Array Nat n) (b : Array Nat 2) => a = b` is type correct, but + `(fun (n : Nat) (a : Array Nat n) (b : Array Nat 2) => a = b) 2` is not. + The let-expression `let x : Nat := 2; Nat.succ x` is represented as + ``` + .letE `x (.const `Nat []) (.lit (.natVal 2)) (.bvar 0) true + ``` + -/ + letE (declName : Name) (type : Expr) (value : Expr) (body : Expr) (nonDep : Bool) + | /-- + Natural number and string literal values. They are not really needed, but provide a more + compact representation in memory for these two kinds of literals, and are used to implement + efficient reduction in the elaborator and kernel. + The "raw" natural number `2` can be represented as `.lit (.natVal 2)`. Note that, it is + definitionally equal to + ```lean4 + .app (.const `Nat.succ []) (.app (.const `Nat.succ []) (.const `Nat.zero [])) + ``` + -/ + lit : Literal → Expr + | /-- + Metadata (aka annotations). We use annotations to provide hints to the pretty-printer, + store references to `Syntax` nodes, position information, and save information for + elaboration procedures (e.g., we use the `inaccessible` annotation during elaboration to + mark `Expr`s that correspond to inaccessible patterns). + Note that `.mdata data e` is definitionally equal to `e`. + -/ + mdata (data : MData) (expr : Expr) + | /-- + Projection-expressions. They are redundant, but are used to create more compact + terms, speedup reduction, and implement eta for structures. + The type of `struct` must be an structure-like inductive type. That is, it has only one + constructor, is not recursive, and it is not an inductive predicate. The kernel and elaborators + check whether the `typeName` matches the type of `struct`, and whether the (zero-based) index + is valid (i.e., it is smaller than the numbef of constructor fields). + When exporting Lean developments to other systems, `proj` can be replaced with `typeName`.`rec` + applications. + Example, given `a : Nat x Bool`, `a.1` is represented as + ```lean4 + .proj `Prod 0 a + ``` + -/ + proj (typeName : Name) (idx : Nat) (struct : Expr) with @[computedField, extern c inline "lean_ctor_get_uint64(#1, lean_ctor_num_objs(#1)*sizeof(void*))"] data : @& Expr → Data @@ -299,6 +470,7 @@ deriving Inhabited, Repr namespace Expr +/-- The constructor name for the given expression. This is used for debugging purposes. -/ def ctorName : Expr → String | bvar .. => "bvar" | fvar .. => "fvar" @@ -318,27 +490,52 @@ protected def hash (e : Expr) : UInt64 := instance : Hashable Expr := ⟨Expr.hash⟩ +/-- +Return `true` if `e` contains free variables. +This is a constant time operation. +-/ def hasFVar (e : Expr) : Bool := e.data.hasFVar +/-- +Return `true` if `e` contains expression metavariables. +This is a constant time operation. +-/ def hasExprMVar (e : Expr) : Bool := e.data.hasExprMVar +/-- +Return `true` if `e` contains universe (aka `Level`) metavariables. +This is a constant time operation. +-/ def hasLevelMVar (e : Expr) : Bool := e.data.hasLevelMVar -/-- Does the expression contain level or expression metavariables?-/ +/-- +Does the expression contain level (aka universe) or expression metavariables? +This is a constant time operation. +-/ def hasMVar (e : Expr) : Bool := let d := e.data d.hasExprMVar || d.hasLevelMVar +/-- +Return true if `e` contains universe level parameters. +This is a constant time operation. +-/ def hasLevelParam (e : Expr) : Bool := e.data.hasLevelParam +/-- +Return the approximated depth of an expression. This information is used to compute +the expression hash code, and speedup comparisons. +This is a constant time operation. We say it is approximate because it maxes out at `255`. +-/ def approxDepth (e : Expr) : UInt32 := e.data.approxDepth.toUInt32 -/-- The range of de-Bruijn variables that are loose. +/-- +The range of de-Bruijn variables that are loose. That is, bvars that are not bound by a binder. For example, `bvar i` has range `i + 1` and an expression with no loose bvars has range `0`. @@ -346,9 +543,15 @@ an expression with no loose bvars has range `0`. def looseBVarRange (e : Expr) : Nat := e.data.looseBVarRange.toNat +/-- +Return the binder information if `e` is a lambda or forall expression, and `.default` otherwise. +-/ def binderInfo (e : Expr) : BinderInfo := e.data.binderInfo +/-! +Export functions. +-/ @[export lean_expr_hash] def hashEx : Expr → UInt64 := hash @[export lean_expr_has_fvar] def hasFVarEx : Expr → Bool := hasFVar @[export lean_expr_has_expr_mvar] def hasExprMVarEx : Expr → Bool := hasExprMVar @@ -360,53 +563,85 @@ def binderInfo (e : Expr) : BinderInfo := end Expr -def mkConst (n : Name) (lvls : List Level := []) : Expr := - Expr.const n lvls +/-- `mkConst declName us` return `.const declName us`. -/ +def mkConst (declName : Name) (us : List Level := []) : Expr := + .const declName us +/-- Return the type of a literal value. -/ def Literal.type : Literal → Expr - | Literal.natVal _ => mkConst `Nat - | Literal.strVal _ => mkConst `String + | .natVal _ => mkConst `Nat + | .strVal _ => mkConst `String @[export lean_lit_type] def Literal.typeEx : Literal → Expr := Literal.type +/-- `.bvar idx` is now the preferred form. -/ def mkBVar (idx : Nat) : Expr := - Expr.bvar idx + .bvar idx -def mkSort (lvl : Level) : Expr := - Expr.sort lvl +/-- `.sort u` is now the preferred form. -/ +def mkSort (u : Level) : Expr := + .sort u +/-- +`.fvar fvarId` is now the preferred form. +This function is seldom used, free variables are often automatically created using the +telescope functions (e.g., `forallTelescope` and `lambdaTelescope`) at `MetaM`. +-/ def mkFVar (fvarId : FVarId) : Expr := - Expr.fvar fvarId + .fvar fvarId -def mkMVar (fvarId : MVarId) : Expr := - Expr.mvar fvarId +/-- +`.mvar mvarId` is now the preferred form. +This function is seldom used, metavariables are often created using functions such +as `mkFresheExprMVar` at `MetaM`. +-/ +def mkMVar (mvarId : MVarId) : Expr := + .mvar mvarId +/-- +`.mdata m e` is now the preferred form. +-/ def mkMData (m : MData) (e : Expr) : Expr := - Expr.mdata m e + .mdata m e -def mkProj (s : Name) (i : Nat) (e : Expr) : Expr := - Expr.proj s i e +/-- +`.proj structName idx struct` is now the preferred form. +-/ +def mkProj (structName : Name) (idx : Nat) (struct : Expr) : Expr := + .proj structName idx struct +/-- +`.app f a` is now the preferred form. +-/ def mkApp (f a : Expr) : Expr := - Expr.app f a + .app f a +/-- +`.lam x t b bi` is now the preferred form. +-/ def mkLambda (x : Name) (bi : BinderInfo) (t : Expr) (b : Expr) : Expr := - Expr.lam x t b bi + .lam x t b bi +/-- +`.forallE x t b bi` is now the preferred form. +-/ def mkForall (x : Name) (bi : BinderInfo) (t : Expr) (b : Expr) : Expr := - Expr.forallE x t b bi + .forallE x t b bi /-- Return `Unit -> type`. Do not confuse with `Thunk type` -/ def mkSimpleThunkType (type : Expr) : Expr := - mkForall Name.anonymous BinderInfo.default (Lean.mkConst `Unit) type + mkForall Name.anonymous .default (mkConst `Unit) type /-- Return `fun (_ : Unit), e` -/ def mkSimpleThunk (type : Expr) : Expr := - mkLambda `_ BinderInfo.default (Lean.mkConst `Unit) type + mkLambda `_ BinderInfo.default (mkConst `Unit) type +/-- +`.letE x t v b nonDep` is now the preferred form. +-/ def mkLet (x : Name) (t : Expr) (v : Expr) (b : Expr) (nonDep : Bool := false) : Expr := - Expr.letE x t v b nonDep + .letE x t v b nonDep def mkAppB (f a b : Expr) := mkApp (mkApp f a) b def mkApp2 (f a b : Expr) := mkAppB f a b @@ -419,18 +654,32 @@ def mkApp8 (f a b c d e₁ e₂ e₃ e₄ : Expr) := mkApp4 (mkApp4 f a b c d) e def mkApp9 (f a b c d e₁ e₂ e₃ e₄ e₅ : Expr) := mkApp5 (mkApp4 f a b c d) e₁ e₂ e₃ e₄ e₅ def mkApp10 (f a b c d e₁ e₂ e₃ e₄ e₅ e₆ : Expr) := mkApp6 (mkApp4 f a b c d) e₁ e₂ e₃ e₄ e₅ e₆ +/-- +`.lit l` is now the preferred form. +-/ def mkLit (l : Literal) : Expr := - Expr.lit l + .lit l +/-- +Return the "raw" natural number `.lit (.natVal n)`. +This is not the default representation used by the Lean frontend. +See `mkNatLit`. +-/ def mkRawNatLit (n : Nat) : Expr := - mkLit (Literal.natVal n) + mkLit (.natVal n) +/-- +Return a natural number literal used in the frontend. It is a `OfNat.ofNat` application. +Recall that all theorems and definitions containing numeric literals are encoded using +`OfNat.ofNat` applications in the frontend. +-/ def mkNatLit (n : Nat) : Expr := let r := mkRawNatLit n mkApp3 (mkConst ``OfNat.ofNat [levelZero]) (mkConst ``Nat) r (mkApp (mkConst ``instOfNatNat) r) +/-- Return the string literal `.lit (.strVal s)` -/ def mkStrLit (s : String) : Expr := - mkLit (Literal.strVal s) + mkLit (.strVal s) @[export lean_expr_mk_bvar] def mkBVarEx : Nat → Expr := mkBVar @[export lean_expr_mk_fvar] def mkFVarEx : FVarId → Expr := mkFVar @@ -465,105 +714,136 @@ namespace Expr @[extern "lean_expr_dbg_to_string"] opaque dbgToString (e : @& Expr) : String +/-- A total order for expressions. We say it is quick because it first compares the hashcodes. -/ @[extern "lean_expr_quick_lt"] opaque quickLt (a : @& Expr) (b : @& Expr) : Bool +/-- A total order for expressions that takes the structure into account (e.g., variable names). -/ @[extern "lean_expr_lt"] opaque lt (a : @& Expr) (b : @& Expr) : Bool -/-- Return true iff `a` and `b` are alpha equivalent. - Binder annotations are ignored. -/ +/-- +Return true iff `a` and `b` are alpha equivalent. +Binder annotations are ignored. +-/ @[extern "lean_expr_eqv"] opaque eqv (a : @& Expr) (b : @& Expr) : Bool instance : BEq Expr where beq := Expr.eqv -protected unsafe def ptrEq (a b : Expr) : Bool := - ptrAddrUnsafe a == ptrAddrUnsafe b - -/- Return true iff `a` and `b` are equal. - Binder names and annotations are taking into account. -/ +/-- +Return true iff `a` and `b` are equal. +Binder names and annotations are taking into account. +-/ @[extern "lean_expr_equal"] opaque equal (a : @& Expr) (b : @& Expr) : Bool +/-- Return `true` if the given expression is a `.sort ..` -/ def isSort : Expr → Bool | sort .. => true | _ => false +/-- Return `true` if the given expression is of the form `.sort (.succ ..)`. -/ def isType : Expr → Bool - | sort (Level.succ ..) => true + | sort (.succ ..) => true | _ => false +/-- Return `true` if the given expression is a `.sort .zero` -/ def isProp : Expr → Bool - | sort (Level.zero ..) => true + | sort (.zero ..) => true | _ => false +/-- Return `true` if the given expression is a bound variable. -/ def isBVar : Expr → Bool | bvar .. => true | _ => false +/-- Return `true` if the given expression is a metavariable. -/ def isMVar : Expr → Bool | mvar .. => true | _ => false +/-- Return `true` if the given expression is a free variable. -/ def isFVar : Expr → Bool | fvar .. => true | _ => false +/-- Return `true` if the given expression is an application. -/ def isApp : Expr → Bool | app .. => true | _ => false +/-- Return `true` if the given expression is a projection `.proj ..` -/ def isProj : Expr → Bool | proj .. => true | _ => false +/-- Return `true` if the given expression is a constant. -/ def isConst : Expr → Bool | const .. => true | _ => false +/-- +Return `true` if the given expression is a constant of the give name. +Examples: +- `` (.const `Nat []).isConstOf `Nat `` is `true` +- `` (.const `Nat []).isConstOf `False `` is `false` +-/ def isConstOf : Expr → Name → Bool | const n .., m => n == m | _, _ => false +/-- Return `true` if the given expression is a forall-expression aka (dependent) arrow. -/ def isForall : Expr → Bool | forallE .. => true | _ => false +/-- Return `true` if the given expression is a lambda abstraction aka anonymous function. -/ def isLambda : Expr → Bool | lam .. => true | _ => false +/-- Return `true` if the given expression is a forall or lambda expression. -/ def isBinding : Expr → Bool | lam .. => true | forallE .. => true | _ => false +/-- Return `true` if the given expression is a let-expression. -/ def isLet : Expr → Bool | letE .. => true | _ => false +/-- Return `true` if the given expression is a metadata. -/ def isMData : Expr → Bool | mdata .. => true | _ => false +/-- Return `true` if the given expression is a literal value. -/ def isLit : Expr → Bool | lit .. => true | _ => false +/-- +Return the "body" of a forall expression. +Example: let `e` be the representation for `forall (p : Prop) (q : Prop), p ∧ q`, then +`getForallBody e` returns ``.app (.app (.const `And []) (.bvar 1)) (.bvar 0)`` +-/ def getForallBody : Expr → Expr | forallE _ _ b .. => getForallBody b | e => e -/-- If the given expression is a sequence of +/-- +If the given expression is a sequence of function applications `f a₁ .. aₙ`, return `f`. -Otherwise return the input expression. -/ +Otherwise return the input expression. +-/ def getAppFn : Expr → Expr | app f _ => getAppFn f | e => e -def getAppNumArgsAux : Expr → Nat → Nat +private def getAppNumArgsAux : Expr → Nat → Nat | app f _, n => getAppNumArgsAux f (n+1) | _, n => n @@ -637,8 +917,10 @@ def isAppOf (e : Expr) (n : Name) : Bool := | const c _ => c == n | _ => false -/-- Given `f a₁ ... aᵢ`, returns true if `f` is a constant -with name `n` and has the correct number of arguments. -/ +/-- +Given `f a₁ ... aᵢ`, returns true if `f` is a constant +with name `n` and has the correct number of arguments. +-/ def isAppOfArity : Expr → Name → Nat → Bool | const c _, n, 0 => c == n | app f _, n, a+1 => isAppOfArity f n a @@ -771,7 +1053,10 @@ def projIdx! : Expr → Nat def hasLooseBVars (e : Expr) : Bool := e.looseBVarRange > 0 -/- Remark: the following function assumes `e` does not have loose bound variables. -/ +/-- +Return `true` if `e` is a non-dependent arrow. +Remark: the following function assumes `e` does not have loose bound variables. +-/ def isArrow (e : Expr) : Bool := match e with | forallE _ _ b _ => !b.hasLooseBVars @@ -787,11 +1072,12 @@ def hasLooseBVarInExplicitDomain : Expr → Nat → Bool → Bool | e, bvarIdx, tryRange => tryRange && hasLooseBVar e bvarIdx /-- - Lower the loose bound variables `>= s` in `e` by `d`. - That is, a loose bound variable `bvar i`. - `i >= s` is mapped into `bvar (i-d)`. +Lower the loose bound variables `>= s` in `e` by `d`. +That is, a loose bound variable `bvar i`. +`i >= s` is mapped into `bvar (i-d)`. - Remark: if `s < d`, then result is `e` -/ +Remark: if `s < d`, then result is `e` +-/ @[extern "lean_expr_lower_loose_bvars"] opaque lowerLooseBVars (e : @& Expr) (s d : @& Nat) : Expr @@ -801,12 +1087,12 @@ opaque lowerLooseBVars (e : @& Expr) (s d : @& Nat) : Expr opaque liftLooseBVars (e : @& Expr) (s d : @& Nat) : Expr /-- - `inferImplicit e numParams considerRange` updates the first `numParams` parameter binder annotations of the `e` forall type. - It marks any parameter with an explicit binder annotation if there is another explicit arguments that depends on it or - the resulting type if `considerRange == true`. +`inferImplicit e numParams considerRange` updates the first `numParams` parameter binder annotations of the `e` forall type. +It marks any parameter with an explicit binder annotation if there is another explicit arguments that depends on it or +the resulting type if `considerRange == true`. - Remark: we use this function to infer the bind annotations of inductive datatype constructors, and structure projections. - When the `{}` annotation is used in these commands, we set `considerRange == false`. +Remark: we use this function to infer the bind annotations of inductive datatype constructors, and structure projections. +When the `{}` annotation is used in these commands, we set `considerRange == false`. -/ def inferImplicit : Expr → Nat → Bool → Expr | Expr.forallE n d b bi, i+1, considerRange => @@ -816,8 +1102,10 @@ def inferImplicit : Expr → Nat → Bool → Expr | e, 0, _ => e | e, _, _ => e -/-- Instantiate the loose bound variables in `e` using `subst`. - That is, a loose `Expr.bvar i` is replaced with `subst[i]`. -/ +/-- +Instantiate the loose bound variables in `e` using `subst`. +That is, a loose `Expr.bvar i` is replaced with `subst[i]`. +-/ @[extern "lean_expr_instantiate"] opaque instantiate (e : @& Expr) (subst : @& Array Expr) : Expr @@ -828,13 +1116,17 @@ opaque instantiate1 (e : @& Expr) (subst : @& Expr) : Expr @[extern "lean_expr_instantiate_rev"] opaque instantiateRev (e : @& Expr) (subst : @& Array Expr) : Expr -/-- Similar to `instantiate`, but consider only the variables `xs` in the range `[beginIdx, endIdx)`. - Function panics if `beginIdx <= endIdx <= xs.size` does not hold. -/ +/-- +Similar to `instantiate`, but consider only the variables `xs` in the range `[beginIdx, endIdx)`. +Function panics if `beginIdx <= endIdx <= xs.size` does not hold. +-/ @[extern "lean_expr_instantiate_range"] opaque instantiateRange (e : @& Expr) (beginIdx endIdx : @& Nat) (xs : @& Array Expr) : Expr -/-- Similar to `instantiateRev`, but consider only the variables `xs` in the range `[beginIdx, endIdx)`. - Function panics if `beginIdx <= endIdx <= xs.size` does not hold. -/ +/-- +Similar to `instantiateRev`, but consider only the variables `xs` in the range `[beginIdx, endIdx)`. +Function panics if `beginIdx <= endIdx <= xs.size` does not hold. +-/ @[extern "lean_expr_instantiate_rev_range"] opaque instantiateRevRange (e : @& Expr) (beginIdx endIdx : @& Nat) (xs : @& Array Expr) : Expr @@ -887,7 +1179,7 @@ abbrev ExprSet := HashSet Expr abbrev PersistentExprSet := PHashSet Expr abbrev PExprSet := PersistentExprSet -/- Auxiliary type for forcing `==` to be structural equality for `Expr` -/ +/-- Auxiliary type for forcing `==` to be structural equality for `Expr` -/ structure ExprStructEq where val : Expr deriving Inhabited @@ -924,19 +1216,19 @@ def mkAppRevRange (f : Expr) (beginIdx endIdx : Nat) (revArgs : Array Expr) : Ex mkAppRevRangeAux revArgs beginIdx f endIdx /-- - If `f` is a lambda expression, than "beta-reduce" it using `revArgs`. - This function is often used with `getAppRev` or `withAppRev`. - Examples: - - `betaRev (fun x y => t x y) #[]` ==> `fun x y => t x y` - - `betaRev (fun x y => t x y) #[a]` ==> `fun y => t a y` - - `betaRev (fun x y => t x y) #[a, b]` ==> `t b a` - - `betaRev (fun x y => t x y) #[a, b, c, d]` ==> `t d c b a` - Suppose `t` is `(fun x y => t x y) a b c d`, then - `args := t.getAppRev` is `#[d, c, b, a]`, - and `betaRev (fun x y => t x y) #[d, c, b, a]` is `t a b c d`. - - If `useZeta` is true, the function also performs zeta-reduction (reduction of let binders) to create further - opportunities for beta reduction. +If `f` is a lambda expression, than "beta-reduce" it using `revArgs`. +This function is often used with `getAppRev` or `withAppRev`. +Examples: +- `betaRev (fun x y => t x y) #[]` ==> `fun x y => t x y` +- `betaRev (fun x y => t x y) #[a]` ==> `fun y => t a y` +- `betaRev (fun x y => t x y) #[a, b]` ==> `t b a` +- `betaRev (fun x y => t x y) #[a, b, c, d]` ==> `t d c b a` +Suppose `t` is `(fun x y => t x y) a b c d`, then +`args := t.getAppRev` is `#[d, c, b, a]`, +and `betaRev (fun x y => t x y) #[d, c, b, a]` is `t a b c d`. + +If `useZeta` is true, the function also performs zeta-reduction (reduction of let binders) to create further +opportunities for beta reduction. -/ partial def betaRev (f : Expr) (revArgs : Array Expr) (useZeta := false) (preserveMData := false) : Expr := if revArgs.size == 0 then f @@ -967,11 +1259,20 @@ partial def betaRev (f : Expr) (revArgs : Array Expr) (useZeta := false) (preser mkAppRevRange (b.instantiateRange n sz revArgs) 0 n revArgs go f 0 -/-- Apply the given arguments to `f`, beta-reducing if `f` is a -lambda expression. See docstring for `betaRev` for examples. -/ +/-- +Apply the given arguments to `f`, beta-reducing if `f` is a +lambda expression. See docstring for `betaRev` for examples. +-/ def beta (f : Expr) (args : Array Expr) : Expr := betaRev f args.reverse +/-- +Return true if the given expression is the function of an expression that is target for (head) beta reduction. +If `useZeta = true`, then `let`-expressions are visited. That is, it assumes +that zeta-reduction (aka let-expansion) is going to be used. + +See `isHeadBetaTarget`. +-/ def isHeadBetaTargetFn (useZeta : Bool) : Expr → Bool | Expr.lam .. => true | Expr.letE _ _ _ b _ => useZeta && isHeadBetaTargetFn useZeta b @@ -983,6 +1284,11 @@ def headBeta (e : Expr) : Expr := let f := e.getAppFn if f.isHeadBetaTargetFn false then betaRev f e.getAppRevArgs else e +/-- +Return true if the given expression is a target for (head) beta reduction. +If `useZeta = true`, then `let`-expressions are visited. That is, it assumes +that zeta-reduction (aka let-expansion) is going to be used. +-/ def isHeadBetaTarget (e : Expr) (useZeta := false) : Bool := e.getAppFn.isHeadBetaTargetFn useZeta @@ -996,12 +1302,13 @@ private def etaExpandedAux : Expr → Nat → Option Expr | e, n => etaExpandedBody e n 0 /-- - If `e` is of the form `(fun x₁ ... xₙ => f x₁ ... xₙ)` and `f` does not contain `x₁`, ..., `xₙ`, - then return `some f`. Otherwise, return `none`. +If `e` is of the form `(fun x₁ ... xₙ => f x₁ ... xₙ)` and `f` does not contain `x₁`, ..., `xₙ`, +then return `some f`. Otherwise, return `none`. - It assumes `e` does not have loose bound variables. +It assumes `e` does not have loose bound variables. - Remark: `ₙ` may be 0 -/ +Remark: `ₙ` may be 0 +-/ def etaExpanded? (e : Expr) : Option Expr := etaExpandedAux e 0 @@ -1010,28 +1317,40 @@ def etaExpandedStrict? : Expr → Option Expr | lam _ _ b _ => etaExpandedAux b 1 | _ => none +/-- Return `some e'` if `e` is of the form `optParam _ e'` -/ def getOptParamDefault? (e : Expr) : Option Expr := if e.isAppOfArity ``optParam 2 then some e.appArg! else none +/-- Return `some e'` if `e` is of the form `autoParam _ e'` -/ def getAutoParamTactic? (e : Expr) : Option Expr := if e.isAppOfArity ``autoParam 2 then some e.appArg! else none +/-- Return `true` if `e` is of the form `outParam _` -/ @[export lean_is_out_param] def isOutParam (e : Expr) : Bool := e.isAppOfArity ``outParam 1 +/-- Return `true` if `e` is of the form `optParam _ _` -/ def isOptParam (e : Expr) : Bool := e.isAppOfArity ``optParam 2 +/-- Return `true` if `e` is of the form `autoParam _ _` -/ def isAutoParam (e : Expr) : Bool := e.isAppOfArity ``autoParam 2 +/-- +Remove `outParam`, `optParam`, and `autoParam` applications/annotations from `e`. +Note that it does not remove nested annotations. +Examples: +- Given `e` of the form `outParam (optParam Nat b)`, `consumeTypeAnnotations e = b`. +- Given `e` of the form `Nat → outParam (optParam Nat b)`, `consumeTypeAnnotations e = e`. +-/ @[export lean_expr_consume_type_annotations] partial def consumeTypeAnnotations (e : Expr) : Expr := if e.isOptParam || e.isAutoParam then @@ -1041,9 +1360,16 @@ partial def consumeTypeAnnotations (e : Expr) : Expr := else e -partial def consumeMDataAndTypeAnnotations (e : Expr) : Expr := +/-- +Remove metadata annotations and `outParam`, `optParam`, and `autoParam` applications/annotations from `e`. +Note that it does not remove nested annotations. +Examples: +- Given `e` of the form `outParam (optParam Nat b)`, `cleanupAnnotations e = b`. +- Given `e` of the form `Nat → outParam (optParam Nat b)`, `cleanupAnnotations e = e`. +-/ +partial def cleanupAnnotations (e : Expr) : Expr := let e' := e.consumeMData.consumeTypeAnnotations - if e' == e then e else consumeMDataAndTypeAnnotations e' + if e' == e then e else cleanupAnnotations e' /-- Return true iff `e` contains a free variable which statisfies `p`. -/ @[inline] def hasAnyFVar (e : Expr) (p : FVarId → Bool) : Bool := @@ -1059,108 +1385,133 @@ partial def consumeMDataAndTypeAnnotations (e : Expr) : Expr := | _ => false visit e +/-- Return `true` if `e` contains the given free variable. -/ def containsFVar (e : Expr) (fvarId : FVarId) : Bool := e.hasAnyFVar (· == fvarId) -/- The update functions here are defined using C code. They will try to avoid - allocating new values using pointer equality. - The hypotheses `(h : e.is...)` are used to ensure Lean will not crash - at runtime. - The `update*!` functions are inlined and provide a convenient way of using the - update proofs without providing proofs. - Note that if they are used under a match-expression, the compiler will eliminate - the double-match. -/ - -@[extern "lean_expr_update_app"] -def updateApp (e : Expr) (newFn : Expr) (newArg : Expr) (h : e.isApp) : Expr := - mkApp newFn newArg - -@[inline] def updateApp! (e : Expr) (newFn : Expr) (newArg : Expr) : Expr := - match h : e with - | app .. => updateApp e newFn newArg (h ▸ rfl) - | _ => panic! "application expected" - -@[extern "lean_expr_update_const"] -def updateConst (e : Expr) (newLevels : List Level) (h : e.isConst) : Expr := - mkConst e.constName! newLevels - -@[inline] def updateConst! (e : Expr) (newLevels : List Level) : Expr := - match h : e with - | const .. => updateConst e newLevels (h ▸ rfl) - | _ => panic! "constant expected" - -@[extern "lean_expr_update_sort"] -def updateSort (e : Expr) (newLevel : Level) (h : e.isSort) : Expr := - mkSort newLevel - -@[inline] def updateSort! (e : Expr) (newLevel : Level) : Expr := - match h : e with - | sort .. => updateSort e newLevel (h ▸ rfl) - | _ => panic! "level expected" - -@[extern "lean_expr_update_proj"] -def updateProj (e : Expr) (newExpr : Expr) (h : e.isProj) : Expr := +/-! +The update functions try to avoid allocating new values using pointer equality. +Note that if the `update*!` functions are used under a match-expression, +the compiler will eliminate the double-match. +-/ + +@[inline] private unsafe def updateApp!Impl (e : Expr) (newFn : Expr) (newArg : Expr) : Expr := + match e with + | app fn arg => if ptrEq fn newFn && ptrEq arg newArg then e else mkApp newFn newArg + | _ => panic! "application expected" + +@[implementedBy updateApp!Impl] +def updateApp! (e : Expr) (newFn : Expr) (newArg : Expr) : Expr := match e with - | proj s i .. => mkProj s i newExpr - | _ => e -- unreachable because of `h` + | app _ _ => mkApp newFn newArg + | _ => panic! "application expected" -@[extern "lean_expr_update_mdata"] -def updateMData (e : Expr) (newExpr : Expr) (h : e.isMData) : Expr := +@[inline] private unsafe def updateConst!Impl (e : Expr) (newLevels : List Level) : Expr := match e with - | mdata d .. => mkMData d newExpr - | _ => e -- unreachable because of `h` + | const n ls => if ptrEqList ls newLevels then e else mkConst n newLevels + | _ => panic! "constant expected" -@[inline] def updateMData! (e : Expr) (newExpr : Expr) : Expr := - match h : e with - | mdata .. => updateMData e newExpr (h ▸ rfl) - | _ => panic! "mdata expected" +@[implementedBy updateConst!Impl] +def updateConst! (e : Expr) (newLevels : List Level) : Expr := + match e with + | const n _ => mkConst n newLevels + | _ => panic! "constant expected" -@[inline] def updateProj! (e : Expr) (newExpr : Expr) : Expr := - match h : e with - | proj .. => updateProj e newExpr (h ▸ rfl) - | _ => panic! "proj expected" +@[inline] private unsafe def updateSort!Impl (e : Expr) (u' : Level) : Expr := + match e with + | sort u => if ptrEq u u' then e else mkSort u' + | _ => panic! "level expected" -@[extern "lean_expr_update_forall"] -def updateForall (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) (h : e.isForall) : Expr := - mkForall e.bindingName! newBinfo newDomain newBody +@[implementedBy updateSort!Impl] +def updateSort! (e : Expr) (newLevel : Level) : Expr := + match e with + | sort _ => mkSort newLevel + | _ => panic! "level expected" -@[inline] def updateForall! (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := - match h : e with - | forallE .. => updateForall e newBinfo newDomain newBody (h ▸ rfl) - | _ => panic! "forall expected" +@[inline] private unsafe def updateMData!Impl (e : Expr) (newExpr : Expr) : Expr := + match e with + | mdata d a => if ptrEq a newExpr then e else mkMData d newExpr + | _ => panic! "mdata expected" -@[inline] def updateForallE! (e : Expr) (newDomain : Expr) (newBody : Expr) : Expr := - match h : e with - | forallE _ _ _ c => updateForall e c newDomain newBody (h ▸ rfl) +@[implementedBy updateMData!Impl] +def updateMData! (e : Expr) (newExpr : Expr) : Expr := + match e with + | mdata d _ => mkMData d newExpr + | _ => panic! "mdata expected" + +@[inline] private unsafe def updateProj!Impl (e : Expr) (newExpr : Expr) : Expr := + match e with + | proj s i a => if ptrEq a newExpr then e else mkProj s i newExpr + | _ => panic! "proj expected" + +@[implementedBy updateProj!Impl] +def updateProj! (e : Expr) (newExpr : Expr) : Expr := + match e with + | proj s i _ => mkProj s i newExpr + | _ => panic! "proj expected" + +@[inline] private unsafe def updateForall!Impl (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | forallE n d b bi => + if ptrEq d newDomain && ptrEq b newBody && bi == newBinfo then + e + else + mkForall n newBinfo newDomain newBody | _ => panic! "forall expected" -@[extern "lean_expr_update_lambda"] -def updateLambda (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) (h : e.isLambda) : Expr := - mkLambda e.bindingName! newBinfo newDomain newBody +@[implementedBy updateForall!Impl] +def updateForall! (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | forallE n _ _ _ => mkForall n newBinfo newDomain newBody + | _ => panic! "forall expected" -@[inline] def updateLambda! (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := - match h : e with - | lam .. => updateLambda e newBinfo newDomain newBody (h ▸ rfl) - | _ => panic! "lambda expected" +@[inline] def updateForallE! (e : Expr) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | forallE n d b bi => updateForall! (forallE n d b bi) bi newDomain newBody + | _ => panic! "forall expected" -@[inline] def updateLambdaE! (e : Expr) (newDomain : Expr) (newBody : Expr) : Expr := - match h : e with - | lam _ _ _ c => updateLambda e c newDomain newBody (h ▸ rfl) +@[inline] private unsafe def updateLambda!Impl (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | lam n d b bi => + if ptrEq d newDomain && ptrEq b newBody && bi == newBinfo then + e + else + mkLambda n newBinfo newDomain newBody | _ => panic! "lambda expected" -@[extern "lean_expr_update_let"] -def updateLet (e : Expr) (newType : Expr) (newVal : Expr) (newBody : Expr) (h : e.isLet) : Expr := - mkLet e.letName! newType newVal newBody +@[implementedBy updateLambda!Impl] +def updateLambda! (e : Expr) (newBinfo : BinderInfo) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | lam n _ _ _ => mkLambda n newBinfo newDomain newBody + | _ => panic! "lambda expected" -@[inline] def updateLet! (e : Expr) (newType : Expr) (newVal : Expr) (newBody : Expr) : Expr := - match h : e with - | letE .. => updateLet e newType newVal newBody (h ▸ rfl) - | _ => panic! "let expression expected" +@[inline] def updateLambdaE! (e : Expr) (newDomain : Expr) (newBody : Expr) : Expr := + match e with + | lam n d b bi => updateLambda! (lam n d b bi) bi newDomain newBody + | _ => panic! "lambda expected" + +@[inline] private unsafe def updateLet!Impl (e : Expr) (newType : Expr) (newVal : Expr) (newBody : Expr) : Expr := + match e with + | letE n t v b nonDep => + if ptrEq t newType && ptrEq v newVal && ptrEq b newBody then + e + else + letE n newType newVal newBody nonDep + | _ => panic! "let expression expected" + +@[implementedBy updateLet!Impl] +def updateLet! (e : Expr) (newType : Expr) (newVal : Expr) (newBody : Expr) : Expr := + match e with + | letE n _ _ _ c => letE n newType newVal newBody c + | _ => panic! "let expression expected" def updateFn : Expr → Expr → Expr | e@(app f a), g => e.updateApp! (updateFn f g) a | _, g => g +/-- +Eta reduction. If `e` is of the form `(fun x => f x)`, then return `f`. +-/ partial def eta (e : Expr) : Expr := match e with | Expr.lam _ d b _ => @@ -1174,8 +1525,9 @@ partial def eta (e : Expr) : Expr := | _ => e.updateLambdaE! d b' | _ => e -/- Instantiate level parameters -/ - +/-- +Instantiate level parameters +-/ @[inline] def instantiateLevelParamsCore (s : Name → Option Level) (e : Expr) : Expr := let rec @[specialize] visit (e : Expr) : Expr := if !e.hasLevelParam then e @@ -1195,6 +1547,10 @@ private def getParamSubst : List Name → List Level → Name → Option Level | p::ps, u::us, p' => if p == p' then some u else getParamSubst ps us p' | _, _, _ => none +/-- +Instantiate univeres level parameters names `paramNames` with `lvls` in `e`. +If the two lists have different length, the smallest one is used. +-/ def instantiateLevelParams (e : Expr) (paramNames : List Name) (lvls : List Level) : Expr := instantiateLevelParamsCore (getParamSubst paramNames lvls) e @@ -1207,23 +1563,38 @@ private partial def getParamSubstArray (ps : Array Name) (us : Array Level) (p' else none else none +/-- +Instantiate univeres level parameters names `paramNames` with `lvls` in `e`. +If the two arrays have different length, the smallest one is used. +-/ def instantiateLevelParamsArray (e : Expr) (paramNames : Array Name) (lvls : Array Level) : Expr := instantiateLevelParamsCore (fun p => getParamSubstArray paramNames lvls p 0) e -/-- Annotate `e` with the given option. -/ +/-- +Annotate `e` with the given option. +The information is stored using metadata around `e`. +-/ def setOption (e : Expr) (optionName : Name) [KVMap.Value α] (val : α) : Expr := mkMData (MData.empty.set optionName val) e -/-- Annotate `e` with `pp.explicit := true` - The delaborator uses `pp` options. -/ +/-- +Annotate `e` with `pp.explicit := flag` +The delaborator uses `pp` options. +-/ def setPPExplicit (e : Expr) (flag : Bool) := e.setOption `pp.explicit flag +/-- +Annotate `e` with `pp.universes := flag` +The delaborator uses `pp` options. +-/ def setPPUniverses (e : Expr) (flag : Bool) := e.setOption `pp.universes flag -/-- If `e` is an application `f a_1 ... a_n` annotate `f`, `a_1` ... `a_n` with `pp.explicit := false`, - and annotate `e` with `pp.explicit := true`. -/ +/-- +If `e` is an application `f a_1 ... a_n` annotate `f`, `a_1` ... `a_n` with `pp.explicit := false`, +and annotate `e` with `pp.explicit := true`. +-/ def setAppPPExplicit (e : Expr) : Expr := match e with | app .. => @@ -1232,8 +1603,10 @@ def setAppPPExplicit (e : Expr) : Expr := mkAppN f args |>.setPPExplicit true | _ => e -/-- Similar for `setAppPPExplicit`, but only annotate children with `pp.explicit := false` if - `e` does not contain metavariables. -/ +/-- +Similar for `setAppPPExplicit`, but only annotate children with `pp.explicit := false` if +`e` does not contain metavariables. +-/ def setAppPPExplicitForExposingMVars (e : Expr) : Expr := match e with | app .. => @@ -1244,40 +1617,60 @@ def setAppPPExplicitForExposingMVars (e : Expr) : Expr := end Expr +/-- +Annotate `e` with the given annotation name `kind`. +It uses metadata to store the annotation. +-/ def mkAnnotation (kind : Name) (e : Expr) : Expr := mkMData (KVMap.empty.insert kind (DataValue.ofBool true)) e +/-- +Return `some e'` if `e = mkAnnotation kind e'` +-/ def annotation? (kind : Name) (e : Expr) : Option Expr := match e with | .mdata d b => if d.size == 1 && d.getBool kind false then some b else none | _ => none +/-- +Annotate `e` with the `let_fun` annotation. This annotation is used as hint for the delaborator. +If `e` is of the form `(fun x : t => b) v`, then `mkLetFunAnnotation e` is delaborated at +`let_fun x : t := v; b` +-/ def mkLetFunAnnotation (e : Expr) : Expr := mkAnnotation `let_fun e +/-- +Return `some e'` if `e = mkLetFunAnnotation e'` +-/ def letFunAnnotation? (e : Expr) : Option Expr := annotation? `let_fun e +/-- +Return true if `e = mkLetFunAnnotation e'`, and `e'` is of the form `(fun x : t => b) v` +-/ def isLetFun (e : Expr) : Bool := match letFunAnnotation? e with | none => false | some e => e.isApp && e.appFn!.isLambda /-- - Auxiliary annotation used to mark terms marked with the "inaccessible" annotation `.(t)` and - `_` in patterns. -/ +Auxiliary annotation used to mark terms marked with the "inaccessible" annotation `.(t)` and +`_` in patterns. +-/ def mkInaccessible (e : Expr) : Expr := mkAnnotation `_inaccessible e +/-- Return `some e'` if `e = mkInaccessible e'`. -/ def inaccessible? (e : Expr) : Option Expr := annotation? `_inaccessible e private def patternRefAnnotationKey := `_patWithRef /-- - During elaboration expressions corresponding to pattern matching terms - are annotated with `Syntax` objects. This function returns `some (stx, p')` if - `p` is the pattern `p'` annotated with `stx` +During elaboration expressions corresponding to pattern matching terms +are annotated with `Syntax` objects. This function returns `some (stx, p')` if +`p` is the pattern `p'` annotated with `stx` -/ def patternWithRef? (p : Expr) : Option (Syntax × Expr) := match p with @@ -1288,8 +1681,8 @@ def patternWithRef? (p : Expr) : Option (Syntax × Expr) := | _ => none /-- - Annotate the pattern `p` with `stx`. This is an auxiliary annotation - for producing better hover information. +Annotate the pattern `p` with `stx`. This is an auxiliary annotation +for producing better hover information. -/ def mkPatternWithRef (p : Expr) (stx : Syntax) : Expr := if patternWithRef? p |>.isSome then @@ -1307,12 +1700,14 @@ def patternAnnotation? (e : Expr) : Option Expr := none /-- - Annotate `e` with the LHS annotation. The delaborator displays - expressions of the form `lhs = rhs` as `lhs` when they have this annotation. +Annotate `e` with the LHS annotation. The delaborator displays +expressions of the form `lhs = rhs` as `lhs` when they have this annotation. +This is used to implement the infoview for the `conv` mode. -/ def mkLHSGoal (e : Expr) : Expr := mkAnnotation `_lhsGoal e +/-- Return `some lhs` if `e = mkLHGoal e'`, where `e'` is of the form `lhs = rhs`. -/ def isLHSGoal? (e : Expr) : Option Expr := match annotation? `_lhsGoal e with | none => none @@ -1322,15 +1717,27 @@ def isLHSGoal? (e : Expr) : Option Expr := else none -def mkFreshFVarId {m : Type → Type} [Monad m] [MonadNameGenerator m] : m FVarId := +/-- +Polymorphic operation for generating unique/fresh free variable identifiers. +It is available in any monad `m` that implements the inferface `MonadNameGenerator`. +-/ +def mkFreshFVarId [Monad m] [MonadNameGenerator m] : m FVarId := return { name := (← mkFreshId) } -def mkFreshMVarId {m : Type → Type} [Monad m] [MonadNameGenerator m] : m MVarId := +/-- +Polymorphic operation for generating unique/fresh metavariable identifiers. +It is available in any monad `m` that implements the inferface `MonadNameGenerator`. +-/ +def mkFreshMVarId [Monad m] [MonadNameGenerator m] : m MVarId := return { name := (← mkFreshId) } +/-- Return `Not p` -/ def mkNot (p : Expr) : Expr := mkApp (mkConst ``Not) p +/-- Return `p ∨ q` -/ def mkOr (p q : Expr) : Expr := mkApp2 (mkConst ``Or) p q +/-- Return `p ∧ q` -/ def mkAnd (p q : Expr) : Expr := mkApp2 (mkConst ``And) p q +/-- Return `Classical.em p` -/ def mkEM (p : Expr) : Expr := mkApp (mkConst ``Classical.em) p end Lean diff --git a/stage0/src/Lean/Level.lean b/stage0/src/Lean/Level.lean index c5efb8df8e67..4e93c0b56fc5 100644 --- a/stage0/src/Lean/Level.lean +++ b/stage0/src/Lean/Level.lean @@ -493,11 +493,9 @@ end Level elseK () /- Similar to `mkLevelMax`, but applies cheap simplifications -/ -@[export lean_level_mk_max_simp] def mkLevelMax' (u v : Level) : Level := mkLevelMaxCore u v fun _ => mkLevelMax u v -@[export lean_level_simp_max] def simpLevelMax' (u v : Level) (d : Level) : Level := mkLevelMaxCore u v fun _ => d @@ -509,51 +507,52 @@ def simpLevelMax' (u v : Level) (d : Level) : Level := else elseK () /- Similar to `mkLevelIMax`, but applies cheap simplifications -/ -@[export lean_level_mk_imax_simp] def mkLevelIMax' (u v : Level) : Level := mkLevelIMaxCore u v fun _ => mkLevelIMax u v -@[export lean_level_simp_imax] def simpLevelIMax' (u v : Level) (d : Level) := mkLevelIMaxCore u v fun _ => d namespace Level -/- The update functions here are defined using C code. They will try to avoid - allocating new values using pointer equality. - The hypotheses `(h : e.is...)` are used to ensure Lean will not crash - at runtime. - The `update*!` functions are inlined and provide a convenient way of using the - update proofs without providing proofs. - Note that if they are used under a match-expression, the compiler will eliminate - the double-match. -/ - -@[extern "lean_level_update_succ"] -def updateSucc (lvl : Level) (newLvl : Level) (h : lvl.isSucc) : Level := - mkLevelSucc newLvl - -@[inline] def updateSucc! (lvl : Level) (newLvl : Level) : Level := -match h : lvl with - | succ .. => updateSucc lvl newLvl (h ▸ rfl) - | _ => panic! "succ level expected" - -@[extern "lean_level_update_max"] -def updateMax (lvl : Level) (newLhs : Level) (newRhs : Level) (h : lvl.isMax) : Level := - mkLevelMax' newLhs newRhs - -@[inline] def updateMax! (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := - match h : lvl with - | max .. => updateMax lvl newLhs newRhs (h ▸ rfl) - | _ => panic! "max level expected" - -@[extern "lean_level_update_imax"] -def updateIMax (lvl : Level) (newLhs : Level) (newRhs : Level) (h : lvl.isIMax) : Level := - mkLevelIMax' newLhs newRhs - -@[inline] def updateIMax! (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := - match h : lvl with - | imax .. => updateIMax lvl newLhs newRhs (h ▸ rfl) - | _ => panic! "imax level expected" +/-! +The update functions try to avoid allocating new values using pointer equality. +Note that if the `update*!` functions are used under a match-expression, +the compiler will eliminate the double-match. +-/ + +@[inline] private unsafe def updateSucc!Impl (lvl : Level) (newLvl : Level) : Level := + match lvl with + | succ l => if ptrEq l newLvl then lvl else mkLevelSucc newLvl + | _ => panic! "succ level expected" + +@[implementedBy updateSucc!Impl] +def updateSucc! (lvl : Level) (newLvl : Level) : Level := + match lvl with + | succ _ => mkLevelSucc newLvl + | _ => panic! "succ level expected" + +@[inline] private unsafe def updateMax!Impl (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := + match lvl with + | max lhs rhs => if ptrEq lhs newLhs && ptrEq rhs newRhs then simpLevelMax' newLhs newRhs lvl else mkLevelMax' newLhs newRhs + | _ => panic! "max level expected" + +@[implementedBy updateMax!Impl] +def updateMax! (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := + match lvl with + | max _ _ => mkLevelMax' newLhs newRhs + | _ => panic! "max level expected" + +@[inline] private unsafe def updateIMax!Impl (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := + match lvl with + | imax lhs rhs => if ptrEq lhs newLhs && ptrEq rhs newRhs then simpLevelIMax' newLhs newRhs lvl else mkLevelIMax' newLhs newRhs + | _ => panic! "imax level expected" + +@[implementedBy updateIMax!Impl] +def updateIMax! (lvl : Level) (newLhs : Level) (newRhs : Level) : Level := + match lvl with + | imax _ _ => mkLevelIMax' newLhs newRhs + | _ => panic! "imax level expected" def mkNaryMax : List Level → Level | [] => levelZero diff --git a/stage0/src/Lean/Linter/Basic.lean b/stage0/src/Lean/Linter/Basic.lean index dc627c584d40..c2f28b5abc76 100644 --- a/stage0/src/Lean/Linter/Basic.lean +++ b/stage0/src/Lean/Linter/Basic.lean @@ -25,12 +25,12 @@ def getLinterUnusedVariables (o : Options) : Bool := o.get linter.unusedVariable def getLinterUnusedVariablesFunArgs (o : Options) : Bool := o.get linter.unusedVariables.funArgs.name (getLinterUnusedVariables o) def getLinterUnusedVariablesPatternVars (o : Options) : Bool := o.get linter.unusedVariables.patternVars.name (getLinterUnusedVariables o) -def unusedVariables : Linter := fun stx => do +def unusedVariables : Linter := fun cmdStx => do -- NOTE: `messages` is local to the current command if (← get).messages.hasErrors then return - let some stxRange := stx.getRange? + let some cmdStxRange := cmdStx.getRange? | pure () let infoTrees := (← get).infoState.trees.toArray @@ -40,7 +40,7 @@ def unusedVariables : Linter := fun stx => do return -- collect references - let refs := findModuleRefs fileMap infoTrees + let refs := findModuleRefs fileMap infoTrees (allowSimultaneousBinderUse := true) let mut vars : HashMap FVarId RefInfo := .empty let mut constDecls : HashSet String.Range := .empty @@ -76,6 +76,7 @@ def unusedVariables : Linter := fun stx => do -- determine unused variables for (id, ⟨decl?, uses⟩) in vars.toList do + -- process declaration let some decl := decl? | continue let declStx := skipDeclIdIfPresent decl.stx @@ -83,43 +84,63 @@ def unusedVariables : Linter := fun stx => do | continue let some localDecl := decl.info.lctx.find? id | continue - if !stxRange.contains range.start || localDecl.userName.hasMacroScopes then + if !cmdStxRange.contains range.start || localDecl.userName.hasMacroScopes then continue + -- check if variable is used + if !uses.isEmpty || tacticFVarUses.contains id || decl.aliases.any (match · with | .fvar id => tacticFVarUses.contains id | _ => false) then + continue + + -- check linter options let opts := decl.ci.options if !getLinterUnusedVariables opts then continue - let mut ignoredPatternFns := #[ + -- collect ignore functions + let mut ignoreFns := #[ isTopLevelDecl constDecls, matchesUnusedPattern, isVariable, isInStructure, isInInductive, isInCtorOrStructBinder, - isInConstantOrAxiom, + isInOpaqueOrAxiom, isInDefWithForeignDefinition, isInDepArrow ] if !getLinterUnusedVariablesFunArgs opts then - ignoredPatternFns := ignoredPatternFns.append #[ + ignoreFns := ignoreFns.append #[ isInLetDeclaration, isInDeclarationSignature, isInFun ] if !getLinterUnusedVariablesPatternVars opts then - ignoredPatternFns := ignoredPatternFns.append #[ + ignoreFns := ignoreFns.append #[ isPatternVar ] - let some stack := findSyntaxStack? stx declStx - | continue - if ignoredPatternFns.any (· declStx stack) then + -- evaluate ignore functions on original syntax + if let some stack := findSyntaxStack? cmdStx declStx then + if ignoreFns.any (· declStx stack) then + continue + else + continue + + -- evaluate ignore functions on macro expansion outputs + if ← infoTrees.anyM fun tree => do + if let some macroExpansions ← collectMacroExpansions? range tree then + return macroExpansions.any fun expansion => + if let some stack := findSyntaxStack? expansion.output declStx then + ignoreFns.any (· declStx stack) + else + false + else + return false + then continue - if uses.isEmpty && !tacticFVarUses.contains id && - decl.aliases.all (match · with | .fvar id => !tacticFVarUses.contains id | _ => false) then - publishMessage s!"unused variable `{localDecl.userName}`" range + -- publish warning if variable is unused and not ignored + publishMessage s!"unused variable `{localDecl.userName}`" range return () where @@ -149,7 +170,7 @@ where stackMatches stack [`null, none, `null, ``Lean.Parser.Command.optDeclSig, none] && (stack.get? 4 |>.any fun (stx, _) => [``Lean.Parser.Command.ctor, ``Lean.Parser.Command.structSimpleBinder].any (stx.isOfKind ·)) - isInConstantOrAxiom (_ : Syntax) (stack : SyntaxStack) := + isInOpaqueOrAxiom (_ : Syntax) (stack : SyntaxStack) := stackMatches stack [`null, none, `null, ``Lean.Parser.Command.declSig, none] && (stack.get? 4 |>.any fun (stx, _) => [``Lean.Parser.Command.opaque, ``Lean.Parser.Command.axiom].any (stx.isOfKind ·)) diff --git a/stage0/src/Lean/Linter/Util.lean b/stage0/src/Lean/Linter/Util.lean index 9203e86bf05b..90f4ee0fd4bd 100644 --- a/stage0/src/Lean/Linter/Util.lean +++ b/stage0/src/Lean/Linter/Util.lean @@ -20,8 +20,45 @@ do let messages := (← get).messages |>.add (mkMessageCore ctx.fileName ctx.fileMap content severity range.start range.stop) modify ({ · with messages := messages }) +/-- Go upwards through the given `tree` starting from the smallest node that +contains the given `range` and collect all `MacroExpansionInfo`s on the way up. +The result is `some []` if no `MacroExpansionInfo` was found on the way and +`none` if no `InfoTree` node was found that covers the given `range`. + +Return the result reversed, s.t. the macro expansion that would be applied to +the original syntax first is the first element of the returned list. -/ +def collectMacroExpansions? {m} [Monad m] (range : String.Range) (tree : Elab.InfoTree) : m <| Option <| List Elab.MacroExpansionInfo := do + if let .some <| .some result ← go then + return some result.reverse + else + return none +where + go : m <| Option <| Option <| List Elab.MacroExpansionInfo := tree.visitM (postNode := fun _ i _ results => do + let results := results |>.filterMap id |>.filterMap id + + -- we expect that at most one InfoTree child returns a result + if let results :: _ := results then + if let .ofMacroExpansionInfo i := i then + return some <| i :: results + else + return some results + else if i.contains range.start && i.contains (includeStop := true) range.stop then + if let .ofMacroExpansionInfo i := i then + return some [i] + else + return some [] + else + return none) + +/-- List of `Syntax` nodes in which each succeeding element is the parent of +the current. The associated index is the index of the preceding element in the +list of children of the current element. -/ abbrev SyntaxStack := List (Syntax × Nat) +/-- Go upwards through the given `root` syntax starting from `child` and +collect all `Syntax` nodes on the way up. + +Return `none` if the `child` is not found in `root`. -/ partial def findSyntaxStack? (root child : Syntax) : Option SyntaxStack := Id.run <| do let some childRange := child.getRange? | none @@ -40,6 +77,8 @@ partial def findSyntaxStack? (root child : Syntax) : Option SyntaxStack := Id.ru return none go [] root +/-- Compare the `SyntaxNodeKind`s in `pattern` to those of the `Syntax` +elements in `stack`. Return `false` if `stack` is shorter than `pattern`. -/ def stackMatches (stack : SyntaxStack) (pattern : List $ Option SyntaxNodeKind) : Bool := stack.length >= pattern.length && (stack diff --git a/stage0/src/Lean/LocalContext.lean b/stage0/src/Lean/LocalContext.lean index a3290c47df31..f82ffda85a97 100644 --- a/stage0/src/Lean/LocalContext.lean +++ b/stage0/src/Lean/LocalContext.lean @@ -318,6 +318,9 @@ instance : ForIn m LocalContext LocalDecl where @[inline] def foldr (lctx : LocalContext) (f : LocalDecl → β → β) (init : β) : β := Id.run <| lctx.foldrM f init +def size (lctx : LocalContext) : Nat := + lctx.foldl (fun n _ => n+1) 0 + @[inline] def findDecl? (lctx : LocalContext) (f : LocalDecl → Option β) : Option β := Id.run <| lctx.findDeclM? f diff --git a/stage0/src/Lean/Meta/AppBuilder.lean b/stage0/src/Lean/Meta/AppBuilder.lean index 2a1f646027f9..450108cab796 100644 --- a/stage0/src/Lean/Meta/AppBuilder.lean +++ b/stage0/src/Lean/Meta/AppBuilder.lean @@ -24,11 +24,13 @@ def mkExpectedTypeHint (e : Expr) (expectedType : Expr) : MetaM Expr := do let u ← getLevel expectedType return mkApp2 (mkConst ``id [u]) expectedType e +/-- Return `a = b`. -/ def mkEq (a b : Expr) : MetaM Expr := do let aType ← inferType a let u ← getLevel aType return mkApp3 (mkConst ``Eq [u]) aType a b +/-- Return `HEq a b`. -/ def mkHEq (a b : Expr) : MetaM Expr := do let aType ← inferType a let bType ← inferType b @@ -47,21 +49,25 @@ def mkEqHEq (a b : Expr) : MetaM Expr := do else return mkApp4 (mkConst ``HEq [u]) aType a bType b +/-- Return a proof of `a = a`. -/ def mkEqRefl (a : Expr) : MetaM Expr := do let aType ← inferType a let u ← getLevel aType return mkApp2 (mkConst ``Eq.refl [u]) aType a +/-- Return a proof of `HEq a a`. -/ def mkHEqRefl (a : Expr) : MetaM Expr := do let aType ← inferType a let u ← getLevel aType return mkApp2 (mkConst ``HEq.refl [u]) aType a +/-- Given `hp : P` and `nhp : Not P` returns an instance of type `e`. -/ def mkAbsurd (e : Expr) (hp hnp : Expr) : MetaM Expr := do let p ← inferType hp let u ← getLevel e return mkApp4 (mkConst ``absurd [u]) p e hp hnp +/-- Given `h : False`, return an instance of type `e`. -/ def mkFalseElim (e : Expr) (h : Expr) : MetaM Expr := do let u ← getLevel e return mkApp2 (mkConst ``False.elim [u]) e h @@ -76,6 +82,7 @@ private def hasTypeMsg (e type : Expr) : MessageData := private def throwAppBuilderException {α} (op : Name) (msg : MessageData) : MetaM α := throwError "AppBuilder for '{op}', {msg}" +/-- Given `h : a = b`, returns a proof of `b = a`. -/ def mkEqSymm (h : Expr) : MetaM Expr := do if h.isAppOf ``Eq.refl then return h @@ -87,6 +94,7 @@ def mkEqSymm (h : Expr) : MetaM Expr := do return mkApp4 (mkConst ``Eq.symm [u]) α a b h | none => throwAppBuilderException ``Eq.symm ("equality proof expected" ++ hasTypeMsg h hType) +/-- Given `h₁ : a = b` and `h₂ : b = c` returns a proof of `a = c`. -/ def mkEqTrans (h₁ h₂ : Expr) : MetaM Expr := do if h₁.isAppOf ``Eq.refl then return h₂ @@ -102,6 +110,7 @@ def mkEqTrans (h₁ h₂ : Expr) : MetaM Expr := do | none, _ => throwAppBuilderException ``Eq.trans ("equality proof expected" ++ hasTypeMsg h₁ hType₁) | _, none => throwAppBuilderException ``Eq.trans ("equality proof expected" ++ hasTypeMsg h₂ hType₂) +/-- Given `h : HEq a b`, returns a proof of `HEq b a`. -/ def mkHEqSymm (h : Expr) : MetaM Expr := do if h.isAppOf ``HEq.refl then return h @@ -114,6 +123,7 @@ def mkHEqSymm (h : Expr) : MetaM Expr := do | none => throwAppBuilderException ``HEq.symm ("heterogeneous equality proof expected" ++ hasTypeMsg h hType) +/-- Given `h₁ : HEq a b`, `h₂ : HEq b c`, returns a proof of `HEq a c`. -/ def mkHEqTrans (h₁ h₂ : Expr) : MetaM Expr := do if h₁.isAppOf ``HEq.refl then return h₂ @@ -129,6 +139,7 @@ def mkHEqTrans (h₁ h₂ : Expr) : MetaM Expr := do | none, _ => throwAppBuilderException ``HEq.trans ("heterogeneous equality proof expected" ++ hasTypeMsg h₁ hType₁) | _, none => throwAppBuilderException ``HEq.trans ("heterogeneous equality proof expected" ++ hasTypeMsg h₂ hType₂) +/-- Given `h : Eq a b`, returns a proof of `HEq a b`. -/ def mkEqOfHEq (h : Expr) : MetaM Expr := do let hType ← infer h match hType.heq? with @@ -140,6 +151,7 @@ def mkEqOfHEq (h : Expr) : MetaM Expr := do | _ => throwAppBuilderException ``HEq.trans m!"heterogeneous equality proof expected{indentExpr h}" +/-- Given `f : α → β` and `h : a = b`, returns a proof of `f a = f b`.-/ def mkCongrArg (f h : Expr) : MetaM Expr := do if h.isAppOf ``Eq.refl then mkEqRefl (mkApp f h.appArg!) @@ -154,6 +166,7 @@ def mkCongrArg (f h : Expr) : MetaM Expr := do | none, _ => throwAppBuilderException ``congrArg ("non-dependent function expected" ++ hasTypeMsg f fType) | _, none => throwAppBuilderException ``congrArg ("equality proof expected" ++ hasTypeMsg h hType) +/-- Given `h : f = g` and `a : α`, returns a proof of `f a = g a`.-/ def mkCongrFun (h a : Expr) : MetaM Expr := do if h.isAppOf ``Eq.refl then mkEqRefl (mkApp h.appArg! a) @@ -171,6 +184,7 @@ def mkCongrFun (h a : Expr) : MetaM Expr := do | _ => throwAppBuilderException ``congrFun ("equality proof between functions expected" ++ hasTypeMsg h hType) | _ => throwAppBuilderException ``congrFun ("equality proof expected" ++ hasTypeMsg h hType) +/-- Given `h₁ : f = g` and `h₂ : a = b`, returns a proof of `f a = g b`. -/ def mkCongr (h₁ h₂ : Expr) : MetaM Expr := do if h₁.isAppOf ``Eq.refl then mkCongrArg h₁.appArg! h₂ @@ -369,6 +383,7 @@ def mkNoConfusion (target : Expr) (h : Expr) : MetaM Expr := do let u ← getLevel target return mkAppN (mkConst (Name.mkStr v.name "noConfusion") (u :: us)) (α.getAppArgs ++ #[target, a, b, h]) +/-- Given a `monad` and `e : α`, makes `pure e`.-/ def mkPure (monad : Expr) (e : Expr) : MetaM Expr := mkAppOptM ``Pure.pure #[monad, none, none, e] diff --git a/stage0/src/Lean/Meta/Basic.lean b/stage0/src/Lean/Meta/Basic.lean index 65f195760507..48a6a0daadf6 100644 --- a/stage0/src/Lean/Meta/Basic.lean +++ b/stage0/src/Lean/Meta/Basic.lean @@ -34,31 +34,31 @@ namespace Lean.Meta builtin_initialize isDefEqStuckExceptionId : InternalExceptionId ← registerInternalExceptionId `isDefEqStuck /-- - Configuration flags for the `MetaM` monad. - Many of them are used to control the `isDefEq` function that checks whether two terms are definitionally equal or not. - Recall that when `isDefEq` is trying to check whether - `?m@C a₁ ... aₙ` and `t` are definitionally equal (`?m@C a₁ ... aₙ =?= t`), where - `?m@C` as a shorthand for `C |- ?m : t` where `t` is the type of `?m`. - We solve it using the assignment `?m := fun a₁ ... aₙ => t` if - 1) `a₁ ... aₙ` are pairwise distinct free variables that are ​*not*​ let-variables. - 2) `a₁ ... aₙ` are not in `C` - 3) `t` only contains free variables in `C` and/or `{a₁, ..., aₙ}` - 4) For every metavariable `?m'@C'` occurring in `t`, `C'` is a subprefix of `C` - 5) `?m` does not occur in `t` +Configuration flags for the `MetaM` monad. +Many of them are used to control the `isDefEq` function that checks whether two terms are definitionally equal or not. +Recall that when `isDefEq` is trying to check whether +`?m@C a₁ ... aₙ` and `t` are definitionally equal (`?m@C a₁ ... aₙ =?= t`), where +`?m@C` as a shorthand for `C |- ?m : t` where `t` is the type of `?m`. +We solve it using the assignment `?m := fun a₁ ... aₙ => t` if +1) `a₁ ... aₙ` are pairwise distinct free variables that are ​*not*​ let-variables. +2) `a₁ ... aₙ` are not in `C` +3) `t` only contains free variables in `C` and/or `{a₁, ..., aₙ}` +4) For every metavariable `?m'@C'` occurring in `t`, `C'` is a subprefix of `C` +5) `?m` does not occur in `t` -/ structure Config where /-- If `foApprox` is set to true, and some `aᵢ` is not a free variable, - then we use first-order unification - ``` - ?m a_1 ... a_i a_{i+1} ... a_{i+k} =?= f b_1 ... b_k - ``` - reduces to - ``` - ?m a_1 ... a_i =?= f - a_{i+1} =?= b_1 - ... - a_{i+k} =?= b_k + then we use first-order unification + ``` + ?m a_1 ... a_i a_{i+1} ... a_{i+k} =?= f b_1 ... b_k + ``` + reduces to + ``` + ?m a_1 ... a_i =?= f + a_{i+1} =?= b_1 + ... + a_{i+k} =?= b_k ``` -/ foApprox : Bool := false @@ -136,6 +136,34 @@ structure ParamInfo where This information affects the generation of congruence theorems. -/ isDecInst : Bool := false + /-- + `higherOrderOutParam` is true if this parameter is a higher-order output parameter + of local instance. + Example: + ``` + getElem : + {Cont : Type u_1} → {Idx : Type u_2} → {Elem : Type u_3} → + {Dom : Cont → Idx → Prop} → [self : GetElem Cont Idx Elem Dom] → + (xs : Cont) → (i : Idx) → Dom xs i → Elem + ``` + This flag is true for the parameter `Dom` because it is output parameter of + `[self : GetElem Cont Idx Elem Dom]` + -/ + higherOrderOutParam : Bool := false + /-- + `dependsOnHigherOrderOutParam` is true if the type of this parameter depends on + the higher-order output parameter of a previous local instance. + Example: + ``` + getElem : + {Cont : Type u_1} → {Idx : Type u_2} → {Elem : Type u_3} → + {Dom : Cont → Idx → Prop} → [self : GetElem Cont Idx Elem Dom] → + (xs : Cont) → (i : Idx) → Dom xs i → Elem + ``` + This flag is true for the parameter with type `Dom xs i` since `Dom` is an output parameter + of the instance `[self : GetElem Cont Idx Elem Dom]` + -/ + dependsOnHigherOrderOutParam : Bool := false deriving Inhabited def ParamInfo.isImplicit (p : ParamInfo) : Bool := diff --git a/stage0/src/Lean/Meta/ExprDefEq.lean b/stage0/src/Lean/Meta/ExprDefEq.lean index eb4c2c71955a..47bb528b0655 100644 --- a/stage0/src/Lean/Meta/ExprDefEq.lean +++ b/stage0/src/Lean/Meta/ExprDefEq.lean @@ -133,7 +133,51 @@ def isEtaUnassignedMVar (e : Expr) : MetaM Bool := do pure true | _ => pure false -/- +private def trySynthPending (e : Expr) : MetaM Bool := do + let mvarId? ← getStuckMVar? e + match mvarId? with + | some mvarId => Meta.synthPending mvarId + | none => pure false + +/-- + Result type for `isDefEqArgsFirstPass`. +-/ +inductive DefEqArgsFirstPassResult where + | /-- + Failed to establish that explicit arguments are def-eq. + Remark: higher output parameters, and parameters that depend on them + are postponed. + -/ + failed + | /-- + Succeeded. The array `postponedImplicit` contains the position + of the implicit arguments for which def-eq has been postponed. + `postponedHO` contains the higher order output parameters, and parameters + that depend on them. They should be processed after the implict ones. + `postponedHO` is used to handle applications involving functions that + contain higher order output parameters. Example: + ```lean + getElem : + {Cont : Type u_1} → {Idx : Type u_2} → {Elem : Type u_3} → + {Dom : Cont → Idx → Prop} → [self : GetElem Cont Idx Elem Dom] → + (xs : Cont) → (i : Idx) → (h : Dom xs i) → Elem + ``` + The argumengs `Dom` and `h` must be processed after all implicit arguments + otherwise higher-order unification problems are generated. See issue #1299, + when trying to solve + ``` + getElem ?a ?i ?h =?= getElem a i (Fin.val_lt_of_le i ...) + ``` + we have to solve the constraint + ``` + ?Dom a i.val =?= LT.lt i.val (Array.size a) + ``` + by solving after the instance has been synthesized, we reduce this constraint to + a simple check. + -/ + ok (postponedImplicit : Array Nat) (postponedHO : Array Nat) + +/-- First pass for `isDefEqArgs`. We unify explicit arguments, *and* easy cases Here, we say a case is easy if it is of the form @@ -161,66 +205,61 @@ def isEtaUnassignedMVar (e : Expr) : MetaM Bool := do introduce counter intuitive behavior. Pre: `paramInfo.size <= args₁.size = args₂.size` + + See `DefEqArgsFirstPassResult` for additional information. -/ -private partial def isDefEqArgsFirstPass - (paramInfo : Array ParamInfo) (args₁ args₂ : Array Expr) : MetaM (Option (Array Nat)) := do - let rec loop (i : Nat) (postponed : Array Nat) := do - if h : i < paramInfo.size then - let info := paramInfo.get ⟨i, h⟩ - let a₁ := args₁[i]! - let a₂ := args₂[i]! - if !info.isExplicit then - if (← isEtaUnassignedMVar a₁ <||> isEtaUnassignedMVar a₂) then - if (← Meta.isExprDefEqAux a₁ a₂) then - loop (i+1) postponed - else - pure none - else - loop (i+1) (postponed.push i) - else if (← Meta.isExprDefEqAux a₁ a₂) then - loop (i+1) postponed - else - pure none +private def isDefEqArgsFirstPass + (paramInfo : Array ParamInfo) (args₁ args₂ : Array Expr) : MetaM DefEqArgsFirstPassResult := do + let mut postponedImplicit := #[] + let mut postponedHO := #[] + for i in [:paramInfo.size] do + let info := paramInfo[i]! + let a₁ := args₁[i]! + let a₂ := args₂[i]! + if info.dependsOnHigherOrderOutParam || info.higherOrderOutParam then + trace[Meta.isDefEq] "found messy {a₁} =?= {a₂}" + postponedHO := postponedHO.push i + else if info.isExplicit then + unless (← Meta.isExprDefEqAux a₁ a₂) do + return .failed + else if (← isEtaUnassignedMVar a₁ <||> isEtaUnassignedMVar a₂) then + unless (← Meta.isExprDefEqAux a₁ a₂) do + return .failed else - pure (some postponed) - loop 0 #[] - -private def trySynthPending (e : Expr) : MetaM Bool := do - let mvarId? ← getStuckMVar? e - match mvarId? with - | some mvarId => Meta.synthPending mvarId - | none => pure false - -private partial def isDefEqArgs (f : Expr) (args₁ args₂ : Array Expr) : MetaM Bool := - if h : args₁.size = args₂.size then do - let finfo ← getFunInfoNArgs f args₁.size - let (some postponed) ← isDefEqArgsFirstPass finfo.paramInfo args₁ args₂ | pure false - let rec processOtherArgs (i : Nat) : MetaM Bool := do - if h₁ : i < args₁.size then - let a₁ := args₁.get ⟨i, h₁⟩ - let a₂ := args₂.get ⟨i, Eq.subst h h₁⟩ - if (← Meta.isExprDefEqAux a₁ a₂) then - processOtherArgs (i+1) - else - pure false - else - pure true - if (← processOtherArgs finfo.paramInfo.size) then - postponed.allM fun i => do - /- Second pass: unify implicit arguments. - In the second pass, we make sure we are unfolding at - least non reducible definitions (default setting). -/ - let a₁ := args₁[i]! - let a₂ := args₂[i]! - let info := finfo.paramInfo[i]! - if info.isInstImplicit then - discard <| trySynthPending a₁ - discard <| trySynthPending a₂ - withAtLeastTransparency TransparencyMode.default <| Meta.isExprDefEqAux a₁ a₂ + postponedImplicit := postponedImplicit.push i + return .ok postponedImplicit postponedHO + +private partial def isDefEqArgs (f : Expr) (args₁ args₂ : Array Expr) : MetaM Bool := do + unless args₁.size == args₂.size do return false + let finfo ← getFunInfoNArgs f args₁.size + let .ok postponedImplicit postponedHO ← isDefEqArgsFirstPass finfo.paramInfo args₁ args₂ | pure false + -- finfo.paramInfo.size may be smaller than args₁.size + for i in [finfo.paramInfo.size:args₁.size] do + unless (← Meta.isExprDefEqAux args₁[i]! args₂[i]!) do + return false + for i in postponedImplicit do + /- Second pass: unify implicit arguments. + In the second pass, we make sure we are unfolding at + least non reducible definitions (default setting). -/ + let a₁ := args₁[i]! + let a₂ := args₂[i]! + let info := finfo.paramInfo[i]! + if info.isInstImplicit then + discard <| trySynthPending a₁ + discard <| trySynthPending a₂ + unless (← withAtLeastTransparency TransparencyMode.default <| Meta.isExprDefEqAux a₁ a₂) do + return false + for i in postponedHO do + let a₁ := args₁[i]! + let a₂ := args₂[i]! + let info := finfo.paramInfo[i]! + if info.isInstImplicit then + unless (← withAtLeastTransparency TransparencyMode.default <| Meta.isExprDefEqAux a₁ a₂) do + return false else - pure false - else - pure false + unless (← Meta.isExprDefEqAux a₁ a₂) do + return false + return true /-- Check whether the types of the free variables at `fvars` are @@ -851,12 +890,13 @@ def checkAssignment (mvarId : MVarId) (fvars : Array Expr) (v : Expr) : MetaM (O private def processAssignmentFOApproxAux (mvar : Expr) (args : Array Expr) (v : Expr) : MetaM Bool := match v with + | .mdata _ e => processAssignmentFOApproxAux mvar args e | Expr.app f a => if args.isEmpty then pure false else Meta.isExprDefEqAux args.back a <&&> Meta.isExprDefEqAux (mkAppRange mvar 0 (args.size - 1) args) f - | _ => pure false + | _ => pure false /- Auxiliary method for applying first-order unification. It is an approximation. @@ -1294,15 +1334,6 @@ private def expandDelayedAssigned? (t : Expr) : MetaM (Option Expr) := do if tArgs.size < fvars.size then return none return some (mkAppRange (mkMVar mvarIdPending) fvars.size tArgs.size tArgs) -private def isSynthetic : Expr → MetaM Bool - | Expr.mvar mvarId => do - let mvarDecl ← getMVarDecl mvarId - match mvarDecl.kind with - | MetavarKind.synthetic => pure true - | MetavarKind.syntheticOpaque => pure true - | MetavarKind.natural => pure false - | _ => pure false - private def isAssignable : Expr → MetaM Bool | Expr.mvar mvarId => do let b ← isReadOnlyOrSyntheticOpaqueExprMVar mvarId; pure (!b) | _ => pure false diff --git a/stage0/src/Lean/Meta/FunInfo.lean b/stage0/src/Lean/Meta/FunInfo.lean index e1a37d3b5405..9194fa7bd53f 100644 --- a/stage0/src/Lean/Meta/FunInfo.lean +++ b/stage0/src/Lean/Meta/FunInfo.lean @@ -9,9 +9,8 @@ import Lean.Meta.InferType namespace Lean.Meta @[inline] private def checkFunInfoCache (fn : Expr) (maxArgs? : Option Nat) (k : MetaM FunInfo) : MetaM FunInfo := do - let s ← get let t ← getTransparency - match s.cache.funInfo.find? ⟨t, fn, maxArgs?⟩ with + match (← get).cache.funInfo.find? ⟨t, fn, maxArgs?⟩ with | some finfo => pure finfo | none => do let finfo ← k @@ -57,21 +56,38 @@ private def getFunInfoAux (fn : Expr) (maxArgs? : Option Nat) : MetaM FunInfo := let fnType ← inferType fn withTransparency TransparencyMode.default do forallBoundedTelescope fnType maxArgs? fun fvars type => do - let mut pinfo := #[] + let mut paramInfo := #[] + let mut higherOrderOutParams : FVarIdSet := {} for i in [:fvars.size] do let fvar := fvars[i]! let decl ← getFVarLocalDecl fvar let backDeps := collectDeps fvars decl.type - pinfo := updateHasFwdDeps pinfo backDeps - pinfo := pinfo.push { - backDeps := backDeps - binderInfo := decl.binderInfo - isProp := (← isProp decl.type) - isDecInst := (← forallTelescopeReducing decl.type fun _ type => return type.isAppOf ``Decidable) + let dependsOnHigherOrderOutParam := + !higherOrderOutParams.isEmpty + && Option.isSome (decl.type.find? fun e => e.isFVar && higherOrderOutParams.contains e.fvarId!) + paramInfo := updateHasFwdDeps paramInfo backDeps + paramInfo := paramInfo.push { + backDeps, dependsOnHigherOrderOutParam + binderInfo := decl.binderInfo + isProp := (← isProp decl.type) + isDecInst := (← forallTelescopeReducing decl.type fun _ type => return type.isAppOf ``Decidable) } + if decl.binderInfo == .instImplicit then + /- Collect higher order output parameters of this class -/ + if let some className ← isClass? decl.type then + if let some outParamPositions := getOutParamPositions? (← getEnv) className then + unless outParamPositions.isEmpty do + let args := decl.type.getAppArgs + for i in [:args.size] do + if outParamPositions.contains i then + let arg := args[i]! + if let some idx := fvars.indexOf? arg then + if (← whnf (← inferType arg)).isForall then + paramInfo := paramInfo.modify idx fun info => { info with higherOrderOutParam := true } + higherOrderOutParams := higherOrderOutParams.insert arg.fvarId! let resultDeps := collectDeps fvars type - pinfo := updateHasFwdDeps pinfo resultDeps - pure { resultDeps := resultDeps, paramInfo := pinfo } + paramInfo := updateHasFwdDeps paramInfo resultDeps + return { resultDeps, paramInfo } def getFunInfo (fn : Expr) : MetaM FunInfo := getFunInfoAux fn none diff --git a/stage0/src/Lean/Meta/Match/Match.lean b/stage0/src/Lean/Meta/Match/Match.lean index b2ba02d2c82d..c3f9aa937848 100644 --- a/stage0/src/Lean/Meta/Match/Match.lean +++ b/stage0/src/Lean/Meta/Match/Match.lean @@ -188,18 +188,18 @@ private def processAsPattern (p : Problem) : MetaM Problem := match alt.patterns with | Pattern.as fvarId p h :: ps => /- We used to use `checkAndReplaceFVarId` here, but `x` and `fvarId` may have different types - when dependent types are beind used. Let's consider the repro for issue #471 - ``` - inductive vec : Nat → Type - | nil : vec 0 - | cons : Int → vec n → vec n.succ - - def vec_len : vec n → Nat - | vec.nil => 0 - | x@(vec.cons h t) => vec_len t + 1 - - ``` - we reach the state + when dependent types are beind used. Let's consider the repro for issue #471 + ``` + inductive vec : Nat → Type + | nil : vec 0 + | cons : Int → vec n → vec n.succ + + def vec_len : vec n → Nat + | vec.nil => 0 + | x@(vec.cons h t) => vec_len t + 1 + + ``` + we reach the state ``` [Meta.Match.match] remaining variables: [x✝:(vec n✝)] alternatives: @@ -297,7 +297,7 @@ def assign (fvarId : FVarId) (v : Expr) : M Bool := do The first step is a variable-transition which replaces `β` with `β✝` in the first and third alternatives. The constraint `β✝ === α` in the second alternative is lost. Note that `α` is not an alternative variable. After applying the variable-transition step twice, we reach the following state - ``lean + ```lean [Meta.Match.match] remaining variables: [f✝:(Arrow β✝ γ✝), g✝:(Arrow α β✝)] alternatives: [g:(Arrow α β✝)] |- [(Arrow.id .(β✝)), g] => h_1 β✝ g diff --git a/stage0/src/Lean/Meta/MatchUtil.lean b/stage0/src/Lean/Meta/MatchUtil.lean index e8dcb817fdbb..06d1a924c49e 100644 --- a/stage0/src/Lean/Meta/MatchUtil.lean +++ b/stage0/src/Lean/Meta/MatchUtil.lean @@ -19,6 +19,7 @@ namespace Lean.Meta | none => p? (← whnf e) | s => return s +/-- Matches `e` with `lhs = (rhs : α)` and returns `(α, lhs, rhs)`. -/ def matchEq? (e : Expr) : MetaM (Option (Expr × Expr × Expr)) := matchHelper? e fun e => return Expr.eq? e diff --git a/stage0/src/Lean/Meta/Tactic/Constructor.lean b/stage0/src/Lean/Meta/Tactic/Constructor.lean index 29b6132866c8..93ab1236602e 100644 --- a/stage0/src/Lean/Meta/Tactic/Constructor.lean +++ b/stage0/src/Lean/Meta/Tactic/Constructor.lean @@ -9,7 +9,11 @@ import Lean.Meta.Tactic.Apply namespace Lean.Meta -def constructor (mvarId : MVarId) : MetaM (List MVarId) := do +/-- +When the goal `mvarId` is an inductive datatype, +`constructor` calls `apply` with the first matching constructor. +-/ +def constructor (mvarId : MVarId) (cfg : ApplyConfig := {}) : MetaM (List MVarId) := do withMVarContext mvarId do checkNotAssigned mvarId `constructor let target ← getMVarType' mvarId @@ -18,7 +22,7 @@ def constructor (mvarId : MVarId) : MetaM (List MVarId) := do fun ival us => do for ctor in ival.ctors do try - return ← apply mvarId (Lean.mkConst ctor us) + return ← apply mvarId (Lean.mkConst ctor us) cfg catch _ => pure () throwTacticEx `constructor mvarId "no applicable constructor found" diff --git a/stage0/src/Lean/Meta/Tactic/Intro.lean b/stage0/src/Lean/Meta/Tactic/Intro.lean index 1ebbee1c9f51..43c9e1cd4f9b 100644 --- a/stage0/src/Lean/Meta/Tactic/Intro.lean +++ b/stage0/src/Lean/Meta/Tactic/Intro.lean @@ -53,7 +53,7 @@ namespace Lean.Meta `whnf` instantiates metavariables, and consumes `MData`, but it also expands the `let`. -/ - let newType := (← instantiateMVars type).consumeMDataAndTypeAnnotations + let newType := (← instantiateMVars type).cleanupAnnotations if newType.isForall || newType.isLet then loop (i+1) lctx fvars fvars.size s newType else diff --git a/stage0/src/Lean/Meta/WHNF.lean b/stage0/src/Lean/Meta/WHNF.lean index cdeb894d3c4f..273c5ed7e883 100644 --- a/stage0/src/Lean/Meta/WHNF.lean +++ b/stage0/src/Lean/Meta/WHNF.lean @@ -254,24 +254,23 @@ mutual /-- Return `some (Expr.mvar mvarId)` if metavariable `mvarId` is blocking reduction. -/ partial def getStuckMVar? (e : Expr) : MetaM (Option MVarId) := do match e with - | Expr.mdata _ e => getStuckMVar? e - | Expr.proj _ _ e => getStuckMVar? (← whnf e) - | Expr.mvar .. => do + | .mdata _ e => getStuckMVar? e + | .proj _ _ e => getStuckMVar? (← whnf e) + | .mvar .. => do let e ← instantiateMVars e match e with | Expr.mvar mvarId => pure (some mvarId) | _ => getStuckMVar? e - | Expr.app f .. => + | .app f .. => let f := f.getAppFn match f with - | Expr.mvar mvarId => return some mvarId - | Expr.const fName _ => - let cinfo? ← getConstNoEx? fName - match cinfo? with - | some $ ConstantInfo.recInfo recVal => isRecStuck? recVal e.getAppArgs - | some $ ConstantInfo.quotInfo recVal => isQuotRecStuck? recVal e.getAppArgs - | _ => return none - | Expr.proj _ _ e => getStuckMVar? (← whnf e) + | .mvar mvarId => return some mvarId + | .const fName _ => + match (← getConstNoEx? fName) with + | some <| .recInfo recVal => isRecStuck? recVal e.getAppArgs + | some <| .quotInfo recVal => isQuotRecStuck? recVal e.getAppArgs + | _ => return none + | .proj _ _ e => getStuckMVar? (← whnf e) | _ => return none | _ => return none end diff --git a/stage0/src/Lean/MetavarContext.lean b/stage0/src/Lean/MetavarContext.lean index d32ea9e63310..cd76382a576b 100644 --- a/stage0/src/Lean/MetavarContext.lean +++ b/stage0/src/Lean/MetavarContext.lean @@ -420,6 +420,12 @@ def hasAssignableMVar [Monad m] [MonadMCtx m] : Expr → m Bool def assignLevelMVar [MonadMCtx m] (mvarId : MVarId) (val : Level) : m Unit := modifyMCtx fun m => { m with lAssignment := m.lAssignment.insert mvarId val, usedAssignment := true } +/-- +Add `mvarId := x` to the metavariable assignment. +This method does not check whether `mvarId` is already assigned, nor it checks whether +a cycle is being introduced, or whether the expression has the right type. +This is a low-level API, and it is safer to use `isDefEq (mkMVar mvarId) x`. +-/ def assignExprMVar [MonadMCtx m] (mvarId : MVarId) (val : Expr) : m Unit := modifyMCtx fun m => { m with eAssignment := m.eAssignment.insert mvarId val, usedAssignment := true } diff --git a/stage0/src/Lean/Parser/Command.lean b/stage0/src/Lean/Parser/Command.lean index be0f7bcc2fb2..54c4bb73d72d 100644 --- a/stage0/src/Lean/Parser/Command.lean +++ b/stage0/src/Lean/Parser/Command.lean @@ -132,8 +132,8 @@ def openDecl := openHiding <|> openRenaming <|> openOnly <|> openSimple @[builtinCommandParser] def «open» := leading_parser withPosition ("open " >> openDecl) @[builtinCommandParser] def «mutual» := leading_parser "mutual " >> many1 (ppLine >> notSymbol "end" >> commandParser) >> ppDedent (ppLine >> "end") >> terminationSuffix -@[builtinCommandParser] def «initialize» := leading_parser optional visibility >> "initialize " >> optional (atomic (ident >> Term.typeSpec >> Term.leftArrow)) >> Term.doSeq -@[builtinCommandParser] def «builtin_initialize» := leading_parser optional visibility >> "builtin_initialize " >> optional (atomic (ident >> Term.typeSpec >> Term.leftArrow)) >> Term.doSeq +def initializeKeyword := leading_parser "initialize " <|> "builtin_initialize " +@[builtinCommandParser] def «initialize» := leading_parser declModifiers false >> initializeKeyword >> optional (atomic (ident >> Term.typeSpec >> Term.leftArrow)) >> Term.doSeq @[builtinCommandParser] def «in» := trailing_parser withOpen (" in " >> commandParser) @@ -153,6 +153,7 @@ builtin_initialize register_parser_alias declVal register_parser_alias optDeclSig register_parser_alias openDecl + register_parser_alias docComment end Command diff --git a/stage0/src/Lean/Parser/Extension.lean b/stage0/src/Lean/Parser/Extension.lean index 9daeccd190d6..3edef816d1c4 100644 --- a/stage0/src/Lean/Parser/Extension.lean +++ b/stage0/src/Lean/Parser/Extension.lean @@ -358,7 +358,10 @@ def leadingIdentBehavior (env : Environment) (catName : Name) : LeadingIdentBeha unsafe def evalParserConstUnsafe (declName : Name) : ParserFn := fun ctx s => unsafeBaseIO do let categories := (parserExtension.getState ctx.env).categories match (← (mkParserOfConstant categories declName { env := ctx.env, opts := ctx.options }).toBaseIO) with - | .ok (_, p) => return p.fn ctx s + | .ok (_, p) => + -- We should manually register `p`'s tokens before invoking it as it might not be part of any syntax category (yet) + let ctx := { ctx with tokens := p.info.collectTokens [] |>.foldl (fun tks tk => tks.insert tk tk) ctx.tokens } + return p.fn ctx s | .error e => return s.mkUnexpectedError e.toString @[implementedBy evalParserConstUnsafe] diff --git a/stage0/src/Lean/Parser/Syntax.lean b/stage0/src/Lean/Parser/Syntax.lean index 1c44599a65bc..9eaddf7db810 100644 --- a/stage0/src/Lean/Parser/Syntax.lean +++ b/stage0/src/Lean/Parser/Syntax.lean @@ -69,7 +69,7 @@ def optKind : Parser := optional ("(" >> nonReservedSymbol "kind" >> ":=" >> ide def notationItem := ppSpace >> withAntiquot (mkAntiquot "notationItem" `Lean.Parser.Command.notationItem) (strLit <|> identPrec) @[builtinCommandParser] def «notation» := leading_parser Term.attrKind >> "notation" >> optPrecedence >> optNamedName >> optNamedPrio >> many notationItem >> darrow >> termParser @[builtinCommandParser] def «macro_rules» := suppressInsideQuot (leading_parser optional docComment >> Term.attrKind >> "macro_rules" >> optKind >> Term.matchAlts) -@[builtinCommandParser] def «syntax» := leading_parser optional docComment >> Term.attrKind >> "syntax " >> optPrecedence >> optNamedName >> optNamedPrio >> many1 (syntaxParser argPrec) >> " : " >> ident +@[builtinCommandParser] def «syntax» := leading_parser optional docComment >> optional (Term.«attributes») >> Term.attrKind >> "syntax " >> optPrecedence >> optNamedName >> optNamedPrio >> many1 (syntaxParser argPrec) >> " : " >> ident @[builtinCommandParser] def syntaxAbbrev := leading_parser optional docComment >> "syntax " >> ident >> " := " >> many1 syntaxParser def catBehaviorBoth := leading_parser nonReservedSymbol "both" def catBehaviorSymbol := leading_parser nonReservedSymbol "symbol" diff --git a/stage0/src/Lean/PrettyPrinter.lean b/stage0/src/Lean/PrettyPrinter.lean index 297dc796a8a3..808532b07a92 100644 --- a/stage0/src/Lean/PrettyPrinter.lean +++ b/stage0/src/Lean/PrettyPrinter.lean @@ -20,10 +20,12 @@ def PPContext.runMetaM {α : Type} (ppCtx : PPContext) (x : MetaM α) : IO α := namespace PrettyPrinter -def ppTerm (stx : Term) : CoreM Format := do +def ppCategory (cat : Name) (stx : Syntax) : CoreM Format := do let opts ← getOptions let stx := (sanitizeSyntax stx).run' { options := opts } - parenthesizeTerm stx >>= formatTerm + parenthesizeCategory cat stx >>= formatCategory cat + +def ppTerm (stx : Term) : CoreM Format := ppCategory `term stx def ppUsing (e : Expr) (delab : Expr → MetaM Term) : MetaM Format := do let lctx := (← getLCtx).sanitizeNames.run' { options := (← getOptions) } @@ -50,11 +52,9 @@ def ppConst (e : Expr) : MetaM Format := do def ppExprLegacy (env : Environment) (mctx : MetavarContext) (lctx : LocalContext) (opts : Options) (e : Expr) : IO Format := Prod.fst <$> ((ppExpr e).run' { lctx := lctx } { mctx := mctx }).toIO { options := opts, fileName := "", fileMap := default } { env := env } -def ppTactic (stx : TSyntax `tactic) : CoreM Format := - parenthesizeTactic stx >>= formatTactic +def ppTactic (stx : TSyntax `tactic) : CoreM Format := ppCategory `tactic stx -def ppCommand (stx : Syntax.Command) : CoreM Format := - parenthesizeCommand stx >>= formatCommand +def ppCommand (stx : Syntax.Command) : CoreM Format := ppCategory `command stx def ppModule (stx : TSyntax ``Parser.Module.module) : CoreM Format := do parenthesize Lean.Parser.Module.module.parenthesizer stx >>= format Lean.Parser.Module.module.formatter diff --git a/stage0/src/Lean/PrettyPrinter/Formatter.lean b/stage0/src/Lean/PrettyPrinter/Formatter.lean index eaff61d972b6..50c1757f0c7d 100644 --- a/stage0/src/Lean/PrettyPrinter/Formatter.lean +++ b/stage0/src/Lean/PrettyPrinter/Formatter.lean @@ -530,7 +530,7 @@ def format (formatter : Formatter) (stx : Syntax) : CoreM Format := do pure $ Format.fill $ st.stack.get! 0) (fun _ => throwError "format: uncaught backtrack exception") -def formatCategory (cat : Name) := format $ categoryFormatter cat +def formatCategory (cat : Name) := format <| categoryFormatter cat def formatTerm := formatCategory `term def formatTactic := formatCategory `tactic diff --git a/stage0/src/Lean/PrettyPrinter/Parenthesizer.lean b/stage0/src/Lean/PrettyPrinter/Parenthesizer.lean index 15066a22056b..f40e94208ed4 100644 --- a/stage0/src/Lean/PrettyPrinter/Parenthesizer.lean +++ b/stage0/src/Lean/PrettyPrinter/Parenthesizer.lean @@ -533,9 +533,11 @@ def parenthesize (parenthesizer : Parenthesizer) (stx : Syntax) : CoreM Syntax : pure st.stxTrav.cur) (fun _ => throwError "parenthesize: uncaught backtrack exception") -def parenthesizeTerm := parenthesize $ categoryParser.parenthesizer `term 0 -def parenthesizeTactic := parenthesize $ categoryParser.parenthesizer `tactic 0 -def parenthesizeCommand := parenthesize $ categoryParser.parenthesizer `command 0 +def parenthesizeCategory (cat : Name) := parenthesize <| categoryParser.parenthesizer cat 0 + +def parenthesizeTerm := parenthesizeCategory `term +def parenthesizeTactic := parenthesizeCategory `tactic +def parenthesizeCommand := parenthesizeCategory `command builtin_initialize registerTraceClass `PrettyPrinter.parenthesize diff --git a/stage0/src/Lean/Server/FileWorker/RequestHandling.lean b/stage0/src/Lean/Server/FileWorker/RequestHandling.lean index 411c58e37527..208323b607cc 100644 --- a/stage0/src/Lean/Server/FileWorker/RequestHandling.lean +++ b/stage0/src/Lean/Server/FileWorker/RequestHandling.lean @@ -237,18 +237,10 @@ open Parser.Command in partial def handleDocumentSymbol (_ : DocumentSymbolParams) : RequestM (RequestTask DocumentSymbolResult) := do let doc ← readDoc - mapTask (← doc.cmdSnaps.waitHead?) fun _ => do - let ⟨cmdSnaps, e?⟩ ← doc.cmdSnaps.getFinishedPrefix - let mut stxs := cmdSnaps.map (·.stx) - match e? with - | some ElabTaskError.aborted => - throw RequestError.fileChanged - | some (ElabTaskError.ioError e) => - throw (e : RequestError) - | _ => pure () - - let lastSnap := cmdSnaps.getLast! -- see `waitHead?` above - stxs := stxs ++ (← parseAhead doc.meta.mkInputContext lastSnap).toList + -- bad: we have to wait on elaboration of the entire file before we can report document symbols + let t ← doc.cmdSnaps.waitAll + mapTask t fun (snaps, _) => do + let mut stxs := snaps.map (·.stx) let (syms, _) := toDocumentSymbols doc.meta.text stxs return { syms := syms.toArray } where diff --git a/stage0/src/Lean/Server/References.lean b/stage0/src/Lean/Server/References.lean index dc48abf3f669..d3b86b3395b1 100644 --- a/stage0/src/Lean/Server/References.lean +++ b/stage0/src/Lean/Server/References.lean @@ -178,13 +178,11 @@ partial def combineFvars (refs : Array Reference) : Array Reference := Id.run do let mut refs' := #[] for ref in refs do match ref with - | { ident := ident@(RefIdent.fvar id), isBinder, .. } => - if isBinder && idMap.contains id then - -- downgrade chained definitions to usages - -- (we shouldn't completely remove them in case they do not have usages) - refs' := refs'.push { ref with ident := applyIdMap idMap ident, isBinder := false, aliases := #[ident] } - else - refs' := refs'.push { ref with ident := applyIdMap idMap ident } + | { ident := ident@(RefIdent.fvar id), .. } => + if idMap.contains id then + refs' := refs'.push { ref with ident := applyIdMap idMap ident, aliases := #[ident] } + else if !idMap.contains id then + refs' := refs'.push ref | _ => refs' := refs'.push ref refs' @@ -198,20 +196,24 @@ where | m, RefIdent.fvar id => RefIdent.fvar <| findCanonicalBinder m id | _, ident => ident -def dedupReferences (refs : Array Reference) : Array Reference := Id.run do - let mut refsByIdAndRange : HashMap (RefIdent × Lsp.Range) Reference := HashMap.empty +def dedupReferences (refs : Array Reference) (allowSimultaneousBinderUse := false) : Array Reference := Id.run do + let mut refsByIdAndRange : HashMap (RefIdent × Option Bool × Lsp.Range) Reference := HashMap.empty for ref in refs do - let key := (ref.ident, ref.range) + let isBinder := if allowSimultaneousBinderUse then some ref.isBinder else none + let key := (ref.ident, isBinder, ref.range) refsByIdAndRange := match refsByIdAndRange[key] with - | some ref' => refsByIdAndRange.insert key { ref' with isBinder := ref'.isBinder || ref.isBinder, aliases := ref'.aliases ++ ref.aliases } + | some ref' => refsByIdAndRange.insert key { ref' with aliases := ref'.aliases ++ ref.aliases } | none => refsByIdAndRange.insert key ref let dedupedRefs := refsByIdAndRange.fold (init := #[]) fun refs _ ref => refs.push ref return dedupedRefs.qsort (·.range < ·.range) def findModuleRefs (text : FileMap) (trees : Array InfoTree) (localVars : Bool := true) - : ModuleRefs := Id.run do - let mut refs := dedupReferences <| combineFvars <| findReferences text trees + (allowSimultaneousBinderUse := false) : ModuleRefs := Id.run do + let mut refs := + dedupReferences (allowSimultaneousBinderUse := allowSimultaneousBinderUse) <| + combineFvars <| + findReferences text trees if !localVars then refs := refs.filter fun | { ident := RefIdent.fvar _, .. } => false diff --git a/stage0/src/Lean/Server/Requests.lean b/stage0/src/Lean/Server/Requests.lean index dd905307b86d..cd034d4fc5e1 100644 --- a/stage0/src/Lean/Server/Requests.lean +++ b/stage0/src/Lean/Server/Requests.lean @@ -132,7 +132,7 @@ structure RequestHandler where builtin_initialize requestHandlers : IO.Ref (Std.PersistentHashMap String RequestHandler) ← IO.mkRef {} -/-- NB: This method may only be called in `builtin_initialize` blocks. +/-- NB: This method may only be called in `initialize` blocks (user or builtin). A registration consists of: - a type of JSON-parsable request data `paramType` @@ -148,7 +148,7 @@ def registerLspRequestHandler (method : String) paramType [FromJson paramType] [FileSource paramType] respType [ToJson respType] (handler : paramType → RequestM (RequestTask respType)) : IO Unit := do - if !(← IO.initializing) then + if !(← Lean.initializing) then throw <| IO.userError s!"Failed to register LSP request handler for '{method}': only possible during initialization" if (← requestHandlers.get).contains method then throw <| IO.userError s!"Failed to register LSP request handler for '{method}': already registered" @@ -164,7 +164,7 @@ def registerLspRequestHandler (method : String) def lookupLspRequestHandler (method : String) : IO (Option RequestHandler) := return (← requestHandlers.get).find? method -/-- NB: This method may only be called in `builtin_initialize` blocks. +/-- NB: This method may only be called in `initialize` blocks (user or builtin). Register another handler to invoke after the last one registered for a method. At least one handler for the method must have already been registered to perform @@ -175,7 +175,7 @@ def chainLspRequestHandler (method : String) paramType [FromJson paramType] respType [FromJson respType] [ToJson respType] (handler : paramType → RequestTask respType → RequestM (RequestTask respType)) : IO Unit := do - if !(← IO.initializing) then + if !(← Lean.initializing) then throw <| IO.userError s!"Failed to chain LSP request handler for '{method}': only possible during initialization" if let some oldHandler ← lookupLspRequestHandler method then let handle := fun j => do diff --git a/stage0/src/Lean/Server/Rpc/Basic.lean b/stage0/src/Lean/Server/Rpc/Basic.lean index 1d1c5f93c0a5..b0e451048126 100644 --- a/stage0/src/Lean/Server/Rpc/Basic.lean +++ b/stage0/src/Lean/Server/Rpc/Basic.lean @@ -42,10 +42,13 @@ non-JSON-serializable fields can be auto-encoded in two ways: -- TODO(WN): for Lean.js, have third parameter defining the client-side structure; -- or, compile `WithRpcRef` to "opaque reference" on the client class RpcEncoding (α : Type) (β : outParam Type) where - rpcEncode {m : Type → Type} [Monad m] [MonadRpcSession m] : α → m β + rpcEncode {m : Type → Type} [Monad m] [MonadRpcSession m] : α → ExceptT String m β rpcDecode {m : Type → Type} [Monad m] [MonadRpcSession m] : β → ExceptT String m α export RpcEncoding (rpcEncode rpcDecode) +instance : Nonempty (RpcEncoding α β) := + ⟨{ rpcEncode := fun _ => throw "unreachable", rpcDecode := fun _ => throw "unreachable" }⟩ + instance [FromJson α] [ToJson α] : RpcEncoding α α where rpcEncode := pure rpcDecode := pure diff --git a/stage0/src/Lean/Server/Rpc/Deriving.lean b/stage0/src/Lean/Server/Rpc/Deriving.lean index c106b84d0747..8ad3231d0797 100644 --- a/stage0/src/Lean/Server/Rpc/Deriving.lean +++ b/stage0/src/Lean/Server/Rpc/Deriving.lean @@ -20,26 +20,14 @@ private def deriveWithRefInstance (typeNm : Name) : CommandElabM Bool := do -- TODO(WN): check that `typeNm` is not a scalar type let typeId := mkIdent typeNm let cmds ← `( - section - variable {m : Type → Type} - unsafe def encodeUnsafe [Monad m] [MonadRpcSession m] (r : WithRpcRef $typeId:ident) : m Lsp.RpcRef := - WithRpcRef.encodeUnsafe $(quote typeNm) r - - @[implementedBy encodeUnsafe] - opaque encode [Monad m] [MonadRpcSession m] (r : WithRpcRef $typeId:ident) : m Lsp.RpcRef := - pure ⟨0⟩ - - unsafe def decodeUnsafe [Monad m] [MonadRpcSession m] (r : Lsp.RpcRef) : ExceptT String m (WithRpcRef $typeId:ident) := - WithRpcRef.decodeUnsafeAs $typeId:ident $(quote typeNm) r - - @[implementedBy decodeUnsafe] - opaque decode [Monad m] [MonadRpcSession m] (r : Lsp.RpcRef) : ExceptT String m (WithRpcRef $typeId:ident) := - throw "unreachable" - - instance : RpcEncoding (WithRpcRef $typeId:ident) Lsp.RpcRef := - { rpcEncode := encode - rpcDecode := decode } - end + unsafe def unsafeInst : RpcEncoding (WithRpcRef $typeId:ident) Lsp.RpcRef where + rpcEncode := WithRpcRef.encodeUnsafe $(quote typeNm) + rpcDecode := WithRpcRef.decodeUnsafeAs $typeId:ident $(quote typeNm) + + @[implementedBy unsafeInst] + opaque inst : RpcEncoding (WithRpcRef $typeId) Lsp.RpcRef + + instance : RpcEncoding (WithRpcRef $typeId) Lsp.RpcRef := inst ) elabCommand cmds return true @@ -85,45 +73,27 @@ def withFieldsFlattened (indVal : InductiveVal) (params : Array Expr) end -def isOptField (n : Name) : Bool := - n.toString.endsWith "?" +private def getRpcPacketFor (ty : Expr) : MetaM Expr := do + let packetTy ← mkFreshExprMVar (Expr.sort levelOne) + let _ ← synthInstance (mkApp2 (mkConst ``RpcEncoding) ty packetTy) + instantiateMVars packetTy -private def deriveStructureInstance (indVal : InductiveVal) (params : Array Expr) : TermElabM Command := +private def deriveStructureInstance (indVal : InductiveVal) (params : Array Expr) + (paramBinders packetParamBinders encInstBinders : Array (TSyntax ``Parser.Term.bracketedBinder)) : TermElabM Command := do withFields indVal params fun fields => do trace[Elab.Deriving.RpcEncoding] "for structure {indVal.name} with params {params}" - -- Postulate that every field have a rpc encoding, storing the encoding type ident - -- in `fieldEncIds`. When multiple fields have the same type, we reuse the encoding type - -- as otherwise typeclass synthesis fails. let mut binders := #[] let mut fieldIds := #[] - let mut fieldEncIds : Array Term := #[] - let mut uniqFieldEncIds : Array Ident := #[] - let mut fieldEncIds' : DiscrTree Ident := {} + let mut fieldEncTypeStxs := #[] for (fieldName, fieldTp) in fields do let mut fieldTp := fieldTp - if isOptField fieldName then - if !fieldTp.isAppOf ``Option then - throwError "optional field '{fieldName}' has type{indentD m!"{fieldTp}"}\nbut is expected to have type{indentD "Option _"}" --" - fieldTp := fieldTp.getArg! 0 - -- postulate that the field has an encoding and remember the encoding's binder name + let fieldEncTypeStx ← PrettyPrinter.delab (← getRpcPacketFor fieldTp) + let stx ← PrettyPrinter.delab fieldTp fieldIds := fieldIds.push <| mkIdent fieldName - let mut fieldEncId : Ident := ⟨Syntax.missing⟩ - match (← fieldEncIds'.getMatch fieldTp).back? with - | none => - fieldEncId ← mkIdent <$> mkFreshUserName fieldName - binders := binders.push (← `(bracketedBinder| ( $fieldEncId:ident ))) - let stx ← PrettyPrinter.delab fieldTp - binders := binders.push - (← `(bracketedBinder| [ $(mkIdent ``Lean.Server.RpcEncoding) $stx $fieldEncId:ident ])) - fieldEncIds' ← fieldEncIds'.insert fieldTp fieldEncId - uniqFieldEncIds := uniqFieldEncIds.push fieldEncId - | some fid => fieldEncId := fid - - if isOptField fieldName then - fieldEncIds := fieldEncIds.push <| ← ``(Option $fieldEncId:ident) - else - fieldEncIds := fieldEncIds.push fieldEncId + fieldEncTypeStxs := fieldEncTypeStxs.push fieldEncTypeStx + binders := binders.push + (← `(bracketedBinder| [ RpcEncoding $stx $fieldEncTypeStx ])) -- helpers for field initialization syntax let fieldInits (func : Name) := fieldIds.mapM fun fid => @@ -134,115 +104,88 @@ private def deriveStructureInstance (indVal : InductiveVal) (params : Array Expr -- helpers for type name syntax let paramIds ← params.mapM fun p => return mkIdent (← getFVarLocalDecl p).userName let typeId := Syntax.mkApp (← `(@$(mkIdent indVal.name))) paramIds - let packetId ← mkIdent <$> mkFreshUserName `RpcEncodingPacket - let packetAppliedId := Syntax.mkApp packetId uniqFieldEncIds - - `(variable $binders* - - structure $packetId:ident where - $[($fieldIds : $fieldEncIds)]* - deriving $(mkIdent ``FromJson), $(mkIdent ``ToJson) - - instance : $(mkIdent ``RpcEncoding) $typeId $packetAppliedId where - rpcEncode a := return { - $[$encInits],* - } - rpcDecode a := return { - $[$decInits],* - } + let instId := mkIdent (`_root_ ++ indVal.name.appendBefore "instRpcEncoding") + + `(variable $packetParamBinders* in + structure RpcEncodingPacket where + $[($fieldIds : $fieldEncTypeStxs)]* + deriving FromJson, ToJson + + variable $(paramBinders ++ packetParamBinders ++ encInstBinders)* in + @[instance] def $instId := show RpcEncoding $typeId (RpcEncodingPacket ..) from { + rpcEncode := fun a => return { $[$encInits],* } + rpcDecode := fun a => return { $[$decInits],* } + } ) private structure CtorState where - -- names of encoded argument types in the RPC packet - encArgTypes : DiscrTree Name := {} - uniqEncArgTypes : Array Name := #[] - -- binders for `encArgTypes` as well as the relevant `RpcEncoding`s - binders : Array (TSyntax ``Parser.Term.bracketedBinder) := #[] -- the syntax of each constructor in the packet ctors : Array (TSyntax ``Parser.Command.ctor) := #[] -- syntax of each arm of the `rpcEncode` pattern-match encodes : Array (TSyntax ``Parser.Term.matchAlt) := #[] -- syntax of each arm of the `rpcDecode` pattern-match decodes : Array (TSyntax ``Parser.Term.matchAlt) := #[] - deriving Inhabited private def matchF := Lean.Parser.Term.matchAlt (rhsParser := Lean.Parser.termParser) -private def deriveInductiveInstance (indVal : InductiveVal) (params : Array Expr) : TermElabM Command := do +private def deriveInductiveInstance (indVal : InductiveVal) (params : Array Expr) + (paramBinders packetParamBinders encInstBinders : Array (TSyntax ``Parser.Term.bracketedBinder)) : TermElabM Command := do trace[Elab.Deriving.RpcEncoding] "for inductive {indVal.name} with params {params}" - - -- produce all encoding types and binders for them - let st ← foldWithConstructors indVal params (init := { : CtorState}) fun acc ctor argVars tp => do - trace[Elab.Deriving.RpcEncoding] "{ctor} : {argVars} → {tp}" - let mut acc := acc - let argFVars ← argVars.mapM (LocalDecl.fvarId <$> getFVarLocalDecl ·) - for arg in argVars do - let argTp ← inferType arg - if (← findExprDependsOn argTp (pf := fun fv => argFVars.contains fv)) then - throwError "cross-argument dependencies are not supported ({arg} : {argTp})" - - if (← acc.encArgTypes.getMatch argTp).isEmpty then - let tid ← mkFreshUserName `_rpcEnc - let argTpStx ← PrettyPrinter.delab argTp - acc := { acc with encArgTypes := ← acc.encArgTypes.insert argTp tid - uniqEncArgTypes := acc.uniqEncArgTypes.push tid - binders := acc.binders.append #[ - (← `(bracketedBinder| ( $(mkIdent tid):ident ))), - (← `(bracketedBinder| [ $(mkIdent ``Lean.Server.RpcEncoding) $argTpStx $(mkIdent tid):ident ])) - ] } - return acc - - -- introduce encoding types into the local context so that we can use the delaborator to print them - withLocalDecls - (st.uniqEncArgTypes.map fun tid => (tid, BinderInfo.default, fun _ => pure <| mkSort levelOne)) - fun ts => do - trace[Elab.Deriving.RpcEncoding] m!"RpcEncoding type binders : {ts}" - - let packetNm ← mkFreshUserName `RpcEncodingPacket - let st ← foldWithConstructors indVal params (init := st) fun acc ctor argVars _ => do - -- create the constructor - let mut pktCtorTp := Lean.mkConst packetNm - for arg in argVars.reverse do - let argTp ← inferType arg - let encTpNm := (← acc.encArgTypes.getMatch argTp).back - let encTp ← elabTerm (mkIdent encTpNm) none - pktCtorTp := mkForall (← getFVarLocalDecl arg).userName BinderInfo.default encTp pktCtorTp - -- TODO(WN): this relies on delab printing non-macro-scoped user names in non-dependent foralls - -- to generate the expected JSON encoding - let pktCtorTpStx ← PrettyPrinter.delab pktCtorTp - let pktCtor ← `(Lean.Parser.Command.ctor| | $(mkIdent ctor.getString!):ident : $pktCtorTpStx:term) - - -- create encoder and decoder match arms - let nms ← argVars.mapM fun _ => mkIdent <$> mkFreshBinderName - let mkPattern (src : Name) := Syntax.mkApp (mkIdent <| Name.mkStr src ctor.getString!) nms - let mkBody (tgt : Name) (func : Name) : TermElabM Term := do - let items ← nms.mapM fun nm => `(← $(mkIdent func) $nm) - let tm := Syntax.mkApp (mkIdent <| Name.mkStr tgt ctor.getString!) items - `(return $tm:term) - - let encArm ← `(matchF| | $(mkPattern indVal.name):term => $(← mkBody packetNm ``rpcEncode)) - let decArm ← `(matchF| | $(mkPattern packetNm):term => $(← mkBody indVal.name ``rpcDecode)) - - return { acc with ctors := acc.ctors.push pktCtor - encodes := acc.encodes.push ⟨encArm⟩ - decodes := acc.decodes.push ⟨decArm⟩ } - - -- helpers for type name syntax - let paramIds ← params.mapM fun p => return mkIdent (← getFVarLocalDecl p).userName - let typeId := Syntax.mkApp (← `(@$(mkIdent indVal.name))) paramIds - let packetAppliedId := Syntax.mkApp (mkIdent packetNm) (st.uniqEncArgTypes.map (mkIdent ·)) - - `(variable $st.binders* - - inductive $(mkIdent packetNm) where - $[$(st.ctors):ctor]* - deriving $(mkIdent ``FromJson), $(mkIdent ``ToJson) - - instance : $(mkIdent ``RpcEncoding) $typeId $packetAppliedId where - rpcEncode := fun x => match x with - $[$(st.encodes):matchAlt]* - rpcDecode := fun x => match x with - $[$(st.decodes):matchAlt]* - ) + withoutModifyingEnv do + let packetNm := (← `(RpcEncodingPacket)).1.getId + addDecl <| .axiomDecl { + name := packetNm + levelParams := [] + type := mkSort levelOne + isUnsafe := true + } + let pktCtorTp := mkConst packetNm + let recInstTp := mkApp2 (mkConst ``RpcEncoding) (mkAppN (mkConst indVal.name) params) pktCtorTp + withLocalDecl `inst .instImplicit recInstTp fun _ => do + let st ← foldWithConstructors indVal params (init := { : CtorState }) fun acc ctor argVars _ => do + -- create the constructor + let fieldStxs ← argVars.mapM fun arg => do + let packetTp ← getRpcPacketFor (← inferType arg) + let tyStx ← PrettyPrinter.delab packetTp + let name := (← getFVarLocalDecl arg).userName + `(bracketedBinder| ($(mkIdent name) : $tyStx)) + let pktCtor ← `(Parser.Command.ctor| | $(mkIdent ctor.getString!):ident $[$fieldStxs]* : RpcEncodingPacket) + + -- create encoder and decoder match arms + let nms ← argVars.mapM fun _ => mkIdent <$> mkFreshBinderName + let mkPattern (src : Name) := Syntax.mkApp (mkIdent <| Name.mkStr src ctor.getString!) nms + let mkBody (tgt : Name) (func : Name) : TermElabM Term := do + let items ← nms.mapM fun nm => `(← $(mkIdent func) $nm) + let tm := Syntax.mkApp (mkIdent <| Name.mkStr tgt ctor.getString!) items + `(return $tm:term) + + let encArm ← `(matchF| | $(mkPattern indVal.name):term => $(← mkBody packetNm ``rpcEncode)) + let decArm ← `(matchF| | $(mkPattern packetNm):term => $(← mkBody indVal.name ``rpcDecode)) + + return { acc with ctors := acc.ctors.push pktCtor + encodes := acc.encodes.push ⟨encArm⟩ + decodes := acc.decodes.push ⟨decArm⟩ } + + -- helpers for type name syntax + let paramIds ← params.mapM fun p => return mkIdent (← getFVarLocalDecl p).userName + let typeId := Syntax.mkApp (← `(@$(mkIdent indVal.name))) paramIds + let instId := mkIdent (`_root_ ++ indVal.name.appendBefore "instRpcEncoding") + + `(variable $packetParamBinders:bracketedBinder* in + inductive RpcEncodingPacket where + $[$(st.ctors):ctor]* + deriving FromJson, ToJson + + variable $(paramBinders ++ packetParamBinders ++ encInstBinders)* in + @[instance] partial def $instId := show RpcEncoding $typeId (RpcEncodingPacket ..) from + { rpcEncode, rpcDecode } + where + rpcEncode {m} [Monad m] [MonadRpcSession m] (x : $typeId) : ExceptT String m (RpcEncodingPacket ..) := + have inst : RpcEncoding $typeId (RpcEncodingPacket ..) := { rpcEncode, rpcDecode } + match x with $[$(st.encodes):matchAlt]* + rpcDecode {m} [Monad m] [MonadRpcSession m] (x : RpcEncodingPacket ..) : ExceptT String m $typeId := + have inst : RpcEncoding $typeId (RpcEncodingPacket ..) := { rpcEncode, rpcDecode } + match x with $[$(st.decodes):matchAlt]* + ) /-- Creates an `RpcEncodingPacket` for `typeName`. For structures, the packet is a structure with the same field names. For inductives, it mirrors the inductive structure with every field @@ -255,33 +198,35 @@ private def deriveInstance (typeName : Name) : CommandElabM Bool := do if indVal.numIndices ≠ 0 then throwError "indexed inductive families are not supported" - let cmds ← liftTermElabM none <| + let (paramBinders, packetParamBinders, encInstBinders) ← liftTermElabM none do -- introduce fvars for all the parameters forallTelescopeReducing indVal.type fun params _ => do - assert! params.size == indVal.numParams + let mut paramBinders := #[] -- input parameters + let mut packetParamBinders := #[] -- RPC encoding packets for type input parameters + let mut encInstBinders := #[] -- RPC encoding instance binders corresponding to packetParamBinders - -- bind every parameter and *some* (not named) `RpcEncoding` for it - let mut binders := #[] for param in params do - let paramNm := (←getFVarLocalDecl param).userName - binders := binders.push (← `(bracketedBinder| ( $(mkIdent paramNm) ))) + let paramNm := (← getFVarLocalDecl param).userName + let ty ← PrettyPrinter.delab (← inferType param) + paramBinders := paramBinders.push (← `(bracketedBinder| ($(mkIdent paramNm) : $ty))) + let packet := mkIdent (← mkFreshUserName (paramNm.appendAfter "Packet")) -- only look for encodings for `Type` parameters - if !(← inferType param).isType then continue - binders := binders.push - (← `(bracketedBinder| [ $(mkIdent ``Lean.Server.RpcEncoding) $(mkIdent paramNm) _ ])) - - return #[ - ← `(section), - ← `(variable $binders*), - ← if isStructure (← getEnv) typeName then - deriveStructureInstance indVal params + if (← inferType param).isType then + packetParamBinders := packetParamBinders.push (← `(bracketedBinder| ($packet : Type))) + encInstBinders := encInstBinders.push (← `(bracketedBinder| [RpcEncoding $(mkIdent paramNm) $packet])) else - deriveInductiveInstance indVal params, - ← `(end) - ] + packetParamBinders := packetParamBinders.push paramBinders.back + + return (paramBinders, packetParamBinders, encInstBinders) + + elabCommand <| ← liftTermElabM none do + Term.elabBinders (paramBinders ++ packetParamBinders ++ encInstBinders) fun locals => do + let params := locals[:paramBinders.size] + if isStructure (← getEnv) typeName then + deriveStructureInstance indVal params paramBinders packetParamBinders encInstBinders + else + deriveInductiveInstance indVal params paramBinders packetParamBinders encInstBinders - for cmd in cmds do - elabCommand cmd.raw return true private unsafe def dispatchDeriveInstanceUnsafe (declNames : Array Name) (args? : Option (TSyntax ``Parser.Term.structInst)) : CommandElabM Bool := do @@ -289,8 +234,7 @@ private unsafe def dispatchDeriveInstanceUnsafe (declNames : Array Name) (args? return false let args ← if let some args := args? then - let n ← liftCoreM <| mkFreshUserName `_args - liftTermElabM (some n) do + liftTermElabM none do let argsT := mkConst ``DerivingParams let args ← elabTerm args argsT evalExpr' DerivingParams ``DerivingParams args diff --git a/stage0/src/Lean/Server/Rpc/RequestHandling.lean b/stage0/src/Lean/Server/Rpc/RequestHandling.lean index 1da7da08fd8c..5ad94572cf28 100644 --- a/stage0/src/Lean/Server/Rpc/RequestHandling.lean +++ b/stage0/src/Lean/Server/Rpc/RequestHandling.lean @@ -82,8 +82,18 @@ def wrapRpcProcedure (method : Name) paramType respType RequestM.mapTask t fun | Except.error e => throw e | Except.ok ret => do - let act := rpcEncode (α := respType) (β := respLspType) (m := StateM FileWorker.RpcSession) ret - return toJson (← seshRef.modifyGet act.run)⟩ + let act : StateM FileWorker.RpcSession (Except String respLspType) := do + let s ← get + match ← rpcEncode (α := respType) (β := respLspType) (m := StateM FileWorker.RpcSession) ret with + | .ok x => return .ok x + | .error e => set s; return .error e + match ← seshRef.modifyGet act.run with + | .ok x => return toJson x + | .error e => + throwThe RequestError { + code := JsonRpc.ErrorCode.invalidParams + message := s!"Cannot encode result of RPC call '{method}'\n{e}" + }⟩ def registerBuiltinRpcProcedure (method : Name) paramType respType {paramLspType} [RpcEncoding paramType paramLspType] [FromJson paramLspType] diff --git a/stage0/src/Lean/Server/Snapshots.lean b/stage0/src/Lean/Server/Snapshots.lean index 3afe0e8565cb..f3b6d77627cb 100644 --- a/stage0/src/Lean/Server/Snapshots.lean +++ b/stage0/src/Lean/Server/Snapshots.lean @@ -83,22 +83,6 @@ def parseNextCmd (inputCtx : Parser.InputContext) (snap : Snapshot) : IO Syntax Parser.parseCommand inputCtx pmctx snap.mpState snap.msgLog return cmdStx -/-- - Parse remaining file without elaboration. NOTE that doing so can lead to parse errors or even wrong syntax objects, - so it should only be done for reporting preliminary results! -/ -partial def parseAhead (inputCtx : Parser.InputContext) (snap : Snapshot) : IO (Array Syntax) := do - let cmdState := snap.cmdState - let scope := cmdState.scopes.head! - let pmctx := { env := cmdState.env, options := scope.opts, currNamespace := scope.currNamespace, openDecls := scope.openDecls } - go inputCtx pmctx snap.mpState #[] - where - go inputCtx pmctx cmdParserState stxs := do - let (cmdStx, cmdParserState, _) := Parser.parseCommand inputCtx pmctx cmdParserState snap.msgLog - if Parser.isEOI cmdStx || Parser.isExitCommand cmdStx then - return stxs.push cmdStx - else - go inputCtx pmctx cmdParserState (stxs.push cmdStx) - register_builtin_option server.stderrAsMessages : Bool := { defValue := true group := "server" diff --git a/stage0/src/Lean/Server/Watchdog.lean b/stage0/src/Lean/Server/Watchdog.lean index ce09f372cf30..9831d6d31c52 100644 --- a/stage0/src/Lean/Server/Watchdog.lean +++ b/stage0/src/Lean/Server/Watchdog.lean @@ -682,7 +682,7 @@ def mkLeanServerCapabilities : ServerCapabilities := { semanticTokensProvider? := some { legend := { tokenTypes := SemanticTokenType.names - tokenModifiers := #[] + tokenModifiers := SemanticTokenModifier.names } full := true range := true diff --git a/stage0/src/Lean/Util/HasConstCache.lean b/stage0/src/Lean/Util/HasConstCache.lean index a131d7172864..bad4046f9bed 100644 --- a/stage0/src/Lean/Util/HasConstCache.lean +++ b/stage0/src/Lean/Util/HasConstCache.lean @@ -11,7 +11,7 @@ structure HasConstCache (declName : Name) where cache : Std.HashMapImp Expr Bool := Std.mkHashMapImp unsafe def HasConstCache.containsUnsafe (e : Expr) : StateM (HasConstCache declName) Bool := do - if let some r := (← get).cache.find? (beq := ⟨Expr.ptrEq⟩) e then + if let some r := (← get).cache.find? (beq := ⟨ptrEq⟩) e then return r else match e with @@ -25,7 +25,7 @@ unsafe def HasConstCache.containsUnsafe (e : Expr) : StateM (HasConstCache declN | _ => return false where cache (e : Expr) (r : Bool) : StateM (HasConstCache declName) Bool := do - modify fun ⟨cache⟩ => ⟨cache.insert (beq := ⟨Expr.ptrEq⟩) e r |>.1⟩ + modify fun ⟨cache⟩ => ⟨cache.insert (beq := ⟨ptrEq⟩) e r |>.1⟩ return r /-- diff --git a/stage0/src/kernel/expr.cpp b/stage0/src/kernel/expr.cpp index 4904d97f2406..ebce32cbf184 100644 --- a/stage0/src/kernel/expr.cpp +++ b/stage0/src/kernel/expr.cpp @@ -330,97 +330,6 @@ expr update_let(expr const & e, expr const & new_type, expr const & new_value, e return e; } -extern "C" LEAN_EXPORT object * lean_expr_update_mdata(obj_arg e, obj_arg new_expr) { - if (mdata_expr(TO_REF(expr, e)).raw() != new_expr) { - object * r = lean_expr_mk_mdata(mdata_data(TO_REF(expr, e)).to_obj_arg(), new_expr); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_expr); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_const(obj_arg e, obj_arg new_levels) { - if (const_levels(TO_REF(expr, e)).raw() != new_levels) { - object * r = lean_expr_mk_const(const_name(TO_REF(expr, e)).to_obj_arg(), new_levels); - lean_dec_ref(e); - return r; - } else { - lean_dec(new_levels); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_sort(obj_arg e, obj_arg new_level) { - if (sort_level(TO_REF(expr, e)).raw() != new_level) { - object * r = lean_expr_mk_sort(new_level); - lean_dec_ref(e); - return r; - } else { - lean_dec(new_level); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_proj(obj_arg e, obj_arg new_expr) { - if (proj_expr(TO_REF(expr, e)).raw() != new_expr) { - object * r = lean_expr_mk_proj(proj_sname(TO_REF(expr, e)).to_obj_arg(), proj_idx(TO_REF(expr, e)).to_obj_arg(), new_expr); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_expr); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_app(obj_arg e, obj_arg new_fn, obj_arg new_arg) { - if (app_fn(TO_REF(expr, e)).raw() != new_fn || app_arg(TO_REF(expr, e)).raw() != new_arg) { - object * r = lean_expr_mk_app(new_fn, new_arg); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_fn); lean_dec_ref(new_arg); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_forall(obj_arg e, uint8 new_binfo, obj_arg new_domain, obj_arg new_body) { - if (binding_domain(TO_REF(expr, e)).raw() != new_domain || binding_body(TO_REF(expr, e)).raw() != new_body || - binding_info(TO_REF(expr, e)) != static_cast(new_binfo)) { - object * r = lean_expr_mk_forall(binding_name(TO_REF(expr, e)).to_obj_arg(), new_domain, new_body, new_binfo); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_domain); lean_dec_ref(new_body); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_lambda(obj_arg e, uint8 new_binfo, obj_arg new_domain, obj_arg new_body) { - if (binding_domain(TO_REF(expr, e)).raw() != new_domain || binding_body(TO_REF(expr, e)).raw() != new_body || - binding_info(TO_REF(expr, e)) != static_cast(new_binfo)) { - object * r = lean_expr_mk_lambda(binding_name(TO_REF(expr, e)).to_obj_arg(), new_domain, new_body, new_binfo); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_domain); lean_dec_ref(new_body); - return e; - } -} - -extern "C" LEAN_EXPORT object * lean_expr_update_let(obj_arg e, obj_arg new_type, obj_arg new_val, obj_arg new_body) { - if (let_type(TO_REF(expr, e)).raw() != new_type || let_value(TO_REF(expr, e)).raw() != new_val || - let_body(TO_REF(expr, e)).raw() != new_body) { - object * r = lean_expr_mk_let(let_name(TO_REF(expr, e)).to_obj_arg(), new_type, new_val, new_body); - lean_dec_ref(e); - return r; - } else { - lean_dec_ref(new_type); lean_dec_ref(new_val); lean_dec_ref(new_body); - return e; - } -} - extern "C" object * lean_expr_consume_type_annotations(obj_arg e); expr consume_type_annotations(expr const & e) { return expr(lean_expr_consume_type_annotations(e.to_obj_arg())); } diff --git a/stage0/src/kernel/level.cpp b/stage0/src/kernel/level.cpp index 9ed8d461d9b5..06652dc8ca67 100644 --- a/stage0/src/kernel/level.cpp +++ b/stage0/src/kernel/level.cpp @@ -29,10 +29,6 @@ extern "C" object * lean_level_mk_mvar(obj_arg); extern "C" object * lean_level_mk_param(obj_arg); extern "C" object * lean_level_mk_max(obj_arg, obj_arg); extern "C" object * lean_level_mk_imax(obj_arg, obj_arg); -extern "C" object * lean_level_mk_max_simp(obj_arg, obj_arg); -extern "C" object * lean_level_mk_imax_simp(obj_arg, obj_arg); -extern "C" object * lean_level_simp_max(obj_arg, obj_arg, obj_arg); -extern "C" object * lean_level_simp_imax(obj_arg, obj_arg, obj_arg); level mk_succ(level const & l) { return level(lean_level_mk_succ(l.to_obj_arg())); } level mk_max_core(level const & l1, level const & l2) { return level(lean_level_mk_max(l1.to_obj_arg(), l2.to_obj_arg())); } @@ -293,34 +289,6 @@ level update_max(level const & l, level const & new_lhs, level const & new_rhs) return mk_imax(new_lhs, new_rhs); } -extern "C" LEAN_EXPORT object * lean_level_update_succ(obj_arg l, obj_arg new_arg) { - if (succ_of(TO_REF(level, l)).raw() == new_arg) { - lean_dec(new_arg); - return l; - } else { - lean_dec_ref(l); - return lean_level_mk_succ(new_arg); - } -} - -extern "C" LEAN_EXPORT object * lean_level_update_max(obj_arg l, obj_arg new_lhs, obj_arg new_rhs) { - if (max_lhs(TO_REF(level, l)).raw() == new_lhs && max_rhs(TO_REF(level, l)).raw() == new_rhs) { - return lean_level_simp_max(new_lhs, new_rhs, l); - } else { - lean_dec_ref(l); - return lean_level_mk_max_simp(new_lhs, new_rhs); - } -} - -extern "C" LEAN_EXPORT object * lean_level_update_imax(obj_arg l, obj_arg new_lhs, obj_arg new_rhs) { - if (imax_lhs(TO_REF(level, l)).raw() == new_lhs && imax_rhs(TO_REF(level, l)).raw() == new_rhs) { - return lean_level_simp_imax(new_lhs, new_rhs, l); - } else { - lean_dec_ref(l); - return lean_level_mk_imax_simp(new_lhs, new_rhs); - } -} - level instantiate(level const & l, names const & ps, levels const & ls) { lean_assert(length(ps) == length(ls)); return replace(l, [=](level const & l) { diff --git a/stage0/stdlib/Init/Data/List/Control.c b/stage0/stdlib/Init/Data/List/Control.c index 7ce9d4c315ad..8e706c1232d8 100644 --- a/stage0/stdlib/Init/Data/List/Control.c +++ b/stage0/stdlib/Init/Data/List/Control.c @@ -21,6 +21,7 @@ LEAN_EXPORT lean_object* l_List_instForIn_x27ListInferInstanceMembershipInstMemb LEAN_EXPORT lean_object* l_List_findSomeM_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterAuxM___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instForIn_x27ListInferInstanceMembershipInstMembershipList(lean_object*, lean_object*, lean_object*); +static lean_object* l_List_instFunctorList___closed__1; LEAN_EXPORT lean_object* l_List_mapM___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_firstM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_anyM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t); @@ -34,6 +35,7 @@ LEAN_EXPORT lean_object* l_List_findM_x3f___rarg___lambda__1(lean_object*, lean_ LEAN_EXPORT lean_object* l_List_anyM(lean_object*); LEAN_EXPORT lean_object* l_List_allM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapA___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_instFunctorList___closed__3; LEAN_EXPORT lean_object* l_List_forIn_loop(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_x27_loop(lean_object*, lean_object*, lean_object*); @@ -43,12 +45,15 @@ LEAN_EXPORT lean_object* l_List_findSomeM_x3f___rarg___lambda__1(lean_object*, l LEAN_EXPORT lean_object* l_List_filterRevM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instForInList(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_findM_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapTRAux___at_List_instFunctorList___spec__1___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_List_instFunctorList___closed__2; LEAN_EXPORT lean_object* l_List_forIn_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forA___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forA___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_allM___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterAuxM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_instFunctorList___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapM_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_instForMList___rarg(lean_object*, lean_object*, lean_object*); @@ -75,6 +80,7 @@ LEAN_EXPORT lean_object* l_List_filterRevM(lean_object*); LEAN_EXPORT lean_object* l_List_filterM(lean_object*); LEAN_EXPORT lean_object* l_List_anyM___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapTRAux___at_List_instFunctorList___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterAuxM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_List_findSomeM_x3f(lean_object*); LEAN_EXPORT lean_object* l_List_foldrM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -82,12 +88,15 @@ LEAN_EXPORT lean_object* l___private_Init_Data_List_Control_0__List_forIn_x27_lo LEAN_EXPORT lean_object* l_List_findM_x3f(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Control_0__List_forIn_loop_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM(lean_object*); +LEAN_EXPORT lean_object* l_List_instFunctorList; LEAN_EXPORT lean_object* l_List_foldrM(lean_object*); +LEAN_EXPORT lean_object* l_List_instFunctorList___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Control_0__List_forIn_loop_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_findM_x3f___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_x27_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapA___rarg___lambda__1(lean_object*, lean_object*); +lean_object* l_List_mapTRAux___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_List_Control_0__List_forIn_loop_match__2_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: @@ -1413,6 +1422,116 @@ x_3 = lean_alloc_closure((void*)(l_List_instForMList___rarg), 3, 0); return x_3; } } +LEAN_EXPORT lean_object* l_List_mapTRAux___at_List_instFunctorList___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_4; +lean_dec(x_1); +x_4 = l_List_reverse___rarg(x_3); +return x_4; +} +else +{ +uint8_t x_5; +x_5 = !lean_is_exclusive(x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_2, 1); +x_7 = lean_ctor_get(x_2, 0); +lean_dec(x_7); +lean_inc(x_1); +lean_ctor_set(x_2, 1, x_3); +lean_ctor_set(x_2, 0, x_1); +{ +lean_object* _tmp_1 = x_6; +lean_object* _tmp_2 = x_2; +x_2 = _tmp_1; +x_3 = _tmp_2; +} +goto _start; +} +else +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_dec(x_2); +lean_inc(x_1); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_3); +x_2 = x_9; +x_3 = x_10; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_List_mapTRAux___at_List_instFunctorList___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_List_mapTRAux___at_List_instFunctorList___spec__1___rarg), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_List_instFunctorList___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_box(0); +x_6 = l_List_mapTRAux___rarg(x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_List_instFunctorList___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_box(0); +x_6 = l_List_mapTRAux___at_List_instFunctorList___spec__1___rarg(x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_List_instFunctorList___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_List_instFunctorList___lambda__1), 4, 0); +return x_1; +} +} +static lean_object* _init_l_List_instFunctorList___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_List_instFunctorList___lambda__2), 4, 0); +return x_1; +} +} +static lean_object* _init_l_List_instFunctorList___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_List_instFunctorList___closed__1; +x_2 = l_List_instFunctorList___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_List_instFunctorList() { +_start: +{ +lean_object* x_1; +x_1 = l_List_instFunctorList___closed__3; +return x_1; +} +} lean_object* initialize_Init_Control_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Basic(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -1428,6 +1547,14 @@ if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_List_mapA___rarg___closed__1 = _init_l_List_mapA___rarg___closed__1(); lean_mark_persistent(l_List_mapA___rarg___closed__1); +l_List_instFunctorList___closed__1 = _init_l_List_instFunctorList___closed__1(); +lean_mark_persistent(l_List_instFunctorList___closed__1); +l_List_instFunctorList___closed__2 = _init_l_List_instFunctorList___closed__2(); +lean_mark_persistent(l_List_instFunctorList___closed__2); +l_List_instFunctorList___closed__3 = _init_l_List_instFunctorList___closed__3(); +lean_mark_persistent(l_List_instFunctorList___closed__3); +l_List_instFunctorList = _init_l_List_instFunctorList(); +lean_mark_persistent(l_List_instFunctorList); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Data/String/Extra.c b/stage0/stdlib/Init/Data/String/Extra.c index c0f4055608d1..c819cb3feb2a 100644 --- a/stage0/stdlib/Init/Data/String/Extra.c +++ b/stage0/stdlib/Init/Data/String/Extra.c @@ -25,14 +25,17 @@ LEAN_EXPORT lean_object* l_String_toNat_x21___lambda__1(lean_object*, uint32_t); lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__2___closed__1; +uint8_t l_String_Iterator_atEnd(lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__2___closed__6; lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__24; +LEAN_EXPORT lean_object* l_String_Iterator_foldUntil(lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__16; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__7; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__10; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__20; +LEAN_EXPORT lean_object* l_String_Iterator_find(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__2(lean_object*, lean_object*, lean_object*); lean_object* lean_string_from_utf8_unchecked(lean_object*); @@ -43,12 +46,14 @@ static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__t static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__22; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__28; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__14; +LEAN_EXPORT lean_object* l_String_Iterator_foldUntil___rarg(lean_object*, lean_object*, lean_object*); uint8_t l_String_isNat(lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__29; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__25; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__2___closed__3; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__6; +lean_object* l_String_Iterator_next(lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__1; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__13; @@ -56,6 +61,7 @@ static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__t lean_object* lean_string_to_utf8(lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__2; static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__21; +uint32_t l_String_Iterator_curr(lean_object*); LEAN_EXPORT lean_object* l_String_toNat_x21___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_String_foldlAux_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_String___aux__Init__Data__String__Extra______macroRules__tacticDecreasing__trivial__1___closed__3; @@ -937,6 +943,94 @@ return x_77; } } } +LEAN_EXPORT lean_object* l_String_Iterator_find(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; +x_3 = l_String_Iterator_atEnd(x_1); +if (x_3 == 0) +{ +uint32_t x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_4 = l_String_Iterator_curr(x_1); +x_5 = lean_box_uint32(x_4); +lean_inc(x_2); +x_6 = lean_apply_1(x_2, x_5); +x_7 = lean_unbox(x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +lean_object* x_8; +x_8 = l_String_Iterator_next(x_1); +x_1 = x_8; +goto _start; +} +else +{ +lean_dec(x_2); +return x_1; +} +} +else +{ +lean_dec(x_2); +return x_1; +} +} +} +LEAN_EXPORT lean_object* l_String_Iterator_foldUntil___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = l_String_Iterator_atEnd(x_1); +if (x_4 == 0) +{ +uint32_t x_5; lean_object* x_6; lean_object* x_7; +x_5 = l_String_Iterator_curr(x_1); +x_6 = lean_box_uint32(x_5); +lean_inc(x_3); +lean_inc(x_2); +x_7 = lean_apply_2(x_3, x_2, x_6); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; +lean_dec(x_3); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_2); +lean_ctor_set(x_8, 1, x_1); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_String_Iterator_next(x_1); +x_1 = x_10; +x_2 = x_9; +goto _start; +} +} +else +{ +lean_object* x_12; +lean_dec(x_3); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_2); +lean_ctor_set(x_12, 1, x_1); +return x_12; +} +} +} +LEAN_EXPORT lean_object* l_String_Iterator_foldUntil(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_String_Iterator_foldUntil___rarg), 3, 0); +return x_2; +} +} lean_object* initialize_Init_Control_Except(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_ByteArray(uint8_t builtin, lean_object*); lean_object* initialize_Init_SimpLemmas(uint8_t builtin, lean_object*); diff --git a/stage0/stdlib/Init/Meta.c b/stage0/stdlib/Init/Meta.c index b0a84c07b1c6..be8086359c42 100644 --- a/stage0/stdlib/Init/Meta.c +++ b/stage0/stdlib/Init/Meta.c @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__9; lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_getSepElems___rarg___boxed(lean_object*); static uint8_t l_Lean_versionString___closed__2; @@ -21,17 +20,17 @@ 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__commandDeclare__simp__like__tactic____________1___closed__73; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__32; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__10; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__13; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decode___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkCIdentFrom(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__3; static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__7; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__6; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_version_getMajor___boxed(lean_object*); lean_object* lean_string_push(lean_object*, uint32_t); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeOctalLitAux___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__81; LEAN_EXPORT lean_object* l_Lean_Syntax_isIdOrAtom_x3f___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10346____boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__2; lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_dsimpKind; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__97; @@ -39,6 +38,7 @@ LEAN_EXPORT lean_object* l_Lean_TSyntax_getChar(lean_object*); LEAN_EXPORT lean_object* l_Lean_instQuoteNameStrAnonymous(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllArith___closed__3; lean_object* l_Lean_extractMacroScopes(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__17; LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef(lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__6; static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__2; @@ -46,20 +46,18 @@ size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Syntax_isNatLit_x3f___boxed(lean_object*); static lean_object* l_Lean_Syntax_unsetTrailing___closed__1; static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__6; -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__19; LEAN_EXPORT lean_object* l_Lean_Syntax_setTailInfoAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTailSepArrayArraySyntax___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__20; static lean_object* l_Lean_Syntax_mkNumLit___closed__2; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__7; LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateFirst___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__2; LEAN_EXPORT uint8_t l_Lean_Meta_DSimp_Config_decide___default; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeDecimalLitAux___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_DSimp_Config_zeta___default; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1___closed__1; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__17; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decodeAfterExp___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_mkSepArray___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__5; @@ -79,11 +77,10 @@ static lean_object* l_Lean_Name_toString_maybePseudoSyntax___closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__11; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Option_hasQuote___rarg___closed__2; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__16; LEAN_EXPORT lean_object* l_Lean_Syntax_getTrailingSize(lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__8; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__90; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__24; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__4; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__10; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__6; static lean_object* l_Lean_Name_reprPrec___closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__12; @@ -95,7 +92,6 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__14; LEAN_EXPORT lean_object* l_Lean_Syntax_getSepArgs___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__38; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_filterSepElemsMAux___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpArith___closed__8; static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__23; @@ -113,6 +109,7 @@ static lean_object* l_Lean_termEval__prio_____closed__9; LEAN_EXPORT lean_object* l_Lean_versionStringCore; static lean_object* l_Lean_versionString___closed__8; LEAN_EXPORT uint32_t l_Lean_idBeginEscape; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__26; LEAN_EXPORT lean_object* l_Lean_instQuote___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__75; @@ -121,6 +118,7 @@ LEAN_EXPORT lean_object* l_Lean_TSyntax_Compat_instCoeTailSyntaxTSyntax(lean_obj lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_instInhabitedEtaStructMode; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__87; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__1; LEAN_EXPORT lean_object* l_Lean_termEval__prio__; static lean_object* l_Array_forInUnsafe_loop___at_Lean_TSyntax_expandInterpolatedStrChunks___spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeQuotedChar(lean_object*, lean_object*); @@ -135,18 +133,18 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__11; static lean_object* l_Lean_quoteNameMk___closed__5; static lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___closed__1; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__8; LEAN_EXPORT lean_object* l_Array_filterSepElemsM___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__12; static lean_object* l_Lean_toolchain___closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__58; lean_object* l_Lean_SourceInfo_fromRef(lean_object*); uint8_t l_String_anyAux_loop(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Name_capitalize(lean_object*); static lean_object* l_Lean_versionString___closed__9; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__16; LEAN_EXPORT lean_object* l_Lean_Syntax_isAtom___boxed(lean_object*); static lean_object* l_Lean_termEval__prec_____closed__6; static lean_object* l_Lean_version_specialDesc___closed__1; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__8; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__68; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__35; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateFirst(lean_object*); @@ -154,27 +152,27 @@ LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeIdentTerm(lean_object*); LEAN_EXPORT lean_object* l_Lean_monadNameGeneratorLift(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapSepElemsM___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_toolchain___closed__9; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__3; extern lean_object* l_Lean_maxRecDepthErrorMessage; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l_panic___at_Lean_TSyntax_getScientific___spec__1___closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__13; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__48; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decodeAfterDot(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_toNat___boxed(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__11; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__6; LEAN_EXPORT uint8_t l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__10; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_memoize___default; static lean_object* l_Lean_toolchain___closed__4; LEAN_EXPORT lean_object* l_Lean_TSyntax_getNat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic__________; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__11; LEAN_EXPORT lean_object* l_Lean_Syntax_getHead_x3f(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__16; static lean_object* l_Lean_instQuoteProdStrAnonymous___rarg___closed__3; static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__8; LEAN_EXPORT uint8_t l_Lean_Meta_DSimp_Config_eta___default; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__20; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__25; LEAN_EXPORT uint8_t l_Lean_Syntax_structEq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTailSepArrayArraySyntax(lean_object*); @@ -187,20 +185,16 @@ LEAN_EXPORT lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__termEva static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__7; static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__14; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeIdentLevel___boxed(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__14; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__68; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5; static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__1; lean_object* lean_string_utf8_prev(lean_object*, lean_object*); static lean_object* l_Lean_instQuoteSubstringStrAnonymous___closed__2; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_isNatLitAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_ofElemsUsingRef___rarg___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__tacticErw______1___closed__40; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__12; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__87; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__7; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__11; lean_object* l_id___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeOctalLitAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instQuote(lean_object*, lean_object*, lean_object*); @@ -218,8 +212,10 @@ static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____ LEAN_EXPORT lean_object* l_Lean_withHeadRefOnly___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__26; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decodeExp(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__11; uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isGreek___boxed(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__16; static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__1; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeBinLitAux(lean_object*, lean_object*, lean_object*); @@ -241,13 +237,12 @@ LEAN_EXPORT lean_object* l_Lean_mkIdentFrom(lean_object*, lean_object*); static lean_object* l_Lean_quoteNameMk___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__1; LEAN_EXPORT uint8_t l_Lean_isIdBeginEscape(uint32_t); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; static lean_object* l_List_foldr___at_Lean_Syntax_decodeNameLit___spec__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_EtaStructMode_toCtorIdx(uint8_t); static lean_object* l_Lean_Syntax_mkNumLit___closed__1; LEAN_EXPORT uint8_t l_Lean_Name_escapePart___lambda__1(uint32_t); -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__7; LEAN_EXPORT lean_object* l_Lean_Syntax_mkScientificLit(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_instInhabitedNat; lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__63; @@ -257,12 +252,10 @@ static lean_object* l_Lean_termEval__prec_____closed__3; static lean_object* l_Lean_Option_hasQuote___rarg___closed__7; static lean_object* l_Lean_TSyntax_expandInterpolatedStr___closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__24; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__15; LEAN_EXPORT lean_object* l_Lean_instQuoteSubstringStrAnonymous___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__9; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__9; LEAN_EXPORT lean_object* l___private_Init_Data_String_Basic_0__Substring_takeWhileAux___at___private_Init_Meta_0__Lean_Syntax_splitNameLitAux___spec__2___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__18; static lean_object* l_Lean_Parser_Tactic_simpAllArith___closed__6; LEAN_EXPORT lean_object* l_Lean_isIdFirst___boxed(lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__4; @@ -273,10 +266,11 @@ LEAN_EXPORT lean_object* l_Lean_Name_toString___boxed(lean_object*, lean_object* lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__27; static lean_object* l_Lean_Syntax_isInterpolatedStrLit_x3f___closed__1; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__14; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__7; lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l_Lean_instQuoteSubstringStrAnonymous___closed__1; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__4; +LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionSepArray(lean_object*); static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__4; LEAN_EXPORT lean_object* l_Lean_version_getSpecialDesc___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeHexDigit___boxed(lean_object*, lean_object*); @@ -284,14 +278,15 @@ lean_object* lean_get_githash(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__19; LEAN_EXPORT lean_object* l_Lean_Syntax_setTailInfo(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__6; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__6; lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__8; static lean_object* l_Lean_instQuoteBoolStrAnonymous___closed__7; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSyntaxArrayArraySyntax(lean_object*); static lean_object* l_Lean_quoteNameMk___closed__4; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_decide___default; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__51; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__31; +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10792____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__59; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__2; lean_object* l_Lean_TSyntaxArray_rawImpl___rarg___boxed(lean_object*); @@ -302,40 +297,43 @@ lean_object* l_Std_Format_joinSep___at_instReprProd___spec__1(lean_object*, lean static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__65; lean_object* l___private_Init_Data_Repr_0__reprSourceInfo____x40_Init_Data_Repr___hyg_1755_(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__39; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__4; LEAN_EXPORT lean_object* l_Array_filterSepElemsM___at_Array_filterSepElems___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10040____boxed(lean_object*, lean_object*); static lean_object* l_Lean_quoteNameMk___closed__9; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_contextual___default; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_TransparencyMode_toCtorIdx(uint8_t); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__13; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__23; lean_object* lean_string_utf8_byte_size(lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_instInhabitedTransparencyMode; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; LEAN_EXPORT lean_object* l_Lean_NameGenerator_namePrefix___default; static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__16; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__9; 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__commandDeclare__simp__like__tactic____________1___lambda__1___closed__82; -LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(uint8_t, uint8_t); +LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Syntax_setHeadInfo(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__61; static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__8; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeTSyntaxConsSyntaxNodeKindNil(lean_object*, lean_object*); static lean_object* l_Lean_toolchain___closed__5; uint8_t lean_usize_dec_lt(size_t, size_t); +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Option_hasQuote___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_version_patch; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__8; static lean_object* l___private_Init_Meta_0__Lean_quoteList___rarg___closed__5; static lean_object* l_Lean_versionString___closed__11; LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Syntax_decodeNameLit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_isNatLitAux___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeTSyntaxConsSyntaxNodeKind(lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13; LEAN_EXPORT lean_object* l_Lean_withHeadRefOnly___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Name_instDecidableEqName(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__61; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__8; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____boxed(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_Lean_version_specialDesc; @@ -345,6 +343,7 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_mkSep___boxed(lean_object*, lean_object*) LEAN_EXPORT lean_object* l_Lean_Syntax_decodeQuotedChar___boxed__const__6; LEAN_EXPORT lean_object* l_Lean_isSubScriptAlnum___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_mapSepElems(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__9; static lean_object* l_Lean_Meta_DSimp_instBEqConfig___closed__1; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__5; static lean_object* l_Lean_versionStringCore___closed__2; @@ -353,7 +352,7 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_Lean_TSyntax_getNat___closed__3; LEAN_EXPORT lean_object* l_Lean_Name_instReprName; static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__5; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__3; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__59; LEAN_EXPORT lean_object* l_Lean_Name_toStringWithSep(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__7; @@ -361,7 +360,6 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_ofElems(lean_object*, lean_object*); static lean_object* l_Lean_Name_escapePart___closed__4; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__19; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__11; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__82; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSepArrayTSyntaxArray(lean_object*, lean_object*); @@ -374,12 +372,12 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_Lean_termEval__prio_____closed__4; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__51; static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__15; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__1; static lean_object* l_Lean_version_major___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_EtaStructMode_toCtorIdx___boxed(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_expandInterpolatedStr___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__6; static lean_object* l_Lean_Option_hasQuote___rarg___closed__4; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__12; static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__7; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_etaStruct___default; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__45; @@ -392,14 +390,17 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_Lean_termEval__prio_____closed__2; LEAN_EXPORT lean_object* l_Lean_TSyntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_expandInterpolatedStrChunks___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__1; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__1; LEAN_EXPORT lean_object* l_Lean_Name_toStringWithSep_maybeEscape(uint8_t, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__25; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__83; LEAN_EXPORT lean_object* l_Lean_Syntax_isLit_x3f___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__3; LEAN_EXPORT uint8_t l_Lean_Meta_DSimp_Config_proj___default; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__39; LEAN_EXPORT lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrio__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionTSepArray___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_hasArgs___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__4; static lean_object* l_Lean_Name_reprPrec___closed__6; @@ -412,10 +413,10 @@ LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_singlePass___default; LEAN_EXPORT lean_object* l_Lean_Syntax_mkApp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapSepElems___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__40; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__7; LEAN_EXPORT lean_object* l_Lean_Syntax_instBEqTSyntax___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__67; LEAN_EXPORT lean_object* l_Lean_Meta_Simp_Config_maxSteps___default; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_getElems___rarg___boxed(lean_object*); static lean_object* l_Lean_TSyntax_expandInterpolatedStrChunks___closed__1; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_version_getMinor___boxed(lean_object*); @@ -431,7 +432,6 @@ static lean_object* l_Lean_termEval__prec_____closed__10; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__69; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decodeExp___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_isLit_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Name_reprPrec___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Simp_instInhabitedConfig; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__17; @@ -445,7 +445,6 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_isNatLit_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_Compat_instCoeTailArraySyntaxTSyntaxArray(lean_object*); static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__5; LEAN_EXPORT lean_object* l_Lean_version_major; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__94; LEAN_EXPORT lean_object* l_Lean_Syntax_instBEqSyntax; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_zeta___default; @@ -462,10 +461,9 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_ofElemsUsingRef___rarg___lambda_ static lean_object* l_Lean_Name_appendIndexAfter___closed__1; uint8_t l_instDecidableNot___rarg(uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_neutralConfig; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__18; uint8_t l_String_contains(lean_object*, uint32_t); +LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_push___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__1; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__15; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); static lean_object* l_Lean_instQuoteBoolStrAnonymous___closed__5; LEAN_EXPORT lean_object* l_Lean_Syntax_mkStrLit___boxed(lean_object*, lean_object*); @@ -475,8 +473,10 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__17; static lean_object* l_Lean_instQuoteBoolStrAnonymous___closed__3; static lean_object* l_Lean_termEval__prec_____closed__7; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__4; static lean_object* l_Lean_Parser_Tactic_simpAllArith___closed__9; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__83; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__3; static lean_object* l_Lean_instQuoteSubstringStrAnonymous___closed__4; LEAN_EXPORT lean_object* l_Lean_instQuoteNatNumLitKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeScientificLitTerm___boxed(lean_object*); @@ -485,6 +485,7 @@ LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeDecimalLitAu LEAN_EXPORT lean_object* l_Array_mapSepElemsM(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkGroupNode(lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__2; static lean_object* l_Lean_termEval__prio_____closed__1; static lean_object* l_Lean_mkGroupNode___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__35; @@ -495,11 +496,9 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_Lean_Name_reprPrec___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decode(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_mkGroupNode___closed__2; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__8; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_mapSepElemsMAux(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_mkCApp(lean_object*, lean_object*); static lean_object* l_Lean_Syntax_mkNameLit___closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; static lean_object* l_Lean_termEval__prio_____closed__6; static lean_object* l_Lean_versionStringCore___closed__5; LEAN_EXPORT lean_object* l_Lean_Syntax_isStrLit_x3f(lean_object*); @@ -509,33 +508,33 @@ static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__70; LEAN_EXPORT lean_object* l_Array_getSepElems(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_String_Basic_0__Substring_takeWhileAux___at___private_Init_Meta_0__Lean_Syntax_splitNameLitAux___spec__3(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__11; static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__19; LEAN_EXPORT lean_object* l_Lean_monadNameGeneratorLift___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_getElems(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10701____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_structEq___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__5; static lean_object* l_panic___at_Lean_TSyntax_getScientific___spec__1___closed__1; -LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10701_(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10792_(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Simp_ConfigCtx_contextual___default; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____lambda__1___closed__1; LEAN_EXPORT lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_quoteList___rarg(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__8; LEAN_EXPORT lean_object* l_Lean_Syntax_isFieldIdx_x3f(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__36; LEAN_EXPORT lean_object* l_Lean_TSyntax_expandInterpolatedStr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSyntaxArrayTSepArray___boxed(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__20; LEAN_EXPORT lean_object* l_Lean_instQuoteStringStrLitKind(lean_object*); lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_ofElems___boxed(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__17; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__36; -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeHexLitAux(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1___closed__4; LEAN_EXPORT uint8_t l_Lean_isNumericSubscript(uint32_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_mkSepArray___spec__1___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__10; +LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionSepArray___boxed(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; LEAN_EXPORT lean_object* l_Lean_Syntax_isScientificLit_x3f(lean_object*); static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__1; LEAN_EXPORT lean_object* l_Lean_Name_toString(lean_object*, uint8_t); @@ -544,26 +543,27 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_Lean_toolchain___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_DSimp_instInhabitedConfig; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__17; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__17; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instReprTransparencyMode; static lean_object* l_Lean_Parser_Tactic_simpAllArith___closed__4; LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshId___rarg(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__4; lean_object* l_String_capitalize(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_TSyntax_getString___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_NameGenerator_next(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_decodeCharLit___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_decodeNatLitVal_x3f(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056_(uint8_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147_(uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_getElems___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__10; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Syntax_getTailInfo_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_Compat_instCoeTailSyntaxTSyntax___boxed(lean_object*); static lean_object* l_Lean_mkNullNode___closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__10; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__19; static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__6; +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Option_hasQuote___rarg___closed__6; extern lean_object* l_Lean_Parser_Tactic_simpStar; static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__11; @@ -573,26 +573,24 @@ LEAN_EXPORT uint8_t l_Lean_Internal_isStage0(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__94; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__31; static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__20; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__6; static lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_withHeadRefOnly___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_TransparencyMode_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__5; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__22; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__12; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeStrLitTerm(lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_expandInterpolatedStrChunks(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_setKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* lean_name_append_index_after(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__1; LEAN_EXPORT lean_object* l_Lean_Name_eraseSuffix_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Simp_instReprConfig___closed__1; LEAN_EXPORT lean_object* l_Array_getSepElems___rarg(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__14; extern lean_object* l_Lean_reservedMacroScope; static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__6; static lean_object* l_Lean_Syntax_instCoeIdentTSyntaxConsSyntaxNodeKindStrAnonymousNil___closed__3; static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__10; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__8; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__7; static lean_object* l_Lean_Syntax_unsetTrailing___closed__2; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__10; static lean_object* l_Lean_NameGenerator_namePrefix___default___closed__1; @@ -603,7 +601,6 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_Lean_Name_instToStringName(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__90; static lean_object* l_Lean_quoteNameMk___closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__21; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__38; static lean_object* l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg___closed__4; @@ -615,8 +612,11 @@ 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__commandDeclare__simp__like__tactic____________1___closed__72; LEAN_EXPORT lean_object* l_Lean_instQuote___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Rewrite_Config_transparency___default; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__8; lean_object* l_Nat_repr(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7; LEAN_EXPORT lean_object* l_Array_mapSepElemsM___at_Array_mapSepElems___spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__96; static lean_object* l___private_Init_Meta_0__Lean_Syntax_splitNameLitAux___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -628,17 +628,15 @@ static lean_object* l_Lean_mkNullNode___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__23; static lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1___closed__1; static lean_object* l_Lean_instQuoteBoolStrAnonymous___closed__6; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__10; static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__3; static lean_object* l_Lean_versionStringCore___closed__8; static lean_object* l_Lean_Name_instReprSyntax___closed__1; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__64; LEAN_EXPORT lean_object* l_Lean_Internal_isStage0___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__10; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__34; LEAN_EXPORT lean_object* l_Lean_instQuoteArrayStrAnonymous___rarg(lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__16; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSyntaxArrayTSepArray(lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_splitNameLitAux(lean_object*, lean_object*); @@ -647,17 +645,15 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNameLitTerm(lean_object*); static lean_object* l_Lean_versionStringCore___closed__4; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeInterpStrQuotedChar___boxed(lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__2; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Parser_Tactic_rwRuleSeq; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__88; static lean_object* l_Lean_instQuoteArrayStrAnonymous___rarg___closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__74; static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__12; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__10; static lean_object* l_Lean_Syntax_instBEqSyntax___closed__1; static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__19; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__89; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__20; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__47; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeTSyntaxConsSyntaxNodeKind___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_NameGenerator_idx___default; @@ -667,7 +663,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_EtaStructMode_noConfusion___rarg___boxed(le static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__6; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__60; static lean_object* l_Lean_Meta_instBEqTransparencyMode___closed__1; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__2; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__9; 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*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1___closed__6; lean_object* lean_array_to_list(lean_object*, lean_object*); @@ -679,9 +675,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_TransparencyMode_toCtorIdx___boxed(lean_obj LEAN_EXPORT lean_object* l_Lean_mkCIdent(lean_object*); static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__16; LEAN_EXPORT lean_object* l_Lean_version_getIsRelease___boxed(lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_dsimp___default; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; 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_simpArithAutoUnfold___closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__1; @@ -707,17 +701,22 @@ LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_version_getPatch___boxed( static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__12; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001_(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__81; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__16; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__13; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_copyHeadTailInfoFrom(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_TSyntax_getChar___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeIdentTSyntaxConsSyntaxNodeKindStrAnonymousNil(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSyntaxArray(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_pred(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__5; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeHexLitAux___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_filterSepElemsMAux(lean_object*); static lean_object* l_Lean_Name_reprPrec___closed__4; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__72; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__4; static lean_object* l_Lean_instQuoteBoolStrAnonymous___closed__1; +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____boxed(lean_object*, lean_object*); lean_object* l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(lean_object*); static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__9; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__23; @@ -730,13 +729,13 @@ static lean_object* l_Lean_version_patch___closed__1; uint8_t l_Array_isEmpty___rarg(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__60; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTermTSyntaxConsSyntaxNodeKindStrAnonymousNil___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282_(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_20090_(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132_(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222_(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19156_(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226_(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17170_(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391_(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_20199_(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241_(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331_(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_19265_(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335_(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_17279_(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__88; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__47; uint8_t l_Substring_beq(lean_object*, lean_object*); @@ -751,25 +750,23 @@ extern lean_object* l_Lean_instInhabitedSyntax; LEAN_EXPORT lean_object* l_Lean_version_getSpecialDesc(lean_object*); static lean_object* l_Lean_toolchain___closed__6; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__41; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__6; static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrio__1___closed__2; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__17; static lean_object* l_Lean_version_minor___closed__1; static lean_object* l_Lean_Name_reprPrec___closed__9; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__96; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__22; LEAN_EXPORT lean_object* l_Lean_mkCIdentFromRef___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__4; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__9; LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_ofElemsUsingRef___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_Config_maxDischargeDepth___default; LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_getElems(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isNumericSubscript___boxed(lean_object*); lean_object* l_Substring_nextn(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__16; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__5; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__14; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__8; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11; LEAN_EXPORT lean_object* l_Lean_evalOptPrio(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__10; static lean_object* l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg___closed__3; @@ -778,62 +775,58 @@ LEAN_EXPORT lean_object* l_Lean_instQuoteProdStrAnonymous(lean_object*, lean_obj static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__25; 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_Syntax_mkApp___closed__2; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__1; LEAN_EXPORT lean_object* l_Lean_NameGenerator_mkChild(lean_object*); LEAN_EXPORT lean_object* l_Lean_getGithash___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instReprEtaStructMode; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__6; static lean_object* l_Lean_Syntax_isCharLit_x3f___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__86; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateFirst___at_Lean_Syntax_setHeadInfoAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNumLitTerm___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__46; lean_object* l_String_dropRight(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_isCharLit_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_splitNameLit(lean_object*); static lean_object* l___private_Init_Meta_0__Lean_quoteList___rarg___closed__6; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__13; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__38; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__21; -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10255____boxed(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__23; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeInterpStrLit(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__6; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__4; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__6; LEAN_EXPORT lean_object* l_Lean_version_minor; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeStrLit___boxed(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422_(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__8; +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_mapSepElemsMAux___at_Array_mapSepElems___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_NameGenerator_namePrefix___default___closed__2; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9; +LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionTSepArray(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_isIdEndEscape(uint32_t); -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__5; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__52; static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__4; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__50; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_version_getMajor(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_TSyntax_getScientific___spec__1(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__2; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_decodeNatLitVal_x3f___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__14; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeCharLit(lean_object*); LEAN_EXPORT uint8_t l_Lean_version_isRelease; -LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10255_(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10346_(lean_object*, lean_object*); static lean_object* l_Lean_Syntax_decodeNatLitVal_x3f___closed__1; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_arith___default; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_TransparencyMode_noConfusion___rarg(uint8_t, uint8_t, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__18; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__29; static lean_object* l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg___closed__1; static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrio__1___closed__1; uint8_t l_Char_isAlpha(uint32_t); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__7; static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__8; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__14; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__1; LEAN_EXPORT lean_object* l_Lean_Option_hasQuote(lean_object*); LEAN_EXPORT uint8_t l_Lean_Syntax_isAtom(lean_object*); static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__5; @@ -843,6 +836,10 @@ LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeDepTermMkConsSyntaxNodeKindStrAno static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__15; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__37; LEAN_EXPORT uint8_t l_Lean_isLetterLike(uint32_t); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__2; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__4; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__14; LEAN_EXPORT uint8_t l_Lean_Meta_DSimp_Config_beta___default; LEAN_EXPORT lean_object* l_Lean_evalPrec(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_isStrLit_x3f___boxed(lean_object*); @@ -850,12 +847,13 @@ static lean_object* l_Lean_Syntax_getHead_x3f___closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__80; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__6; lean_object* l_Lean_Macro_expandMacro_x3f(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_simpArith; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__15; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__9; extern lean_object* l_Lean_Parser_Tactic_simpLemma; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__14; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__34; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__55; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__9; lean_object* l_Lean_mkAtomFrom(lean_object*, lean_object*); lean_object* l_Lean_TSyntaxArray_mkImpl___rarg___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__48; @@ -865,12 +863,13 @@ extern uint32_t l_Char_instInhabitedChar; static lean_object* l_Lean_instInhabitedNameGenerator___closed__1; static lean_object* l_Lean_Meta_TransparencyMode_noConfusion___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__21; LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_ofElemsUsingRef(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__5; static lean_object* l_Lean_versionString___closed__7; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__3; static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__13; LEAN_EXPORT lean_object* l_Lean_Syntax_unsetTrailing(lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; static lean_object* l_Lean_termEval__prio_____closed__7; static lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_isLetterLike___boxed(lean_object*); @@ -880,18 +879,16 @@ LEAN_EXPORT lean_object* l_Lean_Syntax_isIdOrAtom_x3f(lean_object*); static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__13; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSyntaxArray___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNumLitPrec___boxed(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__5; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__4; LEAN_EXPORT lean_object* l_Lean_mkIdentFromRef___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; 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___private_Init_Meta_0__Lean_Name_beq_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_decodeQuotedChar___boxed__const__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__50; -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____boxed(lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__11; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__4; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; static lean_object* l_Lean_Syntax_mkApp___closed__1; uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__24; @@ -902,9 +899,9 @@ static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____ lean_object* l_String_intercalate(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_EtaStructMode_noConfusion(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__25; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__22; static lean_object* l_Lean_Syntax_instCoeIdentTSyntaxConsSyntaxNodeKindStrAnonymousNil___closed__1; static lean_object* l_Lean_Syntax_instCoeTSepArrayTSyntaxArray___closed__1; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__14; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSepArrayTSyntaxArray___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Syntax_mkNameLit___closed__1; LEAN_EXPORT uint8_t l_Lean_version_getIsRelease(lean_object*); @@ -913,28 +910,24 @@ LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_version_getMinor(lean_obj LEAN_EXPORT lean_object* l_Lean_Syntax_getSepArgs(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__80; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__6; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__2; uint8_t l_String_isEmpty(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__5; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__25; extern uint8_t l_instInhabitedBool; LEAN_EXPORT lean_object* l_Lean_Meta_TransparencyMode_noConfusion(lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg___closed__2; static lean_object* l_Lean_TSyntax_expandInterpolatedStr___lambda__1___closed__4; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__4; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__5; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__1; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__1; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__9; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__6; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__14; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__28; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__21; static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__7; LEAN_EXPORT lean_object* l_Lean_mkHole(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_getSepElems___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_isEqvAux___at_Lean_Syntax_structEq___spec__1(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__tacticErw______1___closed__20; lean_object* l_Lean_Syntax_setArg(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__13; static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__29; LEAN_EXPORT lean_object* l_Lean_instQuoteListStrAnonymous(lean_object*); @@ -943,10 +936,11 @@ static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__9; 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 uint8_t l_Lean_Meta_Simp_Config_eta___default; static lean_object* l_Lean_instQuoteBoolStrAnonymous___closed__4; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__21; static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__10; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTermTSyntaxConsSyntaxNodeKindStrAnonymousNil(lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__20; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__1; +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10131____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__8; LEAN_EXPORT uint8_t l_Lean_Syntax_hasArgs(lean_object*); static lean_object* l_Lean_toolchain___closed__1; @@ -962,7 +956,6 @@ LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_quoteList(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__15; static lean_object* l_Lean_Syntax_isFieldIdx_x3f___closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__3; LEAN_EXPORT lean_object* l_Lean_withHeadRefOnly(lean_object*); lean_object* l_String_quote(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__5; @@ -975,13 +968,15 @@ static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__22; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__18; LEAN_EXPORT lean_object* l_Lean_Meta_Simp_instReprConfig; LEAN_EXPORT lean_object* l_Lean_instInhabitedNameGenerator; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__11; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__40; LEAN_EXPORT uint8_t l_Lean_Syntax_instBEqTSyntax___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__67; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__9; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__23; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__10; static lean_object* l_Lean_TSyntax_getNat___closed__2; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__5; lean_object* l_Lean_Syntax_getArgs(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*); static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__8; @@ -995,38 +990,42 @@ lean_object* l_Lean_Syntax_getKind(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllArith___closed__8; LEAN_EXPORT lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__subPrec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MacroScopesView_review(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__4; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__3; LEAN_EXPORT lean_object* l_Lean_quoteNameMk(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeInterpStrQuotedChar___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNumLitPrio___boxed(lean_object*); static lean_object* l_Lean_toolchain___closed__2; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15; LEAN_EXPORT lean_object* l_Array_filterSepElems(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapSepElemsM___at_Array_mapSepElems___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__53; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__42; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__22; static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__1; -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071_(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Name_hasNum(lean_object*); static lean_object* l_Lean_Syntax_mkScientificLit___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__93; LEAN_EXPORT lean_object* l_Lean_Meta_instBEqEtaStructMode; static lean_object* l_Lean_Syntax_mkScientificLit___closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__5; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__9; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__9; lean_object* l_panic___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Name_isInaccessibleUserName___boxed(lean_object*); static uint8_t l_Lean_versionString___closed__3; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__3; LEAN_EXPORT lean_object* l_Lean_Name_replacePrefix___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__91; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; static lean_object* l_Lean_versionString___closed__5; LEAN_EXPORT lean_object* l_Lean_TSyntax_getScientific(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__15; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__78; static lean_object* l_Lean_termEval__prec_____closed__11; LEAN_EXPORT lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__4___boxed(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__7; LEAN_EXPORT lean_object* l_Lean_Syntax_getOptionalIdent_x3f(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_TSyntax_getChar___spec__1___boxed__const__1; static lean_object* l_Lean_evalPrec___closed__1; @@ -1037,27 +1036,32 @@ static lean_object* l_Lean_Name_toStringWithSep___closed__1; LEAN_EXPORT lean_object* l_Lean_NameGenerator_curr(lean_object*); static lean_object* l_Lean_Parser_Tactic_dsimpKind___closed__3; static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__4; +LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_push___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_SepArray_getElems___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_DSimp_instBEqConfig; +LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_push(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__18; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_TSyntax_expandInterpolatedStrChunks___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__17; static lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1___lambda__1___closed__7; -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891_(uint8_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982_(uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_isNameLit_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_instQuoteBoolStrAnonymous___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_mapSepElemsMAux___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__5; LEAN_EXPORT lean_object* l_Lean_instQuoteListStrAnonymous___rarg(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__1; static lean_object* l_Lean_mkHole___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__64; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__6; static lean_object* l_Lean_Syntax_mkApp___closed__3; -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_versionStringCore___closed__6; LEAN_EXPORT lean_object* l_Lean_isIdBeginEscape___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__6; static lean_object* l_Lean_instQuoteNameStrAnonymous___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__54; static lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__2; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__6; LEAN_EXPORT lean_object* l_Lean_mkFreshId___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instQuoteBoolStrAnonymous___closed__2; LEAN_EXPORT uint8_t l_Lean_Meta_Rewrite_Config_offsetCnstrs___default; @@ -1068,11 +1072,11 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__12; static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__subPrio__1___closed__1; LEAN_EXPORT lean_object* l_List_beq___at_Lean_Syntax_structEq___spec__2___boxed(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__6; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__23; lean_object* lean_nat_mul(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__7; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__12; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__91; LEAN_EXPORT lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpArithAutoUnfold___closed__9; @@ -1102,6 +1106,7 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_Lean_Syntax_setInfo(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__13; static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__24; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__24; LEAN_EXPORT lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__15; LEAN_EXPORT lean_object* l_panic___at_Lean_TSyntax_getNat___spec__1(lean_object*); @@ -1114,10 +1119,11 @@ static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean LEAN_EXPORT lean_object* l_List_beq___at_Lean_Syntax_structEq___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_decodeScientificLitVal_x3f_decodeAfterDot___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Name_toString_maybePseudoSyntax___boxed(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__12; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__3; LEAN_EXPORT lean_object* l_Lean_expandMacros(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_updateLast(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__10; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeNameLit(lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__7; static lean_object* l_Lean_Name_toString_maybePseudoSyntax___closed__1; @@ -1135,16 +1141,16 @@ lean_object* l_String_trim(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__24; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeQuotedChar___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isIdEndEscape___boxed(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__20; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__10; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_mkSepArray___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_getTailInfo_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_getTailInfo(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_getOptionalIdent_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeStrLitTerm___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__18; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__14; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__79; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__7; static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__15; LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Syntax_decodeNameLit___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_termEval__prec_____closed__5; @@ -1154,18 +1160,19 @@ LEAN_EXPORT lean_object* l_Lean_mkCIdentFromRef(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__49; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__95; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeStrLit(lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__12; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__76; LEAN_EXPORT uint8_t l_Lean_isIdFirst(uint32_t); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__16; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_isNone___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_getString(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNameLitTerm___boxed(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__6; LEAN_EXPORT lean_object* l_Lean_TSyntax_getName(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__18; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__1; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__19; LEAN_EXPORT lean_object* l_Lean_Syntax_isToken___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__15; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeTSyntaxConsSyntaxNodeKind___rarg(lean_object*); @@ -1176,6 +1183,7 @@ extern lean_object* l_Lean_Parser_Tactic_simpErase; static lean_object* l_Lean_mkCIdentFrom___closed__1; static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_getElems___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__4; LEAN_EXPORT lean_object* l_Lean_Syntax_getTailInfo___boxed(lean_object*); static lean_object* l_Lean_TSyntax_expandInterpolatedStr___closed__5; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeIdentTerm___boxed(lean_object*); @@ -1183,7 +1191,6 @@ static lean_object* l_Lean_termEval__prec_____closed__8; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeQuotedChar___boxed__const__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__85; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__12; static lean_object* l_Lean_toolchain___closed__7; static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrec__1___closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__56; @@ -1193,6 +1200,7 @@ LEAN_EXPORT lean_object* l_Lean_origin; static lean_object* l_Lean_Syntax_isInterpolatedStrLit_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Name_instReprSyntax; lean_object* lean_string_length(lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Syntax_findAux___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_String_Basic_0__Substring_takeWhileAux___at___private_Init_Meta_0__Lean_Syntax_splitNameLitAux___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__10; @@ -1201,10 +1209,12 @@ LEAN_EXPORT lean_object* l_Lean_instQuoteTermStrAnonymous; static lean_object* l_Lean_Name_reprPrec___closed__10; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_beta___default; LEAN_EXPORT lean_object* l_Lean_Syntax_getHead_x3f___lambda__1(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__12; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__3; static lean_object* l_Lean_Option_hasQuote___rarg___closed__3; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__4; LEAN_EXPORT uint8_t l_List_beq___at_Lean_Syntax_structEq___spec__2(lean_object*, lean_object*); static lean_object* l_Lean_TSyntax_expandInterpolatedStr___lambda__1___closed__1; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__12; LEAN_EXPORT lean_object* l_Lean_withHeadRefOnly___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* lean_mk_syntax_ident(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__70; @@ -1212,6 +1222,7 @@ extern lean_object* l_Lean_Parser_Tactic_discharger; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_TransparencyMode_noConfusion___rarg___lambda__1(lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__71; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__15; static lean_object* l_Lean_Syntax_getHead_x3f___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_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__42; @@ -1222,6 +1233,7 @@ lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lean_termEval__prec_____closed__1; LEAN_EXPORT lean_object* l_Lean_Syntax_toNat(lean_object*); static lean_object* l_Lean_versionString___closed__6; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__18; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__37; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__53; LEAN_EXPORT lean_object* lean_name_append_before(lean_object*, lean_object*); @@ -1234,11 +1246,15 @@ static lean_object* l_Lean_mkCIdentFrom___closed__2; static lean_object* l_Lean_origin___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold; lean_object* lean_nat_mod(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__14; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__37; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5; static lean_object* l_Lean_TSyntax_getNat___closed__1; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_dsimpAutoUnfold; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__55; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__16; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__22; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__6; lean_object* l_Lean_SourceInfo_getPos_x3f(lean_object*, uint8_t); static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__6; @@ -1246,48 +1262,47 @@ LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_filterSepElemsMAux___at_ static lean_object* l_Lean_Meta_Simp_instBEqConfig___closed__1; LEAN_EXPORT lean_object* l_Lean_mkFreshId___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_termEval__prec_____closed__4; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_proj___default; -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_instBEqTransparencyMode; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeArraySyntaxSepArray(lean_object*); static lean_object* l_Lean_instQuoteTermStrAnonymous___closed__1; +static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__16; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1___closed__1; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__11; static lean_object* l_Lean_Option_hasQuote___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_instQuoteStringStrLitKind___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_find_x3f(lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__6; static lean_object* l_Lean_Parser_Tactic_tacticErw_______closed__12; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__63; LEAN_EXPORT lean_object* l_Lean_Syntax_decodeStrLitAux___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); lean_object* l_String_drop(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__7; -LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10040_(uint8_t, uint8_t); +LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10131_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeTSyntaxConsSyntaxNodeKindNil___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_filterSepElemsM___at_Array_filterSepElems___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAllAutoUnfold___closed__9; -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__17; LEAN_EXPORT lean_object* l_Lean_monadNameGeneratorLift___rarg___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__71; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__15; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__13; static lean_object* l_Lean_TSyntax_expandInterpolatedStr___closed__2; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__1; static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__14; LEAN_EXPORT lean_object* l_Lean_instQuoteArrayStrAnonymous(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__16; lean_object* l_Nat_min(lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__18; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__1; static lean_object* l___private_Init_Meta_0__Lean_quoteList___rarg___closed__4; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__33; static lean_object* l_Lean_mkSepArray___closed__1; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__5; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__10; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__8; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__3; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__12; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_TSyntax_expandInterpolatedStrChunks___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_Syntax_instCoeTSyntaxArrayArraySyntax___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Name_getRoot___boxed(lean_object*); @@ -1300,10 +1315,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__commandDeclare__simp__like__tactic____________1___closed__79; LEAN_EXPORT lean_object* l_Lean_mkSepArray___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__43; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__15; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__18; static lean_object* l_Lean_Syntax_instCoeTSyntaxArrayArraySyntax___closed__1; static lean_object* l_Lean_Name_reprPrec___closed__3; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__11; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__46; static lean_object* l___private_Init_Meta_0__Lean_quoteList___rarg___closed__2; LEAN_EXPORT uint8_t l_Lean_Name_toString_maybePseudoSyntax(lean_object*); @@ -1314,20 +1328,18 @@ static lean_object* l_Lean_termEval__prec_____closed__9; LEAN_EXPORT lean_object* l_Lean_Meta_TransparencyMode_noConfusion___rarg___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNumLitPrec(lean_object*); static lean_object* l_Array_getSepElems___rarg___closed__1; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__21; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_getSepElems___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Parser_Tactic_commandDeclare__simp__like__tactic_____________closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__95; static lean_object* l_Lean_Parser_Tactic_simpAllArith___closed__7; LEAN_EXPORT lean_object* l_Lean_Syntax_findAux(lean_object*, lean_object*); static lean_object* l_Lean_Name_escapePart___closed__3; +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__3; LEAN_EXPORT lean_object* l_Lean_Syntax_instCoeTSyntaxArrayTSepArray___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_decodeStrLitAux(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__49; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__10; uint8_t lean_string_utf8_at_end(lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__8; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__2; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__7; LEAN_EXPORT lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3(lean_object*); @@ -1335,9 +1347,9 @@ static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Me LEAN_EXPORT lean_object* l_Lean_mkNode(lean_object*, lean_object*); static lean_object* l___private_Init_Meta_0__Lean_quoteList___rarg___closed__1; static lean_object* l_Lean_instQuoteSubstringStrAnonymous___closed__3; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; lean_object* lean_uint32_to_nat(uint32_t); static lean_object* l_Array_forInUnsafe_loop___at_Lean_mkSepArray___spec__1___closed__1; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__17; LEAN_EXPORT lean_object* l_Lean_Name_replacePrefix(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_termEval__prio_____closed__5; LEAN_EXPORT lean_object* l_Lean_TSyntax_instCoeNumLitPrio(lean_object*); @@ -1352,31 +1364,27 @@ LEAN_EXPORT lean_object* l_Lean_TSyntax_expandInterpolatedStr___boxed(lean_objec static lean_object* l_List_foldr___at_Lean_Syntax_decodeNameLit___spec__1___closed__4; lean_object* lean_nat_to_int(lean_object*); LEAN_EXPORT uint8_t l_Lean_Syntax_isToken(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__15; LEAN_EXPORT lean_object* l_Lean_Syntax_isFieldIdx_x3f___boxed(lean_object*); static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__24; LEAN_EXPORT uint8_t l_Lean_Meta_Simp_Config_autoUnfold___default; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__92; LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Name_beq_match__1_splitter(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Syntax_decodeInterpStrLit___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__12; LEAN_EXPORT lean_object* l_Lean_evalPrio(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__18; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__32; static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__5; +LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_defaultMaxSteps; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__10; -static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__4; static lean_object* l_Lean___aux__Init__Meta______macroRules__Lean__Parser__Syntax__addPrec__1___closed__4; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__13; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__12; LEAN_EXPORT lean_object* l___private_Init_Data_String_Basic_0__Substring_takeWhileAux___at___private_Init_Meta_0__Lean_Syntax_splitNameLitAux___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__18; LEAN_EXPORT lean_object* l_Lean_TSyntax_Compat_instCoeTailArraySyntaxTSyntaxArray___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_setHeadInfoAux(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__20; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__9; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__2; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__30; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__77; LEAN_EXPORT lean_object* l_Lean_Option_hasQuote___rarg(lean_object*, lean_object*); @@ -1391,35 +1399,35 @@ static lean_object* l_Lean_Meta_Simp_instInhabitedConfig___closed__1; static lean_object* l_Lean_TSyntax_expandInterpolatedStr___lambda__1___closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__54; static lean_object* l_Lean_Syntax_instCoeIdentTSyntaxConsSyntaxNodeKindStrAnonymousNil___closed__2; -static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__3; static lean_object* l_Lean_Parser_Tactic_simpAllKind___closed__1; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__3; 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__tacticErw______1___closed__29; 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*); -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Syntax_isFieldIdx_x3f___closed__1; LEAN_EXPORT uint8_t l_Lean_isIdRest(uint32_t); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__43; static lean_object* l_Lean_Parser_Tactic_simpAllArithAutoUnfold___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_DSimp_instReprConfig; -static lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__3; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__66; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___lambda__1___closed__56; static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__33; static lean_object* l_repr___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__3___closed__9; static lean_object* l_Lean_Parser_Tactic_simpAutoUnfold___closed__9; -static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__1; +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_mkLit(lean_object*, lean_object*, lean_object*); lean_object* l_Char_ofNat(lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__7; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Meta_0__Array_mapSepElemsMAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_versionStringCore___closed__7; static lean_object* l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__22; +static lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__6; LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____spec__5___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__62; lean_object* l_Repr_addAppParen(lean_object*, lean_object*); +static lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__7; static lean_object* l_Lean_Parser_Tactic_simpArith___closed__2; LEAN_EXPORT lean_object* l___private_Init_Data_String_Basic_0__Substring_takeWhileAux___at___private_Init_Meta_0__Lean_Syntax_splitNameLitAux___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__15; @@ -6621,7 +6629,7 @@ static lean_object* _init_l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg___closed__1; x_2 = l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Init_Meta_0__Lean_Syntax_updateLast___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -16545,6 +16553,85 @@ lean_dec(x_1); return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_push___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = l_Array_isEmpty___rarg(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_box(2); +x_6 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_6, 0, x_5); +lean_ctor_set(x_6, 1, x_1); +x_7 = lean_array_push(x_2, x_6); +x_8 = lean_array_push(x_7, x_3); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_Lean_mkOptionalNode___closed__2; +x_10 = lean_array_push(x_9, x_3); +return x_10; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_push(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Syntax_TSepArray_push___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Syntax_TSepArray_push___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Syntax_TSepArray_push(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionSepArray(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_mkSepArray___closed__1; +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionSepArray___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Syntax_instEmptyCollectionSepArray(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionTSepArray(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_mkSepArray___closed__1; +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Syntax_instEmptyCollectionTSepArray___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Syntax_instEmptyCollectionTSepArray(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} static lean_object* _init_l_Lean_Syntax_instCoeTailSepArrayArraySyntax___closed__1() { _start: { @@ -17995,7 +18082,7 @@ x_1 = 0; return x_1; } } -LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(uint8_t x_1, uint8_t x_2) { +LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(uint8_t x_1, uint8_t x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -18007,7 +18094,7 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966____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; @@ -18015,7 +18102,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_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_3, x_4); +x_5 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_3, x_4); x_6 = lean_box(x_5); return x_6; } @@ -18024,7 +18111,7 @@ static lean_object* _init_l_Lean_Meta_instBEqTransparencyMode___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966____boxed), 2, 0); return x_1; } } @@ -18036,7 +18123,7 @@ x_1 = l_Lean_Meta_instBEqTransparencyMode___closed__1; return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__1() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__1() { _start: { lean_object* x_1; @@ -18044,33 +18131,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.TransparencyMode.all", 30); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__2() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__1; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__1; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__3() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__2; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__2; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__4() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__4() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__3; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__3; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18078,23 +18165,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__5() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__6; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__2; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__2; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__6() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__6() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__5; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__5; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18102,7 +18189,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__7() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__7() { _start: { lean_object* x_1; @@ -18110,33 +18197,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.TransparencyMode.default", 34); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__8() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__7; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__7; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__9() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__8; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__8; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__10() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__10() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__9; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__9; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18144,23 +18231,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__11() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__6; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__8; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__8; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__12() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__12() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__11; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__11; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18168,7 +18255,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__13() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__13() { _start: { lean_object* x_1; @@ -18176,33 +18263,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.TransparencyMode.reducible", 36); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__14() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__13; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__13; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__15() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__14; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__14; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__16() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__16() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__15; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__15; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18210,23 +18297,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__17() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__6; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__14; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__14; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__18() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__18() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__17; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__17; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18234,7 +18321,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__19() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__19() { _start: { lean_object* x_1; @@ -18242,33 +18329,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.TransparencyMode.instances", 36); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__20() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__20() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__19; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__19; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__21() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__20; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__20; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__22() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__22() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__21; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__21; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18276,23 +18363,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__23() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__6; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__20; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__20; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__24() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__24() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__23; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__23; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18300,7 +18387,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891_(uint8_t x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982_(uint8_t x_1, lean_object* x_2) { _start: { switch (x_1) { @@ -18312,14 +18399,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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__4; +x_5 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__6; +x_7 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__6; x_8 = l_Repr_addAppParen(x_7, x_2); return x_8; } @@ -18332,14 +18419,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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__10; +x_11 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__12; +x_13 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__12; x_14 = l_Repr_addAppParen(x_13, x_2); return x_14; } @@ -18352,14 +18439,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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__16; +x_17 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__18; +x_19 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__18; x_20 = l_Repr_addAppParen(x_19, x_2); return x_20; } @@ -18372,14 +18459,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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__22; +x_23 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__24; +x_25 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__24; x_26 = l_Repr_addAppParen(x_25, x_2); return x_26; } @@ -18387,13 +18474,13 @@ return x_26; } } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____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_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891_(x_3, x_2); +x_4 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982_(x_3, x_2); lean_dec(x_2); return x_4; } @@ -18402,7 +18489,7 @@ static lean_object* _init_l_Lean_Meta_instReprTransparencyMode___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____boxed), 2, 0); return x_1; } } @@ -18485,7 +18572,7 @@ x_1 = 0; return x_1; } } -LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10040_(uint8_t x_1, uint8_t x_2) { +LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10131_(uint8_t x_1, uint8_t x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -18497,7 +18584,7 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10040____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10131____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; @@ -18505,7 +18592,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_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10040_(x_3, x_4); +x_5 = l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10131_(x_3, x_4); x_6 = lean_box(x_5); return x_6; } @@ -18514,7 +18601,7 @@ static lean_object* _init_l_Lean_Meta_instBEqEtaStructMode___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10040____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10131____boxed), 2, 0); return x_1; } } @@ -18526,7 +18613,7 @@ x_1 = l_Lean_Meta_instBEqEtaStructMode___closed__1; return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__1() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__1() { _start: { lean_object* x_1; @@ -18534,33 +18621,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.EtaStructMode.all", 27); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__2() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__1; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__1; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__3() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__2; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__2; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__4() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__4() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__3; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__3; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18568,23 +18655,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__5() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__6; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__2; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__2; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__6() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__6() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__5; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__5; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18592,7 +18679,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__7() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__7() { _start: { lean_object* x_1; @@ -18600,33 +18687,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.EtaStructMode.notClasses", 34); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__8() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__7; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__7; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__9() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__8; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__8; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__10() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__10() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__9; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__9; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18634,23 +18721,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__11() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__6; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__8; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__8; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__12() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__12() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__11; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__11; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18658,7 +18745,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__13() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__13() { _start: { lean_object* x_1; @@ -18666,33 +18753,33 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.EtaStructMode.none", 28); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__14() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__13; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__13; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__15() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__14; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__14; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__16() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__16() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__15; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__15; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18700,23 +18787,23 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__17() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Init_Meta_0__Lean_Name_reprSyntax____x40_Init_Meta___hyg_1001____closed__6; -x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__14; +x_2 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__14; x_3 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__18() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__18() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__17; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__17; x_2 = 0; x_3 = lean_alloc_ctor(5, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -18724,7 +18811,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056_(uint8_t x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147_(uint8_t x_1, lean_object* x_2) { _start: { switch (x_1) { @@ -18736,14 +18823,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_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__4; +x_5 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____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_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__6; +x_7 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__6; x_8 = l_Repr_addAppParen(x_7, x_2); return x_8; } @@ -18756,14 +18843,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_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__10; +x_11 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____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_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__12; +x_13 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__12; x_14 = l_Repr_addAppParen(x_13, x_2); return x_14; } @@ -18776,14 +18863,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_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__16; +x_17 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____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_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__18; +x_19 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__18; x_20 = l_Repr_addAppParen(x_19, x_2); return x_20; } @@ -18791,13 +18878,13 @@ return x_20; } } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____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_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056_(x_3, x_2); +x_4 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147_(x_3, x_2); lean_dec(x_2); return x_4; } @@ -18806,7 +18893,7 @@ static lean_object* _init_l_Lean_Meta_instReprEtaStructMode___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____boxed), 2, 0); return x_1; } } @@ -18908,7 +18995,7 @@ x_1 = l_Lean_Meta_DSimp_instInhabitedConfig___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10255_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10346_(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; uint8_t x_4; uint8_t x_5; uint8_t x_6; uint8_t x_7; uint8_t x_8; uint8_t x_9; uint8_t x_10; uint8_t x_11; uint8_t x_12; uint8_t x_13; uint8_t x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; uint8_t x_18; lean_object* x_19; lean_object* x_23; lean_object* x_29; lean_object* x_35; lean_object* x_43; uint8_t x_49; @@ -19061,7 +19148,7 @@ goto block_28; { uint8_t x_36; lean_dec(x_35); -x_36 = l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10040_(x_6, x_14); +x_36 = l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10131_(x_6, x_14); if (x_36 == 0) { uint8_t x_37; @@ -19186,11 +19273,11 @@ goto block_48; } } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10255____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10346____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10255_(x_1, x_2); +x_3 = l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10346_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -19201,7 +19288,7 @@ static lean_object* _init_l_Lean_Meta_DSimp_instBEqConfig___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10255____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_DSimp_beqConfig____x40_Init_Meta___hyg_10346____boxed), 2, 0); return x_1; } } @@ -19213,7 +19300,7 @@ x_1 = l_Lean_Meta_DSimp_instBEqConfig___closed__1; return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__1() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__1() { _start: { lean_object* x_1; @@ -19221,29 +19308,29 @@ x_1 = lean_mk_string_from_bytes("zeta", 4); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__2() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__1; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__1; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__3() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__2; +x_2 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____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_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__4() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__4() { _start: { lean_object* x_1; @@ -19251,29 +19338,29 @@ x_1 = lean_mk_string_from_bytes(" := ", 4); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__4; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__4; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__6() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__3; +x_2 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__7() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__7() { _start: { lean_object* x_1; @@ -19281,17 +19368,17 @@ x_1 = lean_mk_string_from_bytes("beta", 4); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__8() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__7; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__7; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__9() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__9() { _start: { lean_object* x_1; @@ -19299,17 +19386,17 @@ x_1 = lean_mk_string_from_bytes("eta", 3); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__10() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__9; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__9; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__11() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__11() { _start: { lean_object* x_1; @@ -19317,17 +19404,17 @@ x_1 = lean_mk_string_from_bytes("etaStruct", 9); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__12() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__11; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__11; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__13() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__13() { _start: { lean_object* x_1; @@ -19335,17 +19422,17 @@ x_1 = lean_mk_string_from_bytes("iota", 4); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__14() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__13; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__13; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__15() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__15() { _start: { lean_object* x_1; @@ -19353,17 +19440,17 @@ x_1 = lean_mk_string_from_bytes("proj", 4); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__16() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__15; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__15; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__17() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__17() { _start: { lean_object* x_1; @@ -19371,17 +19458,17 @@ x_1 = lean_mk_string_from_bytes("decide", 6); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__18() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__18() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__17; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__17; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19() { _start: { lean_object* x_1; @@ -19389,17 +19476,17 @@ x_1 = lean_mk_string_from_bytes("autoUnfold", 10); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__20() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__20() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__21() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__21() { _start: { lean_object* x_1; @@ -19407,35 +19494,35 @@ x_1 = lean_mk_string_from_bytes("{ ", 2); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__22() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__21; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__21; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__22; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__22; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__21; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__21; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__25() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__25() { _start: { lean_object* x_1; @@ -19443,17 +19530,17 @@ x_1 = lean_mk_string_from_bytes(" }", 2); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__25; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__25; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27() { _start: { lean_object* x_1; lean_object* x_2; @@ -19463,7 +19550,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28() { _start: { lean_object* x_1; lean_object* x_2; @@ -19473,7 +19560,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513_(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; uint8_t x_4; uint8_t x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; uint8_t x_10; uint8_t x_11; uint8_t x_12; lean_object* x_13; @@ -19482,7 +19569,7 @@ x_4 = lean_ctor_get_uint8(x_1, 1); x_5 = lean_ctor_get_uint8(x_1, 2); x_6 = lean_ctor_get_uint8(x_1, 3); x_7 = lean_unsigned_to_nat(0u); -x_8 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056_(x_6, x_7); +x_8 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147_(x_6, x_7); x_9 = lean_ctor_get_uint8(x_1, 4); x_10 = lean_ctor_get_uint8(x_1, 5); x_11 = lean_ctor_get_uint8(x_1, 6); @@ -19490,21 +19577,21 @@ x_12 = lean_ctor_get_uint8(x_1, 7); if (x_3 == 0) { lean_object* x_123; -x_123 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_123 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_13 = x_123; goto block_122; } else { lean_object* x_124; -x_124 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_124 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_13 = x_124; goto block_122; } block_122: { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_14 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__6; +x_14 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__6; x_15 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); @@ -19516,25 +19603,25 @@ x_18 = lean_box(1); x_19 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); -x_20 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__8; +x_20 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__8; x_21 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_21, 0, x_19); lean_ctor_set(x_21, 1, x_20); -x_22 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5; +x_22 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5; x_23 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_23, 0, x_21); lean_ctor_set(x_23, 1, x_22); if (x_4 == 0) { lean_object* x_120; -x_120 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_120 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_24 = x_120; goto block_119; } else { lean_object* x_121; -x_121 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_121 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_24 = x_121; goto block_119; } @@ -19550,7 +19637,7 @@ lean_ctor_set(x_26, 1, x_16); x_27 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_27, 0, x_26); lean_ctor_set(x_27, 1, x_18); -x_28 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__10; +x_28 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__10; x_29 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); @@ -19560,14 +19647,14 @@ lean_ctor_set(x_30, 1, x_22); if (x_5 == 0) { lean_object* x_117; -x_117 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_117 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_31 = x_117; goto block_116; } else { lean_object* x_118; -x_118 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_118 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_31 = x_118; goto block_116; } @@ -19583,7 +19670,7 @@ lean_ctor_set(x_33, 1, x_16); x_34 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_34, 0, x_33); lean_ctor_set(x_34, 1, x_18); -x_35 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__12; +x_35 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__12; x_36 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_36, 0, x_34); lean_ctor_set(x_36, 1, x_35); @@ -19599,7 +19686,7 @@ lean_ctor_set(x_39, 1, x_16); x_40 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_40, 0, x_39); lean_ctor_set(x_40, 1, x_18); -x_41 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__14; +x_41 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__14; x_42 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_42, 0, x_40); lean_ctor_set(x_42, 1, x_41); @@ -19609,14 +19696,14 @@ lean_ctor_set(x_43, 1, x_22); if (x_9 == 0) { lean_object* x_114; -x_114 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_114 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_44 = x_114; goto block_113; } else { lean_object* x_115; -x_115 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_115 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_44 = x_115; goto block_113; } @@ -19632,7 +19719,7 @@ lean_ctor_set(x_46, 1, x_16); x_47 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_47, 0, x_46); lean_ctor_set(x_47, 1, x_18); -x_48 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__16; +x_48 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__16; x_49 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_49, 0, x_47); lean_ctor_set(x_49, 1, x_48); @@ -19642,14 +19729,14 @@ lean_ctor_set(x_50, 1, x_22); if (x_10 == 0) { lean_object* x_111; -x_111 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_111 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_51 = x_111; goto block_110; } else { lean_object* x_112; -x_112 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_112 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_51 = x_112; goto block_110; } @@ -19665,7 +19752,7 @@ lean_ctor_set(x_53, 1, x_16); x_54 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_54, 0, x_53); lean_ctor_set(x_54, 1, x_18); -x_55 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__18; +x_55 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__18; x_56 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_56, 0, x_54); lean_ctor_set(x_56, 1, x_55); @@ -19675,7 +19762,7 @@ lean_ctor_set(x_57, 1, x_22); if (x_11 == 0) { lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_58 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_58 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_59 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_59, 0, x_57); lean_ctor_set(x_59, 1, x_58); @@ -19685,7 +19772,7 @@ lean_ctor_set(x_60, 1, x_16); x_61 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_61, 0, x_60); lean_ctor_set(x_61, 1, x_18); -x_62 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__20; +x_62 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__20; x_63 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_63, 0, x_61); lean_ctor_set(x_63, 1, x_62); @@ -19698,15 +19785,15 @@ lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean x_65 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_65, 0, x_64); lean_ctor_set(x_65, 1, x_58); -x_66 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; +x_66 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; x_67 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_67, 0, x_66); lean_ctor_set(x_67, 1, x_65); -x_68 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +x_68 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; x_69 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_69, 0, x_67); lean_ctor_set(x_69, 1, x_68); -x_70 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +x_70 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; x_71 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_71, 0, x_70); lean_ctor_set(x_71, 1, x_69); @@ -19719,19 +19806,19 @@ return x_73; else { lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; lean_object* x_83; -x_74 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_74 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_75 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_75, 0, x_64); lean_ctor_set(x_75, 1, x_74); -x_76 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; +x_76 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; x_77 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_77, 0, x_76); lean_ctor_set(x_77, 1, x_75); -x_78 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +x_78 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; x_79 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_79, 0, x_77); lean_ctor_set(x_79, 1, x_78); -x_80 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +x_80 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; x_81 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_81, 0, x_80); lean_ctor_set(x_81, 1, x_79); @@ -19745,7 +19832,7 @@ return x_83; else { lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_84 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_84 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_85 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_85, 0, x_57); lean_ctor_set(x_85, 1, x_84); @@ -19755,7 +19842,7 @@ lean_ctor_set(x_86, 1, x_16); x_87 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_87, 0, x_86); lean_ctor_set(x_87, 1, x_18); -x_88 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__20; +x_88 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__20; x_89 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_89, 0, x_87); lean_ctor_set(x_89, 1, x_88); @@ -19765,19 +19852,19 @@ lean_ctor_set(x_90, 1, x_22); if (x_12 == 0) { lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; lean_object* x_100; -x_91 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_91 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_92 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_92, 0, x_90); lean_ctor_set(x_92, 1, x_91); -x_93 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; +x_93 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; x_94 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_94, 0, x_93); lean_ctor_set(x_94, 1, x_92); -x_95 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +x_95 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; x_96 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_96, 0, x_94); lean_ctor_set(x_96, 1, x_95); -x_97 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +x_97 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; x_98 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_98, 0, x_97); lean_ctor_set(x_98, 1, x_96); @@ -19793,15 +19880,15 @@ lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; x_101 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_101, 0, x_90); lean_ctor_set(x_101, 1, x_84); -x_102 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; +x_102 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; x_103 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_103, 0, x_102); lean_ctor_set(x_103, 1, x_101); -x_104 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +x_104 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; x_105 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_105, 0, x_103); lean_ctor_set(x_105, 1, x_104); -x_106 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +x_106 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; x_107 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_107, 0, x_106); lean_ctor_set(x_107, 1, x_105); @@ -19819,11 +19906,11 @@ return x_109; } } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422_(x_1, x_2); +x_3 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; @@ -19833,7 +19920,7 @@ static lean_object* _init_l_Lean_Meta_DSimp_instReprConfig___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____boxed), 2, 0); return x_1; } } @@ -20007,7 +20094,7 @@ x_1 = l_Lean_Meta_Simp_instInhabitedConfig___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10701_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10792_(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; uint8_t x_6; uint8_t x_7; uint8_t x_8; uint8_t x_9; uint8_t x_10; uint8_t x_11; uint8_t x_12; uint8_t x_13; uint8_t x_14; uint8_t x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; uint8_t x_21; uint8_t x_22; uint8_t x_23; uint8_t x_24; uint8_t x_25; uint8_t x_26; uint8_t x_27; uint8_t x_28; uint8_t x_29; uint8_t x_30; uint8_t x_31; uint8_t x_32; lean_object* x_33; lean_object* x_37; lean_object* x_43; lean_object* x_49; lean_object* x_55; lean_object* x_61; lean_object* x_69; lean_object* x_75; lean_object* x_81; lean_object* x_87; lean_object* x_93; uint8_t x_99; @@ -20265,7 +20352,7 @@ goto block_54; { uint8_t x_62; lean_dec(x_61); -x_62 = l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10040_(x_11, x_26); +x_62 = l___private_Init_Meta_0__Lean_Meta_beqEtaStructMode____x40_Init_Meta___hyg_10131_(x_11, x_26); if (x_62 == 0) { uint8_t x_63; @@ -20490,11 +20577,11 @@ goto block_92; } } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10701____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10792____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10701_(x_1, x_2); +x_3 = l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10792_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -20505,7 +20592,7 @@ static lean_object* _init_l_Lean_Meta_Simp_instBEqConfig___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10701____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_Simp_beqConfig____x40_Init_Meta___hyg_10792____boxed), 2, 0); return x_1; } } @@ -20517,7 +20604,7 @@ x_1 = l_Lean_Meta_Simp_instBEqConfig___closed__1; return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__1() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__1() { _start: { lean_object* x_1; @@ -20525,41 +20612,41 @@ x_1 = lean_mk_string_from_bytes("maxSteps", 8); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__2() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__1; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__1; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__3() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__2; +x_2 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____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_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__4() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__3; -x_2 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__3; +x_2 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5; x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__5() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__5() { _start: { lean_object* x_1; @@ -20567,17 +20654,17 @@ x_1 = lean_mk_string_from_bytes("maxDischargeDepth", 17); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__6() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__5; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__5; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__7() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__7() { _start: { lean_object* x_1; @@ -20585,17 +20672,17 @@ x_1 = lean_mk_string_from_bytes("contextual", 10); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__8() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__7; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__7; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__9() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__9() { _start: { lean_object* x_1; @@ -20603,17 +20690,17 @@ x_1 = lean_mk_string_from_bytes("memoize", 7); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__10() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__9; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__9; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__11() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__11() { _start: { lean_object* x_1; @@ -20621,17 +20708,17 @@ x_1 = lean_mk_string_from_bytes("singlePass", 10); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__12() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__11; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__11; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13() { _start: { lean_object* x_1; @@ -20639,17 +20726,17 @@ x_1 = lean_mk_string_from_bytes("arith", 5); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__14() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15() { _start: { lean_object* x_1; @@ -20657,17 +20744,17 @@ x_1 = lean_mk_string_from_bytes("dsimp", 5); return x_1; } } -static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__16() { +static lean_object* _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071_(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; uint8_t x_26; uint8_t x_27; uint8_t x_28; uint8_t x_29; uint8_t x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; uint8_t x_35; uint8_t x_36; uint8_t x_37; uint8_t x_38; uint8_t x_39; lean_object* x_40; @@ -20676,7 +20763,7 @@ lean_inc(x_3); x_4 = l_Nat_repr(x_3); x_5 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_5, 0, x_4); -x_6 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__4; +x_6 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__4; x_7 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); @@ -20688,11 +20775,11 @@ x_10 = lean_box(1); x_11 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_11, 0, x_9); lean_ctor_set(x_11, 1, x_10); -x_12 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__6; +x_12 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__6; x_13 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_13, 0, x_11); lean_ctor_set(x_13, 1, x_12); -x_14 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5; +x_14 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5; x_15 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_15, 0, x_13); lean_ctor_set(x_15, 1, x_14); @@ -20710,7 +20797,7 @@ lean_ctor_set(x_20, 1, x_8); x_21 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_21, 0, x_20); lean_ctor_set(x_21, 1, x_10); -x_22 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__8; +x_22 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__8; x_23 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_23, 0, x_21); lean_ctor_set(x_23, 1, x_22); @@ -20725,7 +20812,7 @@ x_29 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 4); x_30 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 5); x_31 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 6); x_32 = lean_unsigned_to_nat(0u); -x_33 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056_(x_31, x_32); +x_33 = l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147_(x_31, x_32); x_34 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 7); x_35 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 8); x_36 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 9); @@ -20736,14 +20823,14 @@ lean_dec(x_1); if (x_25 == 0) { lean_object* x_196; -x_196 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_196 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_40 = x_196; goto block_195; } else { lean_object* x_197; -x_197 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_197 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_40 = x_197; goto block_195; } @@ -20759,7 +20846,7 @@ lean_ctor_set(x_42, 1, x_8); x_43 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_43, 0, x_42); lean_ctor_set(x_43, 1, x_10); -x_44 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__10; +x_44 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__10; x_45 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_45, 0, x_43); lean_ctor_set(x_45, 1, x_44); @@ -20769,14 +20856,14 @@ lean_ctor_set(x_46, 1, x_14); if (x_26 == 0) { lean_object* x_193; -x_193 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_193 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_47 = x_193; goto block_192; } else { lean_object* x_194; -x_194 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_194 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_47 = x_194; goto block_192; } @@ -20792,7 +20879,7 @@ lean_ctor_set(x_49, 1, x_8); x_50 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_50, 0, x_49); lean_ctor_set(x_50, 1, x_10); -x_51 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__12; +x_51 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__12; x_52 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_52, 0, x_50); lean_ctor_set(x_52, 1, x_51); @@ -20802,14 +20889,14 @@ lean_ctor_set(x_53, 1, x_14); if (x_27 == 0) { lean_object* x_190; -x_190 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_190 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_54 = x_190; goto block_189; } else { lean_object* x_191; -x_191 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_191 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_54 = x_191; goto block_189; } @@ -20825,7 +20912,7 @@ lean_ctor_set(x_56, 1, x_8); x_57 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_57, 0, x_56); lean_ctor_set(x_57, 1, x_10); -x_58 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__2; +x_58 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__2; x_59 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_59, 0, x_57); lean_ctor_set(x_59, 1, x_58); @@ -20835,14 +20922,14 @@ lean_ctor_set(x_60, 1, x_14); if (x_28 == 0) { lean_object* x_187; -x_187 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_187 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_61 = x_187; goto block_186; } else { lean_object* x_188; -x_188 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_188 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_61 = x_188; goto block_186; } @@ -20858,7 +20945,7 @@ lean_ctor_set(x_63, 1, x_8); x_64 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_64, 0, x_63); lean_ctor_set(x_64, 1, x_10); -x_65 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__8; +x_65 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__8; x_66 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_66, 0, x_64); lean_ctor_set(x_66, 1, x_65); @@ -20868,14 +20955,14 @@ lean_ctor_set(x_67, 1, x_14); if (x_29 == 0) { lean_object* x_184; -x_184 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_184 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_68 = x_184; goto block_183; } else { lean_object* x_185; -x_185 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_185 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_68 = x_185; goto block_183; } @@ -20891,7 +20978,7 @@ lean_ctor_set(x_70, 1, x_8); x_71 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_71, 0, x_70); lean_ctor_set(x_71, 1, x_10); -x_72 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__10; +x_72 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__10; x_73 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_73, 0, x_71); lean_ctor_set(x_73, 1, x_72); @@ -20901,14 +20988,14 @@ lean_ctor_set(x_74, 1, x_14); if (x_30 == 0) { lean_object* x_181; -x_181 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_181 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_75 = x_181; goto block_180; } else { lean_object* x_182; -x_182 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_182 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_75 = x_182; goto block_180; } @@ -20924,7 +21011,7 @@ lean_ctor_set(x_77, 1, x_8); x_78 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_78, 0, x_77); lean_ctor_set(x_78, 1, x_10); -x_79 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__12; +x_79 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__12; x_80 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_80, 0, x_78); lean_ctor_set(x_80, 1, x_79); @@ -20940,7 +21027,7 @@ lean_ctor_set(x_83, 1, x_8); x_84 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_84, 0, x_83); lean_ctor_set(x_84, 1, x_10); -x_85 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__14; +x_85 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__14; x_86 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_86, 0, x_84); lean_ctor_set(x_86, 1, x_85); @@ -20950,14 +21037,14 @@ lean_ctor_set(x_87, 1, x_14); if (x_34 == 0) { lean_object* x_178; -x_178 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_178 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_88 = x_178; goto block_177; } else { lean_object* x_179; -x_179 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_179 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_88 = x_179; goto block_177; } @@ -20973,7 +21060,7 @@ lean_ctor_set(x_90, 1, x_8); x_91 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_91, 0, x_90); lean_ctor_set(x_91, 1, x_10); -x_92 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__16; +x_92 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__16; x_93 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_93, 0, x_91); lean_ctor_set(x_93, 1, x_92); @@ -20983,14 +21070,14 @@ lean_ctor_set(x_94, 1, x_14); if (x_35 == 0) { lean_object* x_175; -x_175 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_175 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_95 = x_175; goto block_174; } else { lean_object* x_176; -x_176 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_176 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_95 = x_176; goto block_174; } @@ -21006,7 +21093,7 @@ lean_ctor_set(x_97, 1, x_8); x_98 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_98, 0, x_97); lean_ctor_set(x_98, 1, x_10); -x_99 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__18; +x_99 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__18; x_100 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_100, 0, x_98); lean_ctor_set(x_100, 1, x_99); @@ -21016,14 +21103,14 @@ lean_ctor_set(x_101, 1, x_14); if (x_36 == 0) { lean_object* x_172; -x_172 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_172 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_102 = x_172; goto block_171; } else { lean_object* x_173; -x_173 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_173 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_102 = x_173; goto block_171; } @@ -21039,7 +21126,7 @@ lean_ctor_set(x_104, 1, x_8); x_105 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_105, 0, x_104); lean_ctor_set(x_105, 1, x_10); -x_106 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__14; +x_106 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__14; x_107 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_107, 0, x_105); lean_ctor_set(x_107, 1, x_106); @@ -21049,14 +21136,14 @@ lean_ctor_set(x_108, 1, x_14); if (x_37 == 0) { lean_object* x_169; -x_169 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_169 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_109 = x_169; goto block_168; } else { lean_object* x_170; -x_170 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_170 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_109 = x_170; goto block_168; } @@ -21072,7 +21159,7 @@ lean_ctor_set(x_111, 1, x_8); x_112 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_112, 0, x_111); lean_ctor_set(x_112, 1, x_10); -x_113 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__20; +x_113 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__20; x_114 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_114, 0, x_112); lean_ctor_set(x_114, 1, x_113); @@ -21082,7 +21169,7 @@ lean_ctor_set(x_115, 1, x_14); if (x_38 == 0) { lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_116 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_116 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_117 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_117, 0, x_115); lean_ctor_set(x_117, 1, x_116); @@ -21092,7 +21179,7 @@ lean_ctor_set(x_118, 1, x_8); x_119 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_119, 0, x_118); lean_ctor_set(x_119, 1, x_10); -x_120 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__16; +x_120 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__16; x_121 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_121, 0, x_119); lean_ctor_set(x_121, 1, x_120); @@ -21105,15 +21192,15 @@ lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; x_123 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_123, 0, x_122); lean_ctor_set(x_123, 1, x_116); -x_124 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; +x_124 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; x_125 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_125, 0, x_124); lean_ctor_set(x_125, 1, x_123); -x_126 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +x_126 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; x_127 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_127, 0, x_125); lean_ctor_set(x_127, 1, x_126); -x_128 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +x_128 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; x_129 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_129, 0, x_128); lean_ctor_set(x_129, 1, x_127); @@ -21126,19 +21213,19 @@ return x_131; else { 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; uint8_t x_140; lean_object* x_141; -x_132 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_132 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_133 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_133, 0, x_122); lean_ctor_set(x_133, 1, x_132); -x_134 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; +x_134 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; x_135 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_135, 0, x_134); lean_ctor_set(x_135, 1, x_133); -x_136 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +x_136 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; x_137 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_137, 0, x_135); lean_ctor_set(x_137, 1, x_136); -x_138 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +x_138 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; x_139 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_139, 0, x_138); lean_ctor_set(x_139, 1, x_137); @@ -21152,7 +21239,7 @@ return x_141; else { lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_142 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28; +x_142 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28; x_143 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_143, 0, x_115); lean_ctor_set(x_143, 1, x_142); @@ -21162,7 +21249,7 @@ lean_ctor_set(x_144, 1, x_8); x_145 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_145, 0, x_144); lean_ctor_set(x_145, 1, x_10); -x_146 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__16; +x_146 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__16; x_147 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_147, 0, x_145); lean_ctor_set(x_147, 1, x_146); @@ -21172,19 +21259,19 @@ lean_ctor_set(x_148, 1, x_14); if (x_39 == 0) { lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; uint8_t x_157; lean_object* x_158; -x_149 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27; +x_149 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27; x_150 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_150, 0, x_148); lean_ctor_set(x_150, 1, x_149); -x_151 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; +x_151 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; x_152 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_152, 0, x_151); lean_ctor_set(x_152, 1, x_150); -x_153 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +x_153 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; x_154 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_154, 0, x_152); lean_ctor_set(x_154, 1, x_153); -x_155 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +x_155 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; x_156 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_156, 0, x_155); lean_ctor_set(x_156, 1, x_154); @@ -21200,15 +21287,15 @@ lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; x_159 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_159, 0, x_148); lean_ctor_set(x_159, 1, x_142); -x_160 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24; +x_160 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24; x_161 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_161, 0, x_160); lean_ctor_set(x_161, 1, x_159); -x_162 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26; +x_162 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26; x_163 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_163, 0, x_161); lean_ctor_set(x_163, 1, x_162); -x_164 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23; +x_164 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23; x_165 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_165, 0, x_164); lean_ctor_set(x_165, 1, x_163); @@ -21231,11 +21318,11 @@ return x_167; } } } -LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980_(x_1, x_2); +x_3 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -21244,7 +21331,7 @@ static lean_object* _init_l_Lean_Meta_Simp_instReprConfig___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____boxed), 2, 0); return x_1; } } @@ -21643,7 +21730,7 @@ static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__7; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__7; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } @@ -21652,7 +21739,7 @@ static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__7; +x_1 = l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__7; x_2 = lean_unsigned_to_nat(0u); x_3 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__21; x_4 = lean_alloc_ctor(0, 3, 0); @@ -22205,7 +22292,7 @@ static lean_object* _init_l_Lean_Parser_Tactic_simpAllKind___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__4; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__4; x_2 = lean_alloc_ctor(5, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; @@ -22319,7 +22406,7 @@ static lean_object* _init_l_Lean_Parser_Tactic_dsimpKind___closed__3() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -27957,7 +28044,7 @@ static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } @@ -27966,7 +28053,7 @@ static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15; x_2 = lean_unsigned_to_nat(0u); x_3 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__3; x_4 = lean_alloc_ctor(0, 3, 0); @@ -27981,7 +28068,7 @@ static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15; +x_2 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -27991,7 +28078,7 @@ static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic_tacticErw_______closed__2; -x_2 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15; +x_2 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -28633,7 +28720,7 @@ static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(9u); +x_1 = lean_unsigned_to_nat(10u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } @@ -28653,7 +28740,7 @@ static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__71; -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__14; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__12; x_3 = lean_array_push(x_1, x_2); return x_3; } @@ -28661,27 +28748,37 @@ return x_3; static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__73() { _start: { +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__72; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__14; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__74() { +_start: +{ lean_object* x_1; x_1 = lean_mk_string_from_bytes("simpAll", 7); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__74() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__75() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__73; +x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__74; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__75() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__76() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__73; +x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__74; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__74; +x_3 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__75; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -28689,51 +28786,51 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__76() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__77() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__73; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__74; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__77() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__78() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic_tacticErw_______closed__2; -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__73; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__74; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__78() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__79() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__77; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__78; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__79() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__80() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__78; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__79; 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___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__80() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__81() { _start: { lean_object* x_1; @@ -28741,7 +28838,7 @@ x_1 = lean_mk_string_from_bytes("\"simp_all \"", 11); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__81() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__82() { _start: { lean_object* x_1; @@ -28749,22 +28846,22 @@ x_1 = lean_mk_string_from_bytes("simp", 4); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__82() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__83() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__81; +x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__82; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__83() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__84() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__81; +x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__82; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__82; +x_3 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__83; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -28772,51 +28869,51 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__84() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__85() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__81; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__82; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__85() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__86() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic_tacticErw_______closed__2; -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__81; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__82; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__86() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__87() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__85; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__86; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__87() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__88() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__86; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__87; 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___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__88() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__89() { _start: { lean_object* x_1; @@ -28824,7 +28921,7 @@ x_1 = lean_mk_string_from_bytes("\"simp \"", 7); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__89() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__90() { _start: { lean_object* x_1; @@ -28832,22 +28929,22 @@ x_1 = lean_mk_string_from_bytes("simpStar", 8); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__90() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__91() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__89; +x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__90; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__91() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__92() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__89; +x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__90; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__90; +x_3 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__91; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -28855,44 +28952,44 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__92() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__93() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__89; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__90; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__93() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__94() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic_tacticErw_______closed__2; -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__89; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__90; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__94() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__95() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__93; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__94; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__95() { +static lean_object* _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__96() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__94; +x_2 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__95; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); @@ -29372,7 +29469,7 @@ lean_ctor_set(x_221, 0, x_52); lean_ctor_set(x_221, 1, x_220); lean_ctor_set(x_221, 2, x_219); lean_ctor_set(x_221, 3, x_31); -x_222 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__72; +x_222 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__73; x_223 = lean_array_push(x_222, x_55); x_224 = lean_array_push(x_223, x_85); x_225 = lean_array_push(x_224, x_74); @@ -29417,13 +29514,13 @@ lean_inc(x_240); x_245 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_245, 0, x_240); lean_ctor_set(x_245, 1, x_244); -x_246 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__76; +x_246 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__77; lean_inc(x_242); lean_inc(x_243); x_247 = l_Lean_addMacroScope(x_243, x_246, x_242); x_248 = lean_box(0); -x_249 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__75; -x_250 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__79; +x_249 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__76; +x_250 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__80; x_251 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_251, 0, x_240); lean_ctor_set(x_251, 1, x_249); @@ -29447,7 +29544,7 @@ lean_inc(x_260); x_261 = lean_ctor_get(x_259, 1); lean_inc(x_261); lean_dec(x_259); -x_262 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__80; +x_262 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__81; x_263 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_263, 0, x_260); lean_ctor_set(x_263, 1, x_262); @@ -29790,7 +29887,7 @@ lean_ctor_set(x_420, 0, x_269); lean_ctor_set(x_420, 1, x_419); lean_ctor_set(x_420, 2, x_418); lean_ctor_set(x_420, 3, x_248); -x_421 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__72; +x_421 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__73; x_422 = lean_array_push(x_421, x_272); x_423 = lean_array_push(x_422, x_302); x_424 = lean_array_push(x_423, x_291); @@ -29837,13 +29934,13 @@ lean_inc(x_439); x_444 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_444, 0, x_439); lean_ctor_set(x_444, 1, x_443); -x_445 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__84; +x_445 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__85; lean_inc(x_441); lean_inc(x_442); x_446 = l_Lean_addMacroScope(x_442, x_445, x_441); x_447 = lean_box(0); -x_448 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__83; -x_449 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__87; +x_448 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__84; +x_449 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__88; x_450 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_450, 0, x_439); lean_ctor_set(x_450, 1, x_448); @@ -29867,7 +29964,7 @@ lean_inc(x_459); x_460 = lean_ctor_get(x_458, 1); lean_inc(x_460); lean_dec(x_458); -x_461 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__88; +x_461 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__89; x_462 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_462, 0, x_459); lean_ctor_set(x_462, 1, x_461); @@ -30080,12 +30177,12 @@ x_557 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_557, 0, x_455); lean_ctor_set(x_557, 1, x_492); lean_ctor_set(x_557, 2, x_556); -x_558 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__92; +x_558 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__93; lean_inc(x_441); lean_inc(x_442); x_559 = l_Lean_addMacroScope(x_442, x_558, x_441); -x_560 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__91; -x_561 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__95; +x_560 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__92; +x_561 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__96; lean_inc(x_468); x_562 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_562, 0, x_468); @@ -30276,7 +30373,7 @@ lean_ctor_set(x_649, 0, x_468); lean_ctor_set(x_649, 1, x_648); lean_ctor_set(x_649, 2, x_647); lean_ctor_set(x_649, 3, x_447); -x_650 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__72; +x_650 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__73; x_651 = lean_array_push(x_650, x_471); x_652 = lean_array_push(x_651, x_501); x_653 = lean_array_push(x_652, x_490); @@ -30613,7 +30710,7 @@ x_1 = l_Lean_Parser_Tactic_simpAutoUnfold___closed__25; return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -30621,15 +30718,15 @@ x_1 = lean_mk_string_from_bytes("simp ", 5); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____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_15391____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; lean_object* x_10; 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; -x_5 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__85; +x_5 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__86; 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_15282____lambda__1___closed__1; +x_9 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1___closed__1; x_10 = l_Lean_mkAtomFrom(x_8, x_9); x_11 = l_Lean_Syntax_setArg(x_6, x_7, x_10); x_12 = l_Lean_mkOptionalNode___closed__2; @@ -30648,7 +30745,7 @@ lean_ctor_set(x_19, 1, x_4); return x_19; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -30658,7 +30755,7 @@ 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_15282____closed__2() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -30668,7 +30765,7 @@ 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_15282____closed__3() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__3() { _start: { lean_object* x_1; @@ -30676,22 +30773,22 @@ x_1 = lean_mk_string_from_bytes("Lean.Meta.Simp.Config", 21); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__4() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__3; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__3; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__3; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__3; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__4; +x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__4; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -30699,7 +30796,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__6() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__6() { _start: { lean_object* x_1; @@ -30707,17 +30804,17 @@ x_1 = lean_mk_string_from_bytes("Simp", 4); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__7() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__24; -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__6; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__6; 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_15282____closed__8() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__8() { _start: { lean_object* x_1; @@ -30725,56 +30822,56 @@ x_1 = lean_mk_string_from_bytes("Config", 6); return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__7; -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__8; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__7; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__8; 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_15282____closed__10() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____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_15282____closed__9; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11() { _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_15282____closed__10; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__10; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__12() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19; +x_1 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__12; +x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__12; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -30782,17 +30879,17 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19; +x_2 = l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19; 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_15282____closed__15() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__15() { _start: { lean_object* x_1; lean_object* x_2; @@ -30801,13 +30898,13 @@ x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_instQuoteBoolStrAnonymous___closed__6; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__15; +x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__15; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -30815,7 +30912,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -30825,7 +30922,7 @@ 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_15282____closed__18() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -30837,19 +30934,19 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19() { _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_15282____closed__18; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__18; 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_15282____closed__20() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; @@ -30863,7 +30960,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282_(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_15391_(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; @@ -30927,12 +31024,12 @@ lean_inc(x_11); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9; 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_15282____closed__5; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11; lean_inc(x_11); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_11); @@ -31009,11 +31106,11 @@ x_68 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_68, 0, x_38); lean_ctor_set(x_68, 1, x_43); lean_ctor_set(x_68, 2, x_67); -x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; lean_inc(x_13); lean_inc(x_14); x_70 = l_Lean_addMacroScope(x_14, x_69, x_13); -x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_11); x_72 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_72, 0, x_11); @@ -31028,10 +31125,10 @@ x_77 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_77, 0, x_38); lean_ctor_set(x_77, 1, x_76); lean_ctor_set(x_77, 2, x_75); -x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_79 = l_Lean_addMacroScope(x_14, x_78, x_13); -x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_11); x_82 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_82, 0, x_11); @@ -31062,7 +31159,7 @@ x_93 = lean_array_push(x_92, x_61); lean_inc(x_93); x_94 = lean_array_push(x_93, x_68); x_95 = lean_array_push(x_94, x_89); -x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_97 = lean_array_push(x_95, x_96); x_98 = lean_array_push(x_97, x_74); lean_inc(x_91); @@ -31077,14 +31174,14 @@ x_103 = lean_array_push(x_102, x_57); x_104 = lean_array_push(x_103, x_74); x_105 = lean_array_push(x_104, x_59); x_106 = lean_array_push(x_105, x_101); -x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_108 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_108, 0, x_38); lean_ctor_set(x_108, 1, x_107); lean_ctor_set(x_108, 2, x_106); x_109 = lean_array_push(x_35, x_22); x_110 = lean_array_push(x_109, x_108); -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_112 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_112, 0, x_38); lean_ctor_set(x_112, 1, x_111); @@ -31135,7 +31232,7 @@ x_139 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_139, 0, x_38); lean_ctor_set(x_139, 1, x_8); lean_ctor_set(x_139, 2, x_138); -x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1(x_1, x_139, x_2, x_12); +x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1(x_1, x_139, x_2, x_12); lean_dec(x_2); return x_140; } @@ -31193,12 +31290,12 @@ lean_inc(x_144); x_162 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_162, 0, x_144); lean_ctor_set(x_162, 1, x_161); -x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9; +x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9; lean_inc(x_146); lean_inc(x_147); x_164 = l_Lean_addMacroScope(x_147, x_163, x_146); -x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__5; -x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11; +x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5; +x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11; lean_inc(x_144); x_167 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_167, 0, x_144); @@ -31275,11 +31372,11 @@ x_201 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_201, 0, x_171); lean_ctor_set(x_201, 1, x_176); lean_ctor_set(x_201, 2, x_200); -x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; lean_inc(x_146); lean_inc(x_147); x_203 = l_Lean_addMacroScope(x_147, x_202, x_146); -x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_144); x_205 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_205, 0, x_144); @@ -31294,10 +31391,10 @@ x_210 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_210, 0, x_171); lean_ctor_set(x_210, 1, x_209); lean_ctor_set(x_210, 2, x_208); -x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_212 = l_Lean_addMacroScope(x_147, x_211, x_146); -x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_144); x_215 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_215, 0, x_144); @@ -31326,7 +31423,7 @@ x_225 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Ta x_226 = lean_array_push(x_225, x_194); x_227 = lean_array_push(x_226, x_201); x_228 = lean_array_push(x_227, x_222); -x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_230 = lean_array_push(x_228, x_229); x_231 = lean_array_push(x_230, x_207); x_232 = lean_array_push(x_231, x_224); @@ -31340,14 +31437,14 @@ x_236 = lean_array_push(x_235, x_190); x_237 = lean_array_push(x_236, x_207); x_238 = lean_array_push(x_237, x_192); x_239 = lean_array_push(x_238, x_234); -x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_241 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_241, 0, x_171); lean_ctor_set(x_241, 1, x_240); lean_ctor_set(x_241, 2, x_239); x_242 = lean_array_push(x_168, x_155); x_243 = lean_array_push(x_242, x_241); -x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_245 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_245, 0, x_171); lean_ctor_set(x_245, 1, x_244); @@ -31374,17 +31471,17 @@ x_258 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_258, 0, x_171); lean_ctor_set(x_258, 1, x_8); lean_ctor_set(x_258, 2, x_257); -x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1(x_1, x_258, x_2, x_145); +x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1(x_1, x_258, x_2, x_145); lean_dec(x_2); return x_259; } } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____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_15391____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_15282____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -31519,22 +31616,22 @@ x_1 = l_Lean_Parser_Tactic_simpArith___closed__10; return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13; +x_1 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__1; +x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__1; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -31542,17 +31639,17 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13; +x_2 = l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226_(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_16335_(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; @@ -31616,12 +31713,12 @@ lean_inc(x_11); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9; 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_15282____closed__5; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11; lean_inc(x_11); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_11); @@ -31698,11 +31795,11 @@ x_68 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_68, 0, x_38); lean_ctor_set(x_68, 1, x_43); lean_ctor_set(x_68, 2, x_67); -x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; lean_inc(x_13); lean_inc(x_14); x_70 = l_Lean_addMacroScope(x_14, x_69, x_13); -x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; +x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; lean_inc(x_11); x_72 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_72, 0, x_11); @@ -31717,10 +31814,10 @@ x_77 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_77, 0, x_38); lean_ctor_set(x_77, 1, x_76); lean_ctor_set(x_77, 2, x_75); -x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_79 = l_Lean_addMacroScope(x_14, x_78, x_13); -x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_11); x_82 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_82, 0, x_11); @@ -31751,7 +31848,7 @@ x_93 = lean_array_push(x_92, x_61); lean_inc(x_93); x_94 = lean_array_push(x_93, x_68); x_95 = lean_array_push(x_94, x_89); -x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_97 = lean_array_push(x_95, x_96); x_98 = lean_array_push(x_97, x_74); lean_inc(x_91); @@ -31766,14 +31863,14 @@ x_103 = lean_array_push(x_102, x_57); x_104 = lean_array_push(x_103, x_74); x_105 = lean_array_push(x_104, x_59); x_106 = lean_array_push(x_105, x_101); -x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_108 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_108, 0, x_38); lean_ctor_set(x_108, 1, x_107); lean_ctor_set(x_108, 2, x_106); x_109 = lean_array_push(x_35, x_22); x_110 = lean_array_push(x_109, x_108); -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_112 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_112, 0, x_38); lean_ctor_set(x_112, 1, x_111); @@ -31824,7 +31921,7 @@ x_139 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_139, 0, x_38); lean_ctor_set(x_139, 1, x_8); lean_ctor_set(x_139, 2, x_138); -x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1(x_1, x_139, x_2, x_12); +x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1(x_1, x_139, x_2, x_12); lean_dec(x_2); return x_140; } @@ -31882,12 +31979,12 @@ lean_inc(x_144); x_162 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_162, 0, x_144); lean_ctor_set(x_162, 1, x_161); -x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9; +x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9; lean_inc(x_146); lean_inc(x_147); x_164 = l_Lean_addMacroScope(x_147, x_163, x_146); -x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__5; -x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11; +x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5; +x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11; lean_inc(x_144); x_167 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_167, 0, x_144); @@ -31964,11 +32061,11 @@ x_201 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_201, 0, x_171); lean_ctor_set(x_201, 1, x_176); lean_ctor_set(x_201, 2, x_200); -x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; +x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; lean_inc(x_146); lean_inc(x_147); x_203 = l_Lean_addMacroScope(x_147, x_202, x_146); -x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; +x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; lean_inc(x_144); x_205 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_205, 0, x_144); @@ -31983,10 +32080,10 @@ x_210 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_210, 0, x_171); lean_ctor_set(x_210, 1, x_209); lean_ctor_set(x_210, 2, x_208); -x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_212 = l_Lean_addMacroScope(x_147, x_211, x_146); -x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_144); x_215 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_215, 0, x_144); @@ -32015,7 +32112,7 @@ x_225 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Ta x_226 = lean_array_push(x_225, x_194); x_227 = lean_array_push(x_226, x_201); x_228 = lean_array_push(x_227, x_222); -x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_230 = lean_array_push(x_228, x_229); x_231 = lean_array_push(x_230, x_207); x_232 = lean_array_push(x_231, x_224); @@ -32029,14 +32126,14 @@ x_236 = lean_array_push(x_235, x_190); x_237 = lean_array_push(x_236, x_207); x_238 = lean_array_push(x_237, x_192); x_239 = lean_array_push(x_238, x_234); -x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_241 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_241, 0, x_171); lean_ctor_set(x_241, 1, x_240); lean_ctor_set(x_241, 2, x_239); x_242 = lean_array_push(x_168, x_155); x_243 = lean_array_push(x_242, x_241); -x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_245 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_245, 0, x_171); lean_ctor_set(x_245, 1, x_244); @@ -32063,7 +32160,7 @@ x_258 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_258, 0, x_171); lean_ctor_set(x_258, 1, x_8); lean_ctor_set(x_258, 2, x_257); -x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1(x_1, x_258, x_2, x_145); +x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1(x_1, x_258, x_2, x_145); lean_dec(x_2); return x_259; } @@ -32199,7 +32296,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_17170_(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_17279_(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; @@ -32263,12 +32360,12 @@ lean_inc(x_11); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9; 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_15282____closed__5; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11; lean_inc(x_11); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_11); @@ -32345,11 +32442,11 @@ x_68 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_68, 0, x_38); lean_ctor_set(x_68, 1, x_43); lean_ctor_set(x_68, 2, x_67); -x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; lean_inc(x_13); lean_inc(x_14); x_70 = l_Lean_addMacroScope(x_14, x_69, x_13); -x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; +x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; lean_inc(x_11); x_72 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_72, 0, x_11); @@ -32364,12 +32461,12 @@ x_77 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_77, 0, x_38); lean_ctor_set(x_77, 1, x_76); lean_ctor_set(x_77, 2, x_75); -x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; lean_inc(x_13); lean_inc(x_14); x_79 = l_Lean_addMacroScope(x_14, x_78, x_13); -x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_11); x_82 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_82, 0, x_11); @@ -32391,9 +32488,9 @@ lean_inc(x_11); x_89 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_89, 0, x_11); lean_ctor_set(x_89, 1, x_88); -x_90 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_90 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; x_91 = l_Lean_addMacroScope(x_14, x_90, x_13); -x_92 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_92 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_11); x_93 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_93, 0, x_11); @@ -32431,7 +32528,7 @@ x_108 = lean_array_push(x_107, x_61); lean_inc(x_108); x_109 = lean_array_push(x_108, x_68); x_110 = lean_array_push(x_109, x_104); -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_112 = lean_array_push(x_110, x_111); x_113 = lean_array_push(x_112, x_74); lean_inc(x_106); @@ -32446,14 +32543,14 @@ x_118 = lean_array_push(x_117, x_57); x_119 = lean_array_push(x_118, x_74); x_120 = lean_array_push(x_119, x_59); x_121 = lean_array_push(x_120, x_116); -x_122 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_122 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_123 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_123, 0, x_38); lean_ctor_set(x_123, 1, x_122); lean_ctor_set(x_123, 2, x_121); x_124 = lean_array_push(x_35, x_22); x_125 = lean_array_push(x_124, x_123); -x_126 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_126 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_127 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_127, 0, x_38); lean_ctor_set(x_127, 1, x_126); @@ -32504,7 +32601,7 @@ x_154 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_154, 0, x_38); lean_ctor_set(x_154, 1, x_8); lean_ctor_set(x_154, 2, x_153); -x_155 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1(x_1, x_154, x_2, x_12); +x_155 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1(x_1, x_154, x_2, x_12); lean_dec(x_2); return x_155; } @@ -32562,12 +32659,12 @@ lean_inc(x_159); x_177 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_177, 0, x_159); lean_ctor_set(x_177, 1, x_176); -x_178 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9; +x_178 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9; lean_inc(x_161); lean_inc(x_162); x_179 = l_Lean_addMacroScope(x_162, x_178, x_161); -x_180 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__5; -x_181 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11; +x_180 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5; +x_181 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11; lean_inc(x_159); x_182 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_182, 0, x_159); @@ -32644,11 +32741,11 @@ x_216 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_216, 0, x_186); lean_ctor_set(x_216, 1, x_191); lean_ctor_set(x_216, 2, x_215); -x_217 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; +x_217 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; lean_inc(x_161); lean_inc(x_162); x_218 = l_Lean_addMacroScope(x_162, x_217, x_161); -x_219 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; +x_219 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; lean_inc(x_159); x_220 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_220, 0, x_159); @@ -32663,12 +32760,12 @@ x_225 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_225, 0, x_186); lean_ctor_set(x_225, 1, x_224); lean_ctor_set(x_225, 2, x_223); -x_226 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_226 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; lean_inc(x_161); lean_inc(x_162); x_227 = l_Lean_addMacroScope(x_162, x_226, x_161); -x_228 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_228 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_159); x_230 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_230, 0, x_159); @@ -32690,9 +32787,9 @@ lean_inc(x_159); x_237 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_237, 0, x_159); lean_ctor_set(x_237, 1, x_236); -x_238 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_238 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; x_239 = l_Lean_addMacroScope(x_162, x_238, x_161); -x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_159); x_241 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_241, 0, x_159); @@ -32728,7 +32825,7 @@ x_255 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Ta x_256 = lean_array_push(x_255, x_209); x_257 = lean_array_push(x_256, x_216); x_258 = lean_array_push(x_257, x_252); -x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_260 = lean_array_push(x_258, x_259); x_261 = lean_array_push(x_260, x_222); x_262 = lean_array_push(x_261, x_254); @@ -32742,14 +32839,14 @@ x_266 = lean_array_push(x_265, x_205); x_267 = lean_array_push(x_266, x_222); x_268 = lean_array_push(x_267, x_207); x_269 = lean_array_push(x_268, x_264); -x_270 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_270 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_271 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_271, 0, x_186); lean_ctor_set(x_271, 1, x_270); lean_ctor_set(x_271, 2, x_269); x_272 = lean_array_push(x_183, x_170); x_273 = lean_array_push(x_272, x_271); -x_274 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_274 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_275 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_275, 0, x_186); lean_ctor_set(x_275, 1, x_274); @@ -32776,7 +32873,7 @@ x_288 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_288, 0, x_186); lean_ctor_set(x_288, 1, x_8); lean_ctor_set(x_288, 2, x_287); -x_289 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1(x_1, x_288, x_2, x_160); +x_289 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1(x_1, x_288, x_2, x_160); lean_dec(x_2); return x_289; } @@ -32954,7 +33051,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_18222____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -32962,15 +33059,15 @@ x_1 = lean_mk_string_from_bytes("simp_all ", 9); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____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_18331____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; lean_object* x_10; 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; -x_5 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__77; +x_5 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__78; 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_18222____lambda__1___closed__1; +x_9 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1___closed__1; x_10 = l_Lean_mkAtomFrom(x_8, x_9); x_11 = l_Lean_Syntax_setArg(x_6, x_7, x_10); x_12 = l_Lean_mkOptionalNode___closed__2; @@ -32989,7 +33086,7 @@ lean_ctor_set(x_19, 1, x_4); return x_19; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__1() { _start: { lean_object* x_1; @@ -32997,22 +33094,22 @@ 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_18222____closed__2() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__1; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__1; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__3() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__1; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__1; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__2; +x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__2; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -33020,7 +33117,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__4() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__4() { _start: { lean_object* x_1; @@ -33028,41 +33125,41 @@ 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_18222____closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__7; -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__4; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__7; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____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_18222____closed__6() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____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_18222____closed__5; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____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_18222____closed__6; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____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; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222_(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_18331_(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; @@ -33126,12 +33223,12 @@ lean_inc(x_11); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5; 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_18222____closed__3; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7; lean_inc(x_11); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_11); @@ -33208,11 +33305,11 @@ x_68 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_68, 0, x_38); lean_ctor_set(x_68, 1, x_43); lean_ctor_set(x_68, 2, x_67); -x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; lean_inc(x_13); lean_inc(x_14); x_70 = l_Lean_addMacroScope(x_14, x_69, x_13); -x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_11); x_72 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_72, 0, x_11); @@ -33227,10 +33324,10 @@ x_77 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_77, 0, x_38); lean_ctor_set(x_77, 1, x_76); lean_ctor_set(x_77, 2, x_75); -x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_79 = l_Lean_addMacroScope(x_14, x_78, x_13); -x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_11); x_82 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_82, 0, x_11); @@ -33261,7 +33358,7 @@ x_93 = lean_array_push(x_92, x_61); lean_inc(x_93); x_94 = lean_array_push(x_93, x_68); x_95 = lean_array_push(x_94, x_89); -x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_97 = lean_array_push(x_95, x_96); x_98 = lean_array_push(x_97, x_74); lean_inc(x_91); @@ -33276,14 +33373,14 @@ x_103 = lean_array_push(x_102, x_57); x_104 = lean_array_push(x_103, x_74); x_105 = lean_array_push(x_104, x_59); x_106 = lean_array_push(x_105, x_101); -x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_108 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_108, 0, x_38); lean_ctor_set(x_108, 1, x_107); lean_ctor_set(x_108, 2, x_106); x_109 = lean_array_push(x_35, x_22); x_110 = lean_array_push(x_109, x_108); -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_112 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_112, 0, x_38); lean_ctor_set(x_112, 1, x_111); @@ -33334,7 +33431,7 @@ x_139 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_139, 0, x_38); lean_ctor_set(x_139, 1, x_8); lean_ctor_set(x_139, 2, x_138); -x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1(x_1, x_139, x_2, x_12); +x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1(x_1, x_139, x_2, x_12); lean_dec(x_2); return x_140; } @@ -33392,12 +33489,12 @@ lean_inc(x_144); x_162 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_162, 0, x_144); lean_ctor_set(x_162, 1, x_161); -x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5; +x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5; lean_inc(x_146); lean_inc(x_147); x_164 = l_Lean_addMacroScope(x_147, x_163, x_146); -x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__3; -x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7; +x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3; +x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7; lean_inc(x_144); x_167 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_167, 0, x_144); @@ -33474,11 +33571,11 @@ x_201 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_201, 0, x_171); lean_ctor_set(x_201, 1, x_176); lean_ctor_set(x_201, 2, x_200); -x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; lean_inc(x_146); lean_inc(x_147); x_203 = l_Lean_addMacroScope(x_147, x_202, x_146); -x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_144); x_205 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_205, 0, x_144); @@ -33493,10 +33590,10 @@ x_210 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_210, 0, x_171); lean_ctor_set(x_210, 1, x_209); lean_ctor_set(x_210, 2, x_208); -x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_212 = l_Lean_addMacroScope(x_147, x_211, x_146); -x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_144); x_215 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_215, 0, x_144); @@ -33525,7 +33622,7 @@ x_225 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Ta x_226 = lean_array_push(x_225, x_194); x_227 = lean_array_push(x_226, x_201); x_228 = lean_array_push(x_227, x_222); -x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_230 = lean_array_push(x_228, x_229); x_231 = lean_array_push(x_230, x_207); x_232 = lean_array_push(x_231, x_224); @@ -33539,14 +33636,14 @@ x_236 = lean_array_push(x_235, x_190); x_237 = lean_array_push(x_236, x_207); x_238 = lean_array_push(x_237, x_192); x_239 = lean_array_push(x_238, x_234); -x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_241 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_241, 0, x_171); lean_ctor_set(x_241, 1, x_240); lean_ctor_set(x_241, 2, x_239); x_242 = lean_array_push(x_168, x_155); x_243 = lean_array_push(x_242, x_241); -x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_245 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_245, 0, x_171); lean_ctor_set(x_245, 1, x_244); @@ -33573,17 +33670,17 @@ x_258 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_258, 0, x_171); lean_ctor_set(x_258, 1, x_8); lean_ctor_set(x_258, 2, x_257); -x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1(x_1, x_258, x_2, x_145); +x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1(x_1, x_258, x_2, x_145); lean_dec(x_2); return x_259; } } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____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_18331____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_18222____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -33704,7 +33801,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_19156_(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_19265_(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; @@ -33768,12 +33865,12 @@ lean_inc(x_11); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5; 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_18222____closed__3; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7; lean_inc(x_11); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_11); @@ -33850,11 +33947,11 @@ x_68 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_68, 0, x_38); lean_ctor_set(x_68, 1, x_43); lean_ctor_set(x_68, 2, x_67); -x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; lean_inc(x_13); lean_inc(x_14); x_70 = l_Lean_addMacroScope(x_14, x_69, x_13); -x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; +x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; lean_inc(x_11); x_72 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_72, 0, x_11); @@ -33869,10 +33966,10 @@ x_77 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_77, 0, x_38); lean_ctor_set(x_77, 1, x_76); lean_ctor_set(x_77, 2, x_75); -x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_79 = l_Lean_addMacroScope(x_14, x_78, x_13); -x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_11); x_82 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_82, 0, x_11); @@ -33903,7 +34000,7 @@ x_93 = lean_array_push(x_92, x_61); lean_inc(x_93); x_94 = lean_array_push(x_93, x_68); x_95 = lean_array_push(x_94, x_89); -x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_97 = lean_array_push(x_95, x_96); x_98 = lean_array_push(x_97, x_74); lean_inc(x_91); @@ -33918,14 +34015,14 @@ x_103 = lean_array_push(x_102, x_57); x_104 = lean_array_push(x_103, x_74); x_105 = lean_array_push(x_104, x_59); x_106 = lean_array_push(x_105, x_101); -x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_108 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_108, 0, x_38); lean_ctor_set(x_108, 1, x_107); lean_ctor_set(x_108, 2, x_106); x_109 = lean_array_push(x_35, x_22); x_110 = lean_array_push(x_109, x_108); -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_112 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_112, 0, x_38); lean_ctor_set(x_112, 1, x_111); @@ -33976,7 +34073,7 @@ x_139 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_139, 0, x_38); lean_ctor_set(x_139, 1, x_8); lean_ctor_set(x_139, 2, x_138); -x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1(x_1, x_139, x_2, x_12); +x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1(x_1, x_139, x_2, x_12); lean_dec(x_2); return x_140; } @@ -34034,12 +34131,12 @@ lean_inc(x_144); x_162 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_162, 0, x_144); lean_ctor_set(x_162, 1, x_161); -x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5; +x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5; lean_inc(x_146); lean_inc(x_147); x_164 = l_Lean_addMacroScope(x_147, x_163, x_146); -x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__3; -x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7; +x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3; +x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7; lean_inc(x_144); x_167 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_167, 0, x_144); @@ -34116,11 +34213,11 @@ x_201 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_201, 0, x_171); lean_ctor_set(x_201, 1, x_176); lean_ctor_set(x_201, 2, x_200); -x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; +x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; lean_inc(x_146); lean_inc(x_147); x_203 = l_Lean_addMacroScope(x_147, x_202, x_146); -x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; +x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; lean_inc(x_144); x_205 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_205, 0, x_144); @@ -34135,10 +34232,10 @@ x_210 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_210, 0, x_171); lean_ctor_set(x_210, 1, x_209); lean_ctor_set(x_210, 2, x_208); -x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_212 = l_Lean_addMacroScope(x_147, x_211, x_146); -x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_144); x_215 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_215, 0, x_144); @@ -34167,7 +34264,7 @@ x_225 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Ta x_226 = lean_array_push(x_225, x_194); x_227 = lean_array_push(x_226, x_201); x_228 = lean_array_push(x_227, x_222); -x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_230 = lean_array_push(x_228, x_229); x_231 = lean_array_push(x_230, x_207); x_232 = lean_array_push(x_231, x_224); @@ -34181,14 +34278,14 @@ x_236 = lean_array_push(x_235, x_190); x_237 = lean_array_push(x_236, x_207); x_238 = lean_array_push(x_237, x_192); x_239 = lean_array_push(x_238, x_234); -x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_241 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_241, 0, x_171); lean_ctor_set(x_241, 1, x_240); lean_ctor_set(x_241, 2, x_239); x_242 = lean_array_push(x_168, x_155); x_243 = lean_array_push(x_242, x_241); -x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_245 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_245, 0, x_171); lean_ctor_set(x_245, 1, x_244); @@ -34215,7 +34312,7 @@ x_258 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_258, 0, x_171); lean_ctor_set(x_258, 1, x_8); lean_ctor_set(x_258, 2, x_257); -x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1(x_1, x_258, x_2, x_145); +x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1(x_1, x_258, x_2, x_145); lean_dec(x_2); return x_259; } @@ -34337,7 +34434,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_20090_(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_20199_(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; @@ -34401,12 +34498,12 @@ lean_inc(x_11); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5; 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_18222____closed__3; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7; lean_inc(x_11); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_11); @@ -34483,11 +34580,11 @@ x_68 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_68, 0, x_38); lean_ctor_set(x_68, 1, x_43); lean_ctor_set(x_68, 2, x_67); -x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; lean_inc(x_13); lean_inc(x_14); x_70 = l_Lean_addMacroScope(x_14, x_69, x_13); -x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; +x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; lean_inc(x_11); x_72 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_72, 0, x_11); @@ -34502,12 +34599,12 @@ x_77 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_77, 0, x_38); lean_ctor_set(x_77, 1, x_76); lean_ctor_set(x_77, 2, x_75); -x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; lean_inc(x_13); lean_inc(x_14); x_79 = l_Lean_addMacroScope(x_14, x_78, x_13); -x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_11); x_82 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_82, 0, x_11); @@ -34529,9 +34626,9 @@ lean_inc(x_11); x_89 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_89, 0, x_11); lean_ctor_set(x_89, 1, x_88); -x_90 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_90 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; x_91 = l_Lean_addMacroScope(x_14, x_90, x_13); -x_92 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_92 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_11); x_93 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_93, 0, x_11); @@ -34569,7 +34666,7 @@ x_108 = lean_array_push(x_107, x_61); lean_inc(x_108); x_109 = lean_array_push(x_108, x_68); x_110 = lean_array_push(x_109, x_104); -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_112 = lean_array_push(x_110, x_111); x_113 = lean_array_push(x_112, x_74); lean_inc(x_106); @@ -34584,14 +34681,14 @@ x_118 = lean_array_push(x_117, x_57); x_119 = lean_array_push(x_118, x_74); x_120 = lean_array_push(x_119, x_59); x_121 = lean_array_push(x_120, x_116); -x_122 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_122 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_123 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_123, 0, x_38); lean_ctor_set(x_123, 1, x_122); lean_ctor_set(x_123, 2, x_121); x_124 = lean_array_push(x_35, x_22); x_125 = lean_array_push(x_124, x_123); -x_126 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_126 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_127 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_127, 0, x_38); lean_ctor_set(x_127, 1, x_126); @@ -34642,7 +34739,7 @@ x_154 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_154, 0, x_38); lean_ctor_set(x_154, 1, x_8); lean_ctor_set(x_154, 2, x_153); -x_155 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1(x_1, x_154, x_2, x_12); +x_155 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1(x_1, x_154, x_2, x_12); lean_dec(x_2); return x_155; } @@ -34700,12 +34797,12 @@ lean_inc(x_159); x_177 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_177, 0, x_159); lean_ctor_set(x_177, 1, x_176); -x_178 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5; +x_178 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5; lean_inc(x_161); lean_inc(x_162); x_179 = l_Lean_addMacroScope(x_162, x_178, x_161); -x_180 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__3; -x_181 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7; +x_180 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3; +x_181 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7; lean_inc(x_159); x_182 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_182, 0, x_159); @@ -34782,11 +34879,11 @@ x_216 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_216, 0, x_186); lean_ctor_set(x_216, 1, x_191); lean_ctor_set(x_216, 2, x_215); -x_217 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3; +x_217 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3; lean_inc(x_161); lean_inc(x_162); x_218 = l_Lean_addMacroScope(x_162, x_217, x_161); -x_219 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2; +x_219 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2; lean_inc(x_159); x_220 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_220, 0, x_159); @@ -34801,12 +34898,12 @@ x_225 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_225, 0, x_186); lean_ctor_set(x_225, 1, x_224); lean_ctor_set(x_225, 2, x_223); -x_226 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_226 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; lean_inc(x_161); lean_inc(x_162); x_227 = l_Lean_addMacroScope(x_162, x_226, x_161); -x_228 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_228 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_159); x_230 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_230, 0, x_159); @@ -34828,9 +34925,9 @@ lean_inc(x_159); x_237 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_237, 0, x_159); lean_ctor_set(x_237, 1, x_236); -x_238 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_238 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; x_239 = l_Lean_addMacroScope(x_162, x_238, x_161); -x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_159); x_241 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_241, 0, x_159); @@ -34866,7 +34963,7 @@ x_255 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Ta x_256 = lean_array_push(x_255, x_209); x_257 = lean_array_push(x_256, x_216); x_258 = lean_array_push(x_257, x_252); -x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_260 = lean_array_push(x_258, x_259); x_261 = lean_array_push(x_260, x_222); x_262 = lean_array_push(x_261, x_254); @@ -34880,14 +34977,14 @@ x_266 = lean_array_push(x_265, x_205); x_267 = lean_array_push(x_266, x_222); x_268 = lean_array_push(x_267, x_207); x_269 = lean_array_push(x_268, x_264); -x_270 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_270 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_271 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_271, 0, x_186); lean_ctor_set(x_271, 1, x_270); lean_ctor_set(x_271, 2, x_269); x_272 = lean_array_push(x_183, x_170); x_273 = lean_array_push(x_272, x_271); -x_274 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_274 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_275 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_275, 0, x_186); lean_ctor_set(x_275, 1, x_274); @@ -34914,7 +35011,7 @@ x_288 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_288, 0, x_186); lean_ctor_set(x_288, 1, x_8); lean_ctor_set(x_288, 2, x_287); -x_289 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1(x_1, x_288, x_2, x_160); +x_289 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1(x_1, x_288, x_2, x_160); lean_dec(x_2); return x_289; } @@ -35050,7 +35147,7 @@ x_1 = l_Lean_Parser_Tactic_dsimpAutoUnfold___closed__10; return x_1; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -35058,7 +35155,7 @@ x_1 = lean_mk_string_from_bytes("dsimp ", 6); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____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_21241____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; lean_object* x_10; 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; @@ -35066,7 +35163,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_21132____lambda__1___closed__1; +x_9 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1___closed__1; x_10 = l_Lean_mkAtomFrom(x_8, x_9); x_11 = l_Lean_Syntax_setArg(x_6, x_7, x_10); x_12 = l_Lean_mkOptionalNode___closed__2; @@ -35085,7 +35182,7 @@ lean_ctor_set(x_19, 1, x_4); return x_19; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__1() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__1() { _start: { lean_object* x_1; @@ -35093,22 +35190,22 @@ 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_21132____closed__2() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__1; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__1; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__3() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__1; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__1; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__2; +x_3 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__2; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -35116,7 +35213,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__4() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__4() { _start: { lean_object* x_1; @@ -35124,51 +35221,51 @@ 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_21132____closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__tacticErw______1___closed__24; -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__4; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____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_21132____closed__6() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__5; -x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__8; +x_1 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__5; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__8; 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_21132____closed__7() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____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_21132____closed__6; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__6; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__8() { +static lean_object* _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__8() { _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_21132____closed__7; +x_2 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__7; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132_(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_21241_(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; @@ -35232,12 +35329,12 @@ lean_inc(x_11); x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_11); lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__6; +x_30 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__6; 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_21132____closed__3; -x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__8; +x_32 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__3; +x_33 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__8; lean_inc(x_11); x_34 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_34, 0, x_11); @@ -35314,11 +35411,11 @@ x_68 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_68, 0, x_38); lean_ctor_set(x_68, 1, x_43); lean_ctor_set(x_68, 2, x_67); -x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_69 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; lean_inc(x_13); lean_inc(x_14); x_70 = l_Lean_addMacroScope(x_14, x_69, x_13); -x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_71 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_11); x_72 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_72, 0, x_11); @@ -35333,10 +35430,10 @@ x_77 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_77, 0, x_38); lean_ctor_set(x_77, 1, x_76); lean_ctor_set(x_77, 2, x_75); -x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_78 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_79 = l_Lean_addMacroScope(x_14, x_78, x_13); -x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_80 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_81 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_11); x_82 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_82, 0, x_11); @@ -35367,7 +35464,7 @@ x_93 = lean_array_push(x_92, x_61); lean_inc(x_93); x_94 = lean_array_push(x_93, x_68); x_95 = lean_array_push(x_94, x_89); -x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_96 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_97 = lean_array_push(x_95, x_96); x_98 = lean_array_push(x_97, x_74); lean_inc(x_91); @@ -35382,14 +35479,14 @@ x_103 = lean_array_push(x_102, x_57); x_104 = lean_array_push(x_103, x_74); x_105 = lean_array_push(x_104, x_59); x_106 = lean_array_push(x_105, x_101); -x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_107 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_108 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_108, 0, x_38); lean_ctor_set(x_108, 1, x_107); lean_ctor_set(x_108, 2, x_106); x_109 = lean_array_push(x_35, x_22); x_110 = lean_array_push(x_109, x_108); -x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_111 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_112 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_112, 0, x_38); lean_ctor_set(x_112, 1, x_111); @@ -35440,7 +35537,7 @@ x_139 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_139, 0, x_38); lean_ctor_set(x_139, 1, x_8); lean_ctor_set(x_139, 2, x_138); -x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____lambda__1(x_1, x_139, x_2, x_12); +x_140 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1(x_1, x_139, x_2, x_12); lean_dec(x_2); return x_140; } @@ -35498,12 +35595,12 @@ lean_inc(x_144); x_162 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_162, 0, x_144); lean_ctor_set(x_162, 1, x_161); -x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__6; +x_163 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__6; lean_inc(x_146); lean_inc(x_147); x_164 = l_Lean_addMacroScope(x_147, x_163, x_146); -x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__3; -x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__8; +x_165 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__3; +x_166 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__8; lean_inc(x_144); x_167 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_167, 0, x_144); @@ -35580,11 +35677,11 @@ x_201 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_201, 0, x_171); lean_ctor_set(x_201, 1, x_176); lean_ctor_set(x_201, 2, x_200); -x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14; +x_202 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14; lean_inc(x_146); lean_inc(x_147); x_203 = l_Lean_addMacroScope(x_147, x_202, x_146); -x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13; +x_204 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13; lean_inc(x_144); x_205 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_205, 0, x_144); @@ -35599,10 +35696,10 @@ x_210 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_210, 0, x_171); lean_ctor_set(x_210, 1, x_209); lean_ctor_set(x_210, 2, x_208); -x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17; +x_211 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17; x_212 = l_Lean_addMacroScope(x_147, x_211, x_146); -x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16; -x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19; +x_213 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16; +x_214 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19; lean_inc(x_144); x_215 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_215, 0, x_144); @@ -35631,7 +35728,7 @@ x_225 = l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Ta x_226 = lean_array_push(x_225, x_194); x_227 = lean_array_push(x_226, x_201); x_228 = lean_array_push(x_227, x_222); -x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20; +x_229 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20; x_230 = lean_array_push(x_228, x_229); x_231 = lean_array_push(x_230, x_207); x_232 = lean_array_push(x_231, x_224); @@ -35645,14 +35742,14 @@ x_236 = lean_array_push(x_235, x_190); x_237 = lean_array_push(x_236, x_207); x_238 = lean_array_push(x_237, x_192); x_239 = lean_array_push(x_238, x_234); -x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2; +x_240 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2; x_241 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_241, 0, x_171); lean_ctor_set(x_241, 1, x_240); lean_ctor_set(x_241, 2, x_239); x_242 = lean_array_push(x_168, x_155); x_243 = lean_array_push(x_242, x_241); -x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1; +x_244 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1; x_245 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_245, 0, x_171); lean_ctor_set(x_245, 1, x_244); @@ -35679,17 +35776,17 @@ x_258 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_258, 0, x_171); lean_ctor_set(x_258, 1, x_8); lean_ctor_set(x_258, 2, x_257); -x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____lambda__1(x_1, x_258, x_2, x_145); +x_259 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1(x_1, x_258, x_2, x_145); lean_dec(x_2); return x_259; } } } -LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____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_21241____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_21132____lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -36280,54 +36377,54 @@ l_Lean_Meta_instBEqTransparencyMode___closed__1 = _init_l_Lean_Meta_instBEqTrans lean_mark_persistent(l_Lean_Meta_instBEqTransparencyMode___closed__1); l_Lean_Meta_instBEqTransparencyMode = _init_l_Lean_Meta_instBEqTransparencyMode(); lean_mark_persistent(l_Lean_Meta_instBEqTransparencyMode); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__1 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__1(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__1); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__2 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__2(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__2); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__3 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__3(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__3); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__4 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__4(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__4); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__5 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__5(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__5); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__6 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__6(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__6); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__7 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__7(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__7); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__8 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__8(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__8); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__9 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__9(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__9); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__10 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__10(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__10); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__11 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__11(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__11); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__12 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__12(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__12); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__13 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__13(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__13); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__14 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__14(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__14); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__15 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__15(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__15); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__16 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__16(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__16); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__17 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__17(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__17); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__18 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__18(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__18); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__19 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__19(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__19); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__20 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__20(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__20); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__21 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__21(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__21); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__22 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__22(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__22); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__23 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__23(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__23); -l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__24 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__24(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9891____closed__24); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__1 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__1(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__1); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__2 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__2(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__2); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__3 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__3(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__3); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__4 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__4(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__4); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__5 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__5(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__5); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__6 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__6(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__6); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__7 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__7(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__7); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__8 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__8(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__8); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__9 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__9(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__9); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__10 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__10(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__10); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__11 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__11(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__11); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__12 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__12(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__12); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__13 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__13(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__13); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__14 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__14(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__14); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__15 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__15(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__15); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__16 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__16(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__16); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__17 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__17(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__17); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__18 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__18(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__18); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__19 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__19(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__19); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__20 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__20(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__20); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__21 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__21(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__21); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__22 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__22(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__22); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__23 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__23(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__23); +l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__24 = _init_l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__24(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprTransparencyMode____x40_Init_Meta___hyg_9982____closed__24); l_Lean_Meta_instReprTransparencyMode___closed__1 = _init_l_Lean_Meta_instReprTransparencyMode___closed__1(); lean_mark_persistent(l_Lean_Meta_instReprTransparencyMode___closed__1); l_Lean_Meta_instReprTransparencyMode = _init_l_Lean_Meta_instReprTransparencyMode(); @@ -36337,42 +36434,42 @@ l_Lean_Meta_instBEqEtaStructMode___closed__1 = _init_l_Lean_Meta_instBEqEtaStruc lean_mark_persistent(l_Lean_Meta_instBEqEtaStructMode___closed__1); l_Lean_Meta_instBEqEtaStructMode = _init_l_Lean_Meta_instBEqEtaStructMode(); lean_mark_persistent(l_Lean_Meta_instBEqEtaStructMode); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__1 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__1(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__1); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__2 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__2(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__2); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__3 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__3(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__3); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__4 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__4(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__4); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__5 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__5(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__5); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__6 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__6(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__6); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__7 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__7(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__7); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__8 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__8(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__8); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__9 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__9(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__9); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__10 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__10(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__10); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__11 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__11(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__11); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__12 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__12(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__12); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__13 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__13(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__13); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__14 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__14(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__14); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__15 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__15(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__15); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__16 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__16(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__16); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__17 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__17(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__17); -l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__18 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__18(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10056____closed__18); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__1 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__1(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__1); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__2 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__2(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__2); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__3 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__3(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__3); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__4 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__4(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__4); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__5 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__5(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__5); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__6 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__6(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__6); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__7 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__7(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__7); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__8 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__8(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__8); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__9 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__9(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__9); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__10 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__10(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__10); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__11 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__11(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__11); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__12 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__12(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__12); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__13 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__13(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__13); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__14 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__14(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__14); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__15 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__15(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__15); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__16 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__16(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__16); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__17 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__17(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__17); +l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__18 = _init_l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__18(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_reprEtaStructMode____x40_Init_Meta___hyg_10147____closed__18); l_Lean_Meta_instReprEtaStructMode___closed__1 = _init_l_Lean_Meta_instReprEtaStructMode___closed__1(); lean_mark_persistent(l_Lean_Meta_instReprEtaStructMode___closed__1); l_Lean_Meta_instReprEtaStructMode = _init_l_Lean_Meta_instReprEtaStructMode(); @@ -36393,62 +36490,62 @@ l_Lean_Meta_DSimp_instBEqConfig___closed__1 = _init_l_Lean_Meta_DSimp_instBEqCon lean_mark_persistent(l_Lean_Meta_DSimp_instBEqConfig___closed__1); l_Lean_Meta_DSimp_instBEqConfig = _init_l_Lean_Meta_DSimp_instBEqConfig(); lean_mark_persistent(l_Lean_Meta_DSimp_instBEqConfig); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__1 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__1(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__1); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__2 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__2(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__2); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__3 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__3(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__3); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__4 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__4(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__4); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__5); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__6 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__6(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__6); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__7 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__7(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__7); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__8 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__8(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__8); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__9 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__9(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__9); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__10 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__10(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__10); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__11 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__11(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__11); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__12 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__12(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__12); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__13 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__13(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__13); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__14 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__14(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__14); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__15 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__15(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__15); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__16 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__16(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__16); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__17 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__17(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__17); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__18 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__18(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__18); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__19); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__20 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__20(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__20); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__21 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__21(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__21); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__22 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__22(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__22); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__23); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__24); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__25 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__25(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__25); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__26); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__27); -l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10422____closed__28); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__1 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__1(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__1); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__2 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__2(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__2); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__3 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__3(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__3); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__4 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__4(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__4); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__5); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__6 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__6(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__6); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__7 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__7(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__7); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__8 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__8(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__8); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__9 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__9(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__9); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__10 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__10(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__10); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__11 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__11(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__11); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__12 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__12(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__12); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__13 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__13(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__13); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__14 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__14(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__14); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__15 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__15(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__15); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__16 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__16(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__16); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__17 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__17(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__17); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__18 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__18(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__18); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__19); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__20 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__20(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__20); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__21 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__21(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__21); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__22 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__22(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__22); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__23); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__24); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__25 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__25(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__25); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__26); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__27); +l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28 = _init_l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_DSimp_reprConfig____x40_Init_Meta___hyg_10513____closed__28); l_Lean_Meta_DSimp_instReprConfig___closed__1 = _init_l_Lean_Meta_DSimp_instReprConfig___closed__1(); lean_mark_persistent(l_Lean_Meta_DSimp_instReprConfig___closed__1); l_Lean_Meta_DSimp_instReprConfig = _init_l_Lean_Meta_DSimp_instReprConfig(); @@ -36480,38 +36577,38 @@ l_Lean_Meta_Simp_instBEqConfig___closed__1 = _init_l_Lean_Meta_Simp_instBEqConfi lean_mark_persistent(l_Lean_Meta_Simp_instBEqConfig___closed__1); l_Lean_Meta_Simp_instBEqConfig = _init_l_Lean_Meta_Simp_instBEqConfig(); lean_mark_persistent(l_Lean_Meta_Simp_instBEqConfig); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__1 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__1(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__1); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__2 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__2(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__2); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__3 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__3(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__3); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__4 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__4(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__4); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__5 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__5(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__5); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__6 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__6(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__6); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__7 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__7(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__7); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__8 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__8(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__8); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__9 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__9(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__9); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__10 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__10(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__10); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__11 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__11(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__11); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__12 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__12(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__12); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__13); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__14 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__14(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__14); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__15); -l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__16 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__16(); -lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_10980____closed__16); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__1 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__1(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__1); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__2 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__2(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__2); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__3 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__3(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__3); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__4 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__4(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__4); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__5 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__5(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__5); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__6 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__6(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__6); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__7 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__7(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__7); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__8 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__8(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__8); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__9 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__9(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__9); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__10 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__10(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__10); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__11 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__11(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__11); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__12 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__12(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__12); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__13); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__14 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__14(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__14); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__15); +l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__16 = _init_l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__16(); +lean_mark_persistent(l___private_Init_Meta_0__Lean_Meta_Simp_reprConfig____x40_Init_Meta___hyg_11071____closed__16); l_Lean_Meta_Simp_instReprConfig___closed__1 = _init_l_Lean_Meta_Simp_instReprConfig___closed__1(); lean_mark_persistent(l_Lean_Meta_Simp_instReprConfig___closed__1); l_Lean_Meta_Simp_instReprConfig = _init_l_Lean_Meta_Simp_instReprConfig(); @@ -37109,6 +37206,8 @@ l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__co lean_mark_persistent(l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__94); l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__95 = _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__95(); lean_mark_persistent(l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__95); +l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__96 = _init_l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__96(); +lean_mark_persistent(l_Lean_Parser_Tactic___aux__Init__Meta______macroRules__Lean__Parser__Tactic__commandDeclare__simp__like__tactic____________1___closed__96); l_Lean_Parser_Tactic_simpAutoUnfold___closed__1 = _init_l_Lean_Parser_Tactic_simpAutoUnfold___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_simpAutoUnfold___closed__1); l_Lean_Parser_Tactic_simpAutoUnfold___closed__2 = _init_l_Lean_Parser_Tactic_simpAutoUnfold___closed__2(); @@ -37161,48 +37260,48 @@ l_Lean_Parser_Tactic_simpAutoUnfold___closed__25 = _init_l_Lean_Parser_Tactic_si lean_mark_persistent(l_Lean_Parser_Tactic_simpAutoUnfold___closed__25); l_Lean_Parser_Tactic_simpAutoUnfold = _init_l_Lean_Parser_Tactic_simpAutoUnfold(); lean_mark_persistent(l_Lean_Parser_Tactic_simpAutoUnfold); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1___closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____lambda__1___closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__2); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__3(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__3); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__4(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__4); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__5(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__5); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__6(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__6); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__7(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__7); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__8(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__8); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__9); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__10 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__10(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__10); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__11); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__12 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__12(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__12); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__13); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__14); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__15 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__15(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__15); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__16); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__17); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__18 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__18(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__18); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__19); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15282____closed__20); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1___closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____lambda__1___closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__2); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__3(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__3); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__4(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__4); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__5); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__6(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__6); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__7(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__7); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__8(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__8); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__9); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__10 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__10(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__10); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__11); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__12 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__12(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__12); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__13); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__14); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__15 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__15(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__15); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__16); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__17); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__18 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__18(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__18); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__19); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_15391____closed__20); l_Lean_Parser_Tactic_simpArith___closed__1 = _init_l_Lean_Parser_Tactic_simpArith___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_simpArith___closed__1); l_Lean_Parser_Tactic_simpArith___closed__2 = _init_l_Lean_Parser_Tactic_simpArith___closed__2(); @@ -37225,12 +37324,12 @@ l_Lean_Parser_Tactic_simpArith___closed__10 = _init_l_Lean_Parser_Tactic_simpAri lean_mark_persistent(l_Lean_Parser_Tactic_simpArith___closed__10); l_Lean_Parser_Tactic_simpArith = _init_l_Lean_Parser_Tactic_simpArith(); lean_mark_persistent(l_Lean_Parser_Tactic_simpArith); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__2); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16226____closed__3); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__2); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_16335____closed__3); 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(); @@ -37281,22 +37380,22 @@ 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_18222____lambda__1___closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____lambda__1___closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__2(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__2); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__3(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__3); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__4(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__4); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__5); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__6(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__6); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18222____closed__7); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1___closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____lambda__1___closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__2(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__2); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__3); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__4(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__4); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__5); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__6(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__6); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_18331____closed__7); 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(); @@ -37359,24 +37458,24 @@ 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_21132____lambda__1___closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____lambda__1___closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__1(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__1); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__2(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__2); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__3(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__3); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__4(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__4); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__5(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__5); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__6(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__6); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__7(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__7); -l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__8(); -lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21132____closed__8); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1___closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____lambda__1___closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__1 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__1(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__1); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__2 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__2(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__2); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__3 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__3(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__3); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__4 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__4(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__4); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__5 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__5(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__5); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__6 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__6(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__6); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__7 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__7(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__7); +l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__8 = _init_l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__8(); +lean_mark_persistent(l_Lean_Parser_Tactic_expandSimp____x40_Init_Meta___hyg_21241____closed__8); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Notation.c b/stage0/stdlib/Init/Notation.c index 4b2c825b47d5..bc19914ce534 100644 --- a/stage0/stdlib/Init/Notation.c +++ b/stage0/stdlib/Init/Notation.c @@ -200,6 +200,7 @@ static lean_object* l_Lean_Parser_Syntax_addPrec___closed__13; LEAN_EXPORT lean_object* l_term___xd7__; static lean_object* l___aux__Init__Notation______macroRules__term___x3c_x7c_x3e____1___closed__12; static lean_object* l_Lean___aux__Init__Notation______macroRules__Lean__termThis__1___closed__1; +LEAN_EXPORT lean_object* l___aux__Init__Notation______macroRules__term___x5e____2(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Notation______macroRules__term___u2218____1___closed__4; LEAN_EXPORT lean_object* l___aux__Init__Notation______macroRules__term___x2a____2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_rawNatLit; @@ -13658,6 +13659,118 @@ return x_51; } } } +LEAN_EXPORT lean_object* l___aux__Init__Notation______macroRules__term___x5e____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_term___x5e_____closed__2; +lean_inc(x_1); +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +lean_dec(x_1); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_8 = lean_unsigned_to_nat(0u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = lean_unsigned_to_nat(2u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +lean_dec(x_1); +lean_inc(x_2); +x_12 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_2, x_3); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_2, 2); +lean_inc(x_15); +x_16 = lean_ctor_get(x_2, 1); +lean_inc(x_16); +lean_dec(x_2); +x_17 = l___aux__Init__Notation______macroRules__term___x7c_x7c_x7c____2___closed__3; +lean_inc(x_14); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_14); +lean_ctor_set(x_18, 1, x_17); +x_19 = l___aux__Init__Notation______macroRules__term___x5e____1___closed__7; +x_20 = l_Lean_addMacroScope(x_16, x_19, x_15); +x_21 = l___aux__Init__Notation______macroRules__term___x5e____1___closed__3; +x_22 = l___aux__Init__Notation______macroRules__term___x5e____1___closed__9; +x_23 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_23, 0, x_14); +lean_ctor_set(x_23, 1, x_21); +lean_ctor_set(x_23, 2, x_20); +lean_ctor_set(x_23, 3, x_22); +x_24 = l___aux__Init__Notation______macroRules__stx___x2b__1___closed__9; +x_25 = lean_array_push(x_24, x_18); +x_26 = lean_array_push(x_25, x_23); +x_27 = lean_array_push(x_26, x_9); +x_28 = lean_array_push(x_27, x_11); +x_29 = lean_box(2); +x_30 = l___aux__Init__Notation______macroRules__term___x7c_x7c_x7c____2___closed__2; +x_31 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +lean_ctor_set(x_31, 2, x_28); +lean_ctor_set(x_12, 0, x_31); +return x_12; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_32 = lean_ctor_get(x_12, 0); +x_33 = lean_ctor_get(x_12, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_12); +x_34 = lean_ctor_get(x_2, 2); +lean_inc(x_34); +x_35 = lean_ctor_get(x_2, 1); +lean_inc(x_35); +lean_dec(x_2); +x_36 = l___aux__Init__Notation______macroRules__term___x7c_x7c_x7c____2___closed__3; +lean_inc(x_32); +x_37 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_37, 0, x_32); +lean_ctor_set(x_37, 1, x_36); +x_38 = l___aux__Init__Notation______macroRules__term___x5e____1___closed__7; +x_39 = l_Lean_addMacroScope(x_35, x_38, x_34); +x_40 = l___aux__Init__Notation______macroRules__term___x5e____1___closed__3; +x_41 = l___aux__Init__Notation______macroRules__term___x5e____1___closed__9; +x_42 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_42, 0, x_32); +lean_ctor_set(x_42, 1, x_40); +lean_ctor_set(x_42, 2, x_39); +lean_ctor_set(x_42, 3, x_41); +x_43 = l___aux__Init__Notation______macroRules__stx___x2b__1___closed__9; +x_44 = lean_array_push(x_43, x_37); +x_45 = lean_array_push(x_44, x_42); +x_46 = lean_array_push(x_45, x_9); +x_47 = lean_array_push(x_46, x_11); +x_48 = lean_box(2); +x_49 = l___aux__Init__Notation______macroRules__term___x7c_x7c_x7c____2___closed__2; +x_50 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +lean_ctor_set(x_50, 2, x_47); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_33); +return x_51; +} +} +} +} LEAN_EXPORT lean_object* l___aux__Init__Notation______macroRules__term___x2b_x2b____2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { diff --git a/stage0/stdlib/Init/NotationExtra.c b/stage0/stdlib/Init/NotationExtra.c index 799aa220756d..2154a93b8cba 100644 --- a/stage0/stdlib/Init/NotationExtra.c +++ b/stage0/stdlib/Init/NotationExtra.c @@ -16,7 +16,6 @@ extern "C" { static lean_object* l_calcStep___closed__7; static lean_object* l_Lean_termMacro_x2etrace_x5b___x5d_____closed__3; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__28; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13; static lean_object* l_Lean_unbracketedExplicitBinders___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__14; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__termExists___x2c____1(lean_object*, lean_object*, lean_object*); @@ -55,6 +54,7 @@ LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at___aux__Init__NotationExtr static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__19; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__32; static lean_object* l_unexpandListNil___rarg___closed__2; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__7; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__10; static lean_object* l_Lean_doElemWhile__Do_____closed__5; LEAN_EXPORT lean_object* l_term_u03a3___x2c__; @@ -68,11 +68,13 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHeadInfo_x3f(lean_object*); static lean_object* l___aux__Init__NotationExtra______macroRules__command__ClassAbbrev_____x3a___x3a_x3d_____x2c__1___lambda__3___closed__6; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__5; LEAN_EXPORT lean_object* l_unexpandSorryAx(lean_object*, lean_object*, lean_object*); static lean_object* l_termExists___x2c_____closed__5; static lean_object* l_Lean_explicitBinders___closed__4; static lean_object* l_unexpandSubtype___closed__4; static lean_object* l_Lean_unbracketedExplicitBinders___closed__2; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__3; LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at___aux__Init__NotationExtra______macroRules__tactic_xb7_x2e_____x3b____1___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_unifConstraint___closed__8; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__4; @@ -81,6 +83,7 @@ static lean_object* l_calc___closed__12; static lean_object* l_Lean_unifConstraint___closed__2; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___spec__4___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__15; static lean_object* l_tactic_xb7_x2e_____x3b_____closed__5; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__22; static lean_object* l___aux__Init__NotationExtra______macroRules__command__ClassAbbrev_____x3a___x3a_x3d_____x2c__1___lambda__3___closed__5; @@ -91,11 +94,11 @@ uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Array_sequenceMap___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__1___boxed(lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l_Lean_explicitBinders___closed__3; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; static lean_object* l_termExists___x2c_____closed__1; static lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRules__solve__1___spec__3___closed__1; static lean_object* l_Lean_expandExplicitBinders___closed__1; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__solve__1___lambda__1(lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__2; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__23; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__5___closed__7; static lean_object* l_Lean_unifConstraint___closed__3; @@ -136,6 +139,7 @@ static lean_object* l_tactic_xb7_x2e_____x3b_____closed__14; LEAN_EXPORT lean_object* l_Array_sequenceMap___at___aux__Init__NotationExtra______macroRules__solve__1___spec__1(lean_object*, lean_object*); static lean_object* l_unexpandGetElem___closed__3; static lean_object* l_calcStep___closed__10; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; static lean_object* l_calcStep___closed__11; static lean_object* l_unexpandSubtype___closed__2; size_t lean_usize_sub(size_t, size_t); @@ -157,7 +161,6 @@ static lean_object* l_Lean_bracketedExplicitBinders___closed__7; static lean_object* l_unexpandIte___closed__2; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__13; uint8_t lean_name_eq(lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__4; static lean_object* l_term_u03a3___x2c_____closed__5; static lean_object* l_unexpandGetElem_x27___closed__3; static lean_object* l_Lean_doElemRepeat__Until_____closed__6; @@ -193,6 +196,7 @@ lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_expandExplicitBindersAux_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__32; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__10; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; LEAN_EXPORT lean_object* l_unexpandListToArray(lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandGetElem_x3f___closed__5; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__26; @@ -201,8 +205,10 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doE static lean_object* l___aux__Init__NotationExtra______macroRules__command__ClassAbbrev_____x3a___x3a_x3d_____x2c__1___lambda__3___closed__9; static lean_object* l_Lean_bracketedExplicitBinders___closed__3; static lean_object* l_unexpandListToArray___closed__1; +LEAN_EXPORT lean_object* l_Lean_doElemWhile___x3a__Do__; static lean_object* l_Lean_doElemWhile__Do_____closed__2; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__21; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; static lean_object* l_Lean_explicitBinders___closed__1; static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3_x27___x2c____1___closed__1; static lean_object* l_tactic_xb7_x2e_____x3b_____closed__16; @@ -223,7 +229,6 @@ static lean_object* l_tacticFunext_______closed__5; static lean_object* l_unexpandListToArray___closed__2; static lean_object* l___aux__Init__NotationExtra______macroRules__solve__1___closed__2; LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9; static lean_object* l_Lean_unifConstraint___closed__6; static lean_object* l_Lean_doElemRepeat__Until_____closed__2; static lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3_x27___x2c____1___closed__2; @@ -254,7 +259,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__ter static lean_object* l_tactic_xb7_x2e_____x3b_____closed__1; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__20; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__20; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3; static lean_object* l_solve___closed__11; static lean_object* l_Lean_termMacro_x2etrace_x5b___x5d_____closed__13; static lean_object* l_calc___closed__11; @@ -275,6 +279,7 @@ LEAN_EXPORT lean_object* l_Lean_expandBrackedBindersAux_loop___boxed(lean_object static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__7; LEAN_EXPORT lean_object* l_Lean_expandBrackedBindersAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_unexpandSorryAx___closed__1; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__6; LEAN_EXPORT lean_object* l_unexpandGetElem_x3f(lean_object*, lean_object*, lean_object*); static lean_object* l_term___xd7_x27_____closed__2; static lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext______1___closed__8; @@ -315,6 +320,7 @@ static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra___ static lean_object* l___aux__Init__NotationExtra______macroRules__command__ClassAbbrev_____x3a___x3a_x3d_____x2c__1___lambda__3___closed__10; static lean_object* l_Lean_doElemRepeat_____closed__8; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__13; LEAN_EXPORT lean_object* l_Lean_term__Matches___x7c; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__19; static lean_object* l_Lean_unbracketedExplicitBinders___closed__9; @@ -345,7 +351,6 @@ LEAN_EXPORT lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2__; LEAN_EXPORT lean_object* l_unexpandIte(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__16; LEAN_EXPORT lean_object* l_solve; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5; static lean_object* l_termExists___x2c_____closed__4; static lean_object* l_calc___closed__9; static lean_object* l_term___xd7____1___closed__1; @@ -364,7 +369,7 @@ static lean_object* l_solve___closed__6; static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__10; static lean_object* l_tactic_xb7_x2e_____x3b_____closed__23; LEAN_EXPORT lean_object* l_term___xd7____1; -static lean_object* l_Lean_doElemWhile__Do_____closed__7; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__14; static lean_object* l_Lean_explicitBinders___closed__5; static lean_object* l_tactic_xb7_x2e_____x3b_____closed__13; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_expandExplicitBinders___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -400,6 +405,7 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__4; static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__16; static lean_object* l_Lean_unifConstraintElem___closed__11; +LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lean_termMacro_x2etrace_x5b___x5d_____closed__14; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__34; @@ -413,6 +419,7 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__ter static lean_object* l_termExists___x2c_____closed__6; static lean_object* l_Lean_unbracketedExplicitBinders___closed__6; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__7; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; static lean_object* l___aux__Init__NotationExtra______macroRules__command__ClassAbbrev_____x3a___x3a_x3d_____x2c__1___lambda__3___closed__12; static lean_object* l_solve___closed__13; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1(lean_object*, lean_object*, lean_object*); @@ -431,9 +438,8 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__ter LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__5; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__6; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___lambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile__Do_____closed__10; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; static lean_object* l___aux__Init__NotationExtra______macroRules__solve__1___closed__3; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_u03a3_x27___x2c____1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_unifConstraint___closed__10; @@ -473,6 +479,7 @@ static lean_object* l___aux__Init__NotationExtra______macroRules__tactic_xb7_x2e static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__8; static lean_object* l_Array_forInUnsafe_loop___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___spec__5___closed__3; static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__14; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; LEAN_EXPORT lean_object* l_Lean_Loop_forIn(lean_object*, lean_object*); static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__28; static lean_object* l_tacticFunext_______closed__8; @@ -485,6 +492,7 @@ static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__1 static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__18; static lean_object* l_term_u03a3___x2c_____closed__2; static lean_object* l_term___xd7____1___closed__4; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_term_u2203___x2c_____closed__8; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__12; @@ -499,7 +507,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_Lean_bracketedExplicitBinders___closed__8; static lean_object* l_calc___closed__8; static lean_object* l_unexpandListNil___rarg___closed__3; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10; LEAN_EXPORT lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__13; @@ -513,6 +520,7 @@ static lean_object* l_unexpandPSigma___closed__1; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__9; LEAN_EXPORT lean_object* l_unexpandPSigma(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__11; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__40; static lean_object* l_solve___closed__12; static lean_object* l_Lean_termMacro_x2etrace_x5b___x5d_____closed__9; @@ -539,6 +547,7 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doE static lean_object* l_calc___closed__6; lean_object* l_Lean_Macro_throwError___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__2; static lean_object* l_unexpandGetElem___closed__6; LEAN_EXPORT lean_object* l_unexpandListNil___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandTSyntaxArray(lean_object*, lean_object*, lean_object*); @@ -558,11 +567,10 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_unexpandListToArray___closed__3; static lean_object* l_Lean_doElemRepeat_____closed__7; static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__6; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__28; -static lean_object* l_Lean_doElemWhile__Do_____closed__12; static lean_object* l_term_u2203___x2c_____closed__1; static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__6; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_expandExplicitBindersAux_loop___spec__1(lean_object*); static lean_object* l_Lean_termMacro_x2etrace_x5b___x5d_____closed__21; @@ -582,9 +590,11 @@ static lean_object* l_term_u03a3_x27___x2c_____closed__3; static lean_object* l_tactic_xb7_x2e_____x3b_____closed__9; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__25; static lean_object* l_Lean_unbracketedExplicitBinders___closed__10; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__4; static lean_object* l_Lean_termMacro_x2etrace_x5b___x5d_____closed__2; LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__8; lean_object* l_Lean_MacroScopesView_review(lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__42; lean_object* l_Lean_quoteNameMk(lean_object*); @@ -608,6 +618,7 @@ static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra___ static lean_object* l___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___closed__16; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_sequenceMap___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__1; LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__23; LEAN_EXPORT lean_object* l_Lean_doElemRepeat__; @@ -616,10 +627,9 @@ static lean_object* l_tacticFunext_______closed__10; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__13; static lean_object* l_Lean_term__Matches___x7c___closed__2; static lean_object* l_Lean_term__Matches___x7c___closed__1; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; lean_object* l_Array_ofSubarray___rarg(lean_object*); -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7; static lean_object* l_solve___closed__15; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__11; static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__9; lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); static lean_object* l_calc___closed__5; @@ -634,7 +644,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__ter LEAN_EXPORT lean_object* l_unexpandUnit___boxed(lean_object*); static lean_object* l_solve___closed__5; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__2; -static lean_object* l_Lean_doElemWhile__Do_____closed__13; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__17; static lean_object* l_calc___closed__3; static lean_object* l_tactic_xb7_x2e_____x3b_____closed__10; @@ -646,6 +655,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra_ LEAN_EXPORT lean_object* l_Lean_instForInLoopUnit(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_expandBrackedBindersAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__13; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__12; static lean_object* l_tacticCalc_____closed__7; static lean_object* l_term_u2203___x2c_____closed__5; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__22; @@ -676,7 +686,6 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__com static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__14; LEAN_EXPORT lean_object* l_termExists___x2c__; static lean_object* l_Lean_unifConstraintElem___closed__7; -static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__8; LEAN_EXPORT lean_object* l_Lean_expandExplicitBindersAux_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__21; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tactic_xb7_x2e_____x3b____1(lean_object*, lean_object*, lean_object*); @@ -723,6 +732,7 @@ static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__2; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__3; static lean_object* l_term_u03a3___x2c_____closed__4; static lean_object* l___aux__Init__NotationExtra______macroRules__solve__1___closed__4; +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__10; static lean_object* l_Lean_doElemWhile__Do_____closed__4; static lean_object* l___aux__Init__NotationExtra______macroRules__command__ClassAbbrev_____x3a___x3a_x3d_____x2c__1___lambda__3___closed__1; static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__5; @@ -731,8 +741,8 @@ static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__ter static lean_object* l_Lean_expandExplicitBindersAux_loop___closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__24; static lean_object* l_solve___closed__9; -static lean_object* l_Lean_doElemWhile__Do_____closed__8; LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tacticFunext______1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_doElemWhile___x3a__Do_____closed__11; static lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__5___closed__1; static lean_object* l_calc___closed__7; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___aux__Init__NotationExtra______macroRules__term_x25_x5b___x7c___x5d__1___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -740,6 +750,7 @@ static lean_object* l_unexpandGetElem___closed__7; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__19; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__7; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRules__tactic_xb7_x2e_____x3b____1___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__29; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___aux__Init__NotationExtra______macroRules__tactic_xb7_x2e_____x3b____1___spec__3___boxed(lean_object*, lean_object*, lean_object*); @@ -755,7 +766,6 @@ LEAN_EXPORT lean_object* l_Lean_Loop_forIn___rarg(lean_object*, lean_object*, le LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__command__ClassAbbrev_____x3a___x3a_x3d_____x2c__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_unexpandGetElem(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___aux__Init__NotationExtra______macroRules__tactic_xb7_x2e_____x3b____1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_doElemWhile__Do_____closed__9; uint8_t l_Lean_Syntax_matchesIdent(lean_object*, lean_object*); static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__15; static lean_object* l_Lean_unifConstraintElem___closed__10; @@ -772,11 +782,11 @@ static lean_object* l_term___xd7_x27_____closed__5; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat__Until____1___closed__3; static lean_object* l_Lean_command__Unif__hint____Where___x7c_x2d_u22a2_____closed__4; static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__22; +static lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; static lean_object* l_term___xd7_x27_____closed__3; static lean_object* l_tactic_xb7_x2e_____x3b_____closed__12; static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__27; static lean_object* l___aux__Init__NotationExtra______macroRules__command__ClassAbbrev_____x3a___x3a_x3d_____x2c__1___lambda__3___closed__8; -static lean_object* l_Lean_doElemWhile__Do_____closed__11; LEAN_EXPORT lean_object* l_Lean_Loop_toCtorIdx(lean_object*); static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__1; static lean_object* l_command__ClassAbbrev_____x3a___x3a_x3d_____x2c___closed__4; @@ -2153,7 +2163,7 @@ static lean_object* _init_l_Lean_expandExplicitBindersAux_loop___closed__16() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_expandExplicitBindersAux_loop___closed__13; x_2 = l_Lean_expandExplicitBindersAux_loop___closed__14; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_expandExplicitBindersAux_loop___closed__15; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -16918,25 +16928,25 @@ return x_87; } } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__1() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("doElemWhile_Do_", 15); +x_1 = lean_mk_string_from_bytes("doElemWhile_:_Do_", 17); return x_1; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__2() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__2; -x_2 = l_Lean_doElemWhile__Do_____closed__1; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__3() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__3() { _start: { lean_object* x_1; @@ -16944,17 +16954,45 @@ x_1 = lean_mk_string_from_bytes("while ", 6); return x_1; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__4() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile__Do_____closed__3; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__3; x_2 = lean_alloc_ctor(5, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__5() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__6; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; +x_3 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__11; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__6; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__5; +x_3 = l_Lean_unbracketedExplicitBinders___closed__9; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__7() { _start: { lean_object* x_1; @@ -16962,33 +17000,33 @@ x_1 = lean_mk_string_from_bytes("termBeforeDo", 12); return x_1; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__6() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_doElemWhile__Do_____closed__5; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__7() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile__Do_____closed__6; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__8; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__8() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__6; -x_2 = l_Lean_doElemWhile__Do_____closed__4; -x_3 = l_Lean_doElemWhile__Do_____closed__7; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__6; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__9; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16996,7 +17034,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__9() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__11() { _start: { lean_object* x_1; @@ -17004,23 +17042,23 @@ x_1 = lean_mk_string_from_bytes(" do ", 4); return x_1; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__10() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_doElemWhile__Do_____closed__9; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__11; x_2 = lean_alloc_ctor(5, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__11() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__6; -x_2 = l_Lean_doElemWhile__Do_____closed__8; -x_3 = l_Lean_doElemWhile__Do_____closed__10; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__10; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__12; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -17028,12 +17066,12 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__12() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__6; -x_2 = l_Lean_doElemWhile__Do_____closed__11; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__13; x_3 = l_Lean_doElemRepeat_____closed__7; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); @@ -17042,13 +17080,13 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_doElemWhile__Do_____closed__13() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do_____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_doElemWhile__Do_____closed__2; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__2; x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_doElemWhile__Do_____closed__12; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__14; x_4 = lean_alloc_ctor(3, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -17056,15 +17094,15 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_doElemWhile__Do__() { +static lean_object* _init_l_Lean_doElemWhile___x3a__Do__() { _start: { lean_object* x_1; -x_1 = l_Lean_doElemWhile__Do_____closed__13; +x_1 = l_Lean_doElemWhile___x3a__Do_____closed__15; return x_1; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1() { _start: { lean_object* x_1; @@ -17072,7 +17110,7 @@ x_1 = lean_mk_string_from_bytes("repeat", 6); return x_1; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__2() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2() { _start: { lean_object* x_1; @@ -17080,17 +17118,17 @@ x_1 = lean_mk_string_from_bytes("doSeqIndent", 11); return x_1; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__4; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__2; +x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__4() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4() { _start: { lean_object* x_1; @@ -17098,17 +17136,17 @@ x_1 = lean_mk_string_from_bytes("doSeqItem", 9); return x_1; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__4; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__4; +x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__6() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6() { _start: { lean_object* x_1; @@ -17116,17 +17154,17 @@ x_1 = lean_mk_string_from_bytes("doIf", 4); return x_1; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__4; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__6; +x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__8() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8() { _start: { lean_object* x_1; @@ -17134,52 +17172,411 @@ x_1 = lean_mk_string_from_bytes("doIfProp", 8); return x_1; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__4; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__8; +x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("doBreak", 7); +return x_1; +} +} +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__26; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__28; -x_3 = lean_array_push(x_1, x_2); +x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__4; +x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__11() { +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("doBreak", 7); +x_1 = lean_mk_string_from_bytes("break", 5); return x_1; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12() { +LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_doElemWhile___x3a__Do_____closed__2; +lean_inc(x_1); +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +lean_dec(x_1); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = lean_unsigned_to_nat(3u); +x_11 = l_Lean_Syntax_getArg(x_1, x_10); +x_12 = lean_unsigned_to_nat(5u); +x_13 = l_Lean_Syntax_getArg(x_1, x_12); +lean_dec(x_1); +x_14 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_2, x_3); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; 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; +x_16 = lean_ctor_get(x_14, 0); +x_17 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +lean_inc(x_16); +x_18 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_unexpandIte___closed__3; +lean_inc(x_16); +x_20 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_19); +x_21 = l_Lean_expandExplicitBindersAux_loop___closed__12; +lean_inc(x_16); +x_22 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_22, 0, x_16); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__26; +x_24 = lean_array_push(x_23, x_9); +x_25 = lean_array_push(x_24, x_22); +x_26 = lean_box(2); +x_27 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__19; +x_28 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +lean_ctor_set(x_28, 2, x_25); +x_29 = lean_array_push(x_23, x_28); +x_30 = lean_array_push(x_29, x_11); +x_31 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_26); +lean_ctor_set(x_32, 1, x_31); +lean_ctor_set(x_32, 2, x_30); +x_33 = l_unexpandIte___closed__4; +lean_inc(x_16); +x_34 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_34, 0, x_16); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_unexpandIte___closed__5; +lean_inc(x_16); +x_36 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_36, 0, x_16); +lean_ctor_set(x_36, 1, x_35); +x_37 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +x_38 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_38, 0, x_16); +lean_ctor_set(x_38, 1, x_37); +x_39 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__35; +x_40 = lean_array_push(x_39, x_38); +x_41 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; +x_42 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_42, 0, x_26); +lean_ctor_set(x_42, 1, x_41); +lean_ctor_set(x_42, 2, x_40); +x_43 = lean_array_push(x_23, x_42); +x_44 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__28; +x_45 = lean_array_push(x_43, x_44); +x_46 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_26); +lean_ctor_set(x_47, 1, x_46); +lean_ctor_set(x_47, 2, x_45); +x_48 = lean_array_push(x_39, x_47); +x_49 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_49, 0, x_26); +lean_ctor_set(x_49, 1, x_27); +lean_ctor_set(x_49, 2, x_48); +x_50 = lean_array_push(x_39, x_49); +x_51 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +x_52 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_52, 0, x_26); +lean_ctor_set(x_52, 1, x_51); +lean_ctor_set(x_52, 2, x_50); +x_53 = lean_array_push(x_23, x_36); +x_54 = lean_array_push(x_53, x_52); +x_55 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_55, 0, x_26); +lean_ctor_set(x_55, 1, x_27); +lean_ctor_set(x_55, 2, x_54); +x_56 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__28; +x_57 = lean_array_push(x_56, x_20); +x_58 = lean_array_push(x_57, x_32); +x_59 = lean_array_push(x_58, x_34); +x_60 = lean_array_push(x_59, x_13); +x_61 = lean_array_push(x_60, x_44); +x_62 = lean_array_push(x_61, x_55); +x_63 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +x_64 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_64, 0, x_26); +lean_ctor_set(x_64, 1, x_63); +lean_ctor_set(x_64, 2, x_62); +x_65 = lean_array_push(x_23, x_64); +x_66 = lean_array_push(x_65, x_44); +x_67 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_67, 0, x_26); +lean_ctor_set(x_67, 1, x_46); +lean_ctor_set(x_67, 2, x_66); +x_68 = lean_array_push(x_39, x_67); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_26); +lean_ctor_set(x_69, 1, x_27); +lean_ctor_set(x_69, 2, x_68); +x_70 = lean_array_push(x_39, x_69); +x_71 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_71, 0, x_26); +lean_ctor_set(x_71, 1, x_51); +lean_ctor_set(x_71, 2, x_70); +x_72 = lean_array_push(x_23, x_18); +x_73 = lean_array_push(x_72, x_71); +x_74 = l_Lean_doElemRepeat_____closed__2; +x_75 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_75, 0, x_26); +lean_ctor_set(x_75, 1, x_74); +lean_ctor_set(x_75, 2, x_73); +lean_ctor_set(x_14, 0, x_75); +return x_14; +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_76 = lean_ctor_get(x_14, 0); +x_77 = lean_ctor_get(x_14, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_14); +x_78 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; +lean_inc(x_76); +x_79 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_79, 0, x_76); +lean_ctor_set(x_79, 1, x_78); +x_80 = l_unexpandIte___closed__3; +lean_inc(x_76); +x_81 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_81, 0, x_76); +lean_ctor_set(x_81, 1, x_80); +x_82 = l_Lean_expandExplicitBindersAux_loop___closed__12; +lean_inc(x_76); +x_83 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_83, 0, x_76); +lean_ctor_set(x_83, 1, x_82); +x_84 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__26; +x_85 = lean_array_push(x_84, x_9); +x_86 = lean_array_push(x_85, x_83); +x_87 = lean_box(2); +x_88 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__19; +x_89 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +lean_ctor_set(x_89, 2, x_86); +x_90 = lean_array_push(x_84, x_89); +x_91 = lean_array_push(x_90, x_11); +x_92 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; +x_93 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_93, 0, x_87); +lean_ctor_set(x_93, 1, x_92); +lean_ctor_set(x_93, 2, x_91); +x_94 = l_unexpandIte___closed__4; +lean_inc(x_76); +x_95 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_95, 0, x_76); +lean_ctor_set(x_95, 1, x_94); +x_96 = l_unexpandIte___closed__5; +lean_inc(x_76); +x_97 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_97, 0, x_76); +lean_ctor_set(x_97, 1, x_96); +x_98 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; +x_99 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_99, 0, x_76); +lean_ctor_set(x_99, 1, x_98); +x_100 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__35; +x_101 = lean_array_push(x_100, x_99); +x_102 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; +x_103 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_103, 0, x_87); +lean_ctor_set(x_103, 1, x_102); +lean_ctor_set(x_103, 2, x_101); +x_104 = lean_array_push(x_84, x_103); +x_105 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__28; +x_106 = lean_array_push(x_104, x_105); +x_107 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; +x_108 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_108, 0, x_87); +lean_ctor_set(x_108, 1, x_107); +lean_ctor_set(x_108, 2, x_106); +x_109 = lean_array_push(x_100, x_108); +x_110 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_110, 0, x_87); +lean_ctor_set(x_110, 1, x_88); +lean_ctor_set(x_110, 2, x_109); +x_111 = lean_array_push(x_100, x_110); +x_112 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; +x_113 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_113, 0, x_87); +lean_ctor_set(x_113, 1, x_112); +lean_ctor_set(x_113, 2, x_111); +x_114 = lean_array_push(x_84, x_97); +x_115 = lean_array_push(x_114, x_113); +x_116 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_116, 0, x_87); +lean_ctor_set(x_116, 1, x_88); +lean_ctor_set(x_116, 2, x_115); +x_117 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__command__Unif__hint____Where___x7c_x2d_u22a2____1___closed__28; +x_118 = lean_array_push(x_117, x_81); +x_119 = lean_array_push(x_118, x_93); +x_120 = lean_array_push(x_119, x_95); +x_121 = lean_array_push(x_120, x_13); +x_122 = lean_array_push(x_121, x_105); +x_123 = lean_array_push(x_122, x_116); +x_124 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; +x_125 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_125, 0, x_87); +lean_ctor_set(x_125, 1, x_124); +lean_ctor_set(x_125, 2, x_123); +x_126 = lean_array_push(x_84, x_125); +x_127 = lean_array_push(x_126, x_105); +x_128 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_128, 0, x_87); +lean_ctor_set(x_128, 1, x_107); +lean_ctor_set(x_128, 2, x_127); +x_129 = lean_array_push(x_100, x_128); +x_130 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_130, 0, x_87); +lean_ctor_set(x_130, 1, x_88); +lean_ctor_set(x_130, 2, x_129); +x_131 = lean_array_push(x_100, x_130); +x_132 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_132, 0, x_87); +lean_ctor_set(x_132, 1, x_112); +lean_ctor_set(x_132, 2, x_131); +x_133 = lean_array_push(x_84, x_79); +x_134 = lean_array_push(x_133, x_132); +x_135 = l_Lean_doElemRepeat_____closed__2; +x_136 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_136, 0, x_87); +lean_ctor_set(x_136, 1, x_135); +lean_ctor_set(x_136, 2, x_134); +x_137 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set(x_137, 1, x_77); +return x_137; +} +} +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("doElemWhile_Do_", 15); +return x_1; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__4; -x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__11; +x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__2; +x_2 = l_Lean_doElemWhile__Do_____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13() { +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__6; +x_2 = l_Lean_doElemWhile___x3a__Do_____closed__4; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__9; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__6; +x_2 = l_Lean_doElemWhile__Do_____closed__3; +x_3 = l_Lean_doElemWhile___x3a__Do_____closed__12; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_termMacro_x2etrace_x5b___x5d_____closed__6; +x_2 = l_Lean_doElemWhile__Do_____closed__4; +x_3 = l_Lean_doElemRepeat_____closed__7; +x_4 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do_____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_doElemWhile__Do_____closed__2; +x_2 = lean_unsigned_to_nat(1022u); +x_3 = l_Lean_doElemWhile__Do_____closed__5; +x_4 = lean_alloc_ctor(3, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_doElemWhile__Do__() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("break", 5); +x_1 = l_Lean_doElemWhile__Do_____closed__6; return x_1; } } +static lean_object* _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__26; +x_2 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__28; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -17212,7 +17609,7 @@ if (x_13 == 0) { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; 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; x_14 = lean_ctor_get(x_12, 0); -x_15 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1; +x_15 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; lean_inc(x_14); x_16 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_16, 0, x_14); @@ -17222,10 +17619,10 @@ lean_inc(x_14); x_18 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_18, 0, x_14); lean_ctor_set(x_18, 1, x_17); -x_19 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10; +x_19 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1; x_20 = lean_array_push(x_19, x_9); x_21 = lean_box(2); -x_22 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9; +x_22 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; x_23 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_23, 0, x_21); lean_ctor_set(x_23, 1, x_22); @@ -17240,13 +17637,13 @@ lean_inc(x_14); x_27 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_27, 0, x_14); lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13; +x_28 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; x_29 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_29, 0, x_14); lean_ctor_set(x_29, 1, x_28); x_30 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__35; x_31 = lean_array_push(x_30, x_29); -x_32 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12; +x_32 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; x_33 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_33, 0, x_21); lean_ctor_set(x_33, 1, x_32); @@ -17255,7 +17652,7 @@ x_34 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etra x_35 = lean_array_push(x_34, x_33); x_36 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__28; x_37 = lean_array_push(x_35, x_36); -x_38 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5; +x_38 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; x_39 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_39, 0, x_21); lean_ctor_set(x_39, 1, x_38); @@ -17267,7 +17664,7 @@ lean_ctor_set(x_42, 0, x_21); lean_ctor_set(x_42, 1, x_41); lean_ctor_set(x_42, 2, x_40); x_43 = lean_array_push(x_30, x_42); -x_44 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3; +x_44 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; x_45 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_45, 0, x_21); lean_ctor_set(x_45, 1, x_44); @@ -17285,7 +17682,7 @@ x_52 = lean_array_push(x_51, x_25); x_53 = lean_array_push(x_52, x_11); x_54 = lean_array_push(x_53, x_36); x_55 = lean_array_push(x_54, x_48); -x_56 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7; +x_56 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; x_57 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_57, 0, x_21); lean_ctor_set(x_57, 1, x_56); @@ -17324,7 +17721,7 @@ x_70 = lean_ctor_get(x_12, 1); lean_inc(x_70); lean_inc(x_69); lean_dec(x_12); -x_71 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1; +x_71 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; lean_inc(x_69); x_72 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_72, 0, x_69); @@ -17334,10 +17731,10 @@ lean_inc(x_69); x_74 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_74, 0, x_69); lean_ctor_set(x_74, 1, x_73); -x_75 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10; +x_75 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1; x_76 = lean_array_push(x_75, x_9); x_77 = lean_box(2); -x_78 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9; +x_78 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; x_79 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_79, 0, x_77); lean_ctor_set(x_79, 1, x_78); @@ -17352,13 +17749,13 @@ lean_inc(x_69); x_83 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_83, 0, x_69); lean_ctor_set(x_83, 1, x_82); -x_84 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13; +x_84 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; x_85 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_85, 0, x_69); lean_ctor_set(x_85, 1, x_84); x_86 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__35; x_87 = lean_array_push(x_86, x_85); -x_88 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12; +x_88 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; x_89 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_89, 0, x_77); lean_ctor_set(x_89, 1, x_88); @@ -17367,7 +17764,7 @@ x_90 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etra x_91 = lean_array_push(x_90, x_89); x_92 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__termMacro_x2etrace_x5b___x5d____1___closed__28; x_93 = lean_array_push(x_91, x_92); -x_94 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5; +x_94 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; x_95 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_95, 0, x_77); lean_ctor_set(x_95, 1, x_94); @@ -17379,7 +17776,7 @@ lean_ctor_set(x_98, 0, x_77); lean_ctor_set(x_98, 1, x_97); lean_ctor_set(x_98, 2, x_96); x_99 = lean_array_push(x_86, x_98); -x_100 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3; +x_100 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; x_101 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_101, 0, x_77); lean_ctor_set(x_101, 1, x_100); @@ -17397,7 +17794,7 @@ x_108 = lean_array_push(x_107, x_81); x_109 = lean_array_push(x_108, x_11); x_110 = lean_array_push(x_109, x_92); x_111 = lean_array_push(x_110, x_104); -x_112 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7; +x_112 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; x_113 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_113, 0, x_77); lean_ctor_set(x_113, 1, x_112); @@ -17579,7 +17976,7 @@ if (x_13 == 0) { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; 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; x_14 = lean_ctor_get(x_12, 0); -x_15 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1; +x_15 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; lean_inc(x_14); x_16 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_16, 0, x_14); @@ -17612,7 +18009,7 @@ lean_ctor_set(x_30, 1, x_29); lean_ctor_set(x_30, 2, x_28); x_31 = lean_array_push(x_19, x_24); x_32 = lean_array_push(x_31, x_30); -x_33 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5; +x_33 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; x_34 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_34, 0, x_22); lean_ctor_set(x_34, 1, x_33); @@ -17624,7 +18021,7 @@ lean_ctor_set(x_36, 0, x_14); lean_ctor_set(x_36, 1, x_35); x_37 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat__Until____1___closed__3; x_38 = lean_array_push(x_37, x_11); -x_39 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9; +x_39 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; x_40 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_40, 0, x_22); lean_ctor_set(x_40, 1, x_39); @@ -17634,12 +18031,12 @@ lean_inc(x_14); x_42 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_42, 0, x_14); lean_ctor_set(x_42, 1, x_41); -x_43 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13; +x_43 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; x_44 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_44, 0, x_14); lean_ctor_set(x_44, 1, x_43); x_45 = lean_array_push(x_27, x_44); -x_46 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12; +x_46 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; x_47 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_47, 0, x_22); lean_ctor_set(x_47, 1, x_46); @@ -17657,7 +18054,7 @@ lean_ctor_set(x_53, 0, x_22); lean_ctor_set(x_53, 1, x_29); lean_ctor_set(x_53, 2, x_52); x_54 = lean_array_push(x_27, x_53); -x_55 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3; +x_55 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; x_56 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_56, 0, x_22); lean_ctor_set(x_56, 1, x_55); @@ -17669,7 +18066,7 @@ x_60 = lean_array_push(x_59, x_42); x_61 = lean_array_push(x_60, x_56); x_62 = lean_array_push(x_61, x_49); x_63 = lean_array_push(x_62, x_49); -x_64 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7; +x_64 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; x_65 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_65, 0, x_22); lean_ctor_set(x_65, 1, x_64); @@ -17709,7 +18106,7 @@ x_79 = lean_ctor_get(x_12, 1); lean_inc(x_79); lean_inc(x_78); lean_dec(x_12); -x_80 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1; +x_80 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1; lean_inc(x_78); x_81 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_81, 0, x_78); @@ -17742,7 +18139,7 @@ lean_ctor_set(x_95, 1, x_94); lean_ctor_set(x_95, 2, x_93); x_96 = lean_array_push(x_84, x_89); x_97 = lean_array_push(x_96, x_95); -x_98 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5; +x_98 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5; x_99 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_99, 0, x_87); lean_ctor_set(x_99, 1, x_98); @@ -17754,7 +18151,7 @@ lean_ctor_set(x_101, 0, x_78); lean_ctor_set(x_101, 1, x_100); x_102 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat__Until____1___closed__3; x_103 = lean_array_push(x_102, x_11); -x_104 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9; +x_104 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9; x_105 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_105, 0, x_87); lean_ctor_set(x_105, 1, x_104); @@ -17764,12 +18161,12 @@ lean_inc(x_78); x_107 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_107, 0, x_78); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13; +x_108 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12; x_109 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_109, 0, x_78); lean_ctor_set(x_109, 1, x_108); x_110 = lean_array_push(x_92, x_109); -x_111 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12; +x_111 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11; x_112 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_112, 0, x_87); lean_ctor_set(x_112, 1, x_111); @@ -17787,7 +18184,7 @@ lean_ctor_set(x_118, 0, x_87); lean_ctor_set(x_118, 1, x_94); lean_ctor_set(x_118, 2, x_117); x_119 = lean_array_push(x_92, x_118); -x_120 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3; +x_120 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3; x_121 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_121, 0, x_87); lean_ctor_set(x_121, 1, x_120); @@ -17799,7 +18196,7 @@ x_125 = lean_array_push(x_124, x_107); x_126 = lean_array_push(x_125, x_121); x_127 = lean_array_push(x_126, x_114); x_128 = lean_array_push(x_127, x_114); -x_129 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7; +x_129 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7; x_130 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_130, 0, x_87); lean_ctor_set(x_130, 1, x_129); @@ -18329,7 +18726,7 @@ lean_inc(x_15); x_21 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_21, 0, x_15); lean_ctor_set(x_21, 1, x_20); -x_22 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10; +x_22 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1; x_23 = lean_array_push(x_22, x_9); x_24 = lean_box(2); x_25 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__4; @@ -18551,7 +18948,7 @@ lean_inc(x_124); x_131 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_131, 0, x_124); lean_ctor_set(x_131, 1, x_130); -x_132 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10; +x_132 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1; x_133 = lean_array_push(x_132, x_9); x_134 = lean_box(2); x_135 = l_Lean___aux__Init__NotationExtra______macroRules__Lean__term__Matches___x7c__1___closed__4; @@ -19864,6 +20261,62 @@ l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___clo lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__17); l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__18 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__18(); lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemRepeat____1___closed__18); +l_Lean_doElemWhile___x3a__Do_____closed__1 = _init_l_Lean_doElemWhile___x3a__Do_____closed__1(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__1); +l_Lean_doElemWhile___x3a__Do_____closed__2 = _init_l_Lean_doElemWhile___x3a__Do_____closed__2(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__2); +l_Lean_doElemWhile___x3a__Do_____closed__3 = _init_l_Lean_doElemWhile___x3a__Do_____closed__3(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__3); +l_Lean_doElemWhile___x3a__Do_____closed__4 = _init_l_Lean_doElemWhile___x3a__Do_____closed__4(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__4); +l_Lean_doElemWhile___x3a__Do_____closed__5 = _init_l_Lean_doElemWhile___x3a__Do_____closed__5(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__5); +l_Lean_doElemWhile___x3a__Do_____closed__6 = _init_l_Lean_doElemWhile___x3a__Do_____closed__6(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__6); +l_Lean_doElemWhile___x3a__Do_____closed__7 = _init_l_Lean_doElemWhile___x3a__Do_____closed__7(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__7); +l_Lean_doElemWhile___x3a__Do_____closed__8 = _init_l_Lean_doElemWhile___x3a__Do_____closed__8(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__8); +l_Lean_doElemWhile___x3a__Do_____closed__9 = _init_l_Lean_doElemWhile___x3a__Do_____closed__9(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__9); +l_Lean_doElemWhile___x3a__Do_____closed__10 = _init_l_Lean_doElemWhile___x3a__Do_____closed__10(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__10); +l_Lean_doElemWhile___x3a__Do_____closed__11 = _init_l_Lean_doElemWhile___x3a__Do_____closed__11(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__11); +l_Lean_doElemWhile___x3a__Do_____closed__12 = _init_l_Lean_doElemWhile___x3a__Do_____closed__12(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__12); +l_Lean_doElemWhile___x3a__Do_____closed__13 = _init_l_Lean_doElemWhile___x3a__Do_____closed__13(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__13); +l_Lean_doElemWhile___x3a__Do_____closed__14 = _init_l_Lean_doElemWhile___x3a__Do_____closed__14(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__14); +l_Lean_doElemWhile___x3a__Do_____closed__15 = _init_l_Lean_doElemWhile___x3a__Do_____closed__15(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do_____closed__15); +l_Lean_doElemWhile___x3a__Do__ = _init_l_Lean_doElemWhile___x3a__Do__(); +lean_mark_persistent(l_Lean_doElemWhile___x3a__Do__); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__1); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__2); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__3); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__4); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__5); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__6); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__7); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__8); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__9); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__10); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__11); +l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12(); +lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile___x3a__Do____1___closed__12); l_Lean_doElemWhile__Do_____closed__1 = _init_l_Lean_doElemWhile__Do_____closed__1(); lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__1); l_Lean_doElemWhile__Do_____closed__2 = _init_l_Lean_doElemWhile__Do_____closed__2(); @@ -19876,48 +20329,10 @@ l_Lean_doElemWhile__Do_____closed__5 = _init_l_Lean_doElemWhile__Do_____closed__ lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__5); l_Lean_doElemWhile__Do_____closed__6 = _init_l_Lean_doElemWhile__Do_____closed__6(); lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__6); -l_Lean_doElemWhile__Do_____closed__7 = _init_l_Lean_doElemWhile__Do_____closed__7(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__7); -l_Lean_doElemWhile__Do_____closed__8 = _init_l_Lean_doElemWhile__Do_____closed__8(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__8); -l_Lean_doElemWhile__Do_____closed__9 = _init_l_Lean_doElemWhile__Do_____closed__9(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__9); -l_Lean_doElemWhile__Do_____closed__10 = _init_l_Lean_doElemWhile__Do_____closed__10(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__10); -l_Lean_doElemWhile__Do_____closed__11 = _init_l_Lean_doElemWhile__Do_____closed__11(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__11); -l_Lean_doElemWhile__Do_____closed__12 = _init_l_Lean_doElemWhile__Do_____closed__12(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__12); -l_Lean_doElemWhile__Do_____closed__13 = _init_l_Lean_doElemWhile__Do_____closed__13(); -lean_mark_persistent(l_Lean_doElemWhile__Do_____closed__13); l_Lean_doElemWhile__Do__ = _init_l_Lean_doElemWhile__Do__(); lean_mark_persistent(l_Lean_doElemWhile__Do__); l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1(); lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__1); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__2 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__2(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__2); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__3); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__4 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__4(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__4); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__5); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__6 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__6(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__6); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__7); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__8 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__8(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__8); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__9); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__10); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__11 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__11(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__11); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__12); -l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13 = _init_l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13(); -lean_mark_persistent(l_Lean___aux__Init__NotationExtra______macroRules__Lean__doElemWhile__Do____1___closed__13); l_Lean_doElemRepeat__Until_____closed__1 = _init_l_Lean_doElemRepeat__Until_____closed__1(); lean_mark_persistent(l_Lean_doElemRepeat__Until_____closed__1); l_Lean_doElemRepeat__Until_____closed__2 = _init_l_Lean_doElemRepeat__Until_____closed__2(); diff --git a/stage0/stdlib/Init/Util.c b/stage0/stdlib/Init/Util.c index 5a9ad948b2c7..cd89ed1b87ed 100644 --- a/stage0/stdlib/Init/Util.c +++ b/stage0/stdlib/Init/Util.c @@ -41,6 +41,7 @@ lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______ma lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l___aux__Init__Util______macroRules__term_____x5b___x5d___x3f__1___closed__2; +LEAN_EXPORT uint8_t l_ptrEqList___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_withPtrEqDecEq___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); static lean_object* l___aux__Init__Util______macroRules__term_____x5b___x5d___x3f__1___closed__9; @@ -103,13 +104,18 @@ static lean_object* l_getElem_x21___rarg___closed__4; LEAN_EXPORT lean_object* l_panicWithPos(lean_object*); LEAN_EXPORT lean_object* l_panicWithPosWithDecl(lean_object*); LEAN_EXPORT lean_object* l___aux__Init__Util______macroRules__term_____x5b___x5d___x21__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ptrEqList(lean_object*); +LEAN_EXPORT lean_object* l_ptrEq(lean_object*); LEAN_EXPORT lean_object* l_panicWithPosWithDecl___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ptrEqList___rarg___boxed(lean_object*, lean_object*); lean_object* l_panic___rarg(lean_object*, lean_object*); static lean_object* l___aux__Init__Util______macroRules__term_____x5b___x5d___x3f__1___closed__7; static lean_object* l_term_____x5b___x5d___x3f___closed__19; LEAN_EXPORT lean_object* l_getElem_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl___closed__1; +LEAN_EXPORT uint8_t l_ptrEq___rarg(lean_object*, lean_object*); static lean_object* l_term_____x5b___x5d___x3f___closed__14; +LEAN_EXPORT lean_object* l_ptrEq___rarg___boxed(lean_object*, lean_object*); static lean_object* l_term_____x5b___x5d___x3f___closed__22; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_getElem_x3f(lean_object*, lean_object*, lean_object*, lean_object*); @@ -380,6 +386,106 @@ lean_dec(x_1); return x_4; } } +LEAN_EXPORT uint8_t l_ptrEq___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +size_t x_3; size_t x_4; uint8_t x_5; +x_3 = lean_ptr_addr(x_1); +x_4 = lean_ptr_addr(x_2); +x_5 = lean_usize_dec_eq(x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_ptrEq(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ptrEq___rarg___boxed), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ptrEq___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_ptrEq___rarg(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT uint8_t l_ptrEqList___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = 1; +return x_3; +} +else +{ +uint8_t x_4; +x_4 = 0; +return x_4; +} +} +else +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_5; +x_5 = 0; +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; uint8_t x_12; +x_6 = lean_ctor_get(x_1, 0); +x_7 = lean_ctor_get(x_1, 1); +x_8 = lean_ctor_get(x_2, 0); +x_9 = lean_ctor_get(x_2, 1); +x_10 = lean_ptr_addr(x_6); +x_11 = lean_ptr_addr(x_8); +x_12 = lean_usize_dec_eq(x_10, x_11); +if (x_12 == 0) +{ +uint8_t x_13; +x_13 = 0; +return x_13; +} +else +{ +x_1 = x_7; +x_2 = x_9; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_ptrEqList(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ptrEqList___rarg___boxed), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ptrEqList___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_ptrEqList___rarg(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} LEAN_EXPORT lean_object* l_withPtrEqUnsafe___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -494,7 +600,7 @@ static lean_object* _init_l_getElem_x21___rarg___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_getElem_x21___rarg___closed__1; x_2 = l_getElem_x21___rarg___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_getElem_x21___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Class.c b/stage0/stdlib/Lean/Class.c index 5c0aabc6f62e..004aa317e967 100644 --- a/stage0/stdlib/Lean/Class.c +++ b/stage0/stdlib/Lean/Class.c @@ -14,101 +14,110 @@ extern "C" { #endif lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContextCoreM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_hasOutParams___spec__3(lean_object*, size_t, lean_object*); size_t lean_usize_add(size_t, size_t); lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_hasOutParams___spec__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_moveEntries___at_Lean_ClassState_addEntry___spec__9(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__2; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____closed__5; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__3(lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_throwError___at_Lean_registerTagAttribute___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ClassState_switch(lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at_Lean_ClassState_addEntry___spec__2(lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at_Lean_ClassState_addEntry___spec__2(lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Lean_addClass___lambda__2___closed__2; lean_object* lean_array_uget(lean_object*, size_t); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_ClassState_addEntry___spec__10(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__3(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_ClassState_addEntry(lean_object*, lean_object*); uint8_t l_Lean_Name_quickLt(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____closed__3; LEAN_EXPORT lean_object* l_Lean_SMap_contains___at_Lean_isClass___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_addClass___lambda__2___closed__1; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_instInhabitedClassState; LEAN_EXPORT lean_object* l_Lean_classExtension; -LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_hasOutParams___spec__5(lean_object*, lean_object*); +static lean_object* l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__2; size_t lean_usize_sub(size_t, size_t); lean_object* lean_environment_find(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Class_0__Lean_checkOutParam___closed__3; lean_object* lean_st_ref_get(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_mkStateFromImportedEntries___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__1(lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_ClassState_outParamMap___default___spec__2(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____closed__7; LEAN_EXPORT uint8_t l_Lean_ClassEntry_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_SMap_switch___at_Lean_ClassState_switch___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_getOutParamPositions_x3f___spec__5(lean_object*, lean_object*); static lean_object* l___private_Lean_Class_0__Lean_checkOutParam___closed__1; lean_object* lean_expr_instantiate1(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* l_Std_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Class_0__Lean_consumeNLambdas(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__1; size_t lean_usize_shift_right(size_t, size_t); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____closed__6; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__1; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_contains___at_Lean_isClass___spec__3___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(lean_object*, size_t, size_t, lean_object*, uint8_t); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74____closed__4; +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ClassEntry_lt___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Class_0__Lean_checkOutParam___closed__4; lean_object* l_Lean_registerSimplePersistentEnvExtension___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_ClassState_hasOutParam___default___spec__2(lean_object*); size_t lean_uint64_to_usize(uint64_t); -LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_hasOutParams___spec__6(lean_object*, lean_object*); static lean_object* l_Lean_addClass___lambda__2___closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____closed__3; LEAN_EXPORT lean_object* l_Lean_addClass___lambda__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____closed__5; uint64_t l_Lean_Name_hash___override(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); uint8_t l___private_Lean_Attributes_0__Lean_beqAttributeKind____x40_Lean_Attributes___hyg_135_(uint8_t, uint8_t); -LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_ClassState_hasOutParam___default___spec__2___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_SMap_insert___at_Lean_ClassState_addEntry___spec__1(lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l___private_Lean_Class_0__Lean_checkOutParam(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_SMap_insert___at_Lean_ClassState_addEntry___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Class_0__Lean_checkOutParam(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_getOutParamPositions_x3f___spec__2(lean_object*, lean_object*); static lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__3; -static lean_object* l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__1; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAtAux___at_Lean_isClass___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); uint8_t lean_is_out_param(lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_hasOutParams___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkStateFromImportedEntries___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____closed__6; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentHashMap_containsAtAux___at_Lean_isClass___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_isClass___closed__1; +static lean_object* l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__3; LEAN_EXPORT lean_object* l_Lean_isClass___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____closed__7; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); static lean_object* l___private_Lean_Class_0__Lean_checkOutParam___closed__2; lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addClass(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_hasAnyFVar_visit___at___private_Lean_Class_0__Lean_checkOutParam___spec__3(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_hasOutParams___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_left(size_t, size_t); size_t lean_usize_modn(size_t, lean_object*); lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_ClassState_addEntry___spec__6(lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_ClassState_addEntry___spec__6(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1; lean_object* l_Lean_throwError___at_Lean_AttributeImpl_erase___default___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74____closed__6; +uint8_t l_Array_isEmpty___rarg(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78____closed__6; size_t lean_usize_mul(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_addClass___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_getOutParamPositions_x3f___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_hasAnyFVar_visit___at___private_Lean_Class_0__Lean_checkOutParam___spec__3___boxed(lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); @@ -116,86 +125,74 @@ LEAN_EXPORT lean_object* l_Lean_getClassName(lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_value_x3f(lean_object*); lean_object* l_Lean_PersistentEnvExtension_addEntry___rarg(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SimplePersistentEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_getOutParamPositions_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getOutParamPositions_x3f(lean_object*, lean_object*); lean_object* l_Lean_setEnv___at_Lean_registerTagAttribute___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____closed__4; lean_object* l_Lean_Expr_fvar___override(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__2(lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74____closed__5; LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at_Lean_ClassState_addEntry___spec__8(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_getOutParamPositions_x3f___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedClassState___closed__1; static size_t l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__2; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Class_0__Lean_checkOutParam___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_contains___at_Lean_isClass___spec__2___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78____closed__5; static size_t l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__1; lean_object* lean_list_to_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_contains___at_Lean_ClassState_addEntry___spec__7___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_getOutParamPositions_x3f___spec__6___boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_le(size_t, size_t); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78_(lean_object*); static lean_object* l_Lean_instInhabitedClassState___closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____closed__2; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAux___at_Lean_isClass___spec__4___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__2(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74____closed__3; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78____closed__3; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__2(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_addClass___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ClassState_outParamMap___default; LEAN_EXPORT uint8_t l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_addClass___lambda__1___closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____closed__1; lean_object* lean_nat_mul(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78____closed__1; LEAN_EXPORT uint8_t l_Std_PersistentHashMap_contains___at_Lean_isClass___spec__3(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_hasOutParams___spec__6___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__2; -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1; +LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_getOutParamPositions_x3f___spec__6(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentHashMap_containsAux___at_Lean_isClass___spec__4(lean_object*, size_t, lean_object*); LEAN_EXPORT uint8_t l_Std_AssocList_contains___at_Lean_ClassState_addEntry___spec__7(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74____closed__1; -LEAN_EXPORT lean_object* l_Lean_ClassState_hasOutParam___default; -LEAN_EXPORT lean_object* l_Lean_SMap_insert___at_Lean_ClassState_addEntry___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78____closed__4; lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_ClassState_addEntry___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_ClassState_addEntry___spec__4(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Attribute_Builtin_ensureNoArgs(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74____lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at_Lean_ClassState_addEntry___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); -LEAN_EXPORT lean_object* l_Lean_SMap_find_x3f___at_Lean_hasOutParams___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_ClassState_addEntry___spec__6___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____closed__1; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Class_0__Lean_checkOutParam___spec__2(lean_object*, lean_object*, size_t, size_t); +static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78____closed__2; +LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_ClassState_outParamMap___default___spec__2___boxed(lean_object*); lean_object* lean_usize_to_nat(size_t); LEAN_EXPORT lean_object* l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_addClass___closed__1; -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74____closed__2; +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_getOutParamPositions_x3f___spec__3(lean_object*, size_t, lean_object*); uint8_t l_Lean_Expr_hasFVar(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78____lambda__1(lean_object*); LEAN_EXPORT uint8_t l_Lean_SMap_contains___at_Lean_isClass___spec__1(lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); LEAN_EXPORT uint8_t lean_has_out_params(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_hasOutParams___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t lean_is_class(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____closed__4; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_SMap_find_x3f___at_Lean_getOutParamPositions_x3f___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_HashMapImp_contains___at_Lean_isClass___spec__2(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____closed__2; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_hasOutParams___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addClass___lambda__2___closed__4; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_ClassEntry_lt(lean_object* x_1, lean_object* x_2) { _start: { @@ -217,7 +214,7 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_ClassState_hasOutParam___default___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_ClassState_outParamMap___default___spec__2(lean_object* x_1) { _start: { lean_object* x_2; @@ -225,7 +222,7 @@ x_2 = l_Std_mkHashMapImp___rarg(x_1); return x_2; } } -static lean_object* _init_l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__1() { +static lean_object* _init_l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__1() { _start: { lean_object* x_1; @@ -233,21 +230,21 @@ x_1 = l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); return x_1; } } -static lean_object* _init_l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__2() { +static lean_object* _init_l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__1; +x_1 = l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__1; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__3() { +static lean_object* _init_l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__2; +x_1 = l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__2; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -255,14 +252,14 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1() { +static lean_object* _init_l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_1 = lean_unsigned_to_nat(0u); x_2 = l_Std_mkHashMapImp___rarg(x_1); x_3 = 1; -x_4 = l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__3; +x_4 = l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__3; x_5 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_5, 0, x_2); lean_ctor_set(x_5, 1, x_4); @@ -270,19 +267,19 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*2, x_3); return x_5; } } -static lean_object* _init_l_Lean_ClassState_hasOutParam___default() { +static lean_object* _init_l_Lean_ClassState_outParamMap___default() { _start: { lean_object* x_1; -x_1 = l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1; +x_1 = l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1; return x_1; } } -LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_ClassState_hasOutParam___default___spec__2___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_ClassState_outParamMap___default___spec__2___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Std_mkHashMap___at_Lean_ClassState_hasOutParam___default___spec__2(x_1); +x_2 = l_Std_mkHashMap___at_Lean_ClassState_outParamMap___default___spec__2(x_1); lean_dec(x_1); return x_2; } @@ -302,7 +299,7 @@ static lean_object* _init_l_Lean_instInhabitedClassState___closed__2() { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = 1; x_2 = l_Lean_instInhabitedClassState___closed__1; -x_3 = l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__3; +x_3 = l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__3; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_2); lean_ctor_set(x_4, 1, x_3); @@ -332,30 +329,28 @@ return x_6; } else { -lean_object* x_9; lean_object* x_10; uint8_t x_11; uint64_t x_12; size_t x_13; size_t x_14; size_t x_15; size_t x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_9; lean_object* x_10; uint64_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_9 = lean_array_fget(x_2, x_5); x_10 = lean_array_fget(x_3, x_5); -x_11 = lean_unbox(x_10); -lean_dec(x_10); -x_12 = l_Lean_Name_hash___override(x_9); -x_13 = lean_uint64_to_usize(x_12); -x_14 = 1; -x_15 = lean_usize_sub(x_1, x_14); -x_16 = 5; -x_17 = lean_usize_mul(x_16, x_15); -x_18 = lean_usize_shift_right(x_13, x_17); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_add(x_5, x_19); +x_11 = l_Lean_Name_hash___override(x_9); +x_12 = lean_uint64_to_usize(x_11); +x_13 = 1; +x_14 = lean_usize_sub(x_1, x_13); +x_15 = 5; +x_16 = lean_usize_mul(x_15, x_14); +x_17 = lean_usize_shift_right(x_12, x_16); +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_add(x_5, x_18); lean_dec(x_5); -x_21 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_6, x_18, x_1, x_9, x_11); +x_20 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_6, x_17, x_1, x_9, x_10); x_4 = lean_box(0); -x_5 = x_20; -x_6 = x_21; +x_5 = x_19; +x_6 = x_20; goto _start; } } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4) { +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; @@ -373,79 +368,75 @@ lean_dec(x_2); x_9 = !lean_is_exclusive(x_1); if (x_9 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_10 = lean_ctor_get(x_1, 1); lean_dec(x_10); x_11 = lean_ctor_get(x_1, 0); lean_dec(x_11); x_12 = lean_array_push(x_5, x_3); -x_13 = lean_box(x_4); -x_14 = lean_array_push(x_6, x_13); -lean_ctor_set(x_1, 1, x_14); +x_13 = lean_array_push(x_6, x_4); +lean_ctor_set(x_1, 1, x_13); lean_ctor_set(x_1, 0, x_12); return x_1; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_dec(x_1); -x_15 = lean_array_push(x_5, x_3); -x_16 = lean_box(x_4); -x_17 = lean_array_push(x_6, x_16); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_15); -lean_ctor_set(x_18, 1, x_17); -return x_18; +x_14 = lean_array_push(x_5, x_3); +x_15 = lean_array_push(x_6, x_4); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; } } else { -lean_object* x_19; uint8_t x_20; -x_19 = lean_array_fget(x_5, x_2); -x_20 = lean_name_eq(x_3, x_19); -lean_dec(x_19); -if (x_20 == 0) +lean_object* x_17; uint8_t x_18; +x_17 = lean_array_fget(x_5, x_2); +x_18 = lean_name_eq(x_3, x_17); +lean_dec(x_17); +if (x_18 == 0) { -lean_object* x_21; lean_object* x_22; +lean_object* x_19; lean_object* x_20; lean_dec(x_6); lean_dec(x_5); -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_nat_add(x_2, x_21); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_add(x_2, x_19); lean_dec(x_2); -x_2 = x_22; +x_2 = x_20; goto _start; } else { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_1); -if (x_24 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_1); +if (x_22 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_25 = lean_ctor_get(x_1, 1); -lean_dec(x_25); -x_26 = lean_ctor_get(x_1, 0); -lean_dec(x_26); -x_27 = lean_array_fset(x_5, x_2, x_3); -x_28 = lean_box(x_4); -x_29 = lean_array_fset(x_6, x_2, x_28); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = lean_ctor_get(x_1, 1); +lean_dec(x_23); +x_24 = lean_ctor_get(x_1, 0); +lean_dec(x_24); +x_25 = lean_array_fset(x_5, x_2, x_3); +x_26 = lean_array_fset(x_6, x_2, x_4); lean_dec(x_2); -lean_ctor_set(x_1, 1, x_29); -lean_ctor_set(x_1, 0, x_27); +lean_ctor_set(x_1, 1, x_26); +lean_ctor_set(x_1, 0, x_25); return x_1; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_dec(x_1); -x_30 = lean_array_fset(x_5, x_2, x_3); -x_31 = lean_box(x_4); -x_32 = lean_array_fset(x_6, x_2, x_31); +x_27 = lean_array_fset(x_5, x_2, x_3); +x_28 = lean_array_fset(x_6, x_2, x_4); lean_dec(x_2); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_30); -lean_ctor_set(x_33, 1, x_32); -return x_33; +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } @@ -479,7 +470,7 @@ x_1 = l_Std_PersistentHashMap_mkEmptyEntries(lean_box(0), lean_box(0)); return x_1; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, uint8_t x_5) { +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_1) == 0) @@ -501,6 +492,7 @@ lean_dec(x_13); if (x_14 == 0) { lean_dec(x_12); +lean_dec(x_5); lean_dec(x_4); return x_1; } @@ -523,112 +515,107 @@ x_20 = lean_ctor_get(x_15, 1); x_21 = lean_name_eq(x_4, x_19); if (x_21 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_free_object(x_15); -x_22 = lean_box(x_5); -x_23 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_19, x_20, x_4, x_22); -x_24 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_24, 0, x_23); -x_25 = lean_array_fset(x_17, x_12, x_24); +x_22 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_19, x_20, x_4, x_5); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_22); +x_24 = lean_array_fset(x_17, x_12, x_23); lean_dec(x_12); -lean_ctor_set(x_1, 0, x_25); +lean_ctor_set(x_1, 0, x_24); return x_1; } else { -lean_object* x_26; lean_object* x_27; +lean_object* x_25; lean_dec(x_20); lean_dec(x_19); -x_26 = lean_box(x_5); -lean_ctor_set(x_15, 1, x_26); +lean_ctor_set(x_15, 1, x_5); lean_ctor_set(x_15, 0, x_4); -x_27 = lean_array_fset(x_17, x_12, x_15); +x_25 = lean_array_fset(x_17, x_12, x_15); lean_dec(x_12); -lean_ctor_set(x_1, 0, x_27); +lean_ctor_set(x_1, 0, x_25); return x_1; } } else { -lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_28 = lean_ctor_get(x_15, 0); -x_29 = lean_ctor_get(x_15, 1); -lean_inc(x_29); -lean_inc(x_28); +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = lean_ctor_get(x_15, 0); +x_27 = lean_ctor_get(x_15, 1); +lean_inc(x_27); +lean_inc(x_26); lean_dec(x_15); -x_30 = lean_name_eq(x_4, x_28); -if (x_30 == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_31 = lean_box(x_5); -x_32 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_28, x_29, x_4, x_31); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_32); -x_34 = lean_array_fset(x_17, x_12, x_33); +x_28 = lean_name_eq(x_4, x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_26, x_27, x_4, x_5); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = lean_array_fset(x_17, x_12, x_30); lean_dec(x_12); -lean_ctor_set(x_1, 0, x_34); +lean_ctor_set(x_1, 0, x_31); return x_1; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -lean_dec(x_29); -lean_dec(x_28); -x_35 = lean_box(x_5); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_4); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_array_fset(x_17, x_12, x_36); +lean_object* x_32; lean_object* x_33; +lean_dec(x_27); +lean_dec(x_26); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_4); +lean_ctor_set(x_32, 1, x_5); +x_33 = lean_array_fset(x_17, x_12, x_32); lean_dec(x_12); -lean_ctor_set(x_1, 0, x_37); +lean_ctor_set(x_1, 0, x_33); return x_1; } } } case 1: { -uint8_t x_38; -x_38 = !lean_is_exclusive(x_15); -if (x_38 == 0) -{ -lean_object* x_39; size_t x_40; size_t x_41; lean_object* x_42; lean_object* x_43; -x_39 = lean_ctor_get(x_15, 0); -x_40 = lean_usize_shift_right(x_2, x_9); -x_41 = lean_usize_add(x_3, x_8); -x_42 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_39, x_40, x_41, x_4, x_5); -lean_ctor_set(x_15, 0, x_42); -x_43 = lean_array_fset(x_17, x_12, x_15); +uint8_t x_34; +x_34 = !lean_is_exclusive(x_15); +if (x_34 == 0) +{ +lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_39; +x_35 = lean_ctor_get(x_15, 0); +x_36 = lean_usize_shift_right(x_2, x_9); +x_37 = lean_usize_add(x_3, x_8); +x_38 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_35, x_36, x_37, x_4, x_5); +lean_ctor_set(x_15, 0, x_38); +x_39 = lean_array_fset(x_17, x_12, x_15); lean_dec(x_12); -lean_ctor_set(x_1, 0, x_43); +lean_ctor_set(x_1, 0, x_39); return x_1; } else { -lean_object* x_44; size_t x_45; size_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_44 = lean_ctor_get(x_15, 0); -lean_inc(x_44); +lean_object* x_40; size_t x_41; size_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_40 = lean_ctor_get(x_15, 0); +lean_inc(x_40); lean_dec(x_15); -x_45 = lean_usize_shift_right(x_2, x_9); -x_46 = lean_usize_add(x_3, x_8); -x_47 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_44, x_45, x_46, x_4, x_5); -x_48 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_48, 0, x_47); -x_49 = lean_array_fset(x_17, x_12, x_48); +x_41 = lean_usize_shift_right(x_2, x_9); +x_42 = lean_usize_add(x_3, x_8); +x_43 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_40, x_41, x_42, x_4, x_5); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +x_45 = lean_array_fset(x_17, x_12, x_44); lean_dec(x_12); -lean_ctor_set(x_1, 0, x_49); +lean_ctor_set(x_1, 0, x_45); return x_1; } } default: { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_box(x_5); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_4); -lean_ctor_set(x_51, 1, x_50); -x_52 = lean_array_fset(x_17, x_12, x_51); +lean_object* x_46; lean_object* x_47; +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_4); +lean_ctor_set(x_46, 1, x_5); +x_47 = lean_array_fset(x_17, x_12, x_46); lean_dec(x_12); -lean_ctor_set(x_1, 0, x_52); +lean_ctor_set(x_1, 0, x_47); return x_1; } } @@ -636,123 +623,121 @@ return x_1; } else { -lean_object* x_53; size_t x_54; size_t x_55; size_t x_56; size_t x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; -x_53 = lean_ctor_get(x_1, 0); -lean_inc(x_53); +lean_object* x_48; size_t x_49; size_t x_50; size_t x_51; size_t x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_48 = lean_ctor_get(x_1, 0); +lean_inc(x_48); lean_dec(x_1); -x_54 = 1; -x_55 = 5; -x_56 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__2; -x_57 = lean_usize_land(x_2, x_56); -x_58 = lean_usize_to_nat(x_57); -x_59 = lean_array_get_size(x_53); -x_60 = lean_nat_dec_lt(x_58, x_59); -lean_dec(x_59); -if (x_60 == 0) -{ -lean_object* x_61; -lean_dec(x_58); +x_49 = 1; +x_50 = 5; +x_51 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__2; +x_52 = lean_usize_land(x_2, x_51); +x_53 = lean_usize_to_nat(x_52); +x_54 = lean_array_get_size(x_48); +x_55 = lean_nat_dec_lt(x_53, x_54); +lean_dec(x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_53); +lean_dec(x_5); lean_dec(x_4); -x_61 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_61, 0, x_53); -return x_61; +x_56 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_56, 0, x_48); +return x_56; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_array_fget(x_53, x_58); -x_63 = lean_box(0); -x_64 = lean_array_fset(x_53, x_58, x_63); -switch (lean_obj_tag(x_62)) { +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_array_fget(x_48, x_53); +x_58 = lean_box(0); +x_59 = lean_array_fset(x_48, x_53, x_58); +switch (lean_obj_tag(x_57)) { case 0: { -lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; -x_65 = lean_ctor_get(x_62, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_62, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_62)) { - lean_ctor_release(x_62, 0); - lean_ctor_release(x_62, 1); - x_67 = x_62; +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_60 = lean_ctor_get(x_57, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_57, 1); +lean_inc(x_61); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_62 = x_57; } else { - lean_dec_ref(x_62); - x_67 = lean_box(0); -} -x_68 = lean_name_eq(x_4, x_65); -if (x_68 == 0) -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -lean_dec(x_67); -x_69 = lean_box(x_5); -x_70 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_65, x_66, x_4, x_69); -x_71 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_71, 0, x_70); -x_72 = lean_array_fset(x_64, x_58, x_71); -lean_dec(x_58); -x_73 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_73, 0, x_72); -return x_73; -} -else -{ -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -lean_dec(x_66); -lean_dec(x_65); -x_74 = lean_box(x_5); -if (lean_is_scalar(x_67)) { - x_75 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_57); + x_62 = lean_box(0); +} +x_63 = lean_name_eq(x_4, x_60); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_dec(x_62); +x_64 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_60, x_61, x_4, x_5); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = lean_array_fset(x_59, x_53, x_65); +lean_dec(x_53); +x_67 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_67, 0, x_66); +return x_67; +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; +lean_dec(x_61); +lean_dec(x_60); +if (lean_is_scalar(x_62)) { + x_68 = lean_alloc_ctor(0, 2, 0); } else { - x_75 = x_67; + x_68 = x_62; } -lean_ctor_set(x_75, 0, x_4); -lean_ctor_set(x_75, 1, x_74); -x_76 = lean_array_fset(x_64, x_58, x_75); -lean_dec(x_58); -x_77 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_77, 0, x_76); -return x_77; +lean_ctor_set(x_68, 0, x_4); +lean_ctor_set(x_68, 1, x_5); +x_69 = lean_array_fset(x_59, x_53, x_68); +lean_dec(x_53); +x_70 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_70, 0, x_69); +return x_70; } } case 1: { -lean_object* x_78; lean_object* x_79; size_t x_80; size_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_78 = lean_ctor_get(x_62, 0); -lean_inc(x_78); -if (lean_is_exclusive(x_62)) { - lean_ctor_release(x_62, 0); - x_79 = x_62; +lean_object* x_71; lean_object* x_72; size_t x_73; size_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_71 = lean_ctor_get(x_57, 0); +lean_inc(x_71); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + x_72 = x_57; } else { - lean_dec_ref(x_62); - x_79 = lean_box(0); -} -x_80 = lean_usize_shift_right(x_2, x_55); -x_81 = lean_usize_add(x_3, x_54); -x_82 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_78, x_80, x_81, x_4, x_5); -if (lean_is_scalar(x_79)) { - x_83 = lean_alloc_ctor(1, 1, 0); + lean_dec_ref(x_57); + x_72 = lean_box(0); +} +x_73 = lean_usize_shift_right(x_2, x_50); +x_74 = lean_usize_add(x_3, x_49); +x_75 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_71, x_73, x_74, x_4, x_5); +if (lean_is_scalar(x_72)) { + x_76 = lean_alloc_ctor(1, 1, 0); } else { - x_83 = x_79; + x_76 = x_72; } -lean_ctor_set(x_83, 0, x_82); -x_84 = lean_array_fset(x_64, x_58, x_83); -lean_dec(x_58); -x_85 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_85, 0, x_84); -return x_85; +lean_ctor_set(x_76, 0, x_75); +x_77 = lean_array_fset(x_59, x_53, x_76); +lean_dec(x_53); +x_78 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_78, 0, x_77); +return x_78; } default: { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_86 = lean_box(x_5); -x_87 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_87, 0, x_4); -lean_ctor_set(x_87, 1, x_86); -x_88 = lean_array_fset(x_64, x_58, x_87); -lean_dec(x_58); -x_89 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_89, 0, x_88); -return x_89; +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_4); +lean_ctor_set(x_79, 1, x_5); +x_80 = lean_array_fset(x_59, x_53, x_79); +lean_dec(x_53); +x_81 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_81, 0, x_80); +return x_81; } } } @@ -760,96 +745,96 @@ return x_89; } else { -uint8_t x_90; -x_90 = !lean_is_exclusive(x_1); -if (x_90 == 0) +uint8_t x_82; +x_82 = !lean_is_exclusive(x_1); +if (x_82 == 0) { -lean_object* x_91; lean_object* x_92; size_t x_93; uint8_t x_94; -x_91 = lean_unsigned_to_nat(0u); -x_92 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(x_1, x_91, x_4, x_5); -x_93 = 7; -x_94 = lean_usize_dec_le(x_93, x_3); -if (x_94 == 0) +lean_object* x_83; lean_object* x_84; size_t x_85; uint8_t x_86; +x_83 = lean_unsigned_to_nat(0u); +x_84 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(x_1, x_83, x_4, x_5); +x_85 = 7; +x_86 = lean_usize_dec_le(x_85, x_3); +if (x_86 == 0) { -lean_object* x_95; lean_object* x_96; uint8_t x_97; -x_95 = l_Std_PersistentHashMap_getCollisionNodeSize___rarg(x_92); -x_96 = lean_unsigned_to_nat(4u); -x_97 = lean_nat_dec_lt(x_95, x_96); -lean_dec(x_95); -if (x_97 == 0) +lean_object* x_87; lean_object* x_88; uint8_t x_89; +x_87 = l_Std_PersistentHashMap_getCollisionNodeSize___rarg(x_84); +x_88 = lean_unsigned_to_nat(4u); +x_89 = lean_nat_dec_lt(x_87, x_88); +lean_dec(x_87); +if (x_89 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_98 = lean_ctor_get(x_92, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_92, 1); -lean_inc(x_99); -lean_dec(x_92); -x_100 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__3; -x_101 = l_Std_PersistentHashMap_insertAux_traverse___at_Lean_ClassState_addEntry___spec__4(x_3, x_98, x_99, lean_box(0), x_91, x_100); -lean_dec(x_99); -lean_dec(x_98); -return x_101; +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_90 = lean_ctor_get(x_84, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_84, 1); +lean_inc(x_91); +lean_dec(x_84); +x_92 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__3; +x_93 = l_Std_PersistentHashMap_insertAux_traverse___at_Lean_ClassState_addEntry___spec__4(x_3, x_90, x_91, lean_box(0), x_83, x_92); +lean_dec(x_91); +lean_dec(x_90); +return x_93; } else { -return x_92; +return x_84; } } else { -return x_92; +return x_84; } } else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; size_t x_107; uint8_t x_108; -x_102 = lean_ctor_get(x_1, 0); -x_103 = lean_ctor_get(x_1, 1); -lean_inc(x_103); -lean_inc(x_102); +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; size_t x_99; uint8_t x_100; +x_94 = lean_ctor_get(x_1, 0); +x_95 = lean_ctor_get(x_1, 1); +lean_inc(x_95); +lean_inc(x_94); lean_dec(x_1); -x_104 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_104, 0, x_102); -lean_ctor_set(x_104, 1, x_103); -x_105 = lean_unsigned_to_nat(0u); -x_106 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(x_104, x_105, x_4, x_5); -x_107 = 7; -x_108 = lean_usize_dec_le(x_107, x_3); -if (x_108 == 0) -{ -lean_object* x_109; lean_object* x_110; uint8_t x_111; -x_109 = l_Std_PersistentHashMap_getCollisionNodeSize___rarg(x_106); -x_110 = lean_unsigned_to_nat(4u); -x_111 = lean_nat_dec_lt(x_109, x_110); -lean_dec(x_109); -if (x_111 == 0) -{ -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_112 = lean_ctor_get(x_106, 0); -lean_inc(x_112); -x_113 = lean_ctor_get(x_106, 1); -lean_inc(x_113); -lean_dec(x_106); -x_114 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__3; -x_115 = l_Std_PersistentHashMap_insertAux_traverse___at_Lean_ClassState_addEntry___spec__4(x_3, x_112, x_113, lean_box(0), x_105, x_114); -lean_dec(x_113); -lean_dec(x_112); -return x_115; +x_96 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +x_97 = lean_unsigned_to_nat(0u); +x_98 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(x_96, x_97, x_4, x_5); +x_99 = 7; +x_100 = lean_usize_dec_le(x_99, x_3); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; uint8_t x_103; +x_101 = l_Std_PersistentHashMap_getCollisionNodeSize___rarg(x_98); +x_102 = lean_unsigned_to_nat(4u); +x_103 = lean_nat_dec_lt(x_101, x_102); +lean_dec(x_101); +if (x_103 == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_104 = lean_ctor_get(x_98, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_98, 1); +lean_inc(x_105); +lean_dec(x_98); +x_106 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__3; +x_107 = l_Std_PersistentHashMap_insertAux_traverse___at_Lean_ClassState_addEntry___spec__4(x_3, x_104, x_105, lean_box(0), x_97, x_106); +lean_dec(x_105); +lean_dec(x_104); +return x_107; } else { -return x_106; +return x_98; } } else { -return x_106; +return x_98; } } } } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at_Lean_ClassState_addEntry___spec__2(lean_object* x_1, lean_object* x_2, uint8_t x_3) { +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at_Lean_ClassState_addEntry___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -1025,12 +1010,13 @@ lean_ctor_set(x_10, 1, x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(lean_object* x_1, uint8_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) { lean_object* x_4; +lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(0); return x_4; @@ -1055,53 +1041,50 @@ return x_3; } else { -lean_object* x_11; lean_dec(x_7); lean_dec(x_6); -x_11 = lean_box(x_2); -lean_ctor_set(x_3, 1, x_11); +lean_ctor_set(x_3, 1, x_2); lean_ctor_set(x_3, 0, x_1); return x_3; } } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_ctor_get(x_3, 1); -x_14 = lean_ctor_get(x_3, 2); -lean_inc(x_14); +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = lean_ctor_get(x_3, 2); lean_inc(x_13); lean_inc(x_12); +lean_inc(x_11); lean_dec(x_3); -x_15 = lean_name_eq(x_12, x_1); -if (x_15 == 0) +x_14 = lean_name_eq(x_11, x_1); +if (x_14 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(x_1, x_2, x_14); -x_17 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_17, 0, x_12); -lean_ctor_set(x_17, 1, x_13); -lean_ctor_set(x_17, 2, x_16); -return x_17; +lean_object* x_15; lean_object* x_16; +x_15 = l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(x_1, x_2, x_13); +x_16 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_16, 0, x_11); +lean_ctor_set(x_16, 1, x_12); +lean_ctor_set(x_16, 2, x_15); +return x_16; } else { -lean_object* x_18; lean_object* x_19; -lean_dec(x_13); +lean_object* x_17; lean_dec(x_12); -x_18 = lean_box(x_2); -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_1); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set(x_19, 2, x_14); -return x_19; +lean_dec(x_11); +x_17 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_17, 1, x_2); +lean_ctor_set(x_17, 2, x_13); +return x_17; } } } } } -LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_ClassState_addEntry___spec__6(lean_object* x_1, lean_object* x_2, uint8_t x_3) { +LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_ClassState_addEntry___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -1119,104 +1102,102 @@ x_11 = lean_array_uget(x_6, x_10); x_12 = l_Std_AssocList_contains___at_Lean_ClassState_addEntry___spec__7(x_2, x_11); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; x_13 = lean_unsigned_to_nat(1u); x_14 = lean_nat_add(x_5, x_13); lean_dec(x_5); -x_15 = lean_box(x_3); -x_16 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_16, 0, x_2); -lean_ctor_set(x_16, 1, x_15); -lean_ctor_set(x_16, 2, x_11); -x_17 = lean_array_uset(x_6, x_10, x_16); -x_18 = l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(x_14); -x_19 = lean_nat_dec_le(x_18, x_7); +x_15 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_3); +lean_ctor_set(x_15, 2, x_11); +x_16 = lean_array_uset(x_6, x_10, x_15); +x_17 = l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(x_14); +x_18 = lean_nat_dec_le(x_17, x_7); lean_dec(x_7); -lean_dec(x_18); -if (x_19 == 0) +lean_dec(x_17); +if (x_18 == 0) { -lean_object* x_20; +lean_object* x_19; lean_free_object(x_1); -x_20 = l_Std_HashMapImp_expand___at_Lean_ClassState_addEntry___spec__8(x_14, x_17); -return x_20; +x_19 = l_Std_HashMapImp_expand___at_Lean_ClassState_addEntry___spec__8(x_14, x_16); +return x_19; } else { -lean_ctor_set(x_1, 1, x_17); +lean_ctor_set(x_1, 1, x_16); lean_ctor_set(x_1, 0, x_14); return x_1; } } else { -lean_object* x_21; lean_object* x_22; +lean_object* x_20; lean_object* x_21; lean_dec(x_7); -x_21 = l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(x_2, x_3, x_11); -x_22 = lean_array_uset(x_6, x_10, x_21); -lean_ctor_set(x_1, 1, x_22); +x_20 = l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(x_2, x_3, x_11); +x_21 = lean_array_uset(x_6, x_10, x_20); +lean_ctor_set(x_1, 1, x_21); return x_1; } } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint64_t x_26; size_t x_27; size_t x_28; lean_object* x_29; uint8_t x_30; -x_23 = lean_ctor_get(x_1, 0); -x_24 = lean_ctor_get(x_1, 1); -lean_inc(x_24); +lean_object* x_22; lean_object* x_23; lean_object* x_24; uint64_t x_25; size_t x_26; size_t x_27; lean_object* x_28; uint8_t x_29; +x_22 = lean_ctor_get(x_1, 0); +x_23 = lean_ctor_get(x_1, 1); lean_inc(x_23); +lean_inc(x_22); lean_dec(x_1); -x_25 = lean_array_get_size(x_24); -x_26 = l_Lean_Name_hash___override(x_2); -x_27 = lean_uint64_to_usize(x_26); -x_28 = lean_usize_modn(x_27, x_25); -x_29 = lean_array_uget(x_24, x_28); -x_30 = l_Std_AssocList_contains___at_Lean_ClassState_addEntry___spec__7(x_2, x_29); -if (x_30 == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_nat_add(x_23, x_31); -lean_dec(x_23); -x_33 = lean_box(x_3); -x_34 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_34, 0, x_2); -lean_ctor_set(x_34, 1, x_33); -lean_ctor_set(x_34, 2, x_29); -x_35 = lean_array_uset(x_24, x_28, x_34); -x_36 = l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(x_32); -x_37 = lean_nat_dec_le(x_36, x_25); -lean_dec(x_25); -lean_dec(x_36); -if (x_37 == 0) +x_24 = lean_array_get_size(x_23); +x_25 = l_Lean_Name_hash___override(x_2); +x_26 = lean_uint64_to_usize(x_25); +x_27 = lean_usize_modn(x_26, x_24); +x_28 = lean_array_uget(x_23, x_27); +x_29 = l_Std_AssocList_contains___at_Lean_ClassState_addEntry___spec__7(x_2, x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_30 = lean_unsigned_to_nat(1u); +x_31 = lean_nat_add(x_22, x_30); +lean_dec(x_22); +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_2); +lean_ctor_set(x_32, 1, x_3); +lean_ctor_set(x_32, 2, x_28); +x_33 = lean_array_uset(x_23, x_27, x_32); +x_34 = l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(x_31); +x_35 = lean_nat_dec_le(x_34, x_24); +lean_dec(x_24); +lean_dec(x_34); +if (x_35 == 0) { -lean_object* x_38; -x_38 = l_Std_HashMapImp_expand___at_Lean_ClassState_addEntry___spec__8(x_32, x_35); -return x_38; +lean_object* x_36; +x_36 = l_Std_HashMapImp_expand___at_Lean_ClassState_addEntry___spec__8(x_31, x_33); +return x_36; } else { -lean_object* x_39; -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_32); -lean_ctor_set(x_39, 1, x_35); -return x_39; +lean_object* x_37; +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_31); +lean_ctor_set(x_37, 1, x_33); +return x_37; } } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -lean_dec(x_25); -x_40 = l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(x_2, x_3, x_29); -x_41 = lean_array_uset(x_24, x_28, x_40); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_23); -lean_ctor_set(x_42, 1, x_41); -return x_42; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +lean_dec(x_24); +x_38 = l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(x_2, x_3, x_28); +x_39 = lean_array_uset(x_23, x_27, x_38); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_22); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } } } -LEAN_EXPORT lean_object* l_Lean_SMap_insert___at_Lean_ClassState_addEntry___spec__1(lean_object* x_1, lean_object* x_2, uint8_t x_3) { +LEAN_EXPORT lean_object* l_Lean_SMap_insert___at_Lean_ClassState_addEntry___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -1288,10 +1269,11 @@ return x_22; LEAN_EXPORT lean_object* l_Lean_ClassState_addEntry(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; uint8_t x_4; lean_object* x_5; +lean_object* x_3; lean_object* x_4; lean_object* x_5; x_3 = lean_ctor_get(x_2, 0); lean_inc(x_3); -x_4 = lean_ctor_get_uint8(x_2, sizeof(void*)*1); +x_4 = lean_ctor_get(x_2, 1); +lean_inc(x_4); lean_dec(x_2); x_5 = l_Lean_SMap_insert___at_Lean_ClassState_addEntry___spec__1(x_1, x_3, x_4); return x_5; @@ -1309,38 +1291,16 @@ lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -uint8_t x_5; lean_object* x_6; -x_5 = lean_unbox(x_4); -lean_dec(x_4); -x_6 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_ClassState_addEntry___spec__5(x_1, x_2, x_3, x_5); -return x_6; -} -} LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -size_t x_6; size_t x_7; uint8_t x_8; lean_object* x_9; +size_t x_6; size_t x_7; lean_object* x_8; x_6 = lean_unbox_usize(x_2); lean_dec(x_2); x_7 = lean_unbox_usize(x_3); lean_dec(x_3); -x_8 = lean_unbox(x_5); -lean_dec(x_5); -x_9 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_1, x_6, x_7, x_4, x_8); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at_Lean_ClassState_addEntry___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; -x_4 = lean_unbox(x_3); -lean_dec(x_3); -x_5 = l_Std_PersistentHashMap_insert___at_Lean_ClassState_addEntry___spec__2(x_1, x_2, x_4); -return x_5; +x_8 = l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3(x_1, x_6, x_7, x_4, x_5); +return x_8; } } LEAN_EXPORT lean_object* l_Std_AssocList_contains___at_Lean_ClassState_addEntry___spec__7___boxed(lean_object* x_1, lean_object* x_2) { @@ -1354,36 +1314,6 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; -x_4 = lean_unbox(x_2); -lean_dec(x_2); -x_5 = l_Std_AssocList_replace___at_Lean_ClassState_addEntry___spec__11(x_1, x_4, x_3); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_ClassState_addEntry___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; -x_4 = lean_unbox(x_3); -lean_dec(x_3); -x_5 = l_Std_HashMap_insert___at_Lean_ClassState_addEntry___spec__6(x_1, x_2, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_SMap_insert___at_Lean_ClassState_addEntry___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; -x_4 = lean_unbox(x_3); -lean_dec(x_3); -x_5 = l_Lean_SMap_insert___at_Lean_ClassState_addEntry___spec__1(x_1, x_2, x_4); -return x_5; -} -} LEAN_EXPORT lean_object* l_Lean_SMap_switch___at_Lean_ClassState_switch___spec__1(lean_object* x_1) { _start: { @@ -1430,7 +1360,7 @@ x_2 = l_Lean_SMap_switch___at_Lean_ClassState_switch___spec__1(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -1452,7 +1382,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -1490,7 +1420,7 @@ size_t x_15; size_t x_16; lean_object* x_17; x_15 = 0; x_16 = lean_usize_of_nat(x_7); lean_dec(x_7); -x_17 = l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__2(x_6, x_15, x_16, x_4); +x_17 = l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__2(x_6, x_15, x_16, x_4); lean_dec(x_6); x_2 = x_11; x_4 = x_17; @@ -1504,7 +1434,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Lean_mkStateFromImportedEntries___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_mkStateFromImportedEntries___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -1533,24 +1463,24 @@ size_t x_7; size_t x_8; lean_object* x_9; x_7 = 0; x_8 = lean_usize_of_nat(x_3); lean_dec(x_3); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__3(x_2, x_7, x_8, x_1); +x_9 = l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__3(x_2, x_7, x_8, x_1); lean_dec(x_2); return x_9; } } } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1; -x_3 = l_Lean_mkStateFromImportedEntries___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__1(x_2, x_1); +x_2 = l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1; +x_3 = l_Lean_mkStateFromImportedEntries___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__1(x_2, x_1); x_4 = l_Lean_SMap_switch___at_Lean_ClassState_switch___spec__1(x_3); return x_4; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__1() { _start: { lean_object* x_1; @@ -1558,17 +1488,17 @@ x_1 = lean_mk_string_from_bytes("classExt", 8); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_initFn____x40_Lean_Class___hyg_74____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Class___hyg_78____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__3() { _start: { lean_object* x_1; @@ -1577,7 +1507,7 @@ lean_closure_set(x_1, 0, lean_box(0)); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__4() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__4() { _start: { lean_object* x_1; @@ -1585,22 +1515,22 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ClassState_addEntry), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__5() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Class___hyg_74____lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Class___hyg_78____lambda__1), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__6() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_78____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_Class___hyg_74____closed__2; -x_2 = l_Lean_initFn____x40_Lean_Class___hyg_74____closed__4; -x_3 = l_Lean_initFn____x40_Lean_Class___hyg_74____closed__5; -x_4 = l_Lean_initFn____x40_Lean_Class___hyg_74____closed__3; +x_1 = l_Lean_initFn____x40_Lean_Class___hyg_78____closed__2; +x_2 = l_Lean_initFn____x40_Lean_Class___hyg_78____closed__4; +x_3 = l_Lean_initFn____x40_Lean_Class___hyg_78____closed__5; +x_4 = l_Lean_initFn____x40_Lean_Class___hyg_78____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); @@ -1609,16 +1539,16 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_74_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_78_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_initFn____x40_Lean_Class___hyg_74____closed__6; +x_2 = l_Lean_initFn____x40_Lean_Class___hyg_78____closed__6; x_3 = l_Lean_registerSimplePersistentEnvExtension___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -1626,12 +1556,12 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__2(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__2(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -1639,7 +1569,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_74____spec__3(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_initFn____x40_Lean_Class___hyg_78____spec__3(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -1902,7 +1832,7 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_hasOutParams___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_getOutParamPositions_x3f___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; uint8_t x_7; @@ -1934,20 +1864,17 @@ goto _start; } else { -lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_14; lean_object* x_15; x_14 = lean_array_fget(x_2, x_4); lean_dec(x_4); -x_15 = lean_unbox(x_14); -lean_dec(x_14); -x_16 = lean_box(x_15); -x_17 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_17, 0, x_16); -return x_17; +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } } } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_hasOutParams___spec__3(lean_object* x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_getOutParamPositions_x3f___spec__3(lean_object* x_1, size_t x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -2018,14 +1945,14 @@ x_21 = lean_ctor_get(x_1, 1); lean_inc(x_21); lean_dec(x_1); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Std_PersistentHashMap_findAtAux___at_Lean_hasOutParams___spec__4(x_20, x_21, lean_box(0), x_22, x_3); +x_23 = l_Std_PersistentHashMap_findAtAux___at_Lean_getOutParamPositions_x3f___spec__4(x_20, x_21, lean_box(0), x_22, x_3); lean_dec(x_21); lean_dec(x_20); return x_23; } } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_hasOutParams___spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_getOutParamPositions_x3f___spec__2(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; uint64_t x_4; size_t x_5; lean_object* x_6; @@ -2034,12 +1961,12 @@ lean_inc(x_3); lean_dec(x_1); x_4 = l_Lean_Name_hash___override(x_2); x_5 = lean_uint64_to_usize(x_4); -x_6 = l_Std_PersistentHashMap_findAux___at_Lean_hasOutParams___spec__3(x_3, x_5, x_2); +x_6 = l_Std_PersistentHashMap_findAux___at_Lean_getOutParamPositions_x3f___spec__3(x_3, x_5, x_2); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_hasOutParams___spec__6(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_getOutParamPositions_x3f___spec__6(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -2071,7 +1998,7 @@ return x_9; } } } -LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_hasOutParams___spec__5(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_getOutParamPositions_x3f___spec__5(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; uint64_t x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; @@ -2085,13 +2012,13 @@ x_7 = lean_usize_modn(x_6, x_4); lean_dec(x_4); x_8 = lean_array_uget(x_3, x_7); lean_dec(x_3); -x_9 = l_Std_AssocList_find_x3f___at_Lean_hasOutParams___spec__6(x_2, x_8); +x_9 = l_Std_AssocList_find_x3f___at_Lean_getOutParamPositions_x3f___spec__6(x_2, x_8); lean_dec(x_8); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_SMap_find_x3f___at_Lean_hasOutParams___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_SMap_find_x3f___at_Lean_getOutParamPositions_x3f___spec__1(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -2105,11 +2032,11 @@ x_5 = lean_ctor_get(x_1, 1); lean_inc(x_5); lean_dec(x_1); lean_inc(x_2); -x_6 = l_Std_PersistentHashMap_find_x3f___at_Lean_hasOutParams___spec__2(x_5, x_2); +x_6 = l_Std_PersistentHashMap_find_x3f___at_Lean_getOutParamPositions_x3f___spec__2(x_5, x_2); if (lean_obj_tag(x_6) == 0) { lean_object* x_7; -x_7 = l_Std_HashMapImp_find_x3f___at_Lean_hasOutParams___spec__5(x_4, x_2); +x_7 = l_Std_HashMapImp_find_x3f___at_Lean_getOutParamPositions_x3f___spec__5(x_4, x_2); return x_7; } else @@ -2140,12 +2067,12 @@ lean_object* x_11; lean_object* x_12; x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); lean_dec(x_1); -x_12 = l_Std_HashMapImp_find_x3f___at_Lean_hasOutParams___spec__5(x_11, x_2); +x_12 = l_Std_HashMapImp_find_x3f___at_Lean_getOutParamPositions_x3f___spec__5(x_11, x_2); return x_12; } } } -LEAN_EXPORT uint8_t lean_has_out_params(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_getOutParamPositions_x3f(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -2153,57 +2080,76 @@ x_3 = l_Lean_instInhabitedClassState; x_4 = l_Lean_isClass___closed__1; x_5 = l_Lean_SimplePersistentEnvExtension_getState___rarg(x_3, x_4, x_1); lean_dec(x_1); -x_6 = l_Lean_SMap_find_x3f___at_Lean_hasOutParams___spec__1(x_5, x_2); -if (lean_obj_tag(x_6) == 0) -{ -uint8_t x_7; -x_7 = 0; -return x_7; -} -else -{ -lean_object* x_8; uint8_t x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_unbox(x_8); -lean_dec(x_8); -return x_9; -} +x_6 = l_Lean_SMap_find_x3f___at_Lean_getOutParamPositions_x3f___spec__1(x_5, x_2); +return x_6; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_hasOutParams___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_getOutParamPositions_x3f___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Std_PersistentHashMap_findAtAux___at_Lean_hasOutParams___spec__4(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Std_PersistentHashMap_findAtAux___at_Lean_getOutParamPositions_x3f___spec__4(x_1, x_2, x_3, x_4, x_5); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_hasOutParams___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_getOutParamPositions_x3f___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; lean_object* x_5; x_4 = lean_unbox_usize(x_2); lean_dec(x_2); -x_5 = l_Std_PersistentHashMap_findAux___at_Lean_hasOutParams___spec__3(x_1, x_4, x_3); +x_5 = l_Std_PersistentHashMap_findAux___at_Lean_getOutParamPositions_x3f___spec__3(x_1, x_4, x_3); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_hasOutParams___spec__6___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_getOutParamPositions_x3f___spec__6___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_AssocList_find_x3f___at_Lean_hasOutParams___spec__6(x_1, x_2); +x_3 = l_Std_AssocList_find_x3f___at_Lean_getOutParamPositions_x3f___spec__6(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } +LEAN_EXPORT uint8_t lean_has_out_params(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_getOutParamPositions_x3f(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +x_4 = 0; +return x_4; +} +else +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = l_Array_isEmpty___rarg(x_5); +lean_dec(x_5); +if (x_6 == 0) +{ +uint8_t x_7; +x_7 = 1; +return x_7; +} +else +{ +uint8_t x_8; +x_8 = 0; +return x_8; +} +} +} +} LEAN_EXPORT lean_object* l_Lean_hasOutParams___boxed(lean_object* x_1, lean_object* x_2) { _start: { @@ -2447,85 +2393,85 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Class_0__Lean_checkOutParam(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Class_0__Lean_checkOutParam(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -if (lean_obj_tag(x_3) == 7) +if (lean_obj_tag(x_4) == 7) { -lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -x_5 = lean_ctor_get(x_3, 2); +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); -lean_dec(x_3); -lean_inc(x_4); -x_6 = lean_is_out_param(x_4); -if (x_6 == 0) -{ -uint8_t x_7; -x_7 = l_Lean_Expr_hasAnyFVar_visit___at___private_Lean_Class_0__Lean_checkOutParam___spec__3(x_2, x_4); +x_6 = lean_ctor_get(x_4, 2); +lean_inc(x_6); lean_dec(x_4); +lean_inc(x_5); +x_7 = lean_is_out_param(x_5); if (x_7 == 0) { -lean_object* x_8; lean_object* x_9; -x_8 = lean_unsigned_to_nat(1u); -x_9 = lean_nat_add(x_1, x_8); +uint8_t x_8; +x_8 = l_Lean_Expr_hasAnyFVar_visit___at___private_Lean_Class_0__Lean_checkOutParam___spec__3(x_2, x_5); +lean_dec(x_5); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_unsigned_to_nat(1u); +x_10 = lean_nat_add(x_1, x_9); lean_dec(x_1); -x_1 = x_9; -x_3 = x_5; +x_1 = x_10; +x_4 = x_6; goto _start; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_5); +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_dec(x_6); +lean_dec(x_3); lean_dec(x_2); -x_11 = l_Nat_repr(x_1); -x_12 = l___private_Lean_Class_0__Lean_checkOutParam___closed__1; -x_13 = lean_string_append(x_12, x_11); -lean_dec(x_11); -x_14 = l___private_Lean_Class_0__Lean_checkOutParam___closed__2; -x_15 = lean_string_append(x_13, x_14); -x_16 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_16, 0, x_15); -return x_16; +x_12 = lean_unsigned_to_nat(1u); +x_13 = lean_nat_add(x_1, x_12); +lean_dec(x_1); +x_14 = l_Nat_repr(x_13); +x_15 = l___private_Lean_Class_0__Lean_checkOutParam___closed__1; +x_16 = lean_string_append(x_15, x_14); +lean_dec(x_14); +x_17 = l___private_Lean_Class_0__Lean_checkOutParam___closed__2; +x_18 = lean_string_append(x_16, x_17); +x_19 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_19, 0, x_18); +return x_19; } } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_4); -x_17 = lean_array_get_size(x_2); -x_18 = l___private_Lean_Class_0__Lean_checkOutParam___closed__4; -x_19 = l_Lean_Name_num___override(x_18, x_17); -lean_inc(x_19); -x_20 = lean_array_push(x_2, x_19); -x_21 = l_Lean_Expr_fvar___override(x_19); -x_22 = lean_expr_instantiate1(x_5, x_21); -lean_dec(x_21); +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_dec(x_5); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_nat_add(x_1, x_23); -lean_dec(x_1); -x_1 = x_24; -x_2 = x_20; -x_3 = x_22; +x_20 = lean_array_get_size(x_2); +x_21 = l___private_Lean_Class_0__Lean_checkOutParam___closed__4; +x_22 = l_Lean_Name_num___override(x_21, x_20); +lean_inc(x_22); +x_23 = l_Lean_Expr_fvar___override(x_22); +x_24 = lean_expr_instantiate1(x_6, x_23); +lean_dec(x_23); +lean_dec(x_6); +x_25 = lean_unsigned_to_nat(1u); +x_26 = lean_nat_add(x_1, x_25); +x_27 = lean_array_push(x_2, x_22); +x_28 = lean_array_push(x_3, x_1); +x_1 = x_26; +x_2 = x_27; +x_3 = x_28; +x_4 = x_24; goto _start; } } else { -lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; -lean_dec(x_3); -lean_dec(x_1); -x_26 = lean_array_get_size(x_2); +lean_object* x_30; +lean_dec(x_4); lean_dec(x_2); -x_27 = lean_unsigned_to_nat(0u); -x_28 = lean_nat_dec_lt(x_27, x_26); -lean_dec(x_26); -x_29 = lean_box(x_28); +lean_dec(x_1); x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 0, x_3); return x_30; } } @@ -2581,9 +2527,9 @@ LEAN_EXPORT lean_object* l_Lean_addClass___lambda__1(lean_object* x_1, lean_obje { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_5 = l_Lean_ConstantInfo_type(x_1); -x_6 = lean_unsigned_to_nat(1u); +x_6 = lean_unsigned_to_nat(0u); x_7 = l_Lean_addClass___lambda__1___closed__1; -x_8 = l___private_Lean_Class_0__Lean_checkOutParam(x_6, x_7, x_5); +x_8 = l___private_Lean_Class_0__Lean_checkOutParam(x_6, x_7, x_7, x_5); if (lean_obj_tag(x_8) == 0) { uint8_t x_9; @@ -2611,34 +2557,30 @@ uint8_t x_12; x_12 = !lean_is_exclusive(x_8); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; x_13 = lean_ctor_get(x_8, 0); -x_14 = lean_alloc_ctor(0, 1, 1); +x_14 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_14, 0, x_2); -x_15 = lean_unbox(x_13); -lean_dec(x_13); -lean_ctor_set_uint8(x_14, sizeof(void*)*1, x_15); -x_16 = l_Lean_isClass___closed__1; -x_17 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_16, x_3, x_14); -lean_ctor_set(x_8, 0, x_17); +lean_ctor_set(x_14, 1, x_13); +x_15 = l_Lean_isClass___closed__1; +x_16 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_15, x_3, x_14); +lean_ctor_set(x_8, 0, x_16); return x_8; } else { -lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_18 = lean_ctor_get(x_8, 0); -lean_inc(x_18); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_8, 0); +lean_inc(x_17); lean_dec(x_8); -x_19 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_19, 0, x_2); -x_20 = lean_unbox(x_18); -lean_dec(x_18); -lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_20); -x_21 = l_Lean_isClass___closed__1; -x_22 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_21, x_3, x_19); -x_23 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_23, 0, x_22); -return x_23; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_2); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean_isClass___closed__1; +x_20 = l_Lean_PersistentEnvExtension_addEntry___rarg(x_19, x_3, x_18); +x_21 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_21, 0, x_20); +return x_21; } } } @@ -2911,7 +2853,7 @@ x_14 = lean_ctor_get(x_11, 0); lean_inc(x_14); lean_dec(x_11); x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_2, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_15); lean_dec(x_2); x_17 = l___private_Lean_Class_0__Lean_consumeNLambdas(x_16, x_14); if (lean_obj_tag(x_17) == 0) @@ -2969,7 +2911,7 @@ x_26 = lean_ctor_get(x_22, 0); lean_inc(x_26); lean_dec(x_22); x_27 = lean_unsigned_to_nat(0u); -x_28 = l_Lean_Expr_getAppNumArgsAux(x_2, x_27); +x_28 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_27); lean_dec(x_2); x_29 = l___private_Lean_Class_0__Lean_consumeNLambdas(x_28, x_26); if (lean_obj_tag(x_29) == 0) @@ -3004,7 +2946,7 @@ return x_33; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; @@ -3042,7 +2984,7 @@ return x_13; } } } -LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 0) @@ -3055,7 +2997,7 @@ x_6 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_6, 0, x_5); x_7 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_7, 0, x_6); -x_8 = l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__2(x_7, x_2, x_3, x_4); +x_8 = l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__2(x_7, x_2, x_3, x_4); return x_8; } else @@ -3071,12 +3013,12 @@ return x_10; } } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; x_7 = l_Lean_addClass(x_1, x_2); -x_8 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(x_7, x_4, x_5, x_6); +x_8 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(x_7, x_4, x_5, x_6); if (lean_obj_tag(x_8) == 0) { lean_object* x_9; lean_object* x_10; lean_object* x_11; @@ -3112,7 +3054,7 @@ return x_15; } } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__1() { _start: { lean_object* x_1; @@ -3120,16 +3062,16 @@ x_1 = lean_mk_string_from_bytes("invalid attribute 'class', must be global", 41) return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__1; +x_1 = l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; @@ -3158,7 +3100,7 @@ if (x_14 == 0) lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_dec(x_10); lean_dec(x_1); -x_15 = l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__2; +x_15 = l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__2; x_16 = l_Lean_throwError___at_Lean_registerTagAttribute___spec__3(x_15, x_4, x_5, x_12); lean_dec(x_5); lean_dec(x_4); @@ -3185,7 +3127,7 @@ else { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__1(x_10, x_1, x_21, x_4, x_5, x_12); +x_22 = l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__1(x_10, x_1, x_21, x_4, x_5, x_12); lean_dec(x_5); lean_dec(x_4); return x_22; @@ -3219,7 +3161,7 @@ return x_26; } } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__1() { _start: { lean_object* x_1; @@ -3227,25 +3169,25 @@ x_1 = lean_mk_string_from_bytes("attribute cannot be erased", 26); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__1; +x_1 = l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__2; +x_5 = l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__2; x_6 = l_Lean_throwError___at_Lean_AttributeImpl_erase___default___spec__1(x_5, x_2, x_3, x_4); return x_6; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__1() { _start: { lean_object* x_1; @@ -3253,17 +3195,17 @@ x_1 = lean_mk_string_from_bytes("class", 5); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_initFn____x40_Lean_Class___hyg_844____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Class___hyg_853____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__3() { _start: { lean_object* x_1; @@ -3271,12 +3213,12 @@ x_1 = lean_mk_string_from_bytes("type class", 10); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__4() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__4() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; -x_1 = l_Lean_initFn____x40_Lean_Class___hyg_844____closed__2; -x_2 = l_Lean_initFn____x40_Lean_Class___hyg_844____closed__3; +x_1 = l_Lean_initFn____x40_Lean_Class___hyg_853____closed__2; +x_2 = l_Lean_initFn____x40_Lean_Class___hyg_853____closed__3; x_3 = 0; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_1); @@ -3285,29 +3227,29 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__5() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__6() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__7() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_initFn____x40_Lean_Class___hyg_844____closed__4; -x_2 = l_Lean_initFn____x40_Lean_Class___hyg_844____closed__5; -x_3 = l_Lean_initFn____x40_Lean_Class___hyg_844____closed__6; +x_1 = l_Lean_initFn____x40_Lean_Class___hyg_853____closed__4; +x_2 = l_Lean_initFn____x40_Lean_Class___hyg_853____closed__5; +x_3 = l_Lean_initFn____x40_Lean_Class___hyg_853____closed__6; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -3315,61 +3257,61 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_initFn____x40_Lean_Class___hyg_844____closed__7; +x_2 = l_Lean_initFn____x40_Lean_Class___hyg_853____closed__7; x_3 = l_Lean_registerBuiltinAttribute(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__2(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); -x_8 = l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); @@ -3389,16 +3331,16 @@ lean_dec_ref(res); res = initialize_Lean_Attributes(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__1 = _init_l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__1(); -lean_mark_persistent(l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__1); -l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__2 = _init_l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__2(); -lean_mark_persistent(l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__2); -l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__3 = _init_l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__3(); -lean_mark_persistent(l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1___closed__3); -l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1 = _init_l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1(); -lean_mark_persistent(l_Lean_SMap_empty___at_Lean_ClassState_hasOutParam___default___spec__1); -l_Lean_ClassState_hasOutParam___default = _init_l_Lean_ClassState_hasOutParam___default(); -lean_mark_persistent(l_Lean_ClassState_hasOutParam___default); +l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__1 = _init_l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__1(); +lean_mark_persistent(l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__1); +l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__2 = _init_l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__2(); +lean_mark_persistent(l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__2); +l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__3 = _init_l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__3(); +lean_mark_persistent(l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1___closed__3); +l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1 = _init_l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1(); +lean_mark_persistent(l_Lean_SMap_empty___at_Lean_ClassState_outParamMap___default___spec__1); +l_Lean_ClassState_outParamMap___default = _init_l_Lean_ClassState_outParamMap___default(); +lean_mark_persistent(l_Lean_ClassState_outParamMap___default); l_Lean_instInhabitedClassState___closed__1 = _init_l_Lean_instInhabitedClassState___closed__1(); lean_mark_persistent(l_Lean_instInhabitedClassState___closed__1); l_Lean_instInhabitedClassState___closed__2 = _init_l_Lean_instInhabitedClassState___closed__2(); @@ -3409,19 +3351,19 @@ l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___clos l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__2 = _init_l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__2(); l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__3 = _init_l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__3(); lean_mark_persistent(l_Std_PersistentHashMap_insertAux___at_Lean_ClassState_addEntry___spec__3___closed__3); -l_Lean_initFn____x40_Lean_Class___hyg_74____closed__1 = _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_74____closed__1); -l_Lean_initFn____x40_Lean_Class___hyg_74____closed__2 = _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_74____closed__2); -l_Lean_initFn____x40_Lean_Class___hyg_74____closed__3 = _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_74____closed__3); -l_Lean_initFn____x40_Lean_Class___hyg_74____closed__4 = _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__4(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_74____closed__4); -l_Lean_initFn____x40_Lean_Class___hyg_74____closed__5 = _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__5(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_74____closed__5); -l_Lean_initFn____x40_Lean_Class___hyg_74____closed__6 = _init_l_Lean_initFn____x40_Lean_Class___hyg_74____closed__6(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_74____closed__6); -if (builtin) {res = l_Lean_initFn____x40_Lean_Class___hyg_74_(lean_io_mk_world()); +l_Lean_initFn____x40_Lean_Class___hyg_78____closed__1 = _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_78____closed__1); +l_Lean_initFn____x40_Lean_Class___hyg_78____closed__2 = _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_78____closed__2); +l_Lean_initFn____x40_Lean_Class___hyg_78____closed__3 = _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_78____closed__3); +l_Lean_initFn____x40_Lean_Class___hyg_78____closed__4 = _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__4(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_78____closed__4); +l_Lean_initFn____x40_Lean_Class___hyg_78____closed__5 = _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__5(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_78____closed__5); +l_Lean_initFn____x40_Lean_Class___hyg_78____closed__6 = _init_l_Lean_initFn____x40_Lean_Class___hyg_78____closed__6(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_78____closed__6); +if (builtin) {res = l_Lean_initFn____x40_Lean_Class___hyg_78_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_classExtension = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_classExtension); @@ -3448,29 +3390,29 @@ l_Lean_addClass___lambda__2___closed__4 = _init_l_Lean_addClass___lambda__2___cl lean_mark_persistent(l_Lean_addClass___lambda__2___closed__4); l_Lean_addClass___closed__1 = _init_l_Lean_addClass___closed__1(); lean_mark_persistent(l_Lean_addClass___closed__1); -l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__1 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__1); -l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__2 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__2___closed__2); -l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__1 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__1); -l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__2 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____lambda__3___closed__2); -l_Lean_initFn____x40_Lean_Class___hyg_844____closed__1 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____closed__1); -l_Lean_initFn____x40_Lean_Class___hyg_844____closed__2 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____closed__2); -l_Lean_initFn____x40_Lean_Class___hyg_844____closed__3 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____closed__3); -l_Lean_initFn____x40_Lean_Class___hyg_844____closed__4 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__4(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____closed__4); -l_Lean_initFn____x40_Lean_Class___hyg_844____closed__5 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__5(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____closed__5); -l_Lean_initFn____x40_Lean_Class___hyg_844____closed__6 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__6(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____closed__6); -l_Lean_initFn____x40_Lean_Class___hyg_844____closed__7 = _init_l_Lean_initFn____x40_Lean_Class___hyg_844____closed__7(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_844____closed__7); -res = l_Lean_initFn____x40_Lean_Class___hyg_844_(lean_io_mk_world()); +l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__1 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__1); +l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__2 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__2___closed__2); +l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__1 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__1); +l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__2 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____lambda__3___closed__2); +l_Lean_initFn____x40_Lean_Class___hyg_853____closed__1 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____closed__1); +l_Lean_initFn____x40_Lean_Class___hyg_853____closed__2 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____closed__2); +l_Lean_initFn____x40_Lean_Class___hyg_853____closed__3 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____closed__3); +l_Lean_initFn____x40_Lean_Class___hyg_853____closed__4 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__4(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____closed__4); +l_Lean_initFn____x40_Lean_Class___hyg_853____closed__5 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__5(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____closed__5); +l_Lean_initFn____x40_Lean_Class___hyg_853____closed__6 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__6(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____closed__6); +l_Lean_initFn____x40_Lean_Class___hyg_853____closed__7 = _init_l_Lean_initFn____x40_Lean_Class___hyg_853____closed__7(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Class___hyg_853____closed__7); +res = l_Lean_initFn____x40_Lean_Class___hyg_853_(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/ExternAttr.c b/stage0/stdlib/Lean/Compiler/ExternAttr.c index 4c105e49836f..9d3027da538a 100644 --- a/stage0/stdlib/Lean/Compiler/ExternAttr.c +++ b/stage0/stdlib/Lean/Compiler/ExternAttr.c @@ -43,7 +43,6 @@ static lean_object* l___private_Lean_Compiler_ExternAttr_0__Lean_getExternConstA lean_object* lean_environment_find(lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedExternAttrData___closed__1; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Compiler_ExternAttr___hyg_639____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_expandExternPattern(lean_object*, lean_object*); static lean_object* l___private_Lean_Compiler_ExternAttr_0__Lean_getExternConstArity___closed__6; lean_object* lean_st_ref_get(lean_object*, lean_object*); @@ -51,8 +50,10 @@ uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Compiler_ExternAttr___hyg_639____closed__7; lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +lean_object* l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ExternEntry_backend___boxed(lean_object*); +uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExternNameFor(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Compiler_ExternAttr_0__Lean_getExternConstArity___closed__22; LEAN_EXPORT lean_object* l___private_Lean_Compiler_ExternAttr_0__Lean_syntaxToExternAttrData___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -116,7 +117,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Compiler_ExternAt static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Compiler_ExternAttr_0__Lean_syntaxToExternAttrData___spec__3___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Compiler_ExternAttr_0__Lean_syntaxToExternAttrData(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); -uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Compiler_ExternAttr_0__Lean_syntaxToExternAttrData___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -685,7 +685,7 @@ else { lean_object* x_17; uint8_t x_18; x_17 = lean_box(0); -x_18 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_14, x_17); +x_18 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_14, x_17); if (x_18 == 0) { lean_object* x_19; lean_object* x_20; @@ -821,7 +821,7 @@ else lean_object* x_16; lean_object* x_17; lean_free_object(x_6); x_16 = lean_add_extern(x_10, x_1); -x_17 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(x_16, x_3, x_4, x_9); +x_17 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(x_16, x_3, x_4, x_9); if (lean_obj_tag(x_17) == 0) { lean_object* x_18; lean_object* x_19; lean_object* x_20; @@ -862,7 +862,7 @@ else lean_object* x_25; lean_object* x_26; lean_free_object(x_6); x_25 = lean_add_extern(x_10, x_1); -x_26 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(x_25, x_3, x_4, x_9); +x_26 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(x_25, x_3, x_4, x_9); if (lean_obj_tag(x_26) == 0) { lean_object* x_27; lean_object* x_28; lean_object* x_29; @@ -935,7 +935,7 @@ else { lean_object* x_43; lean_object* x_44; x_43 = lean_add_extern(x_36, x_1); -x_44 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(x_43, x_3, x_4, x_35); +x_44 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(x_43, x_3, x_4, x_35); if (lean_obj_tag(x_44) == 0) { lean_object* x_45; lean_object* x_46; lean_object* x_47; @@ -977,7 +977,7 @@ else { lean_object* x_52; lean_object* x_53; x_52 = lean_add_extern(x_36, x_1); -x_53 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_844____spec__1(x_52, x_3, x_4, x_35); +x_53 = l_Lean_ofExcept___at_Lean_initFn____x40_Lean_Class___hyg_853____spec__1(x_52, x_3, x_4, x_35); if (lean_obj_tag(x_53) == 0) { lean_object* x_54; lean_object* x_55; lean_object* x_56; diff --git a/stage0/stdlib/Lean/Compiler/IR/Basic.c b/stage0/stdlib/Lean/Compiler/IR/Basic.c index c34a0434f7d6..16ab2a8556df 100644 --- a/stage0/stdlib/Lean/Compiler/IR/Basic.c +++ b/stage0/stdlib/Lean/Compiler/IR/Basic.c @@ -12616,7 +12616,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_IR_addParamsRename___ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_IR_addParamsRename___spec__2___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_IR_addParamsRename___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_IR_addParamsRename___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Compiler/IR/Borrow.c b/stage0/stdlib/Lean/Compiler/IR/Borrow.c index 0d114aa6de1f..6e531b45a408 100644 --- a/stage0/stdlib/Lean/Compiler/IR/Borrow.c +++ b/stage0/stdlib/Lean/Compiler/IR/Borrow.c @@ -3380,7 +3380,7 @@ static lean_object* _init_l_Nat_forM_loop___at_Lean_IR_Borrow_ownArgsUsingParams 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_Nat_forM_loop___at_Lean_IR_Borrow_ownArgsUsingParams___spec__2___closed__1; x_2 = l_Nat_forM_loop___at_Lean_IR_Borrow_ownArgsUsingParams___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_forM_loop___at_Lean_IR_Borrow_ownArgsUsingParams___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Compiler/IR/Boxing.c b/stage0/stdlib/Lean/Compiler/IR/Boxing.c index 102a3aaec0e1..f330f9ee6fcc 100644 --- a/stage0/stdlib/Lean/Compiler/IR/Boxing.c +++ b/stage0/stdlib/Lean/Compiler/IR/Boxing.c @@ -466,7 +466,7 @@ static lean_object* _init_l_Nat_foldM_loop___at_Lean_IR_ExplicitBoxing_mkBoxedVe 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_Nat_foldM_loop___at_Lean_IR_ExplicitBoxing_mkBoxedVersionAux___spec__2___closed__1; x_2 = l_Nat_foldM_loop___at_Lean_IR_ExplicitBoxing_mkBoxedVersionAux___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_foldM_loop___at_Lean_IR_ExplicitBoxing_mkBoxedVersionAux___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c b/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c index 129c6533c182..0484a2b3745b 100644 --- a/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c +++ b/stage0/stdlib/Lean/Compiler/IR/ElimDeadBranches.c @@ -2112,7 +2112,7 @@ static lean_object* _init_l_Nat_foldAux___at_Lean_IR_UnreachableBranches_Value_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_Nat_foldAux___at_Lean_IR_UnreachableBranches_Value_merge___spec__2___closed__1; x_2 = l_Nat_foldAux___at_Lean_IR_UnreachableBranches_Value_merge___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_foldAux___at_Lean_IR_UnreachableBranches_Value_merge___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Compiler/IR/EmitC.c b/stage0/stdlib/Lean/Compiler/IR/EmitC.c index 746de2504d7a..9df7f7db7e9c 100644 --- a/stage0/stdlib/Lean/Compiler/IR/EmitC.c +++ b/stage0/stdlib/Lean/Compiler/IR/EmitC.c @@ -1782,7 +1782,7 @@ static lean_object* _init_l_Nat_forM_loop___at_Lean_IR_EmitC_emitFnDeclAux___spe 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_Nat_forM_loop___at_Lean_IR_EmitC_emitFnDeclAux___spec__1___lambda__1___closed__1; x_2 = l_Nat_forM_loop___at_Lean_IR_EmitC_emitFnDeclAux___spec__1___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_forM_loop___at_Lean_IR_EmitC_emitFnDeclAux___spec__1___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Compiler/IR/ExpandResetReuse.c b/stage0/stdlib/Lean/Compiler/IR/ExpandResetReuse.c index 328ef095338b..fdf58a671556 100644 --- a/stage0/stdlib/Lean/Compiler/IR/ExpandResetReuse.c +++ b/stage0/stdlib/Lean/Compiler/IR/ExpandResetReuse.c @@ -989,7 +989,7 @@ static lean_object* _init_l_Lean_IR_ExpandResetReuse_eraseProjIncForAux___closed lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_IR_ExpandResetReuse_eraseProjIncForAux___closed__1; x_2 = l_Lean_IR_ExpandResetReuse_eraseProjIncForAux___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_IR_ExpandResetReuse_eraseProjIncForAux___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Compiler/IR/RC.c b/stage0/stdlib/Lean/Compiler/IR/RC.c index 9f47058712ce..60066be95eac 100644 --- a/stage0/stdlib/Lean/Compiler/IR/RC.c +++ b/stage0/stdlib/Lean/Compiler/IR/RC.c @@ -3513,7 +3513,7 @@ static lean_object* _init_l_Nat_anyAux___at___private_Lean_Compiler_IR_RC_0__Lea 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_Nat_anyAux___at___private_Lean_Compiler_IR_RC_0__Lean_IR_ExplicitRC_isFirstOcc___spec__3___closed__1; x_2 = l_Nat_anyAux___at___private_Lean_Compiler_IR_RC_0__Lean_IR_ExplicitRC_isFirstOcc___spec__3___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_anyAux___at___private_Lean_Compiler_IR_RC_0__Lean_IR_ExplicitRC_isFirstOcc___spec__3___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Compiler/IR/SimpCase.c b/stage0/stdlib/Lean/Compiler/IR/SimpCase.c index de8e3607e880..36f44125a71a 100644 --- a/stage0/stdlib/Lean/Compiler/IR/SimpCase.c +++ b/stage0/stdlib/Lean/Compiler/IR/SimpCase.c @@ -261,7 +261,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Compiler_IR lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Compiler_IR_SimpCase_0__Lean_IR_getOccsOf___spec__2___closed__1; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Compiler_IR_SimpCase_0__Lean_IR_getOccsOf___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Compiler_IR_SimpCase_0__Lean_IR_getOccsOf___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Data/Lsp/Capabilities.c b/stage0/stdlib/Lean/Data/Lsp/Capabilities.c index 653d063a0204..ab8fddcb96c4 100644 --- a/stage0/stdlib/Lean/Data/Lsp/Capabilities.c +++ b/stage0/stdlib/Lean/Data/Lsp/Capabilities.c @@ -41,7 +41,7 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonServerCapabilities; LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_399____spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonCompletionClientCapabilities___closed__1; static lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonServerCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_594____closed__2; -lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3468_(lean_object*); +lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5019_(lean_object*); LEAN_EXPORT uint8_t l_Lean_Lsp_ServerCapabilities_workspaceSymbolProvider___default; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_425____spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Lsp_ServerCapabilities_hoverProvider___default; @@ -59,7 +59,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_from LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_toJsonClientCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_399____spec__2(lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_115_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Capabilities_0__Lean_Lsp_fromJsonServerCapabilities____x40_Lean_Data_Lsp_Capabilities___hyg_723____spec__1___boxed(lean_object*, lean_object*); -lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396_(lean_object*); +lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_ClientCapabilities_textDocument_x3f___default; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonTextDocumentClientCapabilities; static lean_object* l_Lean_Lsp_instToJsonShowDocumentClientCapabilities___closed__1; @@ -1777,7 +1777,7 @@ lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_obj x_4 = lean_ctor_get(x_2, 0); lean_inc(x_4); lean_dec(x_2); -x_5 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3468_(x_4); +x_5 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5019_(x_4); x_6 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_6, 0, x_1); lean_ctor_set(x_6, 1, x_5); @@ -2192,7 +2192,7 @@ return x_4; else { lean_object* x_5; -x_5 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396_(x_3); +x_5 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947_(x_3); lean_dec(x_3); if (lean_obj_tag(x_5) == 0) { diff --git a/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c b/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c index fe51517a44e9..0e534c3438fe 100644 --- a/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c +++ b/stage0/stdlib/Lean/Data/Lsp/LanguageFeatures.c @@ -15,12 +15,17 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonSemanticTokens; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__138; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339____spec__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSemanticTokensParams; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_115____spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionOptions; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDocumentHighlightParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2503____boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonReferenceParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2291____closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSymbolInformation____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3135____spec__1(size_t, size_t, lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__11; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__10; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__90; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionItemKind(uint8_t); static lean_object* l_Lean_Lsp_instToJsonReferenceContext___closed__1; @@ -29,22 +34,34 @@ LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Ls static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__102; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSymbolInformation____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3135____spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSemanticTokens___closed__1; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____spec__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonHover____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1715____boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSymbolTag___boxed(lean_object*); lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonLocation____x40_Lean_Data_Lsp_Basic___hyg_900_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonReferenceContext____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2243_(uint8_t); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__31; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___closed__1; lean_object* lean_mk_empty_array_with_capacity(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__14; LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolTag_noConfusion___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instDecidableEqCompletionItemKind___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__3; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonHoverParams; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSymbolInformation____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3135____closed__3; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__143; static lean_object* l_Lean_Lsp_instToJsonDocumentHighlight___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____rarg___closed__3; lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonInsertReplaceEdit; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonHoverParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1781_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__15; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__2; LEAN_EXPORT uint8_t l_Lean_Lsp_CompletionItemKind_ofNat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSemanticTokensRangeParams; @@ -52,37 +69,52 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItemKind_ofNat___boxed(lean_object static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__124; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonReferenceParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2363_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__95; +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_names; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__6; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__27; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItemKind_noConfusion___rarg___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItemKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___closed__1; lean_object* l_Lean_Json_getNat_x3f(lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__9; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__40; static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionItemKind___boxed(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__26; LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toCtorIdx(uint8_t); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__59; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761____spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonInsertReplaceEdit___closed__1; +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_noConfusion(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__31; static lean_object* l_Lean_Lsp_instFromJsonHoverParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__58; static lean_object* l_Lean_Lsp_instToJsonDefinitionParams___closed__1; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__134; +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__92; static lean_object* l_Lean_Lsp_instFromJsonSemanticTokensLegend___closed__1; +lean_object* l_Except_orElseLazy___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSemanticTokensRangeParams___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_FoldingRangeKind_toCtorIdx(uint8_t); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__150; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__97; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__19; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__17; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__94; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__8; LEAN_EXPORT uint8_t l_Lean_Lsp_CompletionOptions_resolveProvider___default; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__23; LEAN_EXPORT lean_object* l_Lean_Lsp_DocumentSymbolAux_children_x3f___default(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolTag_noConfusion___rarg(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__144; @@ -90,6 +122,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_ LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentSymbolAux___rarg(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__64; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__12; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__6; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItemKind_noConfusion___rarg___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____spec__1___boxed(lean_object*, lean_object*); @@ -99,13 +133,19 @@ static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprC static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__74; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__3; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__89; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentSymbol; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__35; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1105_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____spec__1___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__7; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__36; static lean_object* l_Lean_Lsp_CompletionItemKind_noConfusion___rarg___closed__1; lean_object* l_Lean_Json_getStr_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSemanticTokens; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__5; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__122; @@ -114,8 +154,8 @@ lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonDeclarationParams; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItemKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__39; static lean_object* l_Lean_Lsp_instReprCompletionItemKind___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3616____boxed(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDefinitionParams; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonDefinitionParams; @@ -124,74 +164,101 @@ static lean_object* l_Lean_Lsp_instFromJsonDocumentHighlightParams___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instInhabitedCompletionItem; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1460____spec__2(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__27; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__7; LEAN_EXPORT lean_object* l_Lean_Json_opt___at_Lean_Lsp_instToJsonDocumentSymbol_go___spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonReferenceContext____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2205____closed__1; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__42; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDeclarationParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1887_(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__2(size_t, size_t, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__31; static lean_object* l_Lean_Lsp_instFromJsonCompletionItem___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5081____boxed(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__37; static lean_object* l_Lean_Lsp_instFromJsonSemanticTokens___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentHighlightParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2558_(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3468_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5019_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__40; static lean_object* l_Lean_Lsp_instToJsonDeclarationParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__67; LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolKind_noConfusion(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____closed__3; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__131; -static lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind___closed__5; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__4; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__57; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____spec__3(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonTypeDefinitionParams___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__21; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__38; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__139; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__3; +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__10; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__9; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_names; lean_object* l_List_join___rarg(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); +static lean_object* l_Lean_Lsp_instFromJsonSemanticTokenType___closed__1; static lean_object* l_Lean_Lsp_instToJsonHover___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__87; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__22; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__44; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionItem; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonTypeDefinitionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2154_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__2; lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentSymbolParams; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__14; static lean_object* l_Lean_Lsp_instToJsonCompletionOptions___closed__1; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__28; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSymbolTag(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__26; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__5; LEAN_EXPORT lean_object* l_Lean_Lsp_DocumentHighlightKind_toCtorIdx___boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__55; +static lean_object* l_Lean_Lsp_instToJsonSemanticTokenModifier___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__106; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__24; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonDocumentHighlightParams; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__11; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___closed__1; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__18; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____spec__1(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__15; -static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____at_Lean_Lsp_instToJsonDocumentSymbol_go___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_115_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1460____closed__2; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__108; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__10; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__32; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286_(uint8_t); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__37; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396_(lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__19; +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_noConfusion___rarg(uint8_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__20; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__30; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__3; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonFoldingRange; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__10; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__32; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__71; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__7; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__63; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonReferenceContext____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2205_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolKind_toCtorIdx(uint8_t); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__43; -static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__2; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__18; LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolInformation_containerName_x3f___default; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__76; @@ -199,92 +266,125 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionOptions_triggerCharacters_x3f___de static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__15; LEAN_EXPORT lean_object* l_Lean_Lsp_instReprCompletionItemKind; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentHighlightParams; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1105____boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonWorkspaceSymbolParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2425____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonHover____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1682_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__113; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonWorkspaceSymbolParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2425____boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__30; +lean_object* l_Lean_Json_parseTagged(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentHighlight____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2644____spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___boxed(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__5; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1460_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonReferenceContext; -static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___closed__6; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__42; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instFromJsonInsertReplaceEdit___closed__1; +LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSemanticTokenType; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__125; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__16; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instToJsonDocumentSymbol_go___spec__3(size_t, size_t, lean_object*); static lean_object* l_Lean_Lsp_instToJsonReferenceParams___closed__1; lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toNat(uint8_t); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____rarg___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1382____spec__3(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__105; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_Hover_range_x3f___default; static lean_object* l_Lean_Lsp_instToJsonCompletionItem___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__16; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__53; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____rarg___closed__2; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__12; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__100; static lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___closed__4; +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonReferenceParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2291____spec__1___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__12; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____boxed(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__1; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__16; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1621_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Lsp_instInhabitedCompletionItemKind; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__24; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__148; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3530____boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolTag_toCtorIdx(lean_object*); static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__1___closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339_(lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__24; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionOptions_allCommitCharacters_x3f___default; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instToJsonDocumentSymbol_go___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonInsertReplaceEdit; LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolInformation_tags___default; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__19; static lean_object* l_Lean_Lsp_instFromJsonFoldingRangeParams___closed__1; +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__9; static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__7; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__2(size_t, size_t, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___closed__1; +LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonSemanticTokenModifier; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__135; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3801_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5383_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__112; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__114; -static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__26; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__75; static lean_object* l_Lean_Lsp_instFromJsonDefinitionParams___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind(uint8_t); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSemanticTokenModifier; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__82; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3616_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5167_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__11; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDeclarationParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1942_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__20; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonReferenceParams; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDefinitionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1993_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__116; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__34; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__10; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__128; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__68; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSymbolKind(uint8_t); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonDocumentSymbolParams; lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2161____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__61; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__43; static lean_object* l_Lean_Lsp_instToJsonCompletionParams___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__2; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toNat___boxed(lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__8; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSemanticTokensOptions; LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_115____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSemanticTokensLegend___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1105____closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonTypeDefinitionParams; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1460____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__11; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonHover____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1715____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__127; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1515____spec__1(size_t, size_t, lean_object*); @@ -293,31 +393,47 @@ lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_JsonRpc_instFromJsonMessage__ static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__12; static lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___closed__2; static lean_object* l_Lean_Lsp_instFromJsonWorkspaceSymbolParams___closed__1; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__20; LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1382____spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3530_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5081_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__13; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__142; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__41; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__126; LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolKind_toCtorIdx___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__3___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__136; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__29; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1105____closed__3; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__3; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__141; static lean_object* l_Lean_Lsp_instFromJsonTypeDefinitionParams___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentSymbolAux(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__13; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__41; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDefinitionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2048_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_toNat___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDocumentSymbolParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2692_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___boxed(lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentHighlight____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2644_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__1; static lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___closed__5; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instFromJsonCompletionParams___closed__1; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__38; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__21; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__17; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__50; LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion___rarg(uint8_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__8; static lean_object* l_Lean_Lsp_instInhabitedCompletionItem___closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolTag_toCtorIdx___boxed(lean_object*); static lean_object* l_Lean_Lsp_instToJsonHoverParams___closed__1; @@ -325,20 +441,25 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDeclarationParams; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSemanticTokensLegend; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSymbolInformation____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3135_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__22; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__13; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__111; LEAN_EXPORT uint8_t l_Lean_Lsp_instDecidableEqCompletionItemKind(uint8_t, uint8_t); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__11; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__23; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__23; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__20; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1566_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__110; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonFoldingRangeParams; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__80; LEAN_EXPORT lean_object* l_Lean_Lsp_FoldingRange_kind_x3f___default; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__6; -LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_FoldingRangeKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); -static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____closed__1; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__21; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__107; +LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonSemanticTokenType; LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1382____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__21; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__38; @@ -347,29 +468,38 @@ size_t lean_usize_of_nat(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1566____closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonReferenceParams; static lean_object* l_Lean_Lsp_instFromJsonSemanticTokensRangeParams___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3671_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5222_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__48; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionItemKind___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_DocumentHighlightKind_noConfusion(lean_object*); static lean_object* l_Lean_Lsp_instFromJsonSemanticTokensOptions___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1566____boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__72; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__96; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3801____boxed(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___closed__1; lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonTextDocumentIdentifier____x40_Lean_Data_Lsp_Basic___hyg_1472_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__33; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1515_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__25; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSymbolInformation____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3135____closed__2; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761____spec__1(size_t, size_t, lean_object*); static lean_object* l_Lean_Lsp_instFromJsonDeclarationParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__93; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__22; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__24; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonSemanticTokensParams; LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentHighlight____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2644____spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Lsp_instToJsonSemanticTokenType___closed__1; static lean_object* l_Lean_Lsp_instFromJsonCompletionOptions___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____spec__2___rarg(lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__34; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__16; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__7; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__29; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276_(lean_object*); lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_2523_(lean_object*); @@ -380,11 +510,15 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_DocumentSymbolAux_detail_x3f___default; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItemKind_noConfusion(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__73; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1460____closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__42; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__81; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionList; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionItem; +static lean_object* l_Lean_Lsp_instFromJsonSemanticTokenModifier___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__46; static lean_object* l_Lean_Lsp_instToJsonSymbolInformation___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonTypeDefinitionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2099____boxed(lean_object*); @@ -396,37 +530,60 @@ static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprC static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__10; lean_object* l_Lean_JsonNumber_fromNat(lean_object*); lean_object* l_Lean_Json_getObjValD(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__120; lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocationLink____x40_Lean_Data_Lsp_Basic___hyg_1086____spec__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___closed__1; static lean_object* l_Lean_Lsp_instToJsonFoldingRangeParams___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_FoldingRangeKind_noConfusion(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__43; lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonRange____x40_Lean_Data_Lsp_Basic___hyg_663____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_FoldingRangeKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSymbolInformation____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3135____closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__37; LEAN_EXPORT lean_object* l_Lean_Lsp_DocumentHighlightKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339____spec__1(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__13; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonHoverParams; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_toNat(uint8_t); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205_(uint8_t); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1105____closed__2; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__101; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__1; lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonTextDocumentPositionParams____x40_Lean_Data_Lsp_Basic___hyg_2007____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__49; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__28; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__12; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__123; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__14; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonHoverParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1836_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__133; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__4; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDefinitionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1993____boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____spec__2(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__35; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__22; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonCompletionOptions; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__2; +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_toCtorIdx(uint8_t); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__33; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonHover; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__16; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentSymbol_go(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__36; uint8_t lean_nat_dec_le(lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1177_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__115; lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonLocationLink____x40_Lean_Data_Lsp_Basic___hyg_1031____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolAux____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2915____rarg(lean_object*, lean_object*); @@ -435,17 +592,22 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind(uint8_t); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__99; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__19; lean_object* l_Lean_Json_mkObj(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__18; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__88; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1515____spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonDocumentHighlightKind___closed__3; +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__5; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__56; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__66; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__85; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__117; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__77; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__149; +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItem_textEdit_x3f___default; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__39; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__8; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__36; lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_2483_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__11; @@ -455,98 +617,140 @@ static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonReferenceContext____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2243____boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__146; lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__17; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____closed__2; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1382_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__129; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__25; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__104; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__14; LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonFoldingRange___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_DocumentHighlightKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__45; +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__145; static lean_object* l_Lean_Lsp_instToJsonCompletionList___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3329_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4880_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__4; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__83; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__35; static lean_object* l_Lean_Lsp_instToJsonDocumentSymbol___closed__1; static lean_object* l_Lean_Lsp_instToJsonSemanticTokensParams___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_CompletionItemKind_toCtorIdx___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____boxed(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__2; static lean_object* l_Lean_Lsp_SymbolInformation_tags___default___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__3; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__51; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__1; static lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind___closed__2; -static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__2; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__44; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__15; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__18; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257_(uint8_t, lean_object*); static lean_object* l_Lean_Lsp_instFromJsonSemanticTokensParams___closed__1; static lean_object* l_Lean_Lsp_instFromJsonReferenceContext___closed__1; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__44; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonSemanticTokensOptions; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__45; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__151; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonWorkspaceSymbolParams; -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3839_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5421_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__1; lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocation____x40_Lean_Data_Lsp_Basic___hyg_940____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_115____spec__2(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__70; +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_toCtorIdx___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonTypeDefinitionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2099_(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3568_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5119_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDeclarationParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1887____boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__2; lean_object* l_Lean_Json_getBool_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__78; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__91; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentHighlight; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolTag_noConfusion___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSymbolKind___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1382____spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind___closed__3; +static lean_object* l_Lean_Lsp_SemanticTokenModifier_names___closed__7; LEAN_EXPORT lean_object* l_Lean_Lsp_FoldingRangeKind_toCtorIdx___boxed(lean_object*); static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonHover____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1715_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__46; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonHover____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1682____closed__2; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__69; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonWorkspaceSymbolParams; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__17; LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonHoverParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1781____boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentSymbolParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2730_(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__65; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__109; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____boxed(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__9; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonHover____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1682____closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__39; lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonReferenceContext; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonHover; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__2; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__33; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__45; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonSemanticTokensLegend; LEAN_EXPORT lean_object* l_Lean_Lsp_DocumentHighlightKind_toCtorIdx(uint8_t); static lean_object* l_Lean_Lsp_instFromJsonHover___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__13; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__62; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__41; static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__9; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__2(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922_(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__9; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonReferenceParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2291____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__40; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__3; +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5167____boxed(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__3; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__27; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__15; LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolTag_noConfusion(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__28; static lean_object* l_Lean_Lsp_instToJsonSymbolKind___closed__4; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__121; static lean_object* l_Lean_Lsp_instToJsonDocumentSymbolParams___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonSemanticTokensRangeParams; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__6; +static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__17; static lean_object* l_Lean_Lsp_instFromJsonReferenceParams___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__137; static lean_object* l_Lean_Lsp_instToJsonWorkspaceSymbolParams___closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__54; @@ -555,6 +759,7 @@ LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonDocumentSymbolResult(lean_object*) static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__132; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__103; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionParams; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__34; lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonPosition____x40_Lean_Data_Lsp_Basic___hyg_362_(lean_object*); static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__4; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__14; @@ -567,32 +772,45 @@ LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFe LEAN_EXPORT lean_object* l_Lean_Lsp_SymbolKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toCtorIdx___boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__46; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Lsp_instInhabitedCompletionItem___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__2; LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind___boxed(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___closed__1; lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__130; static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__1; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionItemKind(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokens_resultId_x3f___default; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__86; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonWorkspaceSymbolParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2425_(lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__18; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__147; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__52; static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__8; -static lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind___closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonSymbolInformation; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____spec__1___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__1; static lean_object* l_Lean_Lsp_SemanticTokenType_names___closed__2; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__5; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__140; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__118; static lean_object* l_Lean_Lsp_instFromJsonCompletionList___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonWorkspaceSymbolParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2463_(lean_object*); static lean_object* l_Lean_Lsp_instToJsonSemanticTokensOptions___closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__1; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__30; +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5383____boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDocumentHighlightParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2503_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonReferenceParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2291____boxed(lean_object*); static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__119; LEAN_EXPORT lean_object* l_Lean_Lsp_instFromJsonCompletionList; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__29; +static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__1; static lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_reprCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_257____closed__152; lean_object* l_Repr_addAppParen(lean_object*, lean_object*); static lean_object* _init_l_Lean_Lsp_CompletionOptions_triggerCharacters_x3f___default() { @@ -9337,184 +9555,3658 @@ lean_object* x_4; x_4 = lean_unsigned_to_nat(2u); return x_4; } +case 3: +{ +lean_object* x_5; +x_5 = lean_unsigned_to_nat(3u); +return x_5; +} +case 4: +{ +lean_object* x_6; +x_6 = lean_unsigned_to_nat(4u); +return x_6; +} +case 5: +{ +lean_object* x_7; +x_7 = lean_unsigned_to_nat(5u); +return x_7; +} +case 6: +{ +lean_object* x_8; +x_8 = lean_unsigned_to_nat(6u); +return x_8; +} +case 7: +{ +lean_object* x_9; +x_9 = lean_unsigned_to_nat(7u); +return x_9; +} +case 8: +{ +lean_object* x_10; +x_10 = lean_unsigned_to_nat(8u); +return x_10; +} +case 9: +{ +lean_object* x_11; +x_11 = lean_unsigned_to_nat(9u); +return x_11; +} +case 10: +{ +lean_object* x_12; +x_12 = lean_unsigned_to_nat(10u); +return x_12; +} +case 11: +{ +lean_object* x_13; +x_13 = lean_unsigned_to_nat(11u); +return x_13; +} +case 12: +{ +lean_object* x_14; +x_14 = lean_unsigned_to_nat(12u); +return x_14; +} +case 13: +{ +lean_object* x_15; +x_15 = lean_unsigned_to_nat(13u); +return x_15; +} +case 14: +{ +lean_object* x_16; +x_16 = lean_unsigned_to_nat(14u); +return x_16; +} +case 15: +{ +lean_object* x_17; +x_17 = lean_unsigned_to_nat(15u); +return x_17; +} +case 16: +{ +lean_object* x_18; +x_18 = lean_unsigned_to_nat(16u); +return x_18; +} +case 17: +{ +lean_object* x_19; +x_19 = lean_unsigned_to_nat(17u); +return x_19; +} +case 18: +{ +lean_object* x_20; +x_20 = lean_unsigned_to_nat(18u); +return x_20; +} +case 19: +{ +lean_object* x_21; +x_21 = lean_unsigned_to_nat(19u); +return x_21; +} +case 20: +{ +lean_object* x_22; +x_22 = lean_unsigned_to_nat(20u); +return x_22; +} +case 21: +{ +lean_object* x_23; +x_23 = lean_unsigned_to_nat(21u); +return x_23; +} default: { -lean_object* x_5; -x_5 = lean_unsigned_to_nat(3u); -return x_5; +lean_object* x_24; +x_24 = lean_unsigned_to_nat(22u); +return x_24; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toCtorIdx___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = lean_unbox(x_1); +lean_dec(x_1); +x_3 = l_Lean_Lsp_SemanticTokenType_toCtorIdx(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion___rarg(uint8_t x_1, uint8_t x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Lsp_CompletionItemKind_noConfusion___rarg___closed__1; +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Lsp_SemanticTokenType_noConfusion___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; uint8_t x_5; lean_object* x_6; +x_4 = lean_unbox(x_1); +lean_dec(x_1); +x_5 = lean_unbox(x_2); +lean_dec(x_2); +x_6 = l_Lean_Lsp_SemanticTokenType_noConfusion___rarg(x_4, x_5, x_3); +return x_6; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("keyword", 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("variable", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__3; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("property", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__5; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("function", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("namespace", 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__9; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("type", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__11; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("class", 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__15() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("enum", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__15; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("interface", 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__17; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__19() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("struct", 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__21() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("typeParameter", 13); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__21; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__23() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parameter", 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__24() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__23; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__25() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("enumMember", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__26() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__25; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__27() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("event", 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__28() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__27; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__29() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("method", 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__30() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__29; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__31() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("macro", 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__32() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__31; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__33() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("modifier", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__34() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__33; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__35() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("comment", 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__36() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__35; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__37() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("string", 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__38() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__37; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__39() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("number", 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__40() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__39; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__41() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("regexp", 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__42() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__41; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__43() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("operator", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__44() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__43; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__45() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("decorator", 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__46() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__45; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205_(uint8_t x_1) { +_start: +{ +switch (x_1) { +case 0: +{ +lean_object* x_2; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__2; +return x_2; +} +case 1: +{ +lean_object* x_3; +x_3 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__4; +return x_3; +} +case 2: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__6; +return x_4; +} +case 3: +{ +lean_object* x_5; +x_5 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__8; +return x_5; +} +case 4: +{ +lean_object* x_6; +x_6 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__10; +return x_6; +} +case 5: +{ +lean_object* x_7; +x_7 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__12; +return x_7; +} +case 6: +{ +lean_object* x_8; +x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__14; +return x_8; +} +case 7: +{ +lean_object* x_9; +x_9 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__16; +return x_9; +} +case 8: +{ +lean_object* x_10; +x_10 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__18; +return x_10; +} +case 9: +{ +lean_object* x_11; +x_11 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__20; +return x_11; +} +case 10: +{ +lean_object* x_12; +x_12 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__22; +return x_12; +} +case 11: +{ +lean_object* x_13; +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__24; +return x_13; +} +case 12: +{ +lean_object* x_14; +x_14 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__26; +return x_14; +} +case 13: +{ +lean_object* x_15; +x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__28; +return x_15; +} +case 14: +{ +lean_object* x_16; +x_16 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__30; +return x_16; +} +case 15: +{ +lean_object* x_17; +x_17 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__32; +return x_17; +} +case 16: +{ +lean_object* x_18; +x_18 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__34; +return x_18; +} +case 17: +{ +lean_object* x_19; +x_19 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__36; +return x_19; +} +case 18: +{ +lean_object* x_20; +x_20 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__38; +return x_20; +} +case 19: +{ +lean_object* x_21; +x_21 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__40; +return x_21; +} +case 20: +{ +lean_object* x_22; +x_22 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__42; +return x_22; +} +case 21: +{ +lean_object* x_23; +x_23 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__44; +return x_23; +} +default: +{ +lean_object* x_24; +x_24 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__46; +return x_24; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = lean_unbox(x_1); +lean_dec(x_1); +x_3 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205_(x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokenType___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokenType() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Lsp_instToJsonSemanticTokenType___closed__1; +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("no inductive constructor matched", 32); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__2; +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__2() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 21; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__2; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1; +x_3 = l_Except_orElseLazy___rarg(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__43; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1; +x_9 = l_Except_orElseLazy___rarg(x_6, x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1; +x_13 = l_Except_orElseLazy___rarg(x_11, x_12); +return x_13; +} +} +else +{ +lean_object* x_14; +lean_dec(x_6); +x_14 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__3; +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 20; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__41; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 19; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__39; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 18; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__37; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 17; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__35; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 16; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__33; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 15; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__31; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 14; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__29; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 13; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__27; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 12; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__25; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 11; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__23; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 10; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__21; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 9; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__19; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 8; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__17; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 7; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__15; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 6; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__13; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 5; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__11; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 4; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__9; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 3; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__7; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 2; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__5; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 1; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__3; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 0; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__1; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Lsp_SymbolInformation_tags___default___closed__1; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__2() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 22; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__45; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__1; +x_5 = l_Lean_Json_parseTagged(x_1, x_2, x_3, x_4); +x_6 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___boxed), 3, 2); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_4); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; +x_8 = l_Except_orElseLazy___rarg(x_5, x_6); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_5, 0); +lean_inc(x_9); +lean_dec(x_5); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = l_Except_orElseLazy___rarg(x_10, x_6); +return x_11; +} +} +else +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_5); +x_12 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__2; +x_13 = l_Except_orElseLazy___rarg(x_12, x_6); +return x_13; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokenType___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokenType() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Lsp_instFromJsonSemanticTokenType___closed__1; +return x_1; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(23u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__1; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__1; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__2; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__3; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__3; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__5; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__4; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__7; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__5; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__9; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__6; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__11; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__7; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__13; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__8; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__15; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__9; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__17; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__10; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__19; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__11; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__21; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__12; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__23; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__13; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__25; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__14; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__27; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__15; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__29; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__16; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__31; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__17; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__33; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__18; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__35; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__19; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__37; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__20; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__39; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__21; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__41; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__23() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__22; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__43; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__24() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__23; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__45; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__24; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toNat(uint8_t x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Lsp_SemanticTokenType_toCtorIdx(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toNat___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = lean_unbox(x_1); +lean_dec(x_1); +x_3 = l_Lean_Lsp_SemanticTokenType_toNat(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_toCtorIdx(uint8_t x_1) { +_start: +{ +switch (x_1) { +case 0: +{ +lean_object* x_2; +x_2 = lean_unsigned_to_nat(0u); +return x_2; +} +case 1: +{ +lean_object* x_3; +x_3 = lean_unsigned_to_nat(1u); +return x_3; +} +case 2: +{ +lean_object* x_4; +x_4 = lean_unsigned_to_nat(2u); +return x_4; +} +case 3: +{ +lean_object* x_5; +x_5 = lean_unsigned_to_nat(3u); +return x_5; +} +case 4: +{ +lean_object* x_6; +x_6 = lean_unsigned_to_nat(4u); +return x_6; +} +case 5: +{ +lean_object* x_7; +x_7 = lean_unsigned_to_nat(5u); +return x_7; +} +case 6: +{ +lean_object* x_8; +x_8 = lean_unsigned_to_nat(6u); +return x_8; +} +case 7: +{ +lean_object* x_9; +x_9 = lean_unsigned_to_nat(7u); +return x_9; +} +case 8: +{ +lean_object* x_10; +x_10 = lean_unsigned_to_nat(8u); +return x_10; +} +default: +{ +lean_object* x_11; +x_11 = lean_unsigned_to_nat(9u); +return x_11; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_toCtorIdx___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = lean_unbox(x_1); +lean_dec(x_1); +x_3 = l_Lean_Lsp_SemanticTokenModifier_toCtorIdx(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_noConfusion___rarg(uint8_t x_1, uint8_t x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Lsp_CompletionItemKind_noConfusion___rarg___closed__1; +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_noConfusion(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Lsp_SemanticTokenModifier_noConfusion___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_noConfusion___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; uint8_t x_5; lean_object* x_6; +x_4 = lean_unbox(x_1); +lean_dec(x_1); +x_5 = lean_unbox(x_2); +lean_dec(x_2); +x_6 = l_Lean_Lsp_SemanticTokenModifier_noConfusion___rarg(x_4, x_5, x_3); +return x_6; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("declaration", 11); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("definition", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__3; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("readonly", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__5; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("static", 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("deprecated", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__9; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("abstract", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__11; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("async", 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__15() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("modification", 12); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__15; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__3; +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_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__18() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("defaultLibrary", 14); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__18; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286_(uint8_t x_1) { +_start: +{ +switch (x_1) { +case 0: +{ +lean_object* x_2; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__2; +return x_2; +} +case 1: +{ +lean_object* x_3; +x_3 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__4; +return x_3; +} +case 2: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__6; +return x_4; +} +case 3: +{ +lean_object* x_5; +x_5 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__8; +return x_5; +} +case 4: +{ +lean_object* x_6; +x_6 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__10; +return x_6; +} +case 5: +{ +lean_object* x_7; +x_7 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__12; +return x_7; +} +case 6: +{ +lean_object* x_8; +x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__14; +return x_8; +} +case 7: +{ +lean_object* x_9; +x_9 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__16; +return x_9; +} +case 8: +{ +lean_object* x_10; +x_10 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__17; +return x_10; +} +default: +{ +lean_object* x_11; +x_11 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__19; +return x_11; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = lean_unbox(x_1); +lean_dec(x_1); +x_3 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286_(x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokenModifier___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokenModifier() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Lsp_instToJsonSemanticTokenModifier___closed__1; +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 8; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__1; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1; +x_3 = l_Except_orElseLazy___rarg(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__3; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1; +x_9 = l_Except_orElseLazy___rarg(x_6, x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1; +x_13 = l_Except_orElseLazy___rarg(x_11, x_12); +return x_13; +} +} +else +{ +lean_object* x_14; +lean_dec(x_6); +x_14 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__2; +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 7; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__15; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 6; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__13; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 5; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__11; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 4; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__9; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 3; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__7; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 2; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__5; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 1; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__3; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 0; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__1; +x_5 = lean_unsigned_to_nat(0u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_6); +x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___closed__1; +x_14 = l_Except_orElseLazy___rarg(x_13, x_7); +return x_14; +} +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 9; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__18; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__1; +x_5 = l_Lean_Json_parseTagged(x_1, x_2, x_3, x_4); +x_6 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___boxed), 3, 2); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_4); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; +x_8 = l_Except_orElseLazy___rarg(x_5, x_6); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_5, 0); +lean_inc(x_9); +lean_dec(x_5); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = l_Except_orElseLazy___rarg(x_10, x_6); +return x_11; +} +} +else +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_5); +x_12 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____closed__1; +x_13 = l_Except_orElseLazy___rarg(x_12, x_6); +return x_13; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toCtorIdx___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -uint8_t x_2; lean_object* x_3; -x_2 = lean_unbox(x_1); -lean_dec(x_1); -x_3 = l_Lean_Lsp_SemanticTokenType_toCtorIdx(x_2); -return x_3; +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion___rarg(uint8_t x_1, uint8_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Lsp_CompletionItemKind_noConfusion___rarg___closed__1; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7(x_1, x_2, x_3); +lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Lsp_SemanticTokenType_noConfusion___rarg___boxed), 3, 0); -return x_2; +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_noConfusion___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -uint8_t x_4; uint8_t x_5; lean_object* x_6; -x_4 = lean_unbox(x_1); -lean_dec(x_1); -x_5 = lean_unbox(x_2); -lean_dec(x_2); -x_6 = l_Lean_Lsp_SemanticTokenType_noConfusion___rarg(x_4, x_5, x_3); -return x_6; +lean_object* x_4; +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__1() { +static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokenModifier___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(4u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339_), 1, 0); +return x_1; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__2() { +static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokenModifier() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("keyword", 7); +x_1 = l_Lean_Lsp_instFromJsonSemanticTokenModifier___closed__1; return x_1; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__3() { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(10u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__1; -x_2 = l_Lean_Lsp_SemanticTokenType_names___closed__2; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__1; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__1; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__4() { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("variable", 8); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__2; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__3; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__5() { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__3; -x_2 = l_Lean_Lsp_SemanticTokenType_names___closed__4; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__3; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__5; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__6() { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("property", 8); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__4; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__7; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__7() { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__5; -x_2 = l_Lean_Lsp_SemanticTokenType_names___closed__6; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__5; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__9; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__8() { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__7() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("function", 8); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__6; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__11; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names___closed__9() { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__7; -x_2 = l_Lean_Lsp_SemanticTokenType_names___closed__8; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__7; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__13; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Lsp_SemanticTokenType_names() { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__9() { _start: { -lean_object* x_1; -x_1 = l_Lean_Lsp_SemanticTokenType_names___closed__9; -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__8; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__15; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toNat(uint8_t x_1) { +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__10() { _start: { -switch (x_1) { -case 0: -{ -lean_object* x_2; -x_2 = lean_unsigned_to_nat(0u); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__9; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__3; +x_3 = lean_array_push(x_1, x_2); +return x_3; } -case 1: +} +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__11() { +_start: { -lean_object* x_3; -x_3 = lean_unsigned_to_nat(1u); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__10; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__18; +x_3 = lean_array_push(x_1, x_2); return x_3; } -case 2: -{ -lean_object* x_4; -x_4 = lean_unsigned_to_nat(2u); -return x_4; } -default: +static lean_object* _init_l_Lean_Lsp_SemanticTokenModifier_names() { +_start: { -lean_object* x_5; -x_5 = lean_unsigned_to_nat(3u); -return x_5; +lean_object* x_1; +x_1 = l_Lean_Lsp_SemanticTokenModifier_names___closed__11; +return x_1; } } +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_toNat(uint8_t x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Lsp_SemanticTokenModifier_toCtorIdx(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenType_toNat___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Lsp_SemanticTokenModifier_toNat___boxed(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; x_2 = lean_unbox(x_1); lean_dec(x_1); -x_3 = l_Lean_Lsp_SemanticTokenType_toNat(x_2); +x_3 = l_Lean_Lsp_SemanticTokenModifier_toNat(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; @@ -9548,7 +13240,7 @@ return x_15; } } } -static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__1() { +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__1() { _start: { lean_object* x_1; @@ -9556,7 +13248,7 @@ x_1 = lean_mk_string_from_bytes("tokenTypes", 10); return x_1; } } -static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__2() { +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__2() { _start: { lean_object* x_1; @@ -9564,12 +13256,12 @@ x_1 = lean_mk_string_from_bytes("tokenModifiers", 14); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__1; -x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____spec__1(x_1, x_2); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____spec__1(x_1, x_2); if (lean_obj_tag(x_3) == 0) { uint8_t x_4; @@ -9595,8 +13287,8 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_3, 0); lean_inc(x_7); lean_dec(x_3); -x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__2; -x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____spec__1(x_1, x_8); +x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__2; +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____spec__1(x_1, x_8); if (lean_obj_tag(x_9) == 0) { uint8_t x_10; @@ -9648,21 +13340,21 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____spec__1(x_1, x_2); +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____spec__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274_(x_1); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825_(x_1); lean_dec(x_1); return x_2; } @@ -9671,7 +13363,7 @@ static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokensLegend___closed__ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____boxed), 1, 0); return x_1; } } @@ -9683,7 +13375,7 @@ x_1 = l_Lean_Lsp_instFromJsonSemanticTokensLegend___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3329_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4880_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; @@ -9696,7 +13388,7 @@ x_5 = 0; x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_115____spec__2(x_4, x_5, x_2); x_7 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_7, 0, x_6); -x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__1; +x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__1; x_9 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_9, 0, x_8); lean_ctor_set(x_9, 1, x_7); @@ -9713,7 +13405,7 @@ lean_dec(x_13); x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_115____spec__2(x_14, x_5, x_12); x_16 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_16, 0, x_15); -x_17 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__2; +x_17 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__2; x_18 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_18, 0, x_17); lean_ctor_set(x_18, 1, x_16); @@ -9735,7 +13427,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokensLegend___closed__1( _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3329_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4880_), 1, 0); return x_1; } } @@ -9747,17 +13439,17 @@ x_1 = l_Lean_Lsp_instToJsonSemanticTokensLegend___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; x_3 = l_Lean_Json_getObjValD(x_1, x_2); -x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274_(x_3); +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825_(x_3); lean_dec(x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__1() { +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__1() { _start: { lean_object* x_1; @@ -9765,7 +13457,7 @@ x_1 = lean_mk_string_from_bytes("legend", 6); return x_1; } } -static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__2() { +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__2() { _start: { lean_object* x_1; @@ -9773,12 +13465,12 @@ x_1 = lean_mk_string_from_bytes("full", 4); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__1; -x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____spec__1(x_1, x_2); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____spec__1(x_1, x_2); if (lean_obj_tag(x_3) == 0) { uint8_t x_4; @@ -9832,7 +13524,7 @@ lean_object* x_13; lean_object* x_14; lean_object* x_15; x_13 = lean_ctor_get(x_9, 0); lean_inc(x_13); lean_dec(x_9); -x_14 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__2; +x_14 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__2; x_15 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_43____spec__3(x_1, x_14); if (lean_obj_tag(x_15) == 0) { @@ -9897,21 +13589,21 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____spec__1(x_1, x_2); +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____spec__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396_(x_1); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947_(x_1); lean_dec(x_1); return x_2; } @@ -9920,7 +13612,7 @@ static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokensOptions___closed_ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____boxed), 1, 0); return x_1; } } @@ -9932,14 +13624,14 @@ x_1 = l_Lean_Lsp_instFromJsonSemanticTokensOptions___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3468_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5019_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); -x_3 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3329_(x_2); -x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__1; +x_3 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4880_(x_2); +x_4 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__1; x_5 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_5, 0, x_4); lean_ctor_set(x_5, 1, x_3); @@ -9961,7 +13653,7 @@ x_13 = lean_ctor_get_uint8(x_1, sizeof(void*)*1 + 1); lean_dec(x_1); x_14 = lean_alloc_ctor(1, 0, 1); lean_ctor_set_uint8(x_14, 0, x_13); -x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__2; +x_15 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__2; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_14); @@ -9986,7 +13678,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokensOptions___closed__1 _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3468_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5019_), 1, 0); return x_1; } } @@ -9998,7 +13690,7 @@ x_1 = l_Lean_Lsp_instToJsonSemanticTokensOptions___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3530_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5081_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -10044,11 +13736,11 @@ return x_9; } } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3530____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5081____boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3530_(x_1); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5081_(x_1); lean_dec(x_1); return x_2; } @@ -10057,7 +13749,7 @@ static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokensParams___closed__ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3530____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5081____boxed), 1, 0); return x_1; } } @@ -10069,7 +13761,7 @@ x_1 = l_Lean_Lsp_instFromJsonSemanticTokensParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3568_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5119_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; @@ -10094,7 +13786,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokensParams___closed__1( _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3568_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5119_), 1, 0); return x_1; } } @@ -10106,7 +13798,7 @@ x_1 = l_Lean_Lsp_instToJsonSemanticTokensParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3616_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5167_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -10190,11 +13882,11 @@ return x_18; } } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3616____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5167____boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3616_(x_1); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5167_(x_1); lean_dec(x_1); return x_2; } @@ -10203,7 +13895,7 @@ static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokensRangeParams___clo _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3616____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5167____boxed), 1, 0); return x_1; } } @@ -10215,7 +13907,7 @@ x_1 = l_Lean_Lsp_instFromJsonSemanticTokensRangeParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3671_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5222_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; @@ -10256,7 +13948,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokensRangeParams___close _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3671_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5222_), 1, 0); return x_1; } } @@ -10268,7 +13960,15 @@ x_1 = l_Lean_Lsp_instToJsonSemanticTokensRangeParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__2(size_t x_1, size_t x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_Lsp_SemanticTokens_resultId_x3f___default() { +_start: +{ +lean_object* x_1; +x_1 = lean_box(0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__2(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -10324,7 +14024,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; @@ -10341,7 +14041,7 @@ x_5 = lean_array_get_size(x_4); x_6 = lean_usize_of_nat(x_5); lean_dec(x_5); x_7 = 0; -x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__2(x_6, x_7, x_4); +x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__2(x_6, x_7, x_4); return x_8; } else @@ -10360,7 +14060,15 @@ return x_15; } } } -static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____closed__1() { +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("resultId", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__2() { _start: { lean_object* x_1; @@ -10368,15 +14076,16 @@ x_1 = lean_mk_string_from_bytes("data", 4); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____closed__1; -x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__1(x_1, x_2); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2161____spec__1(x_1, x_2); if (lean_obj_tag(x_3) == 0) { uint8_t x_4; +lean_dec(x_1); x_4 = !lean_is_exclusive(x_3); if (x_4 == 0) { @@ -10395,26 +14104,64 @@ return x_6; } else { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_3); -if (x_7 == 0) +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__2; +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__1(x_1, x_8); +if (lean_obj_tag(x_9) == 0) { -return x_3; +uint8_t x_10; +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; } else { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_3, 0); -lean_inc(x_8); -lean_dec(x_3); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_8); +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; +} +} +else +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_9); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_9, 0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_7); +lean_ctor_set(x_15, 1, x_14); +lean_ctor_set(x_9, 0, x_15); return x_9; } +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_9, 0); +lean_inc(x_16); +lean_dec(x_9); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_7); +lean_ctor_set(x_17, 1, x_16); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; +} +} } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -10422,7 +14169,7 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____spec__2(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____spec__2(x_4, x_5, x_3); return x_6; } } @@ -10430,7 +14177,7 @@ static lean_object* _init_l_Lean_Lsp_instFromJsonSemanticTokens___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284_), 1, 0); return x_1; } } @@ -10442,7 +14189,7 @@ x_1 = l_Lean_Lsp_instFromJsonSemanticTokens___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761____spec__1(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339____spec__1(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -10469,34 +14216,45 @@ goto _start; } } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339_(lean_object* x_1) { _start: { -lean_object* x_2; size_t x_3; size_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_2 = lean_array_get_size(x_1); -x_3 = lean_usize_of_nat(x_2); +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__1; +x_4 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2131____spec__1(x_3, x_2); lean_dec(x_2); -x_4 = 0; -x_5 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761____spec__1(x_3, x_4, x_1); -x_6 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_6, 0, x_5); -x_7 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____closed__1; -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -x_9 = lean_box(0); -x_10 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_9); -x_12 = l_List_join___rarg(x_11); -x_13 = l_Lean_Json_mkObj(x_12); -return x_13; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_array_get_size(x_5); +x_7 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_8 = 0; +x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339____spec__1(x_7, x_8, x_5); +x_10 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__2; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_4); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_List_join___rarg(x_16); +x_18 = l_Lean_Json_mkObj(x_17); +return x_18; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -10504,7 +14262,7 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761____spec__1(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339____spec__1(x_4, x_5, x_3); return x_6; } } @@ -10512,7 +14270,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonSemanticTokens___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339_), 1, 0); return x_1; } } @@ -10524,7 +14282,7 @@ x_1 = l_Lean_Lsp_instToJsonSemanticTokens___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3801_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5383_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -10570,11 +14328,11 @@ return x_9; } } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3801____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5383____boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3801_(x_1); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5383_(x_1); lean_dec(x_1); return x_2; } @@ -10583,7 +14341,7 @@ static lean_object* _init_l_Lean_Lsp_instFromJsonFoldingRangeParams___closed__1( _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3801____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5383____boxed), 1, 0); return x_1; } } @@ -10595,7 +14353,7 @@ x_1 = l_Lean_Lsp_instFromJsonFoldingRangeParams___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3839_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5421_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; @@ -10620,7 +14378,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonFoldingRangeParams___closed__1() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3839_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5421_), 1, 0); return x_1; } } @@ -10699,7 +14457,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonFoldingRangeKind___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("comment", 7); +x_1 = lean_mk_string_from_bytes("imports", 7); return x_1; } } @@ -10717,7 +14475,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonFoldingRangeKind___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("imports", 7); +x_1 = lean_mk_string_from_bytes("region", 6); return x_1; } } @@ -10731,24 +14489,6 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Lsp_instToJsonFoldingRangeKind___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("region", 6); -return x_1; -} -} -static lean_object* _init_l_Lean_Lsp_instToJsonFoldingRangeKind___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__5; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Lsp_instToJsonFoldingRangeKind(uint8_t x_1) { _start: { @@ -10756,19 +14496,19 @@ switch (x_1) { case 0: { lean_object* x_2; -x_2 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__2; +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__36; return x_2; } case 1: { lean_object* x_3; -x_3 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__4; +x_3 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__2; return x_3; } default: { lean_object* x_4; -x_4 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__6; +x_4 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__4; return x_4; } } @@ -10792,7 +14532,7 @@ x_1 = lean_box(0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -10812,7 +14552,7 @@ switch (x_6) { case 0: { lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__2; +x_7 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__36; x_8 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_8, 0, x_1); lean_ctor_set(x_8, 1, x_7); @@ -10824,7 +14564,7 @@ return x_9; case 1: { lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__4; +x_10 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__2; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_1); lean_ctor_set(x_11, 1, x_10); @@ -10836,7 +14576,7 @@ return x_12; default: { lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__6; +x_13 = l_Lean_Lsp_instToJsonFoldingRangeKind___closed__4; x_14 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_14, 0, x_1); lean_ctor_set(x_14, 1, x_13); @@ -10849,7 +14589,7 @@ return x_15; } } } -static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__1() { +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__1() { _start: { lean_object* x_1; @@ -10857,7 +14597,7 @@ x_1 = lean_mk_string_from_bytes("startLine", 9); return x_1; } } -static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__2() { +static lean_object* _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__2() { _start: { lean_object* x_1; @@ -10865,7 +14605,7 @@ x_1 = lean_mk_string_from_bytes("endLine", 7); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; @@ -10874,7 +14614,7 @@ lean_inc(x_2); x_3 = l_Lean_JsonNumber_fromNat(x_2); x_4 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_4, 0, x_3); -x_5 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__1; +x_5 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__1; x_6 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_6, 0, x_5); lean_ctor_set(x_6, 1, x_4); @@ -10887,7 +14627,7 @@ lean_inc(x_9); x_10 = l_Lean_JsonNumber_fromNat(x_9); x_11 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_11, 0, x_10); -x_12 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__2; +x_12 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__2; x_13 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_13, 0, x_12); lean_ctor_set(x_13, 1, x_11); @@ -10898,7 +14638,7 @@ x_15 = lean_ctor_get(x_1, 2); lean_inc(x_15); lean_dec(x_1); x_16 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1276____closed__4; -x_17 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____spec__1(x_16, x_15); +x_17 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____spec__1(x_16, x_15); lean_dec(x_15); x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_17); @@ -10914,11 +14654,11 @@ x_22 = l_Lean_Json_mkObj(x_21); return x_22; } } -LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____spec__1(x_1, x_2); +x_3 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____spec__1(x_1, x_2); lean_dec(x_2); return x_3; } @@ -10927,7 +14667,7 @@ static lean_object* _init_l_Lean_Lsp_instToJsonFoldingRange___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504_), 1, 0); return x_1; } } @@ -11586,6 +15326,162 @@ l_Lean_Lsp_instToJsonSymbolInformation___closed__1 = _init_l_Lean_Lsp_instToJson lean_mark_persistent(l_Lean_Lsp_instToJsonSymbolInformation___closed__1); l_Lean_Lsp_instToJsonSymbolInformation = _init_l_Lean_Lsp_instToJsonSymbolInformation(); lean_mark_persistent(l_Lean_Lsp_instToJsonSymbolInformation); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__2); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__3 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__3(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__3); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__4 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__4(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__4); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__5 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__5(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__5); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__6 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__6(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__6); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__7 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__7(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__7); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__8 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__8(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__8); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__9 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__9(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__9); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__10 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__10(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__10); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__11 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__11(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__11); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__12 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__12(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__12); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__13 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__13(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__13); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__14 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__14(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__14); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__15 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__15(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__15); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__16 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__16(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__16); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__17 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__17(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__17); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__18 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__18(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__18); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__19 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__19(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__19); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__20 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__20(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__20); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__21 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__21(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__21); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__22 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__22(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__22); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__23 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__23(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__23); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__24 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__24(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__24); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__25 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__25(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__25); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__26 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__26(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__26); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__27 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__27(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__27); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__28 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__28(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__28); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__29 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__29(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__29); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__30 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__30(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__30); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__31 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__31(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__31); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__32 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__32(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__32); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__33 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__33(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__33); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__34 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__34(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__34); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__35 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__35(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__35); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__36 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__36(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__36); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__37 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__37(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__37); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__38 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__38(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__38); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__39 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__39(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__39); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__40 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__40(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__40); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__41 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__41(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__41); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__42 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__42(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__42); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__43 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__43(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__43); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__44 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__44(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__44); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__45 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__45(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__45); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__46 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__46(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3205____closed__46); +l_Lean_Lsp_instToJsonSemanticTokenType___closed__1 = _init_l_Lean_Lsp_instToJsonSemanticTokenType___closed__1(); +lean_mark_persistent(l_Lean_Lsp_instToJsonSemanticTokenType___closed__1); +l_Lean_Lsp_instToJsonSemanticTokenType = _init_l_Lean_Lsp_instToJsonSemanticTokenType(); +lean_mark_persistent(l_Lean_Lsp_instToJsonSemanticTokenType); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__1___closed__2); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__2); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__3 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__2___closed__3); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__3___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__4___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__5___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__6___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__7___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__8___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__9___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__10___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__11___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__12___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__13___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__14___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__15___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__16___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__17___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__18___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__19___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__20___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__21___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__22___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____lambda__23___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenType____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3310____closed__2); +l_Lean_Lsp_instFromJsonSemanticTokenType___closed__1 = _init_l_Lean_Lsp_instFromJsonSemanticTokenType___closed__1(); +lean_mark_persistent(l_Lean_Lsp_instFromJsonSemanticTokenType___closed__1); +l_Lean_Lsp_instFromJsonSemanticTokenType = _init_l_Lean_Lsp_instFromJsonSemanticTokenType(); +lean_mark_persistent(l_Lean_Lsp_instFromJsonSemanticTokenType); l_Lean_Lsp_SemanticTokenType_names___closed__1 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__1(); lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__1); l_Lean_Lsp_SemanticTokenType_names___closed__2 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__2(); @@ -11604,12 +15500,134 @@ l_Lean_Lsp_SemanticTokenType_names___closed__8 = _init_l_Lean_Lsp_SemanticTokenT lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__8); l_Lean_Lsp_SemanticTokenType_names___closed__9 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__9(); lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__9); +l_Lean_Lsp_SemanticTokenType_names___closed__10 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__10(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__10); +l_Lean_Lsp_SemanticTokenType_names___closed__11 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__11(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__11); +l_Lean_Lsp_SemanticTokenType_names___closed__12 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__12(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__12); +l_Lean_Lsp_SemanticTokenType_names___closed__13 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__13(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__13); +l_Lean_Lsp_SemanticTokenType_names___closed__14 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__14(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__14); +l_Lean_Lsp_SemanticTokenType_names___closed__15 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__15(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__15); +l_Lean_Lsp_SemanticTokenType_names___closed__16 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__16(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__16); +l_Lean_Lsp_SemanticTokenType_names___closed__17 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__17(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__17); +l_Lean_Lsp_SemanticTokenType_names___closed__18 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__18(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__18); +l_Lean_Lsp_SemanticTokenType_names___closed__19 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__19(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__19); +l_Lean_Lsp_SemanticTokenType_names___closed__20 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__20(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__20); +l_Lean_Lsp_SemanticTokenType_names___closed__21 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__21(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__21); +l_Lean_Lsp_SemanticTokenType_names___closed__22 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__22(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__22); +l_Lean_Lsp_SemanticTokenType_names___closed__23 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__23(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__23); +l_Lean_Lsp_SemanticTokenType_names___closed__24 = _init_l_Lean_Lsp_SemanticTokenType_names___closed__24(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names___closed__24); l_Lean_Lsp_SemanticTokenType_names = _init_l_Lean_Lsp_SemanticTokenType_names(); lean_mark_persistent(l_Lean_Lsp_SemanticTokenType_names); -l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__1(); -lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__1); -l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__2(); -lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3274____closed__2); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__2); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__3 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__3(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__3); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__4 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__4(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__4); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__5 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__5(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__5); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__6 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__6(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__6); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__7 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__7(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__7); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__8 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__8(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__8); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__9 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__9(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__9); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__10 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__10(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__10); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__11 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__11(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__11); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__12 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__12(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__12); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__13 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__13(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__13); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__14 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__14(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__14); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__15 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__15(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__15); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__16 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__16(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__16); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__17 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__17(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__17); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__18 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__18(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__18); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__19 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__19(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4286____closed__19); +l_Lean_Lsp_instToJsonSemanticTokenModifier___closed__1 = _init_l_Lean_Lsp_instToJsonSemanticTokenModifier___closed__1(); +lean_mark_persistent(l_Lean_Lsp_instToJsonSemanticTokenModifier___closed__1); +l_Lean_Lsp_instToJsonSemanticTokenModifier = _init_l_Lean_Lsp_instToJsonSemanticTokenModifier(); +lean_mark_persistent(l_Lean_Lsp_instToJsonSemanticTokenModifier); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__1___closed__2); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__2___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__3___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__4___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__5___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__6___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__7___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__8___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____lambda__9___closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokenModifier____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4339____closed__1); +l_Lean_Lsp_instFromJsonSemanticTokenModifier___closed__1 = _init_l_Lean_Lsp_instFromJsonSemanticTokenModifier___closed__1(); +lean_mark_persistent(l_Lean_Lsp_instFromJsonSemanticTokenModifier___closed__1); +l_Lean_Lsp_instFromJsonSemanticTokenModifier = _init_l_Lean_Lsp_instFromJsonSemanticTokenModifier(); +lean_mark_persistent(l_Lean_Lsp_instFromJsonSemanticTokenModifier); +l_Lean_Lsp_SemanticTokenModifier_names___closed__1 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__1(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__1); +l_Lean_Lsp_SemanticTokenModifier_names___closed__2 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__2(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__2); +l_Lean_Lsp_SemanticTokenModifier_names___closed__3 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__3(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__3); +l_Lean_Lsp_SemanticTokenModifier_names___closed__4 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__4(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__4); +l_Lean_Lsp_SemanticTokenModifier_names___closed__5 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__5(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__5); +l_Lean_Lsp_SemanticTokenModifier_names___closed__6 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__6(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__6); +l_Lean_Lsp_SemanticTokenModifier_names___closed__7 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__7(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__7); +l_Lean_Lsp_SemanticTokenModifier_names___closed__8 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__8(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__8); +l_Lean_Lsp_SemanticTokenModifier_names___closed__9 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__9(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__9); +l_Lean_Lsp_SemanticTokenModifier_names___closed__10 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__10(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__10); +l_Lean_Lsp_SemanticTokenModifier_names___closed__11 = _init_l_Lean_Lsp_SemanticTokenModifier_names___closed__11(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names___closed__11); +l_Lean_Lsp_SemanticTokenModifier_names = _init_l_Lean_Lsp_SemanticTokenModifier_names(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokenModifier_names); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensLegend____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4825____closed__2); l_Lean_Lsp_instFromJsonSemanticTokensLegend___closed__1 = _init_l_Lean_Lsp_instFromJsonSemanticTokensLegend___closed__1(); lean_mark_persistent(l_Lean_Lsp_instFromJsonSemanticTokensLegend___closed__1); l_Lean_Lsp_instFromJsonSemanticTokensLegend = _init_l_Lean_Lsp_instFromJsonSemanticTokensLegend(); @@ -11618,10 +15636,10 @@ l_Lean_Lsp_instToJsonSemanticTokensLegend___closed__1 = _init_l_Lean_Lsp_instToJ lean_mark_persistent(l_Lean_Lsp_instToJsonSemanticTokensLegend___closed__1); l_Lean_Lsp_instToJsonSemanticTokensLegend = _init_l_Lean_Lsp_instToJsonSemanticTokensLegend(); lean_mark_persistent(l_Lean_Lsp_instToJsonSemanticTokensLegend); -l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__1(); -lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__1); -l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__2(); -lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3396____closed__2); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensOptions____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4947____closed__2); l_Lean_Lsp_instFromJsonSemanticTokensOptions___closed__1 = _init_l_Lean_Lsp_instFromJsonSemanticTokensOptions___closed__1(); lean_mark_persistent(l_Lean_Lsp_instFromJsonSemanticTokensOptions___closed__1); l_Lean_Lsp_instFromJsonSemanticTokensOptions = _init_l_Lean_Lsp_instFromJsonSemanticTokensOptions(); @@ -11646,8 +15664,12 @@ l_Lean_Lsp_instToJsonSemanticTokensRangeParams___closed__1 = _init_l_Lean_Lsp_in lean_mark_persistent(l_Lean_Lsp_instToJsonSemanticTokensRangeParams___closed__1); l_Lean_Lsp_instToJsonSemanticTokensRangeParams = _init_l_Lean_Lsp_instToJsonSemanticTokensRangeParams(); lean_mark_persistent(l_Lean_Lsp_instToJsonSemanticTokensRangeParams); -l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____closed__1(); -lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3723____closed__1); +l_Lean_Lsp_SemanticTokens_resultId_x3f___default = _init_l_Lean_Lsp_SemanticTokens_resultId_x3f___default(); +lean_mark_persistent(l_Lean_Lsp_SemanticTokens_resultId_x3f___default); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5284____closed__2); l_Lean_Lsp_instFromJsonSemanticTokens___closed__1 = _init_l_Lean_Lsp_instFromJsonSemanticTokens___closed__1(); lean_mark_persistent(l_Lean_Lsp_instFromJsonSemanticTokens___closed__1); l_Lean_Lsp_instFromJsonSemanticTokens = _init_l_Lean_Lsp_instFromJsonSemanticTokens(); @@ -11672,16 +15694,12 @@ l_Lean_Lsp_instToJsonFoldingRangeKind___closed__3 = _init_l_Lean_Lsp_instToJsonF lean_mark_persistent(l_Lean_Lsp_instToJsonFoldingRangeKind___closed__3); l_Lean_Lsp_instToJsonFoldingRangeKind___closed__4 = _init_l_Lean_Lsp_instToJsonFoldingRangeKind___closed__4(); lean_mark_persistent(l_Lean_Lsp_instToJsonFoldingRangeKind___closed__4); -l_Lean_Lsp_instToJsonFoldingRangeKind___closed__5 = _init_l_Lean_Lsp_instToJsonFoldingRangeKind___closed__5(); -lean_mark_persistent(l_Lean_Lsp_instToJsonFoldingRangeKind___closed__5); -l_Lean_Lsp_instToJsonFoldingRangeKind___closed__6 = _init_l_Lean_Lsp_instToJsonFoldingRangeKind___closed__6(); -lean_mark_persistent(l_Lean_Lsp_instToJsonFoldingRangeKind___closed__6); l_Lean_Lsp_FoldingRange_kind_x3f___default = _init_l_Lean_Lsp_FoldingRange_kind_x3f___default(); lean_mark_persistent(l_Lean_Lsp_FoldingRange_kind_x3f___default); -l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__1(); -lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__1); -l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__2(); -lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922____closed__2); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__1 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__1(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__1); +l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__2 = _init_l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__2(); +lean_mark_persistent(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504____closed__2); l_Lean_Lsp_instToJsonFoldingRange___closed__1 = _init_l_Lean_Lsp_instToJsonFoldingRange___closed__1(); lean_mark_persistent(l_Lean_Lsp_instToJsonFoldingRange___closed__1); l_Lean_Lsp_instToJsonFoldingRange = _init_l_Lean_Lsp_instToJsonFoldingRange(); diff --git a/stage0/stdlib/Lean/Data/Options.c b/stage0/stdlib/Lean/Data/Options.c index f425bb98be39..413ff4461298 100644 --- a/stage0/stdlib/Lean/Data/Options.c +++ b/stage0/stdlib/Lean/Data/Options.c @@ -24,15 +24,18 @@ static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Le static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22; LEAN_EXPORT lean_object* l_Lean_Option_register(lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__17; +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__54; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__8; lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__52; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; LEAN_EXPORT lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__1; LEAN_EXPORT lean_object* l_Lean_OptionDecl_group___default; LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_getOptionDecl___spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__46; static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; LEAN_EXPORT lean_object* l_Lean_instMonadWithOptions___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_registerOption___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -89,6 +92,7 @@ static lean_object* l_Lean_registerOption___closed__1; static lean_object* l_Lean_registerOption___closed__2; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__25; LEAN_EXPORT lean_object* l_Lean_Option_setIfNotSet(lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56; lean_object* l_Lean_KVMap_instForInKVMapProdNameDataValue(lean_object*, lean_object*); static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__24; LEAN_EXPORT lean_object* l___private_Lean_Data_Options_0__Lean_optionDeclsRef; @@ -97,8 +101,10 @@ lean_object* l_String_toName(lean_object*); static lean_object* l_Lean_setOptionFromString___closed__4; LEAN_EXPORT lean_object* l_Lean_instMonadOptions(lean_object*, lean_object*); lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57; static lean_object* l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__7; LEAN_EXPORT lean_object* l_Lean_getOptionDecl(lean_object*, lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49; static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__7; static lean_object* l_Lean_withInPattern___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_OptionDecl_descr___default; @@ -111,6 +117,7 @@ static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Le static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__6; LEAN_EXPORT lean_object* l_Lean_instMonadOptions___rarg(lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__50; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__13; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Data_Options___hyg_121_(lean_object*); static lean_object* l_Lean_setOptionFromString___closed__8; @@ -144,6 +151,7 @@ static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Le LEAN_EXPORT lean_object* l_Std_RBNode_fold___at_Lean_getOptionDeclsArray___spec__1(lean_object*, lean_object*); lean_object* l_Lean_KVMap_setName(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Option_register___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__48; LEAN_EXPORT lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__5; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__18; @@ -155,10 +163,12 @@ LEAN_EXPORT lean_object* l_Lean_Option_get_x3f___rarg___boxed(lean_object*, lean LEAN_EXPORT lean_object* l_Lean_instMonadWithOptions___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_registerOption___lambda__2___closed__1; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__24; +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55; LEAN_EXPORT lean_object* l_Lean_setOptionFromString(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__37; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__15; static lean_object* l_Lean_setOptionFromString___closed__6; +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53; static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__28; LEAN_EXPORT lean_object* l_Lean_registerOption___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -196,7 +206,6 @@ lean_object* l_Lean_KVMap_findCore(lean_object*, lean_object*); static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__1; LEAN_EXPORT lean_object* l_Lean_Option_set(lean_object*); lean_object* l_String_trim(lean_object*); -static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2; static lean_object* l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__2; static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; static lean_object* l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__8; @@ -210,6 +219,7 @@ static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Le static lean_object* l_Lean_setOptionFromString___closed__2; static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__45; static lean_object* l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__26; LEAN_EXPORT lean_object* l_Lean_Option_commandRegister__option___x3a___x3a_x3d__; static lean_object* l_Lean_withInPattern___rarg___lambda__1___closed__1; @@ -223,6 +233,7 @@ static lean_object* l_Lean_setOptionFromString___closed__7; LEAN_EXPORT lean_object* l_Lean_instInhabitedOptionDecls; static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__2; LEAN_EXPORT lean_object* l_Lean_getOptionDescr(lean_object*, lean_object*); +static lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47; static lean_object* l_Lean_setOptionFromString___closed__3; LEAN_EXPORT lean_object* l_Lean_getNatOption___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_setOptionFromString___spec__1(lean_object*, lean_object*); @@ -2373,7 +2384,7 @@ static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRul _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("builtin_initialize", 18); +x_1 = lean_mk_string_from_bytes("initialize", 10); return x_1; } } @@ -2391,7 +2402,7 @@ static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRul _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("null", 4); +x_1 = lean_mk_string_from_bytes("declModifiers", 13); return x_1; } } @@ -2399,7 +2410,7 @@ static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRul _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__4; x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -2408,9 +2419,27 @@ return x_3; static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("null", 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__8; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__10; x_3 = l_Lean_getOptionDeclsArray___closed__1; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); @@ -2419,7 +2448,125 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__10() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(6u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__12; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__13; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__14; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__15; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__16; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__17; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__8; +x_3 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__18; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__20() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("initializeKeyword", 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__4; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__20; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("builtin_initialize", 18); +return x_1; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__24() { _start: { lean_object* x_1; @@ -2427,17 +2574,17 @@ x_1 = lean_mk_string_from_bytes("Term", 4); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__2; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__10; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__24; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__12() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__26() { _start: { lean_object* x_1; @@ -2445,17 +2592,17 @@ x_1 = lean_mk_string_from_bytes("typeSpec", 8); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__13() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__12; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__26; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__14() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__28() { _start: { lean_object* x_1; @@ -2463,7 +2610,7 @@ x_1 = lean_mk_string_from_bytes(":", 1); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__15() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29() { _start: { lean_object* x_1; @@ -2471,17 +2618,17 @@ x_1 = lean_mk_string_from_bytes("app", 3); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__16() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__30() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__15; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__17() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31() { _start: { lean_object* x_1; @@ -2489,22 +2636,22 @@ x_1 = lean_mk_string_from_bytes("Lean.Option", 11); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__18() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__32() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__17; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__19() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__17; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__18; +x_3 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__32; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -2512,7 +2659,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__20() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__34() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -2524,28 +2671,19 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__21() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__35() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__20; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__34; 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_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36() { _start: { lean_object* x_1; lean_object* x_2; @@ -2554,7 +2692,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__24() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__37() { _start: { lean_object* x_1; @@ -2562,7 +2700,7 @@ x_1 = lean_mk_string_from_bytes("←", 3); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38() { _start: { lean_object* x_1; lean_object* x_2; @@ -2571,7 +2709,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__26() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__39() { _start: { lean_object* x_1; @@ -2579,17 +2717,17 @@ x_1 = lean_mk_string_from_bytes("doSeqIndent", 11); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__26; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__39; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__28() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__41() { _start: { lean_object* x_1; @@ -2597,17 +2735,17 @@ x_1 = lean_mk_string_from_bytes("doSeqItem", 9); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__28; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__41; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__30() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__43() { _start: { lean_object* x_1; @@ -2615,17 +2753,17 @@ x_1 = lean_mk_string_from_bytes("doExpr", 6); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__30; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__43; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__32() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__45() { _start: { lean_object* x_1; @@ -2633,22 +2771,22 @@ x_1 = lean_mk_string_from_bytes("Lean.Option.register", 20); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__33() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__46() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__32; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__45; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__34() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__32; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__45; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__33; +x_3 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__46; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -2656,7 +2794,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__35() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__48() { _start: { lean_object* x_1; @@ -2664,41 +2802,41 @@ x_1 = lean_mk_string_from_bytes("register", 8); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__35; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__48; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__37() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__50() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__37; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__50; 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_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__39() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__52() { _start: { lean_object* x_1; lean_object* x_2; @@ -2707,17 +2845,17 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__39; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__52; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__19; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__41() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__54() { _start: { lean_object* x_1; @@ -2725,17 +2863,17 @@ x_1 = lean_mk_string_from_bytes("quotedName", 10); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__41; +x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__54; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__43() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56() { _start: { lean_object* x_1; @@ -2743,7 +2881,7 @@ x_1 = lean_mk_string_from_bytes(".", 1); return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44() { +static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57() { _start: { lean_object* x_1; @@ -2784,410 +2922,422 @@ x_14 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRul x_15 = !lean_is_exclusive(x_14); if (x_15 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; 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_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; x_16 = lean_ctor_get(x_14, 0); x_17 = lean_ctor_get(x_2, 2); lean_inc(x_17); x_18 = lean_ctor_get(x_2, 1); lean_inc(x_18); lean_dec(x_2); -x_19 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__5; +x_19 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22; lean_inc(x_16); x_20 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_20, 0, x_16); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__14; +x_21 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23; +x_22 = lean_array_push(x_21, x_20); +x_23 = lean_box(2); +x_24 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__21; +x_25 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +lean_ctor_set(x_25, 2, x_22); +x_26 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__28; lean_inc(x_16); -x_22 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_22, 0, x_16); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; +x_27 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_27, 0, x_16); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; lean_inc(x_17); lean_inc(x_18); -x_24 = l_Lean_addMacroScope(x_18, x_23, x_17); -x_25 = lean_box(0); -x_26 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__19; -x_27 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__21; +x_29 = l_Lean_addMacroScope(x_18, x_28, x_17); +x_30 = lean_box(0); +x_31 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__33; +x_32 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__35; lean_inc(x_16); -x_28 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_28, 0, x_16); -lean_ctor_set(x_28, 1, x_26); -lean_ctor_set(x_28, 2, x_24); -lean_ctor_set(x_28, 3, x_27); -x_29 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22; -x_30 = lean_array_push(x_29, x_11); -x_31 = lean_box(2); -x_32 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__8; -x_33 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -lean_ctor_set(x_33, 2, x_30); -x_34 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23; -x_35 = lean_array_push(x_34, x_28); -x_36 = lean_array_push(x_35, x_33); -x_37 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__16; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_31); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_36); -x_39 = lean_array_push(x_34, x_22); -x_40 = lean_array_push(x_39, x_38); -x_41 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__13; -x_42 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_42, 0, x_31); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_40); -x_43 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__24; +x_33 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_33, 0, x_16); +lean_ctor_set(x_33, 1, x_31); +lean_ctor_set(x_33, 2, x_29); +lean_ctor_set(x_33, 3, x_32); +x_34 = lean_array_push(x_21, x_11); +x_35 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__10; +x_36 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_36, 0, x_23); +lean_ctor_set(x_36, 1, x_35); +lean_ctor_set(x_36, 2, x_34); +x_37 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; +x_38 = lean_array_push(x_37, x_33); +x_39 = lean_array_push(x_38, x_36); +x_40 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__30; +x_41 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_41, 0, x_23); +lean_ctor_set(x_41, 1, x_40); +lean_ctor_set(x_41, 2, x_39); +x_42 = lean_array_push(x_37, x_27); +x_43 = lean_array_push(x_42, x_41); +x_44 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; +x_45 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_45, 0, x_23); +lean_ctor_set(x_45, 1, x_44); +lean_ctor_set(x_45, 2, x_43); +x_46 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__37; lean_inc(x_16); -x_44 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_44, 0, x_16); -lean_ctor_set(x_44, 1, x_43); -x_45 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +x_47 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_47, 0, x_16); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38; lean_inc(x_9); -x_46 = lean_array_push(x_45, x_9); -x_47 = lean_array_push(x_46, x_42); -x_48 = lean_array_push(x_47, x_44); -x_49 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_49, 0, x_31); -lean_ctor_set(x_49, 1, x_32); -lean_ctor_set(x_49, 2, x_48); -x_50 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; -x_51 = l_Lean_addMacroScope(x_18, x_50, x_17); -x_52 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__34; -x_53 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38; -x_54 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_54, 0, x_16); -lean_ctor_set(x_54, 1, x_52); -lean_ctor_set(x_54, 2, x_51); -lean_ctor_set(x_54, 3, x_53); -x_55 = l_Lean_Syntax_getId(x_9); +x_49 = lean_array_push(x_48, x_9); +x_50 = lean_array_push(x_49, x_45); +x_51 = lean_array_push(x_50, x_47); +x_52 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_52, 0, x_23); +lean_ctor_set(x_52, 1, x_35); +lean_ctor_set(x_52, 2, x_51); +x_53 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49; +x_54 = l_Lean_addMacroScope(x_18, x_53, x_17); +x_55 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47; +x_56 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51; +x_57 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_57, 0, x_16); +lean_ctor_set(x_57, 1, x_55); +lean_ctor_set(x_57, 2, x_54); +lean_ctor_set(x_57, 3, x_56); +x_58 = l_Lean_Syntax_getId(x_9); lean_dec(x_9); -lean_inc(x_55); -x_56 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_25, x_55); -x_57 = lean_array_push(x_34, x_54); -x_58 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; -x_59 = lean_array_push(x_58, x_20); -x_60 = lean_array_push(x_59, x_49); -if (lean_obj_tag(x_56) == 0) -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; 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_61 = l_Lean_quoteNameMk(x_55); -x_62 = lean_array_push(x_34, x_61); -x_63 = lean_array_push(x_62, x_13); -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_31); -lean_ctor_set(x_64, 1, x_32); -lean_ctor_set(x_64, 2, x_63); -x_65 = lean_array_push(x_57, x_64); -x_66 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_66, 0, x_31); -lean_ctor_set(x_66, 1, x_37); -lean_ctor_set(x_66, 2, x_65); -x_67 = lean_array_push(x_29, x_66); -x_68 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; +lean_inc(x_58); +x_59 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_30, x_58); +x_60 = lean_array_push(x_37, x_57); +x_61 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53; +x_62 = lean_array_push(x_61, x_25); +x_63 = lean_array_push(x_62, x_52); +if (lean_obj_tag(x_59) == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; 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; +x_64 = l_Lean_quoteNameMk(x_58); +x_65 = lean_array_push(x_37, x_64); +x_66 = lean_array_push(x_65, x_13); +x_67 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_67, 0, x_23); +lean_ctor_set(x_67, 1, x_35); +lean_ctor_set(x_67, 2, x_66); +x_68 = lean_array_push(x_60, x_67); x_69 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_69, 0, x_31); -lean_ctor_set(x_69, 1, x_68); -lean_ctor_set(x_69, 2, x_67); -x_70 = lean_array_push(x_34, x_69); -x_71 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; -x_72 = lean_array_push(x_70, x_71); -x_73 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; -x_74 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_74, 0, x_31); -lean_ctor_set(x_74, 1, x_73); -lean_ctor_set(x_74, 2, x_72); -x_75 = lean_array_push(x_29, x_74); -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_31); -lean_ctor_set(x_76, 1, x_32); -lean_ctor_set(x_76, 2, x_75); -x_77 = lean_array_push(x_29, x_76); -x_78 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; +lean_ctor_set(x_69, 0, x_23); +lean_ctor_set(x_69, 1, x_40); +lean_ctor_set(x_69, 2, x_68); +x_70 = lean_array_push(x_21, x_69); +x_71 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; +x_72 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_72, 0, x_23); +lean_ctor_set(x_72, 1, x_71); +lean_ctor_set(x_72, 2, x_70); +x_73 = lean_array_push(x_37, x_72); +x_74 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_75 = lean_array_push(x_73, x_74); +x_76 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; +x_77 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_77, 0, x_23); +lean_ctor_set(x_77, 1, x_76); +lean_ctor_set(x_77, 2, x_75); +x_78 = lean_array_push(x_21, x_77); x_79 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_79, 0, x_31); -lean_ctor_set(x_79, 1, x_78); -lean_ctor_set(x_79, 2, x_77); -x_80 = lean_array_push(x_60, x_79); -x_81 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +lean_ctor_set(x_79, 0, x_23); +lean_ctor_set(x_79, 1, x_35); +lean_ctor_set(x_79, 2, x_78); +x_80 = lean_array_push(x_21, x_79); +x_81 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; x_82 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_82, 0, x_31); +lean_ctor_set(x_82, 0, x_23); lean_ctor_set(x_82, 1, x_81); lean_ctor_set(x_82, 2, x_80); -lean_ctor_set(x_14, 0, x_82); +x_83 = lean_array_push(x_63, x_82); +x_84 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +x_85 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_85, 0, x_23); +lean_ctor_set(x_85, 1, x_84); +lean_ctor_set(x_85, 2, x_83); +lean_ctor_set(x_14, 0, x_85); return x_14; } else { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; 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_dec(x_55); -x_83 = lean_ctor_get(x_56, 0); -lean_inc(x_83); -lean_dec(x_56); -x_84 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__43; -x_85 = l_String_intercalate(x_84, x_83); -x_86 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; -x_87 = lean_string_append(x_86, x_85); -lean_dec(x_85); -x_88 = l_Lean_Syntax_mkNameLit(x_87, x_31); -x_89 = lean_array_push(x_29, x_88); -x_90 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; -x_91 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_91, 0, x_31); -lean_ctor_set(x_91, 1, x_90); -lean_ctor_set(x_91, 2, x_89); -x_92 = lean_array_push(x_34, x_91); -x_93 = lean_array_push(x_92, x_13); +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +lean_dec(x_58); +x_86 = lean_ctor_get(x_59, 0); +lean_inc(x_86); +lean_dec(x_59); +x_87 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56; +x_88 = l_String_intercalate(x_87, x_86); +x_89 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57; +x_90 = lean_string_append(x_89, x_88); +lean_dec(x_88); +x_91 = l_Lean_Syntax_mkNameLit(x_90, x_23); +x_92 = lean_array_push(x_21, x_91); +x_93 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55; x_94 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_94, 0, x_31); -lean_ctor_set(x_94, 1, x_32); -lean_ctor_set(x_94, 2, x_93); -x_95 = lean_array_push(x_57, x_94); -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_31); -lean_ctor_set(x_96, 1, x_37); -lean_ctor_set(x_96, 2, x_95); -x_97 = lean_array_push(x_29, x_96); -x_98 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; +lean_ctor_set(x_94, 0, x_23); +lean_ctor_set(x_94, 1, x_93); +lean_ctor_set(x_94, 2, x_92); +x_95 = lean_array_push(x_37, x_94); +x_96 = lean_array_push(x_95, x_13); +x_97 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_97, 0, x_23); +lean_ctor_set(x_97, 1, x_35); +lean_ctor_set(x_97, 2, x_96); +x_98 = lean_array_push(x_60, x_97); x_99 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_99, 0, x_31); -lean_ctor_set(x_99, 1, x_98); -lean_ctor_set(x_99, 2, x_97); -x_100 = lean_array_push(x_34, x_99); -x_101 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; -x_102 = lean_array_push(x_100, x_101); -x_103 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; -x_104 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_104, 0, x_31); -lean_ctor_set(x_104, 1, x_103); -lean_ctor_set(x_104, 2, x_102); -x_105 = lean_array_push(x_29, x_104); -x_106 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_106, 0, x_31); -lean_ctor_set(x_106, 1, x_32); -lean_ctor_set(x_106, 2, x_105); -x_107 = lean_array_push(x_29, x_106); -x_108 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; +lean_ctor_set(x_99, 0, x_23); +lean_ctor_set(x_99, 1, x_40); +lean_ctor_set(x_99, 2, x_98); +x_100 = lean_array_push(x_21, x_99); +x_101 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; +x_102 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_102, 0, x_23); +lean_ctor_set(x_102, 1, x_101); +lean_ctor_set(x_102, 2, x_100); +x_103 = lean_array_push(x_37, x_102); +x_104 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_105 = lean_array_push(x_103, x_104); +x_106 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; +x_107 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_107, 0, x_23); +lean_ctor_set(x_107, 1, x_106); +lean_ctor_set(x_107, 2, x_105); +x_108 = lean_array_push(x_21, x_107); x_109 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_109, 0, x_31); -lean_ctor_set(x_109, 1, x_108); -lean_ctor_set(x_109, 2, x_107); -x_110 = lean_array_push(x_60, x_109); -x_111 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +lean_ctor_set(x_109, 0, x_23); +lean_ctor_set(x_109, 1, x_35); +lean_ctor_set(x_109, 2, x_108); +x_110 = lean_array_push(x_21, x_109); +x_111 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; x_112 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_112, 0, x_31); +lean_ctor_set(x_112, 0, x_23); lean_ctor_set(x_112, 1, x_111); lean_ctor_set(x_112, 2, x_110); -lean_ctor_set(x_14, 0, x_112); +x_113 = lean_array_push(x_63, x_112); +x_114 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +x_115 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_115, 0, x_23); +lean_ctor_set(x_115, 1, x_114); +lean_ctor_set(x_115, 2, x_113); +lean_ctor_set(x_14, 0, x_115); return x_14; } } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; 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_113 = lean_ctor_get(x_14, 0); -x_114 = lean_ctor_get(x_14, 1); -lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_14); -x_115 = lean_ctor_get(x_2, 2); -lean_inc(x_115); -x_116 = lean_ctor_get(x_2, 1); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; 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; +x_116 = lean_ctor_get(x_14, 0); +x_117 = lean_ctor_get(x_14, 1); +lean_inc(x_117); lean_inc(x_116); +lean_dec(x_14); +x_118 = lean_ctor_get(x_2, 2); +lean_inc(x_118); +x_119 = lean_ctor_get(x_2, 1); +lean_inc(x_119); lean_dec(x_2); -x_117 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__5; -lean_inc(x_113); -x_118 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_118, 0, x_113); -lean_ctor_set(x_118, 1, x_117); -x_119 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__14; -lean_inc(x_113); -x_120 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_120, 0, x_113); -lean_ctor_set(x_120, 1, x_119); -x_121 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; -lean_inc(x_115); +x_120 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22; lean_inc(x_116); -x_122 = l_Lean_addMacroScope(x_116, x_121, x_115); -x_123 = lean_box(0); -x_124 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__19; +x_121 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_121, 0, x_116); +lean_ctor_set(x_121, 1, x_120); +x_122 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23; +x_123 = lean_array_push(x_122, x_121); +x_124 = lean_box(2); x_125 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__21; -lean_inc(x_113); -x_126 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_126, 0, x_113); -lean_ctor_set(x_126, 1, x_124); -lean_ctor_set(x_126, 2, x_122); -lean_ctor_set(x_126, 3, x_125); -x_127 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22; -x_128 = lean_array_push(x_127, x_11); -x_129 = lean_box(2); -x_130 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__8; -x_131 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_131, 0, x_129); -lean_ctor_set(x_131, 1, x_130); -lean_ctor_set(x_131, 2, x_128); -x_132 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23; -x_133 = lean_array_push(x_132, x_126); -x_134 = lean_array_push(x_133, x_131); -x_135 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__16; -x_136 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_136, 0, x_129); -lean_ctor_set(x_136, 1, x_135); -lean_ctor_set(x_136, 2, x_134); -x_137 = lean_array_push(x_132, x_120); -x_138 = lean_array_push(x_137, x_136); -x_139 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__13; -x_140 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_140, 0, x_129); -lean_ctor_set(x_140, 1, x_139); -lean_ctor_set(x_140, 2, x_138); -x_141 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__24; -lean_inc(x_113); -x_142 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_142, 0, x_113); +x_126 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +lean_ctor_set(x_126, 2, x_123); +x_127 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__28; +lean_inc(x_116); +x_128 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_128, 0, x_116); +lean_ctor_set(x_128, 1, x_127); +x_129 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; +lean_inc(x_118); +lean_inc(x_119); +x_130 = l_Lean_addMacroScope(x_119, x_129, x_118); +x_131 = lean_box(0); +x_132 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__33; +x_133 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__35; +lean_inc(x_116); +x_134 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_134, 0, x_116); +lean_ctor_set(x_134, 1, x_132); +lean_ctor_set(x_134, 2, x_130); +lean_ctor_set(x_134, 3, x_133); +x_135 = lean_array_push(x_122, x_11); +x_136 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__10; +x_137 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_137, 0, x_124); +lean_ctor_set(x_137, 1, x_136); +lean_ctor_set(x_137, 2, x_135); +x_138 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; +x_139 = lean_array_push(x_138, x_134); +x_140 = lean_array_push(x_139, x_137); +x_141 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__30; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_124); lean_ctor_set(x_142, 1, x_141); -x_143 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +lean_ctor_set(x_142, 2, x_140); +x_143 = lean_array_push(x_138, x_128); +x_144 = lean_array_push(x_143, x_142); +x_145 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; +x_146 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_146, 0, x_124); +lean_ctor_set(x_146, 1, x_145); +lean_ctor_set(x_146, 2, x_144); +x_147 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__37; +lean_inc(x_116); +x_148 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_148, 0, x_116); +lean_ctor_set(x_148, 1, x_147); +x_149 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38; lean_inc(x_9); -x_144 = lean_array_push(x_143, x_9); -x_145 = lean_array_push(x_144, x_140); -x_146 = lean_array_push(x_145, x_142); -x_147 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_147, 0, x_129); -lean_ctor_set(x_147, 1, x_130); -lean_ctor_set(x_147, 2, x_146); -x_148 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; -x_149 = l_Lean_addMacroScope(x_116, x_148, x_115); -x_150 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__34; -x_151 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38; -x_152 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_152, 0, x_113); -lean_ctor_set(x_152, 1, x_150); -lean_ctor_set(x_152, 2, x_149); -lean_ctor_set(x_152, 3, x_151); -x_153 = l_Lean_Syntax_getId(x_9); +x_150 = lean_array_push(x_149, x_9); +x_151 = lean_array_push(x_150, x_146); +x_152 = lean_array_push(x_151, x_148); +x_153 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_153, 0, x_124); +lean_ctor_set(x_153, 1, x_136); +lean_ctor_set(x_153, 2, x_152); +x_154 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49; +x_155 = l_Lean_addMacroScope(x_119, x_154, x_118); +x_156 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47; +x_157 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51; +x_158 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_158, 0, x_116); +lean_ctor_set(x_158, 1, x_156); +lean_ctor_set(x_158, 2, x_155); +lean_ctor_set(x_158, 3, x_157); +x_159 = l_Lean_Syntax_getId(x_9); lean_dec(x_9); -lean_inc(x_153); -x_154 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_123, x_153); -x_155 = lean_array_push(x_132, x_152); -x_156 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; -x_157 = lean_array_push(x_156, x_118); -x_158 = lean_array_push(x_157, x_147); -if (lean_obj_tag(x_154) == 0) -{ -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; 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; -x_159 = l_Lean_quoteNameMk(x_153); -x_160 = lean_array_push(x_132, x_159); -x_161 = lean_array_push(x_160, x_13); -x_162 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_162, 0, x_129); -lean_ctor_set(x_162, 1, x_130); -lean_ctor_set(x_162, 2, x_161); -x_163 = lean_array_push(x_155, x_162); -x_164 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_164, 0, x_129); -lean_ctor_set(x_164, 1, x_135); -lean_ctor_set(x_164, 2, x_163); -x_165 = lean_array_push(x_127, x_164); -x_166 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; -x_167 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_167, 0, x_129); -lean_ctor_set(x_167, 1, x_166); -lean_ctor_set(x_167, 2, x_165); -x_168 = lean_array_push(x_132, x_167); -x_169 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; -x_170 = lean_array_push(x_168, x_169); -x_171 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; -x_172 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_172, 0, x_129); -lean_ctor_set(x_172, 1, x_171); -lean_ctor_set(x_172, 2, x_170); -x_173 = lean_array_push(x_127, x_172); -x_174 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_174, 0, x_129); -lean_ctor_set(x_174, 1, x_130); -lean_ctor_set(x_174, 2, x_173); -x_175 = lean_array_push(x_127, x_174); -x_176 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; -x_177 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_177, 0, x_129); -lean_ctor_set(x_177, 1, x_176); -lean_ctor_set(x_177, 2, x_175); -x_178 = lean_array_push(x_158, x_177); -x_179 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +lean_inc(x_159); +x_160 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_131, x_159); +x_161 = lean_array_push(x_138, x_158); +x_162 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53; +x_163 = lean_array_push(x_162, x_126); +x_164 = lean_array_push(x_163, x_153); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +x_165 = l_Lean_quoteNameMk(x_159); +x_166 = lean_array_push(x_138, x_165); +x_167 = lean_array_push(x_166, x_13); +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_124); +lean_ctor_set(x_168, 1, x_136); +lean_ctor_set(x_168, 2, x_167); +x_169 = lean_array_push(x_161, x_168); +x_170 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_170, 0, x_124); +lean_ctor_set(x_170, 1, x_141); +lean_ctor_set(x_170, 2, x_169); +x_171 = lean_array_push(x_122, x_170); +x_172 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; +x_173 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_173, 0, x_124); +lean_ctor_set(x_173, 1, x_172); +lean_ctor_set(x_173, 2, x_171); +x_174 = lean_array_push(x_138, x_173); +x_175 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_176 = lean_array_push(x_174, x_175); +x_177 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; +x_178 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_178, 0, x_124); +lean_ctor_set(x_178, 1, x_177); +lean_ctor_set(x_178, 2, x_176); +x_179 = lean_array_push(x_122, x_178); x_180 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_180, 0, x_129); -lean_ctor_set(x_180, 1, x_179); -lean_ctor_set(x_180, 2, x_178); -x_181 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_181, 0, x_180); -lean_ctor_set(x_181, 1, x_114); -return x_181; +lean_ctor_set(x_180, 0, x_124); +lean_ctor_set(x_180, 1, x_136); +lean_ctor_set(x_180, 2, x_179); +x_181 = lean_array_push(x_122, x_180); +x_182 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; +x_183 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_183, 0, x_124); +lean_ctor_set(x_183, 1, x_182); +lean_ctor_set(x_183, 2, x_181); +x_184 = lean_array_push(x_164, x_183); +x_185 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +x_186 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_186, 0, x_124); +lean_ctor_set(x_186, 1, x_185); +lean_ctor_set(x_186, 2, x_184); +x_187 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_187, 0, x_186); +lean_ctor_set(x_187, 1, x_117); +return x_187; } else { -lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; -lean_dec(x_153); -x_182 = lean_ctor_get(x_154, 0); -lean_inc(x_182); -lean_dec(x_154); -x_183 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__43; -x_184 = l_String_intercalate(x_183, x_182); -x_185 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; -x_186 = lean_string_append(x_185, x_184); -lean_dec(x_184); -x_187 = l_Lean_Syntax_mkNameLit(x_186, x_129); -x_188 = lean_array_push(x_127, x_187); -x_189 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; -x_190 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_190, 0, x_129); -lean_ctor_set(x_190, 1, x_189); -lean_ctor_set(x_190, 2, x_188); -x_191 = lean_array_push(x_132, x_190); -x_192 = lean_array_push(x_191, x_13); -x_193 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_193, 0, x_129); -lean_ctor_set(x_193, 1, x_130); -lean_ctor_set(x_193, 2, x_192); -x_194 = lean_array_push(x_155, x_193); -x_195 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_195, 0, x_129); -lean_ctor_set(x_195, 1, x_135); -lean_ctor_set(x_195, 2, x_194); -x_196 = lean_array_push(x_127, x_195); -x_197 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; -x_198 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_198, 0, x_129); -lean_ctor_set(x_198, 1, x_197); -lean_ctor_set(x_198, 2, x_196); -x_199 = lean_array_push(x_132, x_198); -x_200 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; -x_201 = lean_array_push(x_199, x_200); -x_202 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; -x_203 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_203, 0, x_129); -lean_ctor_set(x_203, 1, x_202); -lean_ctor_set(x_203, 2, x_201); -x_204 = lean_array_push(x_127, x_203); -x_205 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_205, 0, x_129); -lean_ctor_set(x_205, 1, x_130); -lean_ctor_set(x_205, 2, x_204); -x_206 = lean_array_push(x_127, x_205); -x_207 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; -x_208 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_208, 0, x_129); -lean_ctor_set(x_208, 1, x_207); -lean_ctor_set(x_208, 2, x_206); -x_209 = lean_array_push(x_158, x_208); -x_210 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; +lean_dec(x_159); +x_188 = lean_ctor_get(x_160, 0); +lean_inc(x_188); +lean_dec(x_160); +x_189 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56; +x_190 = l_String_intercalate(x_189, x_188); +x_191 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57; +x_192 = lean_string_append(x_191, x_190); +lean_dec(x_190); +x_193 = l_Lean_Syntax_mkNameLit(x_192, x_124); +x_194 = lean_array_push(x_122, x_193); +x_195 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55; +x_196 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_196, 0, x_124); +lean_ctor_set(x_196, 1, x_195); +lean_ctor_set(x_196, 2, x_194); +x_197 = lean_array_push(x_138, x_196); +x_198 = lean_array_push(x_197, x_13); +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_124); +lean_ctor_set(x_199, 1, x_136); +lean_ctor_set(x_199, 2, x_198); +x_200 = lean_array_push(x_161, x_199); +x_201 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_201, 0, x_124); +lean_ctor_set(x_201, 1, x_141); +lean_ctor_set(x_201, 2, x_200); +x_202 = lean_array_push(x_122, x_201); +x_203 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; +x_204 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_204, 0, x_124); +lean_ctor_set(x_204, 1, x_203); +lean_ctor_set(x_204, 2, x_202); +x_205 = lean_array_push(x_138, x_204); +x_206 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_207 = lean_array_push(x_205, x_206); +x_208 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; +x_209 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_209, 0, x_124); +lean_ctor_set(x_209, 1, x_208); +lean_ctor_set(x_209, 2, x_207); +x_210 = lean_array_push(x_122, x_209); x_211 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_211, 0, x_129); -lean_ctor_set(x_211, 1, x_210); -lean_ctor_set(x_211, 2, x_209); -x_212 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_212, 0, x_211); -lean_ctor_set(x_212, 1, x_114); -return x_212; +lean_ctor_set(x_211, 0, x_124); +lean_ctor_set(x_211, 1, x_136); +lean_ctor_set(x_211, 2, x_210); +x_212 = lean_array_push(x_122, x_211); +x_213 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; +x_214 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_214, 0, x_124); +lean_ctor_set(x_214, 1, x_213); +lean_ctor_set(x_214, 2, x_212); +x_215 = lean_array_push(x_164, x_214); +x_216 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +x_217 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_217, 0, x_124); +lean_ctor_set(x_217, 1, x_216); +lean_ctor_set(x_217, 2, x_215); +x_218 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_218, 0, x_217); +lean_ctor_set(x_218, 1, x_117); +return x_218; } } } @@ -3321,24 +3471,6 @@ x_1 = l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__10; return x_1; } } -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("initialize", 10); -return x_1; -} -} -static lean_object* _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__4; -x_2 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} LEAN_EXPORT lean_object* l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -3372,410 +3504,422 @@ x_14 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRul x_15 = !lean_is_exclusive(x_14); if (x_15 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; 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_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; x_16 = lean_ctor_get(x_14, 0); x_17 = lean_ctor_get(x_2, 2); lean_inc(x_17); x_18 = lean_ctor_get(x_2, 1); lean_inc(x_18); lean_dec(x_2); -x_19 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__1; +x_19 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__5; lean_inc(x_16); x_20 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_20, 0, x_16); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__14; +x_21 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23; +x_22 = lean_array_push(x_21, x_20); +x_23 = lean_box(2); +x_24 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__21; +x_25 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +lean_ctor_set(x_25, 2, x_22); +x_26 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__28; lean_inc(x_16); -x_22 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_22, 0, x_16); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; +x_27 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_27, 0, x_16); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; lean_inc(x_17); lean_inc(x_18); -x_24 = l_Lean_addMacroScope(x_18, x_23, x_17); -x_25 = lean_box(0); -x_26 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__19; -x_27 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__21; +x_29 = l_Lean_addMacroScope(x_18, x_28, x_17); +x_30 = lean_box(0); +x_31 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__33; +x_32 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__35; lean_inc(x_16); -x_28 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_28, 0, x_16); -lean_ctor_set(x_28, 1, x_26); -lean_ctor_set(x_28, 2, x_24); -lean_ctor_set(x_28, 3, x_27); -x_29 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22; -x_30 = lean_array_push(x_29, x_11); -x_31 = lean_box(2); -x_32 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__8; -x_33 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -lean_ctor_set(x_33, 2, x_30); -x_34 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23; -x_35 = lean_array_push(x_34, x_28); -x_36 = lean_array_push(x_35, x_33); -x_37 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__16; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_31); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_36); -x_39 = lean_array_push(x_34, x_22); -x_40 = lean_array_push(x_39, x_38); -x_41 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__13; -x_42 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_42, 0, x_31); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_40); -x_43 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__24; +x_33 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_33, 0, x_16); +lean_ctor_set(x_33, 1, x_31); +lean_ctor_set(x_33, 2, x_29); +lean_ctor_set(x_33, 3, x_32); +x_34 = lean_array_push(x_21, x_11); +x_35 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__10; +x_36 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_36, 0, x_23); +lean_ctor_set(x_36, 1, x_35); +lean_ctor_set(x_36, 2, x_34); +x_37 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; +x_38 = lean_array_push(x_37, x_33); +x_39 = lean_array_push(x_38, x_36); +x_40 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__30; +x_41 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_41, 0, x_23); +lean_ctor_set(x_41, 1, x_40); +lean_ctor_set(x_41, 2, x_39); +x_42 = lean_array_push(x_37, x_27); +x_43 = lean_array_push(x_42, x_41); +x_44 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; +x_45 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_45, 0, x_23); +lean_ctor_set(x_45, 1, x_44); +lean_ctor_set(x_45, 2, x_43); +x_46 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__37; lean_inc(x_16); -x_44 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_44, 0, x_16); -lean_ctor_set(x_44, 1, x_43); -x_45 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +x_47 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_47, 0, x_16); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38; lean_inc(x_9); -x_46 = lean_array_push(x_45, x_9); -x_47 = lean_array_push(x_46, x_42); -x_48 = lean_array_push(x_47, x_44); -x_49 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_49, 0, x_31); -lean_ctor_set(x_49, 1, x_32); -lean_ctor_set(x_49, 2, x_48); -x_50 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; -x_51 = l_Lean_addMacroScope(x_18, x_50, x_17); -x_52 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__34; -x_53 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38; -x_54 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_54, 0, x_16); -lean_ctor_set(x_54, 1, x_52); -lean_ctor_set(x_54, 2, x_51); -lean_ctor_set(x_54, 3, x_53); -x_55 = l_Lean_Syntax_getId(x_9); +x_49 = lean_array_push(x_48, x_9); +x_50 = lean_array_push(x_49, x_45); +x_51 = lean_array_push(x_50, x_47); +x_52 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_52, 0, x_23); +lean_ctor_set(x_52, 1, x_35); +lean_ctor_set(x_52, 2, x_51); +x_53 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49; +x_54 = l_Lean_addMacroScope(x_18, x_53, x_17); +x_55 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47; +x_56 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51; +x_57 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_57, 0, x_16); +lean_ctor_set(x_57, 1, x_55); +lean_ctor_set(x_57, 2, x_54); +lean_ctor_set(x_57, 3, x_56); +x_58 = l_Lean_Syntax_getId(x_9); lean_dec(x_9); -lean_inc(x_55); -x_56 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_25, x_55); -x_57 = lean_array_push(x_34, x_54); -x_58 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; -x_59 = lean_array_push(x_58, x_20); -x_60 = lean_array_push(x_59, x_49); -if (lean_obj_tag(x_56) == 0) -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; 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_61 = l_Lean_quoteNameMk(x_55); -x_62 = lean_array_push(x_34, x_61); -x_63 = lean_array_push(x_62, x_13); -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_31); -lean_ctor_set(x_64, 1, x_32); -lean_ctor_set(x_64, 2, x_63); -x_65 = lean_array_push(x_57, x_64); -x_66 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_66, 0, x_31); -lean_ctor_set(x_66, 1, x_37); -lean_ctor_set(x_66, 2, x_65); -x_67 = lean_array_push(x_29, x_66); -x_68 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; +lean_inc(x_58); +x_59 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_30, x_58); +x_60 = lean_array_push(x_37, x_57); +x_61 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53; +x_62 = lean_array_push(x_61, x_25); +x_63 = lean_array_push(x_62, x_52); +if (lean_obj_tag(x_59) == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; 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; +x_64 = l_Lean_quoteNameMk(x_58); +x_65 = lean_array_push(x_37, x_64); +x_66 = lean_array_push(x_65, x_13); +x_67 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_67, 0, x_23); +lean_ctor_set(x_67, 1, x_35); +lean_ctor_set(x_67, 2, x_66); +x_68 = lean_array_push(x_60, x_67); x_69 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_69, 0, x_31); -lean_ctor_set(x_69, 1, x_68); -lean_ctor_set(x_69, 2, x_67); -x_70 = lean_array_push(x_34, x_69); -x_71 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; -x_72 = lean_array_push(x_70, x_71); -x_73 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; -x_74 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_74, 0, x_31); -lean_ctor_set(x_74, 1, x_73); -lean_ctor_set(x_74, 2, x_72); -x_75 = lean_array_push(x_29, x_74); -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_31); -lean_ctor_set(x_76, 1, x_32); -lean_ctor_set(x_76, 2, x_75); -x_77 = lean_array_push(x_29, x_76); -x_78 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; +lean_ctor_set(x_69, 0, x_23); +lean_ctor_set(x_69, 1, x_40); +lean_ctor_set(x_69, 2, x_68); +x_70 = lean_array_push(x_21, x_69); +x_71 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; +x_72 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_72, 0, x_23); +lean_ctor_set(x_72, 1, x_71); +lean_ctor_set(x_72, 2, x_70); +x_73 = lean_array_push(x_37, x_72); +x_74 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_75 = lean_array_push(x_73, x_74); +x_76 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; +x_77 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_77, 0, x_23); +lean_ctor_set(x_77, 1, x_76); +lean_ctor_set(x_77, 2, x_75); +x_78 = lean_array_push(x_21, x_77); x_79 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_79, 0, x_31); -lean_ctor_set(x_79, 1, x_78); -lean_ctor_set(x_79, 2, x_77); -x_80 = lean_array_push(x_60, x_79); -x_81 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2; +lean_ctor_set(x_79, 0, x_23); +lean_ctor_set(x_79, 1, x_35); +lean_ctor_set(x_79, 2, x_78); +x_80 = lean_array_push(x_21, x_79); +x_81 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; x_82 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_82, 0, x_31); +lean_ctor_set(x_82, 0, x_23); lean_ctor_set(x_82, 1, x_81); lean_ctor_set(x_82, 2, x_80); -lean_ctor_set(x_14, 0, x_82); +x_83 = lean_array_push(x_63, x_82); +x_84 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +x_85 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_85, 0, x_23); +lean_ctor_set(x_85, 1, x_84); +lean_ctor_set(x_85, 2, x_83); +lean_ctor_set(x_14, 0, x_85); return x_14; } else { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; 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_dec(x_55); -x_83 = lean_ctor_get(x_56, 0); -lean_inc(x_83); -lean_dec(x_56); -x_84 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__43; -x_85 = l_String_intercalate(x_84, x_83); -x_86 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; -x_87 = lean_string_append(x_86, x_85); -lean_dec(x_85); -x_88 = l_Lean_Syntax_mkNameLit(x_87, x_31); -x_89 = lean_array_push(x_29, x_88); -x_90 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; -x_91 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_91, 0, x_31); -lean_ctor_set(x_91, 1, x_90); -lean_ctor_set(x_91, 2, x_89); -x_92 = lean_array_push(x_34, x_91); -x_93 = lean_array_push(x_92, x_13); +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +lean_dec(x_58); +x_86 = lean_ctor_get(x_59, 0); +lean_inc(x_86); +lean_dec(x_59); +x_87 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56; +x_88 = l_String_intercalate(x_87, x_86); +x_89 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57; +x_90 = lean_string_append(x_89, x_88); +lean_dec(x_88); +x_91 = l_Lean_Syntax_mkNameLit(x_90, x_23); +x_92 = lean_array_push(x_21, x_91); +x_93 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55; x_94 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_94, 0, x_31); -lean_ctor_set(x_94, 1, x_32); -lean_ctor_set(x_94, 2, x_93); -x_95 = lean_array_push(x_57, x_94); -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_31); -lean_ctor_set(x_96, 1, x_37); -lean_ctor_set(x_96, 2, x_95); -x_97 = lean_array_push(x_29, x_96); -x_98 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; +lean_ctor_set(x_94, 0, x_23); +lean_ctor_set(x_94, 1, x_93); +lean_ctor_set(x_94, 2, x_92); +x_95 = lean_array_push(x_37, x_94); +x_96 = lean_array_push(x_95, x_13); +x_97 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_97, 0, x_23); +lean_ctor_set(x_97, 1, x_35); +lean_ctor_set(x_97, 2, x_96); +x_98 = lean_array_push(x_60, x_97); x_99 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_99, 0, x_31); -lean_ctor_set(x_99, 1, x_98); -lean_ctor_set(x_99, 2, x_97); -x_100 = lean_array_push(x_34, x_99); -x_101 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; -x_102 = lean_array_push(x_100, x_101); -x_103 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; -x_104 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_104, 0, x_31); -lean_ctor_set(x_104, 1, x_103); -lean_ctor_set(x_104, 2, x_102); -x_105 = lean_array_push(x_29, x_104); -x_106 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_106, 0, x_31); -lean_ctor_set(x_106, 1, x_32); -lean_ctor_set(x_106, 2, x_105); -x_107 = lean_array_push(x_29, x_106); -x_108 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; +lean_ctor_set(x_99, 0, x_23); +lean_ctor_set(x_99, 1, x_40); +lean_ctor_set(x_99, 2, x_98); +x_100 = lean_array_push(x_21, x_99); +x_101 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; +x_102 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_102, 0, x_23); +lean_ctor_set(x_102, 1, x_101); +lean_ctor_set(x_102, 2, x_100); +x_103 = lean_array_push(x_37, x_102); +x_104 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_105 = lean_array_push(x_103, x_104); +x_106 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; +x_107 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_107, 0, x_23); +lean_ctor_set(x_107, 1, x_106); +lean_ctor_set(x_107, 2, x_105); +x_108 = lean_array_push(x_21, x_107); x_109 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_109, 0, x_31); -lean_ctor_set(x_109, 1, x_108); -lean_ctor_set(x_109, 2, x_107); -x_110 = lean_array_push(x_60, x_109); -x_111 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2; +lean_ctor_set(x_109, 0, x_23); +lean_ctor_set(x_109, 1, x_35); +lean_ctor_set(x_109, 2, x_108); +x_110 = lean_array_push(x_21, x_109); +x_111 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; x_112 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_112, 0, x_31); +lean_ctor_set(x_112, 0, x_23); lean_ctor_set(x_112, 1, x_111); lean_ctor_set(x_112, 2, x_110); -lean_ctor_set(x_14, 0, x_112); +x_113 = lean_array_push(x_63, x_112); +x_114 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +x_115 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_115, 0, x_23); +lean_ctor_set(x_115, 1, x_114); +lean_ctor_set(x_115, 2, x_113); +lean_ctor_set(x_14, 0, x_115); return x_14; } } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; 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_113 = lean_ctor_get(x_14, 0); -x_114 = lean_ctor_get(x_14, 1); -lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_14); -x_115 = lean_ctor_get(x_2, 2); -lean_inc(x_115); -x_116 = lean_ctor_get(x_2, 1); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; 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; +x_116 = lean_ctor_get(x_14, 0); +x_117 = lean_ctor_get(x_14, 1); +lean_inc(x_117); lean_inc(x_116); +lean_dec(x_14); +x_118 = lean_ctor_get(x_2, 2); +lean_inc(x_118); +x_119 = lean_ctor_get(x_2, 1); +lean_inc(x_119); lean_dec(x_2); -x_117 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__1; -lean_inc(x_113); -x_118 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_118, 0, x_113); -lean_ctor_set(x_118, 1, x_117); -x_119 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__14; -lean_inc(x_113); -x_120 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_120, 0, x_113); -lean_ctor_set(x_120, 1, x_119); -x_121 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; -lean_inc(x_115); +x_120 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__5; lean_inc(x_116); -x_122 = l_Lean_addMacroScope(x_116, x_121, x_115); -x_123 = lean_box(0); -x_124 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__19; +x_121 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_121, 0, x_116); +lean_ctor_set(x_121, 1, x_120); +x_122 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23; +x_123 = lean_array_push(x_122, x_121); +x_124 = lean_box(2); x_125 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__21; -lean_inc(x_113); -x_126 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_126, 0, x_113); -lean_ctor_set(x_126, 1, x_124); -lean_ctor_set(x_126, 2, x_122); -lean_ctor_set(x_126, 3, x_125); -x_127 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__22; -x_128 = lean_array_push(x_127, x_11); -x_129 = lean_box(2); -x_130 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__8; -x_131 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_131, 0, x_129); -lean_ctor_set(x_131, 1, x_130); -lean_ctor_set(x_131, 2, x_128); -x_132 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__23; -x_133 = lean_array_push(x_132, x_126); -x_134 = lean_array_push(x_133, x_131); -x_135 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__16; -x_136 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_136, 0, x_129); -lean_ctor_set(x_136, 1, x_135); -lean_ctor_set(x_136, 2, x_134); -x_137 = lean_array_push(x_132, x_120); -x_138 = lean_array_push(x_137, x_136); -x_139 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__13; -x_140 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_140, 0, x_129); -lean_ctor_set(x_140, 1, x_139); -lean_ctor_set(x_140, 2, x_138); -x_141 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__24; -lean_inc(x_113); -x_142 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_142, 0, x_113); +x_126 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +lean_ctor_set(x_126, 2, x_123); +x_127 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__28; +lean_inc(x_116); +x_128 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_128, 0, x_116); +lean_ctor_set(x_128, 1, x_127); +x_129 = l_Lean_Option_commandRegister__builtin__option___x3a___x3a_x3d_____closed__4; +lean_inc(x_118); +lean_inc(x_119); +x_130 = l_Lean_addMacroScope(x_119, x_129, x_118); +x_131 = lean_box(0); +x_132 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__33; +x_133 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__35; +lean_inc(x_116); +x_134 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_134, 0, x_116); +lean_ctor_set(x_134, 1, x_132); +lean_ctor_set(x_134, 2, x_130); +lean_ctor_set(x_134, 3, x_133); +x_135 = lean_array_push(x_122, x_11); +x_136 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__10; +x_137 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_137, 0, x_124); +lean_ctor_set(x_137, 1, x_136); +lean_ctor_set(x_137, 2, x_135); +x_138 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; +x_139 = lean_array_push(x_138, x_134); +x_140 = lean_array_push(x_139, x_137); +x_141 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__30; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_124); lean_ctor_set(x_142, 1, x_141); -x_143 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__25; +lean_ctor_set(x_142, 2, x_140); +x_143 = lean_array_push(x_138, x_128); +x_144 = lean_array_push(x_143, x_142); +x_145 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; +x_146 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_146, 0, x_124); +lean_ctor_set(x_146, 1, x_145); +lean_ctor_set(x_146, 2, x_144); +x_147 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__37; +lean_inc(x_116); +x_148 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_148, 0, x_116); +lean_ctor_set(x_148, 1, x_147); +x_149 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38; lean_inc(x_9); -x_144 = lean_array_push(x_143, x_9); -x_145 = lean_array_push(x_144, x_140); -x_146 = lean_array_push(x_145, x_142); -x_147 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_147, 0, x_129); -lean_ctor_set(x_147, 1, x_130); -lean_ctor_set(x_147, 2, x_146); -x_148 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__36; -x_149 = l_Lean_addMacroScope(x_116, x_148, x_115); -x_150 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__34; -x_151 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__38; -x_152 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_152, 0, x_113); -lean_ctor_set(x_152, 1, x_150); -lean_ctor_set(x_152, 2, x_149); -lean_ctor_set(x_152, 3, x_151); -x_153 = l_Lean_Syntax_getId(x_9); +x_150 = lean_array_push(x_149, x_9); +x_151 = lean_array_push(x_150, x_146); +x_152 = lean_array_push(x_151, x_148); +x_153 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_153, 0, x_124); +lean_ctor_set(x_153, 1, x_136); +lean_ctor_set(x_153, 2, x_152); +x_154 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49; +x_155 = l_Lean_addMacroScope(x_119, x_154, x_118); +x_156 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47; +x_157 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51; +x_158 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_158, 0, x_116); +lean_ctor_set(x_158, 1, x_156); +lean_ctor_set(x_158, 2, x_155); +lean_ctor_set(x_158, 3, x_157); +x_159 = l_Lean_Syntax_getId(x_9); lean_dec(x_9); -lean_inc(x_153); -x_154 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_123, x_153); -x_155 = lean_array_push(x_132, x_152); -x_156 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; -x_157 = lean_array_push(x_156, x_118); -x_158 = lean_array_push(x_157, x_147); -if (lean_obj_tag(x_154) == 0) -{ -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; 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; -x_159 = l_Lean_quoteNameMk(x_153); -x_160 = lean_array_push(x_132, x_159); -x_161 = lean_array_push(x_160, x_13); -x_162 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_162, 0, x_129); -lean_ctor_set(x_162, 1, x_130); -lean_ctor_set(x_162, 2, x_161); -x_163 = lean_array_push(x_155, x_162); -x_164 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_164, 0, x_129); -lean_ctor_set(x_164, 1, x_135); -lean_ctor_set(x_164, 2, x_163); -x_165 = lean_array_push(x_127, x_164); -x_166 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; -x_167 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_167, 0, x_129); -lean_ctor_set(x_167, 1, x_166); -lean_ctor_set(x_167, 2, x_165); -x_168 = lean_array_push(x_132, x_167); -x_169 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; -x_170 = lean_array_push(x_168, x_169); -x_171 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; -x_172 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_172, 0, x_129); -lean_ctor_set(x_172, 1, x_171); -lean_ctor_set(x_172, 2, x_170); -x_173 = lean_array_push(x_127, x_172); -x_174 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_174, 0, x_129); -lean_ctor_set(x_174, 1, x_130); -lean_ctor_set(x_174, 2, x_173); -x_175 = lean_array_push(x_127, x_174); -x_176 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; -x_177 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_177, 0, x_129); -lean_ctor_set(x_177, 1, x_176); -lean_ctor_set(x_177, 2, x_175); -x_178 = lean_array_push(x_158, x_177); -x_179 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2; +lean_inc(x_159); +x_160 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_131, x_159); +x_161 = lean_array_push(x_138, x_158); +x_162 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53; +x_163 = lean_array_push(x_162, x_126); +x_164 = lean_array_push(x_163, x_153); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +x_165 = l_Lean_quoteNameMk(x_159); +x_166 = lean_array_push(x_138, x_165); +x_167 = lean_array_push(x_166, x_13); +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_124); +lean_ctor_set(x_168, 1, x_136); +lean_ctor_set(x_168, 2, x_167); +x_169 = lean_array_push(x_161, x_168); +x_170 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_170, 0, x_124); +lean_ctor_set(x_170, 1, x_141); +lean_ctor_set(x_170, 2, x_169); +x_171 = lean_array_push(x_122, x_170); +x_172 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; +x_173 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_173, 0, x_124); +lean_ctor_set(x_173, 1, x_172); +lean_ctor_set(x_173, 2, x_171); +x_174 = lean_array_push(x_138, x_173); +x_175 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_176 = lean_array_push(x_174, x_175); +x_177 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; +x_178 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_178, 0, x_124); +lean_ctor_set(x_178, 1, x_177); +lean_ctor_set(x_178, 2, x_176); +x_179 = lean_array_push(x_122, x_178); x_180 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_180, 0, x_129); -lean_ctor_set(x_180, 1, x_179); -lean_ctor_set(x_180, 2, x_178); -x_181 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_181, 0, x_180); -lean_ctor_set(x_181, 1, x_114); -return x_181; +lean_ctor_set(x_180, 0, x_124); +lean_ctor_set(x_180, 1, x_136); +lean_ctor_set(x_180, 2, x_179); +x_181 = lean_array_push(x_122, x_180); +x_182 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; +x_183 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_183, 0, x_124); +lean_ctor_set(x_183, 1, x_182); +lean_ctor_set(x_183, 2, x_181); +x_184 = lean_array_push(x_164, x_183); +x_185 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +x_186 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_186, 0, x_124); +lean_ctor_set(x_186, 1, x_185); +lean_ctor_set(x_186, 2, x_184); +x_187 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_187, 0, x_186); +lean_ctor_set(x_187, 1, x_117); +return x_187; } else { -lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; -lean_dec(x_153); -x_182 = lean_ctor_get(x_154, 0); -lean_inc(x_182); -lean_dec(x_154); -x_183 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__43; -x_184 = l_String_intercalate(x_183, x_182); -x_185 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; -x_186 = lean_string_append(x_185, x_184); -lean_dec(x_184); -x_187 = l_Lean_Syntax_mkNameLit(x_186, x_129); -x_188 = lean_array_push(x_127, x_187); -x_189 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; -x_190 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_190, 0, x_129); -lean_ctor_set(x_190, 1, x_189); -lean_ctor_set(x_190, 2, x_188); -x_191 = lean_array_push(x_132, x_190); -x_192 = lean_array_push(x_191, x_13); -x_193 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_193, 0, x_129); -lean_ctor_set(x_193, 1, x_130); -lean_ctor_set(x_193, 2, x_192); -x_194 = lean_array_push(x_155, x_193); -x_195 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_195, 0, x_129); -lean_ctor_set(x_195, 1, x_135); -lean_ctor_set(x_195, 2, x_194); -x_196 = lean_array_push(x_127, x_195); -x_197 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__31; -x_198 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_198, 0, x_129); -lean_ctor_set(x_198, 1, x_197); -lean_ctor_set(x_198, 2, x_196); -x_199 = lean_array_push(x_132, x_198); -x_200 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__9; -x_201 = lean_array_push(x_199, x_200); -x_202 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__29; -x_203 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_203, 0, x_129); -lean_ctor_set(x_203, 1, x_202); -lean_ctor_set(x_203, 2, x_201); -x_204 = lean_array_push(x_127, x_203); -x_205 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_205, 0, x_129); -lean_ctor_set(x_205, 1, x_130); -lean_ctor_set(x_205, 2, x_204); -x_206 = lean_array_push(x_127, x_205); -x_207 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__27; -x_208 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_208, 0, x_129); -lean_ctor_set(x_208, 1, x_207); -lean_ctor_set(x_208, 2, x_206); -x_209 = lean_array_push(x_158, x_208); -x_210 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2; +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; +lean_dec(x_159); +x_188 = lean_ctor_get(x_160, 0); +lean_inc(x_188); +lean_dec(x_160); +x_189 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56; +x_190 = l_String_intercalate(x_189, x_188); +x_191 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57; +x_192 = lean_string_append(x_191, x_190); +lean_dec(x_190); +x_193 = l_Lean_Syntax_mkNameLit(x_192, x_124); +x_194 = lean_array_push(x_122, x_193); +x_195 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55; +x_196 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_196, 0, x_124); +lean_ctor_set(x_196, 1, x_195); +lean_ctor_set(x_196, 2, x_194); +x_197 = lean_array_push(x_138, x_196); +x_198 = lean_array_push(x_197, x_13); +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_124); +lean_ctor_set(x_199, 1, x_136); +lean_ctor_set(x_199, 2, x_198); +x_200 = lean_array_push(x_161, x_199); +x_201 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_201, 0, x_124); +lean_ctor_set(x_201, 1, x_141); +lean_ctor_set(x_201, 2, x_200); +x_202 = lean_array_push(x_122, x_201); +x_203 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44; +x_204 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_204, 0, x_124); +lean_ctor_set(x_204, 1, x_203); +lean_ctor_set(x_204, 2, x_202); +x_205 = lean_array_push(x_138, x_204); +x_206 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__11; +x_207 = lean_array_push(x_205, x_206); +x_208 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__42; +x_209 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_209, 0, x_124); +lean_ctor_set(x_209, 1, x_208); +lean_ctor_set(x_209, 2, x_207); +x_210 = lean_array_push(x_122, x_209); x_211 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_211, 0, x_129); -lean_ctor_set(x_211, 1, x_210); -lean_ctor_set(x_211, 2, x_209); -x_212 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_212, 0, x_211); -lean_ctor_set(x_212, 1, x_114); -return x_212; +lean_ctor_set(x_211, 0, x_124); +lean_ctor_set(x_211, 1, x_136); +lean_ctor_set(x_211, 2, x_210); +x_212 = lean_array_push(x_122, x_211); +x_213 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__40; +x_214 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_214, 0, x_124); +lean_ctor_set(x_214, 1, x_213); +lean_ctor_set(x_214, 2, x_212); +x_215 = lean_array_push(x_164, x_214); +x_216 = l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__6; +x_217 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_217, 0, x_124); +lean_ctor_set(x_217, 1, x_216); +lean_ctor_set(x_217, 2, x_215); +x_218 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_218, 0, x_217); +lean_ctor_set(x_218, 1, x_117); +return x_218; } } } @@ -4019,6 +4163,32 @@ l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandR lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__43); l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44(); lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__44); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__45 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__45(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__45); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__46 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__46(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__46); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__47); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__48 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__48(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__48); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__49); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__50 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__50(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__50); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__51); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__52 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__52(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__52); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__53); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__54 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__54(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__54); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__55); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__56); +l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57(); +lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__builtin__option___x3a___x3a_x3d____1___closed__57); l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__1 = _init_l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__1(); lean_mark_persistent(l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__1); l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__2 = _init_l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__2(); @@ -4041,10 +4211,6 @@ l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__10 = _init_l_L lean_mark_persistent(l_Lean_Option_commandRegister__option___x3a___x3a_x3d_____closed__10); l_Lean_Option_commandRegister__option___x3a___x3a_x3d__ = _init_l_Lean_Option_commandRegister__option___x3a___x3a_x3d__(); lean_mark_persistent(l_Lean_Option_commandRegister__option___x3a___x3a_x3d__); -l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__1 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__1(); -lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__1); -l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2 = _init_l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2(); -lean_mark_persistent(l_Lean_Option___aux__Lean__Data__Options______macroRules__Lean__Option__commandRegister__option___x3a___x3a_x3d____1___closed__2); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Data/Position.c b/stage0/stdlib/Lean/Data/Position.c index 08288e237e73..bb7bf686eacf 100644 --- a/stage0/stdlib/Lean/Data/Position.c +++ b/stage0/stdlib/Lean/Data/Position.c @@ -922,7 +922,7 @@ static lean_object* _init_l_Lean_FileMap_toPosition_loop___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_FileMap_toPosition_loop___closed__1; x_2 = l_Lean_FileMap_toPosition_loop___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_FileMap_toPosition_loop___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/DocString.c b/stage0/stdlib/Lean/DocString.c index 0f75e53b5a66..0c54e280a088 100644 --- a/stage0/stdlib/Lean/DocString.c +++ b/stage0/stdlib/Lean/DocString.c @@ -13,62 +13,83 @@ #ifdef __cplusplus extern "C" { #endif +lean_object* lean_string_push(lean_object*, uint32_t); +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_consumeSpaces___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addMainModuleDoc(lean_object*, lean_object*); static lean_object* l_Lean_addMainModuleDoc___closed__1; extern lean_object* l_String_instInhabitedString; lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_PersistentEnvExtension_getModuleEntries___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__1; LEAN_EXPORT lean_object* l_Lean_addDocString_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_docStringExt; +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_consumeSpaces(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__6; +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_findNextLine(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_addDocString___rarg(lean_object*, lean_object*, lean_object*); +uint8_t l_String_Iterator_atEnd(lean_object*); LEAN_EXPORT lean_object* l_Lean_addDocString___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__5; +lean_object* lean_nat_add(lean_object*, lean_object*); lean_object* l_Lean_registerSimplePersistentEnvExtension___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize(lean_object*); LEAN_EXPORT lean_object* l_Lean_addDocString(lean_object*); lean_object* l_Lean_MapDeclarationExtension_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__2; uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); lean_object* l_Lean_mkMapDeclarationExtension___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Std_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_1527____closed__4; lean_object* lean_st_mk_ref(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__1; +static lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces___closed__1; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_saveLine(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_consumeSpaces(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_String_Iterator_find___at___private_Lean_DocString_0__Lean_findLeadingSpacesSize___spec__1(lean_object*); +lean_object* l_String_Iterator_next(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_42____closed__2; LEAN_EXPORT lean_object* l_Lean_getMainModuleDoc(lean_object*); lean_object* l_Std_instInhabitedPersistentArray(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___boxed(lean_object*); lean_object* l_Lean_PersistentEnvExtension_addEntry___rarg(lean_object*, 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_1527____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_getMainModuleDoc___boxed(lean_object*); +uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeLeadingSpaces(lean_object*); static lean_object* l_Lean_addDocString___rarg___lambda__1___closed__1; static lean_object* l_Lean_getMainModuleDoc___closed__1; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_moduleDocExt; static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_42____closed__1; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1(lean_object*); lean_object* lean_list_to_array(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__4; -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__2; +uint32_t l_String_Iterator_curr(lean_object*); LEAN_EXPORT lean_object* l_Lean_findDocString_x3f(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getModuleDoc_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addDocString_x27(lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__2; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527_(lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_4_(lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_42_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197_(lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__6; +static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__3; LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_findDocString_x3f___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___boxed(lean_object*); +lean_object* l_Nat_min(lean_object*, lean_object*); lean_object* l_Lean_Environment_getModuleIdx_x3f(lean_object*, lean_object*); static lean_object* l_Lean_addBuiltinDocString___closed__1; -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__3; -static lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__5; LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_findDocString_x3f___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_builtinDocStrings; +LEAN_EXPORT lean_object* l_String_Iterator_foldUntil___at___private_Lean_DocString_0__Lean_findLeadingSpacesSize___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getModuleDoc_x3f___boxed(lean_object*, lean_object*); static lean_object* l_Lean_getModuleDoc_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_4_(lean_object* x_1) { @@ -125,6 +146,362 @@ x_4 = l_Lean_mkMapDeclarationExtension___rarg(x_2, x_3, x_1); return x_4; } } +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_consumeSpaces(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = l_String_Iterator_atEnd(x_1); +if (x_4 == 0) +{ +uint32_t x_5; uint32_t x_6; uint8_t x_7; +x_5 = l_String_Iterator_curr(x_1); +x_6 = 32; +x_7 = lean_uint32_dec_eq(x_5, x_6); +if (x_7 == 0) +{ +uint32_t x_8; uint8_t x_9; +x_8 = 9; +x_9 = lean_uint32_dec_eq(x_5, x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = l_String_Iterator_next(x_1); +x_11 = l_Nat_min(x_2, x_3); +lean_dec(x_2); +x_12 = l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_findNextLine(x_10, x_11); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = l_String_Iterator_next(x_1); +x_14 = lean_unsigned_to_nat(1u); +x_15 = lean_nat_add(x_2, x_14); +lean_dec(x_2); +x_1 = x_13; +x_2 = x_15; +goto _start; +} +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = l_String_Iterator_next(x_1); +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_add(x_2, x_18); +lean_dec(x_2); +x_1 = x_17; +x_2 = x_19; +goto _start; +} +} +else +{ +lean_dec(x_2); +lean_dec(x_1); +lean_inc(x_3); +return x_3; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_findNextLine(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; +x_3 = l_String_Iterator_atEnd(x_1); +if (x_3 == 0) +{ +uint32_t x_4; uint32_t x_5; uint8_t x_6; +x_4 = l_String_Iterator_curr(x_1); +x_5 = 10; +x_6 = lean_uint32_dec_eq(x_4, x_5); +if (x_6 == 0) +{ +lean_object* x_7; +x_7 = l_String_Iterator_next(x_1); +x_1 = x_7; +goto _start; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = l_String_Iterator_next(x_1); +x_10 = lean_unsigned_to_nat(0u); +x_11 = l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_consumeSpaces(x_9, x_10, x_2); +lean_dec(x_2); +return x_11; +} +} +else +{ +lean_dec(x_1); +return x_2; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_consumeSpaces___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_consumeSpaces(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_String_Iterator_find___at___private_Lean_DocString_0__Lean_findLeadingSpacesSize___spec__1(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = l_String_Iterator_atEnd(x_1); +if (x_2 == 0) +{ +uint32_t x_3; uint32_t x_4; uint8_t x_5; +x_3 = l_String_Iterator_curr(x_1); +x_4 = 10; +x_5 = lean_uint32_dec_eq(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; +x_6 = l_String_Iterator_next(x_1); +x_1 = x_6; +goto _start; +} +else +{ +return x_1; +} +} +else +{ +return x_1; +} +} +} +LEAN_EXPORT lean_object* l_String_Iterator_foldUntil___at___private_Lean_DocString_0__Lean_findLeadingSpacesSize___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; +x_3 = l_String_Iterator_atEnd(x_1); +if (x_3 == 0) +{ +uint32_t x_4; uint32_t x_5; uint8_t x_6; +x_4 = l_String_Iterator_curr(x_1); +x_5 = 32; +x_6 = lean_uint32_dec_eq(x_4, x_5); +if (x_6 == 0) +{ +uint32_t x_7; uint8_t x_8; +x_7 = 9; +x_8 = lean_uint32_dec_eq(x_4, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_2); +lean_ctor_set(x_9, 1, x_1); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_unsigned_to_nat(1u); +x_11 = lean_nat_add(x_2, x_10); +lean_dec(x_2); +x_12 = l_String_Iterator_next(x_1); +x_1 = x_12; +x_2 = x_11; +goto _start; +} +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_unsigned_to_nat(1u); +x_15 = lean_nat_add(x_2, x_14); +lean_dec(x_2); +x_16 = l_String_Iterator_next(x_1); +x_1 = x_16; +x_2 = x_15; +goto _start; +} +} +else +{ +lean_object* x_18; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_2); +lean_ctor_set(x_18, 1, x_1); +return x_18; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_findLeadingSpacesSize(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_2 = lean_unsigned_to_nat(0u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +x_4 = l_String_Iterator_find___at___private_Lean_DocString_0__Lean_findLeadingSpacesSize___spec__1(x_3); +x_5 = l_String_Iterator_next(x_4); +x_6 = l_String_Iterator_foldUntil___at___private_Lean_DocString_0__Lean_findLeadingSpacesSize___spec__2(x_5, x_2); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = l___private_Lean_DocString_0__Lean_findLeadingSpacesSize_findNextLine(x_8, x_7); +return x_9; +} +} +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_consumeSpaces(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_unsigned_to_nat(0u); +x_6 = lean_nat_dec_eq(x_2, x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_7 = lean_unsigned_to_nat(1u); +x_8 = lean_nat_sub(x_2, x_7); +lean_dec(x_2); +x_9 = l_String_Iterator_atEnd(x_3); +if (x_9 == 0) +{ +uint32_t x_10; uint32_t x_11; uint8_t x_12; +x_10 = l_String_Iterator_curr(x_3); +x_11 = 32; +x_12 = lean_uint32_dec_eq(x_10, x_11); +if (x_12 == 0) +{ +uint32_t x_13; uint8_t x_14; +x_13 = 9; +x_14 = lean_uint32_dec_eq(x_10, x_13); +if (x_14 == 0) +{ +lean_object* x_15; +lean_dec(x_8); +x_15 = l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_saveLine(x_1, x_3, x_4); +return x_15; +} +else +{ +lean_object* x_16; +x_16 = l_String_Iterator_next(x_3); +x_2 = x_8; +x_3 = x_16; +goto _start; +} +} +else +{ +lean_object* x_18; +x_18 = l_String_Iterator_next(x_3); +x_2 = x_8; +x_3 = x_18; +goto _start; +} +} +else +{ +lean_dec(x_8); +lean_dec(x_3); +lean_dec(x_1); +return x_4; +} +} +else +{ +lean_object* x_20; +lean_dec(x_2); +x_20 = l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_saveLine(x_1, x_3, x_4); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_saveLine(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = l_String_Iterator_atEnd(x_2); +if (x_4 == 0) +{ +uint32_t x_5; uint32_t x_6; uint8_t x_7; +x_5 = l_String_Iterator_curr(x_2); +x_6 = 10; +x_7 = lean_uint32_dec_eq(x_5, x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +x_8 = l_String_Iterator_next(x_2); +x_9 = lean_string_push(x_3, x_5); +x_2 = x_8; +x_3 = x_9; +goto _start; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = l_String_Iterator_next(x_2); +x_12 = lean_string_push(x_3, x_6); +lean_inc(x_1); +x_13 = l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_consumeSpaces(x_1, x_1, x_11, x_12); +return x_13; +} +} +else +{ +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +} +static lean_object* _init_l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("", 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_unsigned_to_nat(0u); +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces___closed__1; +lean_inc(x_1); +x_6 = l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces_consumeSpaces(x_1, x_1, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_DocString_0__Lean_removeLeadingSpaces(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; +lean_inc(x_1); +x_2 = l___private_Lean_DocString_0__Lean_findLeadingSpacesSize(x_1); +x_3 = lean_unsigned_to_nat(0u); +x_4 = lean_nat_dec_eq(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces(x_2, x_1); +return x_5; +} +else +{ +lean_dec(x_2); +return x_1; +} +} +} static lean_object* _init_l_Lean_addBuiltinDocString___closed__1() { _start: { @@ -136,7 +513,7 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_addBuiltinDocString(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; x_4 = l_Lean_addBuiltinDocString___closed__1; x_5 = lean_st_ref_take(x_4, x_3); x_6 = lean_ctor_get(x_5, 0); @@ -144,25 +521,26 @@ lean_inc(x_6); x_7 = lean_ctor_get(x_5, 1); lean_inc(x_7); lean_dec(x_5); -x_8 = l_Std_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_6, x_1, x_2); -x_9 = lean_st_ref_set(x_4, x_8, x_7); -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) +x_8 = l___private_Lean_DocString_0__Lean_removeLeadingSpaces(x_2); +x_9 = l_Std_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(x_6, x_1, x_8); +x_10 = lean_st_ref_set(x_4, x_9, x_7); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -return x_9; +return x_10; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_9, 1); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); lean_inc(x_12); -lean_inc(x_11); -lean_dec(x_9); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -return x_13; +lean_dec(x_10); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; } } } @@ -177,10 +555,11 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_addDocString___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; -x_4 = l_Lean_addDocString___rarg___lambda__1___closed__1; -x_5 = l_Lean_MapDeclarationExtension_insert___rarg(x_4, x_3, x_1, x_2); -return x_5; +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = l___private_Lean_DocString_0__Lean_removeLeadingSpaces(x_1); +x_5 = l_Lean_addDocString___rarg___lambda__1___closed__1; +x_6 = l_Lean_MapDeclarationExtension_insert___rarg(x_5, x_3, x_2, x_4); +return x_6; } } LEAN_EXPORT lean_object* l_Lean_addDocString___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { @@ -191,8 +570,8 @@ x_4 = lean_ctor_get(x_1, 1); lean_inc(x_4); lean_dec(x_1); x_5 = lean_alloc_closure((void*)(l_Lean_addDocString___rarg___lambda__1), 3, 2); -lean_closure_set(x_5, 0, x_2); -lean_closure_set(x_5, 1, x_3); +lean_closure_set(x_5, 0, x_3); +lean_closure_set(x_5, 1, x_2); x_6 = lean_apply_1(x_4, x_5); return x_6; } @@ -388,7 +767,7 @@ lean_dec(x_1); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -397,23 +776,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_197____lambda__1___closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__1; +x_1 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____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_197____lambda__1___closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____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_197____lambda__1___closed__2; -x_3 = l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__1; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__2; +x_3 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____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); @@ -424,15 +803,15 @@ lean_ctor_set_usize(x_5, 4, x_1); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__3; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__3; return x_2; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__1() { _start: { lean_object* x_1; @@ -440,17 +819,17 @@ x_1 = lean_mk_string_from_bytes("moduleDocExt", 12); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__1; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__3() { _start: { lean_object* x_1; @@ -459,7 +838,7 @@ lean_closure_set(x_1, 0, lean_box(0)); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__4() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__4() { _start: { lean_object* x_1; @@ -467,22 +846,22 @@ x_1 = lean_alloc_closure((void*)(l_Std_PersistentArray_push___rarg), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__5() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__6() { +static lean_object* _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____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_197____closed__2; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__4; -x_3 = l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__5; -x_4 = l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__3; +x_1 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__2; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__4; +x_3 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__5; +x_4 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____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); @@ -491,20 +870,20 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_197_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__6; +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____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_197____lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1(x_1); +x_2 = l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1(x_1); lean_dec(x_1); return x_2; } @@ -648,29 +1027,31 @@ if (lean_io_result_is_error(res)) return res; l___private_Lean_DocString_0__Lean_docStringExt = lean_io_result_get_value(res); lean_mark_persistent(l___private_Lean_DocString_0__Lean_docStringExt); lean_dec_ref(res); -}l_Lean_addBuiltinDocString___closed__1 = _init_l_Lean_addBuiltinDocString___closed__1(); +}l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces___closed__1 = _init_l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces___closed__1(); +lean_mark_persistent(l___private_Lean_DocString_0__Lean_removeNumLeadingSpaces___closed__1); +l_Lean_addBuiltinDocString___closed__1 = _init_l_Lean_addBuiltinDocString___closed__1(); 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_197____lambda__1___closed__1 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__1); -l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__2 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__2); -l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__3 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____lambda__1___closed__3); -l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__1 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__1); -l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__2 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__2); -l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__3 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__3); -l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__4 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__4(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__4); -l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__5 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__5(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__5); -l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__6 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__6(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_197____closed__6); -if (builtin) {res = l_Lean_initFn____x40_Lean_DocString___hyg_197_(lean_io_mk_world()); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__1 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__1); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__2 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__2); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__3 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____lambda__1___closed__3); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__1 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__1); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__2 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__2); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__3 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__3); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__4 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__4(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__4); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__5 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__5(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__5); +l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__6 = _init_l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__6(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_DocString___hyg_1527____closed__6); +if (builtin) {res = l_Lean_initFn____x40_Lean_DocString___hyg_1527_(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/App.c b/stage0/stdlib/Lean/Elab/App.c index 2cf97988c67a..53aa8a45febf 100644 --- a/stage0/stdlib/Lean/Elab/App.c +++ b/stage0/stdlib/Lean/Elab/App.c @@ -24,6 +24,7 @@ lean_object* l_Lean_Expr_bindingInfo_x21(lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_ElabAppArgs_synthesizeAppInstMVars___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__29___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__6; LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__14___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__19(lean_object*, lean_object*, lean_object*); @@ -296,7 +297,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLVal static lean_object* l___regBuiltin_Lean_Elab_Term_elabExplicit___closed__2; static uint8_t l___private_Lean_Elab_App_0__Lean_Elab_Term_getSuccesses___lambda__1___closed__2; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLValsAux_loop___lambda__3___closed__2; -lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_fTypeHasOptAutoParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_isNextOutParamOfLocalInstanceAndResult___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabChoice___closed__3; @@ -376,6 +376,7 @@ static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLVals___c LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId___spec__1___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_propagateExpectedTypeFor(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___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__51___closed__5; +lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_5____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___closed__9; @@ -438,6 +439,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabApp___closed__3; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__20; lean_object* l_Lean_Syntax_identComponents(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabIdent_declRange___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_ElabAppArgs_State_etaArgs___default___closed__1; @@ -666,7 +668,6 @@ static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_tryCoeFun_x3f___ static lean_object* l_Lean_Elab_Term_elabAppArgs___closed__14; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_throwLValError___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_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMCtxImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabAppArgs___closed__15; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLValsAux_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -787,7 +788,7 @@ uint8_t l_Lean_Expr_isFVar(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_getForallBody___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_15126_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_15107_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_5_(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppAux(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -815,7 +816,6 @@ lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_obje LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_consumeMDataAndTypeAnnotations(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__34___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___lambda__5___closed__2; lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -14042,7 +14042,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_App_0_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__51___closed__3; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__51___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_anyNamedArgDependsOnCurrent___spec__51___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -16303,7 +16303,7 @@ x_23 = lean_ctor_get(x_21, 1); lean_inc(x_23); lean_dec(x_21); x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_Expr_getAppNumArgsAux(x_8, x_24); +x_25 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_8, x_24); x_26 = l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_isNextOutParamOfLocalInstanceAndResult_isOutParamOfLocalInstance___closed__1; lean_inc(x_25); x_27 = lean_mk_array(x_25, x_26); @@ -25833,7 +25833,7 @@ x_41 = l_Std_Range_forIn_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_add x_42 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_42, 0, x_40); lean_ctor_set(x_42, 1, x_41); -x_43 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_42, x_11, x_12, x_13, x_14, x_15, x_16, x_27); +x_43 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_42, x_11, x_12, x_13, x_14, x_15, x_16, x_27); lean_dec(x_13); x_44 = !lean_is_exclusive(x_43); if (x_44 == 0) @@ -29761,7 +29761,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -x_20 = l_Lean_Expr_consumeMDataAndTypeAnnotations(x_18); +x_20 = l_Lean_Expr_cleanupAnnotations(x_18); x_21 = l_Lean_Expr_getAppFn(x_20); lean_dec(x_20); lean_inc(x_10); @@ -29777,7 +29777,7 @@ lean_object* x_89; lean_object* x_90; x_89 = lean_ctor_get(x_88, 1); lean_inc(x_89); lean_dec(x_88); -x_90 = l_Lean_Expr_consumeMDataAndTypeAnnotations(x_21); +x_90 = l_Lean_Expr_cleanupAnnotations(x_21); if (lean_obj_tag(x_90) == 4) { lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; @@ -36024,6 +36024,7 @@ lean_object* x_67; lean_object* x_68; lean_object* x_69; x_67 = l_Lean_Expr_mvarId_x21(x_63); lean_dec(x_63); x_68 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(x_67, x_5, x_6, x_7, x_8, x_9, x_10, x_64); +lean_dec(x_67); x_69 = lean_ctor_get(x_68, 0); lean_inc(x_69); if (lean_obj_tag(x_69) == 0) @@ -36043,7 +36044,7 @@ lean_object* x_72; lean_object* x_73; x_72 = lean_ctor_get(x_69, 0); lean_inc(x_72); lean_dec(x_69); -x_73 = lean_ctor_get(x_72, 2); +x_73 = lean_ctor_get(x_72, 1); lean_inc(x_73); lean_dec(x_72); if (lean_obj_tag(x_73) == 1) @@ -37482,7 +37483,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLValsAux_loop___lambda__3___closed__1; x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppAux___spec__4___closed__1; x_3 = lean_unsigned_to_nat(1111u); -x_4 = lean_unsigned_to_nat(35u); +x_4 = lean_unsigned_to_nat(21u); x_5 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLValsAux_loop___lambda__3___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -40194,7 +40195,7 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_15126_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_15107_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -40966,7 +40967,7 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_elabProj_declRange___closed__ res = l___regBuiltin_Lean_Elab_Term_elabProj_declRange(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_15126_(lean_io_mk_world()); +res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_15107_(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/Attributes.c b/stage0/stdlib/Lean/Elab/Attributes.c index 2bdee2844843..a217f6d19b4c 100644 --- a/stage0/stdlib/Lean/Elab/Attributes.c +++ b/stage0/stdlib/Lean/Elab/Attributes.c @@ -17,7 +17,7 @@ lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Attribute_stx___default; static lean_object* l_Lean_Elab_mkAttrKindGlobal___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__5(lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_erase_macro_scopes(lean_object*); @@ -28,6 +28,7 @@ lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Macro_getCurrNamespace(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); @@ -38,6 +39,7 @@ extern lean_object* l_Lean_maxRecDepthErrorMessage; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___rarg___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_instInhabitedAttribute; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_toAttributeKind___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_instToFormatAttribute(lean_object*); @@ -47,6 +49,7 @@ lean_object* l_Lean_Elab_throwUnsupportedSyntax___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_toAttributeKind___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___rarg___lambda__5(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___rarg___lambda__1___boxed(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); @@ -54,7 +57,7 @@ lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__14(lean_object*, lean_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_toAttributeKind___closed__6; static lean_object* l_Lean_Elab_elabAttr___rarg___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -68,17 +71,19 @@ lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___rarg(lean_o LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___rarg___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_toAttributeKind___closed__10; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___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_Elab_logException___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___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* l_Lean_Name_toString(lean_object*, uint8_t); +lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Attribute_kind___default; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -90,7 +95,8 @@ lean_object* lean_format_pretty(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_elabAttr___spec__2___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -98,15 +104,17 @@ static lean_object* l_Lean_Elab_toAttributeKind___closed__5; static lean_object* l_Lean_Elab_instToFormatAttribute___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1(lean_object*); lean_object* l_Lean_throwErrorAt___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__4(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_Elab_elabAttr___rarg___lambda__5___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_elabAttr___spec__2___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Elab_instToFormatAttribute___closed__8; static lean_object* l_Lean_Elab_instInhabitedAttribute___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Elab_toAttributeKind___closed__3; static lean_object* l_Lean_Elab_elabAttr___rarg___lambda__3___closed__3; @@ -129,6 +137,7 @@ static lean_object* l_Lean_Elab_instToFormatAttribute___closed__5; LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_elabAttr___spec__2___rarg___lambda__1(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*); static lean_object* l_Lean_Elab_instToFormatAttribute___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__8(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l_Lean_Elab_instToFormatAttribute___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___rarg(lean_object*, lean_object*, lean_object*); @@ -157,14 +166,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_toAttributeKind___boxed(lean_object*, lean_ static lean_object* l_Lean_Elab_elabAttr___rarg___lambda__6___closed__1; static lean_object* l_Lean_Elab_mkAttrKindGlobal___closed__3; LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_elabAttr___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_toAttributeKind(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_elabAttr___spec__4___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabAttr___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_elabAttr___spec__2___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___rarg___lambda__3___closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_elabAttr___rarg___lambda__1(lean_object*); static lean_object* l_Lean_Elab_mkAttrKindGlobal___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_elabAttr___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -181,7 +189,7 @@ lean_object* l_Lean_Syntax_formatStxAux(lean_object*, uint8_t, lean_object*, lea static lean_object* l_Lean_Elab_elabAttr___rarg___lambda__5___closed__1; LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_elabAttr___spec__2___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static uint8_t _init_l_Lean_Elab_Attribute_kind___default() { _start: { @@ -2475,17 +2483,30 @@ lean_dec(x_1); return x_14; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = l_Lean_replaceRef(x_1, x_4); +x_6 = lean_ctor_get(x_2, 1); +lean_inc(x_6); +lean_dec(x_2); +x_7 = lean_apply_3(x_6, lean_box(0), x_5, x_3); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; -x_4 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_4, 0, x_1); +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_3); +lean_ctor_set(x_4, 1, x_1); x_5 = lean_apply_2(x_2, lean_box(0), x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; @@ -2499,19 +2520,85 @@ lean_dec(x_6); x_8 = lean_box(0); lean_inc(x_7); x_9 = lean_apply_2(x_7, lean_box(0), x_8); -x_10 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1___boxed), 3, 2); +x_10 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__2), 3, 2); lean_closure_set(x_10, 0, x_5); lean_closure_set(x_10, 1, x_7); x_11 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_9, x_10); return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, size_t x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -if (lean_obj_tag(x_14) == 0) +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_2); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_inc(x_1); +x_8 = l_Lean_Elab_logException___rarg(x_1, x_2, x_3, x_4, x_7); +x_9 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__4), 3, 2); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_5); +x_10 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_object* x_4; lean_object* x_5; +x_4 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_4, 0, x_1); +x_5 = lean_apply_2(x_2, lean_box(0), x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_4 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__6___boxed), 3, 2); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_apply_4(x_2, lean_box(0), lean_box(0), x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__8(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, size_t x_15, lean_object* x_16) { +_start: +{ +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -2522,39 +2609,41 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -lean_dec(x_14); -x_16 = lean_ctor_get(x_1, 0); -lean_inc(x_16); -lean_dec(x_1); -x_17 = lean_ctor_get(x_16, 1); +x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); lean_dec(x_16); -x_18 = lean_apply_2(x_17, lean_box(0), x_15); -return x_18; +x_18 = lean_ctor_get(x_1, 0); +lean_inc(x_18); +lean_dec(x_1); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_apply_2(x_19, lean_box(0), x_17); +return x_20; } else { -lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_14, 0); -lean_inc(x_19); -lean_dec(x_14); -x_20 = 1; -x_21 = lean_usize_add(x_2, x_20); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_21, x_19); -return x_22; +lean_object* x_21; size_t x_22; size_t x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_16, 0); +lean_inc(x_21); +lean_dec(x_16); +x_22 = 1; +x_23 = lean_usize_add(x_2, x_22); +x_24 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(x_1, 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_23, x_21); +return x_24; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, size_t x_12, size_t x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, size_t x_14, size_t x_15, lean_object* x_16) { _start: { -uint8_t x_15; -x_15 = lean_usize_dec_lt(x_13, x_12); -if (x_15 == 0) +uint8_t x_17; +x_17 = lean_usize_dec_lt(x_15, x_14); +if (x_17 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2565,21 +2654,26 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_16 = lean_ctor_get(x_1, 0); -lean_inc(x_16); +x_18 = lean_ctor_get(x_1, 0); +lean_inc(x_18); lean_dec(x_1); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = lean_apply_2(x_17, lean_box(0), x_14); -return x_18; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_apply_2(x_19, lean_box(0), x_16); +return x_20; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_19 = lean_array_uget(x_11, x_13); -x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_21 = lean_array_uget(x_13, x_15); +x_22 = lean_ctor_get(x_1, 1); +lean_inc(x_22); +x_23 = lean_ctor_get(x_4, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_4, 1); +lean_inc(x_24); +lean_inc(x_21); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); @@ -2589,33 +2683,67 @@ lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_21 = l_Lean_Elab_elabAttr___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); -lean_inc(x_10); +x_25 = l_Lean_Elab_elabAttr___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +x_26 = lean_ctor_get(x_24, 0); +lean_inc(x_26); +x_27 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1___boxed), 4, 3); +lean_closure_set(x_27, 0, x_21); +lean_closure_set(x_27, 1, x_24); +lean_closure_set(x_27, 2, x_25); +lean_inc(x_12); +x_28 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_26, x_27); +lean_inc(x_12); lean_inc(x_1); -x_22 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__2), 4, 3); -lean_closure_set(x_22, 0, x_14); -lean_closure_set(x_22, 1, x_1); -lean_closure_set(x_22, 2, x_10); +lean_inc(x_16); +x_29 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3), 4, 3); +lean_closure_set(x_29, 0, x_16); +lean_closure_set(x_29, 1, x_1); +lean_closure_set(x_29, 2, x_12); +lean_inc(x_12); +x_30 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_28, x_29); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_9); lean_inc(x_10); -x_23 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_21, x_22); -x_24 = lean_box_usize(x_13); -x_25 = lean_box_usize(x_12); -x_26 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3___boxed), 14, 13); -lean_closure_set(x_26, 0, x_1); -lean_closure_set(x_26, 1, x_24); -lean_closure_set(x_26, 2, x_2); -lean_closure_set(x_26, 3, x_3); -lean_closure_set(x_26, 4, x_4); -lean_closure_set(x_26, 5, x_5); -lean_closure_set(x_26, 6, x_6); -lean_closure_set(x_26, 7, x_7); -lean_closure_set(x_26, 8, x_8); -lean_closure_set(x_26, 9, x_9); -lean_closure_set(x_26, 10, x_10); -lean_closure_set(x_26, 11, x_11); -lean_closure_set(x_26, 12, x_25); -x_27 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_23, x_26); -return x_27; +lean_inc(x_1); +x_31 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__5), 7, 6); +lean_closure_set(x_31, 0, x_1); +lean_closure_set(x_31, 1, x_10); +lean_closure_set(x_31, 2, x_9); +lean_closure_set(x_31, 3, x_11); +lean_closure_set(x_31, 4, x_16); +lean_closure_set(x_31, 5, x_12); +x_32 = lean_ctor_get(x_23, 1); +lean_inc(x_32); +lean_dec(x_23); +x_33 = lean_apply_3(x_32, lean_box(0), x_30, x_31); +lean_inc(x_12); +lean_inc(x_1); +x_34 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__7), 3, 2); +lean_closure_set(x_34, 0, x_1); +lean_closure_set(x_34, 1, x_12); +lean_inc(x_12); +x_35 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_33, x_34); +x_36 = lean_box_usize(x_15); +x_37 = lean_box_usize(x_14); +x_38 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__8___boxed), 16, 15); +lean_closure_set(x_38, 0, x_1); +lean_closure_set(x_38, 1, x_36); +lean_closure_set(x_38, 2, x_2); +lean_closure_set(x_38, 3, x_3); +lean_closure_set(x_38, 4, x_4); +lean_closure_set(x_38, 5, x_5); +lean_closure_set(x_38, 6, x_6); +lean_closure_set(x_38, 7, x_7); +lean_closure_set(x_38, 8, x_8); +lean_closure_set(x_38, 9, x_9); +lean_closure_set(x_38, 10, x_10); +lean_closure_set(x_38, 11, x_11); +lean_closure_set(x_38, 12, x_12); +lean_closure_set(x_38, 13, x_13); +lean_closure_set(x_38, 14, x_37); +x_39 = lean_apply_4(x_22, lean_box(0), lean_box(0), x_35, x_38); +return x_39; } } } @@ -2623,7 +2751,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spe _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___boxed), 14, 0); +x_2 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___boxed), 16, 0); return x_2; } } @@ -2641,94 +2769,104 @@ x_5 = lean_apply_2(x_4, lean_box(0), x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); -x_12 = lean_array_get_size(x_10); -x_13 = lean_usize_of_nat(x_12); -lean_dec(x_12); -x_14 = 0; -x_15 = l_Lean_Elab_mkAttrKindGlobal___closed__3; -lean_inc(x_11); +lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +x_14 = lean_array_get_size(x_12); +x_15 = lean_usize_of_nat(x_14); +lean_dec(x_14); +x_16 = 0; +x_17 = l_Lean_Elab_mkAttrKindGlobal___closed__3; +lean_inc(x_13); lean_inc(x_1); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_11, x_10, x_13, x_14, x_15); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_elabAttrs___rarg___lambda__1), 2, 1); -lean_closure_set(x_17, 0, x_1); -x_18 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_16, x_17); -return x_18; +x_18 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_13, x_12, x_15, x_16, x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_elabAttrs___rarg___lambda__1), 2, 1); +lean_closure_set(x_19, 0, x_1); +x_20 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_18, x_19); +return x_20; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabAttrs(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabAttrs___rarg), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabAttrs___rarg), 12, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__1(x_1, x_2, x_3); +x_4 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__6(x_1, x_2, x_3); lean_dec(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -size_t x_15; size_t x_16; lean_object* x_17; -x_15 = lean_unbox_usize(x_2); +size_t x_17; size_t x_18; lean_object* x_19; +x_17 = lean_unbox_usize(x_2); lean_dec(x_2); -x_16 = lean_unbox_usize(x_13); -lean_dec(x_13); -x_17 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__3(x_1, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16, x_14); -return x_17; +x_18 = lean_unbox_usize(x_15); +lean_dec(x_15); +x_19 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___lambda__8(x_1, x_17, 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_18, x_16); +return x_19; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -size_t x_15; size_t x_16; lean_object* x_17; -x_15 = lean_unbox_usize(x_12); -lean_dec(x_12); -x_16 = lean_unbox_usize(x_13); -lean_dec(x_13); -x_17 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15, x_16, x_14); -return x_17; +size_t x_17; size_t x_18; lean_object* x_19; +x_17 = lean_unbox_usize(x_14); +lean_dec(x_14); +x_18 = lean_unbox_usize(x_15); +lean_dec(x_15); +x_19 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabAttrs___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_17, x_18, x_16); +return x_19; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_unsigned_to_nat(1u); -x_12 = l_Lean_Syntax_getArg(x_10, x_11); -x_13 = l_Lean_Syntax_getSepArgs(x_12); -lean_dec(x_12); -x_14 = l_Lean_Elab_elabAttrs___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_14; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_unsigned_to_nat(1u); +x_14 = l_Lean_Syntax_getArg(x_12, x_13); +x_15 = l_Lean_Syntax_getSepArgs(x_14); +lean_dec(x_14); +x_16 = l_Lean_Elab_elabAttrs___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +return x_16; } } LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabDeclAttrs___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabDeclAttrs___rarg___boxed), 12, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabDeclAttrs___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_11; -x_11 = l_Lean_Elab_elabDeclAttrs___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_10); -return x_11; +lean_object* x_13; +x_13 = l_Lean_Elab_elabDeclAttrs___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_12); +return x_13; } } lean_object* initialize_Init(uint8_t builtin, lean_object*); diff --git a/stage0/stdlib/Lean/Elab/Binders.c b/stage0/stdlib/Lean/Elab/Binders.c index 7fda466f4e10..90d1816d28fb 100644 --- a/stage0/stdlib/Lean/Elab/Binders.c +++ b/stage0/stdlib/Lean/Elab/Binders.c @@ -342,8 +342,8 @@ static lean_object* l_Lean_Elab_Term_elabBinder___rarg___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_expandFunBinders_loop___spec__4(lean_object*, size_t, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetTmpDecl___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Term_expandFun_declRange___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_9159_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_9400_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831_(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabDepArrow___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabLetDeclAux___lambda__6(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_quoteAutoTactic___closed__20; @@ -489,13 +489,13 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabLetTmpDecl(lean_objec static lean_object* l_Lean_Elab_Term_quoteAutoTactic___closed__26; extern lean_object* l_Lean_Elab_Term_termElabAttribute; static lean_object* l___regBuiltin_Lean_Elab_Term_elabDepArrow_declRange___closed__5; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_expandFunBinders_loop___spec__7(lean_object*, size_t, size_t, lean_object*, lean_object*); lean_object* l_Lean_mkAtomFrom(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_quoteAutoTactic___spec__1___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Term_elabDepArrow_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_expandBinderIdent___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_elabFun___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__1; static lean_object* l_Lean_Elab_Term_expandSimpleBinderWithType___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Term_elabFun___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabForall_declRange___closed__7; @@ -544,11 +544,11 @@ static lean_object* l_Lean_Elab_Term_expandWhereDecls___closed__3; static lean_object* l___private_Lean_Elab_Binders_0__Lean_Elab_Term_expandMatchAltsIntoMatchAux___closed__11; static lean_object* l_List_foldlM___at_Lean_Elab_Term_declareTacticSyntax___spec__6___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_matchBinder___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__4; LEAN_EXPORT lean_object* l_Lean_compileDecl___at_Lean_Elab_Term_declareTacticSyntax___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Binders_0__Lean_Elab_Term_expandBinderModifier___closed__6; static lean_object* l_Lean_Elab_Term_elabLetDeclCore___closed__6; uint8_t lean_nat_dec_le(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__4; static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetDecl_declRange___closed__2; static lean_object* l_Lean_Elab_Term_quoteAutoTactic___closed__35; static lean_object* l_Lean_Elab_Term_quoteAutoTactic___closed__39; @@ -602,7 +602,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Term_precheckFun_ LEAN_EXPORT lean_object* l_Lean_Elab_Term_FunBinders_elabFunBindersAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Term_declareTacticSyntax___spec__6___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Term_precheckFun___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__5; lean_object* l_Lean_Elab_Term_elabType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_universeConstraintsCheckpoint___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); @@ -619,6 +618,7 @@ lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMe static lean_object* l_Lean_Elab_Term_quoteAutoTactic___closed__23; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_expandFunBinders_loop___closed__2; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Binders_0__Lean_Elab_Term_expandOptIdent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_quoteAutoTactic___spec__1___closed__7; @@ -705,7 +705,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabDepArrow_declRange___close static lean_object* l___regBuiltin_Lean_Elab_Term_elabForall___closed__2; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_quoteAutoTactic___closed__2; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Binders_0__Lean_Elab_Term_expandMatchAltsIntoMatchAux(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_expandFunBinders_loop___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetFunDecl___closed__3; @@ -721,6 +720,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_FunBinders_State_fvars___default; static lean_object* l_List_foldlM___at_Lean_Elab_Term_declareTacticSyntax___spec__6___closed__1; static lean_object* l___private_Lean_Elab_Binders_0__Lean_Elab_Term_expandBinderModifier___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Term_elabFun_declRange___closed__2; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__3; static lean_object* l_Lean_Elab_Term_quoteAutoTactic___closed__48; static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetDelayedDecl_declRange___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabLetFunDecl(lean_object*); @@ -759,7 +759,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_expandForall___closed__5; LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___at_Lean_Elab_Term_declareTacticSyntax___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldlM___at_Lean_Elab_Term_declareTacticSyntax___spec__6___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_expandBinderIdent___spec__2___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForall_declRange___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Term_expandFun_declRange___closed__2; static lean_object* l_Lean_Elab_Term_expandWhereDecls___closed__10; @@ -785,6 +784,7 @@ static lean_object* l_Lean_Elab_Term_quoteAutoTactic___closed__45; static lean_object* l___regBuiltin_Lean_Elab_Term_elabDepArrow_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabBinder(lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__2; lean_object* lean_add_decl(lean_object*, lean_object*); uint8_t l_Lean_Syntax_isAntiquotSplice(lean_object*); static lean_object* l_Lean_Elab_Term_elabLetDeclAux___closed__7; @@ -6423,7 +6423,7 @@ lean_dec(x_1); return x_10; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__1() { _start: { lean_object* x_1; @@ -6431,17 +6431,17 @@ x_1 = lean_mk_string_from_bytes("checkBinderAnnotations", 22); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__3() { _start: { lean_object* x_1; @@ -6449,7 +6449,7 @@ x_1 = lean_mk_string_from_bytes("", 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__4() { _start: { lean_object* x_1; @@ -6457,13 +6457,13 @@ x_1 = lean_mk_string_from_bytes("check whether type is a class instance whenever return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__5() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 1; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__3; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__4; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__3; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__4; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -6472,12 +6472,12 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__2; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__5; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__2; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__5; x_4 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_1); return x_4; } @@ -7236,7 +7236,7 @@ static lean_object* _init_l_Lean_Elab_Term_elabBinder___rarg___lambda__1___close lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_elabBinder___rarg___lambda__1___closed__1; x_2 = l_Lean_Elab_Term_elabBinder___rarg___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_Term_elabBinder___rarg___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -26689,7 +26689,7 @@ static lean_object* _init_l_Lean_Elab_Term_elabLetDeclAux___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__3; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } @@ -28380,7 +28380,7 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_9159_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_9400_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -28690,17 +28690,17 @@ l___private_Lean_Elab_Binders_0__Lean_Elab_Term_ensureAtomicBinderName___closed_ lean_mark_persistent(l___private_Lean_Elab_Binders_0__Lean_Elab_Term_ensureAtomicBinderName___closed__3); l___private_Lean_Elab_Binders_0__Lean_Elab_Term_ensureAtomicBinderName___closed__4 = _init_l___private_Lean_Elab_Binders_0__Lean_Elab_Term_ensureAtomicBinderName___closed__4(); lean_mark_persistent(l___private_Lean_Elab_Binders_0__Lean_Elab_Term_ensureAtomicBinderName___closed__4); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__4); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845____closed__5); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1845_(lean_io_mk_world()); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__4); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831____closed__5); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_1831_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Term_checkBinderAnnotations = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Term_checkBinderAnnotations); @@ -29218,7 +29218,7 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_elabLetTmpDecl_declRange___cl res = l___regBuiltin_Lean_Elab_Term_elabLetTmpDecl_declRange(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_9159_(lean_io_mk_world()); +res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Binders___hyg_9400_(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/BuiltinCommand.c b/stage0/stdlib/Lean/Elab/BuiltinCommand.c index a069ae45495a..9a495d153e17 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinCommand.c +++ b/stage0/stdlib/Lean/Elab/BuiltinCommand.c @@ -459,7 +459,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd___closed__1; lean_object* lean_expr_dbg_to_string(lean_object*); static lean_object* l_Lean_Elab_Command_elabEvalUnsafe___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInCmd_declRange___closed__6; -lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_withLogging___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_mkRunMetaEval___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabChoice(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd___closed__4; @@ -715,7 +714,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabNonComputableSection___ uint8_t l_Lean_Syntax_isNone(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace_declRange___closed__7; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabNamespace(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEvalUnsafe___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -813,6 +811,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___boxed(lean_ob LEAN_EXPORT lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_elabOpenScoped___at_Lean_Elab_Command_elabOpen___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabEnd_declRange___closed__1; +lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MonadQuotation_addMacroScope___at_Lean_Elab_Command_elabVariable___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCheckCore___closed__4; static lean_object* l_Lean_Elab_Command_elabEnd___lambda__1___closed__1; @@ -832,6 +831,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabUniverse(lean_obje static lean_object* l_Lean_Elab_Command_elabEvalUnsafe___lambda__8___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabVariable___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_hasNoErrorMessages___boxed(lean_object*); +lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_addScope___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_BuiltinCommand_0__Lean_Elab_Command_replaceBinderAnnotation___spec__2___lambda__2___closed__6; @@ -6866,7 +6866,7 @@ static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resol 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_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__1___closed__3; x_2 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__1___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Command_elabExport___spec__3___lambda__1___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -15422,7 +15422,7 @@ lean_inc(x_86); lean_dec(x_79); lean_inc(x_3); lean_inc(x_2); -x_87 = l_Lean_Elab_logException___at_Lean_Elab_Command_withLogging___spec__1(x_85, x_2, x_3, x_86); +x_87 = l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(x_85, x_2, x_3, x_86); if (lean_obj_tag(x_87) == 0) { lean_object* x_88; uint8_t x_89; @@ -15477,7 +15477,7 @@ lean_ctor_set(x_99, 0, x_97); x_100 = 2; lean_inc(x_3); lean_inc(x_2); -x_101 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_99, x_100, x_2, x_3, x_98); +x_101 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_99, x_100, x_2, x_3, x_98); x_102 = lean_ctor_get(x_101, 1); lean_inc(x_102); lean_dec(x_101); @@ -15531,7 +15531,7 @@ lean_ctor_set(x_114, 0, x_112); x_115 = 2; lean_inc(x_3); lean_inc(x_2); -x_116 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_114, x_115, x_2, x_3, x_113); +x_116 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_114, x_115, x_2, x_3, x_113); x_117 = lean_ctor_get(x_116, 1); lean_inc(x_117); lean_dec(x_116); @@ -15803,7 +15803,7 @@ lean_inc(x_192); lean_dec(x_185); lean_inc(x_3); lean_inc(x_2); -x_193 = l_Lean_Elab_logException___at_Lean_Elab_Command_withLogging___spec__1(x_191, x_2, x_3, x_192); +x_193 = l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(x_191, x_2, x_3, x_192); if (lean_obj_tag(x_193) == 0) { lean_object* x_194; uint8_t x_195; @@ -15861,7 +15861,7 @@ lean_ctor_set(x_204, 0, x_202); x_205 = 2; lean_inc(x_3); lean_inc(x_2); -x_206 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_204, x_205, x_2, x_3, x_203); +x_206 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_204, x_205, x_2, x_3, x_203); x_207 = lean_ctor_get(x_206, 1); lean_inc(x_207); lean_dec(x_206); diff --git a/stage0/stdlib/Lean/Elab/BuiltinNotation.c b/stage0/stdlib/Lean/Elab/BuiltinNotation.c index 7ed7130b4349..6a3190ffa277 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinNotation.c +++ b/stage0/stdlib/Lean/Elab/BuiltinNotation.c @@ -1545,7 +1545,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Term_elabAnonymo lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Term_elabAnonymousCtor___spec__3___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Term_elabAnonymousCtor___spec__3___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Term_elabAnonymousCtor___spec__3___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/BuiltinTerm.c b/stage0/stdlib/Lean/Elab/BuiltinTerm.c index 520ceac03d58..25acdfc6161a 100644 --- a/stage0/stdlib/Lean/Elab/BuiltinTerm.c +++ b/stage0/stdlib/Lean/Elab/BuiltinTerm.c @@ -9461,7 +9461,7 @@ lean_dec(x_13); x_15 = lean_st_ref_get(x_4, x_14); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 4); +x_17 = lean_ctor_get(x_16, 5); lean_inc(x_17); lean_dec(x_16); x_18 = lean_ctor_get_uint8(x_17, sizeof(void*)*2); @@ -10176,7 +10176,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_BuiltinTerm_0__Lean_Elab_Term_mkS _start: { lean_object* x_9; lean_object* x_10; -lean_inc(x_1); x_9 = l_Lean_Elab_Term_isTacticOrPostponedHole_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); @@ -13347,7 +13346,7 @@ static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resol 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_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Term_elabOpen___spec__22___lambda__1___closed__3; x_2 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Term_elabOpen___spec__22___lambda__1___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Term_elabOpen___spec__22___lambda__1___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/Command.c b/stage0/stdlib/Lean/Elab/Command.c index f1b180ecb5cf..1e7ef64d94f5 100644 --- a/stage0/stdlib/Lean/Elab/Command.c +++ b/stage0/stdlib/Lean/Elab/Command.c @@ -16,15 +16,16 @@ extern "C" { lean_object* l_List_reverse___rarg(lean_object*); static lean_object* l_Lean_Elab_Command_State_infoState___default___closed__4; static lean_object* l_Lean_Elab_Command_State_scopes___default___closed__1; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); 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_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandDeclId___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadQuotationCommandElabM___closed__4; -static lean_object* l_Lean_Elab_Command_withLogging___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_getVarDecls___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedState; lean_object* l_Lean_extractMacroScopes(lean_object*); @@ -34,55 +35,55 @@ static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_22 LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runTermElabM___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*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__2; lean_object* lean_io_get_num_heartbeats(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_catchExceptions(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_registerTraceClass(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_Elab_Command_elabCommandTopLevel___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadCommandElabM___closed__6; lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___closed__4; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__1; static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__12; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1; lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lean_Elab_Command_runLinters___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__3___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_Elab_Command_runLinters___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instAddMessageContextCommandElabM___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScope___rarg___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Command_withMacroExpansion___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at_Lean_Elab_Command_liftTermElabM___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_mkInfoTree___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__17(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); lean_object* lean_io_error_to_string(lean_object*); uint8_t l_Lean_Elab_isAbortExceptionId(lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2237____closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommandTopLevel___lambda__2___closed__1; lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__11(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l___private_Lean_DocString_0__Lean_docStringExt; LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlMAux___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__10(lean_object*, lean_object*, lean_object*); @@ -103,25 +104,22 @@ LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Command_ LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScope___boxed(lean_object*); static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___closed__2; static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__8; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__1(lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_Context_macroStack___default; -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg___closed__1; LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Command_modifyScope___spec__1(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_runTermElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__4; static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__16; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__9(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_withLogging___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_withFreshMacroScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); @@ -135,7 +133,7 @@ lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__13(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getLevelNames___boxed(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -159,19 +157,16 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_runTermElabM___rarg___lambda__1(lea LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__12(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftEIO(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_addLinter(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___at_Lean_Elab_Command_expandDeclId___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__4; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__5; static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__7(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_State_messages___default___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg(lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__7; static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__10; static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__2___closed__2; @@ -184,19 +179,21 @@ static lean_object* l_Lean_Elab_Command_instMonadCommandElabM___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommandTopLevel___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withMacroExpansion___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___lambda__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__16___closed__1; lean_object* l_Lean_KeyedDeclsAttribute_getEntries___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_foldlM___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_ioErrorToMessage(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_Scope_opts___default; static lean_object* l_Lean_Elab_Command_State_traceState___default___closed__1; static lean_object* l_Lean_Elab_Command_State_infoState___default___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_InfoTree_format(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1; static lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM___closed__1; -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Elab_Command_expandDeclId___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_right(size_t, size_t); @@ -209,6 +206,7 @@ lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_ob lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_runLinters___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_modifyScope___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_State_messages___default; @@ -234,6 +232,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermE static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__5; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__3; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_getVarDecls(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getLevelNames___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -246,19 +245,18 @@ static lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM___closed__ static lean_object* l_Lean_Elab_Command_State_ngen___default___closed__3; static lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__3; extern lean_object* l_Lean_maxRecDepth; +LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_LocalContext_empty; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessages___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_MessageData_hasTag(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__12___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___at_Lean_Elab_Command_expandDeclId___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___lambda__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runTermElabM___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___closed__5; @@ -282,7 +280,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedCommandElabM(lean_obje static lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftEIO___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_runLinters(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__12(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*); uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); @@ -304,9 +301,7 @@ static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__9; LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_withLogging___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__11(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Command_liftTermElabM___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_modifyScope___closed__4; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__6(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -332,7 +327,6 @@ static lean_object* l_Lean_Elab_Command_elabCommand___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_Scope_openDecls___default; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_State_nextInstIdx___default; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRefCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermState___boxed(lean_object*, lean_object*); @@ -340,7 +334,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCo lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* lean_array_get(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_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__2; static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___closed__2; @@ -350,13 +343,11 @@ static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_mkMetaCon LEAN_EXPORT lean_object* l_Lean_Elab_getInfoTrees___at_Lean_Elab_Command_elabCommandTopLevel___spec__1(lean_object*); static lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM___closed__3; static lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM___closed__3; -static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkState(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__2; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___closed__2; static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftCoreM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___lambda__3___closed__3; static lean_object* l_Lean_Elab_Command_liftCoreM___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -367,6 +358,7 @@ LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentA LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Command_liftTermElabM___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__12___lambda__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__10; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___lambda__3___closed__5; @@ -380,10 +372,10 @@ static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__13; lean_object* l_Lean_Core_getMaxHeartbeats(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandDeclId___spec__14(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_417_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2237_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_1842_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535_(lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_State_ngen___default; extern lean_object* l_Lean_Expr_instHashableExpr; @@ -394,21 +386,21 @@ lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_obje static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__14; static lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___closed__1; lean_object* l_Lean_Elab_Term_addAutoBoundImplicits_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__5; +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__12(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__3; lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_runTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_Elab_Command_elabCommandTopLevel___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_State_messages___default___closed__3; static size_t l_Lean_Elab_Command_expandDeclId___closed__2; -static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4; LEAN_EXPORT lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_left(size_t, size_t); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___closed__4; uint8_t l_Lean_Name_isAtomic(lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); lean_object* l_Lean_Meta_InfoCacheKey_instHashableInfoCacheKey___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes(lean_object*); static lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1___closed__3; extern lean_object* l_Lean_protectedExt; @@ -418,8 +410,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCo LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_liftAttrM(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_liftAttrM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_withLogging___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_State_scopes___default; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLiftTIOCommandElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_addUnivLevel___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -427,7 +417,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___lambda__1(le static lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__9(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withLogging(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__2; @@ -459,46 +448,48 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId__ static lean_object* l_Lean_Elab_Command_modifyScope___closed__1; static lean_object* l_Lean_Elab_Command_addLinter___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withMacroExpansion(lean_object*); lean_object* l_Lean_InternalExceptionId_getName(lean_object*, lean_object*); lean_object* l_Lean_Elab_expandDeclIdCore(lean_object*); LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_Elab_Command_runLinters___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__1; lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___lambda__3___closed__4; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runLinters___spec__4___closed__1; static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__12___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_Elab_Command_elabCommandTopLevel___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_EStateM_instMonadEStateM(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Command_liftTermElabM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__7; lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceOptions(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_Context_ref___default; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getMainModule___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(lean_object*); static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__6; static lean_object* l_List_foldl___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_withLogging___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_addUnivLevel(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2; static lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadEnvCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*); uint8_t l_List_elem___at_Lean_NameHashSet_insert___spec__2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1___closed__5; static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_DocString_0__Lean_removeLeadingSpaces(lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___lambda__3___closed__1; LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__2(lean_object*, lean_object*, lean_object*); @@ -516,19 +507,21 @@ lean_object* lean_environment_main_module(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessages(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__6; static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScope(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadQuotationCommandElabM___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__1; lean_object* l_Lean_mkPrivateName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getMainModule(lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__8; +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__6___closed__1; static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__11; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -537,7 +530,6 @@ lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___boxed(lean_object*, lean_object*); lean_object* l_Lean_MacroScopesView_review(lean_object*); uint8_t l_Lean_Name_isSuffixOf(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__5; @@ -547,18 +539,18 @@ LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_runLinters___spec__3_ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_showPartialSyntaxErrors; LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_ioErrorToMessage___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_runTermElabM___rarg___lambda__2___closed__1; static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedScope; -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__17(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_runTermElabM___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM___closed__3; static uint32_t l_Lean_Elab_Command_instInhabitedState___closed__4; static lean_object* l_Lean_Elab_Command_Scope_varDecls___default___closed__1; lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_State_infoState___default___closed__3; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withScope(lean_object*); extern lean_object* l_Lean_Elab_pp_macroStack; @@ -567,9 +559,9 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLiftTIOCommandElabM(lean_o LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadOptionsCommandElabM___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_mkInfoTree(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedCommandElabM___closed__1; static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_expandDeclId___spec__12(lean_object*, lean_object*, lean_object*, lean_object*); @@ -581,22 +573,20 @@ static lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___closed__1; static lean_object* l_Lean_Elab_Command_instMonadCommandElabM___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___closed__2; -static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadResolveNameCommandElabM___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_State_ngen___default___closed__1; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__5; static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__12___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_liftCoreM(lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe(lean_object*); -LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_addTraceAsMessagesCore(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__10; -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__2; static lean_object* l_Lean_Elab_Command_instMonadCommandElabM___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadInfoTreeCommandElabM; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getLevelNames(lean_object*); @@ -607,27 +597,27 @@ static lean_object* l_Lean_Elab_Command_instInhabitedState___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommandTopLevel(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___closed__3; lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__3; lean_object* l_Lean_profileitIOUnsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__1; -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getMainModule___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadCommandElabM___closed__4; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Elab_Command_expandDeclId___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_State_ngen___default___closed__2; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedCommandElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); extern lean_object* l_Lean_Expr_instBEqExpr; lean_object* l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabBinders___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_getBracketedBinderIds___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instMonadTraceCommandElabM___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_instAddMessageContextCommandElabM; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandDeclId___spec__5___closed__6; @@ -640,8 +630,10 @@ LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Comm lean_object* l_ReaderT_instMonadReaderT___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_State_traceState___default; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__3___rarg___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Command_expandDeclId___spec__7___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommandTopLevel___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedCommandElabM___closed__2; LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_Elab_Command_runLinters___spec__5___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -659,6 +651,7 @@ lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoB static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__7; static lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___closed__4; static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__9; +static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__4(lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldl___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Command_expandDeclId___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -669,7 +662,6 @@ LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentA static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__4___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_State_nextMacroScope___default; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); @@ -677,18 +669,20 @@ uint8_t l_Lean_Elab_isFreshInstanceName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instAddErrorMessageContextCommandElabM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadRecDepthCommandElabM; static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__12; +LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__2; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__1___closed__1; lean_object* l_Std_instInhabitedPersistentArrayNode(lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4; lean_object* l_Lean_TagDeclarationExtension_tag(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint32_t lean_uint32_of_nat(lean_object*); static lean_object* l_Lean_Elab_Command_instMonadLogCommandElabM___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_getScopes___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_State_infoState___default; @@ -702,12 +696,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadCommandElabM___lambda__1(l LEAN_EXPORT lean_object* l_Lean_Elab_Command_mkMessageAux(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_Elab_Command_elabCommandTopLevel___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Command_liftTermElabM___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_liftTermElabM___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_liftExcept___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__8___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__1; lean_object* l_Lean_Name_replacePrefix(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_liftTermElabM___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_Elab_Command_getBracketedBinderIds___closed__8; static lean_object* l_Lean_Elab_Command_instInhabitedScope___closed__2; @@ -724,12 +719,15 @@ LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Comm LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabCommand___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec__1(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13(lean_object*, lean_object*); static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Command_expandDeclId___spec__2___lambda__1___closed__2; static lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__1; static lean_object* l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__11; static lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadLiftTIOCommandElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_instInhabitedScope___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwAlreadyDeclaredUniverseLevel___at_Lean_Elab_Command_addUnivLevel___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -750,6 +748,7 @@ static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErro LEAN_EXPORT lean_object* l_Lean_Elab_Command_getRef___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_instMonadMacroAdapterCommandElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__3___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommandTopLevel___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2237____closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Command_0__Lean_Elab_Command_mkTermContext___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -9962,7 +9961,70 @@ x_4 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___ return x_4; } } -LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_withLogging___spec__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____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_Command___hyg_2261____closed__1; +x_2 = l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__18; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__2; +x_3 = l_Lean_registerTraceClass(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_maxRecDepthErrorMessage; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__2; +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_1); +lean_ctor_set(x_6, 1, x_5); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_339; uint8_t x_340; @@ -10989,7 +11051,7 @@ return x_337; } } } -LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; @@ -10999,14 +11061,14 @@ lean_inc(x_7); x_8 = lean_ctor_get(x_6, 1); lean_inc(x_8); lean_dec(x_6); -x_9 = l_Lean_logAt___at_Lean_Elab_Command_withLogging___spec__2(x_7, x_1, x_2, x_3, x_4, x_8); +x_9 = l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(x_7, x_1, x_2, x_3, x_4, x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_7); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_withLogging___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 0) @@ -11018,7 +11080,7 @@ x_6 = lean_ctor_get(x_1, 1); lean_inc(x_6); lean_dec(x_1); x_7 = 2; -x_8 = l_Lean_logAt___at_Lean_Elab_Command_withLogging___spec__2(x_5, x_6, x_7, x_2, x_3, x_4); +x_8 = l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(x_5, x_6, x_7, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_5); @@ -11060,7 +11122,7 @@ x_20 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); x_21 = 2; -x_22 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_20, x_21, x_2, x_3, x_15); +x_22 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_20, x_21, x_2, x_3, x_15); return x_22; } else @@ -11157,7 +11219,7 @@ x_47 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_46); x_48 = 2; -x_49 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_47, x_48, x_2, x_3, x_42); +x_49 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_47, x_48, x_2, x_3, x_42); return x_49; } else @@ -11213,24 +11275,7 @@ return x_60; } } } -static lean_object* _init_l_Lean_Elab_Command_withLogging___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("internal exception ", 19); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_withLogging___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_withLogging___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_withLogging(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; @@ -11245,404 +11290,18 @@ return x_5; } else { -lean_object* x_6; +lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = lean_ctor_get(x_5, 0); lean_inc(x_6); -if (lean_obj_tag(x_6) == 0) -{ -lean_object* x_7; lean_object* x_8; x_7 = lean_ctor_get(x_5, 1); lean_inc(x_7); lean_dec(x_5); -x_8 = l_Lean_Elab_logException___at_Lean_Elab_Command_withLogging___spec__1(x_6, x_2, x_3, x_7); +x_8 = l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(x_6, x_2, x_3, x_7); return x_8; } -else -{ -uint8_t x_9; -x_9 = !lean_is_exclusive(x_5); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_5, 1); -x_11 = lean_ctor_get(x_5, 0); -lean_dec(x_11); -x_12 = !lean_is_exclusive(x_6); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = lean_ctor_get(x_6, 0); -x_14 = lean_ctor_get(x_6, 1); -lean_dec(x_14); -x_15 = l_Lean_Elab_isAbortExceptionId(x_13); -if (x_15 == 0) -{ -lean_object* x_16; -lean_free_object(x_5); -x_16 = l_Lean_InternalExceptionId_getName(x_13, x_10); -lean_dec(x_13); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; -lean_free_object(x_6); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_19, 0, x_17); -x_20 = l_Lean_Elab_Command_withLogging___closed__2; -x_21 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___closed__3; -x_23 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -x_24 = 2; -x_25 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_23, x_24, x_2, x_3, x_18); -return x_25; } -else -{ -uint8_t x_26; -lean_dec(x_3); -x_26 = !lean_is_exclusive(x_16); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_27 = lean_ctor_get(x_16, 0); -x_28 = lean_ctor_get(x_2, 6); -lean_inc(x_28); -lean_dec(x_2); -x_29 = lean_io_error_to_string(x_27); -x_30 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_30, 0, x_29); -x_31 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 1, x_31); -lean_ctor_set(x_6, 0, x_28); -lean_ctor_set(x_16, 0, x_6); -return x_16; } -else -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_32 = lean_ctor_get(x_16, 0); -x_33 = lean_ctor_get(x_16, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_16); -x_34 = lean_ctor_get(x_2, 6); -lean_inc(x_34); -lean_dec(x_2); -x_35 = lean_io_error_to_string(x_32); -x_36 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_36, 0, x_35); -x_37 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 1, x_37); -lean_ctor_set(x_6, 0, x_34); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_6); -lean_ctor_set(x_38, 1, x_33); -return x_38; -} -} -} -else -{ -lean_object* x_39; -lean_free_object(x_6); -lean_dec(x_13); -lean_dec(x_3); -lean_dec(x_2); -x_39 = lean_box(0); -lean_ctor_set_tag(x_5, 0); -lean_ctor_set(x_5, 0, x_39); -return x_5; -} -} -else -{ -lean_object* x_40; uint8_t x_41; -x_40 = lean_ctor_get(x_6, 0); -lean_inc(x_40); -lean_dec(x_6); -x_41 = l_Lean_Elab_isAbortExceptionId(x_40); -if (x_41 == 0) -{ -lean_object* x_42; -lean_free_object(x_5); -x_42 = l_Lean_InternalExceptionId_getName(x_40, x_10); -lean_dec(x_40); -if (lean_obj_tag(x_42) == 0) -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_45, 0, x_43); -x_46 = l_Lean_Elab_Command_withLogging___closed__2; -x_47 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_45); -x_48 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___closed__3; -x_49 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); -x_50 = 2; -x_51 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_49, x_50, x_2, x_3, x_44); -return x_51; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -lean_dec(x_3); -x_52 = lean_ctor_get(x_42, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_42, 1); -lean_inc(x_53); -if (lean_is_exclusive(x_42)) { - lean_ctor_release(x_42, 0); - lean_ctor_release(x_42, 1); - x_54 = x_42; -} else { - lean_dec_ref(x_42); - x_54 = lean_box(0); -} -x_55 = lean_ctor_get(x_2, 6); -lean_inc(x_55); -lean_dec(x_2); -x_56 = lean_io_error_to_string(x_52); -x_57 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_57, 0, x_56); -x_58 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_58, 0, x_57); -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_55); -lean_ctor_set(x_59, 1, x_58); -if (lean_is_scalar(x_54)) { - x_60 = lean_alloc_ctor(1, 2, 0); -} else { - x_60 = x_54; -} -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_53); -return x_60; -} -} -else -{ -lean_object* x_61; -lean_dec(x_40); -lean_dec(x_3); -lean_dec(x_2); -x_61 = lean_box(0); -lean_ctor_set_tag(x_5, 0); -lean_ctor_set(x_5, 0, x_61); -return x_5; -} -} -} -else -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; -x_62 = lean_ctor_get(x_5, 1); -lean_inc(x_62); -lean_dec(x_5); -x_63 = lean_ctor_get(x_6, 0); -lean_inc(x_63); -if (lean_is_exclusive(x_6)) { - lean_ctor_release(x_6, 0); - lean_ctor_release(x_6, 1); - x_64 = x_6; -} else { - lean_dec_ref(x_6); - x_64 = lean_box(0); -} -x_65 = l_Lean_Elab_isAbortExceptionId(x_63); -if (x_65 == 0) -{ -lean_object* x_66; -x_66 = l_Lean_InternalExceptionId_getName(x_63, x_62); -lean_dec(x_63); -if (lean_obj_tag(x_66) == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; lean_object* x_75; -lean_dec(x_64); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_69, 0, x_67); -x_70 = l_Lean_Elab_Command_withLogging___closed__2; -x_71 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_69); -x_72 = l_Lean_Elab_logException___at_Lean_Elab_Command_runLinters___spec__1___closed__3; -x_73 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -x_74 = 2; -x_75 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_73, x_74, x_2, x_3, x_68); -return x_75; -} -else -{ -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -lean_dec(x_3); -x_76 = lean_ctor_get(x_66, 0); -lean_inc(x_76); -x_77 = lean_ctor_get(x_66, 1); -lean_inc(x_77); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - x_78 = x_66; -} else { - lean_dec_ref(x_66); - x_78 = lean_box(0); -} -x_79 = lean_ctor_get(x_2, 6); -lean_inc(x_79); -lean_dec(x_2); -x_80 = lean_io_error_to_string(x_76); -x_81 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_81, 0, x_80); -x_82 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_82, 0, x_81); -if (lean_is_scalar(x_64)) { - x_83 = lean_alloc_ctor(0, 2, 0); -} else { - x_83 = x_64; - lean_ctor_set_tag(x_83, 0); -} -lean_ctor_set(x_83, 0, x_79); -lean_ctor_set(x_83, 1, x_82); -if (lean_is_scalar(x_78)) { - x_84 = lean_alloc_ctor(1, 2, 0); -} else { - x_84 = x_78; -} -lean_ctor_set(x_84, 0, x_83); -lean_ctor_set(x_84, 1, x_77); -return x_84; -} -} -else -{ -lean_object* x_85; lean_object* x_86; -lean_dec(x_64); -lean_dec(x_63); -lean_dec(x_3); -lean_dec(x_2); -x_85 = lean_box(0); -x_86 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_86, 0, x_85); -lean_ctor_set(x_86, 1, x_62); -return x_86; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_withLogging___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 = lean_unbox(x_3); -lean_dec(x_3); -x_8 = l_Lean_logAt___at_Lean_Elab_Command_withLogging___spec__2(x_1, x_2, x_7, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; lean_object* x_7; -x_6 = lean_unbox(x_2); -lean_dec(x_2); -x_7 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_1, x_6, x_3, x_4, x_5); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__3; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____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_Command___hyg_2360____closed__1; -x_2 = l_Lean_Elab_Command_mkCommandElabAttributeUnsafe___closed__18; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__2; -x_3 = l_Lean_registerTraceClass(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_maxRecDepthErrorMessage; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__1; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__2; -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -x_7 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_4); -return x_7; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; uint8_t x_6; @@ -11694,7 +11353,7 @@ return x_22; } } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__1() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__1() { _start: { lean_object* x_1; @@ -11702,17 +11361,17 @@ x_1 = lean_mk_string_from_bytes("_traceMsg", 9); return x_1; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__1; +x_2 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__3() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__3() { _start: { lean_object* x_1; @@ -11720,16 +11379,16 @@ x_1 = lean_mk_string_from_bytes("[", 1); return x_1; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__3; +x_1 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__5() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__5() { _start: { lean_object* x_1; @@ -11737,16 +11396,16 @@ x_1 = lean_mk_string_from_bytes("] ", 2); return x_1; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__5; +x_1 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; @@ -11782,15 +11441,15 @@ if (x_19 == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; x_20 = lean_ctor_get(x_15, 0); -x_21 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2; +x_21 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2; x_22 = l_Lean_Name_append(x_1, x_21); x_23 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_23, 0, x_1); -x_24 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4; +x_24 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4; x_25 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_23); -x_26 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6; +x_26 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6; x_27 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_27, 0, x_25); lean_ctor_set(x_27, 1, x_26); @@ -11840,15 +11499,15 @@ x_41 = lean_ctor_get_uint8(x_15, sizeof(void*)*1); x_42 = lean_ctor_get(x_15, 0); lean_inc(x_42); lean_dec(x_15); -x_43 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2; +x_43 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2; x_44 = l_Lean_Name_append(x_1, x_43); x_45 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_45, 0, x_1); -x_46 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4; +x_46 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4; x_47 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_47, 0, x_46); lean_ctor_set(x_47, 1, x_45); -x_48 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6; +x_48 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6; x_49 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_49, 0, x_47); lean_ctor_set(x_49, 1, x_48); @@ -11922,15 +11581,15 @@ if (lean_is_exclusive(x_15)) { lean_dec_ref(x_15); x_72 = lean_box(0); } -x_73 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2; +x_73 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2; x_74 = l_Lean_Name_append(x_1, x_73); x_75 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_75, 0, x_1); -x_76 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4; +x_76 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4; x_77 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_77, 0, x_76); lean_ctor_set(x_77, 1, x_75); -x_78 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6; +x_78 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6; x_79 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_79, 0, x_77); lean_ctor_set(x_79, 1, x_78); @@ -11988,7 +11647,7 @@ return x_92; } } } -LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 0) @@ -12040,7 +11699,7 @@ x_17 = lean_ctor_get(x_11, 1); lean_inc(x_17); lean_dec(x_11); lean_inc(x_9); -x_18 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(x_9, x_2, x_3, x_17); +x_18 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(x_9, x_2, x_3, x_17); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); x_20 = lean_unbox(x_19); @@ -12067,7 +11726,7 @@ x_24 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_24, 0, x_10); x_25 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_25, 0, x_24); -x_26 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4(x_9, x_25, x_2, x_3, x_23); +x_26 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8(x_9, x_25, x_2, x_3, x_23); x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); lean_dec(x_26); @@ -12079,7 +11738,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; @@ -12133,7 +11792,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; @@ -12153,7 +11812,7 @@ lean_object* x_11; lean_object* x_12; x_11 = lean_ctor_get(x_3, 6); lean_dec(x_11); lean_ctor_set(x_3, 6, x_9); -x_12 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__7(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__11(x_2, x_3, x_4, x_8); lean_dec(x_4); return x_12; } @@ -12184,13 +11843,13 @@ lean_ctor_set(x_20, 4, x_17); lean_ctor_set(x_20, 5, x_18); lean_ctor_set(x_20, 6, x_9); lean_ctor_set(x_20, 7, x_19); -x_21 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__7(x_2, x_20, x_4, x_8); +x_21 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__11(x_2, x_20, x_4, x_8); lean_dec(x_4); return x_21; } } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__12(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; @@ -12204,7 +11863,7 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg___closed__1() { +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -12216,26 +11875,26 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg___closed__1; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg___closed__1; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg), 1, 0); +x_3 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg), 1, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___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; @@ -12404,7 +12063,7 @@ return x_41; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; lean_object* x_7; @@ -12416,7 +12075,7 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; @@ -12427,7 +12086,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; @@ -12438,7 +12097,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_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; @@ -12470,23 +12129,23 @@ x_16 = lean_ctor_get(x_14, 3); lean_inc(x_16); lean_dec(x_14); lean_inc(x_8); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__1___boxed), 4, 1); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__1___boxed), 4, 1); lean_closure_set(x_17, 0, x_8); lean_inc(x_12); x_18 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed), 3, 1); lean_closure_set(x_18, 0, x_12); lean_inc(x_8); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__2___boxed), 4, 1); +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__2___boxed), 4, 1); lean_closure_set(x_19, 0, x_8); lean_inc(x_16); lean_inc(x_12); lean_inc(x_8); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__3___boxed), 6, 3); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__3___boxed), 6, 3); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_12); lean_closure_set(x_20, 2, x_16); lean_inc(x_8); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__4___boxed), 6, 3); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4___boxed), 6, 3); lean_closure_set(x_21, 0, x_8); lean_closure_set(x_21, 1, x_12); lean_closure_set(x_21, 2, x_16); @@ -12572,7 +12231,7 @@ x_53 = lean_ctor_get(x_44, 1); lean_inc(x_53); lean_dec(x_44); x_54 = l_List_reverse___rarg(x_53); -x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_54, x_2, x_3, x_52); +x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_54, x_2, x_3, x_52); lean_dec(x_3); lean_dec(x_2); x_56 = !lean_is_exclusive(x_55); @@ -12634,7 +12293,7 @@ x_71 = lean_ctor_get(x_44, 1); lean_inc(x_71); lean_dec(x_44); x_72 = l_List_reverse___rarg(x_71); -x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_2, x_3, x_70); +x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_72, x_2, x_3, x_70); lean_dec(x_3); lean_dec(x_2); x_74 = lean_ctor_get(x_73, 1); @@ -12680,14 +12339,14 @@ x_82 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_82, 0, x_79); x_83 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_83, 0, x_82); -x_84 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__6(x_78, x_83, x_2, x_3, x_36); +x_84 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__10(x_78, x_83, x_2, x_3, x_36); return x_84; } else { lean_object* x_85; lean_dec(x_79); -x_85 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__8(x_78, x_2, x_3, x_36); +x_85 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__12(x_78, x_2, x_3, x_36); lean_dec(x_3); lean_dec(x_2); return x_85; @@ -12698,13 +12357,13 @@ else lean_object* x_86; lean_dec(x_3); lean_dec(x_2); -x_86 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg(x_36); +x_86 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg(x_36); return x_86; } } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; @@ -12758,7 +12417,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; @@ -12778,7 +12437,7 @@ lean_object* x_11; lean_object* x_12; x_11 = lean_ctor_get(x_3, 6); lean_dec(x_11); lean_ctor_set(x_3, 6, x_9); -x_12 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12(x_2, x_3, x_4, x_8); +x_12 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16(x_2, x_3, x_4, x_8); lean_dec(x_4); return x_12; } @@ -12809,13 +12468,13 @@ lean_ctor_set(x_20, 4, x_17); lean_ctor_set(x_20, 5, x_18); lean_ctor_set(x_20, 6, x_9); lean_ctor_set(x_20, 7, x_19); -x_21 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12(x_2, x_20, x_4, x_8); +x_21 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16(x_2, x_20, x_4, x_8); lean_dec(x_4); return x_21; } } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__17(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; @@ -12829,26 +12488,26 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg___closed__1; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg___closed__1; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg), 1, 0); +x_3 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg), 1, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; 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; @@ -12880,23 +12539,23 @@ x_16 = lean_ctor_get(x_14, 3); lean_inc(x_16); lean_dec(x_14); lean_inc(x_8); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__1___boxed), 4, 1); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__1___boxed), 4, 1); lean_closure_set(x_17, 0, x_8); lean_inc(x_12); x_18 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed), 3, 1); lean_closure_set(x_18, 0, x_12); lean_inc(x_8); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__2___boxed), 4, 1); +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__2___boxed), 4, 1); lean_closure_set(x_19, 0, x_8); lean_inc(x_16); lean_inc(x_12); lean_inc(x_8); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__3___boxed), 6, 3); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__3___boxed), 6, 3); lean_closure_set(x_20, 0, x_8); lean_closure_set(x_20, 1, x_12); lean_closure_set(x_20, 2, x_16); lean_inc(x_8); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__4___boxed), 6, 3); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4___boxed), 6, 3); lean_closure_set(x_21, 0, x_8); lean_closure_set(x_21, 1, x_12); lean_closure_set(x_21, 2, x_16); @@ -12982,7 +12641,7 @@ x_53 = lean_ctor_get(x_44, 1); lean_inc(x_53); lean_dec(x_44); x_54 = l_List_reverse___rarg(x_53); -x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_54, x_2, x_3, x_52); +x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_54, x_2, x_3, x_52); lean_dec(x_3); lean_dec(x_2); x_56 = !lean_is_exclusive(x_55); @@ -13044,7 +12703,7 @@ x_71 = lean_ctor_get(x_44, 1); lean_inc(x_71); lean_dec(x_44); x_72 = l_List_reverse___rarg(x_71); -x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_2, x_3, x_70); +x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_72, x_2, x_3, x_70); lean_dec(x_3); lean_dec(x_2); x_74 = lean_ctor_get(x_73, 1); @@ -13090,14 +12749,14 @@ x_82 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_82, 0, x_79); x_83 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_83, 0, x_82); -x_84 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__11(x_78, x_83, x_2, x_3, x_36); +x_84 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__15(x_78, x_83, x_2, x_3, x_36); return x_84; } else { lean_object* x_85; lean_dec(x_79); -x_85 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__13(x_78, x_2, x_3, x_36); +x_85 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__17(x_78, x_2, x_3, x_36); lean_dec(x_3); lean_dec(x_2); return x_85; @@ -13108,24 +12767,24 @@ else lean_object* x_86; lean_dec(x_3); lean_dec(x_2); -x_86 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_36); +x_86 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_36); return x_86; } } } } -LEAN_EXPORT lean_object* l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_inc(x_1); x_6 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_6, 0, x_1); -x_7 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4; +x_7 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4; x_8 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_8, 0, x_7); lean_ctor_set(x_8, 1, x_6); -x_9 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6; +x_9 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6; x_10 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_10, 0, x_8); lean_ctor_set(x_10, 1, x_9); @@ -13140,11 +12799,11 @@ x_14 = lean_alloc_ctor(11, 2, 0); lean_ctor_set(x_14, 0, x_1); lean_ctor_set(x_14, 1, x_13); x_15 = 0; -x_16 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_14, x_15, x_3, x_4, x_5); +x_16 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_14, x_15, x_3, x_4, x_5); return x_16; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -13395,7 +13054,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommand___lambda__2(lean_object lean_object* x_6; lean_inc(x_4); lean_inc(x_3); -x_6 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(x_1, x_3, x_4, x_5); +x_6 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(x_1, x_3, x_4, x_5); if (lean_obj_tag(x_6) == 0) { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; @@ -13515,7 +13174,7 @@ x_49 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_49, 0, x_1); lean_inc(x_5); lean_inc(x_4); -x_50 = l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__15(x_3, x_49, x_4, x_5, x_43); +x_50 = l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__19(x_3, x_49, x_4, x_5, x_43); x_51 = lean_ctor_get(x_50, 1); lean_inc(x_51); lean_dec(x_50); @@ -13540,7 +13199,7 @@ lean_closure_set(x_12, 0, x_11); lean_closure_set(x_12, 1, x_1); lean_inc(x_5); lean_inc(x_4); -x_13 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2(x_12, x_4, x_5, x_10); +x_13 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6(x_12, x_4, x_5, x_10); if (lean_obj_tag(x_13) == 0) { lean_object* x_14; @@ -13736,7 +13395,7 @@ if (x_8 == 0) { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_dec(x_6); -x_9 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__2; +x_9 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__2; lean_inc(x_1); x_10 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___lambda__3), 6, 3); lean_closure_set(x_10, 0, x_1); @@ -13745,7 +13404,7 @@ lean_closure_set(x_10, 2, x_9); x_11 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___lambda__1), 5, 2); lean_closure_set(x_11, 0, x_1); lean_closure_set(x_11, 1, x_10); -x_12 = l_Lean_Elab_Command_withLogging(x_11, x_2, x_3, x_4); +x_12 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_11, x_2, x_3, x_4); return x_12; } else @@ -13764,7 +13423,7 @@ x_16 = l_Lean_Elab_Command_elabCommand___closed__6; x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___lambda__1), 5, 2); lean_closure_set(x_17, 0, x_1); lean_closure_set(x_17, 1, x_16); -x_18 = l_Lean_Elab_Command_withLogging(x_17, x_2, x_3, x_4); +x_18 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_17, x_2, x_3, x_4); return x_18; } else @@ -13780,7 +13439,7 @@ x_20 = l_Lean_Elab_Command_elabCommand___closed__6; x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___lambda__1), 5, 2); lean_closure_set(x_21, 0, x_1); lean_closure_set(x_21, 1, x_20); -x_22 = l_Lean_Elab_Command_withLogging(x_21, x_2, x_3, x_4); +x_22 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_21, x_2, x_3, x_4); return x_22; } else @@ -13791,7 +13450,7 @@ lean_dec(x_13); x_24 = lean_box(0); x_25 = l_Lean_Elab_Command_elabCommand___boxed__const__1; x_26 = lean_box_usize(x_23); -x_27 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16___boxed), 7, 4); +x_27 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20___boxed), 7, 4); lean_closure_set(x_27, 0, x_6); lean_closure_set(x_27, 1, x_25); lean_closure_set(x_27, 2, x_26); @@ -13799,7 +13458,7 @@ lean_closure_set(x_27, 3, x_24); x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___lambda__1), 5, 2); lean_closure_set(x_28, 0, x_1); lean_closure_set(x_28, 1, x_27); -x_29 = l_Lean_Elab_Command_withLogging(x_28, x_2, x_3, x_4); +x_29 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_28, x_2, x_3, x_4); return x_29; } } @@ -13812,7 +13471,7 @@ x_30 = l_Lean_Elab_Command_elabCommand___closed__3; x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand___lambda__1), 5, 2); lean_closure_set(x_31, 0, x_1); lean_closure_set(x_31, 1, x_30); -x_32 = l_Lean_Elab_Command_withLogging(x_31, x_2, x_3, x_4); +x_32 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_31, x_2, x_3, x_4); return x_32; } } @@ -13827,132 +13486,155 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; +x_7 = lean_unbox(x_3); +lean_dec(x_3); +x_8 = l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(x_1, x_2, x_7, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; lean_object* x_7; +x_6 = lean_unbox(x_2); +lean_dec(x_2); +x_7 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_1, x_6, x_3, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(x_1, x_2, x_3, x_4); +x_5 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); return x_6; } } -LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_1, x_2, x_3, x_4); +x_5 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__7(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__11(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__8(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__12(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9(x_1, x_2); +x_3 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__2(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__2___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__6___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__13(x_1, x_2, x_3, x_4); +x_5 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__17(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14(x_1, x_2); +x_3 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18(x_1, x_2); lean_dec(x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -13960,7 +13642,7 @@ x_8 = lean_unbox_usize(x_2); lean_dec(x_2); x_9 = lean_unbox_usize(x_3); lean_dec(x_3); -x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_1, x_8, x_9, x_4, x_5, x_6, x_7); lean_dec(x_1); return x_10; } @@ -13975,7 +13657,7 @@ lean_dec(x_1); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__1() { _start: { lean_object* x_1; @@ -13983,21 +13665,21 @@ x_1 = lean_mk_string_from_bytes("input", 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__2() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____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_Command___hyg_2360____closed__1; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__1; +x_1 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__2; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__2; x_3 = l_Lean_registerTraceClass(x_2, x_1); return x_3; } @@ -14086,15 +13768,15 @@ if (x_19 == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; x_20 = lean_ctor_get(x_15, 0); -x_21 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2; +x_21 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2; x_22 = l_Lean_Name_append(x_1, x_21); x_23 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_23, 0, x_1); -x_24 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4; +x_24 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4; x_25 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_23); -x_26 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6; +x_26 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6; x_27 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_27, 0, x_25); lean_ctor_set(x_27, 1, x_26); @@ -14144,15 +13826,15 @@ x_41 = lean_ctor_get_uint8(x_15, sizeof(void*)*1); x_42 = lean_ctor_get(x_15, 0); lean_inc(x_42); lean_dec(x_15); -x_43 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2; +x_43 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2; x_44 = l_Lean_Name_append(x_1, x_43); x_45 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_45, 0, x_1); -x_46 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4; +x_46 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4; x_47 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_47, 0, x_46); lean_ctor_set(x_47, 1, x_45); -x_48 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6; +x_48 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6; x_49 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_49, 0, x_47); lean_ctor_set(x_49, 1, x_48); @@ -14226,15 +13908,15 @@ if (lean_is_exclusive(x_15)) { lean_dec_ref(x_15); x_72 = lean_box(0); } -x_73 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2; +x_73 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2; x_74 = l_Lean_Name_append(x_1, x_73); x_75 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_75, 0, x_1); -x_76 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4; +x_76 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4; x_77 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_77, 0, x_76); lean_ctor_set(x_77, 1, x_75); -x_78 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6; +x_78 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6; x_79 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_79, 0, x_77); lean_ctor_set(x_79, 1, x_78); @@ -14579,7 +14261,7 @@ x_65 = lean_ctor_get(x_59, 1); lean_inc(x_65); lean_dec(x_59); lean_inc(x_31); -x_66 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(x_31, x_7, x_8, x_65); +x_66 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(x_31, x_7, x_8, x_65); x_67 = lean_ctor_get(x_66, 0); lean_inc(x_67); x_68 = lean_ctor_get(x_66, 1); @@ -14999,7 +14681,7 @@ x_65 = lean_ctor_get(x_59, 1); lean_inc(x_65); lean_dec(x_59); lean_inc(x_31); -x_66 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(x_31, x_7, x_8, x_65); +x_66 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(x_31, x_7, x_8, x_65); x_67 = lean_ctor_get(x_66, 0); lean_inc(x_67); x_68 = lean_ctor_get(x_66, 1); @@ -15441,7 +15123,7 @@ x_7 = lean_name_eq(x_2, x_6); if (x_7 == 0) { lean_object* x_8; uint8_t x_9; -x_8 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2; +x_8 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2; x_9 = l_Lean_Name_isSuffixOf(x_8, x_2); return x_9; } @@ -16363,7 +16045,7 @@ x_20 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); lean_closure_set(x_20, 0, x_1); lean_inc(x_5); lean_inc(x_4); -x_21 = l_Lean_Elab_Command_withLogging(x_20, x_4, x_5, x_19); +x_21 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_20, x_4, x_5, x_19); if (lean_obj_tag(x_21) == 0) { lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; @@ -16564,7 +16246,7 @@ x_75 = lean_alloc_closure((void*)(l_Lean_Elab_Command_runLinters), 4, 1); lean_closure_set(x_75, 0, x_1); lean_inc(x_5); lean_inc(x_4); -x_76 = l_Lean_Elab_Command_withLogging(x_75, x_4, x_5, x_74); +x_76 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_75, x_4, x_5, x_74); if (lean_obj_tag(x_76) == 0) { lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; @@ -16717,7 +16399,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabCommandTopLevel(lean_object* x_ _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; -x_5 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__2; +x_5 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__2; x_6 = l_Lean_Elab_Command_getRef(x_2, x_3, x_4); x_7 = lean_ctor_get(x_6, 0); lean_inc(x_7); @@ -16758,7 +16440,7 @@ lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint x_30 = lean_ctor_get(x_24, 1); lean_inc(x_30); lean_dec(x_24); -x_31 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(x_5, x_2, x_3, x_30); +x_31 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(x_5, x_2, x_3, x_30); x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); x_33 = lean_ctor_get(x_31, 1); @@ -16775,7 +16457,7 @@ goto block_23; if (x_12 == 0) { lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1; +x_14 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1; x_15 = lean_box(0); x_16 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__2(x_1, x_14, x_15, x_2, x_3, x_13); return x_16; @@ -16786,13 +16468,13 @@ lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean lean_inc(x_1); x_17 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_17, 0, x_1); -x_18 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4(x_5, x_17, x_2, x_3, x_13); +x_18 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8(x_5, x_17, x_2, x_3, x_13); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); lean_inc(x_20); lean_dec(x_18); -x_21 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1; +x_21 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1; x_22 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__2(x_1, x_21, x_19, x_2, x_3, x_20); return x_22; } @@ -16850,7 +16532,7 @@ lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint x_61 = lean_ctor_get(x_55, 1); lean_inc(x_61); lean_dec(x_55); -x_62 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(x_5, x_42, x_3, x_61); +x_62 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(x_5, x_42, x_3, x_61); x_63 = lean_ctor_get(x_62, 0); lean_inc(x_63); x_64 = lean_ctor_get(x_62, 1); @@ -16867,7 +16549,7 @@ goto block_54; if (x_43 == 0) { lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1; +x_45 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1; x_46 = lean_box(0); x_47 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__2(x_1, x_45, x_46, x_42, x_3, x_44); return x_47; @@ -16878,13 +16560,13 @@ lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean lean_inc(x_1); x_48 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_48, 0, x_1); -x_49 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4(x_5, x_48, x_42, x_3, x_44); +x_49 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8(x_5, x_48, x_42, x_3, x_44); x_50 = lean_ctor_get(x_49, 0); lean_inc(x_50); x_51 = lean_ctor_get(x_49, 1); lean_inc(x_51); lean_dec(x_49); -x_52 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1; +x_52 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1; x_53 = l_Lean_Elab_Command_elabCommandTopLevel___lambda__2(x_1, x_52, x_50, x_42, x_3, x_51); return x_53; } @@ -18000,12 +17682,13 @@ x_11 = l_Lean_Elab_Command_State_messages___default___closed__3; lean_ctor_set(x_6, 1, x_11); lean_ctor_set(x_6, 0, x_10); lean_inc(x_3); -x_12 = lean_alloc_ctor(0, 5, 0); +x_12 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_12, 0, x_3); lean_ctor_set(x_12, 1, x_4); lean_ctor_set(x_12, 2, x_5); lean_ctor_set(x_12, 3, x_4); -lean_ctor_set(x_12, 4, x_6); +lean_ctor_set(x_12, 4, x_5); +lean_ctor_set(x_12, 5, x_6); return x_12; } else @@ -18020,12 +17703,13 @@ lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); lean_ctor_set_uint8(x_16, sizeof(void*)*2, x_13); lean_inc(x_3); -x_17 = lean_alloc_ctor(0, 5, 0); +x_17 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_17, 0, x_3); lean_ctor_set(x_17, 1, x_4); lean_ctor_set(x_17, 2, x_5); lean_ctor_set(x_17, 3, x_4); -lean_ctor_set(x_17, 4, x_16); +lean_ctor_set(x_17, 4, x_5); +lean_ctor_set(x_17, 5, x_16); return x_17; } } @@ -18794,7 +18478,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -18845,7 +18529,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 4); +x_29 = lean_ctor_get(x_27, 5); lean_inc(x_29); lean_dec(x_27); x_30 = lean_ctor_get(x_29, 1); @@ -18868,7 +18552,7 @@ lean_dec(x_34); x_36 = lean_st_ref_take(x_3, x_35); x_37 = lean_ctor_get(x_36, 0); lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 4); +x_38 = lean_ctor_get(x_37, 5); lean_inc(x_38); x_39 = lean_ctor_get(x_36, 1); lean_inc(x_39); @@ -18877,7 +18561,7 @@ x_40 = !lean_is_exclusive(x_37); if (x_40 == 0) { lean_object* x_41; uint8_t x_42; -x_41 = lean_ctor_get(x_37, 4); +x_41 = lean_ctor_get(x_37, 5); lean_dec(x_41); x_42 = !lean_is_exclusive(x_38); if (x_42 == 0) @@ -18922,7 +18606,7 @@ x_53 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_50); -lean_ctor_set(x_37, 4, x_53); +lean_ctor_set(x_37, 5, x_53); x_54 = lean_st_ref_set(x_3, x_37, x_39); lean_dec(x_3); x_55 = lean_ctor_get(x_54, 1); @@ -18947,243 +18631,249 @@ return x_57; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_58 = lean_ctor_get(x_37, 0); x_59 = lean_ctor_get(x_37, 1); x_60 = lean_ctor_get(x_37, 2); x_61 = lean_ctor_get(x_37, 3); +x_62 = lean_ctor_get(x_37, 4); +lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); lean_inc(x_58); lean_dec(x_37); -x_62 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); +x_63 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); +x_64 = lean_ctor_get(x_38, 0); +lean_inc(x_64); if (lean_is_exclusive(x_38)) { lean_ctor_release(x_38, 0); lean_ctor_release(x_38, 1); - x_64 = x_38; + x_65 = x_38; } else { lean_dec_ref(x_38); - x_64 = lean_box(0); + x_65 = lean_box(0); } -x_65 = l_Std_PersistentArray_append___rarg(x_19, x_32); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(0, 2, 1); +x_66 = l_Std_PersistentArray_append___rarg(x_19, x_32); +if (lean_is_scalar(x_65)) { + x_67 = lean_alloc_ctor(0, 2, 1); } else { - x_66 = x_64; -} -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_65); -lean_ctor_set_uint8(x_66, sizeof(void*)*2, x_62); -x_67 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_67, 0, x_58); -lean_ctor_set(x_67, 1, x_59); -lean_ctor_set(x_67, 2, x_60); -lean_ctor_set(x_67, 3, x_61); -lean_ctor_set(x_67, 4, x_66); -x_68 = lean_st_ref_set(x_3, x_67, x_39); + x_67 = x_65; +} +lean_ctor_set(x_67, 0, x_64); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_63); +x_68 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_68, 0, x_58); +lean_ctor_set(x_68, 1, x_59); +lean_ctor_set(x_68, 2, x_60); +lean_ctor_set(x_68, 3, x_61); +lean_ctor_set(x_68, 4, x_62); +lean_ctor_set(x_68, 5, x_67); +x_69 = lean_st_ref_set(x_3, x_68, x_39); lean_dec(x_3); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_70 = x_68; +x_70 = lean_ctor_get(x_69, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_71 = x_69; } else { - lean_dec_ref(x_68); - x_70 = lean_box(0); + lean_dec_ref(x_69); + x_71 = lean_box(0); } -if (lean_is_scalar(x_70)) { - x_71 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_70; + x_72 = x_71; } -lean_ctor_set(x_71, 0, x_22); -lean_ctor_set(x_71, 1, x_69); -return x_71; +lean_ctor_set(x_72, 0, x_22); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_72 = lean_ctor_get(x_21, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_21, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_73 = lean_ctor_get(x_21, 0); lean_inc(x_73); +x_74 = lean_ctor_get(x_21, 1); +lean_inc(x_74); lean_dec(x_21); -x_74 = lean_st_ref_get(x_7, x_73); -x_75 = lean_ctor_get(x_74, 1); -lean_inc(x_75); -lean_dec(x_74); -x_76 = lean_st_ref_get(x_3, x_75); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); +x_75 = lean_st_ref_get(x_7, x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_st_ref_get(x_3, x_76); +x_78 = lean_ctor_get(x_77, 0); lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_ctor_get(x_77, 4); +x_79 = lean_ctor_get(x_77, 1); lean_inc(x_79); lean_dec(x_77); -x_80 = lean_ctor_get(x_79, 1); +x_80 = lean_ctor_get(x_78, 5); lean_inc(x_80); -x_81 = l_Std_PersistentArray_mapM___at_Lean_Elab_Command_liftTermElabM___spec__7(x_79, x_80, x_2, x_3, x_4, x_5, x_6, x_7, x_78); +lean_dec(x_78); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +x_82 = l_Std_PersistentArray_mapM___at_Lean_Elab_Command_liftTermElabM___spec__7(x_80, x_81, x_2, x_3, x_4, x_5, x_6, x_7, x_79); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_st_ref_get(x_7, x_83); +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +lean_dec(x_82); +x_85 = lean_st_ref_get(x_7, x_84); lean_dec(x_7); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_3, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_87, 4); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_st_ref_take(x_3, x_86); +x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 1); +x_89 = lean_ctor_get(x_88, 5); lean_inc(x_89); -lean_dec(x_86); -x_90 = !lean_is_exclusive(x_87); -if (x_90 == 0) +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = !lean_is_exclusive(x_88); +if (x_91 == 0) { -lean_object* x_91; uint8_t x_92; -x_91 = lean_ctor_get(x_87, 4); -lean_dec(x_91); -x_92 = !lean_is_exclusive(x_88); -if (x_92 == 0) +lean_object* x_92; uint8_t x_93; +x_92 = lean_ctor_get(x_88, 5); +lean_dec(x_92); +x_93 = !lean_is_exclusive(x_89); +if (x_93 == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; -x_93 = lean_ctor_get(x_88, 1); -lean_dec(x_93); -x_94 = l_Std_PersistentArray_append___rarg(x_19, x_82); -lean_ctor_set(x_88, 1, x_94); -x_95 = lean_st_ref_set(x_3, x_87, x_89); +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_89, 1); +lean_dec(x_94); +x_95 = l_Std_PersistentArray_append___rarg(x_19, x_83); +lean_ctor_set(x_89, 1, x_95); +x_96 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) { -lean_object* x_97; -x_97 = lean_ctor_get(x_95, 0); -lean_dec(x_97); -lean_ctor_set_tag(x_95, 1); -lean_ctor_set(x_95, 0, x_72); -return x_95; +lean_object* x_98; +x_98 = lean_ctor_get(x_96, 0); +lean_dec(x_98); +lean_ctor_set_tag(x_96, 1); +lean_ctor_set(x_96, 0, x_73); +return x_96; } else { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_95, 1); -lean_inc(x_98); -lean_dec(x_95); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_72); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_dec(x_96); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_73); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_100 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_101 = lean_ctor_get(x_88, 0); -lean_inc(x_101); -lean_dec(x_88); -x_102 = l_Std_PersistentArray_append___rarg(x_19, x_82); -x_103 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_100); -lean_ctor_set(x_87, 4, x_103); -x_104 = lean_st_ref_set(x_3, x_87, x_89); +uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_101 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +lean_dec(x_89); +x_103 = l_Std_PersistentArray_append___rarg(x_19, x_83); +x_104 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set_uint8(x_104, sizeof(void*)*2, x_101); +lean_ctor_set(x_88, 5, x_104); +x_105 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_106 = x_104; +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; - lean_ctor_set_tag(x_107, 1); + x_108 = x_107; + lean_ctor_set_tag(x_108, 1); } -lean_ctor_set(x_107, 0, x_72); -lean_ctor_set(x_107, 1, x_105); -return x_107; +lean_ctor_set(x_108, 0, x_73); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_108 = lean_ctor_get(x_87, 0); -x_109 = lean_ctor_get(x_87, 1); -x_110 = lean_ctor_get(x_87, 2); -x_111 = lean_ctor_get(x_87, 3); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_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; +x_109 = lean_ctor_get(x_88, 0); +x_110 = lean_ctor_get(x_88, 1); +x_111 = lean_ctor_get(x_88, 2); +x_112 = lean_ctor_get(x_88, 3); +x_113 = lean_ctor_get(x_88, 4); +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_dec(x_87); -x_112 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_113 = lean_ctor_get(x_88, 0); -lean_inc(x_113); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_114 = x_88; +lean_dec(x_88); +x_114 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_115 = lean_ctor_get(x_89, 0); +lean_inc(x_115); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_116 = x_89; } else { - lean_dec_ref(x_88); - x_114 = lean_box(0); + lean_dec_ref(x_89); + x_116 = lean_box(0); } -x_115 = l_Std_PersistentArray_append___rarg(x_19, x_82); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 1); +x_117 = l_Std_PersistentArray_append___rarg(x_19, x_83); +if (lean_is_scalar(x_116)) { + x_118 = lean_alloc_ctor(0, 2, 1); } else { - x_116 = x_114; -} -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_115); -lean_ctor_set_uint8(x_116, sizeof(void*)*2, x_112); -x_117 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_117, 0, x_108); -lean_ctor_set(x_117, 1, x_109); -lean_ctor_set(x_117, 2, x_110); -lean_ctor_set(x_117, 3, x_111); -lean_ctor_set(x_117, 4, x_116); -x_118 = lean_st_ref_set(x_3, x_117, x_89); + x_118 = x_116; +} +lean_ctor_set(x_118, 0, x_115); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); +x_119 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_119, 0, x_109); +lean_ctor_set(x_119, 1, x_110); +lean_ctor_set(x_119, 2, x_111); +lean_ctor_set(x_119, 3, x_112); +lean_ctor_set(x_119, 4, x_113); +lean_ctor_set(x_119, 5, x_118); +x_120 = lean_st_ref_set(x_3, x_119, x_90); lean_dec(x_3); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_122 = x_120; } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + lean_dec_ref(x_120); + x_122 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); } else { - x_121 = x_120; - lean_ctor_set_tag(x_121, 1); + x_123 = x_122; + lean_ctor_set_tag(x_123, 1); } -lean_ctor_set(x_121, 0, x_72); -lean_ctor_set(x_121, 1, x_119); -return x_121; +lean_ctor_set(x_123, 0, x_73); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } @@ -19507,7 +19197,7 @@ if (x_64 == 0) { lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; x_65 = lean_ctor_get(x_58, 1); -x_66 = lean_ctor_get(x_47, 4); +x_66 = lean_ctor_get(x_47, 5); lean_inc(x_66); lean_dec(x_47); x_67 = lean_ctor_get(x_66, 1); @@ -19591,7 +19281,7 @@ x_84 = lean_ctor_get(x_58, 1); lean_inc(x_84); lean_inc(x_83); lean_dec(x_58); -x_85 = lean_ctor_get(x_47, 4); +x_85 = lean_ctor_get(x_47, 5); lean_inc(x_85); lean_dec(x_47); x_86 = lean_ctor_get(x_85, 1); @@ -19692,7 +19382,7 @@ if (lean_is_exclusive(x_102)) { lean_dec_ref(x_102); x_109 = lean_box(0); } -x_110 = lean_ctor_get(x_47, 4); +x_110 = lean_ctor_get(x_47, 5); lean_inc(x_110); lean_dec(x_47); x_111 = lean_ctor_get(x_110, 1); @@ -20379,7 +20069,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_catchExceptions(lean_object* x_1, l _start: { lean_object* x_5; -x_5 = l_Lean_Elab_Command_withLogging(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_1, x_2, x_3, x_4); if (lean_obj_tag(x_5) == 0) { uint8_t x_6; @@ -20555,7 +20245,7 @@ static lean_object* _init_l_Lean_Elab_Command_modifyScope___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Command_modifyScope___closed__1; x_2 = l_Lean_Elab_Command_modifyScope___closed__2; -x_3 = lean_unsigned_to_nat(428u); +x_3 = lean_unsigned_to_nat(416u); x_4 = lean_unsigned_to_nat(16u); x_5 = l_Lean_Elab_Command_modifyScope___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -23385,47 +23075,49 @@ lean_dec(x_6); x_9 = !lean_is_exclusive(x_7); if (x_9 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; x_10 = lean_ctor_get(x_7, 0); -x_11 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__11___closed__1; -x_12 = l_Lean_MapDeclarationExtension_insert___rarg(x_11, x_10, x_1, x_2); -lean_ctor_set(x_7, 0, x_12); -x_13 = lean_st_ref_set(x_4, x_7, x_8); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +x_11 = l___private_Lean_DocString_0__Lean_removeLeadingSpaces(x_2); +x_12 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__11___closed__1; +x_13 = l_Lean_MapDeclarationExtension_insert___rarg(x_12, x_10, x_1, x_11); +lean_ctor_set(x_7, 0, x_13); +x_14 = lean_st_ref_set(x_4, x_7, x_8); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_13, 0); -lean_dec(x_15); -x_16 = lean_box(0); -lean_ctor_set(x_13, 0, x_16); -return x_13; +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_14, 0); +lean_dec(x_16); +x_17 = lean_box(0); +lean_ctor_set(x_14, 0, x_17); +return x_14; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_13, 1); -lean_inc(x_17); -lean_dec(x_13); -x_18 = lean_box(0); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -return x_19; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; } } else { -lean_object* x_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; -x_20 = lean_ctor_get(x_7, 0); -x_21 = lean_ctor_get(x_7, 1); -x_22 = lean_ctor_get(x_7, 2); -x_23 = lean_ctor_get(x_7, 3); -x_24 = lean_ctor_get(x_7, 4); -x_25 = lean_ctor_get(x_7, 5); -x_26 = lean_ctor_get(x_7, 6); -x_27 = lean_ctor_get(x_7, 7); -x_28 = lean_ctor_get(x_7, 8); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_21 = lean_ctor_get(x_7, 0); +x_22 = lean_ctor_get(x_7, 1); +x_23 = lean_ctor_get(x_7, 2); +x_24 = lean_ctor_get(x_7, 3); +x_25 = lean_ctor_get(x_7, 4); +x_26 = lean_ctor_get(x_7, 5); +x_27 = lean_ctor_get(x_7, 6); +x_28 = lean_ctor_get(x_7, 7); +x_29 = lean_ctor_get(x_7, 8); +lean_inc(x_29); lean_inc(x_28); lean_inc(x_27); lean_inc(x_26); @@ -23434,40 +23126,40 @@ lean_inc(x_24); lean_inc(x_23); lean_inc(x_22); lean_inc(x_21); -lean_inc(x_20); lean_dec(x_7); -x_29 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__11___closed__1; -x_30 = l_Lean_MapDeclarationExtension_insert___rarg(x_29, x_20, x_1, x_2); -x_31 = lean_alloc_ctor(0, 9, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_21); -lean_ctor_set(x_31, 2, x_22); -lean_ctor_set(x_31, 3, x_23); -lean_ctor_set(x_31, 4, x_24); -lean_ctor_set(x_31, 5, x_25); -lean_ctor_set(x_31, 6, x_26); -lean_ctor_set(x_31, 7, x_27); -lean_ctor_set(x_31, 8, x_28); -x_32 = lean_st_ref_set(x_4, x_31, x_8); -x_33 = lean_ctor_get(x_32, 1); -lean_inc(x_33); -if (lean_is_exclusive(x_32)) { - lean_ctor_release(x_32, 0); - lean_ctor_release(x_32, 1); - x_34 = x_32; +x_30 = l___private_Lean_DocString_0__Lean_removeLeadingSpaces(x_2); +x_31 = l_Lean_addDocString___at_Lean_Elab_Command_expandDeclId___spec__11___closed__1; +x_32 = l_Lean_MapDeclarationExtension_insert___rarg(x_31, x_21, x_1, x_30); +x_33 = lean_alloc_ctor(0, 9, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_22); +lean_ctor_set(x_33, 2, x_23); +lean_ctor_set(x_33, 3, x_24); +lean_ctor_set(x_33, 4, x_25); +lean_ctor_set(x_33, 5, x_26); +lean_ctor_set(x_33, 6, x_27); +lean_ctor_set(x_33, 7, x_28); +lean_ctor_set(x_33, 8, x_29); +x_34 = lean_st_ref_set(x_4, x_33, x_8); +x_35 = lean_ctor_get(x_34, 1); +lean_inc(x_35); +if (lean_is_exclusive(x_34)) { + lean_ctor_release(x_34, 0); + lean_ctor_release(x_34, 1); + x_36 = x_34; } else { - lean_dec_ref(x_32); - x_34 = lean_box(0); + lean_dec_ref(x_34); + x_36 = lean_box(0); } -x_35 = lean_box(0); -if (lean_is_scalar(x_34)) { - x_36 = lean_alloc_ctor(0, 2, 0); +x_37 = lean_box(0); +if (lean_is_scalar(x_36)) { + x_38 = lean_alloc_ctor(0, 2, 0); } else { - x_36 = x_34; + x_38 = x_36; } -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_33); -return x_36; +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_35); +return x_38; } } } @@ -25105,35 +24797,31 @@ if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Command_showPartialSyntaxErrors = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Command_showPartialSyntaxErrors); lean_dec_ref(res); -}l_Lean_Elab_Command_withLogging___closed__1 = _init_l_Lean_Elab_Command_withLogging___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_withLogging___closed__1); -l_Lean_Elab_Command_withLogging___closed__2 = _init_l_Lean_Elab_Command_withLogging___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_withLogging___closed__2); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360____closed__2); -res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2360_(lean_io_mk_world()); +}l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261____closed__2); +res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2261_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__1(); lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__1); l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__2(); lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabCommand___spec__1___closed__2); -l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__1 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__1(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__1); -l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__2); -l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__3 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__3(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__3); -l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__4); -l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__5 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__5(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__5); -l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4___closed__6); -l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__9___rarg___closed__1); +l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__1 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__1(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__1); +l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__2); +l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__3 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__3(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__3); +l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__4); +l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__5 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__5(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__5); +l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6 = _init_l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8___closed__6); +l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__13___rarg___closed__1); l_Lean_Elab_Command_elabCommand___lambda__3___closed__1 = _init_l_Lean_Elab_Command_elabCommand___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabCommand___lambda__3___closed__1); l_Lean_Elab_Command_elabCommand___lambda__3___closed__2 = _init_l_Lean_Elab_Command_elabCommand___lambda__3___closed__2(); @@ -25158,11 +24846,11 @@ l_Lean_Elab_Command_elabCommand___closed__6 = _init_l_Lean_Elab_Command_elabComm lean_mark_persistent(l_Lean_Elab_Command_elabCommand___closed__6); l_Lean_Elab_Command_elabCommand___boxed__const__1 = _init_l_Lean_Elab_Command_elabCommand___boxed__const__1(); lean_mark_persistent(l_Lean_Elab_Command_elabCommand___boxed__const__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__1); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634____closed__2); -res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2634_(lean_io_mk_world()); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__1); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__2 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535____closed__2); +res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Command___hyg_2535_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__6___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabCommandTopLevel___spec__6___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/ComputedFields.c b/stage0/stdlib/Lean/Elab/ComputedFields.c index e23606ffdc45..60704186dc11 100644 --- a/stage0/stdlib/Lean/Elab/ComputedFields.c +++ b/stage0/stdlib/Lean/Elab/ComputedFields.c @@ -162,6 +162,7 @@ static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_ComputedFields_isScal static lean_object* l_Lean_getConstInfo___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_ComputedFields_validateComputedFields___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Elab_ComputedFields_initFn____x40_Lean_Elab_ComputedFields___hyg_6____closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_ComputedFields_overrideConstructors___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_ComputedFields_overrideCasesOn___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -231,7 +232,6 @@ LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_ComputedFields_setComputedFie lean_object* l_List_redLength___rarg(lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ComputedFields_overrideCasesOn___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_abstractRange___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -816,7 +816,7 @@ static lean_object* _init_l_Lean_Meta_whnfEasyCases___at_Lean_Elab_ComputedField lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_whnfEasyCases___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__2___closed__1; x_2 = l_Lean_Meta_whnfEasyCases___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(290u); +x_3 = lean_unsigned_to_nat(289u); x_4 = lean_unsigned_to_nat(26u); x_5 = l_Lean_Meta_whnfEasyCases___at_Lean_Elab_ComputedFields_getComputedFieldValue___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2598,7 +2598,7 @@ x_50 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLe lean_dec(x_49); lean_dec(x_47); x_51 = lean_unsigned_to_nat(0u); -x_52 = l_Lean_Expr_getAppNumArgsAux(x_27, x_51); +x_52 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_27, x_51); x_53 = l_Lean_Elab_ComputedFields_getComputedFieldValue___closed__3; lean_inc(x_52); x_54 = lean_mk_array(x_52, x_53); @@ -3332,7 +3332,7 @@ x_14 = l_List_mapM___at_Lean_Elab_ComputedFields_mkImplType___spec__2___lambda__ x_15 = l_Lean_Name_append(x_1, x_14); x_16 = l_Lean_Expr_const___override(x_15, x_2); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_7, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_7, x_17); x_19 = l_Lean_Elab_ComputedFields_getComputedFieldValue___closed__3; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -6512,7 +6512,7 @@ static lean_object* _init_l_Lean_Elab_ComputedFields_overrideCasesOn___lambda__3 lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_ComputedFields_overrideCasesOn___lambda__3___closed__3; x_2 = l_Lean_Elab_ComputedFields_overrideCasesOn___lambda__3___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_ComputedFields_overrideCasesOn___lambda__3___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/DeclModifiers.c b/stage0/stdlib/Lean/Elab/DeclModifiers.c index 464417a552f5..14f68a218452 100644 --- a/stage0/stdlib/Lean/Elab/DeclModifiers.c +++ b/stage0/stdlib/Lean/Elab/DeclModifiers.c @@ -85,7 +85,7 @@ static lean_object* l_Lean_Elab_instToFormatModifiers___closed__25; LEAN_EXPORT lean_object* l_Lean_Elab_instToStringVisibility(uint8_t); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed(lean_object**); static lean_object* l_Lean_Elab_instToFormatModifiers___closed__8; static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___rarg___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_expandDeclId___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -102,7 +102,7 @@ static lean_object* l_Lean_Elab_instToFormatModifiers___closed__21; static lean_object* l_Lean_Elab_instToFormatModifiers___closed__13; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___spec__1___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_expandDeclId___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__8; @@ -111,7 +111,7 @@ lean_object* l_Lean_Name_toString(lean_object*, uint8_t); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___spec__1___rarg___closed__5; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_checkIfShadowingStructureField___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed(lean_object**); static lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__1; static lean_object* l_List_mapTRAux___at_Lean_Elab_instToFormatModifiers___spec__1___closed__10; LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_recKind___default; @@ -158,9 +158,9 @@ LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclIdCore(lean_object*); static lean_object* l_Lean_Elab_instToStringModifiers___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_expandDeclId___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_instToFormatModifiers___closed__19; -lean_object* l_Lean_Elab_elabDeclAttrs___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_Elab_elabDeclAttrs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_instToStringModifiers; -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___rarg___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTRAux___at_Lean_Elab_instToFormatModifiers___spec__1___closed__6; @@ -222,7 +222,7 @@ static lean_object* l_Lean_Elab_expandDeclIdCore___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_length(lean_object*); lean_object* l_Lean_indentD(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkIfShadowingStructureField___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Modifiers_isUnsafe___default; static lean_object* l_Lean_Elab_elabModifiers___rarg___closed__1; @@ -261,7 +261,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Visibility_noConfusion___rarg___lambda__1__ uint8_t l_Lean_isStructure(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___rarg___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_instToStringVisibility___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); @@ -2192,24 +2192,26 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, uint8_t x_15) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, uint8_t x_17) { _start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_box(x_15); -x_17 = lean_box(x_5); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_box(x_17); +x_19 = lean_box(x_5); lean_inc(x_1); -x_18 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed), 7, 6); -lean_closure_set(x_18, 0, x_1); -lean_closure_set(x_18, 1, x_2); -lean_closure_set(x_18, 2, x_3); -lean_closure_set(x_18, 3, x_4); -lean_closure_set(x_18, 4, x_16); -lean_closure_set(x_18, 5, x_17); -x_19 = l_Lean_Syntax_getOptional_x3f(x_6); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__1___boxed), 7, 6); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, x_2); +lean_closure_set(x_20, 2, x_3); +lean_closure_set(x_20, 3, x_4); +lean_closure_set(x_20, 4, x_18); +lean_closure_set(x_20, 5, x_19); +x_21 = l_Lean_Syntax_getOptional_x3f(x_6); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +lean_dec(x_16); +lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -2218,31 +2220,31 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_1, 0); -lean_inc(x_21); -lean_dec(x_1); -x_22 = lean_ctor_get(x_21, 1); +x_22 = lean_ctor_get(x_1, 1); lean_inc(x_22); -lean_dec(x_21); -x_23 = l_Lean_Elab_Modifiers_attrs___default___closed__1; -x_24 = lean_apply_2(x_22, lean_box(0), x_23); -x_25 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_24, x_18); -return x_25; +x_23 = lean_ctor_get(x_1, 0); +lean_inc(x_23); +lean_dec(x_1); +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +x_25 = l_Lean_Elab_Modifiers_attrs___default___closed__1; +x_26 = lean_apply_2(x_24, lean_box(0), x_25); +x_27 = lean_apply_4(x_22, lean_box(0), lean_box(0), x_26, x_20); +return x_27; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_26 = lean_ctor_get(x_19, 0); -lean_inc(x_26); -lean_dec(x_19); -x_27 = lean_ctor_get(x_1, 1); -lean_inc(x_27); -x_28 = l_Lean_Elab_elabDeclAttrs___rarg(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_26); -lean_dec(x_26); -x_29 = lean_apply_4(x_27, lean_box(0), lean_box(0), x_28, x_18); -return x_29; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = lean_ctor_get(x_21, 0); +lean_inc(x_28); +lean_dec(x_21); +x_29 = lean_ctor_get(x_1, 1); +lean_inc(x_29); +x_30 = l_Lean_Elab_elabDeclAttrs___rarg(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_28); +lean_dec(x_28); +x_31 = lean_apply_4(x_29, lean_box(0), lean_box(0), x_30, x_20); +return x_31; } } } @@ -2337,112 +2339,114 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_box(x_4); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_box(x_4); lean_inc(x_8); lean_inc(x_1); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed), 15, 14); -lean_closure_set(x_17, 0, x_1); -lean_closure_set(x_17, 1, x_2); -lean_closure_set(x_17, 2, x_3); -lean_closure_set(x_17, 3, x_15); -lean_closure_set(x_17, 4, x_16); -lean_closure_set(x_17, 5, x_5); -lean_closure_set(x_17, 6, x_6); -lean_closure_set(x_17, 7, x_7); -lean_closure_set(x_17, 8, x_8); -lean_closure_set(x_17, 9, x_9); -lean_closure_set(x_17, 10, x_10); -lean_closure_set(x_17, 11, x_11); -lean_closure_set(x_17, 12, x_12); -lean_closure_set(x_17, 13, x_13); -x_18 = l_Lean_Syntax_getOptional_x3f(x_14); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_19 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed), 17, 16); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, x_2); +lean_closure_set(x_19, 2, x_3); +lean_closure_set(x_19, 3, x_17); +lean_closure_set(x_19, 4, x_18); +lean_closure_set(x_19, 5, x_5); +lean_closure_set(x_19, 6, x_6); +lean_closure_set(x_19, 7, x_7); +lean_closure_set(x_19, 8, x_8); +lean_closure_set(x_19, 9, x_9); +lean_closure_set(x_19, 10, x_10); +lean_closure_set(x_19, 11, x_11); +lean_closure_set(x_19, 12, x_12); +lean_closure_set(x_19, 13, x_13); +lean_closure_set(x_19, 14, x_14); +lean_closure_set(x_19, 15, x_15); +x_20 = l_Lean_Syntax_getOptional_x3f(x_16); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_dec(x_8); -x_19 = lean_ctor_get(x_1, 1); -lean_inc(x_19); -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); -lean_dec(x_1); -x_21 = lean_ctor_get(x_20, 1); +x_21 = lean_ctor_get(x_1, 1); lean_inc(x_21); -lean_dec(x_20); -x_22 = 0; -x_23 = lean_box(x_22); -x_24 = lean_apply_2(x_21, lean_box(0), x_23); -x_25 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_24, x_17); -return x_25; +x_22 = lean_ctor_get(x_1, 0); +lean_inc(x_22); +lean_dec(x_1); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = 0; +x_25 = lean_box(x_24); +x_26 = lean_apply_2(x_23, lean_box(0), x_25); +x_27 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_26, x_19); +return x_27; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_26 = lean_ctor_get(x_18, 0); -lean_inc(x_26); -lean_dec(x_18); -lean_inc(x_26); -x_27 = l_Lean_Syntax_getKind(x_26); -x_28 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__7; -x_29 = lean_name_eq(x_27, x_28); -if (x_29 == 0) -{ -lean_object* x_30; uint8_t x_31; -x_30 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__8; -x_31 = lean_name_eq(x_27, x_30); -lean_dec(x_27); +lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_28 = lean_ctor_get(x_20, 0); +lean_inc(x_28); +lean_dec(x_20); +lean_inc(x_28); +x_29 = l_Lean_Syntax_getKind(x_28); +x_30 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__7; +x_31 = lean_name_eq(x_29, x_30); if (x_31 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_32 = lean_ctor_get(x_1, 1); -lean_inc(x_32); -x_33 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__10; -x_34 = l_Lean_throwErrorAt___rarg(x_1, x_8, x_26, x_33); -x_35 = lean_apply_4(x_32, lean_box(0), lean_box(0), x_34, x_17); -return x_35; +lean_object* x_32; uint8_t x_33; +x_32 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__8; +x_33 = lean_name_eq(x_29, x_32); +lean_dec(x_29); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_34 = lean_ctor_get(x_1, 1); +lean_inc(x_34); +x_35 = l_Lean_Elab_elabModifiers___rarg___lambda__3___closed__10; +x_36 = l_Lean_throwErrorAt___rarg(x_1, x_8, x_28, x_35); +x_37 = lean_apply_4(x_34, lean_box(0), lean_box(0), x_36, x_19); +return x_37; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -lean_dec(x_26); +lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_dec(x_28); lean_dec(x_8); -x_36 = lean_ctor_get(x_1, 1); -lean_inc(x_36); -x_37 = lean_ctor_get(x_1, 0); -lean_inc(x_37); -lean_dec(x_1); -x_38 = lean_ctor_get(x_37, 1); +x_38 = lean_ctor_get(x_1, 1); lean_inc(x_38); -lean_dec(x_37); -x_39 = 1; -x_40 = lean_box(x_39); -x_41 = lean_apply_2(x_38, lean_box(0), x_40); -x_42 = lean_apply_4(x_36, lean_box(0), lean_box(0), x_41, x_17); -return x_42; +x_39 = lean_ctor_get(x_1, 0); +lean_inc(x_39); +lean_dec(x_1); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_41 = 1; +x_42 = lean_box(x_41); +x_43 = lean_apply_2(x_40, lean_box(0), x_42); +x_44 = lean_apply_4(x_38, lean_box(0), lean_box(0), x_43, x_19); +return x_44; } } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -lean_dec(x_27); -lean_dec(x_26); +lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_dec(x_29); +lean_dec(x_28); lean_dec(x_8); -x_43 = lean_ctor_get(x_1, 1); -lean_inc(x_43); -x_44 = lean_ctor_get(x_1, 0); -lean_inc(x_44); -lean_dec(x_1); -x_45 = lean_ctor_get(x_44, 1); +x_45 = lean_ctor_get(x_1, 1); lean_inc(x_45); -lean_dec(x_44); -x_46 = 2; -x_47 = lean_box(x_46); -x_48 = lean_apply_2(x_45, lean_box(0), x_47); -x_49 = lean_apply_4(x_43, lean_box(0), lean_box(0), x_48, x_17); -return x_49; +x_46 = lean_ctor_get(x_1, 0); +lean_inc(x_46); +lean_dec(x_1); +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +x_48 = 2; +x_49 = lean_box(x_48); +x_50 = lean_apply_2(x_47, lean_box(0), x_49); +x_51 = lean_apply_4(x_45, lean_box(0), lean_box(0), x_50, x_19); +return x_51; } } } @@ -2457,207 +2461,209 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; uint8_t x_25; -x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Syntax_getArg(x_10, x_11); -x_13 = lean_unsigned_to_nat(1u); -x_14 = l_Lean_Syntax_getArg(x_10, x_13); -x_15 = lean_unsigned_to_nat(2u); -x_16 = l_Lean_Syntax_getArg(x_10, x_15); -x_17 = lean_unsigned_to_nat(3u); -x_18 = l_Lean_Syntax_getArg(x_10, x_17); -x_19 = lean_unsigned_to_nat(4u); -x_20 = l_Lean_Syntax_getArg(x_10, x_19); -x_21 = lean_unsigned_to_nat(5u); -x_22 = l_Lean_Syntax_getArg(x_10, x_21); -x_23 = l_Lean_Syntax_isNone(x_22); -x_24 = l_Lean_Syntax_getOptional_x3f(x_12); -lean_dec(x_12); -if (x_23 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; uint8_t x_27; +x_13 = lean_unsigned_to_nat(0u); +x_14 = l_Lean_Syntax_getArg(x_12, x_13); +x_15 = lean_unsigned_to_nat(1u); +x_16 = l_Lean_Syntax_getArg(x_12, x_15); +x_17 = lean_unsigned_to_nat(2u); +x_18 = l_Lean_Syntax_getArg(x_12, x_17); +x_19 = lean_unsigned_to_nat(3u); +x_20 = l_Lean_Syntax_getArg(x_12, x_19); +x_21 = lean_unsigned_to_nat(4u); +x_22 = l_Lean_Syntax_getArg(x_12, x_21); +x_23 = lean_unsigned_to_nat(5u); +x_24 = l_Lean_Syntax_getArg(x_12, x_23); +x_25 = l_Lean_Syntax_isNone(x_24); +x_26 = l_Lean_Syntax_getOptional_x3f(x_14); +lean_dec(x_14); +if (x_25 == 0) { -lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; -x_77 = l_Lean_Syntax_getArg(x_22, x_11); -lean_dec(x_22); -x_78 = l_Lean_Syntax_getKind(x_77); -x_79 = l_Lean_Elab_elabModifiers___rarg___closed__1; -x_80 = lean_name_eq(x_78, x_79); -lean_dec(x_78); -if (x_80 == 0) +lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; +x_79 = l_Lean_Syntax_getArg(x_24, x_13); +lean_dec(x_24); +x_80 = l_Lean_Syntax_getKind(x_79); +x_81 = l_Lean_Elab_elabModifiers___rarg___closed__1; +x_82 = lean_name_eq(x_80, x_81); +lean_dec(x_80); +if (x_82 == 0) { -uint8_t x_81; -x_81 = 1; -x_25 = x_81; -goto block_76; +uint8_t x_83; +x_83 = 1; +x_27 = x_83; +goto block_78; } else { -uint8_t x_82; -x_82 = 0; -x_25 = x_82; -goto block_76; +uint8_t x_84; +x_84 = 0; +x_27 = x_84; +goto block_78; } } else { -uint8_t x_83; -lean_dec(x_22); -x_83 = 2; -x_25 = x_83; -goto block_76; +uint8_t x_85; +lean_dec(x_24); +x_85 = 2; +x_27 = x_85; +goto block_78; } -block_76: +block_78: { -lean_object* x_26; lean_object* x_27; -x_26 = lean_box(x_25); +lean_object* x_28; lean_object* x_29; +x_28 = lean_box(x_27); lean_inc(x_4); lean_inc(x_1); -x_27 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed), 15, 14); -lean_closure_set(x_27, 0, x_1); -lean_closure_set(x_27, 1, x_18); -lean_closure_set(x_27, 2, x_20); -lean_closure_set(x_27, 3, x_26); -lean_closure_set(x_27, 4, x_14); -lean_closure_set(x_27, 5, x_2); -lean_closure_set(x_27, 6, x_3); -lean_closure_set(x_27, 7, x_4); -lean_closure_set(x_27, 8, x_5); -lean_closure_set(x_27, 9, x_6); -lean_closure_set(x_27, 10, x_7); -lean_closure_set(x_27, 11, x_8); -lean_closure_set(x_27, 12, x_9); -lean_closure_set(x_27, 13, x_16); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_29 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed), 17, 16); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, x_20); +lean_closure_set(x_29, 2, x_22); +lean_closure_set(x_29, 3, x_28); +lean_closure_set(x_29, 4, x_16); +lean_closure_set(x_29, 5, x_2); +lean_closure_set(x_29, 6, x_3); +lean_closure_set(x_29, 7, x_4); +lean_closure_set(x_29, 8, x_5); +lean_closure_set(x_29, 9, x_6); +lean_closure_set(x_29, 10, x_7); +lean_closure_set(x_29, 11, x_8); +lean_closure_set(x_29, 12, x_9); +lean_closure_set(x_29, 13, x_10); +lean_closure_set(x_29, 14, x_11); +lean_closure_set(x_29, 15, x_18); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_dec(x_4); -x_28 = lean_ctor_get(x_1, 1); -lean_inc(x_28); -x_29 = lean_ctor_get(x_1, 0); -lean_inc(x_29); -lean_dec(x_1); -x_30 = lean_ctor_get(x_29, 1); +x_30 = lean_ctor_get(x_1, 1); lean_inc(x_30); -lean_dec(x_29); -x_31 = lean_box(0); -x_32 = lean_apply_2(x_30, lean_box(0), x_31); -x_33 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_32, x_27); -return x_33; +x_31 = lean_ctor_get(x_1, 0); +lean_inc(x_31); +lean_dec(x_1); +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +lean_dec(x_31); +x_33 = lean_box(0); +x_34 = lean_apply_2(x_32, lean_box(0), x_33); +x_35 = lean_apply_4(x_30, lean_box(0), lean_box(0), x_34, x_29); +return x_35; } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_24); -if (x_34 == 0) +uint8_t x_36; +x_36 = !lean_is_exclusive(x_26); +if (x_36 == 0) { -lean_object* x_35; lean_object* x_36; -x_35 = lean_ctor_get(x_24, 0); -x_36 = l_Lean_Syntax_getArg(x_35, x_13); -if (lean_obj_tag(x_36) == 2) +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_26, 0); +x_38 = l_Lean_Syntax_getArg(x_37, x_15); +if (lean_obj_tag(x_38) == 2) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -lean_dec(x_35); +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_dec(x_37); lean_dec(x_4); -x_37 = lean_ctor_get(x_36, 1); -lean_inc(x_37); -lean_dec(x_36); -x_38 = lean_ctor_get(x_1, 1); -lean_inc(x_38); -x_39 = lean_ctor_get(x_1, 0); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); -lean_dec(x_1); -x_40 = lean_ctor_get(x_39, 1); +lean_dec(x_38); +x_40 = lean_ctor_get(x_1, 1); lean_inc(x_40); -lean_dec(x_39); -x_41 = lean_string_utf8_byte_size(x_37); -x_42 = lean_nat_sub(x_41, x_15); +x_41 = lean_ctor_get(x_1, 0); +lean_inc(x_41); +lean_dec(x_1); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); lean_dec(x_41); -x_43 = lean_string_utf8_extract(x_37, x_11, x_42); -lean_dec(x_42); -lean_dec(x_37); -lean_ctor_set(x_24, 0, x_43); -x_44 = lean_apply_2(x_40, lean_box(0), x_24); -x_45 = lean_apply_4(x_38, lean_box(0), lean_box(0), x_44, x_27); -return x_45; +x_43 = lean_string_utf8_byte_size(x_39); +x_44 = lean_nat_sub(x_43, x_17); +lean_dec(x_43); +x_45 = lean_string_utf8_extract(x_39, x_13, x_44); +lean_dec(x_44); +lean_dec(x_39); +lean_ctor_set(x_26, 0, x_45); +x_46 = lean_apply_2(x_42, lean_box(0), x_26); +x_47 = lean_apply_4(x_40, lean_box(0), lean_box(0), x_46, x_29); +return x_47; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -lean_free_object(x_24); -x_46 = lean_ctor_get(x_1, 1); -lean_inc(x_46); -x_47 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_47, 0, x_36); -x_48 = l_Lean_indentD(x_47); -x_49 = l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__2; -x_50 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_48); -x_51 = l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__3; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +lean_free_object(x_26); +x_48 = lean_ctor_get(x_1, 1); +lean_inc(x_48); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_38); +x_50 = l_Lean_indentD(x_49); +x_51 = l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__2; x_52 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -x_53 = l_Lean_throwErrorAt___rarg(x_1, x_4, x_35, x_52); -x_54 = lean_apply_4(x_46, lean_box(0), lean_box(0), x_53, x_27); -return x_54; +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_50); +x_53 = l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__3; +x_54 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +x_55 = l_Lean_throwErrorAt___rarg(x_1, x_4, x_37, x_54); +x_56 = lean_apply_4(x_48, lean_box(0), lean_box(0), x_55, x_29); +return x_56; } } else { -lean_object* x_55; lean_object* x_56; -x_55 = lean_ctor_get(x_24, 0); -lean_inc(x_55); -lean_dec(x_24); -x_56 = l_Lean_Syntax_getArg(x_55, x_13); -if (lean_obj_tag(x_56) == 2) +lean_object* x_57; lean_object* x_58; +x_57 = lean_ctor_get(x_26, 0); +lean_inc(x_57); +lean_dec(x_26); +x_58 = l_Lean_Syntax_getArg(x_57, x_15); +if (lean_obj_tag(x_58) == 2) { -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_dec(x_55); +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_dec(x_57); lean_dec(x_4); -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); -x_58 = lean_ctor_get(x_1, 1); -lean_inc(x_58); -x_59 = lean_ctor_get(x_1, 0); +x_59 = lean_ctor_get(x_58, 1); lean_inc(x_59); -lean_dec(x_1); -x_60 = lean_ctor_get(x_59, 1); +lean_dec(x_58); +x_60 = lean_ctor_get(x_1, 1); lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_string_utf8_byte_size(x_57); -x_62 = lean_nat_sub(x_61, x_15); +x_61 = lean_ctor_get(x_1, 0); +lean_inc(x_61); +lean_dec(x_1); +x_62 = lean_ctor_get(x_61, 1); +lean_inc(x_62); lean_dec(x_61); -x_63 = lean_string_utf8_extract(x_57, x_11, x_62); -lean_dec(x_62); -lean_dec(x_57); -x_64 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_64, 0, x_63); -x_65 = lean_apply_2(x_60, lean_box(0), x_64); -x_66 = lean_apply_4(x_58, lean_box(0), lean_box(0), x_65, x_27); -return x_66; +x_63 = lean_string_utf8_byte_size(x_59); +x_64 = lean_nat_sub(x_63, x_17); +lean_dec(x_63); +x_65 = lean_string_utf8_extract(x_59, x_13, x_64); +lean_dec(x_64); +lean_dec(x_59); +x_66 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_66, 0, x_65); +x_67 = lean_apply_2(x_62, lean_box(0), x_66); +x_68 = lean_apply_4(x_60, lean_box(0), lean_box(0), x_67, x_29); +return x_68; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_67 = lean_ctor_get(x_1, 1); -lean_inc(x_67); -x_68 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_68, 0, x_56); -x_69 = l_Lean_indentD(x_68); -x_70 = l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__2; -x_71 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_69); -x_72 = l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__3; +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_69 = lean_ctor_get(x_1, 1); +lean_inc(x_69); +x_70 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_70, 0, x_58); +x_71 = l_Lean_indentD(x_70); +x_72 = l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__2; x_73 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -x_74 = l_Lean_throwErrorAt___rarg(x_1, x_4, x_55, x_73); -x_75 = lean_apply_4(x_67, lean_box(0), lean_box(0), x_74, x_27); -return x_75; +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_71); +x_74 = l_Lean_Elab_expandOptDocComment_x3f___rarg___closed__3; +x_75 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +x_76 = l_Lean_throwErrorAt___rarg(x_1, x_4, x_57, x_75); +x_77 = lean_apply_4(x_69, lean_box(0), lean_box(0), x_76, x_29); +return x_77; } } } @@ -2668,7 +2674,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_elabModifiers___rarg___boxed), 12, 0); return x_2; } } @@ -2686,37 +2692,71 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -uint8_t x_16; uint8_t x_17; lean_object* x_18; -x_16 = lean_unbox(x_5); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__2___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +uint8_t x_18; uint8_t x_19; lean_object* x_20; +x_18 = lean_unbox(x_5); lean_dec(x_5); -x_17 = lean_unbox(x_15); -lean_dec(x_15); -x_18 = l_Lean_Elab_elabModifiers___rarg___lambda__2(x_1, x_2, x_3, x_4, x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_17); +x_19 = lean_unbox(x_17); +lean_dec(x_17); +x_20 = l_Lean_Elab_elabModifiers___rarg___lambda__2(x_1, x_2, x_3, x_4, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_19); lean_dec(x_6); -return x_18; +return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -uint8_t x_16; lean_object* x_17; -x_16 = lean_unbox(x_4); +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___lambda__3___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +uint8_t x_18; lean_object* x_19; +x_18 = lean_unbox(x_4); lean_dec(x_4); -x_17 = l_Lean_Elab_elabModifiers___rarg___lambda__3(x_1, x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -return x_17; +x_19 = l_Lean_Elab_elabModifiers___rarg___lambda__3(x_1, x_2, x_3, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_16); +return x_19; } } -LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_11; -x_11 = l_Lean_Elab_elabModifiers___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_10); -return x_11; +lean_object* x_13; +x_13 = l_Lean_Elab_elabModifiers___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_12); +return x_13; } } LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { diff --git a/stage0/stdlib/Lean/Elab/Declaration.c b/stage0/stdlib/Lean/Elab/Declaration.c index 93400194ed2d..7c3aaf0a6eae 100644 --- a/stage0/stdlib/Lean/Elab/Declaration.c +++ b/stage0/stdlib/Lean/Elab/Declaration.c @@ -17,17 +17,13 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange_ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabDeclaration(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize(lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__10; static lean_object* l_Lean_Elab_Command_getTerminationHints___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__5; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__32; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration___closed__4; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__20; lean_object* l_Lean_extractMacroScopes(lean_object*); static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__9; size_t lean_usize_add(size_t, size_t); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_expandOptDeclSig(lean_object*); @@ -43,10 +39,11 @@ lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___closed__6; lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange___closed__4; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__43; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_Elab_getOptDerivingClasses___at_Lean_Elab_Command_elabStructure___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26; +lean_object* l_Lean_Syntax_getHeadInfo_x3f(lean_object*); lean_object* l_Lean_Meta_mkForallFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabDeclaration___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -55,14 +52,12 @@ static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expan LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabDeclaration___spec__5___rarg(lean_object*); lean_object* l_Lean_addDecl___at_Lean_Elab_Term_declareTacticSyntax___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_elabDeclaration___closed__8; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__7; lean_object* l_Lean_Elab_Command_elabMutualDef(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Elab_Modifiers_isPartial(lean_object*); +lean_object* l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__1; lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__4; uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Term_addDotCompletionInfo___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -70,13 +65,17 @@ static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Le static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__2; lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___closed__7; uint8_t l_Lean_Elab_Modifiers_isProtected(lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__3; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange___closed__5; static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__4; +static lean_object* l_Lean_Elab_Command_expandInitialize___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement___closed__2; lean_object* l_Lean_Syntax_getIdAt(lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_commandElabAttribute; @@ -89,20 +88,20 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___priva static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2; static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange___closed__2; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__1; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__16; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutual___spec__1___lambda__1___closed__3; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__2; +static lean_object* l_Lean_Elab_Command_expandInitialize___closed__5; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__39; lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Command_expandDeclId___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Attribute_erase(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange___closed__2; lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Command_mkDefViewOfInstance___spec__11(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___closed__1; lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__12; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_splitMutualPreamble(lean_object*); @@ -114,7 +113,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange__ extern lean_object* l_Lean_declRangeExt; lean_object* l_Lean_Elab_Term_ensureNoUnassignedMVars(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*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__14; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize(lean_object*); @@ -123,8 +121,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration(lean_o LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabDeclaration___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement___closed__3; lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__7; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclIdNamespace_x3f(lean_object*, lean_object*, lean_object*); @@ -140,6 +136,7 @@ uint8_t l_Lean_Name_isPrefixOf(lean_object*, lean_object*); 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_Elab_Command_getTerminationHints(lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__25; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__4; lean_object* l_Std_mkHashSetImp___rarg(lean_object*); @@ -150,6 +147,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual(lean_object static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__9; lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__36; lean_object* l_Lean_Elab_Term_withLevelNames___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -157,6 +155,8 @@ static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMut uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration___closed__1; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__10; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___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*); @@ -165,12 +165,10 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declara extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabDeclaration___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__6___boxed(lean_object**); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__6; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__11; static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_classInductiveSyntaxToView(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabDeclaration___spec__4___closed__2; @@ -182,25 +180,29 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAtt static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___closed__7; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__2; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__3; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__16; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__22; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__19; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualNamespace___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabDeclaration___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getDeclarationRange___at_Lean_Elab_Command_elabAxiom___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_runTermElabM___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__12; lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabMutualDef___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__3; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualNamespace___spec__1___closed__2; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__20; lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_MapDeclarationExtension_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; +static lean_object* l_Lean_Elab_Command_expandInitialize___closed__6; static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__10; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration___closed__5; uint8_t l_Lean_isExtern(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__5; @@ -209,90 +211,80 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declara lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabDeclaration___spec__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__19; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange(lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabDeclaration___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandMutualNamespace___closed__1; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__1; lean_object* l_Lean_Elab_Command_expandDeclId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange___closed__6; lean_object* l_Lean_Syntax_getHeadInfo(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__12; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange___closed__1; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__27; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__45; lean_object* l_Lean_Name_toString(lean_object*, uint8_t); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__7; lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_elabInductiveViews(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__40; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr___closed__3; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabDeclaration___spec__5(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration___closed__6; LEAN_EXPORT uint8_t l_Lean_Elab_Command_elabAxiom___lambda__1(lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__24; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__8; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace(lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__6; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__10; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__19; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Command_elabAttr___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__1; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_getTerminationHints___boxed(lean_object*); lean_object* l_Lean_mkConstWithLevelParams___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___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_expandInitialize___lambda__1___closed__12; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__16; lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabClassInductive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_addAutoBoundImplicits_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__35; lean_object* l_Lean_Expr_sort___override(lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___closed__1; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; lean_object* l_Lean_Macro_throwErrorAt___rarg(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace___closed__5; lean_object* l_Lean_CollectLevelParams_main(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace___closed__3; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualNamespace___spec__1___closed__3; static lean_object* l_Lean_Elab_Command_elabMutual___closed__4; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29; LEAN_EXPORT lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__10; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__2; static lean_object* l_Lean_Elab_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange___closed__7; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__21; static lean_object* l_Lean_Elab_Command_expandMutualElement___closed__1; static lean_object* l_Lean_Elab_Command_expandMutualPreamble___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__21; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__38; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Elab_Command_isDefLike(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__13; static lean_object* l_Lean_Elab_Command_expandMutualPreamble___closed__3; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__41; static lean_object* l_Lean_Elab_Command_elabClassInductive___closed__3; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25; static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabDeclaration___spec__5___rarg___closed__1; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__13; lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclIdNamespace_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration___closed__3; @@ -302,10 +294,12 @@ lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, le static lean_object* l_Lean_Elab_Command_elabMutual___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange___closed__3; +static lean_object* l_Lean_Elab_Command_expandInitialize___closed__4; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__20; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr___closed__4; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30; lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabAttr___closed__1; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___closed__4; size_t lean_usize_of_nat(lean_object*); @@ -314,30 +308,29 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__1___boxed(lean_ lean_object* l_Lean_Elab_expandDeclIdCore(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAttr___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef(lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualElement___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__44; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__23; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__4; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualPreamble(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__21; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabClassInductive___closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutual___spec__1___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange___closed__7; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33; static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabDeclaration___spec__5___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualElement(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabClassInductive___closed__1; lean_object* l_Lean_Macro_expandMacro_x3f(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabDeclaration___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__47; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__13; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabDeclaration___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -345,8 +338,6 @@ static lean_object* l_Lean_Elab_Command_expandMutualPreamble___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutual___spec__1___boxed(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_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitCmd(uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualNamespace___spec__1___closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutual___spec__1___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__10; @@ -359,14 +350,12 @@ lean_object* l_Lean_Syntax_getSepArgs(lean_object*); uint8_t l_Lean_isAttribute(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__7___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange(lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange___closed__1; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__4; lean_object* l_Lean_Syntax_getNumArgs(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__1; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__11; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___closed__10; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15; extern lean_object* l_Lean_Elab_macroAttribute; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace___closed__2; lean_object* l_Lean_Syntax_setArg(lean_object*, lean_object*, lean_object*); @@ -374,45 +363,42 @@ lean_object* l_Lean_Elab_Command_withMacroExpansion___rarg(lean_object*, lean_ob lean_object* lean_environment_main_module(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabDeclaration___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_elabMutualInductive(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; lean_object* l_Lean_compileDecl___at_Lean_Elab_Term_declareTacticSyntax___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__5; lean_object* l_panic___at_Lean_expandExplicitBindersAux_loop___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__17; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__29; LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclIdNamespace_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange___closed__4; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3; lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7; lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabInductive___closed__1; lean_object* l_Lean_Syntax_getKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__7___boxed(lean_object**); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__23; -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MacroScopesView_review(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange___closed__1; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__34; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; lean_object* l_Lean_Elab_Term_applyAttributes(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_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__26; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclIdNamespace_x3f___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange(lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutual___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange___closed__2; static lean_object* l_Lean_Elab_Command_getTerminationHints___closed__5; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__2; lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__3; lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_ensureAtomicBinderName___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -422,21 +408,18 @@ lean_object* l_Lean_Elab_Command_getMainModule___rarg(lean_object*, lean_object* lean_object* l_Lean_Elab_Command_elabStructure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__4; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__13; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__37; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabMutual___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabDeclaration___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutual___spec__1___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__3; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_splitMutualPreamble_loop(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__5; lean_object* l_Lean_Elab_expandDeclSig(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*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -444,28 +427,27 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___s LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualDef___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_setInfo(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__14; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__14; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___closed__4; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__17; static lean_object* l_Lean_Elab_Command_elabMutual___lambda__2___closed__2; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__15; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__18; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__2; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__18; uint8_t l_Lean_Syntax_isNone(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__5; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__18; static lean_object* l_Lean_Elab_Command_getTerminationHints___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7049_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7254_(lean_object*); static lean_object* l_Lean_Elab_Command_getTerminationHints___closed__4; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__4; lean_object* l_Lean_Elab_Modifiers_addAttribute(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__40; LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__4(size_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabMutual___lambda__2___closed__1; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__6; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMutualNamespace(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Command_expandDeclId___spec__6(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -476,11 +458,15 @@ static lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange___closed__3; lean_object* l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__38; lean_object* l_Lean_Elab_Command_checkValidInductiveModifier___at_Lean_Elab_Command_elabStructure___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addDeclarationRanges___at_Lean_Elab_Command_elabAxiom___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21; lean_object* l_Lean_Elab_Term_elabBinders___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___boxed(lean_object**); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclaration_declRange___closed__2; extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; @@ -489,12 +475,9 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ uint8_t l_Lean_Elab_Modifiers_isPrivate(lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__5; static size_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__2; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange___closed__6; lean_object* lean_mk_syntax_ident(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__8; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__3; static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -505,24 +488,22 @@ static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expan static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace___closed__4; lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__3; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___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_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Command_elabAttr___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___closed__1; lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange(lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__34; lean_object* l_Lean_Core_resetMessageLog(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__2; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___closed__1; static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange___closed__5; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13; lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___closed__9; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabDeclaration___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___closed__5; @@ -530,48 +511,41 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAttr(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive___spec__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__24; static lean_object* l_Lean_Elab_Command_elabAxiom___lambda__5___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_addAuxDeclarationRanges___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Command_elabAttr___spec__2___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_elabDeclaration___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_expandMutualNamespace___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_ensureValidNamespace___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualElement_declRange___closed__4; lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMutual___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualInductive(lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__16; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4; lean_object* l_Lean_Elab_Term_withAutoBoundImplicit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualNamespace_declRange___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___closed__3; +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23; static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual_declRange___closed__3; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; static lean_object* l_Lean_Elab_Command_elabDeclaration___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___closed__6; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__4; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__3; lean_object* l_Lean_Name_replacePrefix(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__15; static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual___closed__1; -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__42; +uint8_t l_Lean_Syntax_isToken(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4___closed__11; lean_object* l_Lean_Elab_withSaveInfoContext___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutual___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__1; static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__9; static lean_object* l_Lean_Elab_Command_getTerminationHints___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabDeclaration___spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitCmd___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__3___lambda__2___closed__2; -static lean_object* l_Lean_Elab_Command_expandInitCmd___closed__5; static lean_object* l_Lean_Elab_Command_checkValidCtorModifier___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__1___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Declaration_0__Lean_Elab_Command_inductiveSyntaxToView___spec__4(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandBuiltinInitialize(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_isMutualPreambleCommand___closed__6; lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMutual___closed__2; @@ -3461,7 +3435,9 @@ lean_inc(x_19); lean_dec(x_18); x_20 = 0; lean_inc(x_11); -lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); lean_inc(x_6); lean_inc(x_2); x_21 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_20, x_6, x_7, x_8, x_9, x_10, x_11, x_19); @@ -3488,9 +3464,7 @@ uint8_t x_28; lean_object* x_29; lean_dec(x_1); x_28 = 1; x_29 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_25); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_10); return x_29; } else @@ -3511,9 +3485,7 @@ lean_inc(x_31); lean_dec(x_30); x_32 = 1; x_33 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_4, x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_31); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_10); return x_33; } else @@ -3783,7 +3755,9 @@ x_17 = lean_ctor_get(x_1, 1); lean_inc(x_17); x_18 = 2; lean_inc(x_15); -lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); lean_inc(x_10); lean_inc(x_2); x_19 = l_Lean_Elab_Term_applyAttributesAt(x_2, x_17, x_18, x_10, x_11, x_12, x_13, x_14, x_15, x_16); @@ -4539,9 +4513,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAxiom___lambda__3___boxed(lean_ { lean_object* x_11; x_11 = l_Lean_Elab_Command_elabAxiom___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); return x_11; @@ -6070,7 +6042,7 @@ static lean_object* _init_l_Lean_Elab_Command_getTerminationHints___closed__4() lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Command_getTerminationHints___closed__1; x_2 = l_Lean_Elab_Command_getTerminationHints___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_Command_getTerminationHints___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -6757,7 +6729,7 @@ x_53 = lean_ctor_get(x_44, 1); lean_inc(x_53); lean_dec(x_44); x_54 = l_List_reverse___rarg(x_53); -x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_54, x_2, x_3, x_52); +x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_54, x_2, x_3, x_52); lean_dec(x_3); lean_dec(x_2); x_56 = !lean_is_exclusive(x_55); @@ -6819,7 +6791,7 @@ x_71 = lean_ctor_get(x_44, 1); lean_inc(x_71); lean_dec(x_44); x_72 = l_List_reverse___rarg(x_71); -x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_2, x_3, x_70); +x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_72, x_2, x_3, x_70); lean_dec(x_3); lean_dec(x_2); x_74 = lean_ctor_get(x_73, 1); @@ -6995,233 +6967,349 @@ x_7 = lean_ctor_get(x_6, 0); lean_inc(x_7); if (lean_obj_tag(x_7) == 0) { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; x_8 = lean_ctor_get(x_6, 1); lean_inc(x_8); lean_dec(x_6); -x_9 = lean_unsigned_to_nat(0u); +x_9 = lean_unsigned_to_nat(1u); x_10 = l_Lean_Syntax_getArg(x_1, x_9); -lean_inc(x_3); -lean_inc(x_2); -x_11 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_10, x_2, x_3, x_8); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_unsigned_to_nat(1u); -x_15 = l_Lean_Syntax_getArg(x_1, x_14); -lean_inc(x_15); -x_16 = l_Lean_Syntax_getKind(x_15); -x_17 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__18; -x_18 = lean_name_eq(x_16, x_17); -if (x_18 == 0) +lean_inc(x_10); +x_11 = l_Lean_Syntax_getKind(x_10); +x_12 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__18; +x_13 = lean_name_eq(x_11, x_12); +if (x_13 == 0) { -lean_object* x_19; uint8_t x_20; -x_19 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__20; -x_20 = lean_name_eq(x_16, x_19); -if (x_20 == 0) +lean_object* x_14; uint8_t x_15; +x_14 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__20; +x_15 = lean_name_eq(x_11, x_14); +if (x_15 == 0) { -lean_object* x_21; uint8_t x_22; -x_21 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__22; -x_22 = lean_name_eq(x_16, x_21); -if (x_22 == 0) +lean_object* x_16; uint8_t x_17; +x_16 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__22; +x_17 = lean_name_eq(x_11, x_16); +if (x_17 == 0) { -lean_object* x_23; uint8_t x_24; -x_23 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__24; -x_24 = lean_name_eq(x_16, x_23); -lean_dec(x_16); -if (x_24 == 0) +lean_object* x_18; uint8_t x_19; +x_18 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__24; +x_19 = lean_name_eq(x_11, x_18); +lean_dec(x_11); +if (x_19 == 0) { -uint8_t x_25; -lean_dec(x_12); -x_25 = l_Lean_Elab_Command_isDefLike(x_15); -if (x_25 == 0) +uint8_t x_20; +x_20 = l_Lean_Elab_Command_isDefLike(x_10); +if (x_20 == 0) { -lean_object* x_26; lean_object* x_27; +lean_object* x_21; lean_object* x_22; lean_dec(x_1); -x_26 = l_Lean_Elab_Command_elabDeclaration___closed__2; -x_27 = l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(x_26, x_2, x_3, x_13); +x_21 = l_Lean_Elab_Command_elabDeclaration___closed__2; +x_22 = l_Lean_throwError___at___private_Lean_Elab_Command_0__Lean_Elab_Command_elabCommandUsing___spec__1(x_21, x_2, x_3, x_8); lean_dec(x_3); -return x_27; +return x_22; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = l_Lean_Elab_Command_elabInductive___closed__1; +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = l_Lean_Elab_Command_elabInductive___closed__1; lean_inc(x_1); -x_29 = lean_array_push(x_28, x_1); -x_30 = l_Lean_Elab_Command_getTerminationHints(x_1); +x_24 = lean_array_push(x_23, x_1); +x_25 = l_Lean_Elab_Command_getTerminationHints(x_1); lean_dec(x_1); -x_31 = l_Lean_Elab_Command_elabMutualDef(x_29, x_30, x_2, x_3, x_13); -return x_31; +x_26 = l_Lean_Elab_Command_elabMutualDef(x_24, x_25, x_2, x_3, x_8); +return x_26; } } else { -lean_object* x_32; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_unsigned_to_nat(0u); +x_28 = l_Lean_Syntax_getArg(x_1, x_27); lean_dec(x_1); -x_32 = l_Lean_Elab_Command_elabStructure(x_12, x_15, x_2, x_3, x_13); +lean_inc(x_3); +lean_inc(x_2); +x_29 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_28, x_2, x_3, x_8); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = l_Lean_Elab_Command_elabStructure(x_30, x_10, x_2, x_3, x_31); return x_32; } +else +{ +uint8_t x_33; +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_2); +x_33 = !lean_is_exclusive(x_29); +if (x_33 == 0) +{ +return x_29; } else { -lean_object* x_33; -lean_dec(x_16); -lean_dec(x_1); -x_33 = l_Lean_Elab_Command_elabClassInductive(x_12, x_15, x_2, x_3, x_13); -return x_33; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_29, 0); +x_35 = lean_ctor_get(x_29, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_29); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} } } else { -lean_object* x_34; -lean_dec(x_16); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +lean_dec(x_11); +x_37 = lean_unsigned_to_nat(0u); +x_38 = l_Lean_Syntax_getArg(x_1, x_37); lean_dec(x_1); -x_34 = l_Lean_Elab_Command_elabInductive(x_12, x_15, x_2, x_3, x_13); -return x_34; +lean_inc(x_3); +lean_inc(x_2); +x_39 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_38, x_2, x_3, x_8); +if (lean_obj_tag(x_39) == 0) +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); +x_42 = l_Lean_Elab_Command_elabClassInductive(x_40, x_10, x_2, x_3, x_41); +return x_42; } +else +{ +uint8_t x_43; +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_2); +x_43 = !lean_is_exclusive(x_39); +if (x_43 == 0) +{ +return x_39; } else { -lean_object* x_35; -lean_dec(x_16); -lean_dec(x_1); -x_35 = l_Lean_Elab_Command_elabAxiom(x_12, x_15, x_2, x_3, x_13); -return x_35; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_39, 0); +x_45 = lean_ctor_get(x_39, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_39); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; +} } } +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +lean_dec(x_11); +x_47 = lean_unsigned_to_nat(0u); +x_48 = l_Lean_Syntax_getArg(x_1, x_47); +lean_dec(x_1); +lean_inc(x_3); +lean_inc(x_2); +x_49 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_48, x_2, x_3, x_8); +if (lean_obj_tag(x_49) == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = l_Lean_Elab_Command_elabInductive(x_50, x_10, x_2, x_3, x_51); +return x_52; +} else { -uint8_t x_36; +uint8_t x_53; +lean_dec(x_10); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_36 = !lean_is_exclusive(x_11); -if (x_36 == 0) +x_53 = !lean_is_exclusive(x_49); +if (x_53 == 0) { -return x_11; +return x_49; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_11, 0); -x_38 = lean_ctor_get(x_11, 1); -lean_inc(x_38); -lean_inc(x_37); +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_49, 0); +x_55 = lean_ctor_get(x_49, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_49); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +return x_56; +} +} +} +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_dec(x_11); -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; +x_57 = lean_unsigned_to_nat(0u); +x_58 = l_Lean_Syntax_getArg(x_1, x_57); +lean_dec(x_1); +lean_inc(x_3); +lean_inc(x_2); +x_59 = l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1(x_58, x_2, x_3, x_8); +if (lean_obj_tag(x_59) == 0) +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = l_Lean_Elab_Command_elabAxiom(x_60, x_10, x_2, x_3, x_61); +return x_62; +} +else +{ +uint8_t x_63; +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_2); +x_63 = !lean_is_exclusive(x_59); +if (x_63 == 0) +{ +return x_59; +} +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_59, 0); +x_65 = lean_ctor_get(x_59, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_59); +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +return x_66; +} } } } else { -lean_object* x_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; -x_40 = lean_ctor_get(x_7, 0); -lean_inc(x_40); +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_67 = lean_ctor_get(x_7, 0); +lean_inc(x_67); lean_dec(x_7); -x_41 = lean_ctor_get(x_6, 1); -lean_inc(x_41); +x_68 = lean_ctor_get(x_6, 1); +lean_inc(x_68); lean_dec(x_6); -x_42 = lean_ctor_get(x_40, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_40, 1); -lean_inc(x_43); -lean_dec(x_40); +x_69 = lean_ctor_get(x_67, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_67, 1); +lean_inc(x_70); +lean_dec(x_67); lean_inc(x_1); -x_44 = l_Lean_mkIdentFrom(x_1, x_42); -x_45 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Command_mkDefViewOfInstance___spec__11(x_2, x_3, x_41); -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_48 = l_Lean_Elab_Command_getCurrMacroScope(x_2, x_3, x_47); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -lean_dec(x_48); -x_50 = l_Lean_Elab_Command_getMainModule___rarg(x_3, x_49); -x_51 = lean_ctor_get(x_50, 1); -lean_inc(x_51); -lean_dec(x_50); -x_52 = l_Lean_Elab_Command_elabDeclaration___closed__5; -lean_inc(x_46); -x_53 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_53, 0, x_46); -lean_ctor_set(x_53, 1, x_52); -x_54 = l_Lean_Elab_Command_elabDeclaration___closed__7; -x_55 = lean_array_push(x_54, x_53); -lean_inc(x_44); -x_56 = lean_array_push(x_55, x_44); -x_57 = lean_box(2); -x_58 = l_Lean_Elab_Command_elabDeclaration___closed__6; -x_59 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -lean_ctor_set(x_59, 2, x_56); -x_60 = l_Lean_Elab_Command_elabDeclaration___closed__8; -x_61 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_61, 0, x_46); -lean_ctor_set(x_61, 1, x_60); -x_62 = l_Lean_Elab_Command_elabInductive___closed__1; -x_63 = lean_array_push(x_62, x_44); -x_64 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_65 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_65, 0, x_57); -lean_ctor_set(x_65, 1, x_64); -lean_ctor_set(x_65, 2, x_63); -x_66 = lean_array_push(x_54, x_61); -x_67 = lean_array_push(x_66, x_65); -x_68 = l_Lean_Elab_Command_elabDeclaration___closed__9; -x_69 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_69, 0, x_57); -lean_ctor_set(x_69, 1, x_68); -lean_ctor_set(x_69, 2, x_67); -x_70 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_71 = lean_array_push(x_70, x_59); -x_72 = lean_array_push(x_71, x_43); -x_73 = lean_array_push(x_72, x_69); -x_74 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_74, 0, x_57); -lean_ctor_set(x_74, 1, x_64); -lean_ctor_set(x_74, 2, x_73); +x_71 = l_Lean_mkIdentFrom(x_1, x_69); +x_72 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Command_mkDefViewOfInstance___spec__11(x_2, x_3, x_68); +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_72, 1); lean_inc(x_74); -x_75 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand), 4, 1); -lean_closure_set(x_75, 0, x_74); -x_76 = l_Lean_Elab_Command_withMacroExpansion___rarg(x_1, x_74, x_75, x_2, x_3, x_51); -return x_76; +lean_dec(x_72); +x_75 = l_Lean_Elab_Command_getCurrMacroScope(x_2, x_3, x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_77 = l_Lean_Elab_Command_getMainModule___rarg(x_3, x_76); +x_78 = lean_ctor_get(x_77, 1); +lean_inc(x_78); +lean_dec(x_77); +x_79 = l_Lean_Elab_Command_elabDeclaration___closed__5; +lean_inc(x_73); +x_80 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_80, 0, x_73); +lean_ctor_set(x_80, 1, x_79); +x_81 = l_Lean_Elab_Command_elabDeclaration___closed__7; +x_82 = lean_array_push(x_81, x_80); +lean_inc(x_71); +x_83 = lean_array_push(x_82, x_71); +x_84 = lean_box(2); +x_85 = l_Lean_Elab_Command_elabDeclaration___closed__6; +x_86 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +lean_ctor_set(x_86, 2, x_83); +x_87 = l_Lean_Elab_Command_elabDeclaration___closed__8; +x_88 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_88, 0, x_73); +lean_ctor_set(x_88, 1, x_87); +x_89 = l_Lean_Elab_Command_elabInductive___closed__1; +x_90 = lean_array_push(x_89, x_71); +x_91 = l_Lean_Elab_Command_elabDeclaration___closed__4; +x_92 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_92, 0, x_84); +lean_ctor_set(x_92, 1, x_91); +lean_ctor_set(x_92, 2, x_90); +x_93 = lean_array_push(x_81, x_88); +x_94 = lean_array_push(x_93, x_92); +x_95 = l_Lean_Elab_Command_elabDeclaration___closed__9; +x_96 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_96, 0, x_84); +lean_ctor_set(x_96, 1, x_95); +lean_ctor_set(x_96, 2, x_94); +x_97 = l_Lean_Elab_Command_elabDeclaration___closed__10; +x_98 = lean_array_push(x_97, x_86); +x_99 = lean_array_push(x_98, x_70); +x_100 = lean_array_push(x_99, x_96); +x_101 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_101, 0, x_84); +lean_ctor_set(x_101, 1, x_91); +lean_ctor_set(x_101, 2, x_100); +lean_inc(x_101); +x_102 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabCommand), 4, 1); +lean_closure_set(x_102, 0, x_101); +x_103 = l_Lean_Elab_Command_withMacroExpansion___rarg(x_1, x_101, x_102, x_2, x_3, x_78); +return x_103; } } else { -uint8_t x_77; +uint8_t x_104; lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_77 = !lean_is_exclusive(x_6); -if (x_77 == 0) +x_104 = !lean_is_exclusive(x_6); +if (x_104 == 0) { return x_6; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_6, 0); -x_79 = lean_ctor_get(x_6, 1); -lean_inc(x_79); -lean_inc(x_78); +lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_105 = lean_ctor_get(x_6, 0); +x_106 = lean_ctor_get(x_6, 1); +lean_inc(x_106); +lean_inc(x_105); lean_dec(x_6); -x_80 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_80, 0, x_78); -lean_ctor_set(x_80, 1, x_79); -return x_80; +x_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; } } } @@ -7362,7 +7450,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabDeclaration_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(179u); +x_1 = lean_unsigned_to_nat(178u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7374,7 +7462,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabDeclaration_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(200u); +x_1 = lean_unsigned_to_nat(202u); x_2 = lean_unsigned_to_nat(41u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7402,7 +7490,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabDeclaration_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(179u); +x_1 = lean_unsigned_to_nat(178u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7414,7 +7502,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabDeclaration_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(179u); +x_1 = lean_unsigned_to_nat(178u); x_2 = lean_unsigned_to_nat(19u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -8853,7 +8941,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualNamespace _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(244u); +x_1 = lean_unsigned_to_nat(246u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -8865,7 +8953,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualNamespace _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(261u); +x_1 = lean_unsigned_to_nat(263u); x_2 = lean_unsigned_to_nat(34u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -8893,7 +8981,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualNamespace _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(244u); +x_1 = lean_unsigned_to_nat(246u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -8905,7 +8993,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualNamespace _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(244u); +x_1 = lean_unsigned_to_nat(246u); x_2 = lean_unsigned_to_nat(25u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9329,7 +9417,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualElement_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(264u); +x_1 = lean_unsigned_to_nat(266u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9341,7 +9429,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualElement_d _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(276u); x_2 = lean_unsigned_to_nat(26u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9369,7 +9457,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualElement_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(264u); +x_1 = lean_unsigned_to_nat(266u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9381,7 +9469,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualElement_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(264u); +x_1 = lean_unsigned_to_nat(266u); x_2 = lean_unsigned_to_nat(23u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9629,7 +9717,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(277u); +x_1 = lean_unsigned_to_nat(279u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9641,7 +9729,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(284u); +x_1 = lean_unsigned_to_nat(286u); x_2 = lean_unsigned_to_nat(74u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9669,7 +9757,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(277u); +x_1 = lean_unsigned_to_nat(279u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9681,7 +9769,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandMutualPreamble_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(277u); +x_1 = lean_unsigned_to_nat(279u); x_2 = lean_unsigned_to_nat(24u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10244,7 +10332,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabMutual_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(287u); +x_1 = lean_unsigned_to_nat(289u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10256,7 +10344,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabMutual_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(304u); +x_1 = lean_unsigned_to_nat(306u); x_2 = lean_unsigned_to_nat(37u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10284,7 +10372,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabMutual_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(287u); +x_1 = lean_unsigned_to_nat(289u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10296,7 +10384,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabMutual_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(287u); +x_1 = lean_unsigned_to_nat(289u); x_2 = lean_unsigned_to_nat(14u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10342,22 +10430,6 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_array_push(x_3, x_1); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_2); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_9); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_7); -return x_11; -} -} static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__1() { _start: { @@ -10380,7 +10452,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAt _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("unknown attribute [", 19); +x_1 = lean_mk_string_from_bytes("unknown attribute [{attrName}]", 30); return x_1; } } @@ -10389,24 +10461,18 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAt { lean_object* x_1; lean_object* x_2; x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); return x_2; } } static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("]", 1); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); +x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); return x_2; } } @@ -10418,7 +10484,6 @@ x_8 = lean_usize_dec_lt(x_3, x_2); if (x_8 == 0) { lean_object* x_9; -lean_dec(x_5); x_9 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_9, 0, x_4); lean_ctor_set(x_9, 1, x_7); @@ -10452,10 +10517,8 @@ goto _start; else { lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -lean_free_object(x_4); x_21 = lean_unsigned_to_nat(1u); x_22 = l_Lean_Syntax_getArg(x_10, x_21); -lean_dec(x_10); x_23 = l_Lean_Syntax_getId(x_22); lean_dec(x_22); x_24 = lean_erase_macro_scopes(x_23); @@ -10473,163 +10536,115 @@ x_29 = l_Lean_isAttribute(x_28, x_24); lean_dec(x_28); if (x_29 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -lean_dec(x_13); -lean_dec(x_12); -x_30 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_30, 0, x_24); -x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4; -x_32 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_30); -x_33 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6; -x_34 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_34, x_5, x_6, x_27); -x_36 = !lean_is_exclusive(x_35); -if (x_36 == 0) -{ -return x_35; -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_35, 0); -x_38 = lean_ctor_get(x_35, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_35); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; -} +lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; size_t x_34; size_t x_35; +lean_dec(x_24); +x_30 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; +x_31 = 2; +x_32 = l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(x_10, x_30, x_31, x_5, x_6, x_27); +lean_dec(x_10); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = 1; +x_35 = lean_usize_add(x_3, x_34); +x_3 = x_35; +x_7 = x_33; +goto _start; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; size_t x_45; size_t x_46; -x_40 = lean_box(0); -x_41 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___lambda__1(x_24, x_12, x_13, x_40, x_5, x_6, x_27); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = lean_ctor_get(x_42, 0); -lean_inc(x_44); -lean_dec(x_42); -x_45 = 1; -x_46 = lean_usize_add(x_3, x_45); -x_3 = x_46; -x_4 = x_44; -x_7 = x_43; +lean_object* x_37; size_t x_38; size_t x_39; +lean_dec(x_10); +x_37 = lean_array_push(x_13, x_24); +lean_ctor_set(x_4, 1, x_37); +x_38 = 1; +x_39 = lean_usize_add(x_3, x_38); +x_3 = x_39; +x_7 = x_27; goto _start; } } } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; -x_48 = lean_ctor_get(x_4, 0); -x_49 = lean_ctor_get(x_4, 1); -lean_inc(x_49); -lean_inc(x_48); +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; +x_41 = lean_ctor_get(x_4, 0); +x_42 = lean_ctor_get(x_4, 1); +lean_inc(x_42); +lean_inc(x_41); lean_dec(x_4); lean_inc(x_10); -x_50 = l_Lean_Syntax_getKind(x_10); -x_51 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__2; -x_52 = lean_name_eq(x_50, x_51); -lean_dec(x_50); -if (x_52 == 0) +x_43 = l_Lean_Syntax_getKind(x_10); +x_44 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__2; +x_45 = lean_name_eq(x_43, x_44); +lean_dec(x_43); +if (x_45 == 0) { -lean_object* x_53; lean_object* x_54; size_t x_55; size_t x_56; -x_53 = lean_array_push(x_48, x_10); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_49); -x_55 = 1; -x_56 = lean_usize_add(x_3, x_55); -x_3 = x_56; -x_4 = x_54; +lean_object* x_46; lean_object* x_47; size_t x_48; size_t x_49; +x_46 = lean_array_push(x_41, x_10); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_42); +x_48 = 1; +x_49 = lean_usize_add(x_3, x_48); +x_3 = x_49; +x_4 = x_47; goto _start; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; -x_58 = lean_unsigned_to_nat(1u); -x_59 = l_Lean_Syntax_getArg(x_10, x_58); +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; +x_51 = lean_unsigned_to_nat(1u); +x_52 = l_Lean_Syntax_getArg(x_10, x_51); +x_53 = l_Lean_Syntax_getId(x_52); +lean_dec(x_52); +x_54 = lean_erase_macro_scopes(x_53); +x_55 = lean_st_ref_get(x_6, x_7); +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +lean_dec(x_55); +x_58 = lean_ctor_get(x_56, 0); +lean_inc(x_58); +lean_dec(x_56); +lean_inc(x_54); +x_59 = l_Lean_isAttribute(x_58, x_54); +lean_dec(x_58); +if (x_59 == 0) +{ +lean_object* x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; size_t x_65; size_t x_66; +lean_dec(x_54); +x_60 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; +x_61 = 2; +x_62 = l_Lean_logAt___at_Lean_Elab_Command_runLinters___spec__2(x_10, x_60, x_61, x_5, x_6, x_57); lean_dec(x_10); -x_60 = l_Lean_Syntax_getId(x_59); -lean_dec(x_59); -x_61 = lean_erase_macro_scopes(x_60); -x_62 = lean_st_ref_get(x_6, x_7); -x_63 = lean_ctor_get(x_62, 0); +x_63 = lean_ctor_get(x_62, 1); lean_inc(x_63); -x_64 = lean_ctor_get(x_62, 1); -lean_inc(x_64); lean_dec(x_62); -x_65 = lean_ctor_get(x_63, 0); -lean_inc(x_65); -lean_dec(x_63); -lean_inc(x_61); -x_66 = l_Lean_isAttribute(x_65, x_61); -lean_dec(x_65); -if (x_66 == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -lean_dec(x_49); -lean_dec(x_48); -x_67 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_67, 0, x_61); -x_68 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4; -x_69 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_67); -x_70 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6; -x_71 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_70); -x_72 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_71, x_5, x_6, x_64); -x_73 = lean_ctor_get(x_72, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_72, 1); -lean_inc(x_74); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_75 = x_72; -} else { - lean_dec_ref(x_72); - x_75 = lean_box(0); -} -if (lean_is_scalar(x_75)) { - x_76 = lean_alloc_ctor(1, 2, 0); -} else { - x_76 = x_75; -} -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_74); -return x_76; +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_41); +lean_ctor_set(x_64, 1, x_42); +x_65 = 1; +x_66 = lean_usize_add(x_3, x_65); +x_3 = x_66; +x_4 = x_64; +x_7 = x_63; +goto _start; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; size_t x_82; size_t x_83; -x_77 = lean_box(0); -x_78 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___lambda__1(x_61, x_48, x_49, x_77, x_5, x_6, x_64); -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -lean_dec(x_78); -x_81 = lean_ctor_get(x_79, 0); -lean_inc(x_81); -lean_dec(x_79); -x_82 = 1; -x_83 = lean_usize_add(x_3, x_82); -x_3 = x_83; -x_4 = x_81; -x_7 = x_80; +lean_object* x_68; lean_object* x_69; size_t x_70; size_t x_71; +lean_dec(x_10); +x_68 = lean_array_push(x_42, x_54); +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_41); +lean_ctor_set(x_69, 1, x_68); +x_70 = 1; +x_71 = lean_usize_add(x_3, x_70); +x_3 = x_71; +x_4 = x_69; +x_7 = x_57; goto _start; } } @@ -10674,7 +10689,7 @@ lean_dec(x_13); x_15 = lean_st_ref_get(x_4, x_14); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 4); +x_17 = lean_ctor_get(x_16, 5); lean_inc(x_17); lean_dec(x_16); x_18 = lean_ctor_get_uint8(x_17, sizeof(void*)*2); @@ -10922,7 +10937,9 @@ x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); lean_dec(x_13); lean_inc(x_11); -lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); lean_inc(x_6); lean_inc(x_14); x_16 = l_Lean_Elab_Term_applyAttributes(x_14, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_15); @@ -11167,7 +11184,7 @@ return x_2; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabAttr(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; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_5 = lean_unsigned_to_nat(2u); x_6 = l_Lean_Syntax_getArg(x_1, x_5); x_7 = l_Lean_Syntax_getSepArgs(x_6); @@ -11177,12 +11194,8 @@ x_9 = lean_usize_of_nat(x_8); lean_dec(x_8); x_10 = 0; x_11 = l_Lean_Elab_Command_elabAttr___closed__1; -lean_inc(x_2); x_12 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1(x_7, x_9, x_10, x_11, x_2, x_3, x_4); lean_dec(x_7); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); @@ -11290,42 +11303,6 @@ return x_38; } } } -else -{ -uint8_t x_39; -lean_dec(x_3); -lean_dec(x_2); -x_39 = !lean_is_exclusive(x_12); -if (x_39 == 0) -{ -return x_12; -} -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_12, 0); -x_41 = lean_ctor_get(x_12, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_12); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -return x_42; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_8; -} } LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: @@ -11337,6 +11314,7 @@ x_9 = lean_unbox_usize(x_3); lean_dec(x_3); x_10 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1(x_1, x_8, x_9, x_4, x_5, x_6, x_7); lean_dec(x_6); +lean_dec(x_5); lean_dec(x_1); return x_10; } @@ -11471,7 +11449,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(307u); +x_1 = lean_unsigned_to_nat(309u); x_2 = lean_unsigned_to_nat(34u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -11483,7 +11461,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(324u); +x_1 = lean_unsigned_to_nat(327u); x_2 = lean_unsigned_to_nat(39u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -11511,7 +11489,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(307u); +x_1 = lean_unsigned_to_nat(309u); x_2 = lean_unsigned_to_nat(38u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -11523,7 +11501,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(307u); +x_1 = lean_unsigned_to_nat(309u); x_2 = lean_unsigned_to_nat(46u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -11569,2997 +11547,2975 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declModifiers", 13); +x_1 = lean_mk_string_from_bytes("invalid initialization command, unexpected modifiers", 52); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(6u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Term", 4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__2; +x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__4; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__3; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3; +x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__5() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("attributes", 10); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__4; +x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__5; +x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("@[", 2); +x_1 = lean_mk_string_from_bytes("declId", 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__8() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__8() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("attrInstance", 12); +x_1 = lean_mk_string_from_bytes("initFn", 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__9() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__8; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__8; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__10() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("attrKind", 8); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__8; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__9; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__11() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__10; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__12() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_elabInductive___closed__1; -x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("optDeclSig", 10); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__13() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__11; -x_3 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__12; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("typeSpec", 8); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__14() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Attr", 4); +x_1 = lean_mk_string_from_bytes(":", 1); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__15() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__4; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__14; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("app", 3); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__16() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__16() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("simple", 6); +x_1 = lean_mk_string_from_bytes("IO", 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__17() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__15; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__16; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__16; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__16; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__17; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__18() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_elabDeclaration___closed__7; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__13; -x_3 = lean_array_push(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__16; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__19() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(6u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__19; -x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_3 = lean_array_push(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__21() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declId", 6); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__20; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__21; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l_Lean_Elab_Command_elabDeclaration___closed__7; +x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__23() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("initFn", 6); +x_1 = lean_mk_string_from_bytes("declValSimple", 13); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__24() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__23; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__23; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__24; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__23; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(":=", 2); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__27() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("optDeclSig", 10); +x_1 = lean_mk_string_from_bytes("do", 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__27; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(7u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__29() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("typeSpec", 8); +x_1 = lean_mk_string_from_bytes("attributes", 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__29; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("@[", 2); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes(":", 1); +x_1 = lean_mk_string_from_bytes("attrInstance", 12); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__32() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("app", 3); +x_1 = lean_mk_string_from_bytes("attrKind", 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__32; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l_Lean_Elab_Command_elabInductive___closed__1; +x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__34() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("IO", 2); +x_1 = lean_mk_string_from_bytes("Attr", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__35() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__34; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__34; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__35; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("simple", 6); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__34() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__34; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(",", 1); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__38() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("]", 1); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__36() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__38; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("declSig", 7); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__40() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__37() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Unit", 4); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(4u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__41() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__38() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__40; -x_2 = lean_string_utf8_byte_size(x_1); +x_1 = l_Lean_Elab_Command_elabAxiom___lambda__5___closed__3; +x_2 = l_Array_append___rarg(x_1, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__42() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__39() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__40; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__41; -x_4 = lean_alloc_ctor(0, 3, 0); +x_1 = lean_box(2); +x_2 = l_Lean_Elab_Command_elabDeclaration___closed__4; +x_3 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__38; +x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__43() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__40; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__44() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__40() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__43; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("unsafe", 6); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__45() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___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) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__44; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46() { -_start: +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_unsigned_to_nat(5u); +x_19 = l_Lean_Syntax_getArg(x_1, x_18); +x_20 = lean_unsigned_to_nat(0u); +x_21 = l_Lean_Syntax_matchesNull(x_19, x_20); +if (x_21 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_elabDeclaration___closed__7; -x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} +lean_object* x_22; lean_object* x_23; +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); +x_22 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_23 = l_Lean_Macro_throwErrorAt___rarg(x_2, x_22, x_16, x_17); +return x_23; } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__47() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declValSimple", 13); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48() { -_start: +lean_object* x_24; lean_object* x_25; +x_24 = l_Lean_Syntax_getOptional_x3f(x_3); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__47; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +lean_object* x_223; +x_223 = lean_box(0); +x_25 = x_223; +goto block_222; } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(":=", 2); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50() { -_start: +uint8_t x_224; +x_224 = !lean_is_exclusive(x_24); +if (x_224 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("do", 2); -return x_1; -} +x_25 = x_24; +goto block_222; } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_225; lean_object* x_226; +x_225 = lean_ctor_get(x_24, 0); +lean_inc(x_225); +lean_dec(x_24); +x_226 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_226, 0, x_225); +x_25 = x_226; +goto block_222; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52() { -_start: +block_222: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(7u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; -} +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +lean_inc(x_16); +x_26 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_16, x_17); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +if (lean_is_exclusive(x_26)) { + lean_ctor_release(x_26, 0); + lean_ctor_release(x_26, 1); + x_29 = x_26; +} else { + lean_dec_ref(x_26); + x_29 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; uint8_t x_7; +x_30 = lean_ctor_get(x_16, 2); +lean_inc(x_30); +x_31 = lean_ctor_get(x_16, 1); +lean_inc(x_31); +lean_dec(x_16); +x_32 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__7; lean_inc(x_4); -x_6 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_4, x_5); -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_ctor_get(x_4, 2); -lean_inc(x_9); -x_10 = lean_ctor_get(x_4, 1); -lean_inc(x_10); -lean_dec(x_4); -x_11 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; -lean_inc(x_8); -x_12 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_12, 0, x_8); -lean_ctor_set(x_12, 1, x_11); -x_13 = l_Lean_Elab_Command_elabDeclaration___closed__7; -x_14 = lean_array_push(x_13, x_1); -x_15 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_16 = lean_array_push(x_14, x_15); -x_17 = lean_box(2); -x_18 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set(x_19, 2, x_16); -x_20 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__18; -x_21 = lean_array_push(x_20, x_19); -x_22 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_17); -lean_ctor_set(x_23, 1, x_22); -lean_ctor_set(x_23, 2, x_21); -x_24 = l_Lean_Elab_Command_elabInductive___closed__1; -x_25 = lean_array_push(x_24, x_23); -x_26 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_27 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_27, 0, x_17); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_25); -x_28 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -lean_inc(x_8); -x_29 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_29, 0, x_8); -lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_31 = lean_array_push(x_30, x_12); -x_32 = lean_array_push(x_31, x_27); -x_33 = lean_array_push(x_32, x_29); -x_34 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; -x_35 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_35, 0, x_17); -lean_ctor_set(x_35, 1, x_34); -lean_ctor_set(x_35, 2, x_33); -x_36 = lean_array_push(x_24, x_35); -x_37 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_37, 0, x_17); -lean_ctor_set(x_37, 1, x_26); -lean_ctor_set(x_37, 2, x_36); -x_38 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_39 = lean_array_push(x_38, x_37); -x_40 = lean_array_push(x_39, x_15); -x_41 = lean_array_push(x_40, x_15); -x_42 = lean_array_push(x_41, x_15); -x_43 = lean_array_push(x_42, x_15); -x_44 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_45 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_45, 0, x_17); -lean_ctor_set(x_45, 1, x_44); -lean_ctor_set(x_45, 2, x_43); -x_46 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; -lean_inc(x_8); -x_47 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_47, 0, x_8); -lean_ctor_set(x_47, 1, x_46); -x_48 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; -lean_inc(x_9); -lean_inc(x_10); -x_49 = l_Lean_addMacroScope(x_10, x_48, x_9); -x_50 = lean_box(0); -x_51 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -lean_inc(x_8); -x_52 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_52, 0, x_8); -lean_ctor_set(x_52, 1, x_51); -lean_ctor_set(x_52, 2, x_49); -lean_ctor_set(x_52, 3, x_50); -x_53 = lean_array_push(x_13, x_52); -x_54 = lean_array_push(x_53, x_15); -x_55 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; -x_56 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_56, 0, x_17); -lean_ctor_set(x_56, 1, x_55); -lean_ctor_set(x_56, 2, x_54); -x_57 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; -lean_inc(x_8); -x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_8); -lean_ctor_set(x_58, 1, x_57); -x_59 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -lean_inc(x_9); -lean_inc(x_10); -x_60 = l_Lean_addMacroScope(x_10, x_59, x_9); -x_61 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -x_62 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; -lean_inc(x_8); -x_63 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_63, 0, x_8); -lean_ctor_set(x_63, 1, x_61); -lean_ctor_set(x_63, 2, x_60); -lean_ctor_set(x_63, 3, x_62); -x_64 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__43; -x_65 = l_Lean_addMacroScope(x_10, x_64, x_9); -x_66 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__42; -x_67 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__45; -lean_inc(x_8); -x_68 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_68, 0, x_8); -lean_ctor_set(x_68, 1, x_66); -lean_ctor_set(x_68, 2, x_65); -lean_ctor_set(x_68, 3, x_67); -x_69 = lean_array_push(x_24, x_68); -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_17); -lean_ctor_set(x_70, 1, x_26); -lean_ctor_set(x_70, 2, x_69); -x_71 = lean_array_push(x_13, x_63); -x_72 = lean_array_push(x_71, x_70); -x_73 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; +x_33 = l_Lean_Name_str___override(x_4, x_32); +x_34 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; +lean_inc(x_4); +x_35 = l_Lean_Name_str___override(x_4, x_34); +lean_inc(x_27); +x_36 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_36, 0, x_27); +lean_ctor_set(x_36, 1, x_34); +x_37 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7; +lean_inc(x_4); +x_38 = l_Lean_Name_str___override(x_4, x_37); +x_39 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11; +lean_inc(x_30); +lean_inc(x_31); +x_40 = l_Lean_addMacroScope(x_31, x_39, x_30); +x_41 = lean_box(0); +x_42 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10; +lean_inc(x_27); +x_43 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_43, 0, x_27); +lean_ctor_set(x_43, 1, x_42); +lean_ctor_set(x_43, 2, x_40); +lean_ctor_set(x_43, 3, x_41); +x_44 = l_Lean_Elab_Command_elabDeclaration___closed__7; +lean_inc(x_43); +x_45 = lean_array_push(x_44, x_43); +x_46 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_47 = lean_array_push(x_45, x_46); +x_48 = lean_box(2); +lean_inc(x_38); +x_49 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_38); +lean_ctor_set(x_49, 2, x_47); +x_50 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12; +lean_inc(x_4); +x_51 = l_Lean_Name_str___override(x_4, x_50); +x_52 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13; +lean_inc(x_5); +x_53 = l_Lean_Name_str___override(x_5, x_52); +x_54 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14; +lean_inc(x_27); +x_55 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_55, 0, x_27); +lean_ctor_set(x_55, 1, x_54); +x_56 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15; +lean_inc(x_5); +x_57 = l_Lean_Name_str___override(x_5, x_56); +x_58 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19; +x_59 = l_Lean_addMacroScope(x_31, x_58, x_30); +x_60 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18; +x_61 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21; +lean_inc(x_27); +x_62 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_62, 0, x_27); +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_Elab_Command_elabInductive___closed__1; +lean_inc(x_6); +x_64 = lean_array_push(x_63, x_6); +x_65 = l_Lean_Elab_Command_elabDeclaration___closed__4; +x_66 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_66, 0, x_48); +lean_ctor_set(x_66, 1, x_65); +lean_ctor_set(x_66, 2, x_64); +x_67 = lean_array_push(x_44, x_62); +x_68 = lean_array_push(x_67, x_66); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_48); +lean_ctor_set(x_69, 1, x_57); +lean_ctor_set(x_69, 2, x_68); +x_70 = lean_array_push(x_44, x_55); +lean_inc(x_70); +x_71 = lean_array_push(x_70, x_69); +lean_inc(x_53); +x_72 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_72, 0, x_48); +lean_ctor_set(x_72, 1, x_53); +lean_ctor_set(x_72, 2, x_71); +x_73 = lean_array_push(x_63, x_72); x_74 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_74, 0, x_17); -lean_ctor_set(x_74, 1, x_73); -lean_ctor_set(x_74, 2, x_72); -x_75 = lean_array_push(x_13, x_58); +lean_ctor_set(x_74, 0, x_48); +lean_ctor_set(x_74, 1, x_65); +lean_ctor_set(x_74, 2, x_73); +x_75 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22; x_76 = lean_array_push(x_75, x_74); -x_77 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; -x_78 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_78, 0, x_17); -lean_ctor_set(x_78, 1, x_77); -lean_ctor_set(x_78, 2, x_76); -x_79 = lean_array_push(x_24, x_78); -x_80 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_80, 0, x_17); -lean_ctor_set(x_80, 1, x_26); -lean_ctor_set(x_80, 2, x_79); -x_81 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; -x_82 = lean_array_push(x_81, x_80); -x_83 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; -x_84 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_84, 0, x_17); -lean_ctor_set(x_84, 1, x_83); -lean_ctor_set(x_84, 2, x_82); -x_85 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; -lean_inc(x_8); -x_86 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_86, 0, x_8); -lean_ctor_set(x_86, 1, x_85); -x_87 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -x_88 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_88, 0, x_8); -lean_ctor_set(x_88, 1, x_87); -x_89 = lean_array_push(x_13, x_88); -x_90 = lean_array_push(x_89, x_2); -x_91 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; +x_77 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_77, 0, x_48); +lean_ctor_set(x_77, 1, x_51); +lean_ctor_set(x_77, 2, x_76); +x_78 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23; +lean_inc(x_4); +x_79 = l_Lean_Name_str___override(x_4, x_78); +x_80 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24; +lean_inc(x_27); +x_81 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_81, 0, x_27); +lean_ctor_set(x_81, 1, x_80); +x_82 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25; +lean_inc(x_5); +x_83 = l_Lean_Name_str___override(x_5, x_82); +lean_inc(x_27); +x_84 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_84, 0, x_27); +lean_ctor_set(x_84, 1, x_82); +x_85 = lean_array_push(x_44, x_84); +x_86 = lean_array_push(x_85, x_7); +x_87 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_87, 0, x_48); +lean_ctor_set(x_87, 1, x_83); +lean_ctor_set(x_87, 2, x_86); +x_88 = l_Lean_Elab_Command_elabDeclaration___closed__10; +x_89 = lean_array_push(x_88, x_81); +x_90 = lean_array_push(x_89, x_87); +x_91 = lean_array_push(x_90, x_46); x_92 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_92, 0, x_17); -lean_ctor_set(x_92, 1, x_91); -lean_ctor_set(x_92, 2, x_90); -x_93 = lean_array_push(x_30, x_86); -x_94 = lean_array_push(x_93, x_92); -x_95 = lean_array_push(x_94, x_15); -x_96 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; -x_97 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_97, 0, x_17); -lean_ctor_set(x_97, 1, x_96); -lean_ctor_set(x_97, 2, x_95); -x_98 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; -x_99 = lean_array_push(x_98, x_47); -x_100 = lean_array_push(x_99, x_56); -x_101 = lean_array_push(x_100, x_84); -x_102 = lean_array_push(x_101, x_97); -x_103 = lean_array_push(x_102, x_15); -x_104 = lean_array_push(x_103, x_15); -x_105 = lean_array_push(x_104, x_15); -x_106 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -x_107 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_107, 0, x_17); -lean_ctor_set(x_107, 1, x_106); -lean_ctor_set(x_107, 2, x_105); -x_108 = lean_array_push(x_13, x_45); -x_109 = lean_array_push(x_108, x_107); -x_110 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; +lean_ctor_set(x_92, 0, x_48); +lean_ctor_set(x_92, 1, x_79); +lean_ctor_set(x_92, 2, x_91); +x_93 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26; +x_94 = lean_array_push(x_93, x_36); +x_95 = lean_array_push(x_94, x_49); +x_96 = lean_array_push(x_95, x_77); +x_97 = lean_array_push(x_96, x_92); +x_98 = lean_array_push(x_97, x_46); +x_99 = lean_array_push(x_98, x_46); +x_100 = lean_array_push(x_99, x_46); +x_101 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_101, 0, x_48); +lean_ctor_set(x_101, 1, x_35); +lean_ctor_set(x_101, 2, x_100); +x_102 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27; +lean_inc(x_5); +x_103 = l_Lean_Name_str___override(x_5, x_102); +x_104 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28; +lean_inc(x_27); +x_105 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_105, 0, x_27); +lean_ctor_set(x_105, 1, x_104); +x_106 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29; +lean_inc(x_5); +x_107 = l_Lean_Name_str___override(x_5, x_106); +x_108 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30; +x_109 = l_Lean_Name_str___override(x_5, x_108); +x_110 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31; x_111 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_111, 0, x_17); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_111, 2, x_109); -lean_ctor_set(x_6, 0, x_111); -return x_6; -} -else -{ -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; -x_112 = lean_ctor_get(x_6, 0); -x_113 = lean_ctor_get(x_6, 1); -lean_inc(x_113); -lean_inc(x_112); -lean_dec(x_6); -x_114 = lean_ctor_get(x_4, 2); -lean_inc(x_114); -x_115 = lean_ctor_get(x_4, 1); -lean_inc(x_115); -lean_dec(x_4); -x_116 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; -lean_inc(x_112); -x_117 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_117, 0, x_112); -lean_ctor_set(x_117, 1, x_116); -x_118 = l_Lean_Elab_Command_elabDeclaration___closed__7; -x_119 = lean_array_push(x_118, x_1); -x_120 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_121 = lean_array_push(x_119, x_120); -x_122 = lean_box(2); -x_123 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; -x_124 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_124, 0, x_122); -lean_ctor_set(x_124, 1, x_123); -lean_ctor_set(x_124, 2, x_121); -x_125 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__18; -x_126 = lean_array_push(x_125, x_124); -x_127 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -x_128 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_128, 0, x_122); -lean_ctor_set(x_128, 1, x_127); -lean_ctor_set(x_128, 2, x_126); -x_129 = l_Lean_Elab_Command_elabInductive___closed__1; -x_130 = lean_array_push(x_129, x_128); -x_131 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_132 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_132, 0, x_122); -lean_ctor_set(x_132, 1, x_131); -lean_ctor_set(x_132, 2, x_130); -x_133 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -lean_inc(x_112); -x_134 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_134, 0, x_112); -lean_ctor_set(x_134, 1, x_133); -x_135 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_136 = lean_array_push(x_135, x_117); -x_137 = lean_array_push(x_136, x_132); -x_138 = lean_array_push(x_137, x_134); -x_139 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; +lean_ctor_set(x_111, 0, x_48); +lean_ctor_set(x_111, 1, x_109); +lean_ctor_set(x_111, 2, x_110); +x_112 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32; +x_113 = l_Lean_Name_str___override(x_8, x_112); +x_114 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33; +x_115 = l_Lean_Name_str___override(x_113, x_114); +x_116 = lean_array_push(x_63, x_43); +x_117 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_117, 0, x_48); +lean_ctor_set(x_117, 1, x_65); +lean_ctor_set(x_117, 2, x_116); +x_118 = lean_array_push(x_44, x_9); +x_119 = lean_array_push(x_118, x_117); +x_120 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_120, 0, x_48); +lean_ctor_set(x_120, 1, x_115); +lean_ctor_set(x_120, 2, x_119); +x_121 = lean_array_push(x_44, x_111); +x_122 = lean_array_push(x_121, x_120); +x_123 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_123, 0, x_48); +lean_ctor_set(x_123, 1, x_107); +lean_ctor_set(x_123, 2, x_122); +x_124 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__34; +lean_inc(x_27); +x_125 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_125, 0, x_27); +lean_ctor_set(x_125, 1, x_124); +x_126 = lean_array_push(x_44, x_123); +x_127 = lean_array_push(x_126, x_125); +x_128 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35; +lean_inc(x_27); +x_129 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_129, 0, x_27); +lean_ctor_set(x_129, 1, x_128); +x_130 = lean_array_push(x_88, x_105); +x_131 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__15; +lean_inc(x_4); +x_132 = l_Lean_Name_str___override(x_4, x_131); +lean_inc(x_27); +x_133 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_133, 0, x_27); +lean_ctor_set(x_133, 1, x_131); +x_134 = lean_array_push(x_44, x_10); +x_135 = lean_array_push(x_134, x_46); +x_136 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_136, 0, x_48); +lean_ctor_set(x_136, 1, x_38); +lean_ctor_set(x_136, 2, x_135); +x_137 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__36; +lean_inc(x_4); +x_138 = l_Lean_Name_str___override(x_4, x_137); +x_139 = lean_array_push(x_70, x_6); x_140 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_140, 0, x_122); -lean_ctor_set(x_140, 1, x_139); -lean_ctor_set(x_140, 2, x_138); -x_141 = lean_array_push(x_129, x_140); +lean_ctor_set(x_140, 0, x_48); +lean_ctor_set(x_140, 1, x_53); +lean_ctor_set(x_140, 2, x_139); +x_141 = lean_array_push(x_75, x_140); x_142 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_142, 0, x_122); -lean_ctor_set(x_142, 1, x_131); +lean_ctor_set(x_142, 0, x_48); +lean_ctor_set(x_142, 1, x_138); lean_ctor_set(x_142, 2, x_141); -x_143 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_144 = lean_array_push(x_143, x_142); -x_145 = lean_array_push(x_144, x_120); -x_146 = lean_array_push(x_145, x_120); -x_147 = lean_array_push(x_146, x_120); -x_148 = lean_array_push(x_147, x_120); -x_149 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_150 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_150, 0, x_122); -lean_ctor_set(x_150, 1, x_149); -lean_ctor_set(x_150, 2, x_148); -x_151 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; -lean_inc(x_112); -x_152 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_152, 0, x_112); -lean_ctor_set(x_152, 1, x_151); -x_153 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; -lean_inc(x_114); -lean_inc(x_115); -x_154 = l_Lean_addMacroScope(x_115, x_153, x_114); -x_155 = lean_box(0); -x_156 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -lean_inc(x_112); -x_157 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_157, 0, x_112); -lean_ctor_set(x_157, 1, x_156); -lean_ctor_set(x_157, 2, x_154); -lean_ctor_set(x_157, 3, x_155); -x_158 = lean_array_push(x_118, x_157); -x_159 = lean_array_push(x_158, x_120); -x_160 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; -x_161 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_161, 0, x_122); -lean_ctor_set(x_161, 1, x_160); -lean_ctor_set(x_161, 2, x_159); -x_162 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; -lean_inc(x_112); -x_163 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_163, 0, x_112); -lean_ctor_set(x_163, 1, x_162); -x_164 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -lean_inc(x_114); -lean_inc(x_115); -x_165 = l_Lean_addMacroScope(x_115, x_164, x_114); -x_166 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -x_167 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; -lean_inc(x_112); -x_168 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_168, 0, x_112); -lean_ctor_set(x_168, 1, x_166); -lean_ctor_set(x_168, 2, x_165); -lean_ctor_set(x_168, 3, x_167); -x_169 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__43; -x_170 = l_Lean_addMacroScope(x_115, x_169, x_114); -x_171 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__42; -x_172 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__45; -lean_inc(x_112); -x_173 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_173, 0, x_112); -lean_ctor_set(x_173, 1, x_171); -lean_ctor_set(x_173, 2, x_170); -lean_ctor_set(x_173, 3, x_172); -x_174 = lean_array_push(x_129, x_173); -x_175 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_175, 0, x_122); -lean_ctor_set(x_175, 1, x_131); -lean_ctor_set(x_175, 2, x_174); -x_176 = lean_array_push(x_118, x_168); -x_177 = lean_array_push(x_176, x_175); -x_178 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; -x_179 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_179, 0, x_122); -lean_ctor_set(x_179, 1, x_178); -lean_ctor_set(x_179, 2, x_177); -x_180 = lean_array_push(x_118, x_163); -x_181 = lean_array_push(x_180, x_179); -x_182 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; +x_143 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__37; +x_144 = lean_array_push(x_143, x_133); +x_145 = lean_array_push(x_144, x_136); +x_146 = lean_array_push(x_145, x_142); +x_147 = lean_array_push(x_146, x_46); +x_148 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_148, 0, x_48); +lean_ctor_set(x_148, 1, x_132); +lean_ctor_set(x_148, 2, x_147); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_208; +lean_dec(x_27); +lean_dec(x_4); +x_208 = l_Lean_Elab_Command_elabAxiom___lambda__5___closed__3; +x_149 = x_208; +goto block_207; +} +else +{ +lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_209 = lean_ctor_get(x_15, 0); +x_210 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__40; +x_211 = l_Lean_Name_str___override(x_4, x_210); +x_212 = l_Lean_Syntax_getHeadInfo_x3f(x_209); +if (lean_obj_tag(x_212) == 0) +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +x_213 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_213, 0, x_27); +lean_ctor_set(x_213, 1, x_210); +x_214 = lean_array_push(x_63, x_213); +x_215 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_215, 0, x_48); +lean_ctor_set(x_215, 1, x_211); +lean_ctor_set(x_215, 2, x_214); +x_216 = lean_array_push(x_63, x_215); +x_149 = x_216; +goto block_207; +} +else +{ +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; +lean_dec(x_27); +x_217 = lean_ctor_get(x_212, 0); +lean_inc(x_217); +lean_dec(x_212); +x_218 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_218, 0, x_217); +lean_ctor_set(x_218, 1, x_210); +x_219 = lean_array_push(x_63, x_218); +x_220 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_220, 0, x_48); +lean_ctor_set(x_220, 1, x_211); +lean_ctor_set(x_220, 2, x_219); +x_221 = lean_array_push(x_63, x_220); +x_149 = x_221; +goto block_207; +} +} +block_207: +{ +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; +x_150 = l_Lean_Elab_Command_elabAxiom___lambda__5___closed__3; +x_151 = l_Array_append___rarg(x_150, x_149); +x_152 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_152, 0, x_48); +lean_ctor_set(x_152, 1, x_65); +lean_ctor_set(x_152, 2, x_151); +x_153 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__6; +x_154 = lean_array_push(x_153, x_152); +x_155 = lean_array_push(x_154, x_46); +lean_inc(x_11); +x_156 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_156, 0, x_48); +lean_ctor_set(x_156, 1, x_11); +lean_ctor_set(x_156, 2, x_155); +x_157 = lean_array_push(x_44, x_156); +x_158 = lean_array_push(x_157, x_101); +lean_inc(x_33); +x_159 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_159, 0, x_48); +lean_ctor_set(x_159, 1, x_33); +lean_ctor_set(x_159, 2, x_158); +x_160 = lean_array_push(x_44, x_159); +if (lean_obj_tag(x_13) == 0) +{ +x_161 = x_150; +goto block_204; +} +else +{ +lean_object* x_205; lean_object* x_206; +x_205 = lean_ctor_get(x_13, 0); +lean_inc(x_205); +lean_dec(x_13); +x_206 = lean_array_push(x_63, x_205); +x_161 = x_206; +goto block_204; +} +block_204: +{ +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; +x_162 = l_Array_append___rarg(x_150, x_161); +x_163 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_163, 0, x_48); +lean_ctor_set(x_163, 1, x_65); +lean_ctor_set(x_163, 2, x_162); +x_164 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__2; +x_165 = lean_array_push(x_164, x_163); +if (lean_obj_tag(x_12) == 0) +{ +x_166 = x_150; +goto block_202; +} +else +{ +lean_object* x_203; +x_203 = lean_ctor_get(x_12, 0); +lean_inc(x_203); +lean_dec(x_12); +x_166 = x_203; +goto block_202; +} +block_202: +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; +x_167 = l_Array_append___rarg(x_127, x_166); +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_48); +lean_ctor_set(x_168, 1, x_65); +lean_ctor_set(x_168, 2, x_167); +x_169 = lean_array_push(x_130, x_168); +x_170 = lean_array_push(x_169, x_129); +x_171 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_171, 0, x_48); +lean_ctor_set(x_171, 1, x_103); +lean_ctor_set(x_171, 2, x_170); +x_172 = lean_array_push(x_63, x_171); +x_173 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_173, 0, x_48); +lean_ctor_set(x_173, 1, x_65); +lean_ctor_set(x_173, 2, x_172); +x_174 = lean_array_push(x_165, x_173); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; +x_175 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__39; +x_176 = lean_array_push(x_174, x_175); +x_177 = lean_array_push(x_176, x_46); +x_178 = lean_array_push(x_177, x_46); +x_179 = lean_array_push(x_178, x_46); +x_180 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_180, 0, x_48); +lean_ctor_set(x_180, 1, x_11); +lean_ctor_set(x_180, 2, x_179); +x_181 = lean_array_push(x_44, x_180); +x_182 = lean_array_push(x_181, x_148); x_183 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_183, 0, x_122); -lean_ctor_set(x_183, 1, x_182); -lean_ctor_set(x_183, 2, x_181); -x_184 = lean_array_push(x_129, x_183); +lean_ctor_set(x_183, 0, x_48); +lean_ctor_set(x_183, 1, x_33); +lean_ctor_set(x_183, 2, x_182); +x_184 = lean_array_push(x_160, x_183); x_185 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_185, 0, x_122); -lean_ctor_set(x_185, 1, x_131); +lean_ctor_set(x_185, 0, x_48); +lean_ctor_set(x_185, 1, x_65); lean_ctor_set(x_185, 2, x_184); -x_186 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; -x_187 = lean_array_push(x_186, x_185); -x_188 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; -x_189 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_189, 0, x_122); -lean_ctor_set(x_189, 1, x_188); -lean_ctor_set(x_189, 2, x_187); -x_190 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; -lean_inc(x_112); -x_191 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_191, 0, x_112); -lean_ctor_set(x_191, 1, x_190); -x_192 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -x_193 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_193, 0, x_112); -lean_ctor_set(x_193, 1, x_192); -x_194 = lean_array_push(x_118, x_193); -x_195 = lean_array_push(x_194, x_2); -x_196 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; -x_197 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_197, 0, x_122); -lean_ctor_set(x_197, 1, x_196); -lean_ctor_set(x_197, 2, x_195); -x_198 = lean_array_push(x_135, x_191); -x_199 = lean_array_push(x_198, x_197); -x_200 = lean_array_push(x_199, x_120); -x_201 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; -x_202 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_202, 0, x_122); -lean_ctor_set(x_202, 1, x_201); -lean_ctor_set(x_202, 2, x_200); -x_203 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; -x_204 = lean_array_push(x_203, x_152); -x_205 = lean_array_push(x_204, x_161); -x_206 = lean_array_push(x_205, x_189); -x_207 = lean_array_push(x_206, x_202); -x_208 = lean_array_push(x_207, x_120); -x_209 = lean_array_push(x_208, x_120); -x_210 = lean_array_push(x_209, x_120); -x_211 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -x_212 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_212, 0, x_122); -lean_ctor_set(x_212, 1, x_211); -lean_ctor_set(x_212, 2, x_210); -x_213 = lean_array_push(x_118, x_150); -x_214 = lean_array_push(x_213, x_212); -x_215 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; -x_216 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_216, 0, x_122); -lean_ctor_set(x_216, 1, x_215); -lean_ctor_set(x_216, 2, x_214); -x_217 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_217, 0, x_216); -lean_ctor_set(x_217, 1, x_113); -return x_217; -} -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__1() { -_start: +if (lean_is_scalar(x_29)) { + x_186 = lean_alloc_ctor(0, 2, 0); +} else { + x_186 = x_29; +} +lean_ctor_set(x_186, 0, x_185); +lean_ctor_set(x_186, 1, x_28); +return x_186; +} +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("private", 7); -return x_1; +lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_187 = lean_ctor_get(x_25, 0); +lean_inc(x_187); +lean_dec(x_25); +x_188 = lean_array_push(x_150, x_187); +x_189 = l_Array_append___rarg(x_150, x_188); +x_190 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_190, 0, x_48); +lean_ctor_set(x_190, 1, x_65); +lean_ctor_set(x_190, 2, x_189); +x_191 = lean_array_push(x_174, x_190); +x_192 = lean_array_push(x_191, x_46); +x_193 = lean_array_push(x_192, x_46); +x_194 = lean_array_push(x_193, x_46); +x_195 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_195, 0, x_48); +lean_ctor_set(x_195, 1, x_11); +lean_ctor_set(x_195, 2, x_194); +x_196 = lean_array_push(x_44, x_195); +x_197 = lean_array_push(x_196, x_148); +x_198 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_198, 0, x_48); +lean_ctor_set(x_198, 1, x_33); +lean_ctor_set(x_198, 2, x_197); +x_199 = lean_array_push(x_160, x_198); +x_200 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_200, 0, x_48); +lean_ctor_set(x_200, 1, x_65); +lean_ctor_set(x_200, 2, x_199); +if (lean_is_scalar(x_29)) { + x_201 = lean_alloc_ctor(0, 2, 0); +} else { + x_201 = x_29; +} +lean_ctor_set(x_201, 0, x_200); +lean_ctor_set(x_201, 1, x_28); +return x_201; +} +} +} } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__2() { +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l_Lean_Elab_Command_expandInitCmd___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_dec(x_12); +x_16 = lean_unsigned_to_nat(2u); +x_17 = l_Lean_Syntax_getArg(x_1, x_16); +x_18 = lean_unsigned_to_nat(3u); +x_19 = l_Lean_Syntax_getArg(x_1, x_18); +x_20 = lean_unsigned_to_nat(0u); +x_21 = l_Lean_Syntax_matchesNull(x_19, x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_22 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_23 = l_Lean_Macro_throwErrorAt___rarg(x_2, x_22, x_14, x_15); +return x_23; } +else +{ +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = lean_unsigned_to_nat(4u); +x_25 = l_Lean_Syntax_getArg(x_1, x_24); +x_26 = l_Lean_Syntax_isNone(x_25); +if (x_26 == 0) +{ +lean_object* x_27; uint8_t x_28; +x_27 = lean_unsigned_to_nat(1u); +lean_inc(x_25); +x_28 = l_Lean_Syntax_matchesNull(x_25, x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_25); +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_29 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_30 = l_Lean_Macro_throwErrorAt___rarg(x_2, x_29, x_14, x_15); +return x_30; } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("protected", 9); -return x_1; +lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_31 = l_Lean_Syntax_getArg(x_25, x_20); +lean_dec(x_25); +x_32 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__40; +lean_inc(x_3); +x_33 = l_Lean_Name_str___override(x_3, x_32); +lean_inc(x_31); +x_34 = l_Lean_Syntax_isOfKind(x_31, x_33); +lean_dec(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +lean_dec(x_31); +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_35 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_36 = l_Lean_Macro_throwErrorAt___rarg(x_2, x_35, x_14, x_15); +return x_36; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = l_Lean_Syntax_getArg(x_31, x_20); +lean_dec(x_31); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = lean_box(0); +x_40 = l_Lean_Elab_Command_expandInitialize___lambda__1(x_1, x_2, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_13, x_11, x_39, x_38, x_14, x_15); +lean_dec(x_38); +lean_dec(x_17); +return x_40; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__4() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l_Lean_Elab_Command_expandInitCmd___closed__3; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_dec(x_25); +x_41 = lean_box(0); +x_42 = lean_box(0); +x_43 = l_Lean_Elab_Command_expandInitialize___lambda__1(x_1, x_2, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_13, x_11, x_42, x_41, x_14, x_15); +lean_dec(x_17); +return x_43; +} } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__5() { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("unexpected visibility annotation", 32); -return x_1; +lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_dec(x_11); +x_15 = lean_unsigned_to_nat(1u); +x_16 = l_Lean_Syntax_getArg(x_1, x_15); +x_17 = l_Lean_Syntax_isNone(x_16); +if (x_17 == 0) +{ +uint8_t x_18; +lean_inc(x_16); +x_18 = l_Lean_Syntax_matchesNull(x_16, x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_19 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_20 = l_Lean_Macro_throwErrorAt___rarg(x_2, x_19, x_13, x_14); +return x_20; } +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_21 = lean_unsigned_to_nat(0u); +x_22 = l_Lean_Syntax_getArg(x_16, x_21); +lean_dec(x_16); +x_23 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27; +lean_inc(x_4); +x_24 = l_Lean_Name_str___override(x_4, x_23); +lean_inc(x_22); +x_25 = l_Lean_Syntax_isOfKind(x_22, x_24); +lean_dec(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +lean_dec(x_22); +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_26 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_27 = l_Lean_Macro_throwErrorAt___rarg(x_2, x_26, x_13, x_14); +return x_27; } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__6() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_28 = l_Lean_Syntax_getArg(x_22, x_15); +lean_dec(x_22); +x_29 = l_Lean_Syntax_getArgs(x_28); +lean_dec(x_28); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = lean_box(0); +x_32 = l_Lean_Elab_Command_expandInitialize___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_12, x_31, x_30, x_13, x_14); +return x_32; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__7() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___closed__6; -x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_dec(x_16); +x_33 = lean_box(0); +x_34 = lean_box(0); +x_35 = l_Lean_Elab_Command_expandInitialize___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_12, x_34, x_33, x_13, x_14); +return x_35; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__8() { +} +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___closed__7; -x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Term", 4); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__9() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___closed__8; -x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Unit", 4); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__10() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_expandInitCmd___closed__9; -x_2 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__2; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__11() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_3 = l_Lean_Elab_Command_expandInitCmd___closed__10; -x_4 = lean_alloc_ctor(1, 3, 0); +x_1 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__2; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__3; +x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__12() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_elabDeclaration___closed__7; -x_2 = l_Lean_Elab_Command_expandInitCmd___closed__11; -x_3 = lean_array_push(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__2; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__13() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Command_elabDeclaration___closed__7; -x_2 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__13; -x_3 = lean_array_push(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__14() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declSig", 7); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__15() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l_Lean_Elab_Command_expandInitCmd___closed__14; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__6; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__16() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__8() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(4u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("docComment", 10); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__17() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__9() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("invalid initialization command, 'visibility' modifer is not allowed", 67); +x_1 = lean_mk_string_from_bytes("initialize", 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__18() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__10() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("init", 4); +x_1 = lean_mk_string_from_bytes("builtinInit", 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__19() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___closed__18; +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__20() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__12() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("builtinInit", 11); +x_1 = lean_mk_string_from_bytes("init", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_expandInitCmd___closed__21() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Command_expandInitCmd___closed__20; +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitCmd(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_604; lean_object* x_605; lean_object* x_606; uint8_t x_607; +lean_dec(x_7); +x_12 = lean_unsigned_to_nat(3u); +x_13 = l_Lean_Syntax_getArg(x_1, x_12); +x_14 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__1; +lean_inc(x_2); +x_15 = l_Lean_Name_str___override(x_2, x_14); +x_604 = lean_unsigned_to_nat(0u); +x_605 = l_Lean_Syntax_getArg(x_6, x_604); +lean_dec(x_6); +x_606 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__9; +x_607 = l_Lean_Syntax_isToken(x_606, x_605); +lean_dec(x_605); +if (x_607 == 0) +{ +lean_object* x_608; +x_608 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__11; +x_16 = x_608; +goto block_603; +} +else +{ +lean_object* x_609; +x_609 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__13; +x_16 = x_609; +goto block_603; +} +block_603: +{ +lean_object* x_17; +x_17 = l_Lean_mkIdentFrom(x_1, x_16); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_18; lean_object* x_19; uint8_t x_20; +lean_dec(x_9); +x_18 = lean_unsigned_to_nat(0u); +x_19 = l_Lean_Syntax_getArg(x_3, x_18); +x_20 = l_Lean_Syntax_matchesNull(x_19, x_18); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_21 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_22 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_21, x_10, x_11); +lean_dec(x_3); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_23 = lean_unsigned_to_nat(1u); +x_24 = l_Lean_Syntax_getArg(x_3, x_23); +x_25 = l_Lean_Syntax_matchesNull(x_24, x_18); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_26 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_27 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_26, x_10, x_11); +lean_dec(x_3); +return x_27; +} +else +{ +lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_28 = lean_unsigned_to_nat(2u); +x_29 = l_Lean_Syntax_getArg(x_3, x_28); +x_30 = l_Lean_Syntax_matchesNull(x_29, x_18); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_31 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_32 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_31, x_10, x_11); +lean_dec(x_3); +return x_32; +} +else +{ +lean_object* x_33; uint8_t x_34; +x_33 = l_Lean_Syntax_getArg(x_3, x_12); +x_34 = l_Lean_Syntax_matchesNull(x_33, x_18); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_35 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_36 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_35, x_10, x_11); +lean_dec(x_3); +return x_36; +} +else +{ +lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_37 = lean_unsigned_to_nat(4u); +x_38 = l_Lean_Syntax_getArg(x_3, x_37); +x_39 = l_Lean_Syntax_matchesNull(x_38, x_18); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_40 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_41 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_40, x_10, x_11); +lean_dec(x_3); +return x_41; +} +else +{ +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = lean_unsigned_to_nat(5u); +x_43 = l_Lean_Syntax_getArg(x_3, x_42); +x_44 = l_Lean_Syntax_matchesNull(x_43, x_18); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_45 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_46 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_45, x_10, x_11); +lean_dec(x_3); +return x_46; +} +else +{ +lean_object* x_47; uint8_t x_48; +lean_dec(x_3); +lean_inc(x_10); +x_47 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_10, x_11); +x_48 = !lean_is_exclusive(x_47); +if (x_48 == 0) +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; +x_49 = lean_ctor_get(x_47, 0); +x_50 = lean_ctor_get(x_10, 2); +lean_inc(x_50); +x_51 = lean_ctor_get(x_10, 1); +lean_inc(x_51); +lean_dec(x_10); +x_52 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__7; +lean_inc(x_4); +x_53 = l_Lean_Name_str___override(x_4, x_52); +x_54 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27; +lean_inc(x_15); +x_55 = l_Lean_Name_str___override(x_15, x_54); +x_56 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28; +lean_inc(x_49); +x_57 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_57, 0, x_49); +lean_ctor_set(x_57, 1, x_56); +x_58 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29; +lean_inc(x_15); +x_59 = l_Lean_Name_str___override(x_15, x_58); +x_60 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30; +lean_inc(x_15); +x_61 = l_Lean_Name_str___override(x_15, x_60); +x_62 = lean_box(2); +x_63 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31; +x_64 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_61); +lean_ctor_set(x_64, 2, x_63); +x_65 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32; +x_66 = l_Lean_Name_str___override(x_2, x_65); +x_67 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33; +x_68 = l_Lean_Name_str___override(x_66, x_67); +x_69 = l_Lean_Elab_Command_elabDeclaration___closed__7; +x_70 = lean_array_push(x_69, x_17); +x_71 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_72 = lean_array_push(x_70, x_71); +x_73 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_73, 0, x_62); +lean_ctor_set(x_73, 1, x_68); +lean_ctor_set(x_73, 2, x_72); +x_74 = lean_array_push(x_69, x_64); +x_75 = lean_array_push(x_74, x_73); +x_76 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_76, 0, x_62); +lean_ctor_set(x_76, 1, x_59); +lean_ctor_set(x_76, 2, x_75); +x_77 = l_Lean_Elab_Command_elabInductive___closed__1; +x_78 = lean_array_push(x_77, x_76); +x_79 = l_Lean_Elab_Command_elabDeclaration___closed__4; +x_80 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_80, 0, x_62); +lean_ctor_set(x_80, 1, x_79); +lean_ctor_set(x_80, 2, x_78); +x_81 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35; +lean_inc(x_49); +x_82 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_82, 0, x_49); +lean_ctor_set(x_82, 1, x_81); +x_83 = l_Lean_Elab_Command_elabDeclaration___closed__10; +x_84 = lean_array_push(x_83, x_57); +x_85 = lean_array_push(x_84, x_80); +x_86 = lean_array_push(x_85, x_82); +x_87 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_87, 0, x_62); +lean_ctor_set(x_87, 1, x_55); +lean_ctor_set(x_87, 2, x_86); +x_88 = lean_array_push(x_77, x_87); +x_89 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_89, 0, x_62); +lean_ctor_set(x_89, 1, x_79); +lean_ctor_set(x_89, 2, x_88); +x_90 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3; +x_91 = lean_array_push(x_90, x_89); +x_92 = lean_array_push(x_91, x_71); +x_93 = lean_array_push(x_92, x_71); +x_94 = lean_array_push(x_93, x_71); +x_95 = lean_array_push(x_94, x_71); +x_96 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_96, 0, x_62); +lean_ctor_set(x_96, 1, x_5); +lean_ctor_set(x_96, 2, x_95); +x_97 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; +lean_inc(x_4); +x_98 = l_Lean_Name_str___override(x_4, x_97); +lean_inc(x_49); +x_99 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_99, 0, x_49); +lean_ctor_set(x_99, 1, x_97); +x_100 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7; +lean_inc(x_4); +x_101 = l_Lean_Name_str___override(x_4, x_100); +x_102 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11; +lean_inc(x_50); +lean_inc(x_51); +x_103 = l_Lean_addMacroScope(x_51, x_102, x_50); +x_104 = lean_box(0); +x_105 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10; +lean_inc(x_49); +x_106 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_106, 0, x_49); +lean_ctor_set(x_106, 1, x_105); +lean_ctor_set(x_106, 2, x_103); +lean_ctor_set(x_106, 3, x_104); +x_107 = lean_array_push(x_69, x_106); +x_108 = lean_array_push(x_107, x_71); +x_109 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_109, 0, x_62); +lean_ctor_set(x_109, 1, x_101); +lean_ctor_set(x_109, 2, x_108); +x_110 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12; +lean_inc(x_4); +x_111 = l_Lean_Name_str___override(x_4, x_110); +x_112 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13; +lean_inc(x_15); +x_113 = l_Lean_Name_str___override(x_15, x_112); +x_114 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14; +lean_inc(x_49); +x_115 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_115, 0, x_49); +lean_ctor_set(x_115, 1, x_114); +x_116 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15; +lean_inc(x_15); +x_117 = l_Lean_Name_str___override(x_15, x_116); +x_118 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19; +lean_inc(x_50); +lean_inc(x_51); +x_119 = l_Lean_addMacroScope(x_51, x_118, x_50); +x_120 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18; +x_121 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21; +lean_inc(x_49); +x_122 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_122, 0, x_49); +lean_ctor_set(x_122, 1, x_120); +lean_ctor_set(x_122, 2, x_119); +lean_ctor_set(x_122, 3, x_121); +x_123 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5; +x_124 = l_Lean_addMacroScope(x_51, x_123, x_50); +x_125 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4; +x_126 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7; +lean_inc(x_49); +x_127 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_127, 0, x_49); +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 = lean_array_push(x_77, x_127); +x_129 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_129, 0, x_62); +lean_ctor_set(x_129, 1, x_79); +lean_ctor_set(x_129, 2, x_128); +x_130 = lean_array_push(x_69, x_122); +x_131 = lean_array_push(x_130, x_129); +x_132 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_132, 0, x_62); +lean_ctor_set(x_132, 1, x_117); +lean_ctor_set(x_132, 2, x_131); +x_133 = lean_array_push(x_69, x_115); +x_134 = lean_array_push(x_133, x_132); +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_62); +lean_ctor_set(x_135, 1, x_113); +lean_ctor_set(x_135, 2, x_134); +x_136 = lean_array_push(x_77, x_135); +x_137 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_137, 0, x_62); +lean_ctor_set(x_137, 1, x_79); +lean_ctor_set(x_137, 2, x_136); +x_138 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22; +x_139 = lean_array_push(x_138, x_137); +x_140 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_140, 0, x_62); +lean_ctor_set(x_140, 1, x_111); +lean_ctor_set(x_140, 2, x_139); +x_141 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23; +x_142 = l_Lean_Name_str___override(x_4, x_141); +x_143 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24; +lean_inc(x_49); +x_144 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_144, 0, x_49); +lean_ctor_set(x_144, 1, x_143); +x_145 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25; +x_146 = l_Lean_Name_str___override(x_15, x_145); +x_147 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_147, 0, x_49); +lean_ctor_set(x_147, 1, x_145); +x_148 = lean_array_push(x_69, x_147); +x_149 = lean_array_push(x_148, x_13); +x_150 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_150, 0, x_62); +lean_ctor_set(x_150, 1, x_146); +lean_ctor_set(x_150, 2, x_149); +x_151 = lean_array_push(x_83, x_144); +x_152 = lean_array_push(x_151, x_150); +x_153 = lean_array_push(x_152, x_71); +x_154 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_154, 0, x_62); +lean_ctor_set(x_154, 1, x_142); +lean_ctor_set(x_154, 2, x_153); +x_155 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26; +x_156 = lean_array_push(x_155, x_99); +x_157 = lean_array_push(x_156, x_109); +x_158 = lean_array_push(x_157, x_140); +x_159 = lean_array_push(x_158, x_154); +x_160 = lean_array_push(x_159, x_71); +x_161 = lean_array_push(x_160, x_71); +x_162 = lean_array_push(x_161, x_71); +x_163 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_163, 0, x_62); +lean_ctor_set(x_163, 1, x_98); +lean_ctor_set(x_163, 2, x_162); +x_164 = lean_array_push(x_69, x_96); +x_165 = lean_array_push(x_164, x_163); +x_166 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_166, 0, x_62); +lean_ctor_set(x_166, 1, x_53); +lean_ctor_set(x_166, 2, x_165); +lean_ctor_set(x_47, 0, x_166); +return x_47; +} +else +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; +x_167 = lean_ctor_get(x_47, 0); +x_168 = lean_ctor_get(x_47, 1); +lean_inc(x_168); +lean_inc(x_167); +lean_dec(x_47); +x_169 = lean_ctor_get(x_10, 2); +lean_inc(x_169); +x_170 = lean_ctor_get(x_10, 1); +lean_inc(x_170); +lean_dec(x_10); +x_171 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__7; +lean_inc(x_4); +x_172 = l_Lean_Name_str___override(x_4, x_171); +x_173 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27; +lean_inc(x_15); +x_174 = l_Lean_Name_str___override(x_15, x_173); +x_175 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28; +lean_inc(x_167); +x_176 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_176, 0, x_167); +lean_ctor_set(x_176, 1, x_175); +x_177 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29; +lean_inc(x_15); +x_178 = l_Lean_Name_str___override(x_15, x_177); +x_179 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30; +lean_inc(x_15); +x_180 = l_Lean_Name_str___override(x_15, x_179); +x_181 = lean_box(2); +x_182 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31; +x_183 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_183, 0, x_181); +lean_ctor_set(x_183, 1, x_180); +lean_ctor_set(x_183, 2, x_182); +x_184 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32; +x_185 = l_Lean_Name_str___override(x_2, x_184); +x_186 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33; +x_187 = l_Lean_Name_str___override(x_185, x_186); +x_188 = l_Lean_Elab_Command_elabDeclaration___closed__7; +x_189 = lean_array_push(x_188, x_17); +x_190 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_191 = lean_array_push(x_189, x_190); +x_192 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_192, 0, x_181); +lean_ctor_set(x_192, 1, x_187); +lean_ctor_set(x_192, 2, x_191); +x_193 = lean_array_push(x_188, x_183); +x_194 = lean_array_push(x_193, x_192); +x_195 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_195, 0, x_181); +lean_ctor_set(x_195, 1, x_178); +lean_ctor_set(x_195, 2, x_194); +x_196 = l_Lean_Elab_Command_elabInductive___closed__1; +x_197 = lean_array_push(x_196, x_195); +x_198 = l_Lean_Elab_Command_elabDeclaration___closed__4; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_181); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_197); +x_200 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35; +lean_inc(x_167); +x_201 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_201, 0, x_167); +lean_ctor_set(x_201, 1, x_200); +x_202 = l_Lean_Elab_Command_elabDeclaration___closed__10; +x_203 = lean_array_push(x_202, x_176); +x_204 = lean_array_push(x_203, x_199); +x_205 = lean_array_push(x_204, x_201); +x_206 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_206, 0, x_181); +lean_ctor_set(x_206, 1, x_174); +lean_ctor_set(x_206, 2, x_205); +x_207 = lean_array_push(x_196, x_206); +x_208 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_208, 0, x_181); +lean_ctor_set(x_208, 1, x_198); +lean_ctor_set(x_208, 2, x_207); +x_209 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3; +x_210 = lean_array_push(x_209, x_208); +x_211 = lean_array_push(x_210, x_190); +x_212 = lean_array_push(x_211, x_190); +x_213 = lean_array_push(x_212, x_190); +x_214 = lean_array_push(x_213, x_190); +x_215 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_215, 0, x_181); +lean_ctor_set(x_215, 1, x_5); +lean_ctor_set(x_215, 2, x_214); +x_216 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; +lean_inc(x_4); +x_217 = l_Lean_Name_str___override(x_4, x_216); +lean_inc(x_167); +x_218 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_218, 0, x_167); +lean_ctor_set(x_218, 1, x_216); +x_219 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7; +lean_inc(x_4); +x_220 = l_Lean_Name_str___override(x_4, x_219); +x_221 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11; +lean_inc(x_169); +lean_inc(x_170); +x_222 = l_Lean_addMacroScope(x_170, x_221, x_169); +x_223 = lean_box(0); +x_224 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10; +lean_inc(x_167); +x_225 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_225, 0, x_167); +lean_ctor_set(x_225, 1, x_224); +lean_ctor_set(x_225, 2, x_222); +lean_ctor_set(x_225, 3, x_223); +x_226 = lean_array_push(x_188, x_225); +x_227 = lean_array_push(x_226, x_190); +x_228 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_228, 0, x_181); +lean_ctor_set(x_228, 1, x_220); +lean_ctor_set(x_228, 2, x_227); +x_229 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12; +lean_inc(x_4); +x_230 = l_Lean_Name_str___override(x_4, x_229); +x_231 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13; +lean_inc(x_15); +x_232 = l_Lean_Name_str___override(x_15, x_231); +x_233 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14; +lean_inc(x_167); +x_234 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_234, 0, x_167); +lean_ctor_set(x_234, 1, x_233); +x_235 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15; +lean_inc(x_15); +x_236 = l_Lean_Name_str___override(x_15, x_235); +x_237 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19; +lean_inc(x_169); +lean_inc(x_170); +x_238 = l_Lean_addMacroScope(x_170, x_237, x_169); +x_239 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18; +x_240 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21; +lean_inc(x_167); +x_241 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_241, 0, x_167); +lean_ctor_set(x_241, 1, x_239); +lean_ctor_set(x_241, 2, x_238); +lean_ctor_set(x_241, 3, x_240); +x_242 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5; +x_243 = l_Lean_addMacroScope(x_170, x_242, x_169); +x_244 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4; +x_245 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7; +lean_inc(x_167); +x_246 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_246, 0, x_167); +lean_ctor_set(x_246, 1, x_244); +lean_ctor_set(x_246, 2, x_243); +lean_ctor_set(x_246, 3, x_245); +x_247 = lean_array_push(x_196, x_246); +x_248 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_248, 0, x_181); +lean_ctor_set(x_248, 1, x_198); +lean_ctor_set(x_248, 2, x_247); +x_249 = lean_array_push(x_188, x_241); +x_250 = lean_array_push(x_249, x_248); +x_251 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_251, 0, x_181); +lean_ctor_set(x_251, 1, x_236); +lean_ctor_set(x_251, 2, x_250); +x_252 = lean_array_push(x_188, x_234); +x_253 = lean_array_push(x_252, x_251); +x_254 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_254, 0, x_181); +lean_ctor_set(x_254, 1, x_232); +lean_ctor_set(x_254, 2, x_253); +x_255 = lean_array_push(x_196, x_254); +x_256 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_256, 0, x_181); +lean_ctor_set(x_256, 1, x_198); +lean_ctor_set(x_256, 2, x_255); +x_257 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22; +x_258 = lean_array_push(x_257, x_256); +x_259 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_259, 0, x_181); +lean_ctor_set(x_259, 1, x_230); +lean_ctor_set(x_259, 2, x_258); +x_260 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23; +x_261 = l_Lean_Name_str___override(x_4, x_260); +x_262 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24; +lean_inc(x_167); +x_263 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_263, 0, x_167); +lean_ctor_set(x_263, 1, x_262); +x_264 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25; +x_265 = l_Lean_Name_str___override(x_15, x_264); +x_266 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_266, 0, x_167); +lean_ctor_set(x_266, 1, x_264); +x_267 = lean_array_push(x_188, x_266); +x_268 = lean_array_push(x_267, x_13); +x_269 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_269, 0, x_181); +lean_ctor_set(x_269, 1, x_265); +lean_ctor_set(x_269, 2, x_268); +x_270 = lean_array_push(x_202, x_263); +x_271 = lean_array_push(x_270, x_269); +x_272 = lean_array_push(x_271, x_190); +x_273 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_273, 0, x_181); +lean_ctor_set(x_273, 1, x_261); +lean_ctor_set(x_273, 2, x_272); +x_274 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26; +x_275 = lean_array_push(x_274, x_218); +x_276 = lean_array_push(x_275, x_228); +x_277 = lean_array_push(x_276, x_259); +x_278 = lean_array_push(x_277, x_273); +x_279 = lean_array_push(x_278, x_190); +x_280 = lean_array_push(x_279, x_190); +x_281 = lean_array_push(x_280, x_190); +x_282 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_282, 0, x_181); +lean_ctor_set(x_282, 1, x_217); +lean_ctor_set(x_282, 2, x_281); +x_283 = lean_array_push(x_188, x_215); +x_284 = lean_array_push(x_283, x_282); +x_285 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_285, 0, x_181); +lean_ctor_set(x_285, 1, x_172); +lean_ctor_set(x_285, 2, x_284); +x_286 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_286, 0, x_285); +lean_ctor_set(x_286, 1, x_168); +return x_286; +} +} +} +} +} +} +} +} +else +{ +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_287; lean_object* x_288; uint8_t x_289; +lean_dec(x_8); +x_287 = lean_unsigned_to_nat(0u); +x_288 = l_Lean_Syntax_getArg(x_3, x_287); +x_289 = l_Lean_Syntax_matchesNull(x_288, x_287); +if (x_289 == 0) +{ +lean_object* x_290; lean_object* x_291; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_290 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_291 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_290, x_10, x_11); +lean_dec(x_3); +return x_291; +} +else { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; -x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Lean_Syntax_getArg(x_2, x_5); -x_7 = lean_unsigned_to_nat(2u); -x_8 = l_Lean_Syntax_getArg(x_2, x_7); -x_9 = lean_unsigned_to_nat(3u); -x_10 = l_Lean_Syntax_getArg(x_2, x_9); -x_11 = l_Lean_Syntax_isNone(x_8); -if (x_1 == 0) +lean_object* x_292; lean_object* x_293; uint8_t x_294; +x_292 = lean_unsigned_to_nat(1u); +x_293 = l_Lean_Syntax_getArg(x_3, x_292); +x_294 = l_Lean_Syntax_matchesNull(x_293, x_287); +if (x_294 == 0) { -lean_object* x_799; -x_799 = l_Lean_Elab_Command_expandInitCmd___closed__19; -x_12 = x_799; -goto block_798; +lean_object* x_295; lean_object* x_296; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_295 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_296 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_295, x_10, x_11); +lean_dec(x_3); +return x_296; } else { -lean_object* x_800; -x_800 = l_Lean_Elab_Command_expandInitCmd___closed__21; -x_12 = x_800; -goto block_798; -} -block_798: +lean_object* x_297; lean_object* x_298; uint8_t x_299; +x_297 = lean_unsigned_to_nat(2u); +x_298 = l_Lean_Syntax_getArg(x_3, x_297); +x_299 = l_Lean_Syntax_matchesNull(x_298, x_287); +if (x_299 == 0) { -lean_object* x_13; -x_13 = l_Lean_mkIdentFrom(x_2, x_12); -if (x_11 == 0) +lean_object* x_300; lean_object* x_301; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_300 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_301 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_300, x_10, x_11); +lean_dec(x_3); +return x_301; +} +else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_14 = l_Lean_Syntax_getArg(x_8, x_5); -x_15 = lean_unsigned_to_nat(1u); -x_16 = l_Lean_Syntax_getArg(x_8, x_15); -lean_dec(x_8); -x_17 = l_Lean_Syntax_getArg(x_16, x_15); -lean_dec(x_16); -x_18 = l_Lean_Syntax_isNone(x_6); -if (x_18 == 0) +lean_object* x_302; uint8_t x_303; +x_302 = l_Lean_Syntax_getArg(x_3, x_12); +x_303 = l_Lean_Syntax_matchesNull(x_302, x_287); +if (x_303 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_19 = l_Lean_Syntax_getArg(x_6, x_5); -lean_dec(x_6); -x_20 = l_Lean_Syntax_getKind(x_19); -x_21 = l_Lean_Elab_Command_expandInitCmd___closed__2; -x_22 = lean_name_eq(x_20, x_21); -if (x_22 == 0) +lean_object* x_304; lean_object* x_305; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_304 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_305 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_304, x_10, x_11); +lean_dec(x_3); +return x_305; +} +else { -lean_object* x_23; uint8_t x_24; -x_23 = l_Lean_Elab_Command_expandInitCmd___closed__4; -x_24 = lean_name_eq(x_20, x_23); -lean_dec(x_20); -if (x_24 == 0) +lean_object* x_306; lean_object* x_307; uint8_t x_308; +x_306 = lean_unsigned_to_nat(4u); +x_307 = l_Lean_Syntax_getArg(x_3, x_306); +x_308 = l_Lean_Syntax_matchesNull(x_307, x_287); +if (x_308 == 0) { -lean_object* x_25; lean_object* x_26; +lean_object* x_309; lean_object* x_310; lean_dec(x_17); -lean_dec(x_14); +lean_dec(x_15); lean_dec(x_13); -lean_dec(x_10); -x_25 = l_Lean_Elab_Command_expandInitCmd___closed__5; -x_26 = l_Lean_Macro_throwError___rarg(x_25, x_3, x_4); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_309 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_310 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_309, x_10, x_11); lean_dec(x_3); -return x_26; +return x_310; } else { -lean_object* x_27; uint8_t x_28; -lean_inc(x_3); -x_27 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_3, x_4); -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) +lean_object* x_311; lean_object* x_312; uint8_t x_313; +x_311 = lean_unsigned_to_nat(5u); +x_312 = l_Lean_Syntax_getArg(x_3, x_311); +x_313 = l_Lean_Syntax_matchesNull(x_312, x_287); +if (x_313 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_29 = lean_ctor_get(x_27, 0); -x_30 = lean_ctor_get(x_3, 2); -lean_inc(x_30); -x_31 = lean_ctor_get(x_3, 1); -lean_inc(x_31); +lean_object* x_314; lean_object* x_315; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_314 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_315 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_314, x_10, x_11); lean_dec(x_3); -x_32 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; -lean_inc(x_29); -x_33 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_33, 0, x_29); -lean_ctor_set(x_33, 1, x_32); -x_34 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; -lean_inc(x_30); -lean_inc(x_31); -x_35 = l_Lean_addMacroScope(x_31, x_34, x_30); -x_36 = lean_box(0); -x_37 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -lean_inc(x_29); -x_38 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_38, 0, x_29); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_ctor_set(x_38, 3, x_36); -x_39 = l_Lean_Elab_Command_elabDeclaration___closed__7; -lean_inc(x_38); -x_40 = lean_array_push(x_39, x_38); -x_41 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_42 = lean_array_push(x_40, x_41); -x_43 = lean_box(2); -x_44 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; -x_45 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -lean_ctor_set(x_45, 2, x_42); -x_46 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; -lean_inc(x_29); -x_47 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_47, 0, x_29); -lean_ctor_set(x_47, 1, x_46); -x_48 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -x_49 = l_Lean_addMacroScope(x_31, x_48, x_30); -x_50 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -x_51 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; -lean_inc(x_29); -x_52 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_52, 0, x_29); -lean_ctor_set(x_52, 1, x_50); -lean_ctor_set(x_52, 2, x_49); -lean_ctor_set(x_52, 3, x_51); -x_53 = l_Lean_Elab_Command_elabInductive___closed__1; -lean_inc(x_17); -x_54 = lean_array_push(x_53, x_17); -x_55 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_56 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_56, 0, x_43); -lean_ctor_set(x_56, 1, x_55); -lean_ctor_set(x_56, 2, x_54); -x_57 = lean_array_push(x_39, x_52); -x_58 = lean_array_push(x_57, x_56); -x_59 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; -x_60 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_60, 0, x_43); -lean_ctor_set(x_60, 1, x_59); -lean_ctor_set(x_60, 2, x_58); -x_61 = lean_array_push(x_39, x_47); -lean_inc(x_61); -x_62 = lean_array_push(x_61, x_60); -x_63 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_43); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = lean_array_push(x_53, x_64); -x_66 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_66, 0, x_43); -lean_ctor_set(x_66, 1, x_55); -lean_ctor_set(x_66, 2, x_65); -x_67 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; -x_68 = lean_array_push(x_67, x_66); -x_69 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_43); -lean_ctor_set(x_70, 1, x_69); -lean_ctor_set(x_70, 2, x_68); -x_71 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; -lean_inc(x_29); -x_72 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_72, 0, x_29); -lean_ctor_set(x_72, 1, x_71); -x_73 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -lean_inc(x_29); -x_74 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_74, 0, x_29); -lean_ctor_set(x_74, 1, x_73); -x_75 = lean_array_push(x_39, x_74); -x_76 = lean_array_push(x_75, x_10); -x_77 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; -x_78 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_78, 0, x_43); -lean_ctor_set(x_78, 1, x_77); -lean_ctor_set(x_78, 2, x_76); -x_79 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_80 = lean_array_push(x_79, x_72); -x_81 = lean_array_push(x_80, x_78); -x_82 = lean_array_push(x_81, x_41); -x_83 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; -x_84 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_84, 0, x_43); -lean_ctor_set(x_84, 1, x_83); -lean_ctor_set(x_84, 2, x_82); -x_85 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; -x_86 = lean_array_push(x_85, x_33); -x_87 = lean_array_push(x_86, x_45); -x_88 = lean_array_push(x_87, x_70); -x_89 = lean_array_push(x_88, x_84); -x_90 = lean_array_push(x_89, x_41); -x_91 = lean_array_push(x_90, x_41); -x_92 = lean_array_push(x_91, x_41); -x_93 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -x_94 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_94, 0, x_43); -lean_ctor_set(x_94, 1, x_93); -lean_ctor_set(x_94, 2, x_92); -x_95 = l_Lean_Elab_Command_expandInitCmd___closed__12; -x_96 = lean_array_push(x_95, x_94); -x_97 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; -x_98 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_98, 0, x_43); -lean_ctor_set(x_98, 1, x_97); -lean_ctor_set(x_98, 2, x_96); -x_99 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; -lean_inc(x_29); -x_100 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_100, 0, x_29); -lean_ctor_set(x_100, 1, x_99); -x_101 = lean_array_push(x_53, x_38); -x_102 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_102, 0, x_43); -lean_ctor_set(x_102, 1, x_55); -lean_ctor_set(x_102, 2, x_101); -x_103 = lean_array_push(x_39, x_13); -x_104 = lean_array_push(x_103, x_102); -x_105 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; -x_106 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_106, 0, x_43); -lean_ctor_set(x_106, 1, x_105); -lean_ctor_set(x_106, 2, x_104); -x_107 = l_Lean_Elab_Command_expandInitCmd___closed__13; -x_108 = lean_array_push(x_107, x_106); -x_109 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -x_110 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_110, 0, x_43); -lean_ctor_set(x_110, 1, x_109); -lean_ctor_set(x_110, 2, x_108); -x_111 = lean_array_push(x_53, x_110); -x_112 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_112, 0, x_43); -lean_ctor_set(x_112, 1, x_55); -lean_ctor_set(x_112, 2, x_111); -x_113 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -lean_inc(x_29); -x_114 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_114, 0, x_29); -lean_ctor_set(x_114, 1, x_113); -x_115 = lean_array_push(x_79, x_100); -x_116 = lean_array_push(x_115, x_112); -x_117 = lean_array_push(x_116, x_114); -x_118 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; -x_119 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_119, 0, x_43); -lean_ctor_set(x_119, 1, x_118); -lean_ctor_set(x_119, 2, x_117); -x_120 = lean_array_push(x_53, x_119); -x_121 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_121, 0, x_43); -lean_ctor_set(x_121, 1, x_55); -lean_ctor_set(x_121, 2, x_120); -x_122 = l_Lean_Elab_Command_expandInitCmd___closed__3; -lean_inc(x_29); -x_123 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_123, 0, x_29); -lean_ctor_set(x_123, 1, x_122); -x_124 = lean_array_push(x_53, x_123); -x_125 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_125, 0, x_43); -lean_ctor_set(x_125, 1, x_23); -lean_ctor_set(x_125, 2, x_124); -x_126 = lean_array_push(x_53, x_125); -x_127 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_127, 0, x_43); -lean_ctor_set(x_127, 1, x_55); -lean_ctor_set(x_127, 2, x_126); -x_128 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_129 = lean_array_push(x_128, x_121); -x_130 = lean_array_push(x_129, x_127); -x_131 = lean_array_push(x_130, x_41); -x_132 = lean_array_push(x_131, x_41); -x_133 = lean_array_push(x_132, x_41); -x_134 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_135 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_135, 0, x_43); -lean_ctor_set(x_135, 1, x_134); -lean_ctor_set(x_135, 2, x_133); -x_136 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__15; -x_137 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_137, 0, x_29); -lean_ctor_set(x_137, 1, x_136); -x_138 = lean_array_push(x_61, x_17); -x_139 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_139, 0, x_43); -lean_ctor_set(x_139, 1, x_63); -lean_ctor_set(x_139, 2, x_138); -x_140 = lean_array_push(x_67, x_139); -x_141 = l_Lean_Elab_Command_expandInitCmd___closed__15; -x_142 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_142, 0, x_43); -lean_ctor_set(x_142, 1, x_141); -lean_ctor_set(x_142, 2, x_140); -x_143 = l_Lean_Elab_Command_expandInitCmd___closed__16; -x_144 = lean_array_push(x_143, x_137); -x_145 = lean_array_push(x_144, x_14); -x_146 = lean_array_push(x_145, x_142); -x_147 = lean_array_push(x_146, x_41); -x_148 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__16; -x_149 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_149, 0, x_43); -lean_ctor_set(x_149, 1, x_148); -lean_ctor_set(x_149, 2, x_147); -x_150 = lean_array_push(x_39, x_135); -x_151 = lean_array_push(x_150, x_149); -x_152 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_152, 0, x_43); -lean_ctor_set(x_152, 1, x_97); -lean_ctor_set(x_152, 2, x_151); -x_153 = lean_array_push(x_39, x_98); -x_154 = lean_array_push(x_153, x_152); -x_155 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_155, 0, x_43); -lean_ctor_set(x_155, 1, x_55); -lean_ctor_set(x_155, 2, x_154); -lean_ctor_set(x_27, 0, x_155); -return x_27; +return x_315; } else { -lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; -x_156 = lean_ctor_get(x_27, 0); -x_157 = lean_ctor_get(x_27, 1); -lean_inc(x_157); -lean_inc(x_156); -lean_dec(x_27); -x_158 = lean_ctor_get(x_3, 2); -lean_inc(x_158); -x_159 = lean_ctor_get(x_3, 1); -lean_inc(x_159); +lean_object* x_316; uint8_t x_317; lean_dec(x_3); -x_160 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; -lean_inc(x_156); -x_161 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_161, 0, x_156); -lean_ctor_set(x_161, 1, x_160); -x_162 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; -lean_inc(x_158); -lean_inc(x_159); -x_163 = l_Lean_addMacroScope(x_159, x_162, x_158); -x_164 = lean_box(0); -x_165 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -lean_inc(x_156); -x_166 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_166, 0, x_156); -lean_ctor_set(x_166, 1, x_165); -lean_ctor_set(x_166, 2, x_163); -lean_ctor_set(x_166, 3, x_164); -x_167 = l_Lean_Elab_Command_elabDeclaration___closed__7; -lean_inc(x_166); -x_168 = lean_array_push(x_167, x_166); -x_169 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_170 = lean_array_push(x_168, x_169); -x_171 = lean_box(2); -x_172 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; -x_173 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_173, 0, x_171); -lean_ctor_set(x_173, 1, x_172); -lean_ctor_set(x_173, 2, x_170); -x_174 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; -lean_inc(x_156); -x_175 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_175, 0, x_156); -lean_ctor_set(x_175, 1, x_174); -x_176 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -x_177 = l_Lean_addMacroScope(x_159, x_176, x_158); -x_178 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -x_179 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; -lean_inc(x_156); -x_180 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_180, 0, x_156); -lean_ctor_set(x_180, 1, x_178); -lean_ctor_set(x_180, 2, x_177); -lean_ctor_set(x_180, 3, x_179); -x_181 = l_Lean_Elab_Command_elabInductive___closed__1; -lean_inc(x_17); -x_182 = lean_array_push(x_181, x_17); -x_183 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_184 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_184, 0, x_171); -lean_ctor_set(x_184, 1, x_183); -lean_ctor_set(x_184, 2, x_182); -x_185 = lean_array_push(x_167, x_180); -x_186 = lean_array_push(x_185, x_184); -x_187 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; -x_188 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_188, 0, x_171); -lean_ctor_set(x_188, 1, x_187); -lean_ctor_set(x_188, 2, x_186); -x_189 = lean_array_push(x_167, x_175); -lean_inc(x_189); -x_190 = lean_array_push(x_189, x_188); -x_191 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; -x_192 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_192, 0, x_171); -lean_ctor_set(x_192, 1, x_191); -lean_ctor_set(x_192, 2, x_190); -x_193 = lean_array_push(x_181, x_192); -x_194 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_194, 0, x_171); -lean_ctor_set(x_194, 1, x_183); -lean_ctor_set(x_194, 2, x_193); -x_195 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; -x_196 = lean_array_push(x_195, x_194); -x_197 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; -x_198 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_198, 0, x_171); -lean_ctor_set(x_198, 1, x_197); -lean_ctor_set(x_198, 2, x_196); -x_199 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; -lean_inc(x_156); -x_200 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_200, 0, x_156); -lean_ctor_set(x_200, 1, x_199); -x_201 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -lean_inc(x_156); -x_202 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_202, 0, x_156); -lean_ctor_set(x_202, 1, x_201); -x_203 = lean_array_push(x_167, x_202); -x_204 = lean_array_push(x_203, x_10); -x_205 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; -x_206 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_206, 0, x_171); -lean_ctor_set(x_206, 1, x_205); -lean_ctor_set(x_206, 2, x_204); -x_207 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_208 = lean_array_push(x_207, x_200); -x_209 = lean_array_push(x_208, x_206); -x_210 = lean_array_push(x_209, x_169); -x_211 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; -x_212 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_212, 0, x_171); -lean_ctor_set(x_212, 1, x_211); -lean_ctor_set(x_212, 2, x_210); -x_213 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; -x_214 = lean_array_push(x_213, x_161); -x_215 = lean_array_push(x_214, x_173); -x_216 = lean_array_push(x_215, x_198); -x_217 = lean_array_push(x_216, x_212); -x_218 = lean_array_push(x_217, x_169); -x_219 = lean_array_push(x_218, x_169); -x_220 = lean_array_push(x_219, x_169); -x_221 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -x_222 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_222, 0, x_171); -lean_ctor_set(x_222, 1, x_221); -lean_ctor_set(x_222, 2, x_220); -x_223 = l_Lean_Elab_Command_expandInitCmd___closed__12; -x_224 = lean_array_push(x_223, x_222); -x_225 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; -x_226 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_226, 0, x_171); -lean_ctor_set(x_226, 1, x_225); -lean_ctor_set(x_226, 2, x_224); -x_227 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; -lean_inc(x_156); -x_228 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_228, 0, x_156); -lean_ctor_set(x_228, 1, x_227); -x_229 = lean_array_push(x_181, x_166); -x_230 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_230, 0, x_171); -lean_ctor_set(x_230, 1, x_183); -lean_ctor_set(x_230, 2, x_229); -x_231 = lean_array_push(x_167, x_13); -x_232 = lean_array_push(x_231, x_230); -x_233 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; -x_234 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_234, 0, x_171); -lean_ctor_set(x_234, 1, x_233); -lean_ctor_set(x_234, 2, x_232); -x_235 = l_Lean_Elab_Command_expandInitCmd___closed__13; -x_236 = lean_array_push(x_235, x_234); -x_237 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -x_238 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_238, 0, x_171); -lean_ctor_set(x_238, 1, x_237); -lean_ctor_set(x_238, 2, x_236); -x_239 = lean_array_push(x_181, x_238); -x_240 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_240, 0, x_171); -lean_ctor_set(x_240, 1, x_183); -lean_ctor_set(x_240, 2, x_239); -x_241 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -lean_inc(x_156); -x_242 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_242, 0, x_156); -lean_ctor_set(x_242, 1, x_241); -x_243 = lean_array_push(x_207, x_228); -x_244 = lean_array_push(x_243, x_240); -x_245 = lean_array_push(x_244, x_242); -x_246 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; -x_247 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_247, 0, x_171); -lean_ctor_set(x_247, 1, x_246); -lean_ctor_set(x_247, 2, x_245); -x_248 = lean_array_push(x_181, x_247); -x_249 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_249, 0, x_171); -lean_ctor_set(x_249, 1, x_183); -lean_ctor_set(x_249, 2, x_248); -x_250 = l_Lean_Elab_Command_expandInitCmd___closed__3; -lean_inc(x_156); -x_251 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_251, 0, x_156); -lean_ctor_set(x_251, 1, x_250); -x_252 = lean_array_push(x_181, x_251); -x_253 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_253, 0, x_171); -lean_ctor_set(x_253, 1, x_23); -lean_ctor_set(x_253, 2, x_252); -x_254 = lean_array_push(x_181, x_253); -x_255 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_255, 0, x_171); -lean_ctor_set(x_255, 1, x_183); -lean_ctor_set(x_255, 2, x_254); -x_256 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_257 = lean_array_push(x_256, x_249); -x_258 = lean_array_push(x_257, x_255); -x_259 = lean_array_push(x_258, x_169); -x_260 = lean_array_push(x_259, x_169); -x_261 = lean_array_push(x_260, x_169); -x_262 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_263 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_263, 0, x_171); -lean_ctor_set(x_263, 1, x_262); -lean_ctor_set(x_263, 2, x_261); -x_264 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__15; -x_265 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_265, 0, x_156); -lean_ctor_set(x_265, 1, x_264); -x_266 = lean_array_push(x_189, x_17); -x_267 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_267, 0, x_171); -lean_ctor_set(x_267, 1, x_191); -lean_ctor_set(x_267, 2, x_266); -x_268 = lean_array_push(x_195, x_267); -x_269 = l_Lean_Elab_Command_expandInitCmd___closed__15; -x_270 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_270, 0, x_171); -lean_ctor_set(x_270, 1, x_269); -lean_ctor_set(x_270, 2, x_268); -x_271 = l_Lean_Elab_Command_expandInitCmd___closed__16; -x_272 = lean_array_push(x_271, x_265); -x_273 = lean_array_push(x_272, x_14); -x_274 = lean_array_push(x_273, x_270); -x_275 = lean_array_push(x_274, x_169); -x_276 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__16; -x_277 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_277, 0, x_171); -lean_ctor_set(x_277, 1, x_276); -lean_ctor_set(x_277, 2, x_275); -x_278 = lean_array_push(x_167, x_263); -x_279 = lean_array_push(x_278, x_277); -x_280 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_280, 0, x_171); -lean_ctor_set(x_280, 1, x_225); -lean_ctor_set(x_280, 2, x_279); -x_281 = lean_array_push(x_167, x_226); -x_282 = lean_array_push(x_281, x_280); -x_283 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_283, 0, x_171); -lean_ctor_set(x_283, 1, x_183); -lean_ctor_set(x_283, 2, x_282); -x_284 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_284, 0, x_283); -lean_ctor_set(x_284, 1, x_157); -return x_284; -} -} -} -else -{ -lean_object* x_285; uint8_t x_286; -lean_dec(x_20); -lean_inc(x_3); -x_285 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_3, x_4); -x_286 = !lean_is_exclusive(x_285); -if (x_286 == 0) +lean_inc(x_10); +x_316 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_10, x_11); +x_317 = !lean_is_exclusive(x_316); +if (x_317 == 0) { -lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; -x_287 = lean_ctor_get(x_285, 0); -x_288 = lean_ctor_get(x_3, 2); -lean_inc(x_288); -x_289 = lean_ctor_get(x_3, 1); -lean_inc(x_289); -lean_dec(x_3); -x_290 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; -lean_inc(x_287); -x_291 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_291, 0, x_287); -lean_ctor_set(x_291, 1, x_290); -x_292 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; -lean_inc(x_288); -lean_inc(x_289); -x_293 = l_Lean_addMacroScope(x_289, x_292, x_288); -x_294 = lean_box(0); -x_295 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -lean_inc(x_287); -x_296 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_296, 0, x_287); -lean_ctor_set(x_296, 1, x_295); -lean_ctor_set(x_296, 2, x_293); -lean_ctor_set(x_296, 3, x_294); -x_297 = l_Lean_Elab_Command_elabDeclaration___closed__7; -lean_inc(x_296); -x_298 = lean_array_push(x_297, x_296); -x_299 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_300 = lean_array_push(x_298, x_299); -x_301 = lean_box(2); -x_302 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; -x_303 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_303, 0, x_301); -lean_ctor_set(x_303, 1, x_302); -lean_ctor_set(x_303, 2, x_300); -x_304 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; -lean_inc(x_287); -x_305 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_305, 0, x_287); -lean_ctor_set(x_305, 1, x_304); -x_306 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -x_307 = l_Lean_addMacroScope(x_289, x_306, x_288); -x_308 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -x_309 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; -lean_inc(x_287); -x_310 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_310, 0, x_287); -lean_ctor_set(x_310, 1, x_308); -lean_ctor_set(x_310, 2, x_307); -lean_ctor_set(x_310, 3, x_309); -x_311 = l_Lean_Elab_Command_elabInductive___closed__1; -lean_inc(x_17); -x_312 = lean_array_push(x_311, x_17); -x_313 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_314 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_314, 0, x_301); -lean_ctor_set(x_314, 1, x_313); -lean_ctor_set(x_314, 2, x_312); -x_315 = lean_array_push(x_297, x_310); -x_316 = lean_array_push(x_315, x_314); -x_317 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; -x_318 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_318, 0, x_301); -lean_ctor_set(x_318, 1, x_317); -lean_ctor_set(x_318, 2, x_316); -x_319 = lean_array_push(x_297, x_305); +lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; +x_318 = lean_ctor_get(x_316, 0); +x_319 = lean_ctor_get(x_10, 2); lean_inc(x_319); -x_320 = lean_array_push(x_319, x_318); -x_321 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; -x_322 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_322, 0, x_301); -lean_ctor_set(x_322, 1, x_321); -lean_ctor_set(x_322, 2, x_320); -x_323 = lean_array_push(x_311, x_322); -x_324 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_324, 0, x_301); -lean_ctor_set(x_324, 1, x_313); -lean_ctor_set(x_324, 2, x_323); -x_325 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; -x_326 = lean_array_push(x_325, x_324); -x_327 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; -x_328 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_328, 0, x_301); -lean_ctor_set(x_328, 1, x_327); -lean_ctor_set(x_328, 2, x_326); -x_329 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; -lean_inc(x_287); -x_330 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_330, 0, x_287); -lean_ctor_set(x_330, 1, x_329); -x_331 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -lean_inc(x_287); -x_332 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_332, 0, x_287); -lean_ctor_set(x_332, 1, x_331); -x_333 = lean_array_push(x_297, x_332); -x_334 = lean_array_push(x_333, x_10); -x_335 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; -x_336 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_336, 0, x_301); -lean_ctor_set(x_336, 1, x_335); -lean_ctor_set(x_336, 2, x_334); -x_337 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_338 = lean_array_push(x_337, x_330); -x_339 = lean_array_push(x_338, x_336); -x_340 = lean_array_push(x_339, x_299); -x_341 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; +x_320 = lean_ctor_get(x_10, 1); +lean_inc(x_320); +lean_dec(x_10); +x_321 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__7; +lean_inc(x_4); +x_322 = l_Lean_Name_str___override(x_4, x_321); +x_323 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27; +lean_inc(x_15); +x_324 = l_Lean_Name_str___override(x_15, x_323); +x_325 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28; +lean_inc(x_318); +x_326 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_326, 0, x_318); +lean_ctor_set(x_326, 1, x_325); +x_327 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29; +lean_inc(x_15); +x_328 = l_Lean_Name_str___override(x_15, x_327); +x_329 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30; +lean_inc(x_15); +x_330 = l_Lean_Name_str___override(x_15, x_329); +x_331 = lean_box(2); +x_332 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31; +x_333 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_333, 0, x_331); +lean_ctor_set(x_333, 1, x_330); +lean_ctor_set(x_333, 2, x_332); +x_334 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32; +x_335 = l_Lean_Name_str___override(x_2, x_334); +x_336 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33; +x_337 = l_Lean_Name_str___override(x_335, x_336); +x_338 = l_Lean_Elab_Command_elabDeclaration___closed__7; +x_339 = lean_array_push(x_338, x_17); +x_340 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_341 = lean_array_push(x_339, x_340); x_342 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_342, 0, x_301); -lean_ctor_set(x_342, 1, x_341); -lean_ctor_set(x_342, 2, x_340); -x_343 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; -x_344 = lean_array_push(x_343, x_291); -x_345 = lean_array_push(x_344, x_303); -x_346 = lean_array_push(x_345, x_328); -x_347 = lean_array_push(x_346, x_342); -x_348 = lean_array_push(x_347, x_299); -x_349 = lean_array_push(x_348, x_299); -x_350 = lean_array_push(x_349, x_299); -x_351 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -x_352 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_352, 0, x_301); -lean_ctor_set(x_352, 1, x_351); -lean_ctor_set(x_352, 2, x_350); -x_353 = l_Lean_Elab_Command_expandInitCmd___closed__12; -x_354 = lean_array_push(x_353, x_352); -x_355 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; +lean_ctor_set(x_342, 0, x_331); +lean_ctor_set(x_342, 1, x_337); +lean_ctor_set(x_342, 2, x_341); +x_343 = lean_array_push(x_338, x_333); +x_344 = lean_array_push(x_343, x_342); +x_345 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_345, 0, x_331); +lean_ctor_set(x_345, 1, x_328); +lean_ctor_set(x_345, 2, x_344); +x_346 = l_Lean_Elab_Command_elabInductive___closed__1; +x_347 = lean_array_push(x_346, x_345); +x_348 = l_Lean_Elab_Command_elabDeclaration___closed__4; +x_349 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_349, 0, x_331); +lean_ctor_set(x_349, 1, x_348); +lean_ctor_set(x_349, 2, x_347); +x_350 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35; +lean_inc(x_318); +x_351 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_351, 0, x_318); +lean_ctor_set(x_351, 1, x_350); +x_352 = l_Lean_Elab_Command_elabDeclaration___closed__10; +x_353 = lean_array_push(x_352, x_326); +x_354 = lean_array_push(x_353, x_349); +x_355 = lean_array_push(x_354, x_351); x_356 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_356, 0, x_301); -lean_ctor_set(x_356, 1, x_355); -lean_ctor_set(x_356, 2, x_354); -x_357 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; -lean_inc(x_287); -x_358 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_358, 0, x_287); -lean_ctor_set(x_358, 1, x_357); -x_359 = lean_array_push(x_311, x_296); -x_360 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_360, 0, x_301); -lean_ctor_set(x_360, 1, x_313); -lean_ctor_set(x_360, 2, x_359); -x_361 = lean_array_push(x_297, x_13); -x_362 = lean_array_push(x_361, x_360); -x_363 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; -x_364 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_364, 0, x_301); -lean_ctor_set(x_364, 1, x_363); -lean_ctor_set(x_364, 2, x_362); -x_365 = l_Lean_Elab_Command_expandInitCmd___closed__13; -x_366 = lean_array_push(x_365, x_364); -x_367 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -x_368 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_368, 0, x_301); -lean_ctor_set(x_368, 1, x_367); -lean_ctor_set(x_368, 2, x_366); -x_369 = lean_array_push(x_311, x_368); -x_370 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_370, 0, x_301); -lean_ctor_set(x_370, 1, x_313); -lean_ctor_set(x_370, 2, x_369); -x_371 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -lean_inc(x_287); -x_372 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_372, 0, x_287); -lean_ctor_set(x_372, 1, x_371); -x_373 = lean_array_push(x_337, x_358); -x_374 = lean_array_push(x_373, x_370); -x_375 = lean_array_push(x_374, x_372); -x_376 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; -x_377 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_377, 0, x_301); -lean_ctor_set(x_377, 1, x_376); -lean_ctor_set(x_377, 2, x_375); -x_378 = lean_array_push(x_311, x_377); -x_379 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_379, 0, x_301); -lean_ctor_set(x_379, 1, x_313); -lean_ctor_set(x_379, 2, x_378); -x_380 = l_Lean_Elab_Command_expandInitCmd___closed__1; -lean_inc(x_287); -x_381 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_381, 0, x_287); -lean_ctor_set(x_381, 1, x_380); -x_382 = lean_array_push(x_311, x_381); -x_383 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_383, 0, x_301); -lean_ctor_set(x_383, 1, x_21); -lean_ctor_set(x_383, 2, x_382); -x_384 = lean_array_push(x_311, x_383); -x_385 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_385, 0, x_301); -lean_ctor_set(x_385, 1, x_313); -lean_ctor_set(x_385, 2, x_384); -x_386 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_387 = lean_array_push(x_386, x_379); -x_388 = lean_array_push(x_387, x_385); -x_389 = lean_array_push(x_388, x_299); -x_390 = lean_array_push(x_389, x_299); -x_391 = lean_array_push(x_390, x_299); -x_392 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_393 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_393, 0, x_301); -lean_ctor_set(x_393, 1, x_392); -lean_ctor_set(x_393, 2, x_391); -x_394 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__15; -x_395 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_395, 0, x_287); -lean_ctor_set(x_395, 1, x_394); -x_396 = lean_array_push(x_319, x_17); -x_397 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_397, 0, x_301); -lean_ctor_set(x_397, 1, x_321); -lean_ctor_set(x_397, 2, x_396); -x_398 = lean_array_push(x_325, x_397); -x_399 = l_Lean_Elab_Command_expandInitCmd___closed__15; -x_400 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_400, 0, x_301); -lean_ctor_set(x_400, 1, x_399); -lean_ctor_set(x_400, 2, x_398); -x_401 = l_Lean_Elab_Command_expandInitCmd___closed__16; -x_402 = lean_array_push(x_401, x_395); -x_403 = lean_array_push(x_402, x_14); -x_404 = lean_array_push(x_403, x_400); -x_405 = lean_array_push(x_404, x_299); -x_406 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__16; -x_407 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_407, 0, x_301); -lean_ctor_set(x_407, 1, x_406); -lean_ctor_set(x_407, 2, x_405); -x_408 = lean_array_push(x_297, x_393); -x_409 = lean_array_push(x_408, x_407); -x_410 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_410, 0, x_301); -lean_ctor_set(x_410, 1, x_355); -lean_ctor_set(x_410, 2, x_409); -x_411 = lean_array_push(x_297, x_356); -x_412 = lean_array_push(x_411, x_410); -x_413 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_413, 0, x_301); -lean_ctor_set(x_413, 1, x_313); -lean_ctor_set(x_413, 2, x_412); -lean_ctor_set(x_285, 0, x_413); -return x_285; -} -else -{ -lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; -x_414 = lean_ctor_get(x_285, 0); -x_415 = lean_ctor_get(x_285, 1); -lean_inc(x_415); -lean_inc(x_414); -lean_dec(x_285); -x_416 = lean_ctor_get(x_3, 2); -lean_inc(x_416); -x_417 = lean_ctor_get(x_3, 1); -lean_inc(x_417); -lean_dec(x_3); -x_418 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; -lean_inc(x_414); -x_419 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_419, 0, x_414); -lean_ctor_set(x_419, 1, x_418); -x_420 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; -lean_inc(x_416); -lean_inc(x_417); -x_421 = l_Lean_addMacroScope(x_417, x_420, x_416); -x_422 = lean_box(0); -x_423 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -lean_inc(x_414); -x_424 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_424, 0, x_414); -lean_ctor_set(x_424, 1, x_423); -lean_ctor_set(x_424, 2, x_421); -lean_ctor_set(x_424, 3, x_422); -x_425 = l_Lean_Elab_Command_elabDeclaration___closed__7; -lean_inc(x_424); -x_426 = lean_array_push(x_425, x_424); -x_427 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_428 = lean_array_push(x_426, x_427); -x_429 = lean_box(2); -x_430 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; -x_431 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_431, 0, x_429); -lean_ctor_set(x_431, 1, x_430); -lean_ctor_set(x_431, 2, x_428); -x_432 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; -lean_inc(x_414); -x_433 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_433, 0, x_414); -lean_ctor_set(x_433, 1, x_432); -x_434 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -x_435 = l_Lean_addMacroScope(x_417, x_434, x_416); -x_436 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -x_437 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; -lean_inc(x_414); -x_438 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_438, 0, x_414); -lean_ctor_set(x_438, 1, x_436); -lean_ctor_set(x_438, 2, x_435); -lean_ctor_set(x_438, 3, x_437); -x_439 = l_Lean_Elab_Command_elabInductive___closed__1; -lean_inc(x_17); -x_440 = lean_array_push(x_439, x_17); -x_441 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_442 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_442, 0, x_429); -lean_ctor_set(x_442, 1, x_441); -lean_ctor_set(x_442, 2, x_440); -x_443 = lean_array_push(x_425, x_438); -x_444 = lean_array_push(x_443, x_442); -x_445 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; -x_446 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_446, 0, x_429); -lean_ctor_set(x_446, 1, x_445); -lean_ctor_set(x_446, 2, x_444); -x_447 = lean_array_push(x_425, x_433); -lean_inc(x_447); -x_448 = lean_array_push(x_447, x_446); -x_449 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; -x_450 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_450, 0, x_429); -lean_ctor_set(x_450, 1, x_449); -lean_ctor_set(x_450, 2, x_448); -x_451 = lean_array_push(x_439, x_450); +lean_ctor_set(x_356, 0, x_331); +lean_ctor_set(x_356, 1, x_324); +lean_ctor_set(x_356, 2, x_355); +x_357 = lean_array_push(x_346, x_356); +x_358 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_358, 0, x_331); +lean_ctor_set(x_358, 1, x_348); +lean_ctor_set(x_358, 2, x_357); +x_359 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3; +x_360 = lean_array_push(x_359, x_358); +x_361 = lean_array_push(x_360, x_340); +x_362 = lean_array_push(x_361, x_340); +x_363 = lean_array_push(x_362, x_340); +x_364 = lean_array_push(x_363, x_340); +x_365 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_365, 0, x_331); +lean_ctor_set(x_365, 1, x_5); +lean_ctor_set(x_365, 2, x_364); +x_366 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; +lean_inc(x_4); +x_367 = l_Lean_Name_str___override(x_4, x_366); +lean_inc(x_318); +x_368 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_368, 0, x_318); +lean_ctor_set(x_368, 1, x_366); +x_369 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7; +lean_inc(x_4); +x_370 = l_Lean_Name_str___override(x_4, x_369); +x_371 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11; +lean_inc(x_319); +lean_inc(x_320); +x_372 = l_Lean_addMacroScope(x_320, x_371, x_319); +x_373 = lean_box(0); +x_374 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10; +lean_inc(x_318); +x_375 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_375, 0, x_318); +lean_ctor_set(x_375, 1, x_374); +lean_ctor_set(x_375, 2, x_372); +lean_ctor_set(x_375, 3, x_373); +x_376 = lean_array_push(x_338, x_375); +x_377 = lean_array_push(x_376, x_340); +x_378 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_378, 0, x_331); +lean_ctor_set(x_378, 1, x_370); +lean_ctor_set(x_378, 2, x_377); +x_379 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12; +lean_inc(x_4); +x_380 = l_Lean_Name_str___override(x_4, x_379); +x_381 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13; +lean_inc(x_15); +x_382 = l_Lean_Name_str___override(x_15, x_381); +x_383 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14; +lean_inc(x_318); +x_384 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_384, 0, x_318); +lean_ctor_set(x_384, 1, x_383); +x_385 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15; +lean_inc(x_15); +x_386 = l_Lean_Name_str___override(x_15, x_385); +x_387 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19; +lean_inc(x_319); +lean_inc(x_320); +x_388 = l_Lean_addMacroScope(x_320, x_387, x_319); +x_389 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18; +x_390 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21; +lean_inc(x_318); +x_391 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_391, 0, x_318); +lean_ctor_set(x_391, 1, x_389); +lean_ctor_set(x_391, 2, x_388); +lean_ctor_set(x_391, 3, x_390); +x_392 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5; +x_393 = l_Lean_addMacroScope(x_320, x_392, x_319); +x_394 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4; +x_395 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7; +lean_inc(x_318); +x_396 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_396, 0, x_318); +lean_ctor_set(x_396, 1, x_394); +lean_ctor_set(x_396, 2, x_393); +lean_ctor_set(x_396, 3, x_395); +x_397 = lean_array_push(x_346, x_396); +x_398 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_398, 0, x_331); +lean_ctor_set(x_398, 1, x_348); +lean_ctor_set(x_398, 2, x_397); +x_399 = lean_array_push(x_338, x_391); +x_400 = lean_array_push(x_399, x_398); +x_401 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_401, 0, x_331); +lean_ctor_set(x_401, 1, x_386); +lean_ctor_set(x_401, 2, x_400); +x_402 = lean_array_push(x_338, x_384); +x_403 = lean_array_push(x_402, x_401); +x_404 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_404, 0, x_331); +lean_ctor_set(x_404, 1, x_382); +lean_ctor_set(x_404, 2, x_403); +x_405 = lean_array_push(x_346, x_404); +x_406 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_406, 0, x_331); +lean_ctor_set(x_406, 1, x_348); +lean_ctor_set(x_406, 2, x_405); +x_407 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22; +x_408 = lean_array_push(x_407, x_406); +x_409 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_409, 0, x_331); +lean_ctor_set(x_409, 1, x_380); +lean_ctor_set(x_409, 2, x_408); +x_410 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23; +x_411 = l_Lean_Name_str___override(x_4, x_410); +x_412 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24; +lean_inc(x_318); +x_413 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_413, 0, x_318); +lean_ctor_set(x_413, 1, x_412); +x_414 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25; +x_415 = l_Lean_Name_str___override(x_15, x_414); +x_416 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_416, 0, x_318); +lean_ctor_set(x_416, 1, x_414); +x_417 = lean_array_push(x_338, x_416); +x_418 = lean_array_push(x_417, x_13); +x_419 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_419, 0, x_331); +lean_ctor_set(x_419, 1, x_415); +lean_ctor_set(x_419, 2, x_418); +x_420 = lean_array_push(x_352, x_413); +x_421 = lean_array_push(x_420, x_419); +x_422 = lean_array_push(x_421, x_340); +x_423 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_423, 0, x_331); +lean_ctor_set(x_423, 1, x_411); +lean_ctor_set(x_423, 2, x_422); +x_424 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26; +x_425 = lean_array_push(x_424, x_368); +x_426 = lean_array_push(x_425, x_378); +x_427 = lean_array_push(x_426, x_409); +x_428 = lean_array_push(x_427, x_423); +x_429 = lean_array_push(x_428, x_340); +x_430 = lean_array_push(x_429, x_340); +x_431 = lean_array_push(x_430, x_340); +x_432 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_432, 0, x_331); +lean_ctor_set(x_432, 1, x_367); +lean_ctor_set(x_432, 2, x_431); +x_433 = lean_array_push(x_338, x_365); +x_434 = lean_array_push(x_433, x_432); +x_435 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_435, 0, x_331); +lean_ctor_set(x_435, 1, x_322); +lean_ctor_set(x_435, 2, x_434); +lean_ctor_set(x_316, 0, x_435); +return x_316; +} +else +{ +lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; +x_436 = lean_ctor_get(x_316, 0); +x_437 = lean_ctor_get(x_316, 1); +lean_inc(x_437); +lean_inc(x_436); +lean_dec(x_316); +x_438 = lean_ctor_get(x_10, 2); +lean_inc(x_438); +x_439 = lean_ctor_get(x_10, 1); +lean_inc(x_439); +lean_dec(x_10); +x_440 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__7; +lean_inc(x_4); +x_441 = l_Lean_Name_str___override(x_4, x_440); +x_442 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27; +lean_inc(x_15); +x_443 = l_Lean_Name_str___override(x_15, x_442); +x_444 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28; +lean_inc(x_436); +x_445 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_445, 0, x_436); +lean_ctor_set(x_445, 1, x_444); +x_446 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29; +lean_inc(x_15); +x_447 = l_Lean_Name_str___override(x_15, x_446); +x_448 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30; +lean_inc(x_15); +x_449 = l_Lean_Name_str___override(x_15, x_448); +x_450 = lean_box(2); +x_451 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31; x_452 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_452, 0, x_429); -lean_ctor_set(x_452, 1, x_441); +lean_ctor_set(x_452, 0, x_450); +lean_ctor_set(x_452, 1, x_449); lean_ctor_set(x_452, 2, x_451); -x_453 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; -x_454 = lean_array_push(x_453, x_452); -x_455 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; -x_456 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_456, 0, x_429); -lean_ctor_set(x_456, 1, x_455); -lean_ctor_set(x_456, 2, x_454); -x_457 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; -lean_inc(x_414); -x_458 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_458, 0, x_414); -lean_ctor_set(x_458, 1, x_457); -x_459 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -lean_inc(x_414); -x_460 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_460, 0, x_414); -lean_ctor_set(x_460, 1, x_459); -x_461 = lean_array_push(x_425, x_460); -x_462 = lean_array_push(x_461, x_10); -x_463 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; +x_453 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32; +x_454 = l_Lean_Name_str___override(x_2, x_453); +x_455 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33; +x_456 = l_Lean_Name_str___override(x_454, x_455); +x_457 = l_Lean_Elab_Command_elabDeclaration___closed__7; +x_458 = lean_array_push(x_457, x_17); +x_459 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; +x_460 = lean_array_push(x_458, x_459); +x_461 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_461, 0, x_450); +lean_ctor_set(x_461, 1, x_456); +lean_ctor_set(x_461, 2, x_460); +x_462 = lean_array_push(x_457, x_452); +x_463 = lean_array_push(x_462, x_461); x_464 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_464, 0, x_429); -lean_ctor_set(x_464, 1, x_463); -lean_ctor_set(x_464, 2, x_462); -x_465 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_466 = lean_array_push(x_465, x_458); -x_467 = lean_array_push(x_466, x_464); -x_468 = lean_array_push(x_467, x_427); -x_469 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; -x_470 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_470, 0, x_429); +lean_ctor_set(x_464, 0, x_450); +lean_ctor_set(x_464, 1, x_447); +lean_ctor_set(x_464, 2, x_463); +x_465 = l_Lean_Elab_Command_elabInductive___closed__1; +x_466 = lean_array_push(x_465, x_464); +x_467 = l_Lean_Elab_Command_elabDeclaration___closed__4; +x_468 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_468, 0, x_450); +lean_ctor_set(x_468, 1, x_467); +lean_ctor_set(x_468, 2, x_466); +x_469 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35; +lean_inc(x_436); +x_470 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_470, 0, x_436); lean_ctor_set(x_470, 1, x_469); -lean_ctor_set(x_470, 2, x_468); -x_471 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; -x_472 = lean_array_push(x_471, x_419); -x_473 = lean_array_push(x_472, x_431); -x_474 = lean_array_push(x_473, x_456); -x_475 = lean_array_push(x_474, x_470); -x_476 = lean_array_push(x_475, x_427); -x_477 = lean_array_push(x_476, x_427); -x_478 = lean_array_push(x_477, x_427); -x_479 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -x_480 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_480, 0, x_429); -lean_ctor_set(x_480, 1, x_479); -lean_ctor_set(x_480, 2, x_478); -x_481 = l_Lean_Elab_Command_expandInitCmd___closed__12; -x_482 = lean_array_push(x_481, x_480); -x_483 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; +x_471 = l_Lean_Elab_Command_elabDeclaration___closed__10; +x_472 = lean_array_push(x_471, x_445); +x_473 = lean_array_push(x_472, x_468); +x_474 = lean_array_push(x_473, x_470); +x_475 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_475, 0, x_450); +lean_ctor_set(x_475, 1, x_443); +lean_ctor_set(x_475, 2, x_474); +x_476 = lean_array_push(x_465, x_475); +x_477 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_477, 0, x_450); +lean_ctor_set(x_477, 1, x_467); +lean_ctor_set(x_477, 2, x_476); +x_478 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3; +x_479 = lean_array_push(x_478, x_477); +x_480 = lean_array_push(x_479, x_459); +x_481 = lean_array_push(x_480, x_459); +x_482 = lean_array_push(x_481, x_459); +x_483 = lean_array_push(x_482, x_459); x_484 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_484, 0, x_429); -lean_ctor_set(x_484, 1, x_483); -lean_ctor_set(x_484, 2, x_482); -x_485 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; -lean_inc(x_414); -x_486 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_486, 0, x_414); -lean_ctor_set(x_486, 1, x_485); -x_487 = lean_array_push(x_439, x_424); -x_488 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_488, 0, x_429); -lean_ctor_set(x_488, 1, x_441); -lean_ctor_set(x_488, 2, x_487); -x_489 = lean_array_push(x_425, x_13); -x_490 = lean_array_push(x_489, x_488); -x_491 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; -x_492 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_492, 0, x_429); -lean_ctor_set(x_492, 1, x_491); -lean_ctor_set(x_492, 2, x_490); -x_493 = l_Lean_Elab_Command_expandInitCmd___closed__13; -x_494 = lean_array_push(x_493, x_492); -x_495 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -x_496 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_496, 0, x_429); -lean_ctor_set(x_496, 1, x_495); -lean_ctor_set(x_496, 2, x_494); -x_497 = lean_array_push(x_439, x_496); -x_498 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_498, 0, x_429); -lean_ctor_set(x_498, 1, x_441); -lean_ctor_set(x_498, 2, x_497); -x_499 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -lean_inc(x_414); -x_500 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_500, 0, x_414); -lean_ctor_set(x_500, 1, x_499); -x_501 = lean_array_push(x_465, x_486); -x_502 = lean_array_push(x_501, x_498); -x_503 = lean_array_push(x_502, x_500); -x_504 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; -x_505 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_505, 0, x_429); -lean_ctor_set(x_505, 1, x_504); -lean_ctor_set(x_505, 2, x_503); -x_506 = lean_array_push(x_439, x_505); -x_507 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_507, 0, x_429); -lean_ctor_set(x_507, 1, x_441); -lean_ctor_set(x_507, 2, x_506); -x_508 = l_Lean_Elab_Command_expandInitCmd___closed__1; -lean_inc(x_414); -x_509 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_509, 0, x_414); -lean_ctor_set(x_509, 1, x_508); -x_510 = lean_array_push(x_439, x_509); -x_511 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_511, 0, x_429); -lean_ctor_set(x_511, 1, x_21); -lean_ctor_set(x_511, 2, x_510); -x_512 = lean_array_push(x_439, x_511); -x_513 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_513, 0, x_429); -lean_ctor_set(x_513, 1, x_441); -lean_ctor_set(x_513, 2, x_512); -x_514 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_515 = lean_array_push(x_514, x_507); -x_516 = lean_array_push(x_515, x_513); -x_517 = lean_array_push(x_516, x_427); -x_518 = lean_array_push(x_517, x_427); -x_519 = lean_array_push(x_518, x_427); -x_520 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_521 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_521, 0, x_429); -lean_ctor_set(x_521, 1, x_520); -lean_ctor_set(x_521, 2, x_519); -x_522 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__15; -x_523 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_523, 0, x_414); -lean_ctor_set(x_523, 1, x_522); -x_524 = lean_array_push(x_447, x_17); +lean_ctor_set(x_484, 0, x_450); +lean_ctor_set(x_484, 1, x_5); +lean_ctor_set(x_484, 2, x_483); +x_485 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; +lean_inc(x_4); +x_486 = l_Lean_Name_str___override(x_4, x_485); +lean_inc(x_436); +x_487 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_487, 0, x_436); +lean_ctor_set(x_487, 1, x_485); +x_488 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7; +lean_inc(x_4); +x_489 = l_Lean_Name_str___override(x_4, x_488); +x_490 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11; +lean_inc(x_438); +lean_inc(x_439); +x_491 = l_Lean_addMacroScope(x_439, x_490, x_438); +x_492 = lean_box(0); +x_493 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10; +lean_inc(x_436); +x_494 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_494, 0, x_436); +lean_ctor_set(x_494, 1, x_493); +lean_ctor_set(x_494, 2, x_491); +lean_ctor_set(x_494, 3, x_492); +x_495 = lean_array_push(x_457, x_494); +x_496 = lean_array_push(x_495, x_459); +x_497 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_497, 0, x_450); +lean_ctor_set(x_497, 1, x_489); +lean_ctor_set(x_497, 2, x_496); +x_498 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12; +lean_inc(x_4); +x_499 = l_Lean_Name_str___override(x_4, x_498); +x_500 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13; +lean_inc(x_15); +x_501 = l_Lean_Name_str___override(x_15, x_500); +x_502 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14; +lean_inc(x_436); +x_503 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_503, 0, x_436); +lean_ctor_set(x_503, 1, x_502); +x_504 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15; +lean_inc(x_15); +x_505 = l_Lean_Name_str___override(x_15, x_504); +x_506 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19; +lean_inc(x_438); +lean_inc(x_439); +x_507 = l_Lean_addMacroScope(x_439, x_506, x_438); +x_508 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18; +x_509 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21; +lean_inc(x_436); +x_510 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_510, 0, x_436); +lean_ctor_set(x_510, 1, x_508); +lean_ctor_set(x_510, 2, x_507); +lean_ctor_set(x_510, 3, x_509); +x_511 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5; +x_512 = l_Lean_addMacroScope(x_439, x_511, x_438); +x_513 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4; +x_514 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7; +lean_inc(x_436); +x_515 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_515, 0, x_436); +lean_ctor_set(x_515, 1, x_513); +lean_ctor_set(x_515, 2, x_512); +lean_ctor_set(x_515, 3, x_514); +x_516 = lean_array_push(x_465, x_515); +x_517 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_517, 0, x_450); +lean_ctor_set(x_517, 1, x_467); +lean_ctor_set(x_517, 2, x_516); +x_518 = lean_array_push(x_457, x_510); +x_519 = lean_array_push(x_518, x_517); +x_520 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_520, 0, x_450); +lean_ctor_set(x_520, 1, x_505); +lean_ctor_set(x_520, 2, x_519); +x_521 = lean_array_push(x_457, x_503); +x_522 = lean_array_push(x_521, x_520); +x_523 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_523, 0, x_450); +lean_ctor_set(x_523, 1, x_501); +lean_ctor_set(x_523, 2, x_522); +x_524 = lean_array_push(x_465, x_523); x_525 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_525, 0, x_429); -lean_ctor_set(x_525, 1, x_449); +lean_ctor_set(x_525, 0, x_450); +lean_ctor_set(x_525, 1, x_467); lean_ctor_set(x_525, 2, x_524); -x_526 = lean_array_push(x_453, x_525); -x_527 = l_Lean_Elab_Command_expandInitCmd___closed__15; +x_526 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22; +x_527 = lean_array_push(x_526, x_525); x_528 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_528, 0, x_429); -lean_ctor_set(x_528, 1, x_527); -lean_ctor_set(x_528, 2, x_526); -x_529 = l_Lean_Elab_Command_expandInitCmd___closed__16; -x_530 = lean_array_push(x_529, x_523); -x_531 = lean_array_push(x_530, x_14); -x_532 = lean_array_push(x_531, x_528); -x_533 = lean_array_push(x_532, x_427); -x_534 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__16; -x_535 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_535, 0, x_429); -lean_ctor_set(x_535, 1, x_534); -lean_ctor_set(x_535, 2, x_533); -x_536 = lean_array_push(x_425, x_521); -x_537 = lean_array_push(x_536, x_535); +lean_ctor_set(x_528, 0, x_450); +lean_ctor_set(x_528, 1, x_499); +lean_ctor_set(x_528, 2, x_527); +x_529 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23; +x_530 = l_Lean_Name_str___override(x_4, x_529); +x_531 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24; +lean_inc(x_436); +x_532 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_532, 0, x_436); +lean_ctor_set(x_532, 1, x_531); +x_533 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25; +x_534 = l_Lean_Name_str___override(x_15, x_533); +x_535 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_535, 0, x_436); +lean_ctor_set(x_535, 1, x_533); +x_536 = lean_array_push(x_457, x_535); +x_537 = lean_array_push(x_536, x_13); x_538 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_538, 0, x_429); -lean_ctor_set(x_538, 1, x_483); +lean_ctor_set(x_538, 0, x_450); +lean_ctor_set(x_538, 1, x_534); lean_ctor_set(x_538, 2, x_537); -x_539 = lean_array_push(x_425, x_484); +x_539 = lean_array_push(x_471, x_532); x_540 = lean_array_push(x_539, x_538); -x_541 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_541, 0, x_429); -lean_ctor_set(x_541, 1, x_441); -lean_ctor_set(x_541, 2, x_540); -x_542 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_542, 0, x_541); -lean_ctor_set(x_542, 1, x_415); -return x_542; +x_541 = lean_array_push(x_540, x_459); +x_542 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_542, 0, x_450); +lean_ctor_set(x_542, 1, x_530); +lean_ctor_set(x_542, 2, x_541); +x_543 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26; +x_544 = lean_array_push(x_543, x_487); +x_545 = lean_array_push(x_544, x_497); +x_546 = lean_array_push(x_545, x_528); +x_547 = lean_array_push(x_546, x_542); +x_548 = lean_array_push(x_547, x_459); +x_549 = lean_array_push(x_548, x_459); +x_550 = lean_array_push(x_549, x_459); +x_551 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_551, 0, x_450); +lean_ctor_set(x_551, 1, x_486); +lean_ctor_set(x_551, 2, x_550); +x_552 = lean_array_push(x_457, x_484); +x_553 = lean_array_push(x_552, x_551); +x_554 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_554, 0, x_450); +lean_ctor_set(x_554, 1, x_441); +lean_ctor_set(x_554, 2, x_553); +x_555 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_555, 0, x_554); +lean_ctor_set(x_555, 1, x_437); +return x_555; +} +} +} +} +} } } } else { -lean_object* x_543; uint8_t x_544; -lean_dec(x_6); +lean_object* x_556; uint8_t x_557; +x_556 = lean_ctor_get(x_8, 0); +lean_inc(x_556); +lean_dec(x_8); +x_557 = !lean_is_exclusive(x_9); +if (x_557 == 0) +{ +lean_object* x_558; uint8_t x_559; +x_558 = lean_ctor_get(x_9, 0); lean_inc(x_3); -x_543 = l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(x_3, x_4); -x_544 = !lean_is_exclusive(x_543); -if (x_544 == 0) -{ -lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; lean_object* x_570; lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; -x_545 = lean_ctor_get(x_543, 0); -x_546 = lean_ctor_get(x_3, 2); -lean_inc(x_546); -x_547 = lean_ctor_get(x_3, 1); -lean_inc(x_547); -lean_dec(x_3); -x_548 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; -lean_inc(x_545); -x_549 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_549, 0, x_545); -lean_ctor_set(x_549, 1, x_548); -x_550 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; -lean_inc(x_546); -lean_inc(x_547); -x_551 = l_Lean_addMacroScope(x_547, x_550, x_546); -x_552 = lean_box(0); -x_553 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -lean_inc(x_545); -x_554 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_554, 0, x_545); -lean_ctor_set(x_554, 1, x_553); -lean_ctor_set(x_554, 2, x_551); -lean_ctor_set(x_554, 3, x_552); -x_555 = l_Lean_Elab_Command_elabDeclaration___closed__7; -lean_inc(x_554); -x_556 = lean_array_push(x_555, x_554); -x_557 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_558 = lean_array_push(x_556, x_557); -x_559 = lean_box(2); -x_560 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; -x_561 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_561, 0, x_559); -lean_ctor_set(x_561, 1, x_560); -lean_ctor_set(x_561, 2, x_558); -x_562 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; -lean_inc(x_545); -x_563 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_563, 0, x_545); -lean_ctor_set(x_563, 1, x_562); -x_564 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -x_565 = l_Lean_addMacroScope(x_547, x_564, x_546); -x_566 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -x_567 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; -lean_inc(x_545); -x_568 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_568, 0, x_545); -lean_ctor_set(x_568, 1, x_566); -lean_ctor_set(x_568, 2, x_565); -lean_ctor_set(x_568, 3, x_567); -x_569 = l_Lean_Elab_Command_elabInductive___closed__1; -lean_inc(x_17); -x_570 = lean_array_push(x_569, x_17); -x_571 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_572 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_572, 0, x_559); -lean_ctor_set(x_572, 1, x_571); -lean_ctor_set(x_572, 2, x_570); -x_573 = lean_array_push(x_555, x_568); -x_574 = lean_array_push(x_573, x_572); -x_575 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; -x_576 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_576, 0, x_559); -lean_ctor_set(x_576, 1, x_575); -lean_ctor_set(x_576, 2, x_574); -x_577 = lean_array_push(x_555, x_563); -lean_inc(x_577); -x_578 = lean_array_push(x_577, x_576); -x_579 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; -x_580 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_580, 0, x_559); -lean_ctor_set(x_580, 1, x_579); -lean_ctor_set(x_580, 2, x_578); -x_581 = lean_array_push(x_569, x_580); -x_582 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_582, 0, x_559); -lean_ctor_set(x_582, 1, x_571); -lean_ctor_set(x_582, 2, x_581); -x_583 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; -x_584 = lean_array_push(x_583, x_582); -x_585 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; -x_586 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_586, 0, x_559); -lean_ctor_set(x_586, 1, x_585); -lean_ctor_set(x_586, 2, x_584); -x_587 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; -lean_inc(x_545); -x_588 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_588, 0, x_545); -lean_ctor_set(x_588, 1, x_587); -x_589 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -lean_inc(x_545); -x_590 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_590, 0, x_545); -lean_ctor_set(x_590, 1, x_589); -x_591 = lean_array_push(x_555, x_590); -x_592 = lean_array_push(x_591, x_10); -x_593 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; -x_594 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_594, 0, x_559); -lean_ctor_set(x_594, 1, x_593); -lean_ctor_set(x_594, 2, x_592); -x_595 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_596 = lean_array_push(x_595, x_588); -x_597 = lean_array_push(x_596, x_594); -x_598 = lean_array_push(x_597, x_557); -x_599 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; -x_600 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_600, 0, x_559); -lean_ctor_set(x_600, 1, x_599); -lean_ctor_set(x_600, 2, x_598); -x_601 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; -x_602 = lean_array_push(x_601, x_549); -x_603 = lean_array_push(x_602, x_561); -x_604 = lean_array_push(x_603, x_586); -x_605 = lean_array_push(x_604, x_600); -x_606 = lean_array_push(x_605, x_557); -x_607 = lean_array_push(x_606, x_557); -x_608 = lean_array_push(x_607, x_557); -x_609 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -x_610 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_610, 0, x_559); -lean_ctor_set(x_610, 1, x_609); -lean_ctor_set(x_610, 2, x_608); -x_611 = l_Lean_Elab_Command_expandInitCmd___closed__12; -x_612 = lean_array_push(x_611, x_610); -x_613 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; -x_614 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_614, 0, x_559); -lean_ctor_set(x_614, 1, x_613); -lean_ctor_set(x_614, 2, x_612); -x_615 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; -lean_inc(x_545); -x_616 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_616, 0, x_545); -lean_ctor_set(x_616, 1, x_615); -x_617 = lean_array_push(x_569, x_554); -x_618 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_618, 0, x_559); -lean_ctor_set(x_618, 1, x_571); -lean_ctor_set(x_618, 2, x_617); -x_619 = lean_array_push(x_555, x_13); -x_620 = lean_array_push(x_619, x_618); -x_621 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; -x_622 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_622, 0, x_559); -lean_ctor_set(x_622, 1, x_621); -lean_ctor_set(x_622, 2, x_620); -x_623 = l_Lean_Elab_Command_expandInitCmd___closed__13; -x_624 = lean_array_push(x_623, x_622); -x_625 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -x_626 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_626, 0, x_559); -lean_ctor_set(x_626, 1, x_625); -lean_ctor_set(x_626, 2, x_624); -x_627 = lean_array_push(x_569, x_626); -x_628 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_628, 0, x_559); -lean_ctor_set(x_628, 1, x_571); -lean_ctor_set(x_628, 2, x_627); -x_629 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -lean_inc(x_545); -x_630 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_630, 0, x_545); -lean_ctor_set(x_630, 1, x_629); -x_631 = lean_array_push(x_595, x_616); -x_632 = lean_array_push(x_631, x_628); -x_633 = lean_array_push(x_632, x_630); -x_634 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; -x_635 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_635, 0, x_559); -lean_ctor_set(x_635, 1, x_634); -lean_ctor_set(x_635, 2, x_633); -x_636 = lean_array_push(x_569, x_635); -x_637 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_637, 0, x_559); -lean_ctor_set(x_637, 1, x_571); -lean_ctor_set(x_637, 2, x_636); -x_638 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_639 = lean_array_push(x_638, x_637); -x_640 = lean_array_push(x_639, x_557); -x_641 = lean_array_push(x_640, x_557); -x_642 = lean_array_push(x_641, x_557); -x_643 = lean_array_push(x_642, x_557); -x_644 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_645 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_645, 0, x_559); -lean_ctor_set(x_645, 1, x_644); -lean_ctor_set(x_645, 2, x_643); -x_646 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__15; -x_647 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_647, 0, x_545); -lean_ctor_set(x_647, 1, x_646); -x_648 = lean_array_push(x_577, x_17); -x_649 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_649, 0, x_559); -lean_ctor_set(x_649, 1, x_579); -lean_ctor_set(x_649, 2, x_648); -x_650 = lean_array_push(x_583, x_649); -x_651 = l_Lean_Elab_Command_expandInitCmd___closed__15; -x_652 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_652, 0, x_559); -lean_ctor_set(x_652, 1, x_651); -lean_ctor_set(x_652, 2, x_650); -x_653 = l_Lean_Elab_Command_expandInitCmd___closed__16; -x_654 = lean_array_push(x_653, x_647); -x_655 = lean_array_push(x_654, x_14); -x_656 = lean_array_push(x_655, x_652); -x_657 = lean_array_push(x_656, x_557); -x_658 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__16; -x_659 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_659, 0, x_559); -lean_ctor_set(x_659, 1, x_658); -lean_ctor_set(x_659, 2, x_657); -x_660 = lean_array_push(x_555, x_645); -x_661 = lean_array_push(x_660, x_659); -x_662 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_662, 0, x_559); -lean_ctor_set(x_662, 1, x_613); -lean_ctor_set(x_662, 2, x_661); -x_663 = lean_array_push(x_555, x_614); -x_664 = lean_array_push(x_663, x_662); -x_665 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_665, 0, x_559); -lean_ctor_set(x_665, 1, x_571); -lean_ctor_set(x_665, 2, x_664); -lean_ctor_set(x_543, 0, x_665); -return x_543; -} -else -{ -lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; lean_object* x_677; lean_object* x_678; lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; lean_object* x_713; lean_object* x_714; lean_object* x_715; lean_object* x_716; lean_object* x_717; lean_object* x_718; lean_object* x_719; lean_object* x_720; lean_object* x_721; lean_object* x_722; lean_object* x_723; lean_object* x_724; lean_object* x_725; lean_object* x_726; lean_object* x_727; lean_object* x_728; lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; lean_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; lean_object* x_740; lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; lean_object* x_747; lean_object* x_748; lean_object* x_749; lean_object* x_750; lean_object* x_751; lean_object* x_752; lean_object* x_753; lean_object* x_754; lean_object* x_755; lean_object* x_756; lean_object* x_757; lean_object* x_758; lean_object* x_759; lean_object* x_760; lean_object* x_761; lean_object* x_762; lean_object* x_763; lean_object* x_764; lean_object* x_765; lean_object* x_766; lean_object* x_767; lean_object* x_768; lean_object* x_769; lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; lean_object* x_774; lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; -x_666 = lean_ctor_get(x_543, 0); -x_667 = lean_ctor_get(x_543, 1); -lean_inc(x_667); -lean_inc(x_666); -lean_dec(x_543); -x_668 = lean_ctor_get(x_3, 2); -lean_inc(x_668); -x_669 = lean_ctor_get(x_3, 1); -lean_inc(x_669); +x_559 = l_Lean_Syntax_isOfKind(x_3, x_5); +if (x_559 == 0) +{ +lean_object* x_560; lean_object* x_561; +lean_free_object(x_9); +lean_dec(x_558); +lean_dec(x_556); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_560 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_561 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_560, x_10, x_11); lean_dec(x_3); -x_670 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__11; -lean_inc(x_666); -x_671 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_671, 0, x_666); -lean_ctor_set(x_671, 1, x_670); -x_672 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26; -lean_inc(x_668); -lean_inc(x_669); -x_673 = l_Lean_addMacroScope(x_669, x_672, x_668); -x_674 = lean_box(0); -x_675 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25; -lean_inc(x_666); -x_676 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_676, 0, x_666); -lean_ctor_set(x_676, 1, x_675); -lean_ctor_set(x_676, 2, x_673); -lean_ctor_set(x_676, 3, x_674); -x_677 = l_Lean_Elab_Command_elabDeclaration___closed__7; -lean_inc(x_676); -x_678 = lean_array_push(x_677, x_676); -x_679 = l_Lean_Elab_Command_expandMutualPreamble___closed__3; -x_680 = lean_array_push(x_678, x_679); -x_681 = lean_box(2); -x_682 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22; -x_683 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_683, 0, x_681); -lean_ctor_set(x_683, 1, x_682); -lean_ctor_set(x_683, 2, x_680); -x_684 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31; -lean_inc(x_666); -x_685 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_685, 0, x_666); -lean_ctor_set(x_685, 1, x_684); -x_686 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37; -x_687 = l_Lean_addMacroScope(x_669, x_686, x_668); -x_688 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36; -x_689 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39; -lean_inc(x_666); -x_690 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_690, 0, x_666); -lean_ctor_set(x_690, 1, x_688); -lean_ctor_set(x_690, 2, x_687); -lean_ctor_set(x_690, 3, x_689); -x_691 = l_Lean_Elab_Command_elabInductive___closed__1; -lean_inc(x_17); -x_692 = lean_array_push(x_691, x_17); -x_693 = l_Lean_Elab_Command_elabDeclaration___closed__4; -x_694 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_694, 0, x_681); -lean_ctor_set(x_694, 1, x_693); -lean_ctor_set(x_694, 2, x_692); -x_695 = lean_array_push(x_677, x_690); -x_696 = lean_array_push(x_695, x_694); -x_697 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33; -x_698 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_698, 0, x_681); -lean_ctor_set(x_698, 1, x_697); -lean_ctor_set(x_698, 2, x_696); -x_699 = lean_array_push(x_677, x_685); -lean_inc(x_699); -x_700 = lean_array_push(x_699, x_698); -x_701 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30; -x_702 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_702, 0, x_681); -lean_ctor_set(x_702, 1, x_701); -lean_ctor_set(x_702, 2, x_700); -x_703 = lean_array_push(x_691, x_702); -x_704 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_704, 0, x_681); -lean_ctor_set(x_704, 1, x_693); -lean_ctor_set(x_704, 2, x_703); -x_705 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46; -x_706 = lean_array_push(x_705, x_704); -x_707 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28; -x_708 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_708, 0, x_681); -lean_ctor_set(x_708, 1, x_707); -lean_ctor_set(x_708, 2, x_706); -x_709 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49; -lean_inc(x_666); -x_710 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_710, 0, x_666); -lean_ctor_set(x_710, 1, x_709); -x_711 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50; -lean_inc(x_666); -x_712 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_712, 0, x_666); -lean_ctor_set(x_712, 1, x_711); -x_713 = lean_array_push(x_677, x_712); -x_714 = lean_array_push(x_713, x_10); -x_715 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51; -x_716 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_716, 0, x_681); -lean_ctor_set(x_716, 1, x_715); -lean_ctor_set(x_716, 2, x_714); -x_717 = l_Lean_Elab_Command_elabDeclaration___closed__10; -x_718 = lean_array_push(x_717, x_710); -x_719 = lean_array_push(x_718, x_716); -x_720 = lean_array_push(x_719, x_679); -x_721 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48; -x_722 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_722, 0, x_681); -lean_ctor_set(x_722, 1, x_721); -lean_ctor_set(x_722, 2, x_720); -x_723 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52; -x_724 = lean_array_push(x_723, x_671); -x_725 = lean_array_push(x_724, x_683); -x_726 = lean_array_push(x_725, x_708); -x_727 = lean_array_push(x_726, x_722); -x_728 = lean_array_push(x_727, x_679); -x_729 = lean_array_push(x_728, x_679); -x_730 = lean_array_push(x_729, x_679); -x_731 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__12; -x_732 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_732, 0, x_681); -lean_ctor_set(x_732, 1, x_731); -lean_ctor_set(x_732, 2, x_730); -x_733 = l_Lean_Elab_Command_expandInitCmd___closed__12; -x_734 = lean_array_push(x_733, x_732); -x_735 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__8; -x_736 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_736, 0, x_681); -lean_ctor_set(x_736, 1, x_735); -lean_ctor_set(x_736, 2, x_734); -x_737 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7; -lean_inc(x_666); -x_738 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_738, 0, x_666); -lean_ctor_set(x_738, 1, x_737); -x_739 = lean_array_push(x_691, x_676); -x_740 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_740, 0, x_681); -lean_ctor_set(x_740, 1, x_693); -lean_ctor_set(x_740, 2, x_739); -x_741 = lean_array_push(x_677, x_13); -x_742 = lean_array_push(x_741, x_740); -x_743 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17; -x_744 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_744, 0, x_681); -lean_ctor_set(x_744, 1, x_743); -lean_ctor_set(x_744, 2, x_742); -x_745 = l_Lean_Elab_Command_expandInitCmd___closed__13; -x_746 = lean_array_push(x_745, x_744); -x_747 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9; -x_748 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_748, 0, x_681); -lean_ctor_set(x_748, 1, x_747); -lean_ctor_set(x_748, 2, x_746); -x_749 = lean_array_push(x_691, x_748); -x_750 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_750, 0, x_681); -lean_ctor_set(x_750, 1, x_693); -lean_ctor_set(x_750, 2, x_749); -x_751 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5; -lean_inc(x_666); -x_752 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_752, 0, x_666); -lean_ctor_set(x_752, 1, x_751); -x_753 = lean_array_push(x_717, x_738); -x_754 = lean_array_push(x_753, x_750); -x_755 = lean_array_push(x_754, x_752); -x_756 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6; -x_757 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_757, 0, x_681); -lean_ctor_set(x_757, 1, x_756); -lean_ctor_set(x_757, 2, x_755); -x_758 = lean_array_push(x_691, x_757); -x_759 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_759, 0, x_681); -lean_ctor_set(x_759, 1, x_693); -lean_ctor_set(x_759, 2, x_758); -x_760 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20; -x_761 = lean_array_push(x_760, x_759); -x_762 = lean_array_push(x_761, x_679); -x_763 = lean_array_push(x_762, x_679); -x_764 = lean_array_push(x_763, x_679); -x_765 = lean_array_push(x_764, x_679); -x_766 = l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2; -x_767 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_767, 0, x_681); -lean_ctor_set(x_767, 1, x_766); -lean_ctor_set(x_767, 2, x_765); -x_768 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__15; -x_769 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_769, 0, x_666); -lean_ctor_set(x_769, 1, x_768); -x_770 = lean_array_push(x_699, x_17); -x_771 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_771, 0, x_681); -lean_ctor_set(x_771, 1, x_701); -lean_ctor_set(x_771, 2, x_770); -x_772 = lean_array_push(x_705, x_771); -x_773 = l_Lean_Elab_Command_expandInitCmd___closed__15; -x_774 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_774, 0, x_681); -lean_ctor_set(x_774, 1, x_773); -lean_ctor_set(x_774, 2, x_772); -x_775 = l_Lean_Elab_Command_expandInitCmd___closed__16; -x_776 = lean_array_push(x_775, x_769); -x_777 = lean_array_push(x_776, x_14); -x_778 = lean_array_push(x_777, x_774); -x_779 = lean_array_push(x_778, x_679); -x_780 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__16; -x_781 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_781, 0, x_681); -lean_ctor_set(x_781, 1, x_780); -lean_ctor_set(x_781, 2, x_779); -x_782 = lean_array_push(x_677, x_767); -x_783 = lean_array_push(x_782, x_781); -x_784 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_784, 0, x_681); -lean_ctor_set(x_784, 1, x_735); -lean_ctor_set(x_784, 2, x_783); -x_785 = lean_array_push(x_677, x_736); -x_786 = lean_array_push(x_785, x_784); -x_787 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_787, 0, x_681); -lean_ctor_set(x_787, 1, x_693); -lean_ctor_set(x_787, 2, x_786); -x_788 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_788, 0, x_787); -lean_ctor_set(x_788, 1, x_667); -return x_788; -} -} -} -else -{ -uint8_t x_789; -lean_dec(x_8); -x_789 = l_Lean_Syntax_isNone(x_6); -lean_dec(x_6); -if (x_789 == 0) +return x_561; +} +else { -lean_object* x_790; lean_object* x_791; uint8_t x_792; +lean_object* x_562; lean_object* x_563; uint8_t x_564; +x_562 = lean_unsigned_to_nat(0u); +x_563 = l_Lean_Syntax_getArg(x_3, x_562); +x_564 = l_Lean_Syntax_isNone(x_563); +if (x_564 == 0) +{ +lean_object* x_565; uint8_t x_566; +x_565 = lean_unsigned_to_nat(1u); +lean_inc(x_563); +x_566 = l_Lean_Syntax_matchesNull(x_563, x_565); +if (x_566 == 0) +{ +lean_object* x_567; lean_object* x_568; +lean_dec(x_563); +lean_free_object(x_9); +lean_dec(x_558); +lean_dec(x_556); +lean_dec(x_17); +lean_dec(x_15); lean_dec(x_13); -lean_dec(x_10); -x_790 = l_Lean_Elab_Command_expandInitCmd___closed__17; -x_791 = l_Lean_Macro_throwError___rarg(x_790, x_3, x_4); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_567 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_568 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_567, x_10, x_11); lean_dec(x_3); -x_792 = !lean_is_exclusive(x_791); -if (x_792 == 0) +return x_568; +} +else { -return x_791; +lean_object* x_569; lean_object* x_570; lean_object* x_571; uint8_t x_572; +x_569 = l_Lean_Syntax_getArg(x_563, x_562); +lean_dec(x_563); +x_570 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__8; +lean_inc(x_4); +x_571 = l_Lean_Name_str___override(x_4, x_570); +lean_inc(x_569); +x_572 = l_Lean_Syntax_isOfKind(x_569, x_571); +lean_dec(x_571); +if (x_572 == 0) +{ +lean_object* x_573; lean_object* x_574; +lean_dec(x_569); +lean_free_object(x_9); +lean_dec(x_558); +lean_dec(x_556); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_573 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_574 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_573, x_10, x_11); +lean_dec(x_3); +return x_574; } else { -lean_object* x_793; lean_object* x_794; lean_object* x_795; -x_793 = lean_ctor_get(x_791, 0); -x_794 = lean_ctor_get(x_791, 1); -lean_inc(x_794); -lean_inc(x_793); -lean_dec(x_791); -x_795 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_795, 0, x_793); -lean_ctor_set(x_795, 1, x_794); -return x_795; +lean_object* x_575; lean_object* x_576; +lean_ctor_set(x_9, 0, x_569); +x_575 = lean_box(0); +x_576 = l_Lean_Elab_Command_expandInitialize___lambda__3(x_3, x_3, x_4, x_15, x_558, x_13, x_2, x_17, x_556, x_5, x_575, x_9, x_10, x_11); +lean_dec(x_3); +return x_576; +} } } else { -lean_object* x_796; lean_object* x_797; -x_796 = lean_box(0); -x_797 = l_Lean_Elab_Command_expandInitCmd___lambda__1(x_13, x_10, x_796, x_3, x_4); -return x_797; +lean_object* x_577; lean_object* x_578; lean_object* x_579; +lean_dec(x_563); +lean_free_object(x_9); +x_577 = lean_box(0); +x_578 = lean_box(0); +x_579 = l_Lean_Elab_Command_expandInitialize___lambda__3(x_3, x_3, x_4, x_15, x_558, x_13, x_2, x_17, x_556, x_5, x_578, x_577, x_10, x_11); +lean_dec(x_3); +return x_579; +} } } +else +{ +lean_object* x_580; uint8_t x_581; +x_580 = lean_ctor_get(x_9, 0); +lean_inc(x_580); +lean_dec(x_9); +lean_inc(x_3); +x_581 = l_Lean_Syntax_isOfKind(x_3, x_5); +if (x_581 == 0) +{ +lean_object* x_582; lean_object* x_583; +lean_dec(x_580); +lean_dec(x_556); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_582 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_583 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_582, x_10, x_11); +lean_dec(x_3); +return x_583; } +else +{ +lean_object* x_584; lean_object* x_585; uint8_t x_586; +x_584 = lean_unsigned_to_nat(0u); +x_585 = l_Lean_Syntax_getArg(x_3, x_584); +x_586 = l_Lean_Syntax_isNone(x_585); +if (x_586 == 0) +{ +lean_object* x_587; uint8_t x_588; +x_587 = lean_unsigned_to_nat(1u); +lean_inc(x_585); +x_588 = l_Lean_Syntax_matchesNull(x_585, x_587); +if (x_588 == 0) +{ +lean_object* x_589; lean_object* x_590; +lean_dec(x_585); +lean_dec(x_580); +lean_dec(x_556); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_589 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_590 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_589, x_10, x_11); +lean_dec(x_3); +return x_590; } +else +{ +lean_object* x_591; lean_object* x_592; lean_object* x_593; uint8_t x_594; +x_591 = l_Lean_Syntax_getArg(x_585, x_584); +lean_dec(x_585); +x_592 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__8; +lean_inc(x_4); +x_593 = l_Lean_Name_str___override(x_4, x_592); +lean_inc(x_591); +x_594 = l_Lean_Syntax_isOfKind(x_591, x_593); +lean_dec(x_593); +if (x_594 == 0) +{ +lean_object* x_595; lean_object* x_596; +lean_dec(x_591); +lean_dec(x_580); +lean_dec(x_556); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_595 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1; +x_596 = l_Lean_Macro_throwErrorAt___rarg(x_3, x_595, x_10, x_11); +lean_dec(x_3); +return x_596; } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitCmd___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; -x_6 = l_Lean_Elab_Command_expandInitCmd___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_object* x_597; lean_object* x_598; lean_object* x_599; +x_597 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_597, 0, x_591); +x_598 = lean_box(0); +x_599 = l_Lean_Elab_Command_expandInitialize___lambda__3(x_3, x_3, x_4, x_15, x_580, x_13, x_2, x_17, x_556, x_5, x_598, x_597, x_10, x_11); lean_dec(x_3); -return x_6; +return x_599; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitCmd___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +} +else { -uint8_t x_5; lean_object* x_6; -x_5 = lean_unbox(x_1); -lean_dec(x_1); -x_6 = l_Lean_Elab_Command_expandInitCmd(x_5, x_2, x_3, x_4); -return x_6; +lean_object* x_600; lean_object* x_601; lean_object* x_602; +lean_dec(x_585); +x_600 = lean_box(0); +x_601 = lean_box(0); +x_602 = l_Lean_Elab_Command_expandInitialize___lambda__3(x_3, x_3, x_4, x_15, x_580, x_13, x_2, x_17, x_556, x_5, x_601, x_600, x_10, x_11); +lean_dec(x_3); +return x_602; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; -x_4 = 0; -x_5 = l_Lean_Elab_Command_expandInitCmd(x_4, x_1, x_2, x_3); -return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("initialize", 10); -return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2() { +} +} +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__1; +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("expandInitialize", 16); +x_1 = lean_mk_string_from_bytes("declModifiers", 13); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Command_elabDeclaration___closed__2; -x_2 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__3; +x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; +x_2 = l_Lean_Elab_Command_expandInitialize___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__5() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_expandInitialize), 3, 0); +x_1 = lean_mk_string_from_bytes("initializeKeyword", 17); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize(lean_object* x_1) { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___closed__5() { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Command_expandMutualNamespace___closed__5; -x_3 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2; -x_4 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__4; -x_5 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__5; -x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; +x_2 = l_Lean_Elab_Command_expandInitialize___closed__4; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(350u); -x_2 = lean_unsigned_to_nat(49u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); +x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__4; +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__4___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__2() { +static lean_object* _init_l_Lean_Elab_Command_expandInitialize___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(351u); -x_2 = lean_unsigned_to_nat(34u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); +x_1 = l_Lean_Elab_Command_expandInitialize___closed__6; +x_2 = l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__1; -x_2 = lean_unsigned_to_nat(49u); -x_3 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__2; -x_4 = lean_unsigned_to_nat(34u); -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; -} +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_Elab_Command_expandInitialize___closed__1; +lean_inc(x_1); +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_2); +lean_dec(x_1); +x_6 = lean_box(1); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(350u); -x_2 = lean_unsigned_to_nat(53u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_8 = lean_unsigned_to_nat(0u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +x_10 = l_Lean_Elab_Command_expandInitialize___closed__3; +lean_inc(x_9); +x_11 = l_Lean_Syntax_isOfKind(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_12 = lean_box(1); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_3); +return x_13; } +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_unsigned_to_nat(1u); +x_15 = l_Lean_Syntax_getArg(x_1, x_14); +x_16 = l_Lean_Elab_Command_expandInitialize___closed__5; +lean_inc(x_15); +x_17 = l_Lean_Syntax_isOfKind(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_15); +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_18 = lean_box(1); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_3); +return x_19; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__5() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(350u); -x_2 = lean_unsigned_to_nat(69u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_unsigned_to_nat(2u); +x_21 = l_Lean_Syntax_getArg(x_1, x_20); +x_22 = l_Lean_Syntax_isNone(x_21); +if (x_22 == 0) +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_unsigned_to_nat(3u); +lean_inc(x_21); +x_24 = l_Lean_Syntax_matchesNull(x_21, x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_21); +lean_dec(x_15); +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_25 = lean_box(1); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_3); +return x_26; } +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_27 = l_Lean_Syntax_getArg(x_21, x_8); +x_28 = l_Lean_Syntax_getArg(x_21, x_14); +lean_dec(x_21); +x_29 = l_Lean_Elab_Command_expandInitialize___closed__7; +lean_inc(x_28); +x_30 = l_Lean_Syntax_isOfKind(x_28, x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_15); +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_31 = lean_box(1); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_3); +return x_32; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__6() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__4; -x_2 = lean_unsigned_to_nat(53u); -x_3 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__5; -x_4 = lean_unsigned_to_nat(69u); -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_33 = l_Lean_Syntax_getArg(x_28, x_14); +lean_dec(x_28); +x_34 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_34, 0, x_27); +x_35 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_35, 0, x_33); +x_36 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__4; +x_37 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; +x_38 = lean_box(0); +x_39 = l_Lean_Elab_Command_expandInitialize___lambda__4(x_1, x_36, x_9, x_37, x_10, x_15, x_38, x_34, x_35, x_2, x_3); +return x_39; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__7() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__3; -x_2 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__6; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_dec(x_21); +x_40 = lean_box(0); +x_41 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__4; +x_42 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; +x_43 = lean_box(0); +x_44 = l_Lean_Elab_Command_expandInitialize___lambda__4(x_1, x_41, x_9, x_42, x_10, x_15, x_43, x_40, x_40, x_2, x_3); +return x_44; +} } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__4; -x_3 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__7; -x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); -return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandBuiltinInitialize(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__1___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; _start: { -uint8_t x_4; lean_object* x_5; -x_4 = 1; -x_5 = l_Lean_Elab_Command_expandInitCmd(x_4, x_1, x_2, x_3); -return x_5; +lean_object* x_18; +x_18 = l_Lean_Elab_Command_expandInitialize___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_18; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("builtin_initialize", 18); -return x_1; +lean_object* x_16; +x_16 = l_Lean_Elab_Command_expandInitialize___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_2); +lean_dec(x_1); +return x_16; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandInitialize___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Elab_Declaration_0__Lean_Elab_Command_expandDeclNamespace_x3f___closed__6; -x_2 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_15; +x_15 = l_Lean_Elab_Command_expandInitialize___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_2); +lean_dec(x_1); +return x_15; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("expandBuiltinInitialize", 23); +x_1 = lean_mk_string_from_bytes("expandInitialize", 16); return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__4() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___regBuiltin_Lean_Elab_Command_elabDeclaration___closed__2; -x_2 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__3; +x_2 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__5() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_expandBuiltinInitialize), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_expandInitialize), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_2 = l___regBuiltin_Lean_Elab_Command_expandMutualNamespace___closed__5; -x_3 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__2; -x_4 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__4; -x_5 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__5; +x_3 = l_Lean_Elab_Command_expandInitialize___closed__1; +x_4 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2; +x_5 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__3; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(353u); -x_2 = lean_unsigned_to_nat(57u); +x_1 = lean_unsigned_to_nat(329u); +x_2 = lean_unsigned_to_nat(49u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(354u); -x_2 = lean_unsigned_to_nat(33u); +x_1 = lean_unsigned_to_nat(341u); +x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__1; -x_2 = lean_unsigned_to_nat(57u); -x_3 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__2; -x_4 = lean_unsigned_to_nat(33u); +x_1 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__1; +x_2 = lean_unsigned_to_nat(49u); +x_3 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__2; +x_4 = lean_unsigned_to_nat(31u); x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -14568,38 +14524,38 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__4() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(353u); -x_2 = lean_unsigned_to_nat(61u); +x_1 = lean_unsigned_to_nat(329u); +x_2 = lean_unsigned_to_nat(53u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__5() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(353u); -x_2 = lean_unsigned_to_nat(84u); +x_1 = lean_unsigned_to_nat(329u); +x_2 = lean_unsigned_to_nat(69u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__6() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__4; -x_2 = lean_unsigned_to_nat(61u); -x_3 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__5; -x_4 = lean_unsigned_to_nat(84u); +x_1 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__4; +x_2 = lean_unsigned_to_nat(53u); +x_3 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__5; +x_4 = lean_unsigned_to_nat(69u); x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -14608,29 +14564,29 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__7() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__3; -x_2 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__6; +x_1 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__3; +x_2 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__6; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__4; -x_3 = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__7; +x_2 = l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2; +x_3 = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange___closed__7; x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7049_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7254_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -15051,8 +15007,6 @@ l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4 = lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__4); l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__5); -l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabAttr___spec__1___closed__6); l_Lean_Elab_Command_elabAttr___closed__1 = _init_l_Lean_Elab_Command_elabAttr___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabAttr___closed__1); l___regBuiltin_Lean_Elab_Command_elabAttr___closed__1 = _init_l___regBuiltin_Lean_Elab_Command_elabAttr___closed__1(); @@ -15085,162 +15039,132 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_elabAttr_declRange___close res = l___regBuiltin_Lean_Elab_Command_elabAttr_declRange(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__1 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__1); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__2); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__3 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__3); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__4); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__5 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__5); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__6); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__7); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__8 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__8); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__9); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__10 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__10); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__11 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__11); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__12 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__12); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__13 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__13); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__14 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__14(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__14); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__15 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__15(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__15); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__16 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__16(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__16); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__17); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__18 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__18(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__18); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__19 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__19(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__19); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__20); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__21 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__21(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__21); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__22); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__23 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__23(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__23); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__24 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__24(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__24); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__25); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__26); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__27 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__27(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__27); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__28); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__29 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__29(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__29); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__30); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__31); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__32 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__32(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__32); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__33); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__34 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__34(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__34); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__35 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__35(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__35); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__36); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__37); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__38 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__38(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__38); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__39); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__40 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__40(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__40); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__41 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__41(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__41); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__42 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__42(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__42); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__43 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__43(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__43); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__44 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__44(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__44); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__45 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__45(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__45); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__46); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__47 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__47(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__47); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__48); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__49); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__50); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__51); -l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52 = _init_l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___lambda__1___closed__52); -l_Lean_Elab_Command_expandInitCmd___closed__1 = _init_l_Lean_Elab_Command_expandInitCmd___closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__1); -l_Lean_Elab_Command_expandInitCmd___closed__2 = _init_l_Lean_Elab_Command_expandInitCmd___closed__2(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__2); -l_Lean_Elab_Command_expandInitCmd___closed__3 = _init_l_Lean_Elab_Command_expandInitCmd___closed__3(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__3); -l_Lean_Elab_Command_expandInitCmd___closed__4 = _init_l_Lean_Elab_Command_expandInitCmd___closed__4(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__4); -l_Lean_Elab_Command_expandInitCmd___closed__5 = _init_l_Lean_Elab_Command_expandInitCmd___closed__5(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__5); -l_Lean_Elab_Command_expandInitCmd___closed__6 = _init_l_Lean_Elab_Command_expandInitCmd___closed__6(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__6); -l_Lean_Elab_Command_expandInitCmd___closed__7 = _init_l_Lean_Elab_Command_expandInitCmd___closed__7(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__7); -l_Lean_Elab_Command_expandInitCmd___closed__8 = _init_l_Lean_Elab_Command_expandInitCmd___closed__8(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__8); -l_Lean_Elab_Command_expandInitCmd___closed__9 = _init_l_Lean_Elab_Command_expandInitCmd___closed__9(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__9); -l_Lean_Elab_Command_expandInitCmd___closed__10 = _init_l_Lean_Elab_Command_expandInitCmd___closed__10(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__10); -l_Lean_Elab_Command_expandInitCmd___closed__11 = _init_l_Lean_Elab_Command_expandInitCmd___closed__11(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__11); -l_Lean_Elab_Command_expandInitCmd___closed__12 = _init_l_Lean_Elab_Command_expandInitCmd___closed__12(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__12); -l_Lean_Elab_Command_expandInitCmd___closed__13 = _init_l_Lean_Elab_Command_expandInitCmd___closed__13(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__13); -l_Lean_Elab_Command_expandInitCmd___closed__14 = _init_l_Lean_Elab_Command_expandInitCmd___closed__14(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__14); -l_Lean_Elab_Command_expandInitCmd___closed__15 = _init_l_Lean_Elab_Command_expandInitCmd___closed__15(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__15); -l_Lean_Elab_Command_expandInitCmd___closed__16 = _init_l_Lean_Elab_Command_expandInitCmd___closed__16(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__16); -l_Lean_Elab_Command_expandInitCmd___closed__17 = _init_l_Lean_Elab_Command_expandInitCmd___closed__17(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__17); -l_Lean_Elab_Command_expandInitCmd___closed__18 = _init_l_Lean_Elab_Command_expandInitCmd___closed__18(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__18); -l_Lean_Elab_Command_expandInitCmd___closed__19 = _init_l_Lean_Elab_Command_expandInitCmd___closed__19(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__19); -l_Lean_Elab_Command_expandInitCmd___closed__20 = _init_l_Lean_Elab_Command_expandInitCmd___closed__20(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__20); -l_Lean_Elab_Command_expandInitCmd___closed__21 = _init_l_Lean_Elab_Command_expandInitCmd___closed__21(); -lean_mark_persistent(l_Lean_Elab_Command_expandInitCmd___closed__21); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__1); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__2 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__2); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__3); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__4 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__4); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__5 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__5); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__6 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__6); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__7); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__8 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__8); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__9 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__9); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__10); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__11); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__12); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__13); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__14); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__15); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__16 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__16(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__16); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__17 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__17(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__17); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__18); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__19); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__20 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__20(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__20); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__21); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__22); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__23); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__24); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__25); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__26); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__27); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__28); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__29); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__30); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__31); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__32); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__33); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__34 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__34(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__34); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__35); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__36 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__36(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__36); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__37 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__37(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__37); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__38 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__38(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__38); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__39 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__39(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__39); +l_Lean_Elab_Command_expandInitialize___lambda__1___closed__40 = _init_l_Lean_Elab_Command_expandInitialize___lambda__1___closed__40(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__1___closed__40); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__1 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__1); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__2 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__2); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__3 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__3); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__4); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__5); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__6 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__6); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__7); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__8 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__8(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__8); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__9 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__9(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__9); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__10 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__10(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__10); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__11 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__11(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__11); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__12 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__12(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__12); +l_Lean_Elab_Command_expandInitialize___lambda__4___closed__13 = _init_l_Lean_Elab_Command_expandInitialize___lambda__4___closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___lambda__4___closed__13); +l_Lean_Elab_Command_expandInitialize___closed__1 = _init_l_Lean_Elab_Command_expandInitialize___closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___closed__1); +l_Lean_Elab_Command_expandInitialize___closed__2 = _init_l_Lean_Elab_Command_expandInitialize___closed__2(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___closed__2); +l_Lean_Elab_Command_expandInitialize___closed__3 = _init_l_Lean_Elab_Command_expandInitialize___closed__3(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___closed__3); +l_Lean_Elab_Command_expandInitialize___closed__4 = _init_l_Lean_Elab_Command_expandInitialize___closed__4(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___closed__4); +l_Lean_Elab_Command_expandInitialize___closed__5 = _init_l_Lean_Elab_Command_expandInitialize___closed__5(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___closed__5); +l_Lean_Elab_Command_expandInitialize___closed__6 = _init_l_Lean_Elab_Command_expandInitialize___closed__6(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___closed__6); +l_Lean_Elab_Command_expandInitialize___closed__7 = _init_l_Lean_Elab_Command_expandInitialize___closed__7(); +lean_mark_persistent(l_Lean_Elab_Command_expandInitialize___closed__7); l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__1 = _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__1); l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2 = _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__2); l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__3 = _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__3(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__3); -l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__4 = _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__4); -l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__5 = _init_l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandInitialize___closed__5); res = l___regBuiltin_Lean_Elab_Command_expandInitialize(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); @@ -15261,37 +15185,7 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange res = l___regBuiltin_Lean_Elab_Command_expandInitialize_declRange(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__1 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__1); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__2 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__2); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__3 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__3); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__4 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__4); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__5 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize___closed__5); -res = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__1 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__1); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__2 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__2); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__3 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__3); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__4 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__4); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__5 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__5); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__6 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__6); -l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__7 = _init_l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange___closed__7); -res = l___regBuiltin_Lean_Elab_Command_expandBuiltinInitialize_declRange(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7049_(lean_io_mk_world()); +res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Declaration___hyg_7254_(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/DefView.c b/stage0/stdlib/Lean/Elab/DefView.c index 6df74f2a9ae5..255a0f411759 100644 --- a/stage0/stdlib/Lean/Elab/DefView.c +++ b/stage0/stdlib/Lean/Elab/DefView.c @@ -157,6 +157,7 @@ lean_object* lean_environment_main_module(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_mkDefViewOfInstance___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); +lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_mkDefViewOfOpaque___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_mkInstanceName___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_DefKind_noConfusion___rarg___lambda__1(lean_object*); @@ -202,7 +203,6 @@ lean_object* l_Lean_Elab_Term_elabBinders___rarg(lean_object*, lean_object*, lea static lean_object* l_Lean_Elab_Command_isDefLike___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_mkDefViewOfInstance___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_instBEqDefKind; -lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; static lean_object* l_Lean_Elab_Command_mkDefViewOfOpaque___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_mkInstanceName___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1419,7 +1419,7 @@ x_53 = lean_ctor_get(x_44, 1); lean_inc(x_53); lean_dec(x_44); x_54 = l_List_reverse___rarg(x_53); -x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_54, x_2, x_3, x_52); +x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_54, x_2, x_3, x_52); lean_dec(x_3); lean_dec(x_2); x_56 = !lean_is_exclusive(x_55); @@ -1481,7 +1481,7 @@ x_71 = lean_ctor_get(x_44, 1); lean_inc(x_71); lean_dec(x_44); x_72 = l_List_reverse___rarg(x_71); -x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_2, x_3, x_70); +x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_72, x_2, x_3, x_70); lean_dec(x_3); lean_dec(x_2); x_74 = lean_ctor_get(x_73, 1); @@ -2678,7 +2678,7 @@ x_53 = lean_ctor_get(x_44, 1); lean_inc(x_53); lean_dec(x_44); x_54 = l_List_reverse___rarg(x_53); -x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_54, x_2, x_3, x_52); +x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_54, x_2, x_3, x_52); lean_dec(x_3); lean_dec(x_2); x_56 = !lean_is_exclusive(x_55); @@ -2740,7 +2740,7 @@ x_71 = lean_ctor_get(x_44, 1); lean_inc(x_71); lean_dec(x_44); x_72 = l_List_reverse___rarg(x_71); -x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_2, x_3, x_70); +x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_72, x_2, x_3, x_70); lean_dec(x_3); lean_dec(x_2); x_74 = lean_ctor_get(x_73, 1); @@ -3088,7 +3088,7 @@ x_53 = lean_ctor_get(x_44, 1); lean_inc(x_53); lean_dec(x_44); x_54 = l_List_reverse___rarg(x_53); -x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_54, x_2, x_3, x_52); +x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_54, x_2, x_3, x_52); lean_dec(x_3); lean_dec(x_2); x_56 = !lean_is_exclusive(x_55); @@ -3150,7 +3150,7 @@ x_71 = lean_ctor_get(x_44, 1); lean_inc(x_71); lean_dec(x_44); x_72 = l_List_reverse___rarg(x_71); -x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_2, x_3, x_70); +x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_72, x_2, x_3, x_70); lean_dec(x_3); lean_dec(x_2); x_74 = lean_ctor_get(x_73, 1); diff --git a/stage0/stdlib/Lean/Elab/Deriving/BEq.c b/stage0/stdlib/Lean/Elab/Deriving/BEq.c index 6b1007f04928..e484c4622edd 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/BEq.c +++ b/stage0/stdlib/Lean/Elab/Deriving/BEq.c @@ -54,6 +54,7 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMa static lean_object* l_Lean_Elab_Deriving_BEq_mkMatch_mkElseAlt___closed__1; lean_object* lean_environment_find(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); +lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_BEq_mkMatch_mkElseAlt___closed__13; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_BEq_mkMutualBlock___closed__7; @@ -160,7 +161,6 @@ lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Deriving_BEq_0__Lean_Elab_Deriving_BEq_mkBEqEnumFun___closed__16; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__14; static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__13; -lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Deriving_BEq_mkBEqInstanceHandler___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__5___lambda__1___closed__15; static lean_object* l_Lean_Elab_Deriving_BEq_mkAuxFunction___lambda__1___closed__21; @@ -1306,7 +1306,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkM lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__4___closed__15; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__4___closed__16; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_BEq_mkMatch_mkAlts___spec__4___closed__17; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -6898,7 +6898,7 @@ x_111 = 0; x_112 = lean_usize_of_nat(x_104); lean_dec(x_104); x_113 = lean_box(0); -x_114 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_102, x_111, x_112, x_113, x_2, x_3, x_103); +x_114 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_102, x_111, x_112, x_113, x_2, x_3, x_103); lean_dec(x_102); if (lean_obj_tag(x_114) == 0) { @@ -7002,7 +7002,7 @@ x_138 = 0; x_139 = lean_usize_of_nat(x_129); lean_dec(x_129); x_140 = lean_box(0); -x_141 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_127, x_138, x_139, x_140, x_2, x_3, x_128); +x_141 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_127, x_138, x_139, x_140, x_2, x_3, x_128); lean_dec(x_127); if (lean_obj_tag(x_141) == 0) { @@ -7237,7 +7237,7 @@ x_35 = 0; x_36 = lean_usize_of_nat(x_28); lean_dec(x_28); x_37 = lean_box(0); -x_38 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_26, x_35, x_36, x_37, x_2, x_3, x_27); +x_38 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_26, x_35, x_36, x_37, x_2, x_3, x_27); lean_dec(x_26); if (lean_obj_tag(x_38) == 0) { @@ -7341,7 +7341,7 @@ x_62 = 0; x_63 = lean_usize_of_nat(x_53); lean_dec(x_53); x_64 = lean_box(0); -x_65 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_51, x_62, x_63, x_64, x_2, x_3, x_52); +x_65 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_51, x_62, x_63, x_64, x_2, x_3, x_52); lean_dec(x_51); if (lean_obj_tag(x_65) == 0) { diff --git a/stage0/stdlib/Lean/Elab/Deriving/Basic.c b/stage0/stdlib/Lean/Elab/Deriving/Basic.c index d87a51b177b9..eb0960996d0c 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/Basic.c +++ b/stage0/stdlib/Lean/Elab/Deriving/Basic.c @@ -2216,7 +2216,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_elabDeriving__ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabDeriving___spec__19___closed__1; x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabDeriving___spec__19___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Array_forInUnsafe_loop___at_Lean_Elab_elabDeriving___spec__19___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/Deriving/DecEq.c b/stage0/stdlib/Lean/Elab/Deriving/DecEq.c index 8b19ece39d7b..468520a7c991 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/DecEq.c +++ b/stage0/stdlib/Lean/Elab/Deriving/DecEq.c @@ -85,6 +85,7 @@ lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch___closed__2; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__16; +lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__47; uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__15; @@ -115,7 +116,6 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat_mkDecTree___closed__5 static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqHeader___closed__2; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__3___closed__11; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqHeader___closed__1; -lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkEnumOfNat___lambda__1___closed__3; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__33; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1___closed__12; @@ -125,6 +125,7 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1 lean_object* lean_string_utf8_byte_size(lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__5; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__30; +lean_object* l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__18; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkEnumOfNatThm___spec__1___boxed(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); @@ -158,7 +159,6 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2 static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1___closed__19; static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__1___closed__1; static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__43; -lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__32; LEAN_EXPORT lean_object* l_Lean_isEnumType___at_Lean_Elab_Deriving_DecEq_mkDecEqInstanceHandler___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__3___closed__9; @@ -272,7 +272,6 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2 LEAN_EXPORT lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1___closed__21; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__51; -lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__46; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum(lean_object*, lean_object*, lean_object*, lean_object*); @@ -310,6 +309,7 @@ static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__3 static lean_object* l_Lean_Elab_Deriving_DecEq_mkAuxFunction___closed__22; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__1___closed__25; +lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_DecEq_mkDecEqEnum___closed__61; static lean_object* l_Lean_Elab_Deriving_DecEq_mkMatch_mkSameCtorRhs___lambda__2___closed__32; @@ -2978,7 +2978,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_DecEq_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_Std_Range_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__5___closed__5; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__5___closed__6; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_DecEq_mkMatch_mkAlts___spec__5___closed__7; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -6679,7 +6679,7 @@ x_23 = 0; x_24 = lean_usize_of_nat(x_15); lean_dec(x_15); x_25 = lean_box(0); -x_26 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_13, x_23, x_24, x_25, x_2, x_3, x_14); +x_26 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_13, x_23, x_24, x_25, x_2, x_3, x_14); lean_dec(x_13); if (lean_obj_tag(x_26) == 0) { @@ -6784,7 +6784,7 @@ x_51 = 0; x_52 = lean_usize_of_nat(x_41); lean_dec(x_41); x_53 = lean_box(0); -x_54 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_39, x_51, x_52, x_53, x_2, x_3, x_40); +x_54 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_39, x_51, x_52, x_53, x_2, x_3, x_40); lean_dec(x_39); if (lean_obj_tag(x_54) == 0) { @@ -9236,7 +9236,7 @@ lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; x_364 = lean_ctor_get(x_358, 1); lean_inc(x_364); lean_dec(x_358); -x_365 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__3(x_345, x_2, x_3, x_364); +x_365 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Command_elabCommand___spec__7(x_345, x_2, x_3, x_364); x_366 = lean_ctor_get(x_365, 0); lean_inc(x_366); x_367 = lean_ctor_get(x_365, 1); @@ -9270,7 +9270,7 @@ x_352 = l_Lean_Elab_Deriving_DecEq_mkDecEqCmds___closed__10; x_353 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_353, 0, x_351); lean_ctor_set(x_353, 1, x_352); -x_354 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__4(x_345, x_353, x_2, x_3, x_347); +x_354 = l_Lean_addTrace___at_Lean_Elab_Command_elabCommand___spec__8(x_345, x_353, x_2, x_3, x_347); x_355 = lean_ctor_get(x_354, 1); lean_inc(x_355); lean_dec(x_354); diff --git a/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c b/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c index 34c8334b42b9..da4b96d6a296 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c +++ b/stage0/stdlib/Lean/Elab/Deriving/FromToJson.c @@ -36,7 +36,6 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mk lean_object* l_Lean_LocalDecl_userName(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13; uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__6; @@ -44,6 +43,7 @@ lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__2___closed__15; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__10; +static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__32; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__13; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -59,6 +59,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___la static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__6___closed__1; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__39; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__5(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__2___closed__10; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__35; @@ -66,6 +67,7 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___la lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__4___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__6___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -117,7 +119,6 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___la static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__1; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__10; lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__9___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__3; @@ -186,7 +187,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJs lean_object* l_Lean_Name_toString(lean_object*, uint8_t); lean_object* l_Lean_Elab_Deriving_mkLet(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__20; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); @@ -216,7 +216,7 @@ static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFro static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__5; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__4; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__16; -LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527_(lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__8; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__7; lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -246,12 +246,10 @@ lean_object* l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1 lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__29; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__1; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__6; lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__1___closed__3; -static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__2; LEAN_EXPORT lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; lean_object* l_panic___at_Lean_Elab_Deriving_mkLocalInstanceLetDecls___spec__1(lean_object*); @@ -273,7 +271,6 @@ static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mk static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___spec__6___closed__1; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__6; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__4; -lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__2___closed__12; static lean_object* l_Lean_getConstInfoCtor___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__1___closed__2; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__9; @@ -296,6 +293,7 @@ static lean_object* l_Array_qsort_sort___at_Lean_Elab_Deriving_FromToJson_mkFrom static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__15; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__15; uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); +static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35; lean_object* l_Lean_Name_getString_x21(lean_object*); lean_object* l_String_intercalate(lean_object*, lean_object*); static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___closed__4; @@ -304,8 +302,8 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mk lean_object* l_List_redLength___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__2___closed__8; -static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__11; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__22; static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__21; lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -335,6 +333,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJs LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___spec__3(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__39; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__12; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__3; @@ -343,7 +342,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandl static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__17; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__27; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__4; -static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__8; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__6(size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; @@ -357,6 +355,7 @@ static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFro static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___closed__5; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; +static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__33; lean_object* l_List_toArrayAux___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___boxed(lean_object**); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__1; @@ -393,11 +392,11 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___la static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__12; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__11; lean_object* lean_mk_syntax_ident(lean_object*); -static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__16; static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__10; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__2; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__4; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkJsonField___closed__1; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__8; @@ -428,12 +427,15 @@ static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___la static lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__9; static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__17; LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__5___boxed(lean_object**); +static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__38; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__25; +static lean_object* l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__34; lean_object* l_String_dropRightWhile(lean_object*, lean_object*); lean_object* l_Lean_Elab_Deriving_mkInductiveApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__11; uint8_t l_Lean_isStructure(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__1; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__9(size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__4; @@ -951,7 +953,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -6014,7 +6016,7 @@ static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandle _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declValSimple", 13); +x_1 = lean_mk_string_from_bytes("typeSpec", 8); return x_1; } } @@ -6022,7 +6024,7 @@ static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandle _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__11; +x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__6; x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__26; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -6032,7 +6034,7 @@ static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandle _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes(":=", 2); +x_1 = lean_mk_string_from_bytes(":", 1); return x_1; } } @@ -6040,12 +6042,95 @@ static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandle _start: { lean_object* x_1; lean_object* x_2; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__9; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__9; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__2; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__9; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__32() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__33() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__32; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__34() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("declValSimple", 13); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__11; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__34; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(":=", 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37() { +_start: +{ +lean_object* x_1; lean_object* x_2; x_1 = lean_unsigned_to_nat(7u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__38() { _start: { lean_object* x_1; @@ -6053,12 +6138,12 @@ x_1 = lean_mk_string_from_bytes("partial", 7); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__39() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__11; -x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__38; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -6096,43 +6181,43 @@ x_21 = lean_nat_dec_lt(x_17, x_20); lean_dec(x_20); if (x_18 == 0) { -lean_object* x_218; lean_object* x_219; +lean_object* x_252; lean_object* x_253; lean_dec(x_15); -x_218 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__4; -x_219 = l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(x_218); -x_22 = x_219; -goto block_217; +x_252 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__4; +x_253 = l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(x_252); +x_22 = x_253; +goto block_251; } else { -lean_object* x_220; -x_220 = lean_array_fget(x_15, x_17); +lean_object* x_254; +x_254 = lean_array_fget(x_15, x_17); lean_dec(x_15); -x_22 = x_220; -goto block_217; +x_22 = x_254; +goto block_251; } -block_217: +block_251: { lean_object* x_23; lean_object* x_24; x_23 = lean_mk_syntax_ident(x_22); if (x_21 == 0) { -lean_object* x_214; lean_object* x_215; +lean_object* x_248; lean_object* x_249; lean_dec(x_19); -x_214 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__4; -x_215 = l_panic___at_Lean_Elab_Deriving_mkLocalInstanceLetDecls___spec__1(x_214); -x_24 = x_215; -goto block_213; +x_248 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__4; +x_249 = l_panic___at_Lean_Elab_Deriving_mkLocalInstanceLetDecls___spec__1(x_248); +x_24 = x_249; +goto block_247; } else { -lean_object* x_216; -x_216 = lean_array_fget(x_19, x_17); +lean_object* x_250; +x_250 = lean_array_fget(x_19, x_17); lean_dec(x_19); -x_24 = x_216; -goto block_213; +x_24 = x_250; +goto block_247; } -block_213: +block_247: { lean_object* x_25; lean_object* x_26; lean_object* x_27; x_25 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__2; @@ -6248,7 +6333,7 @@ lean_ctor_set(x_73, 2, x_71); x_74 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); if (x_74 == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_inc(x_8); x_75 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_42); x_76 = lean_ctor_get(x_75, 0); @@ -6256,255 +6341,325 @@ lean_inc(x_76); x_77 = lean_ctor_get(x_75, 1); lean_inc(x_77); lean_dec(x_75); -x_78 = lean_st_ref_get(x_9, x_77); -x_79 = lean_ctor_get(x_78, 1); -lean_inc(x_79); -lean_dec(x_78); -x_80 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__16; +x_78 = lean_ctor_get(x_8, 10); +lean_inc(x_78); +x_79 = lean_st_ref_get(x_9, x_77); +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +lean_dec(x_79); +x_82 = lean_ctor_get(x_80, 0); +lean_inc(x_82); +lean_dec(x_80); +x_83 = lean_environment_main_module(x_82); +x_84 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__16; lean_inc(x_76); -x_81 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_81, 0, x_76); -lean_ctor_set(x_81, 1, x_80); -x_82 = lean_array_push(x_60, x_81); -x_83 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__17; -x_84 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_84, 0, x_53); -lean_ctor_set(x_84, 1, x_83); -lean_ctor_set(x_84, 2, x_82); -x_85 = lean_array_push(x_60, x_84); -x_86 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_86, 0, x_53); -lean_ctor_set(x_86, 1, x_54); -lean_ctor_set(x_86, 2, x_85); -x_87 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__19; -x_88 = lean_array_push(x_87, x_86); -x_89 = lean_array_push(x_88, x_66); -x_90 = lean_array_push(x_89, x_66); -x_91 = lean_array_push(x_90, x_66); -x_92 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__15; -x_93 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_93, 0, x_53); -lean_ctor_set(x_93, 1, x_92); -lean_ctor_set(x_93, 2, x_91); -x_94 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__20; +x_85 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_85, 0, x_76); +lean_ctor_set(x_85, 1, x_84); +x_86 = lean_array_push(x_60, x_85); +x_87 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__17; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_53); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = lean_array_push(x_60, x_88); +x_90 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_90, 0, x_53); +lean_ctor_set(x_90, 1, x_54); +lean_ctor_set(x_90, 2, x_89); +x_91 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__19; +x_92 = lean_array_push(x_91, x_90); +x_93 = lean_array_push(x_92, x_66); +x_94 = lean_array_push(x_93, x_66); +x_95 = lean_array_push(x_94, x_66); +x_96 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__15; +x_97 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_97, 0, x_53); +lean_ctor_set(x_97, 1, x_96); +lean_ctor_set(x_97, 2, x_95); +x_98 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__20; lean_inc(x_76); -x_95 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_95, 0, x_76); -lean_ctor_set(x_95, 1, x_94); -x_96 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__7; -x_97 = lean_array_push(x_96, x_23); -x_98 = lean_array_push(x_97, x_66); -x_99 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; -x_100 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_100, 0, x_53); -lean_ctor_set(x_100, 1, x_99); -lean_ctor_set(x_100, 2, x_98); -x_101 = lean_ctor_get(x_28, 0); -lean_inc(x_101); +x_99 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_99, 0, x_76); +lean_ctor_set(x_99, 1, x_98); +x_100 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__7; +x_101 = lean_array_push(x_100, x_23); +x_102 = lean_array_push(x_101, x_66); +x_103 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_53); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = lean_ctor_get(x_28, 0); +lean_inc(x_105); lean_dec(x_28); -x_102 = l_Array_append___rarg(x_51, x_101); -x_103 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_103, 0, x_53); -lean_ctor_set(x_103, 1, x_54); -lean_ctor_set(x_103, 2, x_102); -x_104 = lean_array_push(x_96, x_103); -x_105 = lean_array_push(x_104, x_66); -x_106 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__25; +x_106 = l_Array_append___rarg(x_51, x_105); x_107 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_107, 0, x_53); -lean_ctor_set(x_107, 1, x_106); -lean_ctor_set(x_107, 2, x_105); +lean_ctor_set(x_107, 1, x_54); +lean_ctor_set(x_107, 2, x_106); x_108 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; +lean_inc(x_76); x_109 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_109, 0, x_76); lean_ctor_set(x_109, 1, x_108); -x_110 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___closed__5; -x_111 = lean_array_push(x_110, x_109); -x_112 = lean_array_push(x_111, x_73); -x_113 = lean_array_push(x_112, x_66); -x_114 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__27; -x_115 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_115, 0, x_53); -lean_ctor_set(x_115, 1, x_114); -lean_ctor_set(x_115, 2, x_113); -x_116 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; -x_117 = lean_array_push(x_116, x_95); -x_118 = lean_array_push(x_117, x_100); -x_119 = lean_array_push(x_118, x_107); -x_120 = lean_array_push(x_119, x_115); -x_121 = lean_array_push(x_120, x_66); -x_122 = lean_array_push(x_121, x_66); -x_123 = lean_array_push(x_122, x_66); -x_124 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__21; -x_125 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_125, 0, x_53); -lean_ctor_set(x_125, 1, x_124); -lean_ctor_set(x_125, 2, x_123); -x_126 = lean_array_push(x_96, x_93); -x_127 = lean_array_push(x_126, x_125); -x_128 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; -x_129 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_129, 0, x_53); -lean_ctor_set(x_129, 1, x_128); -lean_ctor_set(x_129, 2, x_127); -x_130 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__2(x_13, x_25, x_3, x_60, x_129, x_4, x_5, x_6, x_7, x_8, x_9, x_79); +x_110 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__8; +x_111 = l_Lean_addMacroScope(x_83, x_110, x_78); +x_112 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; +x_113 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__33; +lean_inc(x_76); +x_114 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_114, 0, x_76); +lean_ctor_set(x_114, 1, x_112); +lean_ctor_set(x_114, 2, x_111); +lean_ctor_set(x_114, 3, x_113); +x_115 = lean_array_push(x_100, x_109); +x_116 = lean_array_push(x_115, x_114); +x_117 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__27; +x_118 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_118, 0, x_53); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set(x_118, 2, x_116); +x_119 = lean_array_push(x_60, x_118); +x_120 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_120, 0, x_53); +lean_ctor_set(x_120, 1, x_54); +lean_ctor_set(x_120, 2, x_119); +x_121 = lean_array_push(x_100, x_107); +x_122 = lean_array_push(x_121, x_120); +x_123 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__25; +x_124 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_124, 0, x_53); +lean_ctor_set(x_124, 1, x_123); +lean_ctor_set(x_124, 2, x_122); +x_125 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36; +x_126 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_126, 0, x_76); +lean_ctor_set(x_126, 1, x_125); +x_127 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___closed__5; +x_128 = lean_array_push(x_127, x_126); +x_129 = lean_array_push(x_128, x_73); +x_130 = lean_array_push(x_129, x_66); +x_131 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35; +x_132 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_132, 0, x_53); +lean_ctor_set(x_132, 1, x_131); +lean_ctor_set(x_132, 2, x_130); +x_133 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; +x_134 = lean_array_push(x_133, x_99); +x_135 = lean_array_push(x_134, x_104); +x_136 = lean_array_push(x_135, x_124); +x_137 = lean_array_push(x_136, x_132); +x_138 = lean_array_push(x_137, x_66); +x_139 = lean_array_push(x_138, x_66); +x_140 = lean_array_push(x_139, x_66); +x_141 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__21; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_53); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = lean_array_push(x_100, x_97); +x_144 = lean_array_push(x_143, x_142); +x_145 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; +x_146 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_146, 0, x_53); +lean_ctor_set(x_146, 1, x_145); +lean_ctor_set(x_146, 2, x_144); +x_147 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__2(x_13, x_25, x_3, x_60, x_146, x_4, x_5, x_6, x_7, x_8, x_9, x_81); lean_dec(x_13); -return x_130; +return x_147; } else { -lean_object* x_131; lean_object* x_132; -x_131 = lean_ctor_get(x_28, 1); -lean_inc(x_131); +lean_object* x_148; lean_object* x_149; +x_148 = lean_ctor_get(x_28, 1); +lean_inc(x_148); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_132 = l_Lean_Elab_Deriving_mkLocalInstanceLetDecls(x_13, x_25, x_131, x_4, x_5, x_6, x_7, x_8, x_9, x_42); -if (lean_obj_tag(x_132) == 0) +x_149 = l_Lean_Elab_Deriving_mkLocalInstanceLetDecls(x_13, x_25, x_148, x_4, x_5, x_6, x_7, x_8, x_9, x_42); +if (lean_obj_tag(x_149) == 0) { -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; -x_133 = lean_ctor_get(x_132, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_132, 1); -lean_inc(x_134); -lean_dec(x_132); +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; +x_150 = lean_ctor_get(x_149, 0); +lean_inc(x_150); +x_151 = lean_ctor_get(x_149, 1); +lean_inc(x_151); +lean_dec(x_149); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_135 = l_Lean_Elab_Deriving_mkLet(x_133, x_73, x_4, x_5, x_6, x_7, x_8, x_9, x_134); -lean_dec(x_133); -x_136 = lean_ctor_get(x_135, 0); -lean_inc(x_136); -x_137 = lean_ctor_get(x_135, 1); -lean_inc(x_137); -lean_dec(x_135); +x_152 = l_Lean_Elab_Deriving_mkLet(x_150, x_73, x_4, x_5, x_6, x_7, x_8, x_9, x_151); +lean_dec(x_150); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +x_154 = lean_ctor_get(x_152, 1); +lean_inc(x_154); +lean_dec(x_152); lean_inc(x_8); -x_138 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_137); -x_139 = lean_ctor_get(x_138, 0); -lean_inc(x_139); -x_140 = lean_ctor_get(x_138, 1); -lean_inc(x_140); -lean_dec(x_138); -x_141 = lean_st_ref_get(x_9, x_140); -x_142 = lean_ctor_get(x_141, 1); -lean_inc(x_142); -lean_dec(x_141); -x_143 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__16; -lean_inc(x_139); -x_144 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_144, 0, x_139); -lean_ctor_set(x_144, 1, x_143); -x_145 = lean_array_push(x_60, x_144); -x_146 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__17; -x_147 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_147, 0, x_53); -lean_ctor_set(x_147, 1, x_146); -lean_ctor_set(x_147, 2, x_145); -x_148 = lean_array_push(x_60, x_147); -x_149 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_149, 0, x_53); -lean_ctor_set(x_149, 1, x_54); -lean_ctor_set(x_149, 2, x_148); -x_150 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; -lean_inc(x_139); -x_151 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_151, 0, x_139); -lean_ctor_set(x_151, 1, x_150); -x_152 = lean_array_push(x_60, x_151); -x_153 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31; -x_154 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_154, 0, x_53); -lean_ctor_set(x_154, 1, x_153); -lean_ctor_set(x_154, 2, x_152); -x_155 = lean_array_push(x_60, x_154); -x_156 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_156, 0, x_53); -lean_ctor_set(x_156, 1, x_54); -lean_ctor_set(x_156, 2, x_155); -x_157 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__19; -x_158 = lean_array_push(x_157, x_149); -x_159 = lean_array_push(x_158, x_66); -x_160 = lean_array_push(x_159, x_66); -x_161 = lean_array_push(x_160, x_156); -x_162 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__15; -x_163 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_163, 0, x_53); -lean_ctor_set(x_163, 1, x_162); -lean_ctor_set(x_163, 2, x_161); -x_164 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__20; -lean_inc(x_139); +x_155 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_154); +x_156 = lean_ctor_get(x_155, 0); +lean_inc(x_156); +x_157 = lean_ctor_get(x_155, 1); +lean_inc(x_157); +lean_dec(x_155); +x_158 = lean_ctor_get(x_8, 10); +lean_inc(x_158); +x_159 = lean_st_ref_get(x_9, x_157); +x_160 = lean_ctor_get(x_159, 0); +lean_inc(x_160); +x_161 = lean_ctor_get(x_159, 1); +lean_inc(x_161); +lean_dec(x_159); +x_162 = lean_ctor_get(x_160, 0); +lean_inc(x_162); +lean_dec(x_160); +x_163 = lean_environment_main_module(x_162); +x_164 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__16; +lean_inc(x_156); x_165 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_165, 0, x_139); +lean_ctor_set(x_165, 0, x_156); lean_ctor_set(x_165, 1, x_164); -x_166 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__7; -x_167 = lean_array_push(x_166, x_23); -x_168 = lean_array_push(x_167, x_66); -x_169 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; +x_166 = lean_array_push(x_60, x_165); +x_167 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__17; +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_53); +lean_ctor_set(x_168, 1, x_167); +lean_ctor_set(x_168, 2, x_166); +x_169 = lean_array_push(x_60, x_168); x_170 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_170, 0, x_53); -lean_ctor_set(x_170, 1, x_169); -lean_ctor_set(x_170, 2, x_168); -x_171 = lean_ctor_get(x_28, 0); -lean_inc(x_171); -lean_dec(x_28); -x_172 = l_Array_append___rarg(x_51, x_171); -x_173 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_173, 0, x_53); -lean_ctor_set(x_173, 1, x_54); -lean_ctor_set(x_173, 2, x_172); -x_174 = lean_array_push(x_166, x_173); -x_175 = lean_array_push(x_174, x_66); -x_176 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__25; +lean_ctor_set(x_170, 1, x_54); +lean_ctor_set(x_170, 2, x_169); +x_171 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__38; +lean_inc(x_156); +x_172 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_172, 0, x_156); +lean_ctor_set(x_172, 1, x_171); +x_173 = lean_array_push(x_60, x_172); +x_174 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__39; +x_175 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_175, 0, x_53); +lean_ctor_set(x_175, 1, x_174); +lean_ctor_set(x_175, 2, x_173); +x_176 = lean_array_push(x_60, x_175); x_177 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_177, 0, x_53); -lean_ctor_set(x_177, 1, x_176); -lean_ctor_set(x_177, 2, x_175); -x_178 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; -x_179 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_179, 0, x_139); -lean_ctor_set(x_179, 1, x_178); -x_180 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___closed__5; -x_181 = lean_array_push(x_180, x_179); -x_182 = lean_array_push(x_181, x_136); -x_183 = lean_array_push(x_182, x_66); -x_184 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__27; -x_185 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_185, 0, x_53); -lean_ctor_set(x_185, 1, x_184); -lean_ctor_set(x_185, 2, x_183); -x_186 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; -x_187 = lean_array_push(x_186, x_165); -x_188 = lean_array_push(x_187, x_170); -x_189 = lean_array_push(x_188, x_177); -x_190 = lean_array_push(x_189, x_185); -x_191 = lean_array_push(x_190, x_66); -x_192 = lean_array_push(x_191, x_66); -x_193 = lean_array_push(x_192, x_66); -x_194 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__21; -x_195 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_195, 0, x_53); -lean_ctor_set(x_195, 1, x_194); -lean_ctor_set(x_195, 2, x_193); -x_196 = lean_array_push(x_166, x_163); -x_197 = lean_array_push(x_196, x_195); -x_198 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; -x_199 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_199, 0, x_53); -lean_ctor_set(x_199, 1, x_198); -lean_ctor_set(x_199, 2, x_197); -x_200 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__2(x_13, x_25, x_3, x_60, x_199, x_4, x_5, x_6, x_7, x_8, x_9, x_142); +lean_ctor_set(x_177, 1, x_54); +lean_ctor_set(x_177, 2, x_176); +x_178 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__19; +x_179 = lean_array_push(x_178, x_170); +x_180 = lean_array_push(x_179, x_66); +x_181 = lean_array_push(x_180, x_66); +x_182 = lean_array_push(x_181, x_177); +x_183 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__15; +x_184 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_184, 0, x_53); +lean_ctor_set(x_184, 1, x_183); +lean_ctor_set(x_184, 2, x_182); +x_185 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__20; +lean_inc(x_156); +x_186 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_186, 0, x_156); +lean_ctor_set(x_186, 1, x_185); +x_187 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__7; +x_188 = lean_array_push(x_187, x_23); +x_189 = lean_array_push(x_188, x_66); +x_190 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; +x_191 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_191, 0, x_53); +lean_ctor_set(x_191, 1, x_190); +lean_ctor_set(x_191, 2, x_189); +x_192 = lean_ctor_get(x_28, 0); +lean_inc(x_192); +lean_dec(x_28); +x_193 = l_Array_append___rarg(x_51, x_192); +x_194 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_194, 0, x_53); +lean_ctor_set(x_194, 1, x_54); +lean_ctor_set(x_194, 2, x_193); +x_195 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; +lean_inc(x_156); +x_196 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_196, 0, x_156); +lean_ctor_set(x_196, 1, x_195); +x_197 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__8; +x_198 = l_Lean_addMacroScope(x_163, x_197, x_158); +x_199 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; +x_200 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__33; +lean_inc(x_156); +x_201 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_201, 0, x_156); +lean_ctor_set(x_201, 1, x_199); +lean_ctor_set(x_201, 2, x_198); +lean_ctor_set(x_201, 3, x_200); +x_202 = lean_array_push(x_187, x_196); +x_203 = lean_array_push(x_202, x_201); +x_204 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__27; +x_205 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_205, 0, x_53); +lean_ctor_set(x_205, 1, x_204); +lean_ctor_set(x_205, 2, x_203); +x_206 = lean_array_push(x_60, x_205); +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_53); +lean_ctor_set(x_207, 1, x_54); +lean_ctor_set(x_207, 2, x_206); +x_208 = lean_array_push(x_187, x_194); +x_209 = lean_array_push(x_208, x_207); +x_210 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__25; +x_211 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_211, 0, x_53); +lean_ctor_set(x_211, 1, x_210); +lean_ctor_set(x_211, 2, x_209); +x_212 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36; +x_213 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_213, 0, x_156); +lean_ctor_set(x_213, 1, x_212); +x_214 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___closed__5; +x_215 = lean_array_push(x_214, x_213); +x_216 = lean_array_push(x_215, x_153); +x_217 = lean_array_push(x_216, x_66); +x_218 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35; +x_219 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_219, 0, x_53); +lean_ctor_set(x_219, 1, x_218); +lean_ctor_set(x_219, 2, x_217); +x_220 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; +x_221 = lean_array_push(x_220, x_186); +x_222 = lean_array_push(x_221, x_191); +x_223 = lean_array_push(x_222, x_211); +x_224 = lean_array_push(x_223, x_219); +x_225 = lean_array_push(x_224, x_66); +x_226 = lean_array_push(x_225, x_66); +x_227 = lean_array_push(x_226, x_66); +x_228 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__21; +x_229 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_229, 0, x_53); +lean_ctor_set(x_229, 1, x_228); +lean_ctor_set(x_229, 2, x_227); +x_230 = lean_array_push(x_187, x_184); +x_231 = lean_array_push(x_230, x_229); +x_232 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; +x_233 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_233, 0, x_53); +lean_ctor_set(x_233, 1, x_232); +lean_ctor_set(x_233, 2, x_231); +x_234 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__2(x_13, x_25, x_3, x_60, x_233, x_4, x_5, x_6, x_7, x_8, x_9, x_161); lean_dec(x_13); -return x_200; +return x_234; } else { -uint8_t x_201; +uint8_t x_235; lean_dec(x_73); lean_dec(x_28); lean_dec(x_23); @@ -6515,30 +6670,30 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_201 = !lean_is_exclusive(x_132); -if (x_201 == 0) +x_235 = !lean_is_exclusive(x_149); +if (x_235 == 0) { -return x_132; +return x_149; } else { -lean_object* x_202; lean_object* x_203; lean_object* x_204; -x_202 = lean_ctor_get(x_132, 0); -x_203 = lean_ctor_get(x_132, 1); -lean_inc(x_203); -lean_inc(x_202); -lean_dec(x_132); -x_204 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_204, 0, x_202); -lean_ctor_set(x_204, 1, x_203); -return x_204; +lean_object* x_236; lean_object* x_237; lean_object* x_238; +x_236 = lean_ctor_get(x_149, 0); +x_237 = lean_ctor_get(x_149, 1); +lean_inc(x_237); +lean_inc(x_236); +lean_dec(x_149); +x_238 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_238, 0, x_236); +lean_ctor_set(x_238, 1, x_237); +return x_238; } } } } else { -uint8_t x_205; +uint8_t x_239; lean_dec(x_31); lean_dec(x_28); lean_dec(x_23); @@ -6549,29 +6704,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_205 = !lean_is_exclusive(x_35); -if (x_205 == 0) +x_239 = !lean_is_exclusive(x_35); +if (x_239 == 0) { return x_35; } else { -lean_object* x_206; lean_object* x_207; lean_object* x_208; -x_206 = lean_ctor_get(x_35, 0); -x_207 = lean_ctor_get(x_35, 1); -lean_inc(x_207); -lean_inc(x_206); +lean_object* x_240; lean_object* x_241; lean_object* x_242; +x_240 = lean_ctor_get(x_35, 0); +x_241 = lean_ctor_get(x_35, 1); +lean_inc(x_241); +lean_inc(x_240); lean_dec(x_35); -x_208 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_208, 0, x_206); -lean_ctor_set(x_208, 1, x_207); -return x_208; +x_242 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_242, 0, x_240); +lean_ctor_set(x_242, 1, x_241); +return x_242; } } } else { -uint8_t x_209; +uint8_t x_243; lean_dec(x_23); lean_dec(x_13); lean_dec(x_9); @@ -6581,23 +6736,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_209 = !lean_is_exclusive(x_27); -if (x_209 == 0) +x_243 = !lean_is_exclusive(x_27); +if (x_243 == 0) { return x_27; } else { -lean_object* x_210; lean_object* x_211; lean_object* x_212; -x_210 = lean_ctor_get(x_27, 0); -x_211 = lean_ctor_get(x_27, 1); -lean_inc(x_211); -lean_inc(x_210); +lean_object* x_244; lean_object* x_245; lean_object* x_246; +x_244 = lean_ctor_get(x_27, 0); +x_245 = lean_ctor_get(x_27, 1); +lean_inc(x_245); +lean_inc(x_244); lean_dec(x_27); -x_212 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_212, 0, x_210); -lean_ctor_set(x_212, 1, x_211); -return x_212; +x_246 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_246, 0, x_244); +lean_ctor_set(x_246, 1, x_245); +return x_246; } } } @@ -6605,7 +6760,7 @@ return x_212; } else { -uint8_t x_221; +uint8_t x_255; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6613,23 +6768,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_221 = !lean_is_exclusive(x_12); -if (x_221 == 0) +x_255 = !lean_is_exclusive(x_12); +if (x_255 == 0) { return x_12; } else { -lean_object* x_222; lean_object* x_223; lean_object* x_224; -x_222 = lean_ctor_get(x_12, 0); -x_223 = lean_ctor_get(x_12, 1); -lean_inc(x_223); -lean_inc(x_222); +lean_object* x_256; lean_object* x_257; lean_object* x_258; +x_256 = lean_ctor_get(x_12, 0); +x_257 = lean_ctor_get(x_12, 1); +lean_inc(x_257); +lean_inc(x_256); lean_dec(x_12); -x_224 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_224, 0, x_222); -lean_ctor_set(x_224, 1, x_223); -return x_224; +x_258 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_258, 0, x_256); +lean_ctor_set(x_258, 1, x_257); +return x_258; } } } @@ -6656,47 +6811,37 @@ static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandle _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__2; -x_2 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__9; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__3; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31; x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___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_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__5() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__4; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__3; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__6() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__5; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___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_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__7() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__6() { _start: { lean_object* x_1; @@ -6704,7 +6849,7 @@ x_1 = lean_mk_string_from_bytes("<|", 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__8() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__7() { _start: { lean_object* x_1; @@ -6712,22 +6857,22 @@ x_1 = lean_mk_string_from_bytes("List.join", 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__9() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__8; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__7; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__10() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__8; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__7; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__9; +x_3 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__8; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6735,7 +6880,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__11() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__10() { _start: { lean_object* x_1; @@ -6743,17 +6888,17 @@ x_1 = lean_mk_string_from_bytes("List", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__12() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__11; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__13() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__12() { _start: { lean_object* x_1; @@ -6761,34 +6906,34 @@ x_1 = lean_mk_string_from_bytes("join", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__14() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__12; -x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__13; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__11; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__15() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__14; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__13; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__16() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__15; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__14; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); @@ -6810,36 +6955,36 @@ lean_inc(x_1); x_11 = l_Lean_Elab_Deriving_mkContext(x_10, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_11) == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_192; lean_object* x_193; lean_object* x_194; uint8_t x_195; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_192 = lean_ctor_get(x_12, 0); -lean_inc(x_192); -x_193 = lean_array_get_size(x_192); -x_194 = lean_unsigned_to_nat(0u); -x_195 = lean_nat_dec_lt(x_194, x_193); -lean_dec(x_193); -if (x_195 == 0) +x_205 = lean_ctor_get(x_12, 0); +lean_inc(x_205); +x_206 = lean_array_get_size(x_205); +x_207 = lean_unsigned_to_nat(0u); +x_208 = lean_nat_dec_lt(x_207, x_206); +lean_dec(x_206); +if (x_208 == 0) { -lean_object* x_196; lean_object* x_197; -lean_dec(x_192); -x_196 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__4; -x_197 = l_panic___at_Lean_Elab_Deriving_mkLocalInstanceLetDecls___spec__1(x_196); -x_14 = x_197; -goto block_191; +lean_object* x_209; lean_object* x_210; +lean_dec(x_205); +x_209 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__4; +x_210 = l_panic___at_Lean_Elab_Deriving_mkLocalInstanceLetDecls___spec__1(x_209); +x_14 = x_210; +goto block_204; } else { -lean_object* x_198; -x_198 = lean_array_fget(x_192, x_194); -lean_dec(x_192); -x_14 = x_198; -goto block_191; +lean_object* x_211; +x_211 = lean_array_fget(x_205, x_207); +lean_dec(x_205); +x_14 = x_211; +goto block_204; } -block_191: +block_204: { lean_object* x_15; lean_object* x_16; lean_object* x_17; x_15 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__2; @@ -6853,7 +6998,7 @@ lean_inc(x_3); x_17 = l_Lean_Elab_Deriving_mkHeader(x_15, x_16, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_13); if (lean_obj_tag(x_17) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; size_t x_27; size_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; size_t x_27; size_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); @@ -6951,280 +7096,309 @@ x_69 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_69, 0, x_46); lean_ctor_set(x_69, 1, x_50); lean_ctor_set(x_69, 2, x_68); -x_70 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__7; -x_71 = lean_array_push(x_70, x_69); -x_72 = lean_array_push(x_71, x_54); -x_73 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__25; -x_74 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_74, 0, x_46); -lean_ctor_set(x_74, 1, x_73); -lean_ctor_set(x_74, 2, x_72); -x_75 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; +x_70 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; lean_inc(x_34); -x_76 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_76, 0, x_34); -lean_ctor_set(x_76, 1, x_75); -x_77 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__4; +x_71 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_71, 0, x_34); +lean_ctor_set(x_71, 1, x_70); +x_72 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__8; lean_inc(x_36); lean_inc(x_41); -x_78 = l_Lean_addMacroScope(x_41, x_77, x_36); -x_79 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__3; -x_80 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__6; +x_73 = l_Lean_addMacroScope(x_41, x_72, x_36); +x_74 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; +x_75 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__33; lean_inc(x_34); -x_81 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_81, 0, x_34); -lean_ctor_set(x_81, 1, x_79); -lean_ctor_set(x_81, 2, x_78); -lean_ctor_set(x_81, 3, x_80); -x_82 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__7; +x_76 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_76, 0, x_34); +lean_ctor_set(x_76, 1, x_74); +lean_ctor_set(x_76, 2, x_73); +lean_ctor_set(x_76, 3, x_75); +x_77 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__7; +x_78 = lean_array_push(x_77, x_71); +x_79 = lean_array_push(x_78, x_76); +x_80 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__27; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_46); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_79); +x_82 = lean_array_push(x_44, x_81); +x_83 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_83, 0, x_46); +lean_ctor_set(x_83, 1, x_50); +lean_ctor_set(x_83, 2, x_82); +x_84 = lean_array_push(x_77, x_69); +x_85 = lean_array_push(x_84, x_83); +x_86 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__25; +x_87 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_87, 0, x_46); +lean_ctor_set(x_87, 1, x_86); +lean_ctor_set(x_87, 2, x_85); +x_88 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36; lean_inc(x_34); -x_83 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_83, 0, x_34); -lean_ctor_set(x_83, 1, x_82); -x_84 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__14; -x_85 = l_Lean_addMacroScope(x_41, x_84, x_36); -x_86 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__10; -x_87 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__16; +x_89 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_89, 0, x_34); +lean_ctor_set(x_89, 1, x_88); +x_90 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__4; +lean_inc(x_36); +lean_inc(x_41); +x_91 = l_Lean_addMacroScope(x_41, x_90, x_36); +x_92 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___closed__3; +x_93 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__5; lean_inc(x_34); -x_88 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_88, 0, x_34); -lean_ctor_set(x_88, 1, x_86); -lean_ctor_set(x_88, 2, x_85); -lean_ctor_set(x_88, 3, x_87); -x_89 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__3; +x_94 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_94, 0, x_34); +lean_ctor_set(x_94, 1, x_92); +lean_ctor_set(x_94, 2, x_91); +lean_ctor_set(x_94, 3, x_93); +x_95 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__6; lean_inc(x_34); -x_90 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_90, 0, x_34); -lean_ctor_set(x_90, 1, x_89); -x_91 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__14; -x_92 = l_Lean_mkSepArray(x_31, x_91); -lean_dec(x_31); -x_93 = l_Array_append___rarg(x_67, x_92); -x_94 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_94, 0, x_46); -lean_ctor_set(x_94, 1, x_50); -lean_ctor_set(x_94, 2, x_93); -x_95 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__4; x_96 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_96, 0, x_34); lean_ctor_set(x_96, 1, x_95); -x_97 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___closed__5; -x_98 = lean_array_push(x_97, x_90); -x_99 = lean_array_push(x_98, x_94); -x_100 = lean_array_push(x_99, x_96); -x_101 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__2; -x_102 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_102, 0, x_46); -lean_ctor_set(x_102, 1, x_101); -lean_ctor_set(x_102, 2, x_100); -x_103 = lean_array_push(x_44, x_102); -x_104 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_104, 0, x_46); -lean_ctor_set(x_104, 1, x_50); -lean_ctor_set(x_104, 2, x_103); -x_105 = lean_array_push(x_70, x_88); -x_106 = lean_array_push(x_105, x_104); -x_107 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__3; -x_108 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_108, 0, x_46); -lean_ctor_set(x_108, 1, x_107); -lean_ctor_set(x_108, 2, x_106); -x_109 = lean_array_push(x_97, x_81); -x_110 = lean_array_push(x_109, x_83); -x_111 = lean_array_push(x_110, x_108); -x_112 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__2; -x_113 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_113, 0, x_46); -lean_ctor_set(x_113, 1, x_112); -lean_ctor_set(x_113, 2, x_111); -x_114 = lean_array_push(x_97, x_76); -x_115 = lean_array_push(x_114, x_113); -x_116 = lean_array_push(x_115, x_54); -x_117 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__27; -x_118 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_118, 0, x_46); -lean_ctor_set(x_118, 1, x_117); -lean_ctor_set(x_118, 2, x_116); -x_119 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; -x_120 = lean_array_push(x_119, x_61); -x_121 = lean_array_push(x_70, x_59); +x_97 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__13; +x_98 = l_Lean_addMacroScope(x_41, x_97, x_36); +x_99 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__9; +x_100 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__15; +lean_inc(x_34); +x_101 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_101, 0, x_34); +lean_ctor_set(x_101, 1, x_99); +lean_ctor_set(x_101, 2, x_98); +lean_ctor_set(x_101, 3, x_100); +x_102 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__3; +lean_inc(x_34); +x_103 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_103, 0, x_34); +lean_ctor_set(x_103, 1, x_102); +x_104 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__14; +x_105 = l_Lean_mkSepArray(x_31, x_104); +lean_dec(x_31); +x_106 = l_Array_append___rarg(x_67, x_105); +x_107 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_107, 0, x_46); +lean_ctor_set(x_107, 1, x_50); +lean_ctor_set(x_107, 2, x_106); +x_108 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__4; +x_109 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_109, 0, x_34); +lean_ctor_set(x_109, 1, x_108); +x_110 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__4___closed__5; +x_111 = lean_array_push(x_110, x_103); +x_112 = lean_array_push(x_111, x_107); +x_113 = lean_array_push(x_112, x_109); +x_114 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__2; +x_115 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_115, 0, x_46); +lean_ctor_set(x_115, 1, x_114); +lean_ctor_set(x_115, 2, x_113); +x_116 = lean_array_push(x_44, x_115); +x_117 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_117, 0, x_46); +lean_ctor_set(x_117, 1, x_50); +lean_ctor_set(x_117, 2, x_116); +x_118 = lean_array_push(x_77, x_101); +x_119 = lean_array_push(x_118, x_117); +x_120 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__5___lambda__1___closed__3; +x_121 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_121, 0, x_46); +lean_ctor_set(x_121, 1, x_120); +lean_ctor_set(x_121, 2, x_119); +x_122 = lean_array_push(x_110, x_94); +x_123 = lean_array_push(x_122, x_96); +x_124 = lean_array_push(x_123, x_121); +x_125 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__2; +x_126 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_126, 0, x_46); +lean_ctor_set(x_126, 1, x_125); +lean_ctor_set(x_126, 2, x_124); +x_127 = lean_array_push(x_110, x_89); +x_128 = lean_array_push(x_127, x_126); +x_129 = lean_array_push(x_128, x_54); +x_130 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35; +x_131 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_131, 0, x_46); +lean_ctor_set(x_131, 1, x_130); +lean_ctor_set(x_131, 2, x_129); +x_132 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; +x_133 = lean_array_push(x_132, x_61); +x_134 = lean_array_push(x_77, x_59); if (x_65 == 0) { -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; 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; uint8_t x_140; lean_object* x_141; +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; uint8_t x_153; lean_object* x_154; lean_dec(x_62); -x_122 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__4; -x_123 = l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(x_122); -x_124 = lean_mk_syntax_ident(x_123); -x_125 = lean_array_push(x_70, x_124); -x_126 = lean_array_push(x_125, x_54); -x_127 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; -x_128 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_128, 0, x_46); -lean_ctor_set(x_128, 1, x_127); -lean_ctor_set(x_128, 2, x_126); -x_129 = lean_array_push(x_120, x_128); -x_130 = lean_array_push(x_129, x_74); -x_131 = lean_array_push(x_130, x_118); -x_132 = lean_array_push(x_131, x_54); -x_133 = lean_array_push(x_132, x_54); -x_134 = lean_array_push(x_133, x_54); -x_135 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__21; -x_136 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_136, 0, x_46); -lean_ctor_set(x_136, 1, x_135); -lean_ctor_set(x_136, 2, x_134); -x_137 = lean_array_push(x_121, x_136); -x_138 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; -x_139 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_139, 0, x_46); -lean_ctor_set(x_139, 1, x_138); -lean_ctor_set(x_139, 2, x_137); -x_140 = 1; -x_141 = l_Lean_Elab_Deriving_mkInstanceCmds(x_12, x_15, x_2, x_140, x_3, x_4, x_5, x_6, x_7, x_8, x_39); +x_135 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__4___closed__4; +x_136 = l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(x_135); +x_137 = lean_mk_syntax_ident(x_136); +x_138 = lean_array_push(x_77, x_137); +x_139 = lean_array_push(x_138, x_54); +x_140 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; +x_141 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_141, 0, x_46); +lean_ctor_set(x_141, 1, x_140); +lean_ctor_set(x_141, 2, x_139); +x_142 = lean_array_push(x_133, x_141); +x_143 = lean_array_push(x_142, x_87); +x_144 = lean_array_push(x_143, x_131); +x_145 = lean_array_push(x_144, x_54); +x_146 = lean_array_push(x_145, x_54); +x_147 = lean_array_push(x_146, x_54); +x_148 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__21; +x_149 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_149, 0, x_46); +lean_ctor_set(x_149, 1, x_148); +lean_ctor_set(x_149, 2, x_147); +x_150 = lean_array_push(x_134, x_149); +x_151 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; +x_152 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_152, 0, x_46); +lean_ctor_set(x_152, 1, x_151); +lean_ctor_set(x_152, 2, x_150); +x_153 = 1; +x_154 = l_Lean_Elab_Deriving_mkInstanceCmds(x_12, x_15, x_2, x_153, x_3, x_4, x_5, x_6, x_7, x_8, x_39); lean_dec(x_12); -if (lean_obj_tag(x_141) == 0) +if (lean_obj_tag(x_154) == 0) { -uint8_t x_142; -x_142 = !lean_is_exclusive(x_141); -if (x_142 == 0) +uint8_t x_155; +x_155 = !lean_is_exclusive(x_154); +if (x_155 == 0) { -lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_143 = lean_ctor_get(x_141, 0); -x_144 = lean_array_push(x_44, x_139); -x_145 = l_Array_append___rarg(x_144, x_143); -lean_ctor_set(x_141, 0, x_145); -return x_141; +lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_156 = lean_ctor_get(x_154, 0); +x_157 = lean_array_push(x_44, x_152); +x_158 = l_Array_append___rarg(x_157, x_156); +lean_ctor_set(x_154, 0, x_158); +return x_154; } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; -x_146 = lean_ctor_get(x_141, 0); -x_147 = lean_ctor_get(x_141, 1); -lean_inc(x_147); -lean_inc(x_146); -lean_dec(x_141); -x_148 = lean_array_push(x_44, x_139); -x_149 = l_Array_append___rarg(x_148, x_146); -x_150 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_150, 0, x_149); -lean_ctor_set(x_150, 1, x_147); -return x_150; +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_159 = lean_ctor_get(x_154, 0); +x_160 = lean_ctor_get(x_154, 1); +lean_inc(x_160); +lean_inc(x_159); +lean_dec(x_154); +x_161 = lean_array_push(x_44, x_152); +x_162 = l_Array_append___rarg(x_161, x_159); +x_163 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_163, 0, x_162); +lean_ctor_set(x_163, 1, x_160); +return x_163; } } else { -uint8_t x_151; -lean_dec(x_139); -x_151 = !lean_is_exclusive(x_141); -if (x_151 == 0) +uint8_t x_164; +lean_dec(x_152); +x_164 = !lean_is_exclusive(x_154); +if (x_164 == 0) { -return x_141; +return x_154; } else { -lean_object* x_152; lean_object* x_153; lean_object* x_154; -x_152 = lean_ctor_get(x_141, 0); -x_153 = lean_ctor_get(x_141, 1); -lean_inc(x_153); -lean_inc(x_152); -lean_dec(x_141); -x_154 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_154, 0, x_152); -lean_ctor_set(x_154, 1, x_153); -return x_154; +lean_object* x_165; lean_object* x_166; lean_object* x_167; +x_165 = lean_ctor_get(x_154, 0); +x_166 = lean_ctor_get(x_154, 1); +lean_inc(x_166); +lean_inc(x_165); +lean_dec(x_154); +x_167 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_167, 0, x_165); +lean_ctor_set(x_167, 1, x_166); +return x_167; } } } else { -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; uint8_t x_172; lean_object* x_173; -x_155 = lean_array_fget(x_62, x_64); +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; uint8_t x_185; lean_object* x_186; +x_168 = lean_array_fget(x_62, x_64); lean_dec(x_62); -x_156 = lean_mk_syntax_ident(x_155); -x_157 = lean_array_push(x_70, x_156); -x_158 = lean_array_push(x_157, x_54); -x_159 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; -x_160 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_160, 0, x_46); -lean_ctor_set(x_160, 1, x_159); -lean_ctor_set(x_160, 2, x_158); -x_161 = lean_array_push(x_120, x_160); -x_162 = lean_array_push(x_161, x_74); -x_163 = lean_array_push(x_162, x_118); -x_164 = lean_array_push(x_163, x_54); -x_165 = lean_array_push(x_164, x_54); -x_166 = lean_array_push(x_165, x_54); -x_167 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__21; -x_168 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_168, 0, x_46); -lean_ctor_set(x_168, 1, x_167); -lean_ctor_set(x_168, 2, x_166); -x_169 = lean_array_push(x_121, x_168); -x_170 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; -x_171 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_171, 0, x_46); -lean_ctor_set(x_171, 1, x_170); -lean_ctor_set(x_171, 2, x_169); -x_172 = 1; -x_173 = l_Lean_Elab_Deriving_mkInstanceCmds(x_12, x_15, x_2, x_172, x_3, x_4, x_5, x_6, x_7, x_8, x_39); +x_169 = lean_mk_syntax_ident(x_168); +x_170 = lean_array_push(x_77, x_169); +x_171 = lean_array_push(x_170, x_54); +x_172 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__23; +x_173 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_173, 0, x_46); +lean_ctor_set(x_173, 1, x_172); +lean_ctor_set(x_173, 2, x_171); +x_174 = lean_array_push(x_133, x_173); +x_175 = lean_array_push(x_174, x_87); +x_176 = lean_array_push(x_175, x_131); +x_177 = lean_array_push(x_176, x_54); +x_178 = lean_array_push(x_177, x_54); +x_179 = lean_array_push(x_178, x_54); +x_180 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__21; +x_181 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_181, 0, x_46); +lean_ctor_set(x_181, 1, x_180); +lean_ctor_set(x_181, 2, x_179); +x_182 = lean_array_push(x_134, x_181); +x_183 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__13; +x_184 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_184, 0, x_46); +lean_ctor_set(x_184, 1, x_183); +lean_ctor_set(x_184, 2, x_182); +x_185 = 1; +x_186 = l_Lean_Elab_Deriving_mkInstanceCmds(x_12, x_15, x_2, x_185, x_3, x_4, x_5, x_6, x_7, x_8, x_39); lean_dec(x_12); -if (lean_obj_tag(x_173) == 0) +if (lean_obj_tag(x_186) == 0) { -uint8_t x_174; -x_174 = !lean_is_exclusive(x_173); -if (x_174 == 0) +uint8_t x_187; +x_187 = !lean_is_exclusive(x_186); +if (x_187 == 0) { -lean_object* x_175; lean_object* x_176; lean_object* x_177; -x_175 = lean_ctor_get(x_173, 0); -x_176 = lean_array_push(x_44, x_171); -x_177 = l_Array_append___rarg(x_176, x_175); -lean_ctor_set(x_173, 0, x_177); -return x_173; +lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_188 = lean_ctor_get(x_186, 0); +x_189 = lean_array_push(x_44, x_184); +x_190 = l_Array_append___rarg(x_189, x_188); +lean_ctor_set(x_186, 0, x_190); +return x_186; } else { -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_178 = lean_ctor_get(x_173, 0); -x_179 = lean_ctor_get(x_173, 1); -lean_inc(x_179); -lean_inc(x_178); -lean_dec(x_173); -x_180 = lean_array_push(x_44, x_171); -x_181 = l_Array_append___rarg(x_180, x_178); -x_182 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_182, 0, x_181); -lean_ctor_set(x_182, 1, x_179); -return x_182; +lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +x_191 = lean_ctor_get(x_186, 0); +x_192 = lean_ctor_get(x_186, 1); +lean_inc(x_192); +lean_inc(x_191); +lean_dec(x_186); +x_193 = lean_array_push(x_44, x_184); +x_194 = l_Array_append___rarg(x_193, x_191); +x_195 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_192); +return x_195; } } else { -uint8_t x_183; -lean_dec(x_171); -x_183 = !lean_is_exclusive(x_173); -if (x_183 == 0) +uint8_t x_196; +lean_dec(x_184); +x_196 = !lean_is_exclusive(x_186); +if (x_196 == 0) { -return x_173; +return x_186; } else { -lean_object* x_184; lean_object* x_185; lean_object* x_186; -x_184 = lean_ctor_get(x_173, 0); -x_185 = lean_ctor_get(x_173, 1); -lean_inc(x_185); -lean_inc(x_184); -lean_dec(x_173); -x_186 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_186, 0, x_184); -lean_ctor_set(x_186, 1, x_185); -return x_186; +lean_object* x_197; lean_object* x_198; lean_object* x_199; +x_197 = lean_ctor_get(x_186, 0); +x_198 = lean_ctor_get(x_186, 1); +lean_inc(x_198); +lean_inc(x_197); +lean_dec(x_186); +x_199 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +return x_199; } } } } else { -uint8_t x_187; +uint8_t x_200; lean_dec(x_12); lean_dec(x_8); lean_dec(x_7); @@ -7233,30 +7407,30 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_187 = !lean_is_exclusive(x_17); -if (x_187 == 0) +x_200 = !lean_is_exclusive(x_17); +if (x_200 == 0) { return x_17; } else { -lean_object* x_188; lean_object* x_189; lean_object* x_190; -x_188 = lean_ctor_get(x_17, 0); -x_189 = lean_ctor_get(x_17, 1); -lean_inc(x_189); -lean_inc(x_188); +lean_object* x_201; lean_object* x_202; lean_object* x_203; +x_201 = lean_ctor_get(x_17, 0); +x_202 = lean_ctor_get(x_17, 1); +lean_inc(x_202); +lean_inc(x_201); lean_dec(x_17); -x_190 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_190, 0, x_188); -lean_ctor_set(x_190, 1, x_189); -return x_190; +x_203 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_203, 0, x_201); +lean_ctor_set(x_203, 1, x_202); +return x_203; } } } } else { -uint8_t x_199; +uint8_t x_212; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -7264,23 +7438,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_199 = !lean_is_exclusive(x_11); -if (x_199 == 0) +x_212 = !lean_is_exclusive(x_11); +if (x_212 == 0) { return x_11; } else { -lean_object* x_200; lean_object* x_201; lean_object* x_202; -x_200 = lean_ctor_get(x_11, 0); -x_201 = lean_ctor_get(x_11, 1); -lean_inc(x_201); -lean_inc(x_200); +lean_object* x_213; lean_object* x_214; lean_object* x_215; +x_213 = lean_ctor_get(x_11, 0); +x_214 = lean_ctor_get(x_11, 1); +lean_inc(x_214); +lean_inc(x_213); lean_dec(x_11); -x_202 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_202, 0, x_200); -lean_ctor_set(x_202, 1, x_201); -return x_202; +x_215 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_215, 0, x_213); +lean_ctor_set(x_215, 1, x_214); +return x_215; } } } @@ -7410,7 +7584,7 @@ x_34 = 0; x_35 = lean_usize_of_nat(x_26); lean_dec(x_26); x_36 = lean_box(0); -x_37 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_24, x_34, x_35, x_36, x_2, x_3, x_25); +x_37 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_24, x_34, x_35, x_36, x_2, x_3, x_25); lean_dec(x_24); if (lean_obj_tag(x_37) == 0) { @@ -7515,7 +7689,7 @@ x_62 = 0; x_63 = lean_usize_of_nat(x_52); lean_dec(x_52); x_64 = lean_box(0); -x_65 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_50, x_62, x_63, x_64, x_2, x_3, x_51); +x_65 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_50, x_62, x_63, x_64, x_2, x_3, x_51); lean_dec(x_50); if (lean_obj_tag(x_65) == 0) { @@ -7678,7 +7852,7 @@ x_97 = 0; x_98 = lean_usize_of_nat(x_89); lean_dec(x_89); x_99 = lean_box(0); -x_100 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_87, x_97, x_98, x_99, x_2, x_3, x_88); +x_100 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_87, x_97, x_98, x_99, x_2, x_3, x_88); lean_dec(x_87); if (lean_obj_tag(x_100) == 0) { @@ -7783,7 +7957,7 @@ x_125 = 0; x_126 = lean_usize_of_nat(x_115); lean_dec(x_115); x_127 = lean_box(0); -x_128 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_113, x_125, x_126, x_127, x_2, x_3, x_114); +x_128 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_113, x_125, x_126, x_127, x_2, x_3, x_114); lean_dec(x_113); if (lean_obj_tag(x_128) == 0) { @@ -8576,7 +8750,7 @@ x_51 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstance x_52 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_52, 0, x_26); lean_ctor_set(x_52, 1, x_51); -x_53 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; +x_53 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; x_54 = lean_array_push(x_53, x_43); x_55 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__20; x_56 = lean_array_push(x_54, x_55); @@ -8671,7 +8845,7 @@ x_100 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanc x_101 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_101, 0, x_80); lean_ctor_set(x_101, 1, x_100); -x_102 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; +x_102 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; x_103 = lean_array_push(x_102, x_92); x_104 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__20; x_105 = lean_array_push(x_103, x_104); @@ -9075,7 +9249,7 @@ static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__3; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31; x_2 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__7___lambda__1___closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -11753,52 +11927,13 @@ return x_1; static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(":", 1); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__9; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___spec__7___closed__9; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__3; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; x_1 = lean_unsigned_to_nat(5u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("typeSpec", 8); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__7() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -11806,22 +11941,22 @@ x_1 = lean_mk_string_from_bytes("Except", 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__8() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__7; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__3; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__7; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__3; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__8; +x_3 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__4; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -11829,7 +11964,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__10() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__6() { _start: { lean_object* x_1; @@ -11837,22 +11972,22 @@ x_1 = lean_mk_string_from_bytes("String", 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__11() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__10; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__6; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__12() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__10; +x_1 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__6; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__11; +x_3 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__7; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -11860,12 +11995,12 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__10; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -12013,7 +12148,7 @@ x_226 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_226, 0, x_187); lean_ctor_set(x_226, 1, x_8); lean_ctor_set(x_226, 2, x_225); -x_227 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__2; +x_227 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; lean_inc(x_173); x_228 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_228, 0, x_173); @@ -12032,7 +12167,7 @@ lean_inc(x_12); x_234 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_234, 0, x_233); lean_ctor_set(x_234, 1, x_12); -x_235 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__4; +x_235 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; lean_inc(x_173); x_236 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_236, 0, x_173); @@ -12053,7 +12188,7 @@ lean_inc(x_173); x_241 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_241, 0, x_173); lean_ctor_set(x_241, 1, x_240); -x_242 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__5; +x_242 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__2; x_243 = lean_array_push(x_242, x_220); x_244 = lean_array_push(x_243, x_226); x_245 = lean_array_push(x_244, x_239); @@ -12070,7 +12205,7 @@ x_250 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_250, 0, x_187); lean_ctor_set(x_250, 1, x_8); lean_ctor_set(x_250, 2, x_249); -x_251 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__6; +x_251 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__26; x_252 = l_Lean_Name_str___override(x_11, x_251); lean_inc(x_175); lean_inc(x_14); @@ -12084,14 +12219,14 @@ lean_inc(x_12); x_255 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_255, 0, x_254); lean_ctor_set(x_255, 1, x_12); -x_256 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9; +x_256 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__5; lean_inc(x_173); x_257 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_257, 0, x_173); lean_ctor_set(x_257, 1, x_256); lean_ctor_set(x_257, 2, x_253); lean_ctor_set(x_257, 3, x_255); -x_258 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13; +x_258 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9; x_259 = l_Lean_addMacroScope(x_180, x_258, x_175); lean_inc(x_12); x_260 = lean_alloc_ctor(0, 2, 0); @@ -12100,7 +12235,7 @@ lean_ctor_set(x_260, 1, x_12); x_261 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_261, 0, x_260); lean_ctor_set(x_261, 1, x_12); -x_262 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__12; +x_262 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__8; lean_inc(x_173); x_263 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_263, 0, x_173); @@ -12140,9 +12275,9 @@ x_276 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_276, 0, x_187); lean_ctor_set(x_276, 1, x_214); lean_ctor_set(x_276, 2, x_275); -x_277 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__26; +x_277 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__34; x_278 = l_Lean_Name_str___override(x_182, x_277); -x_279 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; +x_279 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36; x_280 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_280, 0, x_173); lean_ctor_set(x_280, 1, x_279); @@ -12155,7 +12290,7 @@ x_285 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_285, 0, x_187); lean_ctor_set(x_285, 1, x_278); lean_ctor_set(x_285, 2, x_284); -x_286 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; +x_286 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; x_287 = lean_array_push(x_286, x_207); x_288 = lean_array_push(x_287, x_212); x_289 = lean_array_push(x_288, x_276); @@ -12260,7 +12395,7 @@ x_55 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_55, 0, x_46); lean_ctor_set(x_55, 1, x_8); lean_ctor_set(x_55, 2, x_54); -x_56 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; +x_56 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__38; lean_inc(x_41); x_57 = l_Lean_Name_str___override(x_41, x_56); lean_inc(x_32); @@ -12347,7 +12482,7 @@ x_92 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_92, 0, x_46); lean_ctor_set(x_92, 1, x_8); lean_ctor_set(x_92, 2, x_91); -x_93 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__2; +x_93 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; lean_inc(x_32); x_94 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_94, 0, x_32); @@ -12366,7 +12501,7 @@ lean_inc(x_12); x_100 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_100, 0, x_99); lean_ctor_set(x_100, 1, x_12); -x_101 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__4; +x_101 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; lean_inc(x_32); x_102 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_102, 0, x_32); @@ -12387,7 +12522,7 @@ lean_inc(x_32); x_107 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_107, 0, x_32); lean_ctor_set(x_107, 1, x_106); -x_108 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__5; +x_108 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__2; x_109 = lean_array_push(x_108, x_86); x_110 = lean_array_push(x_109, x_92); x_111 = lean_array_push(x_110, x_105); @@ -12404,7 +12539,7 @@ x_116 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_116, 0, x_46); lean_ctor_set(x_116, 1, x_8); lean_ctor_set(x_116, 2, x_115); -x_117 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__6; +x_117 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__26; x_118 = l_Lean_Name_str___override(x_11, x_117); lean_inc(x_34); lean_inc(x_14); @@ -12418,14 +12553,14 @@ lean_inc(x_12); x_121 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_121, 0, x_120); lean_ctor_set(x_121, 1, x_12); -x_122 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9; +x_122 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__5; lean_inc(x_32); x_123 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_123, 0, x_32); lean_ctor_set(x_123, 1, x_122); lean_ctor_set(x_123, 2, x_119); lean_ctor_set(x_123, 3, x_121); -x_124 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13; +x_124 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9; x_125 = l_Lean_addMacroScope(x_39, x_124, x_34); lean_inc(x_12); x_126 = lean_alloc_ctor(0, 2, 0); @@ -12434,7 +12569,7 @@ lean_ctor_set(x_126, 1, x_12); x_127 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_127, 0, x_126); lean_ctor_set(x_127, 1, x_12); -x_128 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__12; +x_128 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__8; lean_inc(x_32); x_129 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_129, 0, x_32); @@ -12474,9 +12609,9 @@ x_142 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_142, 0, x_46); lean_ctor_set(x_142, 1, x_80); lean_ctor_set(x_142, 2, x_141); -x_143 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__26; +x_143 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__34; x_144 = l_Lean_Name_str___override(x_41, x_143); -x_145 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; +x_145 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36; x_146 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_146, 0, x_32); lean_ctor_set(x_146, 1, x_145); @@ -12489,7 +12624,7 @@ x_151 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_151, 0, x_46); lean_ctor_set(x_151, 1, x_144); lean_ctor_set(x_151, 2, x_150); -x_152 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; +x_152 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; x_153 = lean_array_push(x_152, x_73); x_154 = lean_array_push(x_153, x_78); x_155 = lean_array_push(x_154, x_142); @@ -12558,7 +12693,7 @@ static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHand { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__7; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -13116,7 +13251,7 @@ static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHand { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__3; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); @@ -13139,16 +13274,6 @@ static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHand _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__6; -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__6; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__5; x_3 = lean_alloc_ctor(0, 2, 0); @@ -13157,43 +13282,43 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__10() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__9; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___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_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__11() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__12() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__11; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__10; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__13() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__12() { _start: { lean_object* x_1; @@ -13201,17 +13326,17 @@ x_1 = lean_mk_string_from_bytes("structInst", 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__14() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__6; -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__13; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__15() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__14() { _start: { lean_object* x_1; @@ -13219,7 +13344,7 @@ x_1 = lean_mk_string_from_bytes("{", 1); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__16() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__15() { _start: { lean_object* x_1; @@ -13227,17 +13352,17 @@ x_1 = lean_mk_string_from_bytes("optEllipsis", 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__17() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__6; -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__16; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__15; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__18() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -13247,13 +13372,13 @@ x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__19() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__17; -x_3 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__18; +x_2 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__16; +x_3 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__17; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -13261,7 +13386,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__20() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__19() { _start: { lean_object* x_1; @@ -13448,7 +13573,7 @@ x_78 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_78, 0, x_48); lean_ctor_set(x_78, 1, x_52); lean_ctor_set(x_78, 2, x_77); -x_79 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__2; +x_79 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; lean_inc(x_36); x_80 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_80, 0, x_36); @@ -13457,7 +13582,7 @@ x_81 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__1___clo lean_inc(x_38); lean_inc(x_43); x_82 = l_Lean_addMacroScope(x_43, x_81, x_38); -x_83 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__4; +x_83 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30; x_84 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__7; lean_inc(x_36); x_85 = lean_alloc_ctor(3, 4, 0); @@ -13478,7 +13603,7 @@ lean_inc(x_36); x_91 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_91, 0, x_36); lean_ctor_set(x_91, 1, x_90); -x_92 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__5; +x_92 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__2; x_93 = lean_array_push(x_92, x_71); x_94 = lean_array_push(x_93, x_78); x_95 = lean_array_push(x_94, x_89); @@ -13498,20 +13623,20 @@ x_102 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___ lean_inc(x_38); lean_inc(x_43); x_103 = l_Lean_addMacroScope(x_43, x_102, x_38); -x_104 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9; -x_105 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__10; +x_104 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__5; +x_105 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__9; lean_inc(x_36); x_106 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_106, 0, x_36); lean_ctor_set(x_106, 1, x_104); lean_ctor_set(x_106, 2, x_103); lean_ctor_set(x_106, 3, x_105); -x_107 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13; +x_107 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9; lean_inc(x_38); lean_inc(x_43); x_108 = l_Lean_addMacroScope(x_43, x_107, x_38); -x_109 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__12; -x_110 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__12; +x_109 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__8; +x_110 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__11; lean_inc(x_36); x_111 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_111, 0, x_36); @@ -13532,7 +13657,7 @@ lean_ctor_set(x_118, 0, x_48); lean_ctor_set(x_118, 1, x_117); lean_ctor_set(x_118, 2, x_116); x_119 = lean_array_push(x_87, x_118); -x_120 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__8; +x_120 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__27; x_121 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_121, 0, x_48); lean_ctor_set(x_121, 1, x_120); @@ -13549,7 +13674,7 @@ x_127 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_127, 0, x_48); lean_ctor_set(x_127, 1, x_126); lean_ctor_set(x_127, 2, x_125); -x_128 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__28; +x_128 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36; lean_inc(x_36); x_129 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_129, 0, x_36); @@ -13565,7 +13690,7 @@ x_133 = lean_array_get_size(x_132); x_134 = lean_usize_of_nat(x_133); lean_dec(x_133); x_135 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler_mkAlts___spec__3___closed__6; -x_136 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__3; +x_136 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31; lean_inc(x_36); x_137 = l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___spec__5(x_36, x_38, x_43, x_52, x_56, x_46, x_86, x_135, x_16, x_74, x_76, x_136, x_74, x_117, x_134, x_28, x_132); x_138 = l_Array_append___rarg(x_68, x_137); @@ -13574,7 +13699,7 @@ lean_inc(x_36); x_140 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_140, 0, x_36); lean_ctor_set(x_140, 1, x_139); -x_141 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__15; +x_141 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__14; lean_inc(x_36); x_142 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_142, 0, x_36); @@ -13594,7 +13719,7 @@ x_150 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_150, 0, x_48); lean_ctor_set(x_150, 1, x_52); lean_ctor_set(x_150, 2, x_149); -x_151 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__20; +x_151 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__19; x_152 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_152, 0, x_36); lean_ctor_set(x_152, 1, x_151); @@ -13602,11 +13727,11 @@ x_153 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___cl x_154 = lean_array_push(x_153, x_142); x_155 = lean_array_push(x_154, x_56); x_156 = lean_array_push(x_155, x_150); -x_157 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__19; +x_157 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__18; x_158 = lean_array_push(x_156, x_157); x_159 = lean_array_push(x_158, x_56); x_160 = lean_array_push(x_159, x_152); -x_161 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__14; +x_161 = l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__13; x_162 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_162, 0, x_48); lean_ctor_set(x_162, 1, x_161); @@ -13652,12 +13777,12 @@ x_182 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceH x_183 = lean_array_push(x_182, x_129); x_184 = lean_array_push(x_183, x_181); x_185 = lean_array_push(x_184, x_56); -x_186 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__27; +x_186 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35; x_187 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_187, 0, x_48); lean_ctor_set(x_187, 1, x_186); lean_ctor_set(x_187, 2, x_185); -x_188 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__29; +x_188 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37; x_189 = lean_array_push(x_188, x_63); x_190 = lean_array_push(x_86, x_61); if (x_66 == 0) @@ -14023,7 +14148,7 @@ x_34 = 0; x_35 = lean_usize_of_nat(x_26); lean_dec(x_26); x_36 = lean_box(0); -x_37 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_24, x_34, x_35, x_36, x_2, x_3, x_25); +x_37 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_24, x_34, x_35, x_36, x_2, x_3, x_25); lean_dec(x_24); if (lean_obj_tag(x_37) == 0) { @@ -14128,7 +14253,7 @@ x_62 = 0; x_63 = lean_usize_of_nat(x_52); lean_dec(x_52); x_64 = lean_box(0); -x_65 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_50, x_62, x_63, x_64, x_2, x_3, x_51); +x_65 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_50, x_62, x_63, x_64, x_2, x_3, x_51); lean_dec(x_50); if (lean_obj_tag(x_65) == 0) { @@ -14291,7 +14416,7 @@ x_97 = 0; x_98 = lean_usize_of_nat(x_89); lean_dec(x_89); x_99 = lean_box(0); -x_100 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_87, x_97, x_98, x_99, x_2, x_3, x_88); +x_100 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_87, x_97, x_98, x_99, x_2, x_3, x_88); lean_dec(x_87); if (lean_obj_tag(x_100) == 0) { @@ -14396,7 +14521,7 @@ x_125 = 0; x_126 = lean_usize_of_nat(x_115); lean_dec(x_115); x_127 = lean_box(0); -x_128 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_113, x_125, x_126, x_127, x_2, x_3, x_114); +x_128 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_113, x_125, x_126, x_127, x_2, x_3, x_114); lean_dec(x_113); if (lean_obj_tag(x_128) == 0) { @@ -14679,7 +14804,7 @@ lean_dec(x_2); return x_10; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__1() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__1() { _start: { lean_object* x_1; @@ -14687,7 +14812,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanc return x_1; } } -static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__2() { +static lean_object* _init_l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__2() { _start: { lean_object* x_1; @@ -14695,12 +14820,12 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInsta return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; x_2 = l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__2; -x_3 = l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__1; +x_3 = l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__1; x_4 = l_Lean_Elab_registerBuiltinDerivingHandler(x_2, x_3, x_1); if (lean_obj_tag(x_4) == 0) { @@ -14709,7 +14834,7 @@ x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); lean_dec(x_4); x_6 = l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__8; -x_7 = l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__2; +x_7 = l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__2; x_8 = l_Lean_Elab_registerBuiltinDerivingHandler(x_6, x_7, x_5); return x_8; } @@ -14964,6 +15089,22 @@ l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30 lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__30); l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31(); lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__31); +l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__32 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__32(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__32); +l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__33 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__33(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__33); +l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__34 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__34(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__34); +l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__35); +l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__36); +l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__37); +l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__38 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__38(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__38); +l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__39 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__39(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__3___closed__39); l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__1 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__1(); lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__1); l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__2 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__2(); @@ -14994,8 +15135,6 @@ l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__14 lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__14); l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__15 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__15(); lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__15); -l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__16 = _init_l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__16(); -lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkToJsonInstanceHandler___lambda__4___closed__16); l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__1 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__1(); lean_mark_persistent(l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__1); l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__2 = _init_l_Array_mapIdxM_map___at_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler_mkAlts___spec__3___closed__2(); @@ -15204,14 +15343,6 @@ l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__ lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__8); l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9(); lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__9); -l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__10 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__10); -l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__11 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__11); -l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__12 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__12); -l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13(); -lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__1___closed__13); l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__1 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__1); l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__2 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__2___closed__2(); @@ -15274,13 +15405,11 @@ l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__ lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__18); l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__19 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__19(); lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__19); -l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__20 = _init_l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__20(); -lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_mkFromJsonInstanceHandler___lambda__3___closed__20); -l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__1 = _init_l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__1(); -lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__1); -l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__2 = _init_l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__2(); -lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449____closed__2); -res = l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6449_(lean_io_mk_world()); +l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__1 = _init_l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__1(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__1); +l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__2 = _init_l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__2(); +lean_mark_persistent(l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527____closed__2); +res = l_Lean_Elab_Deriving_FromToJson_initFn____x40_Lean_Elab_Deriving_FromToJson___hyg_6527_(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/Deriving/Hashable.c b/stage0/stdlib/Lean/Elab/Deriving/Hashable.c index 81387baea286..b9502c3b257a 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/Hashable.c +++ b/stage0/stdlib/Lean/Elab/Deriving/Hashable.c @@ -41,6 +41,7 @@ static lean_object* l_Lean_Elab_Deriving_Hashable_mkAuxFunction___closed__16; lean_object* lean_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Hashable_0__Lean_Elab_Deriving_Hashable_mkHashableInstanceCmds(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); +lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Hashable_mkMatch_mkAlts___spec__4___closed__16; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Deriving_Hashable_mkMatch_mkAlts___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -135,7 +136,6 @@ lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Deriving_Hashable_0__Lean_Elab_Deriving_Hashable_mkHashableInstanceCmds___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_Deriving_Hashable_mkMatch___closed__4; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Hashable_mkMatch_mkAlts___spec__4___closed__5; -lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_Hashable_mkAuxFunction___closed__17; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Hashable_mkMatch_mkAlts___spec__4___closed__1; lean_object* l_Lean_Syntax_mkNumLit(lean_object*, lean_object*); @@ -877,7 +877,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Hashabl lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Hashable_mkMatch_mkAlts___spec__4___closed__26; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Hashable_mkMatch_mkAlts___spec__4___closed__27; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Hashable_mkMatch_mkAlts___spec__4___closed__28; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -5038,7 +5038,7 @@ x_29 = 0; x_30 = lean_usize_of_nat(x_22); lean_dec(x_22); x_31 = lean_box(0); -x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_20, x_29, x_30, x_31, x_2, x_3, x_21); +x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_20, x_29, x_30, x_31, x_2, x_3, x_21); lean_dec(x_20); if (lean_obj_tag(x_32) == 0) { @@ -5142,7 +5142,7 @@ x_56 = 0; x_57 = lean_usize_of_nat(x_47); lean_dec(x_47); x_58 = lean_box(0); -x_59 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_45, x_56, x_57, x_58, x_2, x_3, x_46); +x_59 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_45, x_56, x_57, x_58, x_2, x_3, x_46); lean_dec(x_45); if (lean_obj_tag(x_59) == 0) { diff --git a/stage0/stdlib/Lean/Elab/Deriving/Inhabited.c b/stage0/stdlib/Lean/Elab/Deriving/Inhabited.c index 3f7a9921a427..f26b8692c91f 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/Inhabited.c +++ b/stage0/stdlib/Lean/Elab/Deriving/Inhabited.c @@ -10170,7 +10170,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Derivi lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___closed__5; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___closed__6; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Deriving_Inhabited_0__Lean_Elab_mkInhabitedInstanceUsing_mkInstanceCmd_x3f___spec__1___closed__7; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/Deriving/Ord.c b/stage0/stdlib/Lean/Elab/Deriving/Ord.c index 46ac9f18c68b..ea370db7bda1 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/Ord.c +++ b/stage0/stdlib/Lean/Elab/Deriving/Ord.c @@ -48,6 +48,7 @@ static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_m lean_object* lean_environment_find(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_Ord_mkAuxFunction___lambda__1___closed__16; lean_object* lean_st_ref_get(lean_object*, lean_object*); +lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_mkAlts___spec__5___lambda__1___closed__39; static lean_object* l___private_Lean_Elab_Deriving_Ord_0__Lean_Elab_Deriving_Ord_mkOrdInstanceCmds___closed__5; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_mkAlts___spec__5___lambda__1___closed__36; @@ -157,7 +158,6 @@ lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_mkAlts___spec__7___lambda__2___closed__3; static lean_object* l___private_Lean_Elab_Deriving_Ord_0__Lean_Elab_Deriving_Ord_mkOrdInstanceCmds___closed__6; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_mkAlts___spec__5___lambda__1___closed__20; -lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_mkAlts___spec__5___lambda__1___closed__41; LEAN_EXPORT lean_object* l_Lean_Elab_Deriving_Ord_initFn____x40_Lean_Elab_Deriving_Ord___hyg_2970_(lean_object*); lean_object* l_Lean_Elab_Deriving_mkHeader(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1499,7 +1499,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkM lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_mkAlts___spec__5___closed__5; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_mkAlts___spec__5___closed__6; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Ord_mkMatch_mkAlts___spec__5___closed__7; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -5861,7 +5861,7 @@ x_29 = 0; x_30 = lean_usize_of_nat(x_22); lean_dec(x_22); x_31 = lean_box(0); -x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_20, x_29, x_30, x_31, x_2, x_3, x_21); +x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_20, x_29, x_30, x_31, x_2, x_3, x_21); lean_dec(x_20); if (lean_obj_tag(x_32) == 0) { @@ -5965,7 +5965,7 @@ x_56 = 0; x_57 = lean_usize_of_nat(x_47); lean_dec(x_47); x_58 = lean_box(0); -x_59 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_45, x_56, x_57, x_58, x_2, x_3, x_46); +x_59 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_45, x_56, x_57, x_58, x_2, x_3, x_46); lean_dec(x_45); if (lean_obj_tag(x_59) == 0) { diff --git a/stage0/stdlib/Lean/Elab/Deriving/Repr.c b/stage0/stdlib/Lean/Elab/Deriving/Repr.c index 97ae5286b6c2..d92ed34b6d01 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/Repr.c +++ b/stage0/stdlib/Lean/Elab/Deriving/Repr.c @@ -61,6 +61,7 @@ lean_object* lean_environment_find(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_Repr_mkBodyForInduct_mkAlts___spec__3___lambda__1___closed__46; lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_Repr_mkBodyForInduct_mkAlts___spec__3___lambda__1___closed__29; +lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Deriving_Repr_mkBodyForStruct___lambda__2___closed__11; static lean_object* l_List_forIn_loop___at_Lean_Elab_Deriving_Repr_mkBodyForInduct_mkAlts___spec__3___lambda__1___closed__52; static lean_object* l_Lean_Elab_Deriving_Repr_mkReprHeader___closed__27; @@ -215,7 +216,6 @@ static lean_object* l_Lean_Elab_Deriving_Repr_mkAuxFunction___lambda__1___closed static lean_object* l_Lean_Elab_Deriving_Repr_mkBodyForStruct___lambda__2___closed__5; static lean_object* l_Lean_Elab_Deriving_Repr_mkReprHeader___closed__10; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Repr_mkBodyForInduct_mkAlts___spec__2___boxed(lean_object**); -lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Deriving_Repr_mkBodyForInduct_mkAlts___spec__4(size_t, size_t, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Repr_mkBodyForInduct_mkAlts___spec__2___closed__2; lean_object* l_Lean_Elab_Deriving_mkHeader(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1843,7 +1843,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Repr_mk lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Repr_mkBodyForStruct___spec__3___closed__5; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Repr_mkBodyForStruct___spec__3___closed__6; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_Repr_mkBodyForStruct___spec__3___closed__7; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -7806,7 +7806,7 @@ x_29 = 0; x_30 = lean_usize_of_nat(x_22); lean_dec(x_22); x_31 = lean_box(0); -x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_20, x_29, x_30, x_31, x_2, x_3, x_21); +x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_20, x_29, x_30, x_31, x_2, x_3, x_21); lean_dec(x_20); if (lean_obj_tag(x_32) == 0) { @@ -7910,7 +7910,7 @@ x_56 = 0; x_57 = lean_usize_of_nat(x_47); lean_dec(x_47); x_58 = lean_box(0); -x_59 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__16(x_45, x_56, x_57, x_58, x_2, x_3, x_46); +x_59 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_elabCommand___spec__20(x_45, x_56, x_57, x_58, x_2, x_3, x_46); lean_dec(x_45); if (lean_obj_tag(x_59) == 0) { diff --git a/stage0/stdlib/Lean/Elab/Deriving/Util.c b/stage0/stdlib/Lean/Elab/Deriving/Util.c index 71a76a7ebef6..6a248b03ec5f 100644 --- a/stage0/stdlib/Lean/Elab/Deriving/Util.c +++ b/stage0/stdlib/Lean/Elab/Deriving/Util.c @@ -1109,7 +1109,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkInstI lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkInstImplicitBinders___spec__1___closed__5; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkInstImplicitBinders___spec__1___closed__6; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Deriving_mkInstImplicitBinders___spec__1___closed__7; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/Do.c b/stage0/stdlib/Lean/Elab/Do.c index 1d63ac1e0da0..17fc3c65e5f0 100644 --- a/stage0/stdlib/Lean/Elab/Do.c +++ b/stage0/stdlib/Lean/Elab/Do.c @@ -16444,7 +16444,7 @@ static lean_object* _init_l___private_Lean_Elab_Do_0__Lean_Elab_Term_Do_mkTuple_ 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_Do_0__Lean_Elab_Term_Do_mkTuple___closed__1; x_2 = l___private_Lean_Elab_Do_0__Lean_Elab_Term_Do_mkTuple___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_Do_0__Lean_Elab_Term_Do_mkTuple___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/ElabRules.c b/stage0/stdlib/Lean/Elab/ElabRules.c index dcd391730f8d..6c33d37238d9 100644 --- a/stage0/stdlib/Lean/Elab/ElabRules.c +++ b/stage0/stdlib/Lean/Elab/ElabRules.c @@ -37,7 +37,6 @@ static lean_object* l_Lean_Elab_Command_elabElabRules___lambda__7___closed__2; lean_object* l_Lean_Elab_Command_expandNoKindMacroRulesAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRules___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesAux___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* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l_Lean_Elab_Command_elabElab___lambda__1___closed__5; static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__92; @@ -159,7 +158,6 @@ lean_object* l_Lean_throwError___at_Lean_Elab_Command_resolveSyntaxKind___spec__ lean_object* l_Lean_Elab_Command_adaptExpander(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__42; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesAux___spec__5___closed__4; -lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesAux___spec__5___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabElab___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__100; @@ -196,6 +194,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Command_elabElabRules_declRange___c static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__13; static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__41; static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__88; +lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__23; size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__96; @@ -208,6 +207,7 @@ static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__6 static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__33; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabElab___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__110; +lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesAux___spec__5___lambda__2___closed__13; lean_object* l_Lean_Syntax_mkNumLit(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRules___lambda__7___closed__3; @@ -274,6 +274,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabElabRules___lambda__2(lean_obje LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Command_elabElab_declRange(lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__3; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabElab___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabElabRules___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__98; @@ -293,7 +294,6 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesA static lean_object* l_Lean_Elab_Command_elabElab___lambda__1___closed__1; static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__7; static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__71; -lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(lean_object*); static lean_object* l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__69; static lean_object* l___regBuiltin_Lean_Elab_Command_elabElabRules_declRange___closed__4; lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); @@ -1136,7 +1136,7 @@ static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElab lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesAux___spec__5___closed__9; x_2 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesAux___spec__5___closed__10; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesAux___spec__5___closed__11; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2529,7 +2529,7 @@ x_19 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabElabRulesAux___spec__5_ x_20 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__12(x_20, x_7, x_8, x_9); +x_21 = l_Lean_throwError___at_Lean_Elab_Command_elabCommand___spec__16(x_20, x_7, x_8, x_9); lean_dec(x_8); return x_21; } @@ -4217,7 +4217,7 @@ x_830 = l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__101; x_831 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_831, 0, x_829); lean_ctor_set(x_831, 1, x_830); -x_832 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__11(x_824, x_831, x_7, x_8, x_9); +x_832 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabCommand___spec__15(x_824, x_831, x_7, x_8, x_9); return x_832; } else @@ -5194,7 +5194,7 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_11); +x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_11); return x_17; } else @@ -5276,7 +5276,7 @@ lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_16 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_10); +x_16 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_10); return x_16; } else @@ -5593,7 +5593,7 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_11); +x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_11); return x_17; } else @@ -5685,7 +5685,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_16 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_10); +x_16 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_10); return x_16; } else @@ -5744,7 +5744,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_16 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_8); +x_16 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_8); return x_16; } else @@ -5771,7 +5771,7 @@ lean_dec(x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_23 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_8); +x_23 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_8); return x_23; } else @@ -5798,7 +5798,7 @@ lean_dec(x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_30 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_8); +x_30 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_8); return x_30; } else @@ -5849,7 +5849,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_43 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_8); +x_43 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_8); return x_43; } else @@ -5928,7 +5928,7 @@ lean_object* x_7; lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_4); +x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_4); return x_7; } else @@ -5950,7 +5950,7 @@ lean_dec(x_9); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_4); +x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_4); return x_13; } else @@ -5968,7 +5968,7 @@ lean_dec(x_14); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_4); +x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_4); return x_17; } else @@ -6358,7 +6358,7 @@ static lean_object* _init_l_Lean_Elab_Command_elabElab___lambda__1___closed__6() _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(9u); +x_1 = lean_unsigned_to_nat(10u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } @@ -6611,21 +6611,21 @@ lean_ctor_set(x_120, 2, x_119); if (lean_obj_tag(x_14) == 0) { x_121 = x_76; -goto block_173; +goto block_174; } else { -lean_object* x_174; lean_object* x_175; -x_174 = lean_ctor_get(x_14, 0); -lean_inc(x_174); +lean_object* x_175; lean_object* x_176; +x_175 = lean_ctor_get(x_14, 0); +lean_inc(x_175); lean_dec(x_14); -x_175 = lean_array_push(x_56, x_174); -x_121 = x_175; -goto block_173; +x_176 = lean_array_push(x_56, x_175); +x_121 = x_176; +goto block_174; } -block_173: +block_174: { -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_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; x_122 = l_Array_append___rarg(x_76, x_121); x_123 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_123, 0, x_24); @@ -6634,107 +6634,108 @@ lean_ctor_set(x_123, 2, x_122); x_124 = l_Lean_Elab_Command_elabElab___lambda__1___closed__6; lean_inc(x_123); x_125 = lean_array_push(x_124, x_123); -x_126 = lean_array_push(x_125, x_10); -x_127 = lean_array_push(x_126, x_38); -x_128 = l_Lean_Elab_Command_elabElabRules___lambda__3___closed__2; -x_129 = lean_array_push(x_128, x_123); -x_130 = lean_array_push(x_129, x_84); -x_131 = lean_array_push(x_130, x_85); -x_132 = l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__90; -x_133 = lean_array_push(x_131, x_132); -x_134 = lean_array_push(x_133, x_89); +x_126 = l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__90; +x_127 = lean_array_push(x_125, x_126); +x_128 = lean_array_push(x_127, x_10); +x_129 = lean_array_push(x_128, x_38); +x_130 = l_Lean_Elab_Command_elabElabRules___lambda__3___closed__2; +x_131 = lean_array_push(x_130, x_123); +x_132 = lean_array_push(x_131, x_84); +x_133 = lean_array_push(x_132, x_85); +x_134 = lean_array_push(x_133, x_126); +x_135 = lean_array_push(x_134, x_89); if (lean_obj_tag(x_12) == 0) { lean_dec(x_87); lean_dec(x_13); -x_135 = x_76; -goto block_166; +x_136 = x_76; +goto block_167; } else { -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; -x_167 = lean_ctor_get(x_12, 0); -lean_inc(x_167); +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_168 = lean_ctor_get(x_12, 0); +lean_inc(x_168); lean_dec(x_12); -x_168 = l_Lean_Elab_Command_elabElab___lambda__1___closed__10; -x_169 = l_Lean_Name_str___override(x_13, x_168); -x_170 = lean_array_push(x_87, x_167); -x_171 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_171, 0, x_24); -lean_ctor_set(x_171, 1, x_169); -lean_ctor_set(x_171, 2, x_170); -x_172 = lean_array_push(x_56, x_171); -x_135 = x_172; -goto block_166; -} -block_166: -{ -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_136 = l_Array_append___rarg(x_76, x_135); -x_137 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_137, 0, x_24); -lean_ctor_set(x_137, 1, x_58); -lean_ctor_set(x_137, 2, x_136); -x_138 = lean_array_push(x_127, x_137); -x_139 = lean_array_push(x_138, x_59); -x_140 = lean_array_push(x_139, x_72); -x_141 = lean_array_push(x_140, x_78); -x_142 = lean_array_push(x_141, x_80); -x_143 = lean_array_push(x_142, x_7); -x_144 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_144, 0, x_24); -lean_ctor_set(x_144, 1, x_37); -lean_ctor_set(x_144, 2, x_143); -x_145 = lean_array_push(x_86, x_144); +x_169 = l_Lean_Elab_Command_elabElab___lambda__1___closed__10; +x_170 = l_Lean_Name_str___override(x_13, x_169); +x_171 = lean_array_push(x_87, x_168); +x_172 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_172, 0, x_24); +lean_ctor_set(x_172, 1, x_170); +lean_ctor_set(x_172, 2, x_171); +x_173 = lean_array_push(x_56, x_172); +x_136 = x_173; +goto block_167; +} +block_167: +{ +lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_137 = l_Array_append___rarg(x_76, x_136); +x_138 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_138, 0, x_24); +lean_ctor_set(x_138, 1, x_58); +lean_ctor_set(x_138, 2, x_137); +x_139 = lean_array_push(x_129, x_138); +x_140 = lean_array_push(x_139, x_59); +x_141 = lean_array_push(x_140, x_72); +x_142 = lean_array_push(x_141, x_78); +x_143 = lean_array_push(x_142, x_80); +x_144 = lean_array_push(x_143, x_7); +x_145 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_145, 0, x_24); +lean_ctor_set(x_145, 1, x_37); +lean_ctor_set(x_145, 2, x_144); +x_146 = lean_array_push(x_86, x_145); if (lean_obj_tag(x_11) == 0) { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; +lean_object* x_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_dec(x_30); -x_146 = l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__59; -x_147 = lean_array_push(x_134, x_146); -x_148 = lean_array_push(x_147, x_120); -x_149 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_149, 0, x_24); -lean_ctor_set(x_149, 1, x_82); -lean_ctor_set(x_149, 2, x_148); -x_150 = lean_array_push(x_145, x_149); -x_151 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_151, 0, x_24); -lean_ctor_set(x_151, 1, x_58); -lean_ctor_set(x_151, 2, x_150); -x_152 = l_Lean_Elab_Command_elabCommand(x_151, x_16, x_17, x_35); -return x_152; +x_147 = l_Lean_Elab_Command_elabElabRulesAux___lambda__1___closed__59; +x_148 = lean_array_push(x_135, x_147); +x_149 = lean_array_push(x_148, x_120); +x_150 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_150, 0, x_24); +lean_ctor_set(x_150, 1, x_82); +lean_ctor_set(x_150, 2, x_149); +x_151 = lean_array_push(x_146, x_150); +x_152 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_152, 0, x_24); +lean_ctor_set(x_152, 1, x_58); +lean_ctor_set(x_152, 2, x_151); +x_153 = l_Lean_Elab_Command_elabCommand(x_152, x_16, x_17, x_35); +return x_153; } else { -lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -x_153 = lean_ctor_get(x_11, 0); -lean_inc(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; +x_154 = lean_ctor_get(x_11, 0); +lean_inc(x_154); lean_dec(x_11); -x_154 = l_Lean_Elab_Command_elabElabRules___lambda__3___closed__3; -x_155 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_155, 0, x_30); -lean_ctor_set(x_155, 1, x_154); -x_156 = lean_array_push(x_86, x_155); -x_157 = lean_array_push(x_156, x_153); -x_158 = l_Array_append___rarg(x_76, x_157); -x_159 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_159, 0, x_24); -lean_ctor_set(x_159, 1, x_58); -lean_ctor_set(x_159, 2, x_158); -x_160 = lean_array_push(x_134, x_159); -x_161 = lean_array_push(x_160, x_120); -x_162 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_162, 0, x_24); -lean_ctor_set(x_162, 1, x_82); -lean_ctor_set(x_162, 2, x_161); -x_163 = lean_array_push(x_145, x_162); -x_164 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_164, 0, x_24); -lean_ctor_set(x_164, 1, x_58); -lean_ctor_set(x_164, 2, x_163); -x_165 = l_Lean_Elab_Command_elabCommand(x_164, x_16, x_17, x_35); -return x_165; +x_155 = l_Lean_Elab_Command_elabElabRules___lambda__3___closed__3; +x_156 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_156, 0, x_30); +lean_ctor_set(x_156, 1, x_155); +x_157 = lean_array_push(x_86, x_156); +x_158 = lean_array_push(x_157, x_154); +x_159 = l_Array_append___rarg(x_76, x_158); +x_160 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_160, 0, x_24); +lean_ctor_set(x_160, 1, x_58); +lean_ctor_set(x_160, 2, x_159); +x_161 = lean_array_push(x_135, x_160); +x_162 = lean_array_push(x_161, x_120); +x_163 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_163, 0, x_24); +lean_ctor_set(x_163, 1, x_82); +lean_ctor_set(x_163, 2, x_162); +x_164 = lean_array_push(x_146, x_163); +x_165 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_165, 0, x_24); +lean_ctor_set(x_165, 1, x_58); +lean_ctor_set(x_165, 2, x_164); +x_166 = l_Lean_Elab_Command_elabCommand(x_165, x_16, x_17, x_35); +return x_166; } } } diff --git a/stage0/stdlib/Lean/Elab/Extra.c b/stage0/stdlib/Lean/Elab/Extra.c index 4ab54fe0d575..7efe7b68cbc2 100644 --- a/stage0/stdlib/Lean/Elab/Extra.c +++ b/stage0/stdlib/Lean/Elab/Extra.c @@ -13,9 +13,9 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty_declRange___closed__4; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__13; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__2; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_go___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp___closed__3; @@ -23,7 +23,7 @@ lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Term_elabForall__ size_t lean_usize_add(size_t, size_t); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withNewMCtxDepthImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___closed__4; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -44,8 +44,8 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___closed__32; static lean_object* l_Lean_Elab_Term_elabForIn___closed__10; static lean_object* l_Lean_Elab_Term_elabForIn___lambda__1___closed__4; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__12; static lean_object* l_Lean_Elab_Term_elabForIn___lambda__1___closed__8; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe___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_throwUnknownConstant___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_processOp___spec__1(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_Term_BinOp_elabBinCalc___spec__4___closed__16; static lean_object* l_panic___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__1___closed__1; @@ -53,16 +53,19 @@ static lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary___cl lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__2___closed__1; static lean_object* l_Lean_Elab_Term_elabForIn___closed__20; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__1; lean_object* l_Lean_Meta_mkFunUnit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_declRange___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHomogeneousInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty_declRange___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Level_succ___override(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_declRange___closed__7; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_x27___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_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_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty_declRange___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRange___closed__3; lean_object* l_Lean_Meta_mkAppM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -75,6 +78,7 @@ static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_go___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__16; static lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_declRange___closed__5; static lean_object* l_Lean_Elab_Term_elabForIn___lambda__1___closed__3; @@ -82,23 +86,23 @@ static lean_object* l_Lean_Elab_Term_elabForIn___closed__26; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasCoe___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRange___closed__6; lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__7; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree___lambda__1___closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRange___closed__1; uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_processOp___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__21; LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__8; uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__5___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty_declRange___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRange___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__3; lean_object* l_Lean_Expr_appFn_x21(lean_object*); uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__6___boxed(lean_object**); @@ -133,13 +137,11 @@ lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_obj static lean_object* l_Lean_addTrace___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__3___closed__5; uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_processOp___spec__1___closed__2; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__17; static lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__2___closed__5; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__1; extern lean_object* l_Lean_levelZero; lean_object* lean_nat_add(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___closed__19; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel_declRange___closed__3; lean_object* l_Lean_Elab_Term_ensureHasType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -161,10 +163,10 @@ static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp(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_Extra_0__Lean_Elab_Term_getMonadForIn___closed__1; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__2; lean_object* l_StateRefT_x27_lift___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_throwForInFailure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addTrace___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__3___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy_declRange(lean_object*); @@ -173,7 +175,6 @@ static lean_object* l_Lean_Elab_Term_elabForIn___closed__31; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__12; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc___closed__1; static lean_object* l_Lean_Elab_Term_elabForIn___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___closed__11; lean_object* l_Lean_Elab_Term_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -193,15 +194,15 @@ static lean_object* l_Lean_addTrace___at___private_Lean_Elab_Extra_0__Lean_Elab_ LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinCalc___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__11; lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_processOp___spec__1___closed__1; lean_object* l_Lean_Option_get___at_Std_Format_pretty_x27___spec__1(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_processOp___spec__1___closed__4; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__12; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__6; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__19; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_BinOp_elabBinCalc___closed__1; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__5; @@ -222,10 +223,13 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_ana LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___boxed(lean_object**); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp___closed__4; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__11; static lean_object* l_Lean_addTrace___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__3___closed__1; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRel(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_Term_BinOp_elabBinCalc___spec__4___closed__17; +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__8; @@ -235,13 +239,12 @@ lean_object* l_Lean_Elab_Term_elabAppArgs(lean_object*, lean_object*, lean_objec LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_relation_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn_x27___closed__4; lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__20; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__4; lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_x27_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Term_BinOp_elabBinRelCore___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp___closed__2; static lean_object* l_Lean_addTrace___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__3___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc___closed__2; @@ -263,13 +266,13 @@ lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy_declRange___closed__1; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__19; uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty(lean_object*); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___closed__6; static lean_object* l_Lean_Meta_getDefaultInstances___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_processOp___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__2; static lean_object* l_Lean_Elab_Term_elabForIn_x27___lambda__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_declRange(lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___closed__23; @@ -280,6 +283,7 @@ static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeter extern lean_object* l_Lean_instInhabitedExpr; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_processOp___closed__1; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__3; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__9; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Term_maxCoeSize; static lean_object* l_Lean_Elab_Term_elabForIn___closed__1; @@ -288,14 +292,15 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel_declRang static lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary___closed__5; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_declRange___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withNewMCtxDepth___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_initFn____x40_Lean_Elab_Extra___hyg_6573_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_initFn____x40_Lean_Elab_Extra___hyg_6912_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabForIn_x27___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_throwForInFailure___closed__2; LEAN_EXPORT uint8_t l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_isUnknow(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary___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___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe(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_Extra_0__Lean_Elab_Term_BinOp_applyCoe(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze(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_Extra_0__Lean_Elab_Term_BinOp_toTree___lambda__1___closed__2; static lean_object* l_Lean_Elab_Term_elabForIn___closed__2; @@ -320,12 +325,15 @@ lean_object* l_Lean_SimplePersistentEnvExtension_getState___rarg(lean_object*, l static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_declRange___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty___closed__3; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__4; extern lean_object* l_Lean_Elab_Term_termElabAttribute; static lean_object* l_Lean_Elab_Term_elabForIn_x27___lambda__1___closed__3; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_declRange___closed__3; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_x27(lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___closed__4; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__17; LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_x27_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRange___closed__6; @@ -338,11 +346,9 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn___closed__3; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__16; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc___closed__3; lean_object* l_Lean_Meta_trySynthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___closed__29; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -362,27 +368,31 @@ uint8_t l_Lean_Expr_hasMVar(lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__3; lean_object* l_Lean_Name_append(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty___closed__2; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__7___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabForIn_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy_declRange___closed__3; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__13; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy(lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___closed__6; static lean_object* l_Lean_Elab_Term_elabForIn_x27___lambda__1___closed__1; lean_object* l_Lean_Elab_Term_isTypeApp_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHomogeneousInstance___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_declRange___closed__5; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__15; static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_processOp___spec__1___closed__3; +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__14; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__21; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_x27_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_AnalyzeResult_max_x3f___default; lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc___closed__5; @@ -411,18 +421,15 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_has lean_object* l_Lean_Elab_Term_elabType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore_toBoolIfNecessary___closed__3; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__9; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_x27_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOpLazy(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_Extra_0__Lean_Elab_Term_BinOp_getResultingType(lean_object*); lean_object* l_Lean_Meta_mkArrow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_x27_declRange___closed__1; uint8_t l_Lean_Syntax_isNone(lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__4; lean_object* l_Lean_expandMacros(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -433,7 +440,9 @@ static lean_object* l_Lean_Elab_Term_elabForIn___closed__22; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore___lambda__3___closed__1; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__20; static lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore___lambda__3___closed__2; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__10; static lean_object* l_Lean_Elab_Term_elabForIn___closed__28; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -451,6 +460,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp(le lean_object* l_Lean_indentD(lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn___lambda__1___closed__10; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty_declRange(lean_object*); +lean_object* l_Lean_Expr_getForallBody(lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_tryPostpone(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -468,19 +478,16 @@ lean_object* l_Lean_Expr_getAppFn(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp___closed__2; static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__6; LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Term_BinOp_elabBinRelCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__18; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_go___closed__6; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__5; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__3; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__15; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__5; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__14; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_declRange(lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__14; static lean_object* l___regBuiltin_Lean_Elab_Term_elabForIn_declRange___closed__1; lean_object* l_Lean_indentExpr(lean_object*); -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_docString(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_declRange___closed__2; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_go___closed__4; @@ -490,8 +497,6 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCa LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_isLocalIdent_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_defaultInstanceExtension; -static lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___closed__6; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_getResultingType___boxed(lean_object*); static lean_object* l_Lean_Elab_Term_elabForIn_x27___closed__5; static lean_object* l_Lean_Elab_Term_elabForIn___closed__7; static lean_object* l_Lean_Elab_Term_elabForIn___lambda__1___closed__7; @@ -503,11 +508,14 @@ static lean_object* l_Lean_Elab_Term_elabForIn___closed__30; static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasCoe___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty___closed__5; static lean_object* l_Lean_Elab_Term_elabForIn___closed__5; +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__18; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__15; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRange___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasCoe___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp___closed__5; static lean_object* l_Lean_Elab_Term_elabForIn___closed__15; static lean_object* l_Lean_Elab_Term_elabForIn___closed__18; @@ -7495,7 +7503,7 @@ x_19 = l_Lean_Elab_Term_elabAppArgs(x_1, x_17, x_15, x_16, x_18, x_18, x_18, x_4 return x_19; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { if (lean_obj_tag(x_1) == 0) @@ -7537,7 +7545,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_16 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_16 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_16) == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; @@ -7552,7 +7560,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_19 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_18); +x_19 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_18); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; uint8_t x_22; @@ -7700,7 +7708,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_52 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_50, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_52 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_50, x_2, x_3, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_52) == 0) { lean_object* x_53; lean_object* x_54; lean_object* x_55; @@ -7715,7 +7723,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_55 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_51, x_2, x_3, x_4, x_5, x_6, x_7, x_54); +x_55 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_51, x_2, x_3, x_4, x_5, x_6, x_7, x_54); if (lean_obj_tag(x_55) == 0) { lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; @@ -7854,32 +7862,6 @@ return x_86; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_getResultingType(lean_object* x_1) { -_start: -{ -if (lean_obj_tag(x_1) == 7) -{ -lean_object* x_2; -x_2 = lean_ctor_get(x_1, 2); -x_1 = x_2; -goto _start; -} -else -{ -lean_inc(x_1); -return x_1; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_getResultingType___boxed(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_getResultingType(x_1); -lean_dec(x_1); -return x_2; -} -} static lean_object* _init_l_Lean_Meta_getDefaultInstances___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__1___closed__1() { _start: { @@ -7970,6 +7952,79 @@ return x_29; } } } +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__1() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 1; +x_2 = lean_box(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; +} +} +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__1; +x_2 = lean_box(0); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__2; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +if (x_1 == 0) +{ +uint8_t x_11; +x_11 = l_Lean_Expr_isAppOf(x_2, x_3); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_12, 0, x_4); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_10); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_4); +x_14 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__3; +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_10); +return x_15; +} +} +else +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_4); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_10); +return x_17; +} +} +} LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -7984,200 +8039,186 @@ return x_11; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_21; lean_object* x_22; lean_dec(x_5); x_12 = lean_ctor_get(x_4, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_4, 1); lean_inc(x_13); lean_dec(x_4); -x_14 = lean_ctor_get(x_12, 0); -lean_inc(x_14); +x_21 = lean_ctor_get(x_12, 0); +lean_inc(x_21); lean_dec(x_12); -x_15 = l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(x_14, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_15) == 0) -{ -uint8_t x_16; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +x_22 = l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(x_21, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -x_19 = l_Lean_ConstantInfo_type(x_17); -lean_dec(x_17); -x_20 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_getResultingType(x_19); -lean_dec(x_19); -x_21 = lean_unsigned_to_nat(0u); -x_22 = l_Lean_Expr_getAppNumArgsAux(x_20, x_21); -x_23 = lean_unsigned_to_nat(3u); -x_24 = lean_nat_dec_le(x_23, x_22); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); lean_dec(x_22); -if (x_24 == 0) +x_25 = l_Lean_ConstantInfo_type(x_23); +lean_dec(x_23); +x_26 = l_Lean_Expr_getForallBody(x_25); +lean_dec(x_25); +if (lean_obj_tag(x_26) == 5) { -lean_dec(x_20); -lean_free_object(x_15); -lean_inc(x_3); +lean_object* x_27; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +lean_dec(x_26); +if (lean_obj_tag(x_27) == 5) { -lean_object* _tmp_3 = x_13; -lean_object* _tmp_4 = x_3; -lean_object* _tmp_9 = x_18; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_10 = _tmp_9; -} -goto _start; -} -else +lean_object* x_28; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +if (lean_obj_tag(x_28) == 5) { -lean_dec(x_13); -lean_dec(x_3); if (x_1 == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_26 = l_Lean_Expr_appFn_x21(x_20); -lean_dec(x_20); -x_27 = l_Lean_Expr_appArg_x21(x_26); -lean_dec(x_26); -x_28 = l_Lean_Expr_appArg_x21(x_27); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_dec(x_27); -x_29 = l_Lean_Expr_isAppOf(x_28, x_2); +x_29 = lean_ctor_get(x_28, 1); +lean_inc(x_29); lean_dec(x_28); -x_30 = lean_box(x_29); -x_31 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_31, 0, x_30); -x_32 = lean_box(0); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -lean_ctor_set(x_15, 0, x_33); -return x_15; +x_30 = lean_box(0); +lean_inc(x_3); +x_31 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1(x_1, x_29, x_2, x_3, x_30, x_6, x_7, x_8, x_9, x_24); +lean_dec(x_29); +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_14 = x_32; +x_15 = x_33; +goto block_20; } else { -lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_34 = l_Lean_Expr_appFn_x21(x_20); -lean_dec(x_20); -x_35 = l_Lean_Expr_appArg_x21(x_34); +lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_34 = lean_ctor_get(x_27, 1); +lean_inc(x_34); +lean_dec(x_27); +x_35 = lean_ctor_get(x_28, 1); +lean_inc(x_35); +lean_dec(x_28); +x_36 = l_Lean_Expr_isAppOf(x_34, x_2); lean_dec(x_34); -x_36 = l_Lean_Expr_isAppOf(x_35, x_2); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = lean_box(0); +lean_inc(x_3); +x_38 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1(x_1, x_35, x_2, x_3, x_37, x_6, x_7, x_8, x_9, x_24); lean_dec(x_35); -x_37 = lean_box(x_36); -x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_37); -x_39 = lean_box(0); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -lean_ctor_set(x_15, 0, x_40); -return x_15; +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_14 = x_39; +x_15 = x_40; +goto block_20; +} +else +{ +lean_object* x_41; +lean_dec(x_35); +x_41 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__3; +x_14 = x_41; +x_15 = x_24; +goto block_20; } } } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_41 = lean_ctor_get(x_15, 0); -x_42 = lean_ctor_get(x_15, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_15); -x_43 = l_Lean_ConstantInfo_type(x_41); -lean_dec(x_41); -x_44 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_getResultingType(x_43); -lean_dec(x_43); -x_45 = lean_unsigned_to_nat(0u); -x_46 = l_Lean_Expr_getAppNumArgsAux(x_44, x_45); -x_47 = lean_unsigned_to_nat(3u); -x_48 = lean_nat_dec_le(x_47, x_46); -lean_dec(x_46); -if (x_48 == 0) +lean_object* x_42; +lean_dec(x_28); +lean_dec(x_27); +lean_inc(x_3); +x_42 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_42, 0, x_3); +x_14 = x_42; +x_15 = x_24; +goto block_20; +} +} +else { -lean_dec(x_44); +lean_object* x_43; +lean_dec(x_27); lean_inc(x_3); +x_43 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_43, 0, x_3); +x_14 = x_43; +x_15 = x_24; +goto block_20; +} +} +else { -lean_object* _tmp_3 = x_13; -lean_object* _tmp_4 = x_3; -lean_object* _tmp_9 = x_42; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_10 = _tmp_9; +lean_object* x_44; +lean_dec(x_26); +lean_inc(x_3); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_3); +x_14 = x_44; +x_15 = x_24; +goto block_20; } -goto _start; } else { +uint8_t x_45; lean_dec(x_13); lean_dec(x_3); -if (x_1 == 0) +x_45 = !lean_is_exclusive(x_22); +if (x_45 == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_50 = l_Lean_Expr_appFn_x21(x_44); -lean_dec(x_44); -x_51 = l_Lean_Expr_appArg_x21(x_50); -lean_dec(x_50); -x_52 = l_Lean_Expr_appArg_x21(x_51); -lean_dec(x_51); -x_53 = l_Lean_Expr_isAppOf(x_52, x_2); -lean_dec(x_52); -x_54 = lean_box(x_53); -x_55 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_55, 0, x_54); -x_56 = lean_box(0); -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_42); -return x_58; +return x_22; } else { -lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_59 = l_Lean_Expr_appFn_x21(x_44); -lean_dec(x_44); -x_60 = l_Lean_Expr_appArg_x21(x_59); -lean_dec(x_59); -x_61 = l_Lean_Expr_isAppOf(x_60, x_2); -lean_dec(x_60); -x_62 = lean_box(x_61); -x_63 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_63, 0, x_62); -x_64 = lean_box(0); -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -x_66 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_42); -return x_66; -} -} +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_22, 0); +x_47 = lean_ctor_get(x_22, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_22); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; } } -else +block_20: { -uint8_t x_67; +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_dec(x_13); lean_dec(x_3); -x_67 = !lean_is_exclusive(x_15); -if (x_67 == 0) -{ -return x_15; +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +return x_17; } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_15, 0); -x_69 = lean_ctor_get(x_15, 1); -lean_inc(x_69); -lean_inc(x_68); -lean_dec(x_15); -x_70 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_70, 0, x_68); -lean_ctor_set(x_70, 1, x_69); -return x_70; +lean_object* x_18; +x_18 = lean_ctor_get(x_14, 0); +lean_inc(x_18); +lean_dec(x_14); +x_4 = x_13; +x_5 = x_18; +x_10 = x_15; +goto _start; } } } @@ -8215,96 +8256,90 @@ x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_B return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___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_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = l_Lean_Meta_getDefaultInstances___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__1(x_1, x_5, x_6, x_7, x_8, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__1; -x_14 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2(x_2, x_3, x_13, x_11, x_13, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_14) == 0) +lean_object* x_10; lean_object* x_11; +x_10 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__1; +x_11 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2(x_1, x_2, x_10, x_3, x_10, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -lean_dec(x_15); -if (lean_obj_tag(x_16) == 0) +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +lean_dec(x_12); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_dec(x_14); -x_18 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__2; -x_19 = lean_box(0); -x_20 = lean_apply_6(x_18, x_19, x_5, x_6, x_7, x_8, x_17); -return x_20; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_dec(x_11); +x_15 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__2; +x_16 = lean_box(0); +x_17 = lean_apply_6(x_15, x_16, x_5, x_6, x_7, x_8, x_14); +return x_17; } else { -uint8_t x_21; +uint8_t x_18; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_21 = !lean_is_exclusive(x_14); -if (x_21 == 0) +x_18 = !lean_is_exclusive(x_11); +if (x_18 == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_14, 0); -lean_dec(x_22); -x_23 = lean_ctor_get(x_16, 0); -lean_inc(x_23); -lean_dec(x_16); -lean_ctor_set(x_14, 0, x_23); -return x_14; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_11, 0); +lean_dec(x_19); +x_20 = lean_ctor_get(x_13, 0); +lean_inc(x_20); +lean_dec(x_13); +lean_ctor_set(x_11, 0, x_20); +return x_11; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_14, 1); -lean_inc(x_24); -lean_dec(x_14); -x_25 = lean_ctor_get(x_16, 0); -lean_inc(x_25); -lean_dec(x_16); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -return x_26; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_11, 1); +lean_inc(x_21); +lean_dec(x_11); +x_22 = lean_ctor_get(x_13, 0); +lean_inc(x_22); +lean_dec(x_13); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; } } } else { -uint8_t x_27; +uint8_t x_24; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_27 = !lean_is_exclusive(x_14); -if (x_27 == 0) +x_24 = !lean_is_exclusive(x_11); +if (x_24 == 0) { -return x_14; +return x_11; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_14, 0); -x_29 = lean_ctor_get(x_14, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_14); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_11, 0); +x_26 = lean_ctor_get(x_11, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_11); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } } @@ -8329,6 +8364,7 @@ lean_dec(x_10); x_12 = l_Lean_Name_getPrefix(x_9); lean_dec(x_9); x_13 = l_Lean_Meta_getDefaultInstances___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__1(x_12, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_12); x_14 = !lean_is_exclusive(x_13); if (x_14 == 0) { @@ -8337,7 +8373,6 @@ x_15 = lean_ctor_get(x_13, 0); x_16 = lean_ctor_get(x_13, 1); x_17 = lean_unsigned_to_nat(0u); x_18 = l_List_lengthTRAux___rarg(x_15, x_17); -lean_dec(x_15); x_19 = lean_unsigned_to_nat(1u); x_20 = lean_nat_dec_le(x_18, x_19); lean_dec(x_18); @@ -8346,15 +8381,14 @@ if (x_20 == 0) lean_object* x_21; lean_object* x_22; lean_free_object(x_13); x_21 = lean_box(0); -x_22 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(x_12, x_3, x_11, x_21, x_4, x_5, x_6, x_7, x_16); +x_22 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(x_3, x_11, x_15, x_21, x_4, x_5, x_6, x_7, x_16); lean_dec(x_11); -lean_dec(x_12); return x_22; } else { uint8_t x_23; lean_object* x_24; -lean_dec(x_12); +lean_dec(x_15); lean_dec(x_11); lean_dec(x_7); lean_dec(x_6); @@ -8376,7 +8410,6 @@ lean_inc(x_25); lean_dec(x_13); x_27 = lean_unsigned_to_nat(0u); x_28 = l_List_lengthTRAux___rarg(x_25, x_27); -lean_dec(x_25); x_29 = lean_unsigned_to_nat(1u); x_30 = lean_nat_dec_le(x_28, x_29); lean_dec(x_28); @@ -8384,15 +8417,14 @@ if (x_30 == 0) { lean_object* x_31; lean_object* x_32; x_31 = lean_box(0); -x_32 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(x_12, x_3, x_11, x_31, x_4, x_5, x_6, x_7, x_26); +x_32 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(x_3, x_11, x_25, x_31, x_4, x_5, x_6, x_7, x_26); lean_dec(x_11); -lean_dec(x_12); return x_32; } else { uint8_t x_33; lean_object* x_34; lean_object* x_35; -lean_dec(x_12); +lean_dec(x_25); lean_dec(x_11); lean_dec(x_7); lean_dec(x_6); @@ -8455,6 +8487,23 @@ lean_dec(x_1); return x_7; } } +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_1); +lean_dec(x_1); +x_12 = l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +return x_12; +} +} LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -8487,12 +8536,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_has _start: { uint8_t x_10; lean_object* x_11; -x_10 = lean_unbox(x_2); -lean_dec(x_2); -x_11 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(x_1, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_4); -lean_dec(x_3); +x_10 = lean_unbox(x_1); lean_dec(x_1); +x_11 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2(x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +lean_dec(x_2); return x_11; } } @@ -8506,6 +8554,189 @@ x_10 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefau return x_10; } } +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHomogeneousInstance(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +if (lean_obj_tag(x_1) == 4) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_8 = lean_ctor_get(x_1, 0); +x_9 = l_Lean_Name_getPrefix(x_8); +x_10 = l_Lean_Elab_Term_elabForIn___lambda__1___closed__11; +lean_inc(x_2); +x_11 = lean_array_push(x_10, x_2); +lean_inc(x_2); +x_12 = lean_array_push(x_11, x_2); +x_13 = lean_array_push(x_12, x_2); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_14 = l_Lean_Meta_mkAppM(x_9, x_13, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_box(0); +x_18 = l_Lean_Meta_trySynthInstance(x_15, x_17, x_3, x_4, x_5, x_6, x_16); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +if (lean_obj_tag(x_19) == 1) +{ +uint8_t x_20; +lean_dec(x_19); +x_20 = !lean_is_exclusive(x_18); +if (x_20 == 0) +{ +lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_18, 0); +lean_dec(x_21); +x_22 = 1; +x_23 = lean_box(x_22); +lean_ctor_set(x_18, 0, x_23); +return x_18; +} +else +{ +lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_18, 1); +lean_inc(x_24); +lean_dec(x_18); +x_25 = 1; +x_26 = lean_box(x_25); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +else +{ +uint8_t x_28; +lean_dec(x_19); +x_28 = !lean_is_exclusive(x_18); +if (x_28 == 0) +{ +lean_object* x_29; uint8_t x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_18, 0); +lean_dec(x_29); +x_30 = 0; +x_31 = lean_box(x_30); +lean_ctor_set(x_18, 0, x_31); +return x_18; +} +else +{ +lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; +x_32 = lean_ctor_get(x_18, 1); +lean_inc(x_32); +lean_dec(x_18); +x_33 = 0; +x_34 = lean_box(x_33); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_32); +return x_35; +} +} +} +else +{ +uint8_t x_36; +x_36 = !lean_is_exclusive(x_18); +if (x_36 == 0) +{ +lean_object* x_37; uint8_t x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_18, 0); +lean_dec(x_37); +x_38 = 0; +x_39 = lean_box(x_38); +lean_ctor_set_tag(x_18, 0); +lean_ctor_set(x_18, 0, x_39); +return x_18; +} +else +{ +lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; +x_40 = lean_ctor_get(x_18, 1); +lean_inc(x_40); +lean_dec(x_18); +x_41 = 0; +x_42 = lean_box(x_41); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_40); +return x_43; +} +} +} +else +{ +uint8_t x_44; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_44 = !lean_is_exclusive(x_14); +if (x_44 == 0) +{ +lean_object* x_45; uint8_t x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_14, 0); +lean_dec(x_45); +x_46 = 0; +x_47 = lean_box(x_46); +lean_ctor_set_tag(x_14, 0); +lean_ctor_set(x_14, 0, x_47); +return x_14; +} +else +{ +lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; +x_48 = lean_ctor_get(x_14, 1); +lean_inc(x_48); +lean_dec(x_14); +x_49 = 0; +x_50 = lean_box(x_49); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_48); +return x_51; +} +} +} +else +{ +uint8_t x_52; lean_object* x_53; lean_object* x_54; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_52 = 0; +x_53 = lean_box(x_52); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_7); +return x_54; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHomogeneousInstance___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHomogeneousInstance(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_8; +} +} LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { @@ -9036,461 +9267,507 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { if (lean_obj_tag(x_2) == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_2, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_2, 1); +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_2, 0); lean_inc(x_13); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_13); -x_14 = lean_infer_type(x_13, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_14) == 0) +lean_inc(x_14); +x_15 = lean_infer_type(x_14, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_16); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_17); -x_20 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___closed__2; -x_43 = lean_st_ref_get(x_10, x_19); -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_44, 3); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___closed__2; +x_44 = lean_st_ref_get(x_11, x_20); +x_45 = lean_ctor_get(x_44, 0); lean_inc(x_45); -lean_dec(x_44); -x_46 = lean_ctor_get_uint8(x_45, sizeof(void*)*1); +x_46 = lean_ctor_get(x_45, 3); +lean_inc(x_46); lean_dec(x_45); -if (x_46 == 0) +x_47 = lean_ctor_get_uint8(x_46, sizeof(void*)*1); +lean_dec(x_46); +if (x_47 == 0) { -lean_object* x_47; uint8_t x_48; -x_47 = lean_ctor_get(x_43, 1); -lean_inc(x_47); -lean_dec(x_43); -x_48 = 0; -x_21 = x_48; -x_22 = x_47; -goto block_42; +lean_object* x_48; uint8_t x_49; +x_48 = lean_ctor_get(x_44, 1); +lean_inc(x_48); +lean_dec(x_44); +x_49 = 0; +x_22 = x_49; +x_23 = x_48; +goto block_43; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; -x_49 = lean_ctor_get(x_43, 1); -lean_inc(x_49); -lean_dec(x_43); -x_50 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_49); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_50 = lean_ctor_get(x_44, 1); +lean_inc(x_50); +lean_dec(x_44); +x_51 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_50); +x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -lean_dec(x_50); -x_53 = lean_unbox(x_51); +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); lean_dec(x_51); -x_21 = x_53; -x_22 = x_52; -goto block_42; +x_54 = lean_unbox(x_52); +lean_dec(x_52); +x_22 = x_54; +x_23 = x_53; +goto block_43; } -block_42: +block_43: { -if (x_21 == 0) +if (x_22 == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_box(0); -x_24 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3(x_1, x_18, x_12, x_13, x_20, x_2, x_3, x_4, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_22); -return x_24; +lean_object* x_24; lean_object* x_25; +x_24 = lean_box(0); +x_25 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3(x_1, x_19, x_13, x_14, x_21, x_2, x_3, x_4, x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_23); +return x_25; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; 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_inc(x_13); -x_25 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_25, 0, x_13); -x_26 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__2; -x_27 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_25); -x_28 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__2___closed__4; -x_29 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -lean_inc(x_18); -x_30 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_30, 0, x_18); -x_31 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -x_32 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__4; -x_33 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); +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_inc(x_14); +x_26 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_26, 0, x_14); +x_27 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__2; +x_28 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__2___closed__4; +x_30 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +lean_inc(x_19); +x_31 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_31, 0, x_19); +x_32 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__4; +x_34 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); lean_inc(x_1); -x_34 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_34, 0, x_1); -x_35 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -x_36 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; -x_37 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_20, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_22); -x_39 = lean_ctor_get(x_38, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_38, 1); +x_35 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_35, 0, x_1); +x_36 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +x_37 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; +x_38 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_21, x_38, x_6, x_7, x_8, x_9, x_10, x_11, x_23); +x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); -lean_dec(x_38); -x_41 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3(x_1, x_18, x_12, x_13, x_20, x_2, x_3, x_4, x_39, x_5, x_6, x_7, x_8, x_9, x_10, x_40); -return x_41; +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); +x_42 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3(x_1, x_19, x_13, x_14, x_21, x_2, x_3, x_4, x_40, x_6, x_7, x_8, x_9, x_10, x_11, x_41); +return x_42; } } } else { -uint8_t x_54; +uint8_t x_55; +lean_dec(x_14); lean_dec(x_13); -lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_54 = !lean_is_exclusive(x_14); -if (x_54 == 0) +x_55 = !lean_is_exclusive(x_15); +if (x_55 == 0) { -return x_14; +return x_15; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_14, 0); -x_56 = lean_ctor_get(x_14, 1); +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_15, 0); +x_57 = lean_ctor_get(x_15, 1); +lean_inc(x_57); lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_14); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -return x_57; +lean_dec(x_15); +x_58 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +return x_58; } } } else { -uint8_t x_58; +lean_object* x_59; uint8_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_dec(x_3); -x_58 = !lean_is_exclusive(x_2); -if (x_58 == 0) -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; lean_object* x_65; x_59 = lean_ctor_get(x_2, 0); -x_60 = lean_ctor_get(x_2, 1); -x_61 = lean_ctor_get(x_2, 2); -x_62 = lean_ctor_get(x_2, 3); -lean_inc(x_60); -x_63 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_63, 0, x_60); -x_64 = 1; +lean_inc(x_59); +x_60 = lean_ctor_get_uint8(x_2, sizeof(void*)*4); +x_61 = lean_ctor_get(x_2, 1); +lean_inc(x_61); +x_62 = lean_ctor_get(x_2, 2); +lean_inc(x_62); +x_63 = lean_ctor_get(x_2, 3); +lean_inc(x_63); +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + lean_ctor_release(x_2, 1); + lean_ctor_release(x_2, 2); + lean_ctor_release(x_2, 3); + x_64 = x_2; +} else { + lean_dec_ref(x_2); + x_64 = lean_box(0); +} +if (x_5 == 0) +{ +lean_object* x_117; lean_object* x_118; lean_object* x_119; uint8_t x_120; +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_63); lean_inc(x_1); -x_65 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_1, x_61, x_63, x_64, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_65) == 0) +x_117 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHomogeneousInstance(x_61, x_1, x_8, x_9, x_10, x_11, x_12); +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_117, 1); +lean_inc(x_119); +lean_dec(x_117); +x_120 = lean_unbox(x_118); +lean_dec(x_118); +x_65 = x_120; +x_66 = x_119; +goto block_116; +} +else { -lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -lean_dec(x_65); -x_68 = 0; -x_69 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_1, x_62, x_63, x_68, x_5, x_6, x_7, x_8, x_9, x_10, x_67); -if (lean_obj_tag(x_69) == 0) +x_65 = x_5; +x_66 = x_12; +goto block_116; +} +block_116: { -uint8_t x_70; -x_70 = !lean_is_exclusive(x_69); -if (x_70 == 0) +if (x_65 == 0) { -lean_object* x_71; -x_71 = lean_ctor_get(x_69, 0); -lean_ctor_set(x_2, 3, x_71); -lean_ctor_set(x_2, 2, x_66); -lean_ctor_set(x_69, 0, x_2); -return x_69; -} -else +lean_object* x_67; lean_object* x_68; +lean_dec(x_64); +lean_dec(x_1); +x_67 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_68 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_62, x_67, x_6, x_7, x_8, x_9, x_10, x_11, x_66); +if (lean_obj_tag(x_68) == 0) +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_71 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_63, x_67, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +if (lean_obj_tag(x_71) == 0) { lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_69, 0); -x_73 = lean_ctor_get(x_69, 1); -lean_inc(x_73); +x_72 = lean_ctor_get(x_71, 0); lean_inc(x_72); -lean_dec(x_69); -lean_ctor_set(x_2, 3, x_72); -lean_ctor_set(x_2, 2, x_66); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_2); -lean_ctor_set(x_74, 1, x_73); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_mkOp(x_61, x_69, x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_73); +if (lean_obj_tag(x_74) == 0) +{ +uint8_t x_75; +x_75 = !lean_is_exclusive(x_74); +if (x_75 == 0) +{ +lean_object* x_76; lean_object* x_77; +x_76 = lean_ctor_get(x_74, 0); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_59); +lean_ctor_set(x_77, 1, x_76); +lean_ctor_set(x_74, 0, x_77); return x_74; } +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_78 = lean_ctor_get(x_74, 0); +x_79 = lean_ctor_get(x_74, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_74); +x_80 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_80, 0, x_59); +lean_ctor_set(x_80, 1, x_78); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_79); +return x_81; +} } else { -uint8_t x_75; -lean_dec(x_66); -lean_free_object(x_2); -lean_dec(x_60); +uint8_t x_82; lean_dec(x_59); -x_75 = !lean_is_exclusive(x_69); -if (x_75 == 0) +x_82 = !lean_is_exclusive(x_74); +if (x_82 == 0) { -return x_69; +return x_74; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_69, 0); -x_77 = lean_ctor_get(x_69, 1); -lean_inc(x_77); -lean_inc(x_76); +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_74, 0); +x_84 = lean_ctor_get(x_74, 1); +lean_inc(x_84); +lean_inc(x_83); +lean_dec(x_74); +x_85 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +return x_85; +} +} +} +else +{ +uint8_t x_86; lean_dec(x_69); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +lean_dec(x_61); +lean_dec(x_59); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_86 = !lean_is_exclusive(x_71); +if (x_86 == 0) +{ +return x_71; +} +else +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_71, 0); +x_88 = lean_ctor_get(x_71, 1); +lean_inc(x_88); +lean_inc(x_87); +lean_dec(x_71); +x_89 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +return x_89; } } } else { -uint8_t x_79; +uint8_t x_90; lean_dec(x_63); -lean_free_object(x_2); -lean_dec(x_62); -lean_dec(x_60); +lean_dec(x_61); lean_dec(x_59); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_79 = !lean_is_exclusive(x_65); -if (x_79 == 0) +x_90 = !lean_is_exclusive(x_68); +if (x_90 == 0) { -return x_65; +return x_68; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_80 = lean_ctor_get(x_65, 0); -x_81 = lean_ctor_get(x_65, 1); -lean_inc(x_81); -lean_inc(x_80); -lean_dec(x_65); -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -return x_82; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_68, 0); +x_92 = lean_ctor_get(x_68, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_68); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +return x_93; } } } else { -lean_object* x_83; uint8_t x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; -x_83 = lean_ctor_get(x_2, 0); -x_84 = lean_ctor_get_uint8(x_2, sizeof(void*)*4); -x_85 = lean_ctor_get(x_2, 1); -x_86 = lean_ctor_get(x_2, 2); -x_87 = lean_ctor_get(x_2, 3); -lean_inc(x_87); -lean_inc(x_86); -lean_inc(x_85); -lean_inc(x_83); -lean_dec(x_2); -lean_inc(x_85); -x_88 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_88, 0, x_85); -x_89 = 1; +lean_object* x_94; uint8_t x_95; uint8_t x_96; lean_object* x_97; +lean_inc(x_61); +x_94 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_94, 0, x_61); +x_95 = 1; +x_96 = 0; +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_88); +lean_inc(x_94); lean_inc(x_1); -x_90 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_1, x_86, x_88, x_89, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_90) == 0) +x_97 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_1, x_62, x_94, x_95, x_96, x_6, x_7, x_8, x_9, x_10, x_11, x_66); +if (lean_obj_tag(x_97) == 0) { -lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; -x_91 = lean_ctor_get(x_90, 0); -lean_inc(x_91); -x_92 = lean_ctor_get(x_90, 1); -lean_inc(x_92); -lean_dec(x_90); -x_93 = 0; -x_94 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_1, x_87, x_88, x_93, x_5, x_6, x_7, x_8, x_9, x_10, x_92); -if (lean_obj_tag(x_94) == 0) +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_97, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_97, 1); +lean_inc(x_99); +lean_dec(x_97); +x_100 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_1, x_63, x_94, x_96, x_96, x_6, x_7, x_8, x_9, x_10, x_11, x_99); +if (lean_obj_tag(x_100) == 0) { -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_95 = lean_ctor_get(x_94, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_94, 1); -lean_inc(x_96); -if (lean_is_exclusive(x_94)) { - lean_ctor_release(x_94, 0); - lean_ctor_release(x_94, 1); - x_97 = x_94; -} else { - lean_dec_ref(x_94); - x_97 = lean_box(0); -} -x_98 = lean_alloc_ctor(1, 4, 1); -lean_ctor_set(x_98, 0, x_83); -lean_ctor_set(x_98, 1, x_85); -lean_ctor_set(x_98, 2, x_91); -lean_ctor_set(x_98, 3, x_95); -lean_ctor_set_uint8(x_98, sizeof(void*)*4, x_84); -if (lean_is_scalar(x_97)) { - x_99 = lean_alloc_ctor(0, 2, 0); +uint8_t x_101; +x_101 = !lean_is_exclusive(x_100); +if (x_101 == 0) +{ +lean_object* x_102; lean_object* x_103; +x_102 = lean_ctor_get(x_100, 0); +if (lean_is_scalar(x_64)) { + x_103 = lean_alloc_ctor(1, 4, 1); } else { - x_99 = x_97; + x_103 = x_64; } -lean_ctor_set(x_99, 0, x_98); -lean_ctor_set(x_99, 1, x_96); -return x_99; +lean_ctor_set(x_103, 0, x_59); +lean_ctor_set(x_103, 1, x_61); +lean_ctor_set(x_103, 2, x_98); +lean_ctor_set(x_103, 3, x_102); +lean_ctor_set_uint8(x_103, sizeof(void*)*4, x_60); +lean_ctor_set(x_100, 0, x_103); +return x_100; } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -lean_dec(x_91); -lean_dec(x_85); -lean_dec(x_83); -x_100 = lean_ctor_get(x_94, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_94, 1); -lean_inc(x_101); -if (lean_is_exclusive(x_94)) { - lean_ctor_release(x_94, 0); - lean_ctor_release(x_94, 1); - x_102 = x_94; +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_104 = lean_ctor_get(x_100, 0); +x_105 = lean_ctor_get(x_100, 1); +lean_inc(x_105); +lean_inc(x_104); +lean_dec(x_100); +if (lean_is_scalar(x_64)) { + x_106 = lean_alloc_ctor(1, 4, 1); } else { - lean_dec_ref(x_94); - x_102 = lean_box(0); + x_106 = x_64; +} +lean_ctor_set(x_106, 0, x_59); +lean_ctor_set(x_106, 1, x_61); +lean_ctor_set(x_106, 2, x_98); +lean_ctor_set(x_106, 3, x_104); +lean_ctor_set_uint8(x_106, sizeof(void*)*4, x_60); +x_107 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set(x_107, 1, x_105); +return x_107; } -if (lean_is_scalar(x_102)) { - x_103 = lean_alloc_ctor(1, 2, 0); -} else { - x_103 = x_102; } -lean_ctor_set(x_103, 0, x_100); -lean_ctor_set(x_103, 1, x_101); -return x_103; +else +{ +uint8_t x_108; +lean_dec(x_98); +lean_dec(x_64); +lean_dec(x_61); +lean_dec(x_59); +x_108 = !lean_is_exclusive(x_100); +if (x_108 == 0) +{ +return x_100; +} +else +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_109 = lean_ctor_get(x_100, 0); +x_110 = lean_ctor_get(x_100, 1); +lean_inc(x_110); +lean_inc(x_109); +lean_dec(x_100); +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 { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -lean_dec(x_88); -lean_dec(x_87); -lean_dec(x_85); -lean_dec(x_83); +uint8_t x_112; +lean_dec(x_94); +lean_dec(x_64); +lean_dec(x_63); +lean_dec(x_61); +lean_dec(x_59); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_104 = lean_ctor_get(x_90, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_90, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_90)) { - lean_ctor_release(x_90, 0); - lean_ctor_release(x_90, 1); - x_106 = x_90; -} else { - lean_dec_ref(x_90); - x_106 = lean_box(0); -} -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); -} else { - x_107 = x_106; -} -lean_ctor_set(x_107, 0, x_104); -lean_ctor_set(x_107, 1, x_105); -return x_107; -} -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +x_112 = !lean_is_exclusive(x_97); +if (x_112 == 0) { -lean_object* x_13; -x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_5); -return x_13; -} +return x_97; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +else { -uint8_t x_17; lean_object* x_18; -x_17 = lean_unbox(x_8); -lean_dec(x_8); -x_18 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_17, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -return x_18; +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_97, 0); +x_114 = lean_ctor_get(x_97, 1); +lean_inc(x_114); +lean_inc(x_113); +lean_dec(x_97); +x_115 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_115, 0, x_113); +lean_ctor_set(x_115, 1, x_114); +return x_115; +} } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; lean_object* x_13; -x_12 = lean_unbox(x_4); -lean_dec(x_4); -x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_1, x_2, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_13; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; uint8_t x_11; lean_object* x_12; -x_10 = lean_box(0); -x_11 = 0; -x_12 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_2, x_1, x_10, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; @@ -9499,7 +9776,7 @@ x_12 = l_Lean_Elab_Term_ensureHasType(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x return x_12; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -9507,16 +9784,16 @@ x_1 = lean_mk_string_from_bytes("result: ", 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__1; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; @@ -9538,7 +9815,7 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_15 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_15) == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; @@ -9583,65 +9860,65 @@ return x_23; } else { -lean_object* x_24; lean_object* x_25; +lean_object* x_24; uint8_t x_25; lean_object* x_26; x_24 = lean_ctor_get(x_14, 0); lean_inc(x_24); lean_dec(x_14); +x_25 = 0; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_25 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe(x_2, x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_25) == 0) +x_26 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe(x_2, x_24, x_25, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -lean_dec(x_25); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_28 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_27); -if (lean_obj_tag(x_28) == 0) +x_29 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_27, x_6, x_7, x_8, x_9, x_10, x_11, x_28); +if (lean_obj_tag(x_29) == 0) { -lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); +lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); -lean_dec(x_28); -x_45 = lean_st_ref_get(x_11, x_30); -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_46, 3); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_46 = lean_st_ref_get(x_11, x_31); +x_47 = lean_ctor_get(x_46, 0); lean_inc(x_47); -lean_dec(x_46); -x_48 = lean_ctor_get_uint8(x_47, sizeof(void*)*1); +x_48 = lean_ctor_get(x_47, 3); +lean_inc(x_48); lean_dec(x_47); -if (x_48 == 0) +x_49 = lean_ctor_get_uint8(x_48, sizeof(void*)*1); +lean_dec(x_48); +if (x_49 == 0) { -lean_object* x_49; uint8_t x_50; -x_49 = lean_ctor_get(x_45, 1); -lean_inc(x_49); -lean_dec(x_45); -x_50 = 0; -x_31 = x_50; -x_32 = x_49; -goto block_44; +lean_object* x_50; +x_50 = lean_ctor_get(x_46, 1); +lean_inc(x_50); +lean_dec(x_46); +x_32 = x_25; +x_33 = x_50; +goto block_45; } else { lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_51 = lean_ctor_get(x_45, 1); +x_51 = lean_ctor_get(x_46, 1); lean_inc(x_51); -lean_dec(x_45); +lean_dec(x_46); lean_inc(x_4); x_52 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_4, x_6, x_7, x_8, x_9, x_10, x_11, x_51); x_53 = lean_ctor_get(x_52, 0); @@ -9651,43 +9928,43 @@ lean_inc(x_54); lean_dec(x_52); x_55 = lean_unbox(x_53); lean_dec(x_53); -x_31 = x_55; -x_32 = x_54; -goto block_44; +x_32 = x_55; +x_33 = x_54; +goto block_45; } -block_44: +block_45: { -if (x_31 == 0) +if (x_32 == 0) { -lean_object* x_33; lean_object* x_34; +lean_object* x_34; lean_object* x_35; lean_dec(x_4); -x_33 = lean_box(0); -x_34 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__1(x_3, x_29, x_33, x_6, x_7, x_8, x_9, x_10, x_11, x_32); -return x_34; +x_34 = lean_box(0); +x_35 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__1(x_3, x_30, x_34, x_6, x_7, x_8, x_9, x_10, x_11, x_33); +return x_35; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -lean_inc(x_29); -x_35 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_35, 0, x_29); -x_36 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__2; -x_37 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_35); -x_38 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; -x_39 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -x_40 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_4, x_39, x_6, x_7, x_8, x_9, x_10, x_11, x_32); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_inc(x_30); +x_36 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_36, 0, x_30); +x_37 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__2; +x_38 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +x_39 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; +x_40 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_4, x_40, x_6, x_7, x_8, x_9, x_10, x_11, x_33); +x_42 = lean_ctor_get(x_41, 0); lean_inc(x_42); -lean_dec(x_40); -x_43 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__1(x_3, x_29, x_41, x_6, x_7, x_8, x_9, x_10, x_11, x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); lean_dec(x_41); -return x_43; +x_44 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__1(x_3, x_30, x_42, x_6, x_7, x_8, x_9, x_10, x_11, x_43); +lean_dec(x_42); +return x_44; } } } @@ -9702,19 +9979,19 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); -x_56 = !lean_is_exclusive(x_28); +x_56 = !lean_is_exclusive(x_29); if (x_56 == 0) { -return x_28; +return x_29; } else { lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_28, 0); -x_58 = lean_ctor_get(x_28, 1); +x_57 = lean_ctor_get(x_29, 0); +x_58 = lean_ctor_get(x_29, 1); lean_inc(x_58); lean_inc(x_57); -lean_dec(x_28); +lean_dec(x_29); x_59 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_59, 0, x_57); lean_ctor_set(x_59, 1, x_58); @@ -9733,19 +10010,19 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); -x_60 = !lean_is_exclusive(x_25); +x_60 = !lean_is_exclusive(x_26); if (x_60 == 0) { -return x_25; +return x_26; } else { lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_25, 0); -x_62 = lean_ctor_get(x_25, 1); +x_61 = lean_ctor_get(x_26, 0); +x_62 = lean_ctor_get(x_26, 1); lean_inc(x_62); lean_inc(x_61); -lean_dec(x_25); +lean_dec(x_26); x_63 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_63, 0, x_61); lean_ctor_set(x_63, 1, x_62); @@ -9765,7 +10042,7 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_64 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_64 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_64) == 0) { lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; @@ -9810,7 +10087,7 @@ return x_72; } } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__1() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__1() { _start: { lean_object* x_1; @@ -9818,16 +10095,16 @@ x_1 = lean_mk_string_from_bytes("hasUncomparable: ", 17); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__2() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__1; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__3() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__3() { _start: { lean_object* x_1; @@ -9835,16 +10112,16 @@ x_1 = lean_mk_string_from_bytes(", maxType: ", 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__4() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__3; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__5() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__5() { _start: { lean_object* x_1; @@ -9852,51 +10129,51 @@ x_1 = lean_mk_string_from_bytes("false", 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__6() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__5; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__5; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__7() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__6; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__6; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__8() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__2; -x_2 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__7; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__2; +x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__7; x_3 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__9() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__8; -x_2 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__4; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__8; +x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__4; x_3 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__10() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__10() { _start: { lean_object* x_1; @@ -9904,43 +10181,43 @@ x_1 = lean_mk_string_from_bytes("", 15); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__11() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__10; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__10; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__12() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__11; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__11; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__13() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__9; -x_2 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__12; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__9; +x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__12; x_3 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__14() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__13; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__13; x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; x_3 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9948,7 +10225,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__15() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__15() { _start: { lean_object* x_1; @@ -9956,67 +10233,67 @@ x_1 = lean_mk_string_from_bytes("true", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__16() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__15; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__15; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__17() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__17() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__16; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__16; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__18() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__2; -x_2 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__17; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__2; +x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__17; x_3 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__19() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__18; -x_2 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__4; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__18; +x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__4; x_3 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__20() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__19; -x_2 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__12; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__19; +x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__12; x_3 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__21() { +static lean_object* _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__20; +x_1 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__20; x_2 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; x_3 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10024,7 +10301,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; @@ -10034,169 +10311,154 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_10 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_inc(x_2); +lean_inc(x_1); +x_10 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_10) == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_11); -x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_13) == 0) +x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___closed__2; +x_52 = lean_st_ref_get(x_8, x_12); +x_53 = lean_ctor_get(x_52, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_53, 3); +lean_inc(x_54); +lean_dec(x_53); +x_55 = lean_ctor_get_uint8(x_54, sizeof(void*)*1); +lean_dec(x_54); +if (x_55 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___closed__2; -x_55 = lean_st_ref_get(x_8, x_15); -x_56 = lean_ctor_get(x_55, 0); +lean_object* x_56; uint8_t x_57; +x_56 = lean_ctor_get(x_52, 1); lean_inc(x_56); -x_57 = lean_ctor_get(x_56, 3); -lean_inc(x_57); -lean_dec(x_56); -x_58 = lean_ctor_get_uint8(x_57, sizeof(void*)*1); -lean_dec(x_57); -if (x_58 == 0) -{ -lean_object* x_59; uint8_t x_60; -x_59 = lean_ctor_get(x_55, 1); -lean_inc(x_59); -lean_dec(x_55); -x_60 = 0; -x_17 = x_60; -x_18 = x_59; -goto block_54; +lean_dec(x_52); +x_57 = 0; +x_14 = x_57; +x_15 = x_56; +goto block_51; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; -x_61 = lean_ctor_get(x_55, 1); +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_58 = lean_ctor_get(x_52, 1); +lean_inc(x_58); +lean_dec(x_52); +x_59 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_58); +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); lean_inc(x_61); -lean_dec(x_55); -x_62 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_61); -x_63 = lean_ctor_get(x_62, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_62, 1); -lean_inc(x_64); -lean_dec(x_62); -x_65 = lean_unbox(x_63); -lean_dec(x_63); -x_17 = x_65; -x_18 = x_64; -goto block_54; +lean_dec(x_59); +x_62 = lean_unbox(x_60); +lean_dec(x_60); +x_14 = x_62; +x_15 = x_61; +goto block_51; } -block_54: +block_51: { -if (x_17 == 0) +if (x_14 == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_box(0); -x_20 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2(x_14, x_11, x_2, x_16, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -return x_20; +lean_object* x_16; lean_object* x_17; +x_16 = lean_box(0); +x_17 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2(x_11, x_1, x_2, x_13, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_15); +return x_17; } else { -uint8_t x_21; -x_21 = lean_ctor_get_uint8(x_14, sizeof(void*)*1); -if (x_21 == 0) +uint8_t x_18; +x_18 = lean_ctor_get_uint8(x_11, sizeof(void*)*1); +if (x_18 == 0) { -lean_object* x_22; -x_22 = lean_ctor_get(x_14, 0); -lean_inc(x_22); -if (lean_obj_tag(x_22) == 0) +lean_object* x_19; +x_19 = lean_ctor_get(x_11, 0); +lean_inc(x_19); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_23 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__14; -x_24 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_16, x_23, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2(x_14, x_11, x_2, x_16, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_26); -return x_27; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_20 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__14; +x_21 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_13, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_15); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2(x_11, x_1, x_2, x_13, x_22, x_3, x_4, x_5, x_6, x_7, x_8, x_23); +return x_24; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_28 = lean_ctor_get(x_22, 0); -lean_inc(x_28); -lean_dec(x_22); -x_29 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_29, 0, x_28); -x_30 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__9; -x_31 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_29); -x_32 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; -x_33 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -x_34 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_16, x_33, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2(x_14, x_11, x_2, x_16, x_35, x_3, x_4, x_5, x_6, x_7, x_8, x_36); -return x_37; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_25 = lean_ctor_get(x_19, 0); +lean_inc(x_25); +lean_dec(x_19); +x_26 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_27 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__9; +x_28 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; +x_30 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_13, x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_15); +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___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2(x_11, x_1, x_2, x_13, x_32, x_3, x_4, x_5, x_6, x_7, x_8, x_33); +return x_34; } } else { -lean_object* x_38; -x_38 = lean_ctor_get(x_14, 0); -lean_inc(x_38); -if (lean_obj_tag(x_38) == 0) +lean_object* x_35; +x_35 = lean_ctor_get(x_11, 0); +lean_inc(x_35); +if (lean_obj_tag(x_35) == 0) { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_39 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__21; -x_40 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_16, x_39, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); -x_43 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2(x_14, x_11, x_2, x_16, x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_42); -return x_43; +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_36 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__21; +x_37 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_13, x_36, x_3, x_4, x_5, x_6, x_7, x_8, x_15); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2(x_11, x_1, x_2, x_13, x_38, x_3, x_4, x_5, x_6, x_7, x_8, x_39); +return x_40; } -else -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_44 = lean_ctor_get(x_38, 0); -lean_inc(x_44); -lean_dec(x_38); -x_45 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_45, 0, x_44); -x_46 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__19; -x_47 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_45); -x_48 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; -x_49 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); -x_50 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_16, x_49, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -lean_dec(x_50); -x_53 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2(x_14, x_11, x_2, x_16, x_51, x_3, x_4, x_5, x_6, x_7, x_8, x_52); -return x_53; +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_41 = lean_ctor_get(x_35, 0); +lean_inc(x_41); +lean_dec(x_35); +x_42 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_42, 0, x_41); +x_43 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__19; +x_44 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_42); +x_45 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; +x_46 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +x_47 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_13, x_46, x_3, x_4, x_5, x_6, x_7, x_8, x_15); +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2(x_11, x_1, x_2, x_13, x_48, x_3, x_4, x_5, x_6, x_7, x_8, x_49); +return x_50; } } } @@ -10204,8 +10466,7 @@ return x_53; } else { -uint8_t x_66; -lean_dec(x_11); +uint8_t x_63; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -10213,29 +10474,113 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_66 = !lean_is_exclusive(x_13); -if (x_66 == 0) +lean_dec(x_1); +x_63 = !lean_is_exclusive(x_10); +if (x_63 == 0) { -return x_13; +return x_10; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_13, 0); -x_68 = lean_ctor_get(x_13, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_13); -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_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_10, 0); +x_65 = lean_ctor_get(x_10, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_10); +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +return x_66; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; lean_object* x_13; +x_11 = lean_box(0); +x_12 = 0; +x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_2, x_1, x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_5); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +uint8_t x_17; lean_object* x_18; +x_17 = lean_unbox(x_8); +lean_dec(x_8); +x_18 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_17, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +return x_18; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_13 = lean_unbox(x_4); +lean_dec(x_4); +x_14 = lean_unbox(x_5); +lean_dec(x_5); +x_15 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go(x_1, x_2, x_3, x_13, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_3); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_3); +lean_dec(x_3); +x_12 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_10 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toTree(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_13; } else { -uint8_t x_70; +uint8_t x_14; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -10243,34 +10588,25 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_70 = !lean_is_exclusive(x_10); -if (x_70 == 0) +x_14 = !lean_is_exclusive(x_10); +if (x_14 == 0) { return x_10; } else { -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_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); +lean_inc(x_15); lean_dec(x_10); -x_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; -} -} +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinOp___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_3); -return x_11; } } static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp___closed__1() { @@ -10333,7 +10669,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRang _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(332u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10345,8 +10681,8 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(307u); -x_2 = lean_unsigned_to_nat(38u); +x_1 = lean_unsigned_to_nat(333u); +x_2 = lean_unsigned_to_nat(37u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -10360,7 +10696,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRange___closed__1; x_2 = lean_unsigned_to_nat(0u); x_3 = l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRange___closed__2; -x_4 = lean_unsigned_to_nat(38u); +x_4 = lean_unsigned_to_nat(37u); x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -10373,7 +10709,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRang _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(332u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10385,7 +10721,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp_declRang _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(332u); x_2 = lean_unsigned_to_nat(13u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10481,7 +10817,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(310u); +x_1 = lean_unsigned_to_nat(336u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10493,7 +10829,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(310u); +x_1 = lean_unsigned_to_nat(336u); x_2 = lean_unsigned_to_nat(41u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10521,7 +10857,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(310u); +x_1 = lean_unsigned_to_nat(336u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10533,7 +10869,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOpLazy_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(310u); +x_1 = lean_unsigned_to_nat(336u); x_2 = lean_unsigned_to_nat(17u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10961,87 +11297,88 @@ return x_16; LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_elabBinRelCore___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; +uint8_t x_12; lean_object* x_13; +x_12 = 1; lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_12 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe(x_1, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_12) == 0) +x_13 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe(x_1, x_3, x_12, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -lean_dec(x_12); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_15 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_14); -if (lean_obj_tag(x_15) == 0) +x_16 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -if (lean_is_exclusive(x_15)) { - lean_ctor_release(x_15, 0); - lean_ctor_release(x_15, 1); - x_18 = x_15; +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +if (lean_is_exclusive(x_16)) { + lean_ctor_release(x_16, 0); + lean_ctor_release(x_16, 1); + x_19 = x_16; } else { - lean_dec_ref(x_15); - x_18 = lean_box(0); + lean_dec_ref(x_16); + x_19 = lean_box(0); } -x_33 = lean_st_ref_get(x_10, x_17); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_34, 3); +x_34 = lean_st_ref_get(x_10, x_18); +x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); -lean_dec(x_34); -x_36 = lean_ctor_get_uint8(x_35, sizeof(void*)*1); +x_36 = lean_ctor_get(x_35, 3); +lean_inc(x_36); lean_dec(x_35); -if (x_36 == 0) +x_37 = lean_ctor_get_uint8(x_36, sizeof(void*)*1); +lean_dec(x_36); +if (x_37 == 0) { -lean_object* x_37; uint8_t x_38; -x_37 = lean_ctor_get(x_33, 1); -lean_inc(x_37); -lean_dec(x_33); -x_38 = 0; -x_19 = x_38; -x_20 = x_37; -goto block_32; +lean_object* x_38; uint8_t x_39; +x_38 = lean_ctor_get(x_34, 1); +lean_inc(x_38); +lean_dec(x_34); +x_39 = 0; +x_20 = x_39; +x_21 = x_38; +goto block_33; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_39 = lean_ctor_get(x_33, 1); -lean_inc(x_39); -lean_dec(x_33); +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_40 = lean_ctor_get(x_34, 1); +lean_inc(x_40); +lean_dec(x_34); lean_inc(x_2); -x_40 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_39); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); +x_41 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_40); +x_42 = lean_ctor_get(x_41, 0); lean_inc(x_42); -lean_dec(x_40); -x_43 = lean_unbox(x_41); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); lean_dec(x_41); -x_19 = x_43; -x_20 = x_42; -goto block_32; +x_44 = lean_unbox(x_42); +lean_dec(x_42); +x_20 = x_44; +x_21 = x_43; +goto block_33; } -block_32: +block_33: { -if (x_19 == 0) +if (x_20 == 0) { -lean_object* x_21; +lean_object* x_22; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -11049,63 +11386,63 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -if (lean_is_scalar(x_18)) { - x_21 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_19)) { + x_22 = lean_alloc_ctor(0, 2, 0); } else { - x_21 = x_18; + x_22 = x_19; } -lean_ctor_set(x_21, 0, x_16); -lean_ctor_set(x_21, 1, x_20); -return x_21; +lean_ctor_set(x_22, 0, x_17); +lean_ctor_set(x_22, 1, x_21); +return x_22; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -lean_dec(x_18); -lean_inc(x_16); -x_22 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_22, 0, x_16); -x_23 = l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__2; -x_24 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_22); -x_25 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; -x_26 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -x_27 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_2, x_26, x_5, x_6, x_7, x_8, x_9, x_10, x_20); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +lean_dec(x_19); +lean_inc(x_17); +x_23 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_23, 0, x_17); +x_24 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__2; +x_25 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +x_26 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_getMonadForIn___closed__6; +x_27 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_2, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_21); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) { -lean_object* x_29; -x_29 = lean_ctor_get(x_27, 0); -lean_dec(x_29); -lean_ctor_set(x_27, 0, x_16); -return x_27; +lean_object* x_30; +x_30 = lean_ctor_get(x_28, 0); +lean_dec(x_30); +lean_ctor_set(x_28, 0, x_17); +return x_28; } else { -lean_object* x_30; lean_object* x_31; -x_30 = lean_ctor_get(x_27, 1); -lean_inc(x_30); -lean_dec(x_27); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_16); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_28, 1); +lean_inc(x_31); +lean_dec(x_28); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_17); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } } } else { -uint8_t x_44; +uint8_t x_45; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -11113,29 +11450,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_44 = !lean_is_exclusive(x_15); -if (x_44 == 0) +x_45 = !lean_is_exclusive(x_16); +if (x_45 == 0) { -return x_15; +return x_16; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_15, 0); -x_46 = lean_ctor_get(x_15, 1); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_16, 0); +x_47 = lean_ctor_get(x_16, 1); +lean_inc(x_47); lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_15); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; +lean_dec(x_16); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; } } } else { -uint8_t x_48; +uint8_t x_49; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -11143,23 +11480,23 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_48 = !lean_is_exclusive(x_12); -if (x_48 == 0) +x_49 = !lean_is_exclusive(x_13); +if (x_49 == 0) { -return x_12; +return x_13; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_12, 0); -x_50 = lean_ctor_get(x_12, 1); +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_13, 0); +x_51 = lean_ctor_get(x_13, 1); +lean_inc(x_51); lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_12); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +lean_dec(x_13); +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; } } } @@ -11304,7 +11641,7 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -x_19 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_19 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; @@ -11319,7 +11656,7 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -x_22 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr(x_2, x_11, x_12, x_13, x_14, x_15, x_16, x_21); +x_22 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExprCore(x_2, x_11, x_12, x_13, x_14, x_15, x_16, x_21); if (lean_obj_tag(x_22) == 0) { lean_object* x_23; lean_object* x_24; lean_object* x_25; @@ -11797,7 +12134,7 @@ lean_inc(x_48); if (lean_obj_tag(x_48) == 0) { lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_49 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__14; +x_49 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__14; x_50 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_42, x_49, x_6, x_7, x_8, x_9, x_10, x_11, x_44); x_51 = lean_ctor_get(x_50, 0); lean_inc(x_51); @@ -11815,7 +12152,7 @@ lean_inc(x_54); lean_dec(x_48); x_55 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_55, 0, x_54); -x_56 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__9; +x_56 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__9; x_57 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_57, 0, x_56); lean_ctor_set(x_57, 1, x_55); @@ -11841,7 +12178,7 @@ lean_inc(x_64); if (lean_obj_tag(x_64) == 0) { lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_65 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__21; +x_65 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__21; x_66 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_42, x_65, x_6, x_7, x_8, x_9, x_10, x_11, x_44); x_67 = lean_ctor_get(x_66, 0); lean_inc(x_67); @@ -11859,7 +12196,7 @@ lean_inc(x_70); lean_dec(x_64); x_71 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_71, 0, x_70); -x_72 = l_Lean_Elab_Term_BinOp_elabBinOp___closed__19; +x_72 = l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__19; x_73 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_73, 0, x_72); lean_ctor_set(x_73, 1, x_71); @@ -12217,7 +12554,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(356u); +x_1 = lean_unsigned_to_nat(382u); x_2 = lean_unsigned_to_nat(26u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12229,7 +12566,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(356u); +x_1 = lean_unsigned_to_nat(382u); x_2 = lean_unsigned_to_nat(75u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12257,7 +12594,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(356u); +x_1 = lean_unsigned_to_nat(382u); x_2 = lean_unsigned_to_nat(30u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12269,7 +12606,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRel_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(356u); +x_1 = lean_unsigned_to_nat(382u); x_2 = lean_unsigned_to_nat(40u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12384,7 +12721,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(358u); +x_1 = lean_unsigned_to_nat(384u); x_2 = lean_unsigned_to_nat(34u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12396,7 +12733,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(358u); +x_1 = lean_unsigned_to_nat(384u); x_2 = lean_unsigned_to_nat(88u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12424,7 +12761,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(358u); +x_1 = lean_unsigned_to_nat(384u); x_2 = lean_unsigned_to_nat(38u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12436,7 +12773,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinRelNoProp_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(358u); +x_1 = lean_unsigned_to_nat(384u); x_2 = lean_unsigned_to_nat(54u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12487,7 +12824,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_rel { lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Lean_Expr_getAppNumArgsAux(x_1, x_7); +x_8 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_7); x_9 = lean_unsigned_to_nat(2u); x_10 = lean_nat_dec_lt(x_8, x_9); lean_dec(x_8); @@ -12724,7 +13061,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_ela lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__3; x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__4; -x_3 = lean_unsigned_to_nat(391u); +x_3 = lean_unsigned_to_nat(417u); x_4 = lean_unsigned_to_nat(56u); x_5 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -13412,7 +13749,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabB lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__3; x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__4; -x_3 = lean_unsigned_to_nat(401u); +x_3 = lean_unsigned_to_nat(427u); x_4 = lean_unsigned_to_nat(48u); x_5 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -13425,7 +13762,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabB lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__3; x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__4; -x_3 = lean_unsigned_to_nat(402u); +x_3 = lean_unsigned_to_nat(428u); x_4 = lean_unsigned_to_nat(68u); x_5 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__2___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -13514,7 +13851,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabB lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__9; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__10; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Term_BinOp_elabBinCalc___spec__4___closed__11; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -22008,7 +22345,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRa _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(382u); +x_1 = lean_unsigned_to_nat(408u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -22020,7 +22357,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRa _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(415u); +x_1 = lean_unsigned_to_nat(441u); x_2 = lean_unsigned_to_nat(36u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -22048,7 +22385,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRa _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(382u); +x_1 = lean_unsigned_to_nat(408u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -22060,7 +22397,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinCalc_declRa _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(382u); +x_1 = lean_unsigned_to_nat(408u); x_2 = lean_unsigned_to_nat(15u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -22369,7 +22706,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonem _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(444u); x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -22381,7 +22718,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonem _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(459u); x_2 = lean_unsigned_to_nat(34u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -22409,7 +22746,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonem _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(444u); x_2 = lean_unsigned_to_nat(4u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -22421,7 +22758,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonem _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(444u); x_2 = lean_unsigned_to_nat(25u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -22467,7 +22804,7 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_initFn____x40_Lean_Elab_Extra___hyg_6573_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_BinOp_initFn____x40_Lean_Elab_Extra___hyg_6912_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -22771,6 +23108,12 @@ l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___closed__7 = _in lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_analyze_go___closed__7); l_Lean_Meta_getDefaultInstances___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__1___closed__1 = _init_l_Lean_Meta_getDefaultInstances___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__1___closed__1(); lean_mark_persistent(l_Lean_Meta_getDefaultInstances___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__1___closed__1); +l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__1 = _init_l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__1(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__1); +l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__2 = _init_l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__2(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__2); +l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__3 = _init_l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__3(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___spec__2___lambda__1___closed__3); l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__1 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__1); l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__2 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_hasHeterogeneousDefaultInstances___lambda__2___closed__2(); @@ -22795,52 +23138,52 @@ l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__3 = _i lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__3); l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__4 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__4(); lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_applyCoe_go___closed__4); -l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__1 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__1); -l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__2 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___lambda__2___closed__2); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__1 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__1); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__2 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__2); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__3 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__3); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__4 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__4); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__5 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__5); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__6 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__6); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__7 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__7); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__8 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__8); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__9 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__9); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__10 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__10(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__10); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__11 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__11(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__11); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__12 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__12(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__12); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__13 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__13(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__13); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__14 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__14(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__14); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__15 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__15(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__15); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__16 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__16(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__16); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__17 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__17(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__17); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__18 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__18(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__18); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__19 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__19(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__19); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__20 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__20(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__20); -l_Lean_Elab_Term_BinOp_elabBinOp___closed__21 = _init_l_Lean_Elab_Term_BinOp_elabBinOp___closed__21(); -lean_mark_persistent(l_Lean_Elab_Term_BinOp_elabBinOp___closed__21); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__1 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__1); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__2 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___lambda__2___closed__2); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__1 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__1); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__2 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__2(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__2); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__3 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__3(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__3); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__4 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__4(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__4); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__5 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__5(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__5); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__6 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__6(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__6); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__7 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__7(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__7); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__8 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__8(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__8); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__9 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__9(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__9); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__10 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__10(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__10); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__11 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__11(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__11); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__12 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__12(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__12); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__13 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__13(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__13); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__14 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__14(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__14); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__15 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__15(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__15); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__16 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__16(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__16); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__17 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__17(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__17); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__18 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__18(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__18); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__19 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__19(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__19); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__20 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__20(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__20); +l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__21 = _init_l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__21(); +lean_mark_persistent(l___private_Lean_Elab_Extra_0__Lean_Elab_Term_BinOp_toExpr___closed__21); l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp___closed__1 = _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp___closed__1); l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp___closed__2 = _init_l___regBuiltin_Lean_Elab_Term_BinOp_elabBinOp___closed__2(); @@ -23096,7 +23439,7 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty_d res = l___regBuiltin_Lean_Elab_Term_BinOp_elabDefaultOrNonempty_declRange(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = l_Lean_Elab_Term_BinOp_initFn____x40_Lean_Elab_Extra___hyg_6573_(lean_io_mk_world()); +res = l_Lean_Elab_Term_BinOp_initFn____x40_Lean_Elab_Extra___hyg_6912_(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/Frontend.c b/stage0/stdlib/Lean/Elab/Frontend.c index b48a1a33029f..ce9c31713d1c 100644 --- a/stage0/stdlib/Lean/Elab/Frontend.c +++ b/stage0/stdlib/Lean/Elab/Frontend.c @@ -77,7 +77,7 @@ static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Frontend___hyg_828____cl static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Frontend___hyg_828____closed__2; lean_object* l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_Elab_Frontend_processCommand___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t); +lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_elabCommandAtFrontend___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Parser_isExitCommand(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Frontend_getInputContext(lean_object*, lean_object*, lean_object*); @@ -2368,7 +2368,7 @@ lean_dec(x_16); x_25 = l_Std_PersistentArray_toArray___rarg(x_24); x_26 = l_Lean_FileMap_ofString(x_5); x_27 = 0; -x_28 = l_Lean_Server_findModuleRefs(x_26, x_25, x_27); +x_28 = l_Lean_Server_findModuleRefs(x_26, x_25, x_27, x_27); lean_dec(x_25); x_29 = l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(x_28); x_30 = lean_box(0); diff --git a/stage0/stdlib/Lean/Elab/Inductive.c b/stage0/stdlib/Lean/Elab/Inductive.c index 1a18b675ea10..75a07ec03ea2 100644 --- a/stage0/stdlib/Lean/Elab/Inductive.c +++ b/stage0/stdlib/Lean/Elab/Inductive.c @@ -95,6 +95,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_instInhabitedElabHeaderResult; LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___rarg___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_getResultingUniverse___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Level_succ___override(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__4___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_assignLevelMVar___at_Lean_Elab_Command_accLevelAtCtor___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__8; @@ -292,6 +293,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews___lambda__4___bo LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_levelMVarToParam___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___closed__15; lean_object* l_Lean_mkAppN(lean_object*, lean_object*); +lean_object* l_Lean_simpLevelIMax_x27(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkParamsAndResultType___closed__2; static lean_object* l_List_mapTRAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -382,18 +384,19 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0_ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams(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_Inductive_0__Lean_Elab_Command_throwUnexpectedInductiveType___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_level_update_max(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_ComputedFields_setComputedFields(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabInductiveViews(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_markUsedAssignment___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_simpLevelMax_x27(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_checkParamOccs___spec__1___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__8(uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_isInductiveFamily(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -409,6 +412,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapTRAux___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__7___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__8___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__9___closed__5; static lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___closed__1; +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectLevelParamsInInductive___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_withUsed(lean_object*); @@ -420,6 +424,7 @@ static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCto LEAN_EXPORT lean_object* l_Lean_Elab_Command_accLevelAtCtor___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__9; static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___closed__4; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyDerivingHandlers___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -602,9 +607,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inducti lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkBelow___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___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_Inductive_0__Lean_Elab_Command_isInductiveFamily___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_ptr_addr(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors_elabCtorType___lambda__3___closed__1; lean_object* lean_mk_below(lean_object*, lean_object*); -lean_object* lean_level_update_imax(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkUnsafe___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_accLevelAtCtor___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -614,7 +619,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_wi lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_computeFixedIndexBitMask_go___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_mkRecOn___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkAuxConstructions___spec__1___closed__8; lean_object* l_Array_indexOfAux___at___private_Lean_Elab_PreDefinition_Structural_FindRecArg_0__Lean_Elab_Structural_getIndexMinPos___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabCtors___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*); @@ -759,10 +763,8 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); -lean_object* lean_level_update_succ(lean_object*, lean_object*); lean_object* l_Lean_Level_getLevelOffset(lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkResultingUniverses_check___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__2(lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__4___closed__1; @@ -882,6 +884,7 @@ LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Inductive_0__Lean_ LEAN_EXPORT lean_object* l_Lean_Elab_Command_withCtorRef___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_collectUniverses_go___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_elabHeaderAux___lambda__6___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___lambda__6(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_fixedIndicesToParams___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_checkValidCtorModifier___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -2640,7 +2643,7 @@ static lean_object* _init_l___private_Lean_Elab_Inductive_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_Inductive_0__Lean_Elab_Command_checkNumParams___closed__1; x_2 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_checkNumParams___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -6840,7 +6843,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_re { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Expr_getAppNumArgsAux(x_3, x_9); +x_10 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_9); x_11 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1___closed__1; lean_inc(x_10); x_12 = lean_mk_array(x_10, x_11); @@ -7915,7 +7918,7 @@ else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_3, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_13); x_15 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -10292,205 +10295,391 @@ case 1: lean_object* x_9; lean_object* x_10; uint8_t x_11; x_9 = lean_ctor_get(x_1, 0); lean_inc(x_9); +lean_inc(x_9); x_10 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); x_11 = !lean_is_exclusive(x_10); if (x_11 == 0) { -lean_object* x_12; lean_object* x_13; +lean_object* x_12; size_t x_13; size_t x_14; uint8_t x_15; x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_level_update_succ(x_1, x_12); -lean_ctor_set(x_10, 0, x_13); +x_13 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_14 = lean_ptr_addr(x_12); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_1); +x_16 = l_Lean_Level_succ___override(x_12); +lean_ctor_set(x_10, 0, x_16); return x_10; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_10, 0); -x_15 = lean_ctor_get(x_10, 1); -lean_inc(x_15); -lean_inc(x_14); -lean_dec(x_10); -x_16 = lean_level_update_succ(x_1, x_14); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -return x_17; +lean_dec(x_12); +lean_ctor_set(x_10, 0, x_1); +return x_10; } } -case 2: +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; uint8_t x_24; -x_18 = lean_ctor_get(x_1, 0); +lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; uint8_t x_21; +x_17 = lean_ctor_get(x_10, 0); +x_18 = lean_ctor_get(x_10, 1); lean_inc(x_18); -x_19 = lean_ctor_get(x_1, 1); -lean_inc(x_19); -x_20 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_22); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +lean_inc(x_17); +lean_dec(x_10); +x_19 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_20 = lean_ptr_addr(x_17); +x_21 = lean_usize_dec_eq(x_19, x_20); +if (x_21 == 0) { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_level_update_max(x_1, x_21, x_25); -lean_ctor_set(x_23, 0, x_26); +lean_object* x_22; lean_object* x_23; +lean_dec(x_1); +x_22 = l_Lean_Level_succ___override(x_17); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_18); return x_23; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_23, 0); -x_28 = lean_ctor_get(x_23, 1); +lean_object* x_24; +lean_dec(x_17); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_1); +lean_ctor_set(x_24, 1, x_18); +return x_24; +} +} +} +case 2: +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_1, 1); +lean_inc(x_26); +lean_inc(x_25); +x_27 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_28 = lean_ctor_get(x_27, 0); lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_23); -x_29 = lean_level_update_max(x_1, x_21, x_27); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +lean_inc(x_26); +x_30 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_29); +x_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) +{ +lean_object* x_32; size_t x_33; size_t x_34; uint8_t x_35; +x_32 = lean_ctor_get(x_30, 0); +x_33 = lean_ptr_addr(x_25); +lean_dec(x_25); +x_34 = lean_ptr_addr(x_28); +x_35 = lean_usize_dec_eq(x_33, x_34); +if (x_35 == 0) +{ +lean_object* x_36; +lean_dec(x_26); +lean_dec(x_1); +x_36 = l_Lean_mkLevelMax_x27(x_28, x_32); +lean_ctor_set(x_30, 0, x_36); +return x_30; +} +else +{ +size_t x_37; size_t x_38; uint8_t x_39; +x_37 = lean_ptr_addr(x_26); +lean_dec(x_26); +x_38 = lean_ptr_addr(x_32); +x_39 = lean_usize_dec_eq(x_37, x_38); +if (x_39 == 0) +{ +lean_object* x_40; +lean_dec(x_1); +x_40 = l_Lean_mkLevelMax_x27(x_28, x_32); +lean_ctor_set(x_30, 0, x_40); return x_30; } +else +{ +lean_object* x_41; +x_41 = l_Lean_simpLevelMax_x27(x_28, x_32, x_1); +lean_dec(x_1); +lean_dec(x_32); +lean_dec(x_28); +lean_ctor_set(x_30, 0, x_41); +return x_30; +} +} +} +else +{ +lean_object* x_42; lean_object* x_43; size_t x_44; size_t x_45; uint8_t x_46; +x_42 = lean_ctor_get(x_30, 0); +x_43 = lean_ctor_get(x_30, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_30); +x_44 = lean_ptr_addr(x_25); +lean_dec(x_25); +x_45 = lean_ptr_addr(x_28); +x_46 = lean_usize_dec_eq(x_44, x_45); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; +lean_dec(x_26); +lean_dec(x_1); +x_47 = l_Lean_mkLevelMax_x27(x_28, x_42); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_43); +return x_48; +} +else +{ +size_t x_49; size_t x_50; uint8_t x_51; +x_49 = lean_ptr_addr(x_26); +lean_dec(x_26); +x_50 = lean_ptr_addr(x_42); +x_51 = lean_usize_dec_eq(x_49, x_50); +if (x_51 == 0) +{ +lean_object* x_52; lean_object* x_53; +lean_dec(x_1); +x_52 = l_Lean_mkLevelMax_x27(x_28, x_42); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_43); +return x_53; +} +else +{ +lean_object* x_54; lean_object* x_55; +x_54 = l_Lean_simpLevelMax_x27(x_28, x_42, x_1); +lean_dec(x_1); +lean_dec(x_42); +lean_dec(x_28); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_43); +return x_55; +} +} +} } case 3: { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_31 = lean_ctor_get(x_1, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_1, 1); -lean_inc(x_32); -x_33 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_35); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_56 = lean_ctor_get(x_1, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_1, 1); +lean_inc(x_57); +lean_inc(x_56); +x_58 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_56, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_58, 1); +lean_inc(x_60); +lean_dec(x_58); +lean_inc(x_57); +x_61 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_57, x_2, x_3, x_4, x_5, x_6, x_7, x_60); +x_62 = !lean_is_exclusive(x_61); +if (x_62 == 0) { -lean_object* x_38; lean_object* x_39; -x_38 = lean_ctor_get(x_36, 0); -x_39 = lean_level_update_imax(x_1, x_34, x_38); -lean_ctor_set(x_36, 0, x_39); -return x_36; +lean_object* x_63; size_t x_64; size_t x_65; uint8_t x_66; +x_63 = lean_ctor_get(x_61, 0); +x_64 = lean_ptr_addr(x_56); +lean_dec(x_56); +x_65 = lean_ptr_addr(x_59); +x_66 = lean_usize_dec_eq(x_64, x_65); +if (x_66 == 0) +{ +lean_object* x_67; +lean_dec(x_57); +lean_dec(x_1); +x_67 = l_Lean_mkLevelIMax_x27(x_59, x_63); +lean_ctor_set(x_61, 0, x_67); +return x_61; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_40 = lean_ctor_get(x_36, 0); -x_41 = lean_ctor_get(x_36, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_36); -x_42 = lean_level_update_imax(x_1, x_34, x_40); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_41); -return x_43; +size_t x_68; size_t x_69; uint8_t x_70; +x_68 = lean_ptr_addr(x_57); +lean_dec(x_57); +x_69 = lean_ptr_addr(x_63); +x_70 = lean_usize_dec_eq(x_68, x_69); +if (x_70 == 0) +{ +lean_object* x_71; +lean_dec(x_1); +x_71 = l_Lean_mkLevelIMax_x27(x_59, x_63); +lean_ctor_set(x_61, 0, x_71); +return x_61; +} +else +{ +lean_object* x_72; +x_72 = l_Lean_simpLevelIMax_x27(x_59, x_63, x_1); +lean_dec(x_1); +lean_ctor_set(x_61, 0, x_72); +return x_61; +} +} +} +else +{ +lean_object* x_73; lean_object* x_74; size_t x_75; size_t x_76; uint8_t x_77; +x_73 = lean_ctor_get(x_61, 0); +x_74 = lean_ctor_get(x_61, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_61); +x_75 = lean_ptr_addr(x_56); +lean_dec(x_56); +x_76 = lean_ptr_addr(x_59); +x_77 = lean_usize_dec_eq(x_75, x_76); +if (x_77 == 0) +{ +lean_object* x_78; lean_object* x_79; +lean_dec(x_57); +lean_dec(x_1); +x_78 = l_Lean_mkLevelIMax_x27(x_59, x_73); +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_74); +return x_79; +} +else +{ +size_t x_80; size_t x_81; uint8_t x_82; +x_80 = lean_ptr_addr(x_57); +lean_dec(x_57); +x_81 = lean_ptr_addr(x_73); +x_82 = lean_usize_dec_eq(x_80, x_81); +if (x_82 == 0) +{ +lean_object* x_83; lean_object* x_84; +lean_dec(x_1); +x_83 = l_Lean_mkLevelIMax_x27(x_59, x_73); +x_84 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_74); +return x_84; +} +else +{ +lean_object* x_85; lean_object* x_86; +x_85 = l_Lean_simpLevelIMax_x27(x_59, x_73, x_1); +lean_dec(x_1); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_74); +return x_86; +} +} } } case 5: { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_44 = lean_ctor_get(x_1, 0); -lean_inc(x_44); -x_60 = lean_st_ref_get(x_7, x_8); -x_61 = lean_ctor_get(x_60, 1); -lean_inc(x_61); -lean_dec(x_60); -x_62 = lean_st_ref_get(x_5, x_61); -x_63 = lean_ctor_get(x_62, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_62, 1); -lean_inc(x_64); -lean_dec(x_62); -x_65 = lean_ctor_get(x_63, 0); -lean_inc(x_65); -lean_dec(x_63); -x_66 = lean_ctor_get(x_65, 5); -lean_inc(x_66); -lean_dec(x_65); -lean_inc(x_44); -x_67 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_66, x_44); -if (lean_obj_tag(x_67) == 0) +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_87 = lean_ctor_get(x_1, 0); +lean_inc(x_87); +x_103 = lean_st_ref_get(x_7, x_8); +x_104 = lean_ctor_get(x_103, 1); +lean_inc(x_104); +lean_dec(x_103); +x_105 = lean_st_ref_get(x_5, x_104); +x_106 = lean_ctor_get(x_105, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_105, 1); +lean_inc(x_107); +lean_dec(x_105); +x_108 = lean_ctor_get(x_106, 0); +lean_inc(x_108); +lean_dec(x_106); +x_109 = lean_ctor_get(x_108, 5); +lean_inc(x_109); +lean_dec(x_108); +lean_inc(x_87); +x_110 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_109, x_87); +if (lean_obj_tag(x_110) == 0) { -x_45 = x_67; -x_46 = x_64; -goto block_59; +x_88 = x_110; +x_89 = x_107; +goto block_102; } else { -lean_object* x_68; lean_object* x_69; -x_68 = l_Lean_markUsedAssignment___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3___rarg(x_5, x_6, x_7, x_64); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -lean_dec(x_68); -x_45 = x_67; -x_46 = x_69; -goto block_59; +lean_object* x_111; lean_object* x_112; +x_111 = l_Lean_markUsedAssignment___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3___rarg(x_5, x_6, x_7, x_107); +x_112 = lean_ctor_get(x_111, 1); +lean_inc(x_112); +lean_dec(x_111); +x_88 = x_110; +x_89 = x_112; +goto block_102; } -block_59: +block_102: { -if (lean_obj_tag(x_45) == 0) +if (lean_obj_tag(x_88) == 0) { -lean_object* x_47; -lean_dec(x_44); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_1); -lean_ctor_set(x_47, 1, x_46); -return x_47; +lean_object* x_90; +lean_dec(x_87); +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_1); +lean_ctor_set(x_90, 1, x_89); +return x_90; } else { -lean_object* x_48; uint8_t x_49; +lean_object* x_91; uint8_t x_92; lean_dec(x_1); -x_48 = lean_ctor_get(x_45, 0); -lean_inc(x_48); -lean_dec(x_45); -x_49 = l_Lean_Level_hasMVar(x_48); -if (x_49 == 0) +x_91 = lean_ctor_get(x_88, 0); +lean_inc(x_91); +lean_dec(x_88); +x_92 = l_Lean_Level_hasMVar(x_91); +if (x_92 == 0) { -lean_object* x_50; -lean_dec(x_44); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_46); -return x_50; +lean_object* x_93; +lean_dec(x_87); +x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_89); +return x_93; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_51 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_48, x_2, x_3, x_4, x_5, x_6, x_7, x_46); -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -lean_inc(x_52); -x_54 = l_Lean_assignLevelMVar___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(x_44, x_52, x_2, x_3, x_4, x_5, x_6, x_7, x_53); -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_94 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_shouldInferResultUniverse___spec__1(x_91, x_2, x_3, x_4, x_5, x_6, x_7, x_89); +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +lean_dec(x_94); +lean_inc(x_95); +x_97 = l_Lean_assignLevelMVar___at_Lean_Elab_Command_shouldInferResultUniverse___spec__2(x_87, x_95, x_2, x_3, x_4, x_5, x_6, x_7, x_96); +x_98 = !lean_is_exclusive(x_97); +if (x_98 == 0) { -lean_object* x_56; -x_56 = lean_ctor_get(x_54, 0); -lean_dec(x_56); -lean_ctor_set(x_54, 0, x_52); -return x_54; +lean_object* x_99; +x_99 = lean_ctor_get(x_97, 0); +lean_dec(x_99); +lean_ctor_set(x_97, 0, x_95); +return x_97; } else { -lean_object* x_57; lean_object* x_58; -x_57 = lean_ctor_get(x_54, 1); -lean_inc(x_57); -lean_dec(x_54); -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_52); -lean_ctor_set(x_58, 1, x_57); -return x_58; +lean_object* x_100; lean_object* x_101; +x_100 = lean_ctor_get(x_97, 1); +lean_inc(x_100); +lean_dec(x_97); +x_101 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_101, 0, x_95); +lean_ctor_set(x_101, 1, x_100); +return x_101; } } } @@ -10498,11 +10687,11 @@ return x_58; } default: { -lean_object* x_70; -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_1); -lean_ctor_set(x_70, 1, x_8); -return x_70; +lean_object* x_113; +x_113 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_113, 0, x_1); +lean_ctor_set(x_113, 1, x_8); +return x_113; } } } @@ -12236,205 +12425,391 @@ case 1: lean_object* x_10; lean_object* x_11; uint8_t x_12; x_10 = lean_ctor_get(x_1, 0); lean_inc(x_10); +lean_inc(x_10); x_11 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); x_12 = !lean_is_exclusive(x_11); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; +lean_object* x_13; size_t x_14; size_t x_15; uint8_t x_16; x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_level_update_succ(x_1, x_13); -lean_ctor_set(x_11, 0, x_14); +x_14 = lean_ptr_addr(x_10); +lean_dec(x_10); +x_15 = lean_ptr_addr(x_13); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; +lean_dec(x_1); +x_17 = l_Lean_Level_succ___override(x_13); +lean_ctor_set(x_11, 0, x_17); 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_level_update_succ(x_1, x_15); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_dec(x_13); +lean_ctor_set(x_11, 0, x_1); +return x_11; } } -case 2: +else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_19 = lean_ctor_get(x_1, 0); +lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; uint8_t x_22; +x_18 = lean_ctor_get(x_11, 0); +x_19 = lean_ctor_get(x_11, 1); lean_inc(x_19); -x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); -x_21 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_20, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_23); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) +lean_inc(x_18); +lean_dec(x_11); +x_20 = lean_ptr_addr(x_10); +lean_dec(x_10); +x_21 = lean_ptr_addr(x_18); +x_22 = lean_usize_dec_eq(x_20, x_21); +if (x_22 == 0) { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_24, 0); -x_27 = lean_level_update_max(x_1, x_22, x_26); -lean_ctor_set(x_24, 0, x_27); +lean_object* x_23; lean_object* x_24; +lean_dec(x_1); +x_23 = l_Lean_Level_succ___override(x_18); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_19); return x_24; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = lean_ctor_get(x_24, 0); -x_29 = lean_ctor_get(x_24, 1); +lean_object* x_25; +lean_dec(x_18); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_1); +lean_ctor_set(x_25, 1, x_19); +return x_25; +} +} +} +case 2: +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_1, 1); +lean_inc(x_27); +lean_inc(x_26); +x_28 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_29 = lean_ctor_get(x_28, 0); lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_24); -x_30 = lean_level_update_max(x_1, x_22, x_28); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +lean_inc(x_27); +x_31 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_30); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) +{ +lean_object* x_33; size_t x_34; size_t x_35; uint8_t x_36; +x_33 = lean_ctor_get(x_31, 0); +x_34 = lean_ptr_addr(x_26); +lean_dec(x_26); +x_35 = lean_ptr_addr(x_29); +x_36 = lean_usize_dec_eq(x_34, x_35); +if (x_36 == 0) +{ +lean_object* x_37; +lean_dec(x_27); +lean_dec(x_1); +x_37 = l_Lean_mkLevelMax_x27(x_29, x_33); +lean_ctor_set(x_31, 0, x_37); +return x_31; +} +else +{ +size_t x_38; size_t x_39; uint8_t x_40; +x_38 = lean_ptr_addr(x_27); +lean_dec(x_27); +x_39 = lean_ptr_addr(x_33); +x_40 = lean_usize_dec_eq(x_38, x_39); +if (x_40 == 0) +{ +lean_object* x_41; +lean_dec(x_1); +x_41 = l_Lean_mkLevelMax_x27(x_29, x_33); +lean_ctor_set(x_31, 0, x_41); return x_31; } +else +{ +lean_object* x_42; +x_42 = l_Lean_simpLevelMax_x27(x_29, x_33, x_1); +lean_dec(x_1); +lean_dec(x_33); +lean_dec(x_29); +lean_ctor_set(x_31, 0, x_42); +return x_31; +} +} +} +else +{ +lean_object* x_43; lean_object* x_44; size_t x_45; size_t x_46; uint8_t x_47; +x_43 = lean_ctor_get(x_31, 0); +x_44 = lean_ctor_get(x_31, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_31); +x_45 = lean_ptr_addr(x_26); +lean_dec(x_26); +x_46 = lean_ptr_addr(x_29); +x_47 = lean_usize_dec_eq(x_45, x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; +lean_dec(x_27); +lean_dec(x_1); +x_48 = l_Lean_mkLevelMax_x27(x_29, x_43); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_44); +return x_49; +} +else +{ +size_t x_50; size_t x_51; uint8_t x_52; +x_50 = lean_ptr_addr(x_27); +lean_dec(x_27); +x_51 = lean_ptr_addr(x_43); +x_52 = lean_usize_dec_eq(x_50, x_51); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; +lean_dec(x_1); +x_53 = l_Lean_mkLevelMax_x27(x_29, x_43); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_44); +return x_54; +} +else +{ +lean_object* x_55; lean_object* x_56; +x_55 = l_Lean_simpLevelMax_x27(x_29, x_43, x_1); +lean_dec(x_1); +lean_dec(x_43); +lean_dec(x_29); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_44); +return x_56; +} +} +} } case 3: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_32 = lean_ctor_get(x_1, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_1, 1); -lean_inc(x_33); -x_34 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_33, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_36); -x_38 = !lean_is_exclusive(x_37); -if (x_38 == 0) +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_57 = lean_ctor_get(x_1, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_1, 1); +lean_inc(x_58); +lean_inc(x_57); +x_59 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_57, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +lean_inc(x_58); +x_62 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_61); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_37, 0); -x_40 = lean_level_update_imax(x_1, x_35, x_39); -lean_ctor_set(x_37, 0, x_40); -return x_37; +lean_object* x_64; size_t x_65; size_t x_66; uint8_t x_67; +x_64 = lean_ctor_get(x_62, 0); +x_65 = lean_ptr_addr(x_57); +lean_dec(x_57); +x_66 = lean_ptr_addr(x_60); +x_67 = lean_usize_dec_eq(x_65, x_66); +if (x_67 == 0) +{ +lean_object* x_68; +lean_dec(x_58); +lean_dec(x_1); +x_68 = l_Lean_mkLevelIMax_x27(x_60, x_64); +lean_ctor_set(x_62, 0, x_68); +return x_62; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_41 = lean_ctor_get(x_37, 0); -x_42 = lean_ctor_get(x_37, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_37); -x_43 = lean_level_update_imax(x_1, x_35, x_41); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_42); -return x_44; +size_t x_69; size_t x_70; uint8_t x_71; +x_69 = lean_ptr_addr(x_58); +lean_dec(x_58); +x_70 = lean_ptr_addr(x_64); +x_71 = lean_usize_dec_eq(x_69, x_70); +if (x_71 == 0) +{ +lean_object* x_72; +lean_dec(x_1); +x_72 = l_Lean_mkLevelIMax_x27(x_60, x_64); +lean_ctor_set(x_62, 0, x_72); +return x_62; +} +else +{ +lean_object* x_73; +x_73 = l_Lean_simpLevelIMax_x27(x_60, x_64, x_1); +lean_dec(x_1); +lean_ctor_set(x_62, 0, x_73); +return x_62; +} +} +} +else +{ +lean_object* x_74; lean_object* x_75; size_t x_76; size_t x_77; uint8_t x_78; +x_74 = lean_ctor_get(x_62, 0); +x_75 = lean_ctor_get(x_62, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_62); +x_76 = lean_ptr_addr(x_57); +lean_dec(x_57); +x_77 = lean_ptr_addr(x_60); +x_78 = lean_usize_dec_eq(x_76, x_77); +if (x_78 == 0) +{ +lean_object* x_79; lean_object* x_80; +lean_dec(x_58); +lean_dec(x_1); +x_79 = l_Lean_mkLevelIMax_x27(x_60, x_74); +x_80 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_80, 0, x_79); +lean_ctor_set(x_80, 1, x_75); +return x_80; +} +else +{ +size_t x_81; size_t x_82; uint8_t x_83; +x_81 = lean_ptr_addr(x_58); +lean_dec(x_58); +x_82 = lean_ptr_addr(x_74); +x_83 = lean_usize_dec_eq(x_81, x_82); +if (x_83 == 0) +{ +lean_object* x_84; lean_object* x_85; +lean_dec(x_1); +x_84 = l_Lean_mkLevelIMax_x27(x_60, x_74); +x_85 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_85, 0, x_84); +lean_ctor_set(x_85, 1, x_75); +return x_85; +} +else +{ +lean_object* x_86; lean_object* x_87; +x_86 = l_Lean_simpLevelIMax_x27(x_60, x_74, x_1); +lean_dec(x_1); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_75); +return x_87; +} +} } } case 5: { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_45 = lean_ctor_get(x_1, 0); -lean_inc(x_45); -x_61 = lean_st_ref_get(x_8, x_9); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = lean_st_ref_get(x_6, x_62); -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_63, 1); -lean_inc(x_65); -lean_dec(x_63); -x_66 = lean_ctor_get(x_64, 0); -lean_inc(x_66); -lean_dec(x_64); -x_67 = lean_ctor_get(x_66, 5); -lean_inc(x_67); -lean_dec(x_66); -lean_inc(x_45); -x_68 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_67, x_45); -if (lean_obj_tag(x_68) == 0) +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_88 = lean_ctor_get(x_1, 0); +lean_inc(x_88); +x_104 = lean_st_ref_get(x_8, x_9); +x_105 = lean_ctor_get(x_104, 1); +lean_inc(x_105); +lean_dec(x_104); +x_106 = lean_st_ref_get(x_6, x_105); +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = lean_ctor_get(x_107, 0); +lean_inc(x_109); +lean_dec(x_107); +x_110 = lean_ctor_get(x_109, 5); +lean_inc(x_110); +lean_dec(x_109); +lean_inc(x_88); +x_111 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_110, x_88); +if (lean_obj_tag(x_111) == 0) { -x_46 = x_68; -x_47 = x_65; -goto block_60; +x_89 = x_111; +x_90 = x_108; +goto block_103; } else { -lean_object* x_69; lean_object* x_70; -x_69 = l_Lean_markUsedAssignment___at_Lean_Elab_Command_accLevelAtCtor___spec__3___rarg(x_6, x_7, x_8, x_65); -x_70 = lean_ctor_get(x_69, 1); -lean_inc(x_70); -lean_dec(x_69); -x_46 = x_68; -x_47 = x_70; -goto block_60; +lean_object* x_112; lean_object* x_113; +x_112 = l_Lean_markUsedAssignment___at_Lean_Elab_Command_accLevelAtCtor___spec__3___rarg(x_6, x_7, x_8, x_108); +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +lean_dec(x_112); +x_89 = x_111; +x_90 = x_113; +goto block_103; } -block_60: +block_103: { -if (lean_obj_tag(x_46) == 0) +if (lean_obj_tag(x_89) == 0) { -lean_object* x_48; -lean_dec(x_45); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_1); -lean_ctor_set(x_48, 1, x_47); -return x_48; +lean_object* x_91; +lean_dec(x_88); +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_1); +lean_ctor_set(x_91, 1, x_90); +return x_91; } else { -lean_object* x_49; uint8_t x_50; +lean_object* x_92; uint8_t x_93; lean_dec(x_1); -x_49 = lean_ctor_get(x_46, 0); -lean_inc(x_49); -lean_dec(x_46); -x_50 = l_Lean_Level_hasMVar(x_49); -if (x_50 == 0) +x_92 = lean_ctor_get(x_89, 0); +lean_inc(x_92); +lean_dec(x_89); +x_93 = l_Lean_Level_hasMVar(x_92); +if (x_93 == 0) { -lean_object* x_51; -lean_dec(x_45); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_47); -return x_51; +lean_object* x_94; +lean_dec(x_88); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_90); +return x_94; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; -x_52 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_49, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_47); -x_53 = lean_ctor_get(x_52, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_52, 1); -lean_inc(x_54); -lean_dec(x_52); -lean_inc(x_53); -x_55 = l_Lean_assignLevelMVar___at_Lean_Elab_Command_accLevelAtCtor___spec__2(x_45, x_53, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_54); -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; +x_95 = l_Lean_instantiateLevelMVars___at_Lean_Elab_Command_accLevelAtCtor___spec__1(x_92, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_90); +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); +lean_inc(x_96); +x_98 = l_Lean_assignLevelMVar___at_Lean_Elab_Command_accLevelAtCtor___spec__2(x_88, x_96, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_97); +x_99 = !lean_is_exclusive(x_98); +if (x_99 == 0) { -lean_object* x_57; -x_57 = lean_ctor_get(x_55, 0); -lean_dec(x_57); -lean_ctor_set(x_55, 0, x_53); -return x_55; +lean_object* x_100; +x_100 = lean_ctor_get(x_98, 0); +lean_dec(x_100); +lean_ctor_set(x_98, 0, x_96); +return x_98; } else { -lean_object* x_58; lean_object* x_59; -x_58 = lean_ctor_get(x_55, 1); -lean_inc(x_58); -lean_dec(x_55); -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_53); -lean_ctor_set(x_59, 1, x_58); -return x_59; +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_98, 1); +lean_inc(x_101); +lean_dec(x_98); +x_102 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_102, 0, x_96); +lean_ctor_set(x_102, 1, x_101); +return x_102; } } } @@ -12442,11 +12817,11 @@ return x_59; } default: { -lean_object* x_71; -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_1); -lean_ctor_set(x_71, 1, x_9); -return x_71; +lean_object* x_114; +x_114 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_114, 0, x_1); +lean_ctor_set(x_114, 1, x_9); +return x_114; } } } @@ -24619,7 +24994,7 @@ return x_27; else { lean_object* x_28; uint8_t x_29; -x_28 = l_Lean_Expr_getAppNumArgsAux(x_6, x_13); +x_28 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_6, x_13); x_29 = lean_nat_dec_lt(x_2, x_28); if (x_29 == 0) { @@ -24843,7 +25218,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_co { 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; size_t x_25; lean_object* x_26; size_t x_27; lean_object* x_28; x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Lean_Expr_getAppNumArgsAux(x_6, x_12); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_6, x_12); x_14 = l___private_Lean_Elab_Inductive_0__Lean_Elab_Command_reorderCtorArgs___lambda__1___closed__1; lean_inc(x_13); x_15 = lean_mk_array(x_13, x_14); @@ -28685,7 +29060,9 @@ lean_inc(x_35); lean_dec(x_34); x_36 = 0; lean_inc(x_10); -lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); x_37 = l_Lean_Elab_Term_applyAttributesAt(x_15, x_35, x_36, x_5, x_6, x_7, x_8, x_9, x_10, x_33); lean_dec(x_35); @@ -29581,7 +29958,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -29632,7 +30009,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 4); +x_29 = lean_ctor_get(x_27, 5); lean_inc(x_29); lean_dec(x_27); x_30 = lean_ctor_get(x_29, 1); @@ -29655,7 +30032,7 @@ lean_dec(x_34); x_36 = lean_st_ref_take(x_3, x_35); x_37 = lean_ctor_get(x_36, 0); lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 4); +x_38 = lean_ctor_get(x_37, 5); lean_inc(x_38); x_39 = lean_ctor_get(x_36, 1); lean_inc(x_39); @@ -29664,7 +30041,7 @@ x_40 = !lean_is_exclusive(x_37); if (x_40 == 0) { lean_object* x_41; uint8_t x_42; -x_41 = lean_ctor_get(x_37, 4); +x_41 = lean_ctor_get(x_37, 5); lean_dec(x_41); x_42 = !lean_is_exclusive(x_38); if (x_42 == 0) @@ -29709,7 +30086,7 @@ x_53 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_50); -lean_ctor_set(x_37, 4, x_53); +lean_ctor_set(x_37, 5, x_53); x_54 = lean_st_ref_set(x_3, x_37, x_39); lean_dec(x_3); x_55 = lean_ctor_get(x_54, 1); @@ -29734,243 +30111,249 @@ return x_57; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_58 = lean_ctor_get(x_37, 0); x_59 = lean_ctor_get(x_37, 1); x_60 = lean_ctor_get(x_37, 2); x_61 = lean_ctor_get(x_37, 3); +x_62 = lean_ctor_get(x_37, 4); +lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); lean_inc(x_58); lean_dec(x_37); -x_62 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); +x_63 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); +x_64 = lean_ctor_get(x_38, 0); +lean_inc(x_64); if (lean_is_exclusive(x_38)) { lean_ctor_release(x_38, 0); lean_ctor_release(x_38, 1); - x_64 = x_38; + x_65 = x_38; } else { lean_dec_ref(x_38); - x_64 = lean_box(0); + x_65 = lean_box(0); } -x_65 = l_Std_PersistentArray_append___rarg(x_19, x_32); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(0, 2, 1); +x_66 = l_Std_PersistentArray_append___rarg(x_19, x_32); +if (lean_is_scalar(x_65)) { + x_67 = lean_alloc_ctor(0, 2, 1); } else { - x_66 = x_64; + x_67 = x_65; } -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_65); -lean_ctor_set_uint8(x_66, sizeof(void*)*2, x_62); -x_67 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_67, 0, x_58); -lean_ctor_set(x_67, 1, x_59); -lean_ctor_set(x_67, 2, x_60); -lean_ctor_set(x_67, 3, x_61); -lean_ctor_set(x_67, 4, x_66); -x_68 = lean_st_ref_set(x_3, x_67, x_39); -lean_dec(x_3); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_70 = x_68; +lean_ctor_set(x_67, 0, x_64); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_63); +x_68 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_68, 0, x_58); +lean_ctor_set(x_68, 1, x_59); +lean_ctor_set(x_68, 2, x_60); +lean_ctor_set(x_68, 3, x_61); +lean_ctor_set(x_68, 4, x_62); +lean_ctor_set(x_68, 5, x_67); +x_69 = lean_st_ref_set(x_3, x_68, x_39); +lean_dec(x_3); +x_70 = lean_ctor_get(x_69, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_71 = x_69; } else { - lean_dec_ref(x_68); - x_70 = lean_box(0); + lean_dec_ref(x_69); + x_71 = lean_box(0); } -if (lean_is_scalar(x_70)) { - x_71 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_70; + x_72 = x_71; } -lean_ctor_set(x_71, 0, x_22); -lean_ctor_set(x_71, 1, x_69); -return x_71; +lean_ctor_set(x_72, 0, x_22); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_72 = lean_ctor_get(x_21, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_21, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_73 = lean_ctor_get(x_21, 0); lean_inc(x_73); +x_74 = lean_ctor_get(x_21, 1); +lean_inc(x_74); lean_dec(x_21); -x_74 = lean_st_ref_get(x_7, x_73); -x_75 = lean_ctor_get(x_74, 1); -lean_inc(x_75); -lean_dec(x_74); -x_76 = lean_st_ref_get(x_3, x_75); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); +x_75 = lean_st_ref_get(x_7, x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_st_ref_get(x_3, x_76); +x_78 = lean_ctor_get(x_77, 0); lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_ctor_get(x_77, 4); +x_79 = lean_ctor_get(x_77, 1); lean_inc(x_79); lean_dec(x_77); -x_80 = lean_ctor_get(x_79, 1); +x_80 = lean_ctor_get(x_78, 5); lean_inc(x_80); -x_81 = l_Std_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(x_79, x_80, x_2, x_3, x_4, x_5, x_6, x_7, x_78); +lean_dec(x_78); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +x_82 = l_Std_PersistentArray_mapM___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_mkInductiveDecl___spec__10(x_80, x_81, x_2, x_3, x_4, x_5, x_6, x_7, x_79); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_st_ref_get(x_7, x_83); +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +lean_dec(x_82); +x_85 = lean_st_ref_get(x_7, x_84); lean_dec(x_7); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_3, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_87, 4); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_st_ref_take(x_3, x_86); +x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 1); +x_89 = lean_ctor_get(x_88, 5); lean_inc(x_89); -lean_dec(x_86); -x_90 = !lean_is_exclusive(x_87); -if (x_90 == 0) +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = !lean_is_exclusive(x_88); +if (x_91 == 0) { -lean_object* x_91; uint8_t x_92; -x_91 = lean_ctor_get(x_87, 4); -lean_dec(x_91); -x_92 = !lean_is_exclusive(x_88); -if (x_92 == 0) +lean_object* x_92; uint8_t x_93; +x_92 = lean_ctor_get(x_88, 5); +lean_dec(x_92); +x_93 = !lean_is_exclusive(x_89); +if (x_93 == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; -x_93 = lean_ctor_get(x_88, 1); -lean_dec(x_93); -x_94 = l_Std_PersistentArray_append___rarg(x_19, x_82); -lean_ctor_set(x_88, 1, x_94); -x_95 = lean_st_ref_set(x_3, x_87, x_89); +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_89, 1); +lean_dec(x_94); +x_95 = l_Std_PersistentArray_append___rarg(x_19, x_83); +lean_ctor_set(x_89, 1, x_95); +x_96 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) { -lean_object* x_97; -x_97 = lean_ctor_get(x_95, 0); -lean_dec(x_97); -lean_ctor_set_tag(x_95, 1); -lean_ctor_set(x_95, 0, x_72); -return x_95; +lean_object* x_98; +x_98 = lean_ctor_get(x_96, 0); +lean_dec(x_98); +lean_ctor_set_tag(x_96, 1); +lean_ctor_set(x_96, 0, x_73); +return x_96; } else { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_95, 1); -lean_inc(x_98); -lean_dec(x_95); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_72); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_dec(x_96); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_73); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_100 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_101 = lean_ctor_get(x_88, 0); -lean_inc(x_101); -lean_dec(x_88); -x_102 = l_Std_PersistentArray_append___rarg(x_19, x_82); -x_103 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_100); -lean_ctor_set(x_87, 4, x_103); -x_104 = lean_st_ref_set(x_3, x_87, x_89); +uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_101 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +lean_dec(x_89); +x_103 = l_Std_PersistentArray_append___rarg(x_19, x_83); +x_104 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set_uint8(x_104, sizeof(void*)*2, x_101); +lean_ctor_set(x_88, 5, x_104); +x_105 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_106 = x_104; +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; - lean_ctor_set_tag(x_107, 1); + x_108 = x_107; + lean_ctor_set_tag(x_108, 1); } -lean_ctor_set(x_107, 0, x_72); -lean_ctor_set(x_107, 1, x_105); -return x_107; +lean_ctor_set(x_108, 0, x_73); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_108 = lean_ctor_get(x_87, 0); -x_109 = lean_ctor_get(x_87, 1); -x_110 = lean_ctor_get(x_87, 2); -x_111 = lean_ctor_get(x_87, 3); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_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; +x_109 = lean_ctor_get(x_88, 0); +x_110 = lean_ctor_get(x_88, 1); +x_111 = lean_ctor_get(x_88, 2); +x_112 = lean_ctor_get(x_88, 3); +x_113 = lean_ctor_get(x_88, 4); +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_dec(x_87); -x_112 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_113 = lean_ctor_get(x_88, 0); -lean_inc(x_113); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_114 = x_88; -} else { - lean_dec_ref(x_88); - x_114 = lean_box(0); -} -x_115 = l_Std_PersistentArray_append___rarg(x_19, x_82); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 1); +lean_dec(x_88); +x_114 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_115 = lean_ctor_get(x_89, 0); +lean_inc(x_115); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_116 = x_89; } else { - x_116 = x_114; -} -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_115); -lean_ctor_set_uint8(x_116, sizeof(void*)*2, x_112); -x_117 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_117, 0, x_108); -lean_ctor_set(x_117, 1, x_109); -lean_ctor_set(x_117, 2, x_110); -lean_ctor_set(x_117, 3, x_111); -lean_ctor_set(x_117, 4, x_116); -x_118 = lean_st_ref_set(x_3, x_117, x_89); -lean_dec(x_3); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; + lean_dec_ref(x_89); + x_116 = lean_box(0); +} +x_117 = l_Std_PersistentArray_append___rarg(x_19, x_83); +if (lean_is_scalar(x_116)) { + x_118 = lean_alloc_ctor(0, 2, 1); +} else { + x_118 = x_116; +} +lean_ctor_set(x_118, 0, x_115); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); +x_119 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_119, 0, x_109); +lean_ctor_set(x_119, 1, x_110); +lean_ctor_set(x_119, 2, x_111); +lean_ctor_set(x_119, 3, x_112); +lean_ctor_set(x_119, 4, x_113); +lean_ctor_set(x_119, 5, x_118); +x_120 = lean_st_ref_set(x_3, x_119, x_90); +lean_dec(x_3); +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_122 = x_120; } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + lean_dec_ref(x_120); + x_122 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); } else { - x_121 = x_120; - lean_ctor_set_tag(x_121, 1); + x_123 = x_122; + lean_ctor_set_tag(x_123, 1); } -lean_ctor_set(x_121, 0, x_72); -lean_ctor_set(x_121, 1, x_119); -return x_121; +lean_ctor_set(x_123, 0, x_73); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } @@ -32693,7 +33076,7 @@ lean_ctor_set(x_28, 7, x_27); x_29 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_30 = 2; lean_inc(x_11); -x_31 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_29, x_30, x_28, x_11, x_19); +x_31 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_29, x_30, x_28, x_11, x_19); x_32 = lean_ctor_get(x_31, 1); lean_inc(x_32); lean_dec(x_31); @@ -32787,7 +33170,7 @@ lean_ctor_set(x_71, 7, x_70); x_72 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_73 = 2; lean_inc(x_11); -x_74 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_72, x_73, x_71, x_11, x_62); +x_74 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_73, x_71, x_11, x_62); x_75 = lean_ctor_get(x_74, 1); lean_inc(x_75); lean_dec(x_74); @@ -33023,7 +33406,7 @@ lean_ctor_set(x_29, 7, x_28); x_30 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_31 = 2; lean_inc(x_11); -x_32 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_30, x_31, x_29, x_11, x_20); +x_32 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_30, x_31, x_29, x_11, x_20); x_33 = lean_ctor_get(x_32, 1); lean_inc(x_33); lean_dec(x_32); @@ -33122,7 +33505,7 @@ lean_ctor_set(x_74, 7, x_73); x_75 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_76 = 2; lean_inc(x_11); -x_77 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_75, x_76, x_74, x_11, x_65); +x_77 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_75, x_76, x_74, x_11, x_65); x_78 = lean_ctor_get(x_77, 1); lean_inc(x_78); lean_dec(x_77); @@ -33242,7 +33625,7 @@ lean_ctor_set(x_28, 7, x_27); x_29 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_30 = 2; lean_inc(x_10); -x_31 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_29, x_30, x_28, x_10, x_19); +x_31 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_29, x_30, x_28, x_10, x_19); x_32 = lean_ctor_get(x_31, 1); lean_inc(x_32); lean_dec(x_31); @@ -33375,7 +33758,7 @@ lean_ctor_set(x_27, 7, x_26); x_28 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_29 = 2; lean_inc(x_10); -x_30 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_28, x_29, x_27, x_10, x_18); +x_30 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_28, x_29, x_27, x_10, x_18); x_31 = lean_ctor_get(x_30, 1); lean_inc(x_31); lean_dec(x_30); @@ -33475,7 +33858,7 @@ lean_ctor_set(x_74, 7, x_73); x_75 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_76 = 2; lean_inc(x_10); -x_77 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_75, x_76, x_74, x_10, x_65); +x_77 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_75, x_76, x_74, x_10, x_65); x_78 = lean_ctor_get(x_77, 1); lean_inc(x_78); lean_dec(x_77); @@ -33705,7 +34088,7 @@ lean_ctor_set(x_39, 7, x_38); x_40 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_41 = 2; lean_inc(x_7); -x_42 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_40, x_41, x_39, x_7, x_30); +x_42 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_40, x_41, x_39, x_7, x_30); x_43 = lean_ctor_get(x_42, 1); lean_inc(x_43); lean_dec(x_42); @@ -33817,7 +34200,7 @@ lean_ctor_set(x_88, 7, x_87); x_89 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_90 = 2; lean_inc(x_7); -x_91 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_89, x_90, x_88, x_7, x_79); +x_91 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_89, x_90, x_88, x_7, x_79); x_92 = lean_ctor_get(x_91, 1); lean_inc(x_92); lean_dec(x_91); @@ -33925,7 +34308,7 @@ lean_ctor_set(x_135, 7, x_134); x_136 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Inductive_0__Lean_Elab_Command_applyComputedFields___spec__1___lambda__2___closed__3; x_137 = 2; lean_inc(x_7); -x_138 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_136, x_137, x_135, x_7, x_126); +x_138 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_136, x_137, x_135, x_7, x_126); x_139 = lean_ctor_get(x_138, 1); lean_inc(x_139); lean_dec(x_138); @@ -34880,7 +35263,9 @@ if (x_12 == 0) { lean_object* x_13; lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); x_13 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_13, 0, x_4); @@ -34902,7 +35287,9 @@ lean_inc(x_17); lean_dec(x_16); x_18 = 1; lean_inc(x_10); -lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); x_19 = l_Lean_Elab_Term_applyAttributesAt(x_15, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_17); @@ -34924,7 +35311,9 @@ else { uint8_t x_25; lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); x_25 = !lean_is_exclusive(x_19); if (x_25 == 0) @@ -35567,6 +35956,7 @@ lean_dec(x_13); lean_ctor_set(x_9, 5, x_14); x_15 = lean_box(0); x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__2(x_2, x_3, x_4, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_9); if (lean_obj_tag(x_16) == 0) { uint8_t x_17; @@ -35656,6 +36046,7 @@ lean_ctor_set(x_37, 9, x_34); lean_ctor_set(x_37, 10, x_35); x_38 = lean_box(0); x_39 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__2(x_2, x_3, x_4, x_38, x_5, x_6, x_7, x_8, x_37, x_10, x_11); +lean_dec(x_37); if (lean_obj_tag(x_39) == 0) { lean_object* x_40; lean_object* x_41; lean_object* x_42; @@ -36100,9 +36491,7 @@ lean_dec(x_2); x_13 = lean_unbox_usize(x_3); lean_dec(x_3); x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabInductiveViews___spec__2(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_9); lean_dec(x_1); return x_14; } @@ -36148,9 +36537,6 @@ lean_dec(x_3); x_13 = lean_unbox_usize(x_4); lean_dec(x_4); x_14 = l_Lean_Elab_Command_elabInductiveViews___lambda__4(x_1, x_2, x_12, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); lean_dec(x_2); lean_dec(x_1); return x_14; diff --git a/stage0/stdlib/Lean/Elab/LetRec.c b/stage0/stdlib/Lean/Elab/LetRec.c index a8f6059aac44..d16b15ae3c95 100644 --- a/stage0/stdlib/Lean/Elab/LetRec.c +++ b/stage0/stdlib/Lean/Elab/LetRec.c @@ -17,6 +17,7 @@ lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabLetRec___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_registerLetRecsToLift___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* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabLetRec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); lean_object* l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -98,7 +99,6 @@ LEAN_EXPORT uint8_t l_List_foldr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Te LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec___closed__8; static lean_object* l_Lean_addDeclarationRanges___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__6___closed__9; static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12___closed__2; @@ -210,6 +210,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec_declRange___closed_ static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12___lambda__3___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabLetRec_declRange(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__20___lambda__3___closed__4; @@ -2351,34 +2352,96 @@ return x_13; } else { -lean_object* x_14; lean_object* x_15; +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; x_14 = lean_array_uget(x_1, x_3); +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_9, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_9, 2); +lean_inc(x_17); +x_18 = lean_ctor_get(x_9, 3); +lean_inc(x_18); +x_19 = lean_ctor_get(x_9, 4); +lean_inc(x_19); +x_20 = lean_ctor_get(x_9, 5); +lean_inc(x_20); +x_21 = lean_ctor_get(x_9, 6); +lean_inc(x_21); +x_22 = lean_ctor_get(x_9, 7); +lean_inc(x_22); +x_23 = lean_ctor_get(x_9, 8); +lean_inc(x_23); +x_24 = lean_ctor_get(x_9, 9); +lean_inc(x_24); +x_25 = lean_ctor_get(x_9, 10); +lean_inc(x_25); +x_26 = l_Lean_replaceRef(x_14, x_20); +lean_dec(x_20); +x_27 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_27, 0, x_15); +lean_ctor_set(x_27, 1, x_16); +lean_ctor_set(x_27, 2, x_17); +lean_ctor_set(x_27, 3, x_18); +lean_ctor_set(x_27, 4, x_19); +lean_ctor_set(x_27, 5, x_26); +lean_ctor_set(x_27, 6, x_21); +lean_ctor_set(x_27, 7, x_22); +lean_ctor_set(x_27, 8, x_23); +lean_ctor_set(x_27, 9, x_24); +lean_ctor_set(x_27, 10, x_25); +lean_inc(x_10); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_28 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12(x_14, x_5, x_6, x_7, x_8, x_27, x_10, x_11); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; size_t x_32; size_t x_33; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_array_push(x_4, x_29); +x_32 = 1; +x_33 = lean_usize_add(x_3, x_32); +x_3 = x_33; +x_4 = x_31; +x_11 = x_30; +goto _start; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_28, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_28, 1); +lean_inc(x_36); +lean_dec(x_28); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_15 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_mkLetRecDeclView___spec__12(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_15) == 0) +x_37 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_36); +if (lean_obj_tag(x_37) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_array_push(x_4, x_16); -x_19 = 1; -x_20 = lean_usize_add(x_3, x_19); -x_3 = x_20; -x_4 = x_18; -x_11 = x_17; +lean_object* x_38; size_t x_39; size_t x_40; +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = 1; +x_40 = lean_usize_add(x_3, x_39); +x_3 = x_40; +x_11 = x_38; goto _start; } else { -uint8_t x_22; +uint8_t x_42; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -2386,23 +2449,24 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_22 = !lean_is_exclusive(x_15); -if (x_22 == 0) +x_42 = !lean_is_exclusive(x_37); +if (x_42 == 0) { -return x_15; +return x_37; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_15, 0); -x_24 = lean_ctor_get(x_15, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_15); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_37, 0); +x_44 = lean_ctor_get(x_37, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_37); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} } } } @@ -2907,7 +2971,9 @@ lean_inc(x_28); lean_dec(x_27); x_29 = 2; lean_inc(x_9); -lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); lean_inc(x_4); lean_inc(x_26); x_30 = l_Lean_Elab_Term_applyAttributesAt(x_26, x_3, x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_28); @@ -3868,7 +3934,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Elab_LetRec_0__Lean_Elab_Term_elabLetRecDeclValues___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4571,7 +4637,7 @@ x_31 = l_Lean_replaceRef(x_22, x_30); lean_dec(x_30); lean_dec(x_22); lean_ctor_set(x_10, 5, x_31); -x_32 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_32 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_10); x_33 = !lean_is_exclusive(x_32); if (x_33 == 0) @@ -4633,7 +4699,7 @@ lean_ctor_set(x_49, 7, x_44); lean_ctor_set(x_49, 8, x_45); lean_ctor_set(x_49, 9, x_46); lean_ctor_set(x_49, 10, x_47); -x_50 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_28, x_6, x_7, x_8, x_9, x_49, x_11, x_12); +x_50 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_28, x_6, x_7, x_8, x_9, x_49, x_11, x_12); lean_dec(x_49); x_51 = lean_ctor_get(x_50, 0); lean_inc(x_51); @@ -4834,7 +4900,7 @@ lean_inc(x_14); x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); lean_dec(x_13); -x_16 = lean_ctor_get(x_14, 3); +x_16 = lean_ctor_get(x_14, 4); lean_inc(x_16); lean_dec(x_14); x_17 = lean_array_get_size(x_1); @@ -4877,10 +4943,10 @@ x_35 = !lean_is_exclusive(x_33); if (x_35 == 0) { lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_36 = lean_ctor_get(x_33, 3); +x_36 = lean_ctor_get(x_33, 4); x_37 = lean_array_to_list(lean_box(0), x_29); x_38 = l_List_appendTR___rarg(x_37, x_36); -lean_ctor_set(x_33, 3, x_38); +lean_ctor_set(x_33, 4, x_38); x_39 = lean_st_ref_set(x_5, x_33, x_34); x_40 = !lean_is_exclusive(x_39); if (x_40 == 0) @@ -4905,70 +4971,73 @@ return x_43; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; x_44 = lean_ctor_get(x_33, 0); x_45 = lean_ctor_get(x_33, 1); x_46 = lean_ctor_get(x_33, 2); x_47 = lean_ctor_get(x_33, 3); x_48 = lean_ctor_get(x_33, 4); +x_49 = lean_ctor_get(x_33, 5); +lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); lean_dec(x_33); -x_49 = lean_array_to_list(lean_box(0), x_29); -x_50 = l_List_appendTR___rarg(x_49, x_47); -x_51 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_51, 0, x_44); -lean_ctor_set(x_51, 1, x_45); -lean_ctor_set(x_51, 2, x_46); -lean_ctor_set(x_51, 3, x_50); -lean_ctor_set(x_51, 4, x_48); -x_52 = lean_st_ref_set(x_5, x_51, x_34); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -if (lean_is_exclusive(x_52)) { - lean_ctor_release(x_52, 0); - lean_ctor_release(x_52, 1); - x_54 = x_52; +x_50 = lean_array_to_list(lean_box(0), x_29); +x_51 = l_List_appendTR___rarg(x_50, x_48); +x_52 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_52, 0, x_44); +lean_ctor_set(x_52, 1, x_45); +lean_ctor_set(x_52, 2, x_46); +lean_ctor_set(x_52, 3, x_47); +lean_ctor_set(x_52, 4, x_51); +lean_ctor_set(x_52, 5, x_49); +x_53 = lean_st_ref_set(x_5, x_52, x_34); +x_54 = lean_ctor_get(x_53, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_55 = x_53; } else { - lean_dec_ref(x_52); - x_54 = lean_box(0); + lean_dec_ref(x_53); + x_55 = lean_box(0); } -if (lean_is_scalar(x_54)) { - x_55 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(0, 2, 0); } else { - x_55 = x_54; + x_56 = x_55; } -lean_ctor_set(x_55, 0, x_20); -lean_ctor_set(x_55, 1, x_53); -return x_55; +lean_ctor_set(x_56, 0, x_20); +lean_ctor_set(x_56, 1, x_54); +return x_56; } } else { -uint8_t x_56; +uint8_t x_57; lean_dec(x_17); lean_dec(x_8); lean_dec(x_6); -x_56 = !lean_is_exclusive(x_21); -if (x_56 == 0) +x_57 = !lean_is_exclusive(x_21); +if (x_57 == 0) { return x_21; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_21, 0); -x_58 = lean_ctor_get(x_21, 1); +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_21, 0); +x_59 = lean_ctor_get(x_21, 1); +lean_inc(x_59); lean_inc(x_58); -lean_inc(x_57); lean_dec(x_21); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -return x_59; +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; } } } diff --git a/stage0/stdlib/Lean/Elab/Level.c b/stage0/stdlib/Lean/Elab/Level.c index 599de296a5d4..7d3551fdfa2f 100644 --- a/stage0/stdlib/Lean/Elab/Level.c +++ b/stage0/stdlib/Lean/Elab/Level.c @@ -68,12 +68,12 @@ static lean_object* l_Lean_Elab_Level_elabLevel___closed__25; LEAN_EXPORT lean_object* l_Lean_Elab_Level_mkFreshLevelMVar(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Level_instMonadOptionsLevelElabM___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Level_maxUniverseOffset; -lean_object* lean_level_mk_max_simp(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Level_elabLevel___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshId___at_Lean_Elab_Level_mkFreshLevelMVar___spec__2___boxed(lean_object*); -lean_object* lean_level_mk_imax_simp(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Level_initFn____x40_Lean_Elab_Level___hyg_266_(lean_object*); static lean_object* l_Lean_Elab_Level_elabLevel___closed__12; lean_object* l_Nat_repr(lean_object*); @@ -1074,7 +1074,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = lean_level_mk_imax_simp(x_12, x_4); +x_14 = l_Lean_mkLevelIMax_x27(x_12, x_4); x_2 = x_9; x_4 = x_14; x_6 = x_13; @@ -1137,7 +1137,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = lean_level_mk_max_simp(x_12, x_4); +x_14 = l_Lean_mkLevelMax_x27(x_12, x_4); x_2 = x_9; x_4 = x_14; x_6 = x_13; diff --git a/stage0/stdlib/Lean/Elab/Macro.c b/stage0/stdlib/Lean/Elab/Macro.c index 4eaddba8b320..28d0eabefcde 100644 --- a/stage0/stdlib/Lean/Elab/Macro.c +++ b/stage0/stdlib/Lean/Elab/Macro.c @@ -525,7 +525,7 @@ static lean_object* _init_l_Lean_Elab_Command_elabMacro___lambda__2___closed__27 _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(9u); +x_1 = lean_unsigned_to_nat(10u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } @@ -667,16 +667,16 @@ lean_ctor_set(x_267, 1, x_266); if (lean_obj_tag(x_7) == 0) { x_268 = x_263; -goto block_304; +goto block_306; } else { -lean_object* x_305; lean_object* x_306; -x_305 = lean_ctor_get(x_7, 0); -lean_inc(x_305); -x_306 = lean_array_push(x_243, x_305); -x_268 = x_306; -goto block_304; +lean_object* x_307; lean_object* x_308; +x_307 = lean_ctor_get(x_7, 0); +lean_inc(x_307); +x_308 = lean_array_push(x_243, x_307); +x_268 = x_308; +goto block_306; } block_215: { @@ -1088,9 +1088,9 @@ return x_214; } } } -block_304: +block_306: { -lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; x_269 = l_Array_append___rarg(x_263, x_268); x_270 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_270, 0, x_24); @@ -1098,81 +1098,83 @@ lean_ctor_set(x_270, 1, x_245); lean_ctor_set(x_270, 2, x_269); x_271 = l_Lean_Elab_Command_elabMacro___lambda__2___closed__27; x_272 = lean_array_push(x_271, x_270); -x_273 = lean_array_push(x_272, x_11); +x_273 = l_Lean_Elab_Command_elabMacro___lambda__2___closed__3; +x_274 = lean_array_push(x_272, x_273); +x_275 = lean_array_push(x_274, x_11); if (lean_obj_tag(x_225) == 0) { -x_274 = x_217; -goto block_302; +x_276 = x_217; +goto block_304; } else { -lean_object* x_303; +lean_object* x_305; lean_dec(x_217); -x_303 = lean_ctor_get(x_225, 0); -lean_inc(x_303); +x_305 = lean_ctor_get(x_225, 0); +lean_inc(x_305); lean_dec(x_225); -x_274 = x_303; -goto block_302; +x_276 = x_305; +goto block_304; } -block_302: +block_304: { -lean_object* x_275; lean_object* x_276; -x_275 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_275, 0, x_274); -lean_ctor_set(x_275, 1, x_223); -x_276 = lean_array_push(x_273, x_275); +lean_object* x_277; lean_object* x_278; +x_277 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_277, 0, x_276); +lean_ctor_set(x_277, 1, x_223); +x_278 = lean_array_push(x_275, x_277); if (lean_obj_tag(x_12) == 0) { -lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; +lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_dec(x_14); -x_277 = l_Lean_Elab_Command_elabMacro___lambda__2___closed__17; -x_278 = lean_array_push(x_276, x_277); -x_279 = lean_array_push(x_278, x_246); -x_280 = lean_array_push(x_279, x_259); -x_281 = lean_array_push(x_280, x_265); -x_282 = lean_array_push(x_281, x_267); -x_283 = lean_array_push(x_282, x_13); -x_284 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_284, 0, x_24); -lean_ctor_set(x_284, 1, x_224); -lean_ctor_set(x_284, 2, x_283); -x_29 = x_284; +x_279 = l_Lean_Elab_Command_elabMacro___lambda__2___closed__17; +x_280 = lean_array_push(x_278, x_279); +x_281 = lean_array_push(x_280, x_246); +x_282 = lean_array_push(x_281, x_259); +x_283 = lean_array_push(x_282, x_265); +x_284 = lean_array_push(x_283, x_267); +x_285 = lean_array_push(x_284, x_13); +x_286 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_286, 0, x_24); +lean_ctor_set(x_286, 1, x_224); +lean_ctor_set(x_286, 2, x_285); +x_29 = x_286; x_30 = x_222; goto block_215; } else { -lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; -x_285 = lean_ctor_get(x_12, 0); -lean_inc(x_285); +lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; +x_287 = lean_ctor_get(x_12, 0); +lean_inc(x_287); lean_dec(x_12); -x_286 = l_Lean_Elab_Command_elabMacro___lambda__2___closed__28; -x_287 = l_Lean_Name_str___override(x_14, x_286); -x_288 = l_Lean_Elab_Command_elabMacro___lambda__1___closed__1; +x_288 = l_Lean_Elab_Command_elabMacro___lambda__2___closed__28; +x_289 = l_Lean_Name_str___override(x_14, x_288); +x_290 = l_Lean_Elab_Command_elabMacro___lambda__1___closed__1; lean_inc(x_267); -x_289 = lean_array_push(x_288, x_267); -x_290 = lean_array_push(x_289, x_285); -x_291 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_291, 0, x_24); -lean_ctor_set(x_291, 1, x_287); -lean_ctor_set(x_291, 2, x_290); -x_292 = lean_array_push(x_243, x_291); -x_293 = l_Array_append___rarg(x_263, x_292); -x_294 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_294, 0, x_24); -lean_ctor_set(x_294, 1, x_245); -lean_ctor_set(x_294, 2, x_293); -x_295 = lean_array_push(x_276, x_294); -x_296 = lean_array_push(x_295, x_246); -x_297 = lean_array_push(x_296, x_259); -x_298 = lean_array_push(x_297, x_265); -x_299 = lean_array_push(x_298, x_267); -x_300 = lean_array_push(x_299, x_13); -x_301 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_301, 0, x_24); -lean_ctor_set(x_301, 1, x_224); -lean_ctor_set(x_301, 2, x_300); -x_29 = x_301; +x_291 = lean_array_push(x_290, x_267); +x_292 = lean_array_push(x_291, x_287); +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_24); +lean_ctor_set(x_293, 1, x_289); +lean_ctor_set(x_293, 2, x_292); +x_294 = lean_array_push(x_243, x_293); +x_295 = l_Array_append___rarg(x_263, x_294); +x_296 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_296, 0, x_24); +lean_ctor_set(x_296, 1, x_245); +lean_ctor_set(x_296, 2, x_295); +x_297 = lean_array_push(x_278, x_296); +x_298 = lean_array_push(x_297, x_246); +x_299 = lean_array_push(x_298, x_259); +x_300 = lean_array_push(x_299, x_265); +x_301 = lean_array_push(x_300, x_267); +x_302 = lean_array_push(x_301, x_13); +x_303 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_303, 0, x_24); +lean_ctor_set(x_303, 1, x_224); +lean_ctor_set(x_303, 2, x_302); +x_29 = x_303; x_30 = x_222; goto block_215; } diff --git a/stage0/stdlib/Lean/Elab/MacroArgUtil.c b/stage0/stdlib/Lean/Elab/MacroArgUtil.c index 410239f6bb7e..311ed31c8841 100644 --- a/stage0/stdlib/Lean/Elab/MacroArgUtil.c +++ b/stage0/stdlib/Lean/Elab/MacroArgUtil.c @@ -64,6 +64,7 @@ lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofList(lean_object*); static lean_object* l_Lean_Elab_Command_expandMacroArg_mkSyntaxAndPat___closed__11; +uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstWithInfos___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandMacroArg_mkSplicePat___closed__3; @@ -88,7 +89,6 @@ extern lean_object* l_Lean_LocalContext_empty; static lean_object* l_Lean_Elab_Command_expandMacroArg_mkSyntaxAndPat___closed__26; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandMacroArg_mkSyntaxAndPat___closed__12; -lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__1___closed__4; lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); static lean_object* l_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___closed__7; @@ -162,7 +162,6 @@ lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at___private_Lean_Elab_Syntax_0_ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstWithInfos___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -212,6 +211,7 @@ static lean_object* l_List_filterMap___at_Lean_Elab_Command_expandMacroArg_mkAnt LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandMacroArg_mkSplicePat(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; static lean_object* l_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___closed__4; +lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandMacroArg_mkSyntaxAndPat___closed__19; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___closed__9; @@ -272,7 +272,7 @@ x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); lean_dec(x_9); x_11 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__1___lambda__1___closed__1; -x_12 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_10, x_11); +x_12 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_10, x_11); lean_dec(x_10); if (x_12 == 0) { @@ -303,7 +303,7 @@ x_19 = lean_ctor_get(x_17, 0); lean_inc(x_19); lean_dec(x_17); x_20 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__1___lambda__1___closed__1; -x_21 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_19, x_20); +x_21 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_19, x_20); lean_dec(x_19); if (x_21 == 0) { @@ -439,7 +439,7 @@ x_42 = lean_ctor_get(x_40, 0); lean_inc(x_42); lean_dec(x_40); x_43 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__1___lambda__1___closed__1; -x_44 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_42, x_43); +x_44 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_42, x_43); lean_dec(x_42); if (x_44 == 0) { @@ -670,7 +670,7 @@ x_42 = lean_ctor_get(x_40, 0); lean_inc(x_42); lean_dec(x_40); x_43 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__1___lambda__1___closed__1; -x_44 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_42, x_43); +x_44 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_42, x_43); lean_dec(x_42); if (x_44 == 0) { @@ -2674,7 +2674,7 @@ x_42 = lean_ctor_get(x_40, 0); lean_inc(x_42); lean_dec(x_40); x_43 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__1___lambda__1___closed__1; -x_44 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_42, x_43); +x_44 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_42, x_43); lean_dec(x_42); if (x_44 == 0) { @@ -2904,7 +2904,7 @@ x_42 = lean_ctor_get(x_40, 0); lean_inc(x_42); lean_dec(x_40); x_43 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandMacroArg_mkAntiquotNode___spec__1___lambda__1___closed__1; -x_44 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_42, x_43); +x_44 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_42, x_43); lean_dec(x_42); if (x_44 == 0) { @@ -11529,7 +11529,7 @@ x_1187 = lean_alloc_closure((void*)(l_Lean_Elab_Command_strLitToPattern___boxed) lean_closure_set(x_1187, 0, x_1133); lean_inc(x_5); lean_inc(x_4); -x_1188 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(x_1187, x_4, x_5, x_6); +x_1188 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(x_1187, x_4, x_5, x_6); if (lean_obj_tag(x_1188) == 0) { lean_object* x_1189; lean_object* x_1190; lean_object* x_1191; lean_object* x_1192; lean_object* x_1193; lean_object* x_1194; lean_object* x_1195; lean_object* x_1196; lean_object* x_1197; lean_object* x_1198; lean_object* x_1199; lean_object* x_1200; lean_object* x_1201; @@ -11771,7 +11771,7 @@ x_1261 = lean_alloc_closure((void*)(l_Lean_Elab_Command_strLitToPattern___boxed) lean_closure_set(x_1261, 0, x_1207); lean_inc(x_5); lean_inc(x_4); -x_1262 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(x_1261, x_4, x_5, x_6); +x_1262 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(x_1261, x_4, x_5, x_6); if (lean_obj_tag(x_1262) == 0) { lean_object* x_1263; lean_object* x_1264; lean_object* x_1265; lean_object* x_1266; lean_object* x_1267; lean_object* x_1268; lean_object* x_1269; lean_object* x_1270; lean_object* x_1271; lean_object* x_1272; lean_object* x_1273; lean_object* x_1274; lean_object* x_1275; @@ -12066,7 +12066,7 @@ lean_closure_set(x_6, 0, x_1); lean_closure_set(x_6, 1, x_5); lean_inc(x_3); lean_inc(x_2); -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(x_6, x_2, x_3, x_4); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(x_6, x_2, x_3, x_4); if (lean_obj_tag(x_7) == 0) { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; diff --git a/stage0/stdlib/Lean/Elab/MacroRules.c b/stage0/stdlib/Lean/Elab/MacroRules.c index 8e64a061a7a4..05653192308c 100644 --- a/stage0/stdlib/Lean/Elab/MacroRules.c +++ b/stage0/stdlib/Lean/Elab/MacroRules.c @@ -134,6 +134,7 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMacroRules lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Command_elabMacroRulesAux___spec__4(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMacroRulesAux___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(lean_object*); lean_object* l_Lean_Syntax_getQuotContent(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabMacroRules_declRange___closed__4; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMacroRulesAux___spec__5___lambda__2___closed__16; @@ -187,7 +188,6 @@ static lean_object* l_Lean_Elab_Command_elabMacroRulesAux___closed__44; static lean_object* l_Lean_Elab_Command_elabMacroRulesAux___closed__60; static lean_object* l___regBuiltin_Lean_Elab_Command_elabMacroRules___closed__1; static lean_object* l_Lean_Elab_Command_elabMacroRulesAux___closed__47; -lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(lean_object*); static lean_object* l_Lean_Elab_Command_elabMacroRulesAux___closed__1; static lean_object* l_Lean_Elab_Command_elabMacroRules___lambda__1___closed__5; static lean_object* l_Lean_Elab_Command_elabMacroRules___lambda__2___closed__3; @@ -925,7 +925,7 @@ static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMacr lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMacroRulesAux___spec__5___closed__9; x_2 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMacroRulesAux___spec__5___closed__10; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMacroRulesAux___spec__5___closed__11; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2696,7 +2696,7 @@ lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_9); +x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_9); return x_17; } else @@ -2728,7 +2728,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); lean_dec(x_2); -x_26 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_9); +x_26 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_9); return x_26; } else @@ -2757,7 +2757,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); lean_dec(x_2); -x_33 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_9); +x_33 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_9); return x_33; } else @@ -3515,7 +3515,7 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_316 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_9); +x_316 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_9); return x_316; } else @@ -3633,7 +3633,7 @@ lean_object* x_7; lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_4); +x_7 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_4); return x_7; } else @@ -3655,7 +3655,7 @@ lean_dec(x_9); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_4); +x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_4); return x_13; } else @@ -3673,7 +3673,7 @@ lean_dec(x_14); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__14___rarg(x_4); +x_17 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabCommand___spec__18___rarg(x_4); return x_17; } else diff --git a/stage0/stdlib/Lean/Elab/Match.c b/stage0/stdlib/Lean/Elab/Match.c index cccd5d174563..0a2c515fd2d9 100644 --- a/stage0/stdlib/Lean/Elab/Match.c +++ b/stage0/stdlib/Lean/Elab/Match.c @@ -24,6 +24,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_ToDepElim lean_object* l_Lean_Elab_Term_collectPatternVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_applyRefMap___lambda__1(lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KVMap_setBool(lean_object*, lean_object*, uint8_t); @@ -84,6 +85,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatch LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabMatch_declRange(lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchGeneralizing_x3f___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_toPattern___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Term_runPendingTacticsAt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withPatternVars_loop(lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); @@ -92,11 +94,10 @@ lean_object* l_Lean_Meta_getFVarsToGeneralize(lean_object*, lean_object*, uint8_ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchAlts___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_updateMatchType___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabPatterns___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__5___boxed(lean_object*, lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMatch_elabMatchDefault___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withIncRecDepth___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -114,6 +115,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_normalize_processVar_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withElaboratedLHS___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabInaccessible___closed__1; lean_object* l_Lean_Syntax_mkSep(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchGeneralizing_x3f___closed__10; static lean_object* l_List_forIn_loop___at_Lean_Elab_Term_reportMatcherResultErrors___spec__1___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -141,6 +143,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatch lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_replace___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_mkPatternRefMap_go___spec__7(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_toPattern___closed__3; +lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___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_Match_0__Lean_Elab_Term_withPatternVars_loop___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getHead_x3f(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withoutAuxDiscrs___spec__3(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -169,7 +172,6 @@ lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_markIsDep(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_elabMatch_elabMatchDefault___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___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*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabMatch_docString___closed__1; @@ -178,7 +180,7 @@ uint8_t l_Lean_Expr_isApp(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_reportMatcherResultErrors___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Term_elabMatch_elabMatchDefault___spec__5___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_waitExpectedType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabInaccessible(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*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchAlts___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -213,7 +215,6 @@ static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMa lean_object* l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_ToDepElimPattern_main___spec__5(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__6(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofList(lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__3___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -267,6 +268,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Match_0 LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withoutAuxDiscrs___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__13(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ForEachExpr_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_mkPatternRefMap_go___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__23(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMatch___closed__12; @@ -312,7 +314,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withPatte LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_normalize_addVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_Discr_h_x3f___default; LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___spec__5___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabInaccessible_declRange___closed__4; lean_object* l_Lean_Core_withFreshMacroScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -333,6 +334,7 @@ lean_object* l_Lean_LocalDecl_value(lean_object*); uint8_t l_Lean_Name_hasMacroScopes(lean_object*); lean_object* l_List_mapTRAux___at_Lean_MessageData_instCoeListExprMessageData___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_tryPostponeIfNoneOrMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Match_instantiatePatternMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMatch___closed__6; static lean_object* l_Lean_mkAuxDiscr___at___private_Lean_Elab_Match_0__Lean_Elab_Term_expandNonAtomicDiscrs_x3f_loop___spec__1___rarg___closed__4; @@ -361,6 +363,7 @@ lean_object* l_StateRefT_x27_lift(lean_object*, lean_object*, lean_object*, lean static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMatch___closed__5; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandNonAtomicDiscrs_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallMetaTelescopeReducingAux(lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_elabMatch_elabMatchDefault___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -382,6 +385,7 @@ static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMa lean_object* l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__11___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_ToDepElimPattern_isExplicitPatternVar___spec__1(lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabMatch_declRange___closed__2; static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_ToDepElimPattern_normalize_processInaccessible___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -421,6 +425,7 @@ static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMa LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withEqs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_throwEx___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_hasExprMVar(lean_object*); static lean_object* l_Lean_Meta_transform___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___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*); @@ -442,7 +447,6 @@ lean_object* l_Std_mkHashMapImp___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_inaccessible_x3f(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_isPatternVar_isAtomicIdent___boxed(lean_object*); -static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___lambda__3___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_applyRefMap(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); @@ -458,12 +462,15 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElim LEAN_EXPORT lean_object* l_Lean_Elab_Term_precheckMatch(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Match_isNamedPattern_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__8___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__13___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath_checkCompatibleApps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_TopSort_State_visitedFVars___default; static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabPatterns___spec__2___closed__2; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Expr_isFVar___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getDiscrs___boxed(lean_object*); lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath_goIndex___lambda__1___boxed(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_Match_0__Lean_Elab_Term_elabMatchAux___spec__6___boxed(lean_object*, lean_object*, lean_object*); @@ -487,6 +494,7 @@ lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_applyRefMap___spec__2___boxed(lean_object*, lean_object*); lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMatch___closed__9; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_GeneralizeResult_refined___default; uint64_t l_Lean_Expr_hash(lean_object*); @@ -517,6 +525,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Match_0__Lea lean_object* lean_array_to_list(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_collectDeps___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_isAtomic(lean_object*); +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__2; uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMatch_elabMatchDefault(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_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -537,10 +546,11 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Match_0 static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_resolveId_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_main___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_tryPostponeIfDiscrTypeIsMVar___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_Match_0__Lean_Elab_Term_elabMatchAltView___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12(size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Term_instInhabitedDiscr___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__20(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withoutAuxDiscrs___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -564,7 +574,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withToCle lean_object* l_Array_unzip___rarg(lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_reverse___rarg(lean_object*); -static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isConst(lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); @@ -573,7 +582,6 @@ lean_object* l_Lean_Meta_Match_instantiateAltLHSMVars(lean_object*, lean_object* lean_object* l_Lean_Meta_getLocalInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchOptMotive(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_updateFirst___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_normalize___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__21(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -592,6 +600,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElim LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_topSort(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instInhabitedDiscr___closed__2; +static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__1; lean_object* l_Lean_Elab_Term_elabTermEnsuringType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -601,6 +610,7 @@ static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltVi LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_ToDepElimPattern_normalize___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_List_elem___at_Lean_Occurrences_contains___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withoutAuxDiscrs___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isAtomicDiscr_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchOptMotive___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_eraseIndices___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -624,7 +634,6 @@ static lean_object* l_List_forIn_loop___at_Lean_Elab_Term_reportMatcherResultErr LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__12(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_contains___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_mkPatternRefMap_go___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_elabMatch_elabMatchDefault___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabPatterns___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Match_0__Lean_Elab_Term_expandNonAtomicDiscrs_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_eraseIndices(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -643,11 +652,11 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath_goType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_normalize_processInaccessible(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_Match_0__Lean_Elab_Term_getMatchGeneralizing_x3f___closed__2; -lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_tryPostponeIfDiscrTypeIsMVar___spec__1___closed__1; extern lean_object* l_Lean_Elab_Term_termElabAttribute; static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___lambda__4___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_precheckMatch___closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAtomFrom(lean_object*, lean_object*); @@ -658,12 +667,11 @@ static lean_object* l_Lean_Elab_Term_ToDepElimPattern_main___rarg___lambda__2___ lean_object* l_Lean_LocalDecl_type(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isMissing(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_packMatchTypePatterns___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_topSort___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_expandMacros___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportMatcherResultErrors___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_Term_synthesizeSyntheticMVarsUsingDefault(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withoutAuxDiscrs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -675,6 +683,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_isAtomic uint8_t l_Array_contains___at___private_Lean_Meta_Match_Value_0__Lean_Meta_isUIntTypeName___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withPatternElabConfig___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchAlts___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_reportMatcherResultErrors___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__7___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -689,18 +698,15 @@ lean_object* l_Lean_Syntax_getSepArgs(lean_object*); static lean_object* l_Lean_Elab_Term_ToDepElimPattern_main___rarg___lambda__4___closed__1; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___closed__1; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_packMatchTypePatterns___spec__1___closed__1; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_main___rarg___lambda__4___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_isExplicitPatternVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_isAtomicDiscr_x3f___closed__4; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalInstances___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_throwInvalidPattern(lean_object*); -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___rarg___closed__1; lean_object* l_Lean_mkHole(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -710,8 +716,8 @@ lean_object* l_Lean_Syntax_setArg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_precheckMatch___closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_precheckMatch___spec__5___closed__2; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__1; lean_object* lean_environment_main_module(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__2; uint8_t lean_expr_eqv(lean_object*, lean_object*); lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___lambda__3___closed__2; @@ -719,9 +725,10 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_precheckMa static lean_object* l_Lean_Elab_Term_ToDepElimPattern_main___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Match_0__Lean_Elab_Term_expandNonAtomicDiscrs_x3f___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchGeneralizing_x3f___closed__1; +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_main_unpack(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__4; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Std_HashMap_insert___at_Lean_Meta_ForEachExpr_visit___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_ToDepElimPattern_main_unpack_go___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isMVar(lean_object*); @@ -757,7 +764,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_Matc LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getIndexToInclude_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMatch___closed__10; lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_main___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabInaccessible___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedDiscr; @@ -793,7 +799,6 @@ uint8_t l_Lean_TagAttribute_hasTag(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_mkAuxDiscr___at___private_Lean_Elab_Match_0__Lean_Elab_Term_expandNonAtomicDiscrs_x3f_loop___spec__1___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_generalize___spec__3___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_State_patternVars___default; lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -867,7 +872,6 @@ LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Term_reportMatcherResu lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ToDepElimPattern_TopSort_State_visitedMVars___default; lean_object* l_List_toArrayAux___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getIndexToInclude_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -882,13 +886,12 @@ lean_object* lean_expr_instantiate_rev(lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Term_reportMatcherResultErrors___spec__1___closed__2; lean_object* l_Lean_Expr_arrayLit_x3f(lean_object*); LEAN_EXPORT uint8_t l_Std_AssocList_contains___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_mkPatternRefMap_go___spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11___boxed(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___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath_goIndex___spec__1___closed__2; -LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_precheckMatch___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_collectDeps___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withElaboratedLHS___rarg___closed__2; lean_object* lean_panic_fn(lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabPatterns___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_generalize___lambda__1___closed__1; uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); @@ -910,14 +913,13 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatch lean_object* l_Lean_Meta_mkEqHEq(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_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__10(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_isAtomicDiscr_x3f___spec__1___rarg___closed__1; -uint8_t l_Lean_Expr_binderInfo(lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_toPattern___closed__2; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_precheckMatch___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_eraseInaccessibleAnnotations___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath_goIndex___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabMatch_docString(lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_withoutErrToSorry___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_Match_0__Lean_Elab_Term_tryPostponeIfDiscrTypeIsMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -944,6 +946,7 @@ static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux__ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_ToDepElimPattern_main_unpack_go___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_withMVar___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFreshTypeMVar(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_precheckMatch___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_expandSimpleMatch___closed__11; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___closed__11; @@ -1014,7 +1017,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_precheckMatc static lean_object* l___regBuiltin_Lean_Elab_Term_elabInaccessible___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__5___rarg(lean_object*); static lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_isAtomicDiscr_x3f___spec__1___rarg___closed__2; -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12___boxed(lean_object*, lean_object*); lean_object* l_Lean_Meta_setMVarTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_topSort_visit___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Match_0__Lean_Elab_Term_ToDepElimPattern_packMatchTypePatterns___spec__1___closed__3; @@ -1027,8 +1029,8 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabNoMatch_declRange(lea lean_object* l_Lean_Elab_Term_isLocalIdent_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Closure_mkBinding___spec__1(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_17065_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_17123_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555_(lean_object*); lean_object* l_Lean_mkSimpleThunk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_isAtomicDiscr_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabNoMatch___closed__4; @@ -1042,6 +1044,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_Match_ lean_object* l_Lean_Elab_Term_getPatternsVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabInaccessible_declRange___closed__7; LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_withToClear___spec__13___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_elabMatch___closed__1; static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__4___closed__1; lean_object* l_Lean_Elab_Term_mkTermInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1055,6 +1058,7 @@ uint8_t l_Lean_isAuxFunDiscrName(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withElaboratedLHS(lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___spec__5(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkInaccessible(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___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_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___lambda__1(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1062,7 +1066,6 @@ lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Syntax_SepArray_getElems___spec LEAN_EXPORT lean_object* l_Lean_Elab_Term_withDepElimPatterns___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getIndexToInclude_x3f_go___boxed(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_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___spec__6(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___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_Match_0__Lean_Elab_Term_ToDepElimPattern_packMatchTypePatterns___spec__1___closed__5; static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__4___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withPatternElabConfig___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1073,6 +1076,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_ToDepElimPat LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_withoutAuxDiscrs(lean_object*); lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchGeneralizing_x3f___closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltView___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_ToDepElimPattern_normalize___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2407,7 +2411,7 @@ x_114 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Ter x_115 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_115, 0, x_113); lean_ctor_set(x_115, 1, x_114); -x_116 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_115, x_6, x_7, x_8, x_9, x_10, x_11, x_107); +x_116 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_115, x_6, x_7, x_8, x_9, x_10, x_11, x_107); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4256,7 +4260,7 @@ case 5: { lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_17, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_17, x_18); x_20 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_19); x_21 = lean_mk_array(x_19, x_20); @@ -4289,9 +4293,11 @@ return x_30; } case 10: { -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_17, 1); +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_17, 0); lean_inc(x_31); +x_32 = lean_ctor_get(x_17, 1); +lean_inc(x_32); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -4299,26 +4305,46 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); +lean_inc(x_32); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_32 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2(x_1, x_2, x_3, x_4, x_5, x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_32) == 0) +x_33 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2(x_1, x_2, x_3, x_4, x_5, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); +lean_object* x_34; lean_object* x_35; size_t x_36; size_t x_37; uint8_t x_38; +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_ptr_addr(x_32); lean_dec(x_32); -x_35 = lean_expr_update_mdata(x_17, x_33); -x_36 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__3(x_1, x_2, x_3, x_4, x_5, x_35, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_34); -return x_36; +x_37 = lean_ptr_addr(x_34); +x_38 = lean_usize_dec_eq(x_36, x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +lean_dec(x_17); +x_39 = l_Lean_Expr_mdata___override(x_31, x_34); +x_40 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__3(x_1, x_2, x_3, x_4, x_5, x_39, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_35); +return x_40; } else { -uint8_t x_37; +lean_object* x_41; +lean_dec(x_34); +lean_dec(x_31); +x_41 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__3(x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_35); +return x_41; +} +} +else +{ +uint8_t x_42; +lean_dec(x_32); +lean_dec(x_31); lean_dec(x_17); lean_dec(x_13); lean_dec(x_12); @@ -4331,31 +4357,35 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_37 = !lean_is_exclusive(x_32); -if (x_37 == 0) +x_42 = !lean_is_exclusive(x_33); +if (x_42 == 0) { -return x_32; +return x_33; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_32, 0); -x_39 = lean_ctor_get(x_32, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_32); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_33, 0); +x_44 = lean_ctor_get(x_33, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_33); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } case 11: { -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_17, 2); -lean_inc(x_41); +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_46 = lean_ctor_get(x_17, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_17, 1); +lean_inc(x_47); +x_48 = lean_ctor_get(x_17, 2); +lean_inc(x_48); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -4363,26 +4393,48 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); +lean_inc(x_48); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_42 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2(x_1, x_2, x_3, x_4, x_5, x_41, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_42) == 0) +x_49 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2(x_1, x_2, x_3, x_4, x_5, x_48, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_49) == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_expr_update_proj(x_17, x_43); -x_46 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__3(x_1, x_2, x_3, x_4, x_5, x_45, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_44); -return x_46; +lean_object* x_50; lean_object* x_51; size_t x_52; size_t x_53; uint8_t x_54; +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = lean_ptr_addr(x_48); +lean_dec(x_48); +x_53 = lean_ptr_addr(x_50); +x_54 = lean_usize_dec_eq(x_52, x_53); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; +lean_dec(x_17); +x_55 = l_Lean_Expr_proj___override(x_46, x_47, x_50); +x_56 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__3(x_1, x_2, x_3, x_4, x_5, x_55, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_51); +return x_56; } else { -uint8_t x_47; +lean_object* x_57; +lean_dec(x_50); +lean_dec(x_47); +lean_dec(x_46); +x_57 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__3(x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_51); +return x_57; +} +} +else +{ +uint8_t x_58; +lean_dec(x_48); +lean_dec(x_47); +lean_dec(x_46); lean_dec(x_17); lean_dec(x_13); lean_dec(x_12); @@ -4395,31 +4447,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_47 = !lean_is_exclusive(x_42); -if (x_47 == 0) +x_58 = !lean_is_exclusive(x_49); +if (x_58 == 0) { -return x_42; +return x_49; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_42, 0); -x_49 = lean_ctor_get(x_42, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_42); -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_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_49, 0); +x_60 = lean_ctor_get(x_49, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_49); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } } default: { -lean_object* x_51; -x_51 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__3(x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_51; +lean_object* x_62; +x_62 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__3(x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_62; } } } @@ -8679,8 +8731,8 @@ else lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; lean_dec(x_9); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); -x_15 = l_Lean_Expr_getAppNumArgsAux(x_2, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_15 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_13); x_16 = lean_nat_dec_eq(x_14, x_15); lean_dec(x_15); lean_dec(x_14); @@ -8908,7 +8960,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Match_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath_goIndex___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath_goIndex___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_findDiscrRefinementPath_goIndex___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10027,7 +10079,7 @@ x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); lean_dec(x_37); x_39 = lean_unsigned_to_nat(0u); -x_40 = l_Lean_Expr_getAppNumArgsAux(x_9, x_39); +x_40 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_39); x_41 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_40); x_42 = lean_mk_array(x_40, x_41); @@ -10035,7 +10087,7 @@ x_43 = lean_unsigned_to_nat(1u); x_44 = lean_nat_sub(x_40, x_43); lean_dec(x_40); x_45 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_42, x_44); -x_46 = l_Lean_Expr_getAppNumArgsAux(x_13, x_39); +x_46 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_13, x_39); lean_inc(x_46); x_47 = lean_mk_array(x_46, x_41); x_48 = lean_nat_sub(x_46, x_43); @@ -10332,7 +10384,7 @@ x_102 = lean_ctor_get(x_101, 0); lean_inc(x_102); lean_dec(x_101); x_103 = lean_unsigned_to_nat(0u); -x_104 = l_Lean_Expr_getAppNumArgsAux(x_9, x_103); +x_104 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_103); x_105 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_104); x_106 = lean_mk_array(x_104, x_105); @@ -10340,7 +10392,7 @@ x_107 = lean_unsigned_to_nat(1u); x_108 = lean_nat_sub(x_104, x_107); lean_dec(x_104); x_109 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_106, x_108); -x_110 = l_Lean_Expr_getAppNumArgsAux(x_13, x_103); +x_110 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_13, x_103); lean_inc(x_110); x_111 = lean_mk_array(x_110, x_105); x_112 = lean_nat_sub(x_110, x_107); @@ -10658,7 +10710,7 @@ x_165 = lean_ctor_get(x_164, 0); lean_inc(x_165); lean_dec(x_164); x_166 = lean_unsigned_to_nat(0u); -x_167 = l_Lean_Expr_getAppNumArgsAux(x_9, x_166); +x_167 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_166); x_168 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_167); x_169 = lean_mk_array(x_167, x_168); @@ -10666,7 +10718,7 @@ x_170 = lean_unsigned_to_nat(1u); x_171 = lean_nat_sub(x_167, x_170); lean_dec(x_167); x_172 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_169, x_171); -x_173 = l_Lean_Expr_getAppNumArgsAux(x_13, x_166); +x_173 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_13, x_166); lean_inc(x_173); x_174 = lean_mk_array(x_173, x_168); x_175 = lean_nat_sub(x_173, x_170); @@ -11112,7 +11164,7 @@ x_246 = lean_ctor_get(x_245, 0); lean_inc(x_246); lean_dec(x_245); x_247 = lean_unsigned_to_nat(0u); -x_248 = l_Lean_Expr_getAppNumArgsAux(x_9, x_247); +x_248 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_247); x_249 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_248); x_250 = lean_mk_array(x_248, x_249); @@ -11120,7 +11172,7 @@ x_251 = lean_unsigned_to_nat(1u); x_252 = lean_nat_sub(x_248, x_251); lean_dec(x_248); x_253 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_250, x_252); -x_254 = l_Lean_Expr_getAppNumArgsAux(x_223, x_247); +x_254 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_223, x_247); lean_inc(x_254); x_255 = lean_mk_array(x_254, x_249); x_256 = lean_nat_sub(x_254, x_251); @@ -12939,7 +12991,7 @@ x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); lean_dec(x_34); x_36 = lean_unsigned_to_nat(0u); -x_37 = l_Lean_Expr_getAppNumArgsAux(x_9, x_36); +x_37 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_36); x_38 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_37); x_39 = lean_mk_array(x_37, x_38); @@ -12947,7 +12999,7 @@ x_40 = lean_unsigned_to_nat(1u); x_41 = lean_nat_sub(x_37, x_40); lean_dec(x_37); x_42 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_39, x_41); -x_43 = l_Lean_Expr_getAppNumArgsAux(x_12, x_36); +x_43 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_12, x_36); lean_inc(x_43); x_44 = lean_mk_array(x_43, x_38); x_45 = lean_nat_sub(x_43, x_40); @@ -13170,7 +13222,7 @@ x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); lean_dec(x_82); x_84 = lean_unsigned_to_nat(0u); -x_85 = l_Lean_Expr_getAppNumArgsAux(x_9, x_84); +x_85 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_84); x_86 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_85); x_87 = lean_mk_array(x_85, x_86); @@ -13178,7 +13230,7 @@ x_88 = lean_unsigned_to_nat(1u); x_89 = lean_nat_sub(x_85, x_88); lean_dec(x_85); x_90 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_87, x_89); -x_91 = l_Lean_Expr_getAppNumArgsAux(x_12, x_84); +x_91 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_12, x_84); lean_inc(x_91); x_92 = lean_mk_array(x_91, x_86); x_93 = lean_nat_sub(x_91, x_88); @@ -13425,7 +13477,7 @@ x_133 = lean_ctor_get(x_132, 0); lean_inc(x_133); lean_dec(x_132); x_134 = lean_unsigned_to_nat(0u); -x_135 = l_Lean_Expr_getAppNumArgsAux(x_9, x_134); +x_135 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_134); x_136 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_135); x_137 = lean_mk_array(x_135, x_136); @@ -13433,7 +13485,7 @@ x_138 = lean_unsigned_to_nat(1u); x_139 = lean_nat_sub(x_135, x_138); lean_dec(x_135); x_140 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_137, x_139); -x_141 = l_Lean_Expr_getAppNumArgsAux(x_12, x_134); +x_141 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_12, x_134); lean_inc(x_141); x_142 = lean_mk_array(x_141, x_136); x_143 = lean_nat_sub(x_141, x_138); @@ -13943,7 +13995,7 @@ x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); lean_dec(x_20); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_9, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_22); x_24 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -14148,7 +14200,7 @@ x_69 = lean_ctor_get(x_68, 0); lean_inc(x_69); lean_dec(x_68); x_70 = lean_unsigned_to_nat(0u); -x_71 = l_Lean_Expr_getAppNumArgsAux(x_9, x_70); +x_71 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_70); x_72 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_71); x_73 = lean_mk_array(x_71, x_72); @@ -14385,7 +14437,7 @@ x_121 = lean_ctor_get(x_119, 0); lean_inc(x_121); lean_dec(x_119); x_122 = lean_unsigned_to_nat(0u); -x_123 = l_Lean_Expr_getAppNumArgsAux(x_9, x_122); +x_123 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_122); x_124 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_123); x_125 = lean_mk_array(x_123, x_124); @@ -14668,7 +14720,7 @@ x_180 = lean_ctor_get(x_178, 0); lean_inc(x_180); lean_dec(x_178); x_181 = lean_unsigned_to_nat(0u); -x_182 = l_Lean_Expr_getAppNumArgsAux(x_167, x_181); +x_182 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_167, x_181); x_183 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_182); x_184 = lean_mk_array(x_182, x_183); @@ -20084,7 +20136,7 @@ x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); lean_dec(x_47); x_49 = lean_unsigned_to_nat(0u); -x_50 = l_Lean_Expr_getAppNumArgsAux(x_1, x_49); +x_50 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_49); x_51 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_50); x_52 = lean_mk_array(x_50, x_51); @@ -20456,7 +20508,7 @@ x_130 = lean_ctor_get(x_14, 0); lean_inc(x_130); lean_dec(x_14); x_131 = lean_unsigned_to_nat(0u); -x_132 = l_Lean_Expr_getAppNumArgsAux(x_130, x_131); +x_132 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_130, x_131); x_133 = lean_unsigned_to_nat(1u); x_134 = lean_nat_sub(x_132, x_133); x_135 = lean_nat_sub(x_134, x_133); @@ -20956,7 +21008,7 @@ else { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; x_6 = lean_unsigned_to_nat(0u); -x_7 = l_Lean_Expr_getAppNumArgsAux(x_1, x_6); +x_7 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_6); x_8 = lean_unsigned_to_nat(2u); x_9 = lean_nat_sub(x_7, x_8); x_10 = lean_unsigned_to_nat(1u); @@ -21463,7 +21515,7 @@ x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); lean_dec(x_22); x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_Expr_getAppNumArgsAux(x_1, x_24); +x_25 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_24); x_26 = l_Lean_Meta_transform_visit___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrs___spec__2___lambda__1___closed__1; lean_inc(x_25); x_27 = lean_mk_array(x_25, x_26); @@ -21630,7 +21682,7 @@ x_72 = lean_ctor_get(x_9, 0); lean_inc(x_72); lean_dec(x_9); x_73 = lean_unsigned_to_nat(0u); -x_74 = l_Lean_Expr_getAppNumArgsAux(x_72, x_73); +x_74 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_72, x_73); x_75 = lean_unsigned_to_nat(2u); x_76 = lean_nat_sub(x_74, x_75); x_77 = lean_unsigned_to_nat(1u); @@ -23636,7 +23688,7 @@ lean_inc(x_10); x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); -x_12 = lean_ctor_get(x_10, 4); +x_12 = lean_ctor_get(x_10, 5); lean_inc(x_12); lean_dec(x_10); x_13 = lean_ctor_get(x_12, 1); @@ -23649,7 +23701,7 @@ lean_dec(x_14); x_16 = lean_st_ref_take(x_1, x_15); x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 4); +x_18 = lean_ctor_get(x_17, 5); lean_inc(x_18); x_19 = lean_ctor_get(x_16, 1); lean_inc(x_19); @@ -23658,7 +23710,7 @@ x_20 = !lean_is_exclusive(x_17); if (x_20 == 0) { lean_object* x_21; uint8_t x_22; -x_21 = lean_ctor_get(x_17, 4); +x_21 = lean_ctor_get(x_17, 5); lean_dec(x_21); x_22 = !lean_is_exclusive(x_18); if (x_22 == 0) @@ -23702,7 +23754,7 @@ x_33 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_33, 0, x_31); lean_ctor_set(x_33, 1, x_32); lean_ctor_set_uint8(x_33, sizeof(void*)*2, x_30); -lean_ctor_set(x_17, 4, x_33); +lean_ctor_set(x_17, 5, x_33); x_34 = lean_st_ref_set(x_1, x_17, x_19); x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); @@ -23726,61 +23778,64 @@ return x_37; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_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_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; x_38 = lean_ctor_get(x_17, 0); x_39 = lean_ctor_get(x_17, 1); x_40 = lean_ctor_get(x_17, 2); x_41 = lean_ctor_get(x_17, 3); +x_42 = lean_ctor_get(x_17, 4); +lean_inc(x_42); lean_inc(x_41); lean_inc(x_40); lean_inc(x_39); lean_inc(x_38); lean_dec(x_17); -x_42 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); -x_43 = lean_ctor_get(x_18, 0); -lean_inc(x_43); +x_43 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); +x_44 = lean_ctor_get(x_18, 0); +lean_inc(x_44); if (lean_is_exclusive(x_18)) { lean_ctor_release(x_18, 0); lean_ctor_release(x_18, 1); - x_44 = x_18; + x_45 = x_18; } else { lean_dec_ref(x_18); - x_44 = lean_box(0); + x_45 = lean_box(0); } -x_45 = l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___spec__4___rarg___closed__3; -if (lean_is_scalar(x_44)) { - x_46 = lean_alloc_ctor(0, 2, 1); +x_46 = l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___spec__4___rarg___closed__3; +if (lean_is_scalar(x_45)) { + x_47 = lean_alloc_ctor(0, 2, 1); } else { - x_46 = x_44; + x_47 = x_45; } -lean_ctor_set(x_46, 0, x_43); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_42); -x_47 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_47, 0, x_38); -lean_ctor_set(x_47, 1, x_39); -lean_ctor_set(x_47, 2, x_40); -lean_ctor_set(x_47, 3, x_41); -lean_ctor_set(x_47, 4, x_46); -x_48 = lean_st_ref_set(x_1, x_47, x_19); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; +lean_ctor_set(x_47, 0, x_44); +lean_ctor_set(x_47, 1, x_46); +lean_ctor_set_uint8(x_47, sizeof(void*)*2, x_43); +x_48 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_48, 0, x_38); +lean_ctor_set(x_48, 1, x_39); +lean_ctor_set(x_48, 2, x_40); +lean_ctor_set(x_48, 3, x_41); +lean_ctor_set(x_48, 4, x_42); +lean_ctor_set(x_48, 5, x_47); +x_49 = lean_st_ref_set(x_1, x_48, x_19); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_51 = x_49; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_49); + x_51 = lean_box(0); } -if (lean_is_scalar(x_50)) { - x_51 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_51)) { + x_52 = lean_alloc_ctor(0, 2, 0); } else { - x_51 = x_50; + x_52 = x_51; } -lean_ctor_set(x_51, 0, x_13); -lean_ctor_set(x_51, 1, x_49); -return x_51; +lean_ctor_set(x_52, 0, x_13); +lean_ctor_set(x_52, 1, x_50); +return x_52; } } } @@ -23803,7 +23858,7 @@ lean_dec(x_24); x_26 = lean_st_ref_get(x_5, x_25); x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -x_28 = lean_ctor_get(x_27, 4); +x_28 = lean_ctor_get(x_27, 5); lean_inc(x_28); lean_dec(x_27); x_29 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); @@ -23868,7 +23923,7 @@ lean_dec(x_45); x_47 = lean_st_ref_take(x_5, x_46); x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); -x_49 = lean_ctor_get(x_48, 4); +x_49 = lean_ctor_get(x_48, 5); lean_inc(x_49); if (lean_obj_tag(x_43) == 0) { @@ -23880,7 +23935,7 @@ x_51 = !lean_is_exclusive(x_48); if (x_51 == 0) { lean_object* x_52; uint8_t x_53; -x_52 = lean_ctor_get(x_48, 4); +x_52 = lean_ctor_get(x_48, 5); lean_dec(x_52); x_53 = !lean_is_exclusive(x_49); if (x_53 == 0) @@ -23948,7 +24003,7 @@ x_73 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_73, 0, x_68); lean_ctor_set(x_73, 1, x_72); lean_ctor_set_uint8(x_73, sizeof(void*)*2, x_67); -lean_ctor_set(x_48, 4, x_73); +lean_ctor_set(x_48, 5, x_73); x_74 = lean_st_ref_set(x_5, x_48, x_50); lean_dec(x_5); x_75 = lean_ctor_get(x_74, 1); @@ -23978,439 +24033,448 @@ goto block_23; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; x_80 = lean_ctor_get(x_48, 0); x_81 = lean_ctor_get(x_48, 1); x_82 = lean_ctor_get(x_48, 2); x_83 = lean_ctor_get(x_48, 3); +x_84 = lean_ctor_get(x_48, 4); +lean_inc(x_84); lean_inc(x_83); lean_inc(x_82); lean_inc(x_81); lean_inc(x_80); lean_dec(x_48); -x_84 = lean_ctor_get_uint8(x_49, sizeof(void*)*2); -x_85 = lean_ctor_get(x_49, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_49, 1); +x_85 = lean_ctor_get_uint8(x_49, sizeof(void*)*2); +x_86 = lean_ctor_get(x_49, 0); lean_inc(x_86); +x_87 = lean_ctor_get(x_49, 1); +lean_inc(x_87); if (lean_is_exclusive(x_49)) { lean_ctor_release(x_49, 0); lean_ctor_release(x_49, 1); - x_87 = x_49; + x_88 = x_49; } else { lean_dec_ref(x_49); - x_87 = lean_box(0); + x_88 = lean_box(0); } -x_88 = lean_ctor_get(x_43, 0); -lean_inc(x_88); +x_89 = lean_ctor_get(x_43, 0); +lean_inc(x_89); lean_dec(x_43); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_86); -x_90 = l_Std_PersistentArray_push___rarg(x_35, x_89); -if (lean_is_scalar(x_87)) { - x_91 = lean_alloc_ctor(0, 2, 1); +x_90 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_90, 0, x_89); +lean_ctor_set(x_90, 1, x_87); +x_91 = l_Std_PersistentArray_push___rarg(x_35, x_90); +if (lean_is_scalar(x_88)) { + x_92 = lean_alloc_ctor(0, 2, 1); } else { - x_91 = x_87; + x_92 = x_88; } -lean_ctor_set(x_91, 0, x_85); -lean_ctor_set(x_91, 1, x_90); -lean_ctor_set_uint8(x_91, sizeof(void*)*2, x_84); -x_92 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_92, 0, x_80); -lean_ctor_set(x_92, 1, x_81); -lean_ctor_set(x_92, 2, x_82); -lean_ctor_set(x_92, 3, x_83); -lean_ctor_set(x_92, 4, x_91); -x_93 = lean_st_ref_set(x_5, x_92, x_50); -lean_dec(x_5); -x_94 = lean_ctor_get(x_93, 1); -lean_inc(x_94); -if (lean_is_exclusive(x_93)) { - lean_ctor_release(x_93, 0); - lean_ctor_release(x_93, 1); - x_95 = x_93; +lean_ctor_set(x_92, 0, x_86); +lean_ctor_set(x_92, 1, x_91); +lean_ctor_set_uint8(x_92, sizeof(void*)*2, x_85); +x_93 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_93, 0, x_80); +lean_ctor_set(x_93, 1, x_81); +lean_ctor_set(x_93, 2, x_82); +lean_ctor_set(x_93, 3, x_83); +lean_ctor_set(x_93, 4, x_84); +lean_ctor_set(x_93, 5, x_92); +x_94 = lean_st_ref_set(x_5, x_93, x_50); +lean_dec(x_5); +x_95 = lean_ctor_get(x_94, 1); +lean_inc(x_95); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_96 = x_94; } else { - lean_dec_ref(x_93); - x_95 = lean_box(0); + lean_dec_ref(x_94); + x_96 = lean_box(0); } -x_96 = lean_box(0); -x_97 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_97, 0, x_39); -lean_ctor_set(x_97, 1, x_96); -if (lean_is_scalar(x_95)) { - x_98 = lean_alloc_ctor(0, 2, 0); +x_97 = lean_box(0); +x_98 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_98, 0, x_39); +lean_ctor_set(x_98, 1, x_97); +if (lean_is_scalar(x_96)) { + x_99 = lean_alloc_ctor(0, 2, 0); } else { - x_98 = x_95; + x_99 = x_96; } -lean_ctor_set(x_98, 0, x_97); -lean_ctor_set(x_98, 1, x_94); -x_11 = x_98; +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set(x_99, 1, x_95); +x_11 = x_99; goto block_23; } } else { -lean_object* x_99; uint8_t x_100; -x_99 = lean_ctor_get(x_47, 1); -lean_inc(x_99); +lean_object* x_100; uint8_t x_101; +x_100 = lean_ctor_get(x_47, 1); +lean_inc(x_100); lean_dec(x_47); -x_100 = !lean_is_exclusive(x_48); -if (x_100 == 0) +x_101 = !lean_is_exclusive(x_48); +if (x_101 == 0) { -lean_object* x_101; uint8_t x_102; -x_101 = lean_ctor_get(x_48, 4); -lean_dec(x_101); -x_102 = !lean_is_exclusive(x_49); -if (x_102 == 0) +lean_object* x_102; uint8_t x_103; +x_102 = lean_ctor_get(x_48, 5); +lean_dec(x_102); +x_103 = !lean_is_exclusive(x_49); +if (x_103 == 0) { -lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; -x_103 = lean_ctor_get(x_49, 1); -lean_dec(x_103); -x_104 = lean_ctor_get(x_43, 0); -lean_inc(x_104); +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; uint8_t x_109; +x_104 = lean_ctor_get(x_49, 1); +lean_dec(x_104); +x_105 = lean_ctor_get(x_43, 0); +lean_inc(x_105); lean_dec(x_43); -x_105 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_105, 0, x_104); -x_106 = l_Std_PersistentArray_push___rarg(x_35, x_105); -lean_ctor_set(x_49, 1, x_106); -x_107 = lean_st_ref_set(x_5, x_48, x_99); +x_106 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_106, 0, x_105); +x_107 = l_Std_PersistentArray_push___rarg(x_35, x_106); +lean_ctor_set(x_49, 1, x_107); +x_108 = lean_st_ref_set(x_5, x_48, x_100); lean_dec(x_5); -x_108 = !lean_is_exclusive(x_107); -if (x_108 == 0) +x_109 = !lean_is_exclusive(x_108); +if (x_109 == 0) { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_107, 0); -lean_dec(x_109); -x_110 = lean_box(0); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_39); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_107, 0, x_111); -x_11 = x_107; +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_108, 0); +lean_dec(x_110); +x_111 = lean_box(0); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_39); +lean_ctor_set(x_112, 1, x_111); +lean_ctor_set(x_108, 0, x_112); +x_11 = x_108; goto block_23; } else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -lean_dec(x_107); -x_113 = lean_box(0); -x_114 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_114, 0, x_39); -lean_ctor_set(x_114, 1, x_113); +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_113 = lean_ctor_get(x_108, 1); +lean_inc(x_113); +lean_dec(x_108); +x_114 = lean_box(0); x_115 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_115, 0, x_114); -lean_ctor_set(x_115, 1, x_112); -x_11 = x_115; +lean_ctor_set(x_115, 0, x_39); +lean_ctor_set(x_115, 1, x_114); +x_116 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_116, 0, x_115); +lean_ctor_set(x_116, 1, x_113); +x_11 = x_116; goto block_23; } } else { -uint8_t 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; -x_116 = lean_ctor_get_uint8(x_49, sizeof(void*)*2); -x_117 = lean_ctor_get(x_49, 0); -lean_inc(x_117); -lean_dec(x_49); -x_118 = lean_ctor_get(x_43, 0); +uint8_t x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_117 = lean_ctor_get_uint8(x_49, sizeof(void*)*2); +x_118 = lean_ctor_get(x_49, 0); lean_inc(x_118); +lean_dec(x_49); +x_119 = lean_ctor_get(x_43, 0); +lean_inc(x_119); lean_dec(x_43); -x_119 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_119, 0, x_118); -x_120 = l_Std_PersistentArray_push___rarg(x_35, x_119); -x_121 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_121, 0, x_117); -lean_ctor_set(x_121, 1, x_120); -lean_ctor_set_uint8(x_121, sizeof(void*)*2, x_116); -lean_ctor_set(x_48, 4, x_121); -x_122 = lean_st_ref_set(x_5, x_48, x_99); +x_120 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_120, 0, x_119); +x_121 = l_Std_PersistentArray_push___rarg(x_35, x_120); +x_122 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_122, 0, x_118); +lean_ctor_set(x_122, 1, x_121); +lean_ctor_set_uint8(x_122, sizeof(void*)*2, x_117); +lean_ctor_set(x_48, 5, x_122); +x_123 = lean_st_ref_set(x_5, x_48, x_100); lean_dec(x_5); -x_123 = lean_ctor_get(x_122, 1); -lean_inc(x_123); -if (lean_is_exclusive(x_122)) { - lean_ctor_release(x_122, 0); - lean_ctor_release(x_122, 1); - x_124 = x_122; -} else { - lean_dec_ref(x_122); - x_124 = lean_box(0); -} -x_125 = lean_box(0); -x_126 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_126, 0, x_39); -lean_ctor_set(x_126, 1, x_125); -if (lean_is_scalar(x_124)) { - x_127 = lean_alloc_ctor(0, 2, 0); -} else { - x_127 = x_124; -} -lean_ctor_set(x_127, 0, x_126); -lean_ctor_set(x_127, 1, x_123); -x_11 = x_127; +x_124 = lean_ctor_get(x_123, 1); +lean_inc(x_124); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_125 = x_123; +} else { + lean_dec_ref(x_123); + x_125 = lean_box(0); +} +x_126 = lean_box(0); +x_127 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_127, 0, x_39); +lean_ctor_set(x_127, 1, x_126); +if (lean_is_scalar(x_125)) { + x_128 = lean_alloc_ctor(0, 2, 0); +} else { + x_128 = x_125; +} +lean_ctor_set(x_128, 0, x_127); +lean_ctor_set(x_128, 1, x_124); +x_11 = x_128; goto block_23; } } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; uint8_t x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_128 = lean_ctor_get(x_48, 0); -x_129 = lean_ctor_get(x_48, 1); -x_130 = lean_ctor_get(x_48, 2); -x_131 = lean_ctor_get(x_48, 3); +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; uint8_t x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_129 = lean_ctor_get(x_48, 0); +x_130 = lean_ctor_get(x_48, 1); +x_131 = lean_ctor_get(x_48, 2); +x_132 = lean_ctor_get(x_48, 3); +x_133 = lean_ctor_get(x_48, 4); +lean_inc(x_133); +lean_inc(x_132); lean_inc(x_131); lean_inc(x_130); lean_inc(x_129); -lean_inc(x_128); lean_dec(x_48); -x_132 = lean_ctor_get_uint8(x_49, sizeof(void*)*2); -x_133 = lean_ctor_get(x_49, 0); -lean_inc(x_133); +x_134 = lean_ctor_get_uint8(x_49, sizeof(void*)*2); +x_135 = lean_ctor_get(x_49, 0); +lean_inc(x_135); if (lean_is_exclusive(x_49)) { lean_ctor_release(x_49, 0); lean_ctor_release(x_49, 1); - x_134 = x_49; + x_136 = x_49; } else { lean_dec_ref(x_49); - x_134 = lean_box(0); + x_136 = lean_box(0); } -x_135 = lean_ctor_get(x_43, 0); -lean_inc(x_135); +x_137 = lean_ctor_get(x_43, 0); +lean_inc(x_137); lean_dec(x_43); -x_136 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_136, 0, x_135); -x_137 = l_Std_PersistentArray_push___rarg(x_35, x_136); -if (lean_is_scalar(x_134)) { - x_138 = lean_alloc_ctor(0, 2, 1); -} else { - x_138 = x_134; -} -lean_ctor_set(x_138, 0, x_133); -lean_ctor_set(x_138, 1, x_137); -lean_ctor_set_uint8(x_138, sizeof(void*)*2, x_132); -x_139 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_139, 0, x_128); -lean_ctor_set(x_139, 1, x_129); -lean_ctor_set(x_139, 2, x_130); -lean_ctor_set(x_139, 3, x_131); -lean_ctor_set(x_139, 4, x_138); -x_140 = lean_st_ref_set(x_5, x_139, x_99); -lean_dec(x_5); -x_141 = lean_ctor_get(x_140, 1); -lean_inc(x_141); -if (lean_is_exclusive(x_140)) { - lean_ctor_release(x_140, 0); - lean_ctor_release(x_140, 1); - x_142 = x_140; -} else { - lean_dec_ref(x_140); - x_142 = lean_box(0); -} -x_143 = lean_box(0); -x_144 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_144, 0, x_39); -lean_ctor_set(x_144, 1, x_143); -if (lean_is_scalar(x_142)) { - x_145 = lean_alloc_ctor(0, 2, 0); -} else { - x_145 = x_142; -} -lean_ctor_set(x_145, 0, x_144); -lean_ctor_set(x_145, 1, x_141); -x_11 = x_145; +x_138 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_138, 0, x_137); +x_139 = l_Std_PersistentArray_push___rarg(x_35, x_138); +if (lean_is_scalar(x_136)) { + x_140 = lean_alloc_ctor(0, 2, 1); +} else { + x_140 = x_136; +} +lean_ctor_set(x_140, 0, x_135); +lean_ctor_set(x_140, 1, x_139); +lean_ctor_set_uint8(x_140, sizeof(void*)*2, x_134); +x_141 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_141, 0, x_129); +lean_ctor_set(x_141, 1, x_130); +lean_ctor_set(x_141, 2, x_131); +lean_ctor_set(x_141, 3, x_132); +lean_ctor_set(x_141, 4, x_133); +lean_ctor_set(x_141, 5, x_140); +x_142 = lean_st_ref_set(x_5, x_141, x_100); +lean_dec(x_5); +x_143 = lean_ctor_get(x_142, 1); +lean_inc(x_143); +if (lean_is_exclusive(x_142)) { + lean_ctor_release(x_142, 0); + lean_ctor_release(x_142, 1); + x_144 = x_142; +} else { + lean_dec_ref(x_142); + x_144 = lean_box(0); +} +x_145 = lean_box(0); +x_146 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_146, 0, x_39); +lean_ctor_set(x_146, 1, x_145); +if (lean_is_scalar(x_144)) { + x_147 = lean_alloc_ctor(0, 2, 0); +} else { + x_147 = x_144; +} +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_143); +x_11 = x_147; goto block_23; } } } else { -uint8_t x_146; +uint8_t x_148; lean_dec(x_39); lean_dec(x_35); lean_dec(x_9); lean_dec(x_5); -x_146 = !lean_is_exclusive(x_42); -if (x_146 == 0) +x_148 = !lean_is_exclusive(x_42); +if (x_148 == 0) { x_11 = x_42; goto block_23; } else { -lean_object* x_147; lean_object* x_148; lean_object* x_149; -x_147 = lean_ctor_get(x_42, 0); -x_148 = lean_ctor_get(x_42, 1); -lean_inc(x_148); -lean_inc(x_147); +lean_object* x_149; lean_object* x_150; lean_object* x_151; +x_149 = lean_ctor_get(x_42, 0); +x_150 = lean_ctor_get(x_42, 1); +lean_inc(x_150); +lean_inc(x_149); lean_dec(x_42); -x_149 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_149, 0, x_147); -lean_ctor_set(x_149, 1, x_148); -x_11 = x_149; +x_151 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_151, 0, x_149); +lean_ctor_set(x_151, 1, x_150); +x_11 = x_151; goto block_23; } } } else { -lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; uint8_t x_158; +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; uint8_t x_160; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_2); -x_150 = lean_ctor_get(x_38, 0); -lean_inc(x_150); -x_151 = lean_ctor_get(x_38, 1); -lean_inc(x_151); +x_152 = lean_ctor_get(x_38, 0); +lean_inc(x_152); +x_153 = lean_ctor_get(x_38, 1); +lean_inc(x_153); lean_dec(x_38); -x_152 = lean_st_ref_get(x_9, x_151); +x_154 = lean_st_ref_get(x_9, x_153); lean_dec(x_9); -x_153 = lean_ctor_get(x_152, 1); -lean_inc(x_153); -lean_dec(x_152); -x_154 = lean_st_ref_take(x_5, x_153); -x_155 = lean_ctor_get(x_154, 0); +x_155 = lean_ctor_get(x_154, 1); lean_inc(x_155); -x_156 = lean_ctor_get(x_155, 4); -lean_inc(x_156); -x_157 = lean_ctor_get(x_154, 1); -lean_inc(x_157); lean_dec(x_154); -x_158 = !lean_is_exclusive(x_155); -if (x_158 == 0) -{ -lean_object* x_159; uint8_t x_160; -x_159 = lean_ctor_get(x_155, 4); -lean_dec(x_159); -x_160 = !lean_is_exclusive(x_156); +x_156 = lean_st_ref_take(x_5, x_155); +x_157 = lean_ctor_get(x_156, 0); +lean_inc(x_157); +x_158 = lean_ctor_get(x_157, 5); +lean_inc(x_158); +x_159 = lean_ctor_get(x_156, 1); +lean_inc(x_159); +lean_dec(x_156); +x_160 = !lean_is_exclusive(x_157); if (x_160 == 0) { -lean_object* x_161; lean_object* x_162; uint8_t x_163; -x_161 = lean_ctor_get(x_156, 1); +lean_object* x_161; uint8_t x_162; +x_161 = lean_ctor_get(x_157, 5); lean_dec(x_161); -lean_ctor_set(x_156, 1, x_35); -x_162 = lean_st_ref_set(x_5, x_155, x_157); +x_162 = !lean_is_exclusive(x_158); +if (x_162 == 0) +{ +lean_object* x_163; lean_object* x_164; uint8_t x_165; +x_163 = lean_ctor_get(x_158, 1); +lean_dec(x_163); +lean_ctor_set(x_158, 1, x_35); +x_164 = lean_st_ref_set(x_5, x_157, x_159); lean_dec(x_5); -x_163 = !lean_is_exclusive(x_162); -if (x_163 == 0) +x_165 = !lean_is_exclusive(x_164); +if (x_165 == 0) { -lean_object* x_164; -x_164 = lean_ctor_get(x_162, 0); -lean_dec(x_164); -lean_ctor_set_tag(x_162, 1); -lean_ctor_set(x_162, 0, x_150); -x_11 = x_162; +lean_object* x_166; +x_166 = lean_ctor_get(x_164, 0); +lean_dec(x_166); +lean_ctor_set_tag(x_164, 1); +lean_ctor_set(x_164, 0, x_152); +x_11 = x_164; goto block_23; } else { -lean_object* x_165; lean_object* x_166; -x_165 = lean_ctor_get(x_162, 1); -lean_inc(x_165); -lean_dec(x_162); -x_166 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_166, 0, x_150); -lean_ctor_set(x_166, 1, x_165); -x_11 = x_166; +lean_object* x_167; lean_object* x_168; +x_167 = lean_ctor_get(x_164, 1); +lean_inc(x_167); +lean_dec(x_164); +x_168 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_168, 0, x_152); +lean_ctor_set(x_168, 1, x_167); +x_11 = x_168; goto block_23; } } else { -uint8_t x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -x_167 = lean_ctor_get_uint8(x_156, sizeof(void*)*2); -x_168 = lean_ctor_get(x_156, 0); -lean_inc(x_168); -lean_dec(x_156); -x_169 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_169, 0, x_168); -lean_ctor_set(x_169, 1, x_35); -lean_ctor_set_uint8(x_169, sizeof(void*)*2, x_167); -lean_ctor_set(x_155, 4, x_169); -x_170 = lean_st_ref_set(x_5, x_155, x_157); +uint8_t x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_169 = lean_ctor_get_uint8(x_158, sizeof(void*)*2); +x_170 = lean_ctor_get(x_158, 0); +lean_inc(x_170); +lean_dec(x_158); +x_171 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_171, 0, x_170); +lean_ctor_set(x_171, 1, x_35); +lean_ctor_set_uint8(x_171, sizeof(void*)*2, x_169); +lean_ctor_set(x_157, 5, x_171); +x_172 = lean_st_ref_set(x_5, x_157, x_159); lean_dec(x_5); -x_171 = lean_ctor_get(x_170, 1); -lean_inc(x_171); -if (lean_is_exclusive(x_170)) { - lean_ctor_release(x_170, 0); - lean_ctor_release(x_170, 1); - x_172 = x_170; +x_173 = lean_ctor_get(x_172, 1); +lean_inc(x_173); +if (lean_is_exclusive(x_172)) { + lean_ctor_release(x_172, 0); + lean_ctor_release(x_172, 1); + x_174 = x_172; } else { - lean_dec_ref(x_170); - x_172 = lean_box(0); + lean_dec_ref(x_172); + x_174 = lean_box(0); } -if (lean_is_scalar(x_172)) { - x_173 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_174)) { + x_175 = lean_alloc_ctor(1, 2, 0); } else { - x_173 = x_172; - lean_ctor_set_tag(x_173, 1); + x_175 = x_174; + lean_ctor_set_tag(x_175, 1); } -lean_ctor_set(x_173, 0, x_150); -lean_ctor_set(x_173, 1, x_171); -x_11 = x_173; +lean_ctor_set(x_175, 0, x_152); +lean_ctor_set(x_175, 1, x_173); +x_11 = x_175; goto block_23; } } else { -lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; uint8_t 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; -x_174 = lean_ctor_get(x_155, 0); -x_175 = lean_ctor_get(x_155, 1); -x_176 = lean_ctor_get(x_155, 2); -x_177 = lean_ctor_get(x_155, 3); +lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; uint8_t x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; +x_176 = lean_ctor_get(x_157, 0); +x_177 = lean_ctor_get(x_157, 1); +x_178 = lean_ctor_get(x_157, 2); +x_179 = lean_ctor_get(x_157, 3); +x_180 = lean_ctor_get(x_157, 4); +lean_inc(x_180); +lean_inc(x_179); +lean_inc(x_178); lean_inc(x_177); lean_inc(x_176); -lean_inc(x_175); -lean_inc(x_174); -lean_dec(x_155); -x_178 = lean_ctor_get_uint8(x_156, sizeof(void*)*2); -x_179 = lean_ctor_get(x_156, 0); -lean_inc(x_179); -if (lean_is_exclusive(x_156)) { - lean_ctor_release(x_156, 0); - lean_ctor_release(x_156, 1); - x_180 = x_156; -} else { - lean_dec_ref(x_156); - x_180 = lean_box(0); -} -if (lean_is_scalar(x_180)) { - x_181 = lean_alloc_ctor(0, 2, 1); +lean_dec(x_157); +x_181 = lean_ctor_get_uint8(x_158, sizeof(void*)*2); +x_182 = lean_ctor_get(x_158, 0); +lean_inc(x_182); +if (lean_is_exclusive(x_158)) { + lean_ctor_release(x_158, 0); + lean_ctor_release(x_158, 1); + x_183 = x_158; } else { - x_181 = x_180; -} -lean_ctor_set(x_181, 0, x_179); -lean_ctor_set(x_181, 1, x_35); -lean_ctor_set_uint8(x_181, sizeof(void*)*2, x_178); -x_182 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_182, 0, x_174); -lean_ctor_set(x_182, 1, x_175); -lean_ctor_set(x_182, 2, x_176); -lean_ctor_set(x_182, 3, x_177); -lean_ctor_set(x_182, 4, x_181); -x_183 = lean_st_ref_set(x_5, x_182, x_157); -lean_dec(x_5); -x_184 = lean_ctor_get(x_183, 1); -lean_inc(x_184); -if (lean_is_exclusive(x_183)) { - lean_ctor_release(x_183, 0); - lean_ctor_release(x_183, 1); - x_185 = x_183; + lean_dec_ref(x_158); + x_183 = lean_box(0); +} +if (lean_is_scalar(x_183)) { + x_184 = lean_alloc_ctor(0, 2, 1); +} else { + x_184 = x_183; +} +lean_ctor_set(x_184, 0, x_182); +lean_ctor_set(x_184, 1, x_35); +lean_ctor_set_uint8(x_184, sizeof(void*)*2, x_181); +x_185 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_185, 0, x_176); +lean_ctor_set(x_185, 1, x_177); +lean_ctor_set(x_185, 2, x_178); +lean_ctor_set(x_185, 3, x_179); +lean_ctor_set(x_185, 4, x_180); +lean_ctor_set(x_185, 5, x_184); +x_186 = lean_st_ref_set(x_5, x_185, x_159); +lean_dec(x_5); +x_187 = lean_ctor_get(x_186, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_186)) { + lean_ctor_release(x_186, 0); + lean_ctor_release(x_186, 1); + x_188 = x_186; } else { - lean_dec_ref(x_183); - x_185 = lean_box(0); + lean_dec_ref(x_186); + x_188 = lean_box(0); } -if (lean_is_scalar(x_185)) { - x_186 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_188)) { + x_189 = lean_alloc_ctor(1, 2, 0); } else { - x_186 = x_185; - lean_ctor_set_tag(x_186, 1); + x_189 = x_188; + lean_ctor_set_tag(x_189, 1); } -lean_ctor_set(x_186, 0, x_150); -lean_ctor_set(x_186, 1, x_184); -x_11 = x_186; +lean_ctor_set(x_189, 0, x_152); +lean_ctor_set(x_189, 1, x_187); +x_11 = x_189; goto block_23; } } @@ -24737,13 +24801,14 @@ return x_30; } case 6: { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; x_31 = lean_ctor_get(x_1, 0); lean_inc(x_31); x_32 = lean_ctor_get(x_1, 1); lean_inc(x_32); x_33 = lean_ctor_get(x_1, 2); lean_inc(x_33); +x_34 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); lean_dec(x_1); lean_inc(x_8); lean_inc(x_7); @@ -24751,19 +24816,18 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_34 = l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go(x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_34) == 0) +x_35 = l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go(x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_35) == 0) { -lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_35, 0); lean_inc(x_36); -lean_dec(x_34); -x_37 = l_Lean_Expr_binderInfo(x_33); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); x_38 = lean_alloc_closure((void*)(l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___lambda__1___boxed), 10, 1); lean_closure_set(x_38, 0, x_33); -x_39 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___spec__1___rarg(x_31, x_37, x_35, x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_36); +x_39 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___spec__1___rarg(x_31, x_34, x_36, x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_37); return x_39; } else @@ -24777,19 +24841,19 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_40 = !lean_is_exclusive(x_34); +x_40 = !lean_is_exclusive(x_35); if (x_40 == 0) { -return x_34; +return x_35; } else { lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_34, 0); -x_42 = lean_ctor_get(x_34, 1); +x_41 = lean_ctor_get(x_35, 0); +x_42 = lean_ctor_get(x_35, 1); lean_inc(x_42); lean_inc(x_41); -lean_dec(x_34); +lean_dec(x_35); x_43 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_43, 0, x_41); lean_ctor_set(x_43, 1, x_42); @@ -24799,13 +24863,14 @@ return x_43; } case 7: { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +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_1, 0); lean_inc(x_44); x_45 = lean_ctor_get(x_1, 1); lean_inc(x_45); x_46 = lean_ctor_get(x_1, 2); lean_inc(x_46); +x_47 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); lean_dec(x_1); lean_inc(x_8); lean_inc(x_7); @@ -24813,19 +24878,18 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_47 = l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go(x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_47) == 0) +x_48 = l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go(x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_49 = lean_ctor_get(x_48, 0); lean_inc(x_49); -lean_dec(x_47); -x_50 = l_Lean_Expr_binderInfo(x_46); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); x_51 = lean_alloc_closure((void*)(l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___lambda__2___boxed), 10, 1); lean_closure_set(x_51, 0, x_46); -x_52 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___spec__1___rarg(x_44, x_50, x_48, x_51, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_49); +x_52 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go___spec__1___rarg(x_44, x_47, x_49, x_51, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_50); return x_52; } else @@ -24839,19 +24903,19 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_53 = !lean_is_exclusive(x_47); +x_53 = !lean_is_exclusive(x_48); if (x_53 == 0) { -return x_47; +return x_48; } else { lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_47, 0); -x_55 = lean_ctor_get(x_47, 1); +x_54 = lean_ctor_get(x_48, 0); +x_55 = lean_ctor_get(x_48, 1); lean_inc(x_55); lean_inc(x_54); -lean_dec(x_47); +lean_dec(x_48); x_56 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_56, 0, x_54); lean_ctor_set(x_56, 1, x_55); @@ -25120,74 +25184,119 @@ return x_111; } case 11: { -lean_object* x_112; lean_object* x_113; -x_112 = lean_ctor_get(x_1, 2); +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_112 = lean_ctor_get(x_1, 0); lean_inc(x_112); -x_113 = l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go(x_112, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_113) == 0) +x_113 = lean_ctor_get(x_1, 1); +lean_inc(x_113); +x_114 = lean_ctor_get(x_1, 2); +lean_inc(x_114); +lean_inc(x_114); +x_115 = l_Lean_Elab_Term_ToDepElimPattern_savePatternInfo_go(x_114, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_115) == 0) { -uint8_t x_114; -x_114 = !lean_is_exclusive(x_113); -if (x_114 == 0) +uint8_t x_116; +x_116 = !lean_is_exclusive(x_115); +if (x_116 == 0) { -lean_object* x_115; lean_object* x_116; -x_115 = lean_ctor_get(x_113, 0); -x_116 = lean_expr_update_proj(x_1, x_115); -lean_ctor_set(x_113, 0, x_116); -return x_113; +lean_object* x_117; size_t x_118; size_t x_119; uint8_t x_120; +x_117 = lean_ctor_get(x_115, 0); +x_118 = lean_ptr_addr(x_114); +lean_dec(x_114); +x_119 = lean_ptr_addr(x_117); +x_120 = lean_usize_dec_eq(x_118, x_119); +if (x_120 == 0) +{ +lean_object* x_121; +lean_dec(x_1); +x_121 = l_Lean_Expr_proj___override(x_112, x_113, x_117); +lean_ctor_set(x_115, 0, x_121); +return x_115; } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_117 = lean_ctor_get(x_113, 0); -x_118 = lean_ctor_get(x_113, 1); -lean_inc(x_118); -lean_inc(x_117); +lean_dec(x_117); lean_dec(x_113); -x_119 = lean_expr_update_proj(x_1, x_117); -x_120 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_120, 0, x_119); -lean_ctor_set(x_120, 1, x_118); -return x_120; +lean_dec(x_112); +lean_ctor_set(x_115, 0, x_1); +return x_115; } } else { -uint8_t x_121; +lean_object* x_122; lean_object* x_123; size_t x_124; size_t x_125; uint8_t x_126; +x_122 = lean_ctor_get(x_115, 0); +x_123 = lean_ctor_get(x_115, 1); +lean_inc(x_123); +lean_inc(x_122); +lean_dec(x_115); +x_124 = lean_ptr_addr(x_114); +lean_dec(x_114); +x_125 = lean_ptr_addr(x_122); +x_126 = lean_usize_dec_eq(x_124, x_125); +if (x_126 == 0) +{ +lean_object* x_127; lean_object* x_128; lean_dec(x_1); -x_121 = !lean_is_exclusive(x_113); -if (x_121 == 0) +x_127 = l_Lean_Expr_proj___override(x_112, x_113, x_122); +x_128 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_128, 0, x_127); +lean_ctor_set(x_128, 1, x_123); +return x_128; +} +else { -return x_113; +lean_object* x_129; +lean_dec(x_122); +lean_dec(x_113); +lean_dec(x_112); +x_129 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_129, 0, x_1); +lean_ctor_set(x_129, 1, x_123); +return x_129; +} +} } else { -lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_122 = lean_ctor_get(x_113, 0); -x_123 = lean_ctor_get(x_113, 1); -lean_inc(x_123); -lean_inc(x_122); +uint8_t x_130; +lean_dec(x_114); lean_dec(x_113); -x_124 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_124, 0, x_122); -lean_ctor_set(x_124, 1, x_123); -return x_124; +lean_dec(x_112); +lean_dec(x_1); +x_130 = !lean_is_exclusive(x_115); +if (x_130 == 0) +{ +return x_115; +} +else +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_131 = lean_ctor_get(x_115, 0); +x_132 = lean_ctor_get(x_115, 1); +lean_inc(x_132); +lean_inc(x_131); +lean_dec(x_115); +x_133 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_133, 0, x_131); +lean_ctor_set(x_133, 1, x_132); +return x_133; } } } default: { -lean_object* x_125; +lean_object* x_134; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_125 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_125, 0, x_1); -lean_ctor_set(x_125, 1, x_9); -return x_125; +x_134 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_134, 0, x_1); +lean_ctor_set(x_134, 1, x_9); +return x_134; } } } @@ -26579,7 +26688,7 @@ x_36 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term x_37 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_37, 0, x_35); lean_ctor_set(x_37, 1, x_36); -x_38 = lean_alloc_closure((void*)(l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1___boxed), 8, 1); +x_38 = lean_alloc_closure((void*)(l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___boxed), 8, 1); lean_closure_set(x_38, 0, x_37); lean_inc(x_17); lean_inc(x_16); @@ -33793,7 +33902,7 @@ else { lean_object* x_18; lean_object* x_19; uint8_t x_20; x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_14, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_14, x_18); x_20 = lean_nat_dec_lt(x_10, x_19); if (x_20 == 0) { @@ -33852,7 +33961,7 @@ else { lean_object* x_32; lean_object* x_33; uint8_t x_34; x_32 = lean_unsigned_to_nat(0u); -x_33 = l_Lean_Expr_getAppNumArgsAux(x_27, x_32); +x_33 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_27, x_32); x_34 = lean_nat_dec_lt(x_10, x_33); if (x_34 == 0) { @@ -38671,7 +38780,7 @@ lean_dec(x_2); return x_9; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -38681,7 +38790,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__2() { _start: { lean_object* x_1; @@ -38689,17 +38798,17 @@ x_1 = lean_mk_string_from_bytes("ignoreUnusedAlts", 16); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__1; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__2; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__4() { _start: { lean_object* x_1; @@ -38707,13 +38816,13 @@ x_1 = lean_mk_string_from_bytes("if true, do not generate error if an alternativ return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__5() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 0; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___closed__15; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__4; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__4; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -38722,12 +38831,12 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__3; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__5; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__3; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__5; x_4 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_1); return x_4; } @@ -40312,7 +40421,119 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; +x_9 = l_Lean_Expr_hasMVar(x_1); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_11 = lean_st_ref_get(x_7, x_8); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_st_ref_get(x_5, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_instantiateMVarsCore(x_16, x_1); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_st_ref_get(x_7, x_15); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_st_ref_take(x_5, x_21); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = !lean_is_exclusive(x_23); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = lean_ctor_get(x_23, 0); +lean_dec(x_26); +lean_ctor_set(x_23, 0, x_19); +x_27 = lean_st_ref_set(x_5, x_23, x_24); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +lean_object* x_29; +x_29 = lean_ctor_get(x_27, 0); +lean_dec(x_29); +lean_ctor_set(x_27, 0, x_18); +return x_27; +} +else +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_dec(x_27); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_18); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_32 = lean_ctor_get(x_23, 1); +x_33 = lean_ctor_get(x_23, 2); +x_34 = lean_ctor_get(x_23, 3); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_23); +x_35 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_35, 0, x_19); +lean_ctor_set(x_35, 1, x_32); +lean_ctor_set(x_35, 2, x_33); +lean_ctor_set(x_35, 3, x_34); +x_36 = lean_st_ref_set(x_5, x_35, x_24); +x_37 = lean_ctor_get(x_36, 1); +lean_inc(x_37); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + lean_ctor_release(x_36, 1); + x_38 = x_36; +} else { + lean_dec_ref(x_36); + x_38 = lean_box(0); +} +if (lean_is_scalar(x_38)) { + x_39 = lean_alloc_ctor(0, 2, 0); +} else { + x_39 = x_38; +} +lean_ctor_set(x_39, 0, x_18); +lean_ctor_set(x_39, 1, x_37); +return x_39; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; lean_object* x_11; @@ -40364,15 +40585,15 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7___rarg), 9, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___rarg), 9, 0); return x_2; } } -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__1() { +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -40380,16 +40601,16 @@ x_1 = lean_mk_string_from_bytes("invalid match-expression, type of pattern varia return x_1; } } -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__2() { +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__1; +x_1 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__3() { +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -40397,76 +40618,397 @@ x_1 = lean_mk_string_from_bytes("' contains metavariables", 24); return x_1; } } -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__4() { +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__3; +x_1 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_9; -lean_inc(x_2); -x_9 = l_Lean_Elab_Term_tryPostpone(x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) +lean_object* x_10; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +x_10 = l_Lean_Elab_Term_runPendingTacticsAt(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = l_Lean_LocalDecl_toExpr(x_1); -x_12 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_12, 0, x_11); -x_13 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__2; -x_14 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -x_15 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__4; -x_16 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -x_17 = l_Lean_LocalDecl_type(x_1); -x_18 = l_Lean_indentExpr(x_17); -x_19 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_19, 0, x_16); -lean_ctor_set(x_19, 1, x_18); -x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___closed__16; +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +lean_inc(x_1); +x_12 = l_Lean_instantiateMVars___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_11); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Expr_hasExprMVar(x_14); +lean_dec(x_14); +if (x_16 == 0) +{ +lean_object* x_17; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_17 = lean_box(0); +lean_ctor_set(x_12, 0, x_17); +return x_12; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; 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_free_object(x_12); +x_18 = l_Lean_LocalDecl_toExpr(x_2); +x_19 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_19, 0, x_18); +x_20 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__2; x_21 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -x_22 = l_Lean_Elab_Term_throwMVarError___rarg(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_10); -return x_22; +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +x_22 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__4; +x_23 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_24 = l_Lean_indentExpr(x_1); +x_25 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___closed__16; +x_27 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_Elab_Term_throwMVarError___rarg(x_27, x_3, x_4, x_5, x_6, x_7, x_8, x_15); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_28; +} } else { -uint8_t x_23; +lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_29 = lean_ctor_get(x_12, 0); +x_30 = lean_ctor_get(x_12, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_12); +x_31 = l_Lean_Expr_hasExprMVar(x_29); +lean_dec(x_29); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_32 = lean_box(0); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_30); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_34 = l_Lean_LocalDecl_toExpr(x_2); +x_35 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_35, 0, x_34); +x_36 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__2; +x_37 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +x_38 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__4; +x_39 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +x_40 = l_Lean_indentExpr(x_1); +x_41 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___closed__16; +x_43 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = l_Lean_Elab_Term_throwMVarError___rarg(x_43, x_3, x_4, x_5, x_6, x_7, x_8, x_30); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_44; +} +} +} +else +{ +uint8_t x_45; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_45 = !lean_is_exclusive(x_10); +if (x_45 == 0) +{ +return x_10; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_10, 0); +x_47 = lean_ctor_get(x_10, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_10); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; +} +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_11; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_3); +lean_ctor_set(x_11, 1, x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; +lean_dec(x_3); +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_2, 1); +lean_inc(x_13); lean_dec(x_2); -x_23 = !lean_is_exclusive(x_9); -if (x_23 == 0) +x_14 = l_Lean_LocalDecl_hasExprMVar(x_12); +if (x_14 == 0) { -return x_9; +lean_object* x_15; +lean_dec(x_12); +x_15 = lean_box(0); +x_2 = x_13; +x_3 = x_15; +goto _start; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_9, 0); -x_25 = lean_ctor_get(x_9, 1); -lean_inc(x_25); -lean_inc(x_24); +lean_object* x_17; +lean_inc(x_4); +x_17 = l_Lean_Elab_Term_tryPostpone(x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = l_Lean_LocalDecl_type(x_12); +x_20 = lean_alloc_closure((void*)(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___boxed), 9, 2); +lean_closure_set(x_20, 0, x_19); +lean_closure_set(x_20, 1, x_12); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_21 = l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___rarg(x_1, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_23 = lean_box(0); +x_2 = x_13; +x_3 = x_23; +x_10 = x_22; +goto _start; +} +else +{ +uint8_t x_25; +lean_dec(x_13); lean_dec(x_9); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_25 = !lean_is_exclusive(x_21); +if (x_25 == 0) +{ +return x_21; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_21, 0); +x_27 = lean_ctor_get(x_21, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_21); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} +} +} +else +{ +uint8_t x_29; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_17); +if (x_29 == 0) +{ +return x_17; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_17, 0); +x_31 = lean_ctor_get(x_17, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_17); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} +} +} +} +} +} +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("invalid match-expression, pattern contains metavariables", 56); +return x_1; +} +} +static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___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) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = 0; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_10 = l_Lean_Meta_Match_Pattern_toExpr_visit(x_9, x_1, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = l_Lean_indentExpr(x_11); +x_14 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__2; +x_15 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___closed__16; +x_17 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_Elab_Term_throwMVarError___rarg(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_12); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_18; +} +else +{ +uint8_t x_19; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_10); +if (x_19 == 0) +{ +return x_10; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = 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_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { if (lean_obj_tag(x_2) == 0) @@ -40486,28 +41028,44 @@ return x_11; } else { -lean_object* x_12; lean_object* x_13; uint8_t x_14; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_dec(x_3); x_12 = lean_ctor_get(x_2, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_2, 1); lean_inc(x_13); lean_dec(x_2); -x_14 = l_Lean_LocalDecl_hasExprMVar(x_12); -if (x_14 == 0) +lean_inc(x_12); +x_14 = l_Lean_Meta_Match_instantiatePatternMVars(x_12, x_6, x_7, x_8, x_9, x_10); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_Meta_Match_Pattern_hasExprMVar(x_15); +if (x_17 == 0) { -lean_object* x_15; +lean_object* x_18; lean_dec(x_12); -x_15 = lean_box(0); +x_18 = lean_box(0); x_2 = x_13; -x_3 = x_15; +x_3 = x_18; +x_10 = x_16; goto _start; } else { -lean_object* x_17; lean_object* x_18; -x_17 = lean_alloc_closure((void*)(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___boxed), 8, 1); -lean_closure_set(x_17, 0, x_12); +lean_object* x_20; +lean_inc(x_4); +x_20 = l_Lean_Elab_Term_tryPostpone(x_4, x_5, x_6, x_7, x_8, x_9, x_16); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_alloc_closure((void*)(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___boxed), 8, 1); +lean_closure_set(x_22, 0, x_12); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); @@ -40515,22 +41073,22 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_1); -x_18 = l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7___rarg(x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_18) == 0) +x_23 = l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___rarg(x_1, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_box(0); +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +x_25 = lean_box(0); x_2 = x_13; -x_3 = x_20; -x_10 = x_19; +x_3 = x_25; +x_10 = x_24; goto _start; } else { -uint8_t x_22; +uint8_t x_27; lean_dec(x_13); lean_dec(x_9); lean_dec(x_8); @@ -40539,213 +41097,31 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) -{ -return x_18; -} -else -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_18, 0); -x_24 = lean_ctor_get(x_18, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_18); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; -} -} -} -} -} -} -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("invalid match-expression, pattern contains metavariables", 56); -return x_1; -} -} -static lean_object* _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -lean_inc(x_2); -x_9 = l_Lean_Elab_Term_tryPostpone(x_2, x_3, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_10; uint8_t x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = 0; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_12 = l_Lean_Meta_Match_Pattern_toExpr_visit(x_11, x_1, x_4, x_5, x_6, x_7, x_10); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l_Lean_indentExpr(x_13); -x_16 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__2; -x_17 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchTypeAndDiscrs_elabDiscrsWitMatchType___spec__1___closed__16; -x_19 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -x_20 = l_Lean_Elab_Term_throwMVarError___rarg(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_14); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_20; -} -else -{ -uint8_t x_21; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_21 = !lean_is_exclusive(x_12); -if (x_21 == 0) -{ -return x_12; -} -else -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_12, 0); -x_23 = lean_ctor_get(x_12, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_12); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; -} -} -} -else -{ -uint8_t x_25; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_25 = !lean_is_exclusive(x_9); -if (x_25 == 0) +x_27 = !lean_is_exclusive(x_23); +if (x_27 == 0) { -return x_9; +return x_23; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_9, 0); -x_27 = lean_ctor_get(x_9, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_9); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_23, 0); +x_29 = lean_ctor_get(x_23, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_23); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_11; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_3); -lean_ctor_set(x_11, 1, x_10); -return x_11; } else { -lean_object* x_12; lean_object* x_13; uint8_t x_14; -lean_dec(x_3); -x_12 = lean_ctor_get(x_2, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_2, 1); -lean_inc(x_13); -lean_dec(x_2); -lean_inc(x_12); -x_14 = l_Lean_Meta_Match_Pattern_hasExprMVar(x_12); -if (x_14 == 0) -{ -lean_object* x_15; -lean_dec(x_12); -x_15 = lean_box(0); -x_2 = x_13; -x_3 = x_15; -goto _start; -} -else -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_alloc_closure((void*)(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___boxed), 8, 1); -lean_closure_set(x_17, 0, x_12); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_1); -x_18 = l_Lean_Meta_withExistingLocalDecls___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7___rarg(x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_box(0); -x_2 = x_13; -x_3 = x_20; -x_10 = x_19; -goto _start; -} -else -{ -uint8_t x_22; +uint8_t x_31; lean_dec(x_13); +lean_dec(x_12); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -40753,30 +41129,30 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) +x_31 = !lean_is_exclusive(x_20); +if (x_31 == 0) { -return x_18; +return x_20; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_18, 0); -x_24 = lean_ctor_get(x_18, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_18); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_20, 0); +x_33 = lean_ctor_get(x_20, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_20); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } } } } } } -LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { if (lean_obj_tag(x_1) == 0) @@ -40858,7 +41234,7 @@ lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc_n(x_19, 2); -x_34 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8(x_19, x_19, x_33, x_2, x_3, x_4, x_5, x_32, x_7, x_17); +x_34 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9(x_19, x_19, x_33, x_2, x_3, x_4, x_5, x_32, x_7, x_17); if (lean_obj_tag(x_34) == 0) { lean_object* x_35; lean_object* x_36; lean_object* x_37; @@ -40872,14 +41248,14 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_37 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9(x_19, x_36, x_33, x_2, x_3, x_4, x_5, x_32, x_7, x_35); +x_37 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(x_19, x_36, x_33, x_2, x_3, x_4, x_5, x_32, x_7, x_35); if (lean_obj_tag(x_37) == 0) { lean_object* x_38; lean_object* x_39; x_38 = lean_ctor_get(x_37, 1); lean_inc(x_38); lean_dec(x_37); -x_39 = l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_38); +x_39 = l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_38); if (lean_obj_tag(x_39) == 0) { uint8_t x_40; @@ -41062,7 +41438,7 @@ lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc_n(x_64, 2); -x_79 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8(x_64, x_64, x_78, x_2, x_3, x_4, x_5, x_77, x_7, x_62); +x_79 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9(x_64, x_64, x_78, x_2, x_3, x_4, x_5, x_77, x_7, x_62); if (lean_obj_tag(x_79) == 0) { lean_object* x_80; lean_object* x_81; lean_object* x_82; @@ -41076,14 +41452,14 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_82 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9(x_64, x_81, x_78, x_2, x_3, x_4, x_5, x_77, x_7, x_80); +x_82 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(x_64, x_81, x_78, x_2, x_3, x_4, x_5, x_77, x_7, x_80); if (lean_obj_tag(x_82) == 0) { lean_object* x_83; lean_object* x_84; x_83 = lean_ctor_get(x_82, 1); lean_inc(x_83); lean_dec(x_82); -x_84 = l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_83); +x_84 = l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_83); if (lean_obj_tag(x_84) == 0) { lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; @@ -41206,7 +41582,7 @@ return x_101; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -41270,7 +41646,7 @@ goto _start; } } } -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12(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_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__13(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -41430,7 +41806,7 @@ x_35 = lean_ctor_get(x_33, 1); lean_inc(x_35); lean_dec(x_33); x_36 = lean_array_to_list(lean_box(0), x_23); -x_37 = l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(x_36, x_7, x_8, x_9, x_10, x_11, x_12, x_35); +x_37 = l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(x_36, x_7, x_8, x_9, x_10, x_11, x_12, x_35); lean_dec(x_11); if (lean_obj_tag(x_37) == 0) { @@ -41976,7 +42352,7 @@ if (lean_obj_tag(x_28) == 0) lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_dec(x_21); x_30 = lean_array_get_size(x_22); -x_31 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__1; +x_31 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__1; lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -41995,7 +42371,7 @@ lean_dec(x_32); x_35 = lean_usize_of_nat(x_30); x_36 = 0; lean_inc(x_22); -x_37 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(x_35, x_36, x_22); +x_37 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12(x_35, x_36, x_22); lean_inc(x_24); lean_inc(x_23); x_38 = lean_alloc_ctor(0, 4, 0); @@ -42453,7 +42829,7 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); x_15 = l___private_Lean_Elab_Match_0__Lean_Elab_Term_getMatchGeneralizing_x3f___closed__11; -x_16 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12(x_1, x_15); +x_16 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__13(x_1, x_15); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; @@ -42594,39 +42970,48 @@ x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_el return x_6; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_instantiateMVars___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_1); +lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___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) { _start: { lean_object* x_9; -x_9 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_List_mapM___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_6); return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -42634,15 +43019,15 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__11(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12___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_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__13___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_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__12(x_1, x_2); +x_3 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__13(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -45952,7 +46337,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_elabMatch_declRange___cl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1251u); +x_1 = lean_unsigned_to_nat(1253u); x_2 = lean_unsigned_to_nat(27u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -45964,7 +46349,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_elabMatch_declRange___cl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1268u); +x_1 = lean_unsigned_to_nat(1270u); x_2 = lean_unsigned_to_nat(37u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -45992,7 +46377,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_elabMatch_declRange___cl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1251u); +x_1 = lean_unsigned_to_nat(1253u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -46004,7 +46389,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_elabMatch_declRange___cl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1251u); +x_1 = lean_unsigned_to_nat(1253u); x_2 = lean_unsigned_to_nat(40u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -46050,7 +46435,7 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_17065_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_17123_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -46358,7 +46743,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_elabNoMatch_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1277u); +x_1 = lean_unsigned_to_nat(1279u); x_2 = lean_unsigned_to_nat(29u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -46370,7 +46755,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_elabNoMatch_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1289u); +x_1 = lean_unsigned_to_nat(1291u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -46398,7 +46783,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_elabNoMatch_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1277u); +x_1 = lean_unsigned_to_nat(1279u); x_2 = lean_unsigned_to_nat(33u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -46410,7 +46795,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Term_elabNoMatch_declRange___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1277u); +x_1 = lean_unsigned_to_nat(1279u); x_2 = lean_unsigned_to_nat(44u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -46865,17 +47250,17 @@ l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___closed__1 lean_mark_persistent(l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___closed__1); l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___closed__2 = _init_l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___closed__2(); lean_mark_persistent(l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAltViews_loop___closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__4); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559____closed__5); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13559_(lean_io_mk_world()); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__4); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555____closed__5); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_13555_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Term_match_ignoreUnusedAlts = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Term_match_ignoreUnusedAlts); @@ -46912,18 +47297,18 @@ l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Match_0__Lean_Elab_T lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__5___rarg___closed__1); l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__5___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__5___rarg___closed__2(); lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__5___rarg___closed__2); -l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__1 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__1(); -lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__1); -l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__2 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__2(); -lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__2); -l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__3 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__3(); -lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__3); -l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__4 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__4(); -lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__8___lambda__1___closed__4); l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__1 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__1(); lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__1); l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__2 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__2(); lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__2); +l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__3 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__3(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__3); +l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__4 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__4(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__9___lambda__1___closed__4); +l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__1 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__1(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__1); +l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__2 = _init_l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__2(); +lean_mark_persistent(l_List_forIn_loop___at___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___spec__10___lambda__1___closed__2); l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__2___closed__1 = _init_l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__2___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__2___closed__1); l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__2___closed__2 = _init_l___private_Lean_Elab_Match_0__Lean_Elab_Term_elabMatchAux___lambda__2___closed__2(); @@ -46997,7 +47382,7 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_elabMatch_declRange___closed_ res = l___regBuiltin_Lean_Elab_Term_elabMatch_declRange(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_17065_(lean_io_mk_world()); +res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Match___hyg_17123_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Elab_Term_elabNoMatch___closed__1 = _init_l_Lean_Elab_Term_elabNoMatch___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/MutualDef.c b/stage0/stdlib/Lean/Elab/MutualDef.c index a4a6bd8eab72..1f5837222ad7 100644 --- a/stage0/stdlib/Lean/Elab/MutualDef.c +++ b/stage0/stdlib/Lean/Elab/MutualDef.c @@ -13,7 +13,6 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed__const__1; lean_object* l_List_reverse___rarg(lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -21,6 +20,7 @@ extern lean_object* l_Lean_pp_letVarTypes; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_checkForHiddenUnivLevels_visit___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addTrace___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__4___closed__2; LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Term_processDefDeriving___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldAux___at_Lean_Elab_Term_MutualClosure_insertReplacementForMainFns___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -247,6 +247,7 @@ lean_object* l_Lean_Elab_Term_withLevelNames___rarg(lean_object*, lean_object*, LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_collectUsed___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__6___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_LocalContext_contains(lean_object*, lean_object*); uint8_t l_Lean_Elab_DefKind_isExample(uint8_t); LEAN_EXPORT lean_object* l_Std_RBNode_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); @@ -256,7 +257,7 @@ lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean static lean_object* l_Lean_Elab_elabModifiers___at_Lean_Elab_Command_elabMutualDef___spec__1___lambda__3___closed__2; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_processDefDeriving___spec__3___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkLetRecsToLiftTypes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__5___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__10___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__11___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -307,8 +308,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expan static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_Replacement_apply___lambda__1(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__3___closed__5; -lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getFunName___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withFunLocalDecls_loop(lean_object*); @@ -344,6 +343,7 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualD static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___spec__10___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkClosureForAux___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_MutualClosure_getModifiersForLetRecs___spec__3(lean_object*, size_t, size_t); +lean_object* l_Lean_Meta_mkSorry(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_levelMVarToParamPreDecls(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Closure_mkLambda(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_isModified(lean_object*); @@ -449,6 +449,7 @@ uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_FixPoint_merge___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_MutualClosure_insertReplacementForLetRecs(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__7(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabMutualDef___boxed__const__1; lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -470,7 +471,7 @@ uint8_t l_Std_HashSetImp_contains___at_Lean_CollectLevelParams_visitLevel___spec LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___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_getMax_x3f___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_pickMaxFVar_x3f___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__18(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Expr_instHashableExpr; @@ -543,6 +544,7 @@ lean_object* l_Lean_throwError___at_Lean_Elab_Term_expandDeclId___spec__12(lean_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Command_elabMutualDef___spec__11___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_mkDefViewOfInstance___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_reverse___rarg(lean_object*); static lean_object* l_Lean_Elab_addDeclarationRanges___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__3___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -653,7 +655,6 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_removeUnusedVars(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_isAttribute(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_collectUsed___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___spec__5___closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_checkForHiddenUnivLevels___spec__2___closed__5; @@ -760,6 +761,7 @@ uint8_t l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec_ lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_typeHasRecFun___spec__1___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_HashMap_insert___at___private_Lean_Meta_Check_0__Lean_Meta_checkAux_check___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Term_processDefDeriving___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_registerFailedToInferDefTypeInfo___closed__1; @@ -861,6 +863,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_Mutua static lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Term_elabMutualDef_processDeriving___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Term_processDefDeriving___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_RBNode_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkFreeVarMap___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualDef___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_addAutoBoundImplicits(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -877,6 +880,7 @@ static lean_object* l_Lean_Elab_addDeclarationRanges___at___private_Lean_Elab_Mu LEAN_EXPORT lean_object* l_Std_RBNode_fold___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_List_foldr___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_typeHasRecFun___spec__1(lean_object*, uint8_t, lean_object*); static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkInitialUsedFVarsMap___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__14___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_MutualClosure_mkLetRecClosures___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabHeaders___spec__6___lambda__1___boxed(lean_object**); @@ -929,6 +933,7 @@ LEAN_EXPORT lean_object* l_Std_RBNode_fold___at___private_Lean_Elab_MutualDef_0_ LEAN_EXPORT lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_check___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_checkForHiddenUnivLevels___spec__2___closed__2; static lean_object* l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_expandWhereStructInst___closed__1; +lean_object* l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Command_elabMutualDef___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getDeclarationSelectionRef(lean_object*); @@ -2631,7 +2636,7 @@ static lean_object* _init_l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isMu 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_MutualDef_0__Lean_Elab_Term_isMultiConstant_x3f___closed__1; x_2 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isMultiConstant_x3f___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_isMultiConstant_x3f___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4793,7 +4798,9 @@ x_51 = lean_ctor_get(x_50, 1); lean_inc(x_51); x_52 = 2; lean_inc(x_11); -lean_inc(x_47); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); lean_inc(x_6); lean_inc(x_32); x_53 = l_Lean_Elab_Term_applyAttributesAt(x_32, x_51, x_52, x_6, x_7, x_8, x_9, x_47, x_11, x_49); @@ -4987,7 +4994,9 @@ x_100 = lean_ctor_get(x_99, 1); lean_inc(x_100); x_101 = 2; lean_inc(x_11); -lean_inc(x_96); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); lean_inc(x_6); lean_inc(x_81); x_102 = l_Lean_Elab_Term_applyAttributesAt(x_81, x_100, x_101, x_6, x_7, x_8, x_9, x_96, x_11, x_98); @@ -5236,7 +5245,9 @@ x_158 = lean_ctor_get(x_157, 1); lean_inc(x_158); x_159 = 2; lean_inc(x_11); -lean_inc(x_154); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); lean_inc(x_6); lean_inc(x_139); x_160 = l_Lean_Elab_Term_applyAttributesAt(x_139, x_158, x_159, x_6, x_7, x_8, x_9, x_154, x_11, x_156); @@ -31879,7 +31890,7 @@ case 5: { lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; x_59 = lean_unsigned_to_nat(0u); -x_60 = l_Lean_Expr_getAppNumArgsAux(x_4, x_59); +x_60 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_59); x_61 = l_Lean_Elab_Term_checkForHiddenUnivLevels_visit___closed__1; lean_inc(x_60); x_62 = lean_mk_array(x_60, x_61); @@ -32866,7 +32877,7 @@ case 5: { lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; x_266 = lean_unsigned_to_nat(0u); -x_267 = l_Lean_Expr_getAppNumArgsAux(x_4, x_266); +x_267 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_266); x_268 = l_Lean_Elab_Term_checkForHiddenUnivLevels_visit___closed__1; lean_inc(x_267); x_269 = lean_mk_array(x_267, x_268); @@ -35204,7 +35215,7 @@ x_44 = l_Lean_throwUnknownConstant___at_Lean_Elab_Term_elabMutualDef_processDeri x_45 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_45, 0, x_43); lean_ctor_set(x_45, 1, x_44); -x_46 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_45, x_6, x_7, x_8, x_9, x_32, x_11, x_36); +x_46 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_45, x_6, x_7, x_8, x_9, x_32, x_11, x_36); lean_dec(x_11); lean_dec(x_32); lean_dec(x_9); @@ -36450,6 +36461,84 @@ goto _start; } } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; +x_11 = lean_usize_dec_lt(x_2, x_1); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_3); +lean_ctor_set(x_12, 1, x_10); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_13 = lean_array_uget(x_3, x_2); +x_14 = lean_unsigned_to_nat(0u); +x_15 = lean_array_uset(x_3, x_2, x_14); +x_16 = lean_ctor_get(x_13, 7); +lean_inc(x_16); +lean_dec(x_13); +x_17 = 1; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_18 = l_Lean_Meta_mkSorry(x_16, x_17, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = 1; +x_22 = lean_usize_add(x_2, x_21); +x_23 = lean_array_uset(x_15, x_2, x_19); +x_2 = x_22; +x_3 = x_23; +x_10 = x_20; +goto _start; +} +else +{ +uint8_t x_25; +lean_dec(x_15); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_25 = !lean_is_exclusive(x_18); +if (x_25 == 0) +{ +return x_18; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_18, 0); +x_27 = lean_ctor_get(x_18, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_18); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} +} +} +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { @@ -36730,16 +36819,100 @@ return x_68; } } } -static lean_object* _init_l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed__const__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -size_t x_1; lean_object* x_2; -x_1 = 0; -x_2 = lean_box_usize(x_1); -return x_2; +lean_object* x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_17 = lean_array_get_size(x_1); +x_18 = lean_usize_of_nat(x_17); +lean_dec(x_17); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__3(x_18, x_2, x_1, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l_Lean_Elab_Term_getLetRecsToLift___rarg(x_11, x_12, x_13, x_14, x_15, x_21); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = l_List_mapM___at_Lean_Elab_Term_elabMutualDef_go___spec__2(x_23, x_10, x_11, x_12, x_13, x_14, x_15, x_24); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +lean_inc(x_14); +lean_inc(x_12); +lean_inc(x_10); +lean_inc_n(x_26, 2); +lean_inc(x_3); +x_28 = l_List_forM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkLetRecsToLiftTypes___spec__1(x_3, x_26, x_26, x_10, x_11, x_12, x_13, x_14, x_15, x_27); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_28, 1); +lean_inc(x_29); +lean_dec(x_28); +x_30 = lean_box_usize(x_2); +lean_inc(x_26); +lean_inc(x_9); +lean_inc(x_20); +x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabMutualDef_go___lambda__1___boxed), 17, 9); +lean_closure_set(x_31, 0, x_20); +lean_closure_set(x_31, 1, x_3); +lean_closure_set(x_31, 2, x_9); +lean_closure_set(x_31, 3, x_26); +lean_closure_set(x_31, 4, x_30); +lean_closure_set(x_31, 5, x_4); +lean_closure_set(x_31, 6, x_5); +lean_closure_set(x_31, 7, x_6); +lean_closure_set(x_31, 8, x_7); +x_32 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withUsed___rarg(x_8, x_20, x_9, x_26, x_31, x_10, x_11, x_12, x_13, x_14, x_15, x_29); +lean_dec(x_9); +return x_32; +} +else +{ +uint8_t x_33; +lean_dec(x_26); +lean_dec(x_20); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_33 = !lean_is_exclusive(x_28); +if (x_33 == 0) +{ +return x_28; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_28, 0); +x_35 = lean_ctor_get(x_28, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_28); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; @@ -36760,7 +36933,7 @@ lean_inc(x_8); x_21 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__1(x_1, x_19, x_20, x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14); if (lean_obj_tag(x_21) == 0) { -lean_object* x_22; lean_object* x_23; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_42; x_22 = lean_ctor_get(x_21, 1); lean_inc(x_22); lean_dec(x_21); @@ -36771,95 +36944,108 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_2); -x_23 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues(x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_22); -if (lean_obj_tag(x_23) == 0) +x_42 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_elabFunValues(x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = 0; +lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = 0; lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_27 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_26, x_26, x_8, x_9, x_10, x_11, x_12, x_13, x_25); -if (lean_obj_tag(x_27) == 0) +x_46 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_45, x_45, x_8, x_9, x_10, x_11, x_12, x_13, x_44); +if (lean_obj_tag(x_46) == 0) { -lean_object* x_28; lean_object* x_29; size_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; size_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_28 = lean_ctor_get(x_27, 1); -lean_inc(x_28); -lean_dec(x_27); -x_29 = lean_array_get_size(x_24); -x_30 = lean_usize_of_nat(x_29); -lean_dec(x_29); -x_31 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__2(x_30, x_20, x_24, x_8, x_9, x_10, x_11, x_12, x_13, x_28); -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -x_34 = lean_array_get_size(x_2); -x_35 = lean_usize_of_nat(x_34); -lean_dec(x_34); -x_36 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__3(x_35, x_20, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_33); -x_37 = lean_ctor_get(x_36, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_36, 1); -lean_inc(x_38); -lean_dec(x_36); -x_39 = l_Lean_Elab_Term_getLetRecsToLift___rarg(x_9, x_10, x_11, x_12, x_13, x_38); -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); -lean_inc(x_41); -lean_dec(x_39); -x_42 = l_List_mapM___at_Lean_Elab_Term_elabMutualDef_go___spec__2(x_40, x_8, x_9, x_10, x_11, x_12, x_13, x_41); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); +lean_object* x_47; lean_object* x_48; size_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +x_48 = lean_array_get_size(x_43); +x_49 = lean_usize_of_nat(x_48); +lean_dec(x_48); +x_50 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_MutualClosure_main___spec__2(x_49, x_20, x_43, x_8, x_9, x_10, x_11, x_12, x_13, x_47); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_53 = l_Lean_Elab_Term_elabMutualDef_go___lambda__2(x_2, x_20, x_7, x_3, x_4, x_5, x_1, x_6, x_51, x_8, x_9, x_10, x_11, x_12, x_13, x_52); +lean_dec(x_6); +return x_53; +} +else +{ +lean_object* x_54; lean_object* x_55; +lean_dec(x_43); +x_54 = lean_ctor_get(x_46, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_46, 1); +lean_inc(x_55); +lean_dec(x_46); +x_23 = x_54; +x_24 = x_55; +goto block_41; +} +} +else +{ +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_42, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_42, 1); +lean_inc(x_57); lean_dec(x_42); +x_23 = x_56; +x_24 = x_57; +goto block_41; +} +block_41: +{ +lean_object* x_25; +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_n(x_43, 2); -lean_inc(x_7); -x_45 = l_List_forM___at___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_checkLetRecsToLiftTypes___spec__1(x_7, x_43, x_43, x_8, x_9, x_10, x_11, x_12, x_13, x_44); -if (lean_obj_tag(x_45) == 0) +x_25 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_23, x_8, x_9, x_10, x_11, x_12, x_13, x_24); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_46 = lean_ctor_get(x_45, 1); -lean_inc(x_46); -lean_dec(x_45); -x_47 = l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed__const__1; -lean_inc(x_43); -lean_inc(x_32); -lean_inc(x_37); -x_48 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabMutualDef_go___lambda__1___boxed), 17, 9); -lean_closure_set(x_48, 0, x_37); -lean_closure_set(x_48, 1, x_7); -lean_closure_set(x_48, 2, x_32); -lean_closure_set(x_48, 3, x_43); -lean_closure_set(x_48, 4, x_47); -lean_closure_set(x_48, 5, x_3); -lean_closure_set(x_48, 6, x_4); -lean_closure_set(x_48, 7, x_5); -lean_closure_set(x_48, 8, x_1); -x_49 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_withUsed___rarg(x_6, x_37, x_32, x_43, x_48, x_8, x_9, x_10, x_11, x_12, x_13, x_46); -lean_dec(x_32); -return x_49; +lean_object* x_26; lean_object* x_27; size_t x_28; lean_object* x_29; +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = lean_array_get_size(x_2); +x_28 = lean_usize_of_nat(x_27); +lean_dec(x_27); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_2); +x_29 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6(x_28, x_20, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_26); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = l_Lean_Elab_Term_elabMutualDef_go___lambda__2(x_2, x_20, x_7, x_3, x_4, x_5, x_1, x_6, x_30, x_8, x_9, x_10, x_11, x_12, x_13, x_31); +lean_dec(x_6); +return x_32; } else { -uint8_t x_50; -lean_dec(x_43); -lean_dec(x_37); -lean_dec(x_32); +uint8_t x_33; lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -36867,34 +37053,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_50 = !lean_is_exclusive(x_45); -if (x_50 == 0) +x_33 = !lean_is_exclusive(x_29); +if (x_33 == 0) { -return x_45; +return x_29; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_45, 0); -x_52 = lean_ctor_get(x_45, 1); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_45); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_51); -lean_ctor_set(x_53, 1, x_52); -return x_53; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_29, 0); +x_35 = lean_ctor_get(x_29, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_29); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } } else { -uint8_t x_54; -lean_dec(x_24); +uint8_t x_37; lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -36902,28 +37089,30 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_54 = !lean_is_exclusive(x_27); -if (x_54 == 0) +x_37 = !lean_is_exclusive(x_25); +if (x_37 == 0) { -return x_27; +return x_25; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_27, 0); -x_56 = lean_ctor_get(x_27, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_27); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -return x_57; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_25, 0); +x_39 = lean_ctor_get(x_25, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_25); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} } } } @@ -36937,24 +37126,25 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_58 = !lean_is_exclusive(x_23); +x_58 = !lean_is_exclusive(x_21); if (x_58 == 0) { -return x_23; +return x_21; } else { lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_23, 0); -x_60 = lean_ctor_get(x_23, 1); +x_59 = lean_ctor_get(x_21, 0); +x_60 = lean_ctor_get(x_21, 1); lean_inc(x_60); lean_inc(x_59); -lean_dec(x_23); +lean_dec(x_21); x_61 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_61, 0, x_59); lean_ctor_set(x_61, 1, x_60); @@ -36962,41 +37152,6 @@ return x_61; } } } -else -{ -uint8_t x_62; -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); -lean_dec(x_1); -x_62 = !lean_is_exclusive(x_21); -if (x_62 == 0) -{ -return x_21; -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_21, 0); -x_64 = lean_ctor_get(x_21, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_21); -x_65 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -return x_65; -} -} -} } LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: @@ -37039,7 +37194,7 @@ lean_inc(x_19); lean_dec(x_17); x_20 = l___private_Lean_Elab_MutualDef_0__Lean_Elab_Term_getAllUserLevelNames(x_18); lean_inc(x_18); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed), 14, 6); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabMutualDef_go___lambda__3), 14, 6); lean_closure_set(x_21, 0, x_2); lean_closure_set(x_21, 1, x_18); lean_closure_set(x_21, 2, x_12); @@ -37164,6 +37319,20 @@ lean_dec(x_1); return x_14; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = l_Array_mapMUnsafe_map___at_Lean_Elab_Term_elabMutualDef_go___spec__6(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +return x_13; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__1___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; @@ -37191,13 +37360,15 @@ x_19 = l_Lean_Elab_Term_elabMutualDef_go___lambda__1(x_1, x_2, x_3, x_4, x_18, x return x_19; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_15; -x_15 = l_Lean_Elab_Term_elabMutualDef_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_6); -return x_15; +size_t x_17; lean_object* x_18; +x_17 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_18 = l_Lean_Elab_Term_elabMutualDef_go___lambda__2(x_1, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_8); +return x_18; } } LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabMutualDef(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -37543,7 +37714,7 @@ lean_closure_set(x_14, 0, x_12); lean_closure_set(x_14, 1, x_13); lean_inc(x_3); lean_inc(x_2); -x_15 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__10(x_14, x_2, x_3, x_10); +x_15 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabCommand___spec__14(x_14, x_2, x_3, x_10); if (lean_obj_tag(x_15) == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; @@ -37682,50 +37853,104 @@ return x_9; } else { -lean_object* x_10; lean_object* x_11; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_10 = lean_array_uget(x_1, x_3); -lean_inc(x_6); -lean_inc(x_5); -x_11 = l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4(x_10, x_5, x_6, x_7); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; +x_11 = l_Lean_Elab_Command_getRef(x_5, x_6, x_7); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = lean_array_push(x_4, x_12); -x_15 = 1; -x_16 = lean_usize_add(x_3, x_15); -x_3 = x_16; -x_4 = x_14; -x_7 = x_13; +x_14 = l_Lean_replaceRef(x_10, x_12); +lean_dec(x_12); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_5, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_5, 2); +lean_inc(x_17); +x_18 = lean_ctor_get(x_5, 3); +lean_inc(x_18); +x_19 = lean_ctor_get(x_5, 4); +lean_inc(x_19); +x_20 = lean_ctor_get(x_5, 5); +lean_inc(x_20); +x_21 = lean_ctor_get(x_5, 7); +lean_inc(x_21); +x_22 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_22, 0, x_15); +lean_ctor_set(x_22, 1, x_16); +lean_ctor_set(x_22, 2, x_17); +lean_ctor_set(x_22, 3, x_18); +lean_ctor_set(x_22, 4, x_19); +lean_ctor_set(x_22, 5, x_20); +lean_ctor_set(x_22, 6, x_14); +lean_ctor_set(x_22, 7, x_21); +lean_inc(x_6); +x_23 = l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4(x_10, x_22, x_6, x_13); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; size_t x_27; size_t x_28; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_array_push(x_4, x_24); +x_27 = 1; +x_28 = lean_usize_add(x_3, x_27); +x_3 = x_28; +x_4 = x_26; +x_7 = x_25; goto _start; } else { -uint8_t x_18; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_23, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_23, 1); +lean_inc(x_31); +lean_dec(x_23); +lean_inc(x_6); +lean_inc(x_5); +x_32 = l_Lean_Elab_logException___at_Lean_Elab_Command_elabCommand___spec__3(x_30, x_5, x_6, x_31); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; size_t x_34; size_t x_35; +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = 1; +x_35 = lean_usize_add(x_3, x_34); +x_3 = x_35; +x_7 = x_33; +goto _start; +} +else +{ +uint8_t x_37; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_18 = !lean_is_exclusive(x_11); -if (x_18 == 0) +x_37 = !lean_is_exclusive(x_32); +if (x_37 == 0) { -return x_11; +return x_32; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_11, 0); -x_20 = lean_ctor_get(x_11, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_11); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_32, 0); +x_39 = lean_ctor_get(x_32, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_32); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} } } } @@ -39682,8 +39907,6 @@ l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__5___closed lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__5___closed__1); l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__5___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__5___closed__2(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_elabMutualDef_go___spec__5___closed__2); -l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed__const__1 = _init_l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed__const__1(); -lean_mark_persistent(l_Lean_Elab_Term_elabMutualDef_go___lambda__2___boxed__const__1); l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__1___closed__1 = _init_l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__1___closed__1); l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__1___closed__2 = _init_l_Lean_Elab_elabAttr___at_Lean_Elab_Command_elabMutualDef___spec__4___lambda__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Notation.c b/stage0/stdlib/Lean/Elab/Notation.c index 1e116665bc36..dccf28828a0d 100644 --- a/stage0/stdlib/Lean/Elab/Notation.c +++ b/stage0/stdlib/Lean/Elab/Notation.c @@ -38,6 +38,7 @@ static lean_object* l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNo static lean_object* l_Lean_Elab_Command_mkSimpleDelab___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__36; static lean_object* l_Lean_Elab_Command_mkSimpleDelab___lambda__1___closed__53; static lean_object* l_Lean_Elab_Command_mkSimpleDelab___lambda__1___closed__42; LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandNotation___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1944,7 +1945,7 @@ static lean_object* _init_l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_El lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_Elab_Command_hasDuplicateAntiquot___spec__1___closed__4; x_2 = l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_Elab_Command_hasDuplicateAntiquot___spec__1___closed__5; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_Elab_Command_hasDuplicateAntiquot___spec__1___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -5901,7 +5902,7 @@ static lean_object* _init_l___private_Lean_Elab_Notation_0__Lean_Elab_Command_ex _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(9u); +x_1 = lean_unsigned_to_nat(10u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } @@ -5916,6 +5917,16 @@ x_3 = lean_array_push(x_1, x_2); return x_3; } } +static lean_object* _init_l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__36() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__35; +x_2 = l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__3; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, 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: { @@ -6069,7 +6080,7 @@ x_170 = l_Lean_Elab_Command_expandNotationItemIntoSyntaxItem___lambda__1___close x_171 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_171, 0, x_127); lean_ctor_set(x_171, 1, x_170); -x_172 = l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__35; +x_172 = l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__36; lean_inc(x_7); x_173 = lean_array_push(x_172, x_7); x_174 = lean_array_push(x_173, x_130); @@ -7496,6 +7507,8 @@ l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__ lean_mark_persistent(l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__34); l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__35 = _init_l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__35(); lean_mark_persistent(l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__35); +l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__36 = _init_l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__36(); +lean_mark_persistent(l___private_Lean_Elab_Notation_0__Lean_Elab_Command_expandNotationAux___lambda__2___closed__36); l_Lean_Elab_Command_expandNotation___closed__1 = _init_l_Lean_Elab_Command_expandNotation___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_expandNotation___closed__1); l_Lean_Elab_Command_expandNotation___closed__2 = _init_l_Lean_Elab_Command_expandNotation___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Open.c b/stage0/stdlib/Lean/Elab/Open.c index 361fea89c09f..72dcf379faea 100644 --- a/stage0/stdlib/Lean/Elab/Open.c +++ b/stage0/stdlib/Lean/Elab/Open.c @@ -3641,7 +3641,7 @@ static lean_object* _init_l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resol 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_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___rarg___lambda__2___closed__3; x_2 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___rarg___lambda__2___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___rarg___lambda__2___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/PatternVar.c b/stage0/stdlib/Lean/Elab/PatternVar.c index 1f06e50fc667..907da89ebb95 100644 --- a/stage0/stdlib/Lean/Elab/PatternVar.c +++ b/stage0/stdlib/Lean/Elab/PatternVar.c @@ -1169,7 +1169,7 @@ static lean_object* _init_l___private_Lean_Elab_PatternVar_0__Lean_Elab_Term_Col 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_PatternVar_0__Lean_Elab_Term_CollectPatternVars_getNextParam___closed__1; x_2 = l___private_Lean_Elab_PatternVar_0__Lean_Elab_Term_CollectPatternVars_getNextParam___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_PatternVar_0__Lean_Elab_Term_CollectPatternVars_getNextParam___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c b/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c index f606b36cb098..339156d88b4a 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Basic.c @@ -1127,7 +1127,9 @@ if (x_13 == 0) { lean_object* x_14; lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); x_14 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_14, 0, x_5); @@ -1148,7 +1150,9 @@ x_18 = lean_ctor_get(x_17, 1); lean_inc(x_18); lean_dec(x_17); lean_inc(x_11); -lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); lean_inc(x_6); x_19 = l_Lean_Elab_Term_applyAttributesAt(x_16, x_18, x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_18); @@ -1170,7 +1174,9 @@ else { uint8_t x_25; lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); x_25 = !lean_is_exclusive(x_19); if (x_25 == 0) @@ -1263,9 +1269,7 @@ lean_dec(x_3); x_15 = lean_unbox_usize(x_4); lean_dec(x_4); x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_applyAttributesOf___spec__1(x_13, x_2, x_14, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_10); lean_dec(x_2); return x_16; } @@ -1277,9 +1281,7 @@ uint8_t x_10; lean_object* x_11; x_10 = lean_unbox(x_2); lean_dec(x_2); x_11 = l_Lean_Elab_applyAttributesOf(x_1, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_7); lean_dec(x_1); return x_11; } @@ -2563,7 +2565,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -2614,7 +2616,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 4); +x_29 = lean_ctor_get(x_27, 5); lean_inc(x_29); lean_dec(x_27); x_30 = lean_ctor_get(x_29, 1); @@ -2637,7 +2639,7 @@ lean_dec(x_34); x_36 = lean_st_ref_take(x_3, x_35); x_37 = lean_ctor_get(x_36, 0); lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 4); +x_38 = lean_ctor_get(x_37, 5); lean_inc(x_38); x_39 = lean_ctor_get(x_36, 1); lean_inc(x_39); @@ -2646,7 +2648,7 @@ x_40 = !lean_is_exclusive(x_37); if (x_40 == 0) { lean_object* x_41; uint8_t x_42; -x_41 = lean_ctor_get(x_37, 4); +x_41 = lean_ctor_get(x_37, 5); lean_dec(x_41); x_42 = !lean_is_exclusive(x_38); if (x_42 == 0) @@ -2691,7 +2693,7 @@ x_53 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_50); -lean_ctor_set(x_37, 4, x_53); +lean_ctor_set(x_37, 5, x_53); x_54 = lean_st_ref_set(x_3, x_37, x_39); lean_dec(x_3); x_55 = lean_ctor_get(x_54, 1); @@ -2716,243 +2718,249 @@ return x_57; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_58 = lean_ctor_get(x_37, 0); x_59 = lean_ctor_get(x_37, 1); x_60 = lean_ctor_get(x_37, 2); x_61 = lean_ctor_get(x_37, 3); +x_62 = lean_ctor_get(x_37, 4); +lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); lean_inc(x_58); lean_dec(x_37); -x_62 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); +x_63 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); +x_64 = lean_ctor_get(x_38, 0); +lean_inc(x_64); if (lean_is_exclusive(x_38)) { lean_ctor_release(x_38, 0); lean_ctor_release(x_38, 1); - x_64 = x_38; + x_65 = x_38; } else { lean_dec_ref(x_38); - x_64 = lean_box(0); + x_65 = lean_box(0); } -x_65 = l_Std_PersistentArray_append___rarg(x_19, x_32); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(0, 2, 1); +x_66 = l_Std_PersistentArray_append___rarg(x_19, x_32); +if (lean_is_scalar(x_65)) { + x_67 = lean_alloc_ctor(0, 2, 1); } else { - x_66 = x_64; -} -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_65); -lean_ctor_set_uint8(x_66, sizeof(void*)*2, x_62); -x_67 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_67, 0, x_58); -lean_ctor_set(x_67, 1, x_59); -lean_ctor_set(x_67, 2, x_60); -lean_ctor_set(x_67, 3, x_61); -lean_ctor_set(x_67, 4, x_66); -x_68 = lean_st_ref_set(x_3, x_67, x_39); + x_67 = x_65; +} +lean_ctor_set(x_67, 0, x_64); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_63); +x_68 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_68, 0, x_58); +lean_ctor_set(x_68, 1, x_59); +lean_ctor_set(x_68, 2, x_60); +lean_ctor_set(x_68, 3, x_61); +lean_ctor_set(x_68, 4, x_62); +lean_ctor_set(x_68, 5, x_67); +x_69 = lean_st_ref_set(x_3, x_68, x_39); lean_dec(x_3); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_70 = x_68; +x_70 = lean_ctor_get(x_69, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_71 = x_69; } else { - lean_dec_ref(x_68); - x_70 = lean_box(0); + lean_dec_ref(x_69); + x_71 = lean_box(0); } -if (lean_is_scalar(x_70)) { - x_71 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_70; + x_72 = x_71; } -lean_ctor_set(x_71, 0, x_22); -lean_ctor_set(x_71, 1, x_69); -return x_71; +lean_ctor_set(x_72, 0, x_22); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_72 = lean_ctor_get(x_21, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_21, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_73 = lean_ctor_get(x_21, 0); lean_inc(x_73); +x_74 = lean_ctor_get(x_21, 1); +lean_inc(x_74); lean_dec(x_21); -x_74 = lean_st_ref_get(x_7, x_73); -x_75 = lean_ctor_get(x_74, 1); -lean_inc(x_75); -lean_dec(x_74); -x_76 = lean_st_ref_get(x_3, x_75); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); +x_75 = lean_st_ref_get(x_7, x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_st_ref_get(x_3, x_76); +x_78 = lean_ctor_get(x_77, 0); lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_ctor_get(x_77, 4); +x_79 = lean_ctor_get(x_77, 1); lean_inc(x_79); lean_dec(x_77); -x_80 = lean_ctor_get(x_79, 1); +x_80 = lean_ctor_get(x_78, 5); lean_inc(x_80); -x_81 = l_Std_PersistentArray_mapM___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__8(x_79, x_80, x_2, x_3, x_4, x_5, x_6, x_7, x_78); +lean_dec(x_78); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +x_82 = l_Std_PersistentArray_mapM___at___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___spec__8(x_80, x_81, x_2, x_3, x_4, x_5, x_6, x_7, x_79); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_st_ref_get(x_7, x_83); +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +lean_dec(x_82); +x_85 = lean_st_ref_get(x_7, x_84); lean_dec(x_7); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_3, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_87, 4); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_st_ref_take(x_3, x_86); +x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 1); +x_89 = lean_ctor_get(x_88, 5); lean_inc(x_89); -lean_dec(x_86); -x_90 = !lean_is_exclusive(x_87); -if (x_90 == 0) -{ -lean_object* x_91; uint8_t x_92; -x_91 = lean_ctor_get(x_87, 4); -lean_dec(x_91); -x_92 = !lean_is_exclusive(x_88); -if (x_92 == 0) -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; -x_93 = lean_ctor_get(x_88, 1); -lean_dec(x_93); -x_94 = l_Std_PersistentArray_append___rarg(x_19, x_82); -lean_ctor_set(x_88, 1, x_94); -x_95 = lean_st_ref_set(x_3, x_87, x_89); +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = !lean_is_exclusive(x_88); +if (x_91 == 0) +{ +lean_object* x_92; uint8_t x_93; +x_92 = lean_ctor_get(x_88, 5); +lean_dec(x_92); +x_93 = !lean_is_exclusive(x_89); +if (x_93 == 0) +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_89, 1); +lean_dec(x_94); +x_95 = l_Std_PersistentArray_append___rarg(x_19, x_83); +lean_ctor_set(x_89, 1, x_95); +x_96 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) { -lean_object* x_97; -x_97 = lean_ctor_get(x_95, 0); -lean_dec(x_97); -lean_ctor_set_tag(x_95, 1); -lean_ctor_set(x_95, 0, x_72); -return x_95; +lean_object* x_98; +x_98 = lean_ctor_get(x_96, 0); +lean_dec(x_98); +lean_ctor_set_tag(x_96, 1); +lean_ctor_set(x_96, 0, x_73); +return x_96; } else { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_95, 1); -lean_inc(x_98); -lean_dec(x_95); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_72); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_dec(x_96); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_73); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_100 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_101 = lean_ctor_get(x_88, 0); -lean_inc(x_101); -lean_dec(x_88); -x_102 = l_Std_PersistentArray_append___rarg(x_19, x_82); -x_103 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_100); -lean_ctor_set(x_87, 4, x_103); -x_104 = lean_st_ref_set(x_3, x_87, x_89); +uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_101 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +lean_dec(x_89); +x_103 = l_Std_PersistentArray_append___rarg(x_19, x_83); +x_104 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set_uint8(x_104, sizeof(void*)*2, x_101); +lean_ctor_set(x_88, 5, x_104); +x_105 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_106 = x_104; +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; - lean_ctor_set_tag(x_107, 1); + x_108 = x_107; + lean_ctor_set_tag(x_108, 1); } -lean_ctor_set(x_107, 0, x_72); -lean_ctor_set(x_107, 1, x_105); -return x_107; +lean_ctor_set(x_108, 0, x_73); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_108 = lean_ctor_get(x_87, 0); -x_109 = lean_ctor_get(x_87, 1); -x_110 = lean_ctor_get(x_87, 2); -x_111 = lean_ctor_get(x_87, 3); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_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; +x_109 = lean_ctor_get(x_88, 0); +x_110 = lean_ctor_get(x_88, 1); +x_111 = lean_ctor_get(x_88, 2); +x_112 = lean_ctor_get(x_88, 3); +x_113 = lean_ctor_get(x_88, 4); +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_dec(x_87); -x_112 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_113 = lean_ctor_get(x_88, 0); -lean_inc(x_113); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_114 = x_88; +lean_dec(x_88); +x_114 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_115 = lean_ctor_get(x_89, 0); +lean_inc(x_115); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_116 = x_89; } else { - lean_dec_ref(x_88); - x_114 = lean_box(0); + lean_dec_ref(x_89); + x_116 = lean_box(0); } -x_115 = l_Std_PersistentArray_append___rarg(x_19, x_82); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 1); +x_117 = l_Std_PersistentArray_append___rarg(x_19, x_83); +if (lean_is_scalar(x_116)) { + x_118 = lean_alloc_ctor(0, 2, 1); } else { - x_116 = x_114; -} -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_115); -lean_ctor_set_uint8(x_116, sizeof(void*)*2, x_112); -x_117 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_117, 0, x_108); -lean_ctor_set(x_117, 1, x_109); -lean_ctor_set(x_117, 2, x_110); -lean_ctor_set(x_117, 3, x_111); -lean_ctor_set(x_117, 4, x_116); -x_118 = lean_st_ref_set(x_3, x_117, x_89); + x_118 = x_116; +} +lean_ctor_set(x_118, 0, x_115); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); +x_119 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_119, 0, x_109); +lean_ctor_set(x_119, 1, x_110); +lean_ctor_set(x_119, 2, x_111); +lean_ctor_set(x_119, 3, x_112); +lean_ctor_set(x_119, 4, x_113); +lean_ctor_set(x_119, 5, x_118); +x_120 = lean_st_ref_set(x_3, x_119, x_90); lean_dec(x_3); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_122 = x_120; } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + lean_dec_ref(x_120); + x_122 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); } else { - x_121 = x_120; - lean_ctor_set_tag(x_121, 1); + x_123 = x_122; + lean_ctor_set_tag(x_123, 1); } -lean_ctor_set(x_121, 0, x_72); -lean_ctor_set(x_121, 1, x_119); -return x_121; +lean_ctor_set(x_123, 0, x_73); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } @@ -3019,7 +3027,9 @@ if (x_1 == 0) { lean_object* x_11; lean_object* x_12; lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); x_11 = lean_box(0); x_12 = lean_alloc_ctor(0, 2, 0); @@ -3047,9 +3057,7 @@ lean_dec(x_5); lean_dec(x_4); x_14 = lean_box(0); x_15 = l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___lambda__2(x_1, x_2, x_14, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_11); return x_15; } else @@ -3063,9 +3071,7 @@ lean_object* x_17; lean_object* x_18; lean_dec(x_5); x_17 = lean_box(0); x_18 = l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___lambda__2(x_1, x_2, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_11); return x_18; } else @@ -3125,9 +3131,7 @@ lean_inc(x_28); lean_dec(x_19); x_29 = lean_box(0); x_30 = l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___lambda__2(x_1, x_2, x_29, x_7, x_8, x_9, x_10, x_11, x_12, x_28); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_11); return x_30; } } @@ -3361,7 +3365,9 @@ lean_inc(x_1); x_19 = lean_array_push(x_18, x_1); x_20 = 0; lean_inc(x_10); -lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); x_21 = l_Lean_Elab_applyAttributesOf(x_19, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_17); if (lean_obj_tag(x_21) == 0) @@ -4344,9 +4350,7 @@ uint8_t x_11; lean_object* x_12; x_11 = lean_unbox(x_1); lean_dec(x_1); x_12 = l___private_Lean_Elab_PreDefinition_Basic_0__Lean_Elab_addNonRecAux___lambda__2(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_8); lean_dec(x_3); lean_dec(x_2); return x_12; @@ -5182,7 +5186,7 @@ static lean_object* _init_l_Lean_Elab_addAndCompileUnsafe___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_addAndCompileUnsafe___closed__1; x_2 = l_Lean_Elab_addAndCompileUnsafe___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_addAndCompileUnsafe___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -5350,7 +5354,9 @@ lean_inc(x_49); lean_dec(x_48); x_50 = 0; lean_inc(x_8); -lean_inc(x_37); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); lean_inc(x_3); x_51 = l_Lean_Elab_applyAttributesOf(x_14, x_50, x_3, x_4, x_5, x_6, x_37, x_8, x_49); if (lean_obj_tag(x_51) == 0) @@ -5414,9 +5420,7 @@ lean_inc(x_62); lean_dec(x_53); x_63 = lean_box(0); x_64 = l_Lean_Elab_addAndCompileUnsafe___lambda__2(x_14, x_63, x_3, x_4, x_5, x_6, x_37, x_8, x_62); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_37); lean_dec(x_14); return x_64; } @@ -5639,9 +5643,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_addAndCompileUnsafe___lambda__2___boxed(lea { lean_object* x_10; x_10 = l_Lean_Elab_addAndCompileUnsafe___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); return x_10; diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Eqns.c b/stage0/stdlib/Lean/Elab/PreDefinition/Eqns.c index 71b999e6ac21..9edfa2ec0aff 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Eqns.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Eqns.c @@ -261,6 +261,7 @@ LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at___private_Lean_Elab lean_object* l_Lean_Meta_Match_isNamedPattern_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Eqns_mkUnfoldProof_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Eqns_deltaLHS___lambda__2___closed__6; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Eqns_mkEqnTypes_go___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Eqns_simpEqnType___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Eqns_simpEqnType___lambda__2___closed__4; @@ -337,7 +338,6 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Elab_PreD lean_object* l_Lean_Meta_delta_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_replaceFVarId(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Eqns_deltaRHS_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_saveEqn___spec__27___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_commitWhenSome_x3f___at_Lean_Elab_Eqns_funext_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Eqns_mkEqnTypes_go___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -375,12 +375,12 @@ LEAN_EXPORT lean_object* l_Lean_ForEachExpr_visit___at_Lean_Elab_Eqns_simpEqnTyp LEAN_EXPORT lean_object* l_Lean_Elab_Eqns_simpEqnType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Eqns_removeUnusedEqnHypotheses_go___spec__9___boxed(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_Elab_Eqns_deltaLHS___lambda__2___closed__9; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Eqns_removeUnusedEqnHypotheses_go___spec__21(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Eqns_simpEqnType___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_Elab_Eqns_getUnfoldFor_x3f___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Eqns_removeUnusedEqnHypotheses_go___spec__21___at_Lean_Elab_Eqns_removeUnusedEqnHypotheses_go___spec__22(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -491,6 +491,7 @@ LEAN_EXPORT lean_object* l_Lean_mkFreshId___at_Lean_Elab_Eqns_removeUnusedEqnHyp static lean_object* l_Lean_Elab_Eqns_splitMatch_x3f_go___closed__5; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Eqns_removeUnusedEqnHypotheses_go___spec__11(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Eqns_mkUnfoldProof___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_Elab_Eqns_getUnfoldFor_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Eqns_removeUnusedEqnHypotheses_go___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_saveEqn___spec__31(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1746,7 +1747,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDef lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2238,7 +2239,7 @@ x_21 = lean_ctor_get(x_7, 0); lean_inc(x_21); lean_dec(x_7); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_4, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_22); x_24 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__3___closed__5; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -13620,7 +13621,7 @@ x_5 = lean_ctor_get(x_3, 0); lean_inc(x_5); lean_dec(x_3); x_6 = lean_unsigned_to_nat(0u); -x_7 = l_Lean_Expr_getAppNumArgsAux(x_2, x_6); +x_7 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_6); x_8 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__3___closed__5; lean_inc(x_7); x_9 = lean_mk_array(x_7, x_8); @@ -20116,80 +20117,128 @@ x_10 = lean_ctor_get(x_7, 1); x_11 = l_Lean_Expr_getAppFn(x_9); if (lean_obj_tag(x_11) == 11) { -lean_object* x_12; lean_object* x_13; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_free_object(x_7); -x_12 = lean_ctor_get(x_11, 2); +x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_whnfAux(x_12, x_2, x_3, x_4, x_5, x_10); -if (lean_obj_tag(x_13) == 0) +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +x_14 = lean_ctor_get(x_11, 2); +lean_inc(x_14); +lean_inc(x_14); +x_15 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_whnfAux(x_14, x_2, x_3, x_4, x_5, x_10); +if (lean_obj_tag(x_15) == 0) { -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +uint8_t x_16; +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_expr_update_proj(x_11, x_15); -x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_9, x_17); -x_19 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__3___closed__5; -lean_inc(x_18); -x_20 = lean_mk_array(x_18, x_19); -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_nat_sub(x_18, x_21); -lean_dec(x_18); -x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_20, x_22); -x_24 = l_Lean_mkAppN(x_16, x_23); -lean_ctor_set(x_13, 0, x_24); -return x_13; +lean_object* x_17; size_t x_18; size_t x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ptr_addr(x_14); +lean_dec(x_14); +x_19 = lean_ptr_addr(x_17); +x_20 = lean_usize_dec_eq(x_18, x_19); +x_21 = lean_unsigned_to_nat(0u); +x_22 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_21); +x_23 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__3___closed__5; +lean_inc(x_22); +x_24 = lean_mk_array(x_22, x_23); +x_25 = lean_unsigned_to_nat(1u); +x_26 = lean_nat_sub(x_22, x_25); +lean_dec(x_22); +x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_24, x_26); +if (x_20 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_11); +x_28 = l_Lean_Expr_proj___override(x_12, x_13, x_17); +x_29 = l_Lean_mkAppN(x_28, x_27); +lean_ctor_set(x_15, 0, x_29); +return x_15; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_25 = lean_ctor_get(x_13, 0); -x_26 = lean_ctor_get(x_13, 1); -lean_inc(x_26); -lean_inc(x_25); +lean_object* x_30; +lean_dec(x_17); lean_dec(x_13); -x_27 = lean_expr_update_proj(x_11, x_25); -x_28 = lean_unsigned_to_nat(0u); -x_29 = l_Lean_Expr_getAppNumArgsAux(x_9, x_28); -x_30 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__3___closed__5; -lean_inc(x_29); -x_31 = lean_mk_array(x_29, x_30); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_nat_sub(x_29, x_32); -lean_dec(x_29); -x_34 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_31, x_33); -x_35 = l_Lean_mkAppN(x_27, x_34); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_26); -return x_36; +lean_dec(x_12); +x_30 = l_Lean_mkAppN(x_11, x_27); +lean_ctor_set(x_15, 0, x_30); +return x_15; } } else { -uint8_t x_37; +lean_object* x_31; lean_object* x_32; size_t x_33; size_t x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_31 = lean_ctor_get(x_15, 0); +x_32 = lean_ctor_get(x_15, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_15); +x_33 = lean_ptr_addr(x_14); +lean_dec(x_14); +x_34 = lean_ptr_addr(x_31); +x_35 = lean_usize_dec_eq(x_33, x_34); +x_36 = lean_unsigned_to_nat(0u); +x_37 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_36); +x_38 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__3___closed__5; +lean_inc(x_37); +x_39 = lean_mk_array(x_37, x_38); +x_40 = lean_unsigned_to_nat(1u); +x_41 = lean_nat_sub(x_37, x_40); +lean_dec(x_37); +x_42 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_9, x_39, x_41); +if (x_35 == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_dec(x_11); -lean_dec(x_9); -x_37 = !lean_is_exclusive(x_13); -if (x_37 == 0) +x_43 = l_Lean_Expr_proj___override(x_12, x_13, x_31); +x_44 = l_Lean_mkAppN(x_43, x_42); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_32); +return x_45; +} +else { -return x_13; +lean_object* x_46; lean_object* x_47; +lean_dec(x_31); +lean_dec(x_13); +lean_dec(x_12); +x_46 = l_Lean_mkAppN(x_11, x_42); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_32); +return x_47; +} +} } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_13, 0); -x_39 = lean_ctor_get(x_13, 1); -lean_inc(x_39); -lean_inc(x_38); +uint8_t x_48; +lean_dec(x_14); lean_dec(x_13); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_9); +x_48 = !lean_is_exclusive(x_15); +if (x_48 == 0) +{ +return x_15; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_15, 0); +x_50 = lean_ctor_get(x_15, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_15); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; } } } @@ -20205,120 +20254,153 @@ return x_7; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_7, 0); -x_42 = lean_ctor_get(x_7, 1); -lean_inc(x_42); -lean_inc(x_41); +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_7, 0); +x_53 = lean_ctor_get(x_7, 1); +lean_inc(x_53); +lean_inc(x_52); lean_dec(x_7); -x_43 = l_Lean_Expr_getAppFn(x_41); -if (lean_obj_tag(x_43) == 11) +x_54 = l_Lean_Expr_getAppFn(x_52); +if (lean_obj_tag(x_54) == 11) { -lean_object* x_44; lean_object* x_45; -x_44 = lean_ctor_get(x_43, 2); -lean_inc(x_44); -x_45 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_whnfAux(x_44, x_2, x_3, x_4, x_5, x_42); -if (lean_obj_tag(x_45) == 0) +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +lean_inc(x_57); +x_58 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_whnfAux(x_57, x_2, x_3, x_4, x_5, x_53); +if (lean_obj_tag(x_58) == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_48 = x_45; +lean_object* x_59; lean_object* x_60; lean_object* x_61; size_t x_62; size_t x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_58, 1); +lean_inc(x_60); +if (lean_is_exclusive(x_58)) { + lean_ctor_release(x_58, 0); + lean_ctor_release(x_58, 1); + x_61 = x_58; } else { - lean_dec_ref(x_45); - x_48 = lean_box(0); + lean_dec_ref(x_58); + x_61 = lean_box(0); } -x_49 = lean_expr_update_proj(x_43, x_46); -x_50 = lean_unsigned_to_nat(0u); -x_51 = l_Lean_Expr_getAppNumArgsAux(x_41, x_50); -x_52 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__3___closed__5; -lean_inc(x_51); -x_53 = lean_mk_array(x_51, x_52); -x_54 = lean_unsigned_to_nat(1u); -x_55 = lean_nat_sub(x_51, x_54); -lean_dec(x_51); -x_56 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_41, x_53, x_55); -x_57 = l_Lean_mkAppN(x_49, x_56); -if (lean_is_scalar(x_48)) { - x_58 = lean_alloc_ctor(0, 2, 0); +x_62 = lean_ptr_addr(x_57); +lean_dec(x_57); +x_63 = lean_ptr_addr(x_59); +x_64 = lean_usize_dec_eq(x_62, x_63); +x_65 = lean_unsigned_to_nat(0u); +x_66 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_52, x_65); +x_67 = l___private_Lean_Elab_PreDefinition_Eqns_0__Lean_Elab_Eqns_findMatchToSplit_x3f___lambda__3___closed__5; +lean_inc(x_66); +x_68 = lean_mk_array(x_66, x_67); +x_69 = lean_unsigned_to_nat(1u); +x_70 = lean_nat_sub(x_66, x_69); +lean_dec(x_66); +x_71 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_52, x_68, x_70); +if (x_64 == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_dec(x_54); +x_72 = l_Lean_Expr_proj___override(x_55, x_56, x_59); +x_73 = l_Lean_mkAppN(x_72, x_71); +if (lean_is_scalar(x_61)) { + x_74 = lean_alloc_ctor(0, 2, 0); } else { - x_58 = x_48; + x_74 = x_61; } -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_47); -return x_58; +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_60); +return x_74; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -lean_dec(x_43); -lean_dec(x_41); -x_59 = lean_ctor_get(x_45, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_45, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_61 = x_45; +lean_object* x_75; lean_object* x_76; +lean_dec(x_59); +lean_dec(x_56); +lean_dec(x_55); +x_75 = l_Lean_mkAppN(x_54, x_71); +if (lean_is_scalar(x_61)) { + x_76 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_45); - x_61 = lean_box(0); + x_76 = x_61; } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_60); +return x_76; +} +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +lean_dec(x_57); +lean_dec(x_56); +lean_dec(x_55); +lean_dec(x_54); +lean_dec(x_52); +x_77 = lean_ctor_get(x_58, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_58, 1); +lean_inc(x_78); +if (lean_is_exclusive(x_58)) { + lean_ctor_release(x_58, 0); + lean_ctor_release(x_58, 1); + x_79 = x_58; } else { - x_62 = x_61; + lean_dec_ref(x_58); + x_79 = lean_box(0); } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; +if (lean_is_scalar(x_79)) { + x_80 = lean_alloc_ctor(1, 2, 0); +} else { + x_80 = x_79; +} +lean_ctor_set(x_80, 0, x_77); +lean_ctor_set(x_80, 1, x_78); +return x_80; } } else { -lean_object* x_63; -lean_dec(x_43); +lean_object* x_81; +lean_dec(x_54); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_41); -lean_ctor_set(x_63, 1, x_42); -return x_63; +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_52); +lean_ctor_set(x_81, 1, x_53); +return x_81; } } } else { -uint8_t x_64; +uint8_t x_82; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_64 = !lean_is_exclusive(x_7); -if (x_64 == 0) +x_82 = !lean_is_exclusive(x_7); +if (x_82 == 0) { return x_7; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_7, 0); -x_66 = lean_ctor_get(x_7, 1); -lean_inc(x_66); -lean_inc(x_65); +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_7, 0); +x_84 = lean_ctor_get(x_7, 1); +lean_inc(x_84); +lean_inc(x_83); lean_dec(x_7); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -return x_67; +x_85 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +return x_85; } } } diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/Main.c index 8daa4df95ef0..b6f85e8840d2 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Main.c @@ -16,6 +16,7 @@ extern "C" { lean_object* l_Lean_Elab_WF_TerminationBy_markAsUsed(lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_addPreDefinitions___spec__2___closed__4; +lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_addPreDefinitions___spec__9___rarg___closed__2; size_t lean_usize_add(size_t, size_t); lean_object* l_List_forM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -82,6 +83,7 @@ static lean_object* l_Lean_Elab_addPreDefinitions___closed__11; lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* l_Lean_MessageData_ofList(lean_object*); +uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_addAndCompilePartial___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_addAndCompilePartial___spec__2___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_betaReduceLetRecApps___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -126,7 +128,6 @@ static lean_object* l_Lean_Elab_addPreDefinitions___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Util_SCC_0__Lean_SCC_resetOnStack___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_partitionPreDefs___spec__21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_addAndCompilePartial___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_addPreDefinitions___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_applyAttributesOf(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_partitionPreDefs___spec__23(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_addPreDefinitions___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -178,6 +179,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_SCC_0__Lean_SCC_modifyDataOf___at LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_partitionPreDefs___lambda__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_partitionPreDefs___spec__24___lambda__1___boxed(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_addAndCompilePartial___spec__2___closed__5; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_partitionPreDefs___lambda__2___boxed__const__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_addPreDefinitions___spec__2___closed__1; @@ -238,7 +240,6 @@ size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_addPreDefinitions___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_addPreDefinitions___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_addAndCompilePartialRec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(lean_object*, lean_object*); lean_object* l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isLambda(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_addPreDefinitions___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -256,7 +257,6 @@ lean_object* l_List_redLength___rarg(lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_addPreDefinitions___spec__18(lean_object*, size_t, size_t); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_addAndCompilePartial___spec__1(lean_object*); lean_object* lean_environment_main_module(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_addPreDefinitions___spec__21(lean_object*, size_t, size_t); @@ -2641,7 +2641,7 @@ lean_inc(x_13); x_14 = lean_ctor_get(x_11, 0); lean_inc(x_14); lean_dec(x_11); -x_15 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_13, x_14); +x_15 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_13, x_14); lean_dec(x_14); lean_dec(x_13); if (x_15 == 0) @@ -2674,7 +2674,7 @@ lean_inc(x_20); x_21 = lean_ctor_get(x_18, 0); lean_inc(x_21); lean_dec(x_18); -x_22 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_20, x_21); +x_22 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_20, x_21); lean_dec(x_21); lean_dec(x_20); if (x_22 == 0) @@ -3960,7 +3960,7 @@ else { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_2, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_15); x_17 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_Main_0__Lean_Elab_betaReduceLetRecApps___spec__3___lambda__1___closed__1; lean_inc(x_16); x_18 = lean_mk_array(x_16, x_17); @@ -4463,7 +4463,9 @@ x_28 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Main_0__L x_29 = lean_array_push(x_28, x_14); x_30 = 0; lean_inc(x_10); -lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); x_31 = l_Lean_Elab_applyAttributesOf(x_29, x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_27); if (lean_obj_tag(x_31) == 0) @@ -4474,7 +4476,9 @@ lean_inc(x_32); lean_dec(x_31); x_33 = 1; lean_inc(x_10); -lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); x_34 = l_Lean_Elab_applyAttributesOf(x_29, x_33, x_5, x_6, x_7, x_8, x_9, x_10, x_32); lean_dec(x_29); @@ -6673,7 +6677,7 @@ x_39 = l_Lean_replaceRef(x_26, x_38); lean_dec(x_38); lean_dec(x_26); lean_ctor_set(x_9, 5, x_39); -x_40 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_36, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +x_40 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_36, x_5, x_6, x_7, x_8, x_9, x_10, x_18); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6738,7 +6742,7 @@ lean_ctor_set(x_57, 7, x_52); lean_ctor_set(x_57, 8, x_53); lean_ctor_set(x_57, 9, x_54); lean_ctor_set(x_57, 10, x_55); -x_58 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_36, x_5, x_6, x_7, x_8, x_57, x_10, x_18); +x_58 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_36, x_5, x_6, x_7, x_8, x_57, x_10, x_18); lean_dec(x_10); lean_dec(x_57); lean_dec(x_8); @@ -7505,7 +7509,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_addPreDefiniti lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_addPreDefinitions___spec__22___lambda__3___closed__1; x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_addPreDefinitions___spec__22___lambda__3___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Array_forInUnsafe_loop___at_Lean_Elab_addPreDefinitions___spec__22___lambda__3___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c b/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c index 0d6ed07a99d3..5713d8efad82 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/MkInhabitant.c @@ -570,7 +570,7 @@ static lean_object* _init_l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Le lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_loop___closed__2; x_2 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_loop___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_PreDefinition_MkInhabitant_0__Lean_Elab_mkFnInhabitant_x3f_loop___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c index 7df820069219..0af8e3087558 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/BRecOn.c @@ -201,6 +201,7 @@ static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lea lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_throwToBelowFailed(lean_object*); lean_object* l_Lean_Meta_decLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -276,7 +277,6 @@ lean_object* l_List_redLength___rarg(lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_replaceRecApps_loop___spec__40(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkBRecOn___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__5___closed__4; @@ -739,7 +739,7 @@ x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); lean_dec(x_14); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_15, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_15, x_17); x_19 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -1681,7 +1681,7 @@ static lean_object* _init_l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDef lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__1___rarg___lambda__2___closed__1; x_2 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__1___rarg___lambda__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_withBelowDict___spec__1___rarg___lambda__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2030,7 +2030,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0 lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_dec(x_4); x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_1, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_10); x_12 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_11); x_13 = lean_mk_array(x_11, x_12); @@ -2951,7 +2951,7 @@ if (x_23 == 0) lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; x_24 = lean_ctor_get(x_14, 0); x_25 = lean_unsigned_to_nat(0u); -x_26 = l_Lean_Expr_getAppNumArgsAux(x_2, x_25); +x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_25); x_27 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_26); x_28 = lean_mk_array(x_26, x_27); @@ -3061,7 +3061,7 @@ x_60 = lean_ctor_get(x_14, 0); lean_inc(x_60); lean_dec(x_14); x_61 = lean_unsigned_to_nat(0u); -x_62 = l_Lean_Expr_getAppNumArgsAux(x_2, x_61); +x_62 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_61); x_63 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_62); x_64 = lean_mk_array(x_62, x_63); @@ -3184,7 +3184,7 @@ if (lean_is_exclusive(x_14)) { x_100 = lean_box(0); } x_101 = lean_unsigned_to_nat(0u); -x_102 = l_Lean_Expr_getAppNumArgsAux(x_2, x_101); +x_102 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_101); x_103 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_102); x_104 = lean_mk_array(x_102, x_103); @@ -9384,7 +9384,7 @@ x_24 = lean_ctor_get(x_21, 1); lean_inc(x_24); lean_dec(x_21); x_25 = lean_unsigned_to_nat(0u); -x_26 = l_Lean_Expr_getAppNumArgsAux(x_3, x_25); +x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_25); x_27 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_26); x_28 = lean_mk_array(x_26, x_27); @@ -9834,7 +9834,7 @@ x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_1, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_20); x_22 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_21); x_23 = lean_mk_array(x_21, x_22); @@ -9863,7 +9863,7 @@ if (x_30 == 0) lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_dec(x_28); x_31 = lean_unsigned_to_nat(0u); -x_32 = l_Lean_Expr_getAppNumArgsAux(x_1, x_31); +x_32 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_31); x_33 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_32); x_34 = lean_mk_array(x_32, x_33); @@ -9893,7 +9893,7 @@ x_41 = lean_ctor_get(x_39, 1); lean_inc(x_41); lean_dec(x_39); x_42 = lean_unsigned_to_nat(0u); -x_43 = l_Lean_Expr_getAppNumArgsAux(x_1, x_42); +x_43 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_42); x_44 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_43); x_45 = lean_mk_array(x_43, x_44); @@ -10086,7 +10086,7 @@ if (x_94 == 0) lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_dec(x_92); x_95 = lean_unsigned_to_nat(0u); -x_96 = l_Lean_Expr_getAppNumArgsAux(x_1, x_95); +x_96 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_95); x_97 = l___private_Lean_Elab_PreDefinition_Structural_BRecOn_0__Lean_Elab_Structural_toBelowAux___lambda__4___closed__3; lean_inc(x_96); x_98 = lean_mk_array(x_96, x_97); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Basic.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Basic.c index 2bfa9becdcd4..decc87cca250 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Basic.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Basic.c @@ -30,10 +30,10 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Structural_instInhabit lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_instInhabitedM___closed__2; static lean_object* l_Lean_Elab_Structural_instInhabitedM___closed__1; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_recArgHasLooseBVarsAt___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Structural_instInhabitedM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_State_addMatchers___default; LEAN_EXPORT lean_object* l_Lean_Elab_Structural_run(lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -277,7 +277,7 @@ else { lean_object* x_6; lean_object* x_7; uint8_t x_8; x_6 = lean_unsigned_to_nat(0u); -x_7 = l_Lean_Expr_getAppNumArgsAux(x_3, x_6); +x_7 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_6); x_8 = lean_nat_dec_lt(x_2, x_7); if (x_8 == 0) { diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Eqns.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Eqns.c index 22d87aaa4d5e..668e6e83ca4e 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Eqns.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Eqns.c @@ -1842,7 +1842,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Structural_mkEqn lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Structural_mkEqns___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Structural_mkEqns___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Structural_mkEqns___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c index 95cda092efd5..7c264a1a9c21 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/FindRecArg.c @@ -118,6 +118,7 @@ uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_FindRecArg_0__Lean_Elab_Structural_hasBadParamDep_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_FindRecArg_0__Lean_Elab_Structural_throwStructuralFailed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Elab_PreDefinition_Structural_FindRecArg_0__Lean_Elab_Structural_hasBadIndexDep_x3f___spec__3(lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Structural_findRecArg_go___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); static lean_object* l_Lean_Elab_Structural_findRecArg_go___rarg___closed__10; @@ -167,7 +168,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_PreDefi static lean_object* l_Lean_addTrace___at_Lean_Elab_Structural_findRecArg_go___spec__12___closed__8; static lean_object* l_Lean_addTrace___at_Lean_Elab_Structural_findRecArg_go___spec__12___closed__2; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_indexOfAux___at___private_Lean_Elab_PreDefinition_Structural_FindRecArg_0__Lean_Elab_Structural_getIndexMinPos___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addTrace___at_Lean_Elab_Structural_findRecArg_go___spec__12___closed__1; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Elab_PreDefinition_Structural_FindRecArg_0__Lean_Elab_Structural_hasBadIndexDep_x3f___spec__11(lean_object*, lean_object*, lean_object*); @@ -5375,7 +5375,7 @@ goto block_210; 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_164; lean_object* x_185; uint8_t x_186; lean_dec(x_55); x_56 = lean_unsigned_to_nat(0u); -x_57 = l_Lean_Expr_getAppNumArgsAux(x_22, x_56); +x_57 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_22, x_56); x_58 = l_Lean_Elab_Structural_findRecArg_go___rarg___lambda__3___closed__1; lean_inc(x_57); x_59 = lean_mk_array(x_57, x_58); @@ -9335,7 +9335,7 @@ lean_inc(x_24); lean_dec(x_19); x_25 = lean_nat_add(x_24, x_20); lean_dec(x_20); -x_26 = l_Lean_Expr_getAppNumArgsAux(x_3, x_21); +x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_21); x_27 = lean_nat_dec_eq(x_25, x_26); lean_dec(x_25); if (x_27 == 0) @@ -9514,7 +9514,7 @@ lean_inc(x_64); lean_dec(x_58); x_65 = lean_nat_add(x_64, x_59); lean_dec(x_59); -x_66 = l_Lean_Expr_getAppNumArgsAux(x_3, x_60); +x_66 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_60); x_67 = lean_nat_dec_eq(x_65, x_66); lean_dec(x_65); if (x_67 == 0) diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/IndPred.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/IndPred.c index 87de49827925..09f228516de6 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/IndPred.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/IndPred.c @@ -94,6 +94,7 @@ static lean_object* l___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Le lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Structural_mkIndPredBRecOn___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_EXPORT lean_object* l_Lean_Elab_Structural_mkIndPredBRecOn___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop___spec__9___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); @@ -130,7 +131,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM__ lean_object* l_List_redLength___rarg(lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_mkIndPredBRecOn___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Structural_mkIndPredBRecOn___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Elab_Structural_mkIndPredBRecOn___closed__2; @@ -261,7 +261,7 @@ static lean_object* _init_l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_El lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__2; x_2 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -329,7 +329,7 @@ if (x_21 == 0) lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; x_22 = lean_ctor_get(x_12, 0); x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Lean_Expr_getAppNumArgsAux(x_1, x_23); +x_24 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_23); x_25 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__1; lean_inc(x_24); x_26 = lean_mk_array(x_24, x_25); @@ -439,7 +439,7 @@ x_58 = lean_ctor_get(x_12, 0); lean_inc(x_58); lean_dec(x_12); x_59 = lean_unsigned_to_nat(0u); -x_60 = l_Lean_Expr_getAppNumArgsAux(x_1, x_59); +x_60 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_59); x_61 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__1; lean_inc(x_60); x_62 = lean_mk_array(x_60, x_61); @@ -562,7 +562,7 @@ if (lean_is_exclusive(x_12)) { x_98 = lean_box(0); } x_99 = lean_unsigned_to_nat(0u); -x_100 = l_Lean_Expr_getAppNumArgsAux(x_1, x_99); +x_100 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_99); x_101 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__1; lean_inc(x_100); x_102 = lean_mk_array(x_100, x_101); @@ -2620,7 +2620,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_IndPred_ 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_dec(x_6); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -3036,7 +3036,7 @@ x_14 = lean_ctor_get(x_12, 1); lean_inc(x_14); lean_dec(x_12); x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_5, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_15); x_17 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__1; lean_inc(x_16); x_18 = lean_mk_array(x_16, x_17); @@ -3065,7 +3065,7 @@ if (x_25 == 0) lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_dec(x_23); x_26 = lean_unsigned_to_nat(0u); -x_27 = l_Lean_Expr_getAppNumArgsAux(x_5, x_26); +x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_26); x_28 = l_Lean_Meta_matchMatcherApp_x3f___at___private_Lean_Elab_PreDefinition_Structural_IndPred_0__Lean_Elab_Structural_replaceIndPredRecApps_loop_addBelow___spec__1___closed__1; lean_inc(x_27); x_29 = lean_mk_array(x_27, x_28); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c index 33a0f724331d..9217e7c13ce8 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/Main.c @@ -70,6 +70,7 @@ static lean_object* l_Lean_setEnv___at___private_Lean_Elab_PreDefinition_Structu lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_structuralRecursion___closed__6; static lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimRecursion___closed__3; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Structural_structuralRecursion___closed__3; @@ -102,7 +103,6 @@ static lean_object* l_Lean_setEnv___at___private_Lean_Elab_PreDefinition_Structu LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_getFixedPrefix___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Structural_mkBRecOn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_getFixedPrefix___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_setEnv___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimRecursion___spec__2___closed__7; lean_object* l_Lean_Elab_addNonRec___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_setEnv___at___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_elimRecursion___spec__2___closed__3; @@ -900,7 +900,7 @@ else { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_5, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_15); x_17 = l___private_Lean_Elab_PreDefinition_Structural_Main_0__Lean_Elab_Structural_getFixedPrefix___lambda__2___closed__1; lean_inc(x_16); x_18 = lean_mk_array(x_16, x_17); @@ -2816,7 +2816,7 @@ static lean_object* _init_l_Lean_Elab_Structural_structuralRecursion___closed__9 lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Structural_structuralRecursion___closed__6; x_2 = l_Lean_Elab_Structural_structuralRecursion___closed__7; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_Structural_structuralRecursion___closed__8; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -3061,9 +3061,7 @@ lean_dec(x_50); x_52 = lean_array_push(x_46, x_27); x_53 = 1; x_54 = l_Lean_Elab_applyAttributesOf(x_52, x_53, x_2, x_3, x_4, x_5, x_6, x_7, x_51); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +lean_dec(x_6); lean_dec(x_52); return x_54; } diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c index 092b80924699..4c2ac6d713b1 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/Structural/SmartUnfolding.c @@ -56,6 +56,7 @@ lean_object* l_Lean_Meta_markSmartUnfoldingMatch(lean_object*); static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__4; lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__6___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); @@ -74,7 +75,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___ lean_object* l_Lean_Meta_forallTelescope___at___private_Lean_Meta_InferType_0__Lean_Meta_inferForallType___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__3; lean_object* l_List_redLength___rarg(lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_isPerm___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_MatcherApp_toExpr(lean_object*); @@ -141,7 +141,7 @@ static lean_object* _init_l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structu lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__2; x_2 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -209,7 +209,7 @@ if (x_20 == 0) lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; x_21 = lean_ctor_get(x_11, 0); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_1, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_22); x_24 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__1; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -319,7 +319,7 @@ x_57 = lean_ctor_get(x_11, 0); lean_inc(x_57); lean_dec(x_11); x_58 = lean_unsigned_to_nat(0u); -x_59 = l_Lean_Expr_getAppNumArgsAux(x_1, x_58); +x_59 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_58); x_60 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__1; lean_inc(x_59); x_61 = lean_mk_array(x_59, x_60); @@ -442,7 +442,7 @@ if (lean_is_exclusive(x_11)) { x_97 = lean_box(0); } x_98 = lean_unsigned_to_nat(0u); -x_99 = l_Lean_Expr_getAppNumArgsAux(x_1, x_98); +x_99 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_98); x_100 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__1; lean_inc(x_99); x_101 = lean_mk_array(x_99, x_100); @@ -1823,7 +1823,7 @@ x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Lean_Expr_getAppNumArgsAux(x_3, x_12); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_12); x_14 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__1; lean_inc(x_13); x_15 = lean_mk_array(x_13, x_14); @@ -1852,7 +1852,7 @@ if (x_22 == 0) lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_dec(x_20); x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Lean_Expr_getAppNumArgsAux(x_3, x_23); +x_24 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_23); x_25 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Elab_Structural_addSmartUnfoldingDefAux_visit___spec__1___closed__1; lean_inc(x_24); x_26 = lean_mk_array(x_24, x_25); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Eqns.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Eqns.c index de146d8d7fda..3db98e0591d9 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Eqns.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Eqns.c @@ -134,6 +134,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Ela static lean_object* l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_decodePackedArg_x3f_decodePSigma___closed__4; lean_object* l_Lean_mkMapDeclarationExtension___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_registerEqnsInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_initFn____x40_Lean_Elab_PreDefinition_WF_Eqns___hyg_3112_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_initFn____x40_Lean_Elab_PreDefinition_WF_Eqns___hyg_2936_(lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_getFixedPrefix___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -180,7 +181,6 @@ static lean_object* l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_mkProof_go___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___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_getFixedPrefix___lambda__3___closed__2; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_getFixedPrefix___lambda__3___closed__1; static lean_object* l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_mkProof_go___lambda__1___closed__8; lean_object* l_Lean_Meta_applySimpResultToTarget(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -847,7 +847,7 @@ x_22 = l_Lean_Expr_constLevels_x21(x_21); x_23 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__6; x_24 = l_Lean_Expr_const___override(x_23, x_22); x_25 = lean_unsigned_to_nat(0u); -x_26 = l_Lean_Expr_getAppNumArgsAux(x_19, x_25); +x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_19, x_25); x_27 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__7; lean_inc(x_26); x_28 = lean_mk_array(x_26, x_27); @@ -1096,7 +1096,7 @@ x_84 = l_Lean_Expr_constLevels_x21(x_83); x_85 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__6; x_86 = l_Lean_Expr_const___override(x_85, x_84); x_87 = lean_unsigned_to_nat(0u); -x_88 = l_Lean_Expr_getAppNumArgsAux(x_81, x_87); +x_88 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_81, x_87); x_89 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__7; lean_inc(x_88); x_90 = lean_mk_array(x_88, x_89); @@ -1358,7 +1358,7 @@ x_147 = l_Lean_Expr_constLevels_x21(x_146); x_148 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__6; x_149 = l_Lean_Expr_const___override(x_148, x_147); x_150 = lean_unsigned_to_nat(0u); -x_151 = l_Lean_Expr_getAppNumArgsAux(x_143, x_150); +x_151 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_143, x_150); x_152 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__7; lean_inc(x_151); x_153 = lean_mk_array(x_151, x_152); @@ -1636,7 +1636,7 @@ x_213 = l_Lean_Expr_constLevels_x21(x_212); x_214 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__6; x_215 = l_Lean_Expr_const___override(x_214, x_213); x_216 = lean_unsigned_to_nat(0u); -x_217 = l_Lean_Expr_getAppNumArgsAux(x_209, x_216); +x_217 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_209, x_216); x_218 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__7; lean_inc(x_217); x_219 = lean_mk_array(x_217, x_218); @@ -2207,7 +2207,7 @@ static lean_object* _init_l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_El 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_PreDefinition_WF_Eqns_0__Lean_Elab_WF_decodePackedArg_x3f___closed__1; x_2 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_decodePackedArg_x3f___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_decodePackedArg_x3f___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2645,7 +2645,7 @@ else { lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_10, x_16); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_10, x_16); x_18 = lean_unsigned_to_nat(6u); x_19 = lean_nat_dec_le(x_18, x_17); if (x_19 == 0) @@ -4692,7 +4692,7 @@ x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); lean_dec(x_16); x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_17, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_17, x_18); x_20 = l___private_Lean_Elab_PreDefinition_WF_Eqns_0__Lean_Elab_WF_rwFixEq___lambda__1___closed__7; lean_inc(x_19); x_21 = lean_mk_array(x_19, x_20); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Fix.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Fix.c index 7e62e1499b1a..2a8c3d8cb157 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Fix.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Fix.c @@ -59,7 +59,6 @@ lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_CasesOnApp_addArg_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getRecAppSyntax_x3f(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Tactic_evalTacticAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f___at___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_loop___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_processRec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -69,6 +68,7 @@ lean_object* lean_st_ref_get(lean_object*, lean_object*); uint8_t l_Lean_Elab_Structural_recArgHasLooseBVarsAt(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_loop___spec__9___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* l_Lean_Elab_Tactic_evalTactic(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_mkFix___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_loop___spec__11___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); @@ -145,6 +145,7 @@ static lean_object* l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_p lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_loop___spec__4___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_mkFix___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Elab_WF_mkFix___lambda__1___closed__4; static lean_object* l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps___closed__1; lean_object* l_Lean_Meta_CasesOnApp_toExpr(lean_object*); @@ -191,7 +192,6 @@ static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_PreDefinitio lean_object* l_List_redLength___rarg(lean_object*); lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Term_addDotCompletionInfo___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -498,7 +498,7 @@ x_21 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_21, 0, x_19); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_18); -x_22 = l_Lean_Elab_Tactic_evalTacticAux(x_21, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_14); +x_22 = l_Lean_Elab_Tactic_evalTactic(x_21, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_14); return x_22; } } @@ -985,7 +985,7 @@ static lean_object* _init_l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Ela 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_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_processRec___closed__2; x_2 = l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_processRec___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_processRec___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -997,7 +997,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; x_14 = lean_unsigned_to_nat(0u); -x_15 = l_Lean_Expr_getAppNumArgsAux(x_5, x_14); +x_15 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_14); x_16 = lean_unsigned_to_nat(1u); x_17 = lean_nat_add(x_2, x_16); x_18 = lean_nat_dec_lt(x_15, x_17); @@ -1468,7 +1468,7 @@ if (x_24 == 0) lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; x_25 = lean_ctor_get(x_15, 0); x_26 = lean_unsigned_to_nat(0u); -x_27 = l_Lean_Expr_getAppNumArgsAux(x_2, x_26); +x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_26); x_28 = l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_processRec___closed__1; lean_inc(x_27); x_29 = lean_mk_array(x_27, x_28); @@ -1578,7 +1578,7 @@ x_61 = lean_ctor_get(x_15, 0); lean_inc(x_61); lean_dec(x_15); x_62 = lean_unsigned_to_nat(0u); -x_63 = l_Lean_Expr_getAppNumArgsAux(x_2, x_62); +x_63 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_62); x_64 = l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_processRec___closed__1; lean_inc(x_63); x_65 = lean_mk_array(x_63, x_64); @@ -1701,7 +1701,7 @@ if (lean_is_exclusive(x_15)) { x_101 = lean_box(0); } x_102 = lean_unsigned_to_nat(0u); -x_103 = l_Lean_Expr_getAppNumArgsAux(x_2, x_102); +x_103 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_102); x_104 = l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_processRec___closed__1; lean_inc(x_103); x_105 = lean_mk_array(x_103, x_104); @@ -4698,7 +4698,7 @@ if (x_14 == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_5, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_15); x_17 = l___private_Lean_Elab_PreDefinition_WF_Fix_0__Lean_Elab_WF_replaceRecApps_processRec___closed__1; lean_inc(x_16); x_18 = lean_mk_array(x_16, x_17); @@ -6084,7 +6084,7 @@ 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; uint8_t x_25; x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_3, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_18); x_20 = lean_unsigned_to_nat(3u); x_21 = lean_nat_sub(x_19, x_20); x_22 = lean_unsigned_to_nat(1u); @@ -7133,7 +7133,7 @@ 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; uint8_t x_25; x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_3, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_18); x_20 = lean_unsigned_to_nat(3u); x_21 = lean_nat_sub(x_19, x_20); x_22 = lean_unsigned_to_nat(1u); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Ite.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Ite.c index f1f095d7d4ef..14bc04ef7a4a 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Ite.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Ite.c @@ -31,6 +31,7 @@ lean_object* l_Lean_Expr_constLevels_x21(lean_object*); static lean_object* l_Lean_Meta_iteToDIte___lambda__1___closed__7; lean_object* l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); static lean_object* l_Lean_Meta_iteToDIte___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_iteToDIte___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -42,7 +43,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_iteToDIte___lambda__1___boxed(lean_object*, LEAN_EXPORT lean_object* l_Lean_Meta_iteToDIte(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_iteToDIte___lambda__1___closed__6; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_mkNot(lean_object*); static lean_object* l_Lean_Meta_iteToDIte___lambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Meta_iteToDIte___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -146,7 +146,7 @@ static lean_object* _init_l_Lean_Meta_iteToDIte___lambda__1___closed__11() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_iteToDIte___lambda__1___closed__8; x_2 = l_Lean_Meta_iteToDIte___lambda__1___closed__9; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_iteToDIte___lambda__1___closed__10; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -175,7 +175,7 @@ else lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; x_12 = l_Lean_Expr_getAppFn(x_1); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_Meta_iteToDIte___lambda__1___closed__3; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c index 981869b858d8..8e1aa2fa47d4 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Main.c @@ -105,6 +105,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_wfRecursion___spe lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_Elab_addNonRecPreDefs_mkSum___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_WF_registerEqnsInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_wfRecursion___spec__3___closed__2; lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Meta_CasesOnApp_addArg___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -143,7 +144,6 @@ static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinitio LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_Elab_addNonRecPreDefs___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_getFixedPrefix___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_Elab_addNonRecPreDefs(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_WF_elabWFRel___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_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_Elab_addNonRecPreDefs_mkSum___spec__1___closed__3; @@ -257,7 +257,7 @@ static lean_object* _init_l___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_El 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_PreDefinition_WF_Main_0__Lean_Elab_isOnlyOneUnaryDef___closed__1; x_2 = l___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_Elab_isOnlyOneUnaryDef___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_Elab_isOnlyOneUnaryDef___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -971,7 +971,7 @@ x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_16, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_16, x_18); x_20 = l___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_Elab_addNonRecPreDefs_mkSum___closed__1; lean_inc(x_19); x_21 = lean_mk_array(x_19, x_20); @@ -3507,7 +3507,7 @@ return x_26; else { lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; -x_27 = l_Lean_Expr_getAppNumArgsAux(x_5, x_12); +x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_12); x_28 = l___private_Lean_Elab_PreDefinition_WF_Main_0__Lean_Elab_addNonRecPreDefs_mkSum___closed__1; lean_inc(x_27); x_29 = lean_mk_array(x_27, x_28); @@ -4327,7 +4327,9 @@ if (x_12 == 0) { lean_object* x_13; lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); x_13 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_13, 0, x_4); @@ -4343,7 +4345,9 @@ x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_wfRecursion___spec__1___closed__1 x_16 = lean_array_push(x_15, x_14); x_17 = 1; lean_inc(x_10); -lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); lean_inc(x_5); x_18 = l_Lean_Elab_applyAttributesOf(x_16, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_16); @@ -4365,7 +4369,9 @@ else { uint8_t x_24; lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); x_24 = !lean_is_exclusive(x_18); if (x_24 == 0) @@ -5127,7 +5133,9 @@ x_28 = lean_usize_of_nat(x_27); lean_dec(x_27); x_29 = lean_box(0); lean_inc(x_12); -lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); x_30 = l_Array_forInUnsafe_loop___at_Lean_Elab_wfRecursion___spec__1(x_15, x_28, x_2, x_29, x_7, x_8, x_9, x_10, x_11, x_12, x_26); if (lean_obj_tag(x_30) == 0) @@ -5947,9 +5955,7 @@ lean_dec(x_2); x_13 = lean_unbox_usize(x_3); lean_dec(x_3); x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_wfRecursion___spec__1(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_9); lean_dec(x_1); return x_14; } diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/PackDomain.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/PackDomain.c index 8de12c8d4ab0..7a1014cd435f 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/PackDomain.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/PackDomain.c @@ -102,6 +102,7 @@ lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_PackDomain_0__Lean_Elab_WF_mkTupleElems___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_WF_packDomain___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_packDomain_isAppOfPreDef_x3f___lambda__1___boxed(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_packDomain___spec__4___lambda__2___closed__1; lean_object* l_Nat_repr(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -143,7 +144,6 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Elab_WF_packDomain_pac lean_object* l_Lean_Meta_Cases_cases(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_packDomain_packApplications_visit___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_packDomain_packApplications_visit___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_WF_packDomain___spec__4___closed__4; static lean_object* l_Lean_Elab_WF_packDomain_packApplications___closed__1; @@ -389,7 +389,7 @@ static lean_object* _init_l_Lean_Elab_WF_mkUnaryArg_go___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_WF_mkUnaryArg_go___closed__1; x_2 = l_Lean_Elab_WF_mkUnaryArg_go___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_WF_mkUnaryArg_go___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -13548,7 +13548,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_packDomain_packApplications_visitApp(lea { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_4, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_11); x_13 = l_Lean_Elab_WF_packDomain_packApplications_visitApp___closed__1; lean_inc(x_12); x_14 = lean_mk_array(x_12, x_13); @@ -13722,7 +13722,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_WF_packDomain_packApplications___lambda__1( lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_10 = l_Lean_Expr_getAppFn(x_3); x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_3, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_11); x_13 = l_Lean_Elab_WF_packDomain_packApplications_visitApp___closed__1; lean_inc(x_12); x_14 = lean_mk_array(x_12, x_13); @@ -15159,7 +15159,7 @@ lean_dec(x_7); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_2, x_10); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Lean_Expr_getAppNumArgsAux(x_6, x_12); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_6, x_12); x_14 = lean_nat_dec_lt(x_11, x_13); lean_dec(x_13); lean_dec(x_11); @@ -15610,7 +15610,7 @@ lean_ctor_set(x_55, 0, x_53); lean_ctor_set(x_55, 1, x_54); x_56 = lean_nat_dec_lt(x_48, x_3); lean_dec(x_3); -x_57 = l_Lean_Expr_getAppNumArgsAux(x_39, x_16); +x_57 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_39, x_16); lean_dec(x_39); x_58 = l_Nat_repr(x_57); x_59 = lean_alloc_ctor(2, 1, 0); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/PackMutual.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/PackMutual.c index 2647103dab7b..acabbcd0c67d 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/PackMutual.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/PackMutual.c @@ -107,6 +107,7 @@ lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_getCodomainsLevel___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_post_mkNewArg___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_post_mkNewArg___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_packValues_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_WF_withFixedPrefix___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_getCodomainsLevel___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -149,7 +150,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Le lean_object* l_Lean_Meta_Cases_cases(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_withFixedPrefix_go___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_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_WF_packMutual___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bindingName_x21(lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_getCodomainsLevel___spec__1___lambda__2___closed__6; @@ -947,7 +947,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDef lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_getCodomainsLevel___spec__1___closed__2; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_getCodomainsLevel___spec__1___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_getCodomainsLevel___spec__1___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1812,7 +1812,7 @@ else { lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; uint8_t x_52; uint8_t x_53; lean_object* x_54; x_35 = lean_unsigned_to_nat(0u); -x_36 = l_Lean_Expr_getAppNumArgsAux(x_28, x_35); +x_36 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_28, x_35); x_37 = l___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_mkNewCoDomain_go___closed__7; lean_inc(x_36); x_38 = lean_mk_array(x_36, x_37); @@ -3267,7 +3267,7 @@ x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_16, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_16, x_18); x_20 = l___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_mkNewCoDomain_go___closed__7; lean_inc(x_19); x_21 = lean_mk_array(x_19, x_20); @@ -3396,7 +3396,7 @@ lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean x_21 = lean_ctor_get(x_18, 0); lean_inc(x_21); lean_dec(x_18); -x_22 = l_Lean_Expr_getAppNumArgsAux(x_2, x_17); +x_22 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_17); x_23 = l___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Lean_Elab_WF_mkNewCoDomain_go___closed__7; lean_inc(x_22); x_24 = lean_mk_array(x_22, x_23); @@ -3517,7 +3517,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_PreDefinition_WF_PackMutual_0__Le { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_5, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_11); x_13 = lean_unsigned_to_nat(1u); x_14 = lean_nat_add(x_1, x_13); x_15 = lean_nat_dec_eq(x_12, x_14); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Rel.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Rel.c index f53ea919df52..2cb400fc2656 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/Rel.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/Rel.c @@ -352,7 +352,7 @@ static lean_object* _init_l___private_Lean_Elab_PreDefinition_WF_Rel_0__Lean_Ela 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_PreDefinition_WF_Rel_0__Lean_Elab_WF_getRefFromElems___lambda__1___closed__1; x_2 = l___private_Lean_Elab_PreDefinition_WF_Rel_0__Lean_Elab_WF_getRefFromElems___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_PreDefinition_WF_Rel_0__Lean_Elab_WF_getRefFromElems___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/PreDefinition/WF/TerminationHint.c b/stage0/stdlib/Lean/Elab/PreDefinition/WF/TerminationHint.c index ad8e34f9d8cd..6df323d50e76 100644 --- a/stage0/stdlib/Lean/Elab/PreDefinition/WF/TerminationHint.c +++ b/stage0/stdlib/Lean/Elab/PreDefinition/WF/TerminationHint.c @@ -4057,7 +4057,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreD lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_WF_TerminationHint_0__Lean_Elab_WF_expandTerminationByNonCore___spec__9___closed__3; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_WF_TerminationHint_0__Lean_Elab_WF_expandTerminationByNonCore___spec__9___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_PreDefinition_WF_TerminationHint_0__Lean_Elab_WF_expandTerminationByNonCore___spec__9___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/Print.c b/stage0/stdlib/Lean/Elab/Print.c index f6127e1a9c11..29e923e305ed 100644 --- a/stage0/stdlib/Lean/Elab/Print.c +++ b/stage0/stdlib/Lean/Elab/Print.c @@ -86,6 +86,7 @@ LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_ lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_levelParamsToMessageData___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrint___closed__5; +lean_object* l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__13(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___closed__7; @@ -112,7 +113,6 @@ lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printId___spec__2___closed__3; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintAxioms___closed__2; -lean_object* l_Lean_logAt___at_Lean_Elab_Command_withLogging___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_levelParamsToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabPrint(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); @@ -214,7 +214,6 @@ lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_mkHeader___closed__10; static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_levelParamsToMessageData___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrint_declRange___closed__6; -lean_object* l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printInduct___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrintAxioms___closed__3; LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printId___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); @@ -246,6 +245,7 @@ lean_object* l_Lean_Expr_getUsedConstants(lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printId___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Print_0__Lean_Elab_Command_printAxiomsOf___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Print_0__Lean_Elab_Command_printId___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabPrint___closed__6; @@ -1349,7 +1349,7 @@ x_18 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_18, 0, x_16); lean_ctor_set(x_18, 1, x_17); x_19 = 0; -x_20 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_18, x_19, x_7, x_8, x_12); +x_20 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_18, x_19, x_7, x_8, x_12); return x_20; } } @@ -1375,7 +1375,7 @@ x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); x_12 = 0; -x_13 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_10, x_12, x_6, x_7, x_11); +x_13 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_10, x_12, x_6, x_7, x_11); return x_13; } } @@ -1778,7 +1778,7 @@ x_27 = lean_ctor_get(x_25, 1); lean_inc(x_27); lean_dec(x_25); x_28 = 0; -x_29 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_26, x_28, x_7, x_8, x_27); +x_29 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_26, x_28, x_7, x_8, x_27); return x_29; } else @@ -3447,7 +3447,7 @@ lean_ctor_set(x_20, 0, x_19); x_21 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_21, 0, x_20); x_22 = 0; -x_23 = l_Lean_logAt___at_Lean_Elab_Command_withLogging___spec__2(x_10, x_21, x_22, x_2, x_3, x_4); +x_23 = l_Lean_logAt___at_Lean_Elab_Command_elabCommand___spec__4(x_10, x_21, x_22, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_10); @@ -4888,7 +4888,7 @@ x_25 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_24); x_26 = 0; -x_27 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_25, x_26, x_2, x_3, x_7); +x_27 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_25, x_26, x_2, x_3, x_7); return x_27; } else @@ -4906,7 +4906,7 @@ x_32 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_32, 0, x_30); lean_ctor_set(x_32, 1, x_31); x_33 = 0; -x_34 = l_Lean_log___at_Lean_Elab_Command_withLogging___spec__3(x_32, x_33, x_2, x_3, x_7); +x_34 = l_Lean_log___at_Lean_Elab_Command_elabCommand___spec__5(x_32, x_33, x_2, x_3, x_7); return x_34; } } diff --git a/stage0/stdlib/Lean/Elab/Quotation.c b/stage0/stdlib/Lean/Elab/Quotation.c index ab3347559d6f..dac6a661ede5 100644 --- a/stage0/stdlib/Lean/Elab/Quotation.c +++ b/stage0/stdlib/Lean/Elab/Quotation.c @@ -267,6 +267,7 @@ static lean_object* l_Lean_Elab_Term_Quotation___aux__Lean__Elab__Quotation_____ lean_object* lean_string_utf8_extract(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__26___closed__5; static lean_object* l_Lean_Elab_Term_Quotation_commandElab__stx__quot_____closed__1; +uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__14___closed__14; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Syntax_getAntiquotTerm(lean_object*); @@ -726,7 +727,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_ArrayStxBuilder_empty; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_quoteSyntax___spec__27___lambda__3___closed__16; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_floatOutAntiquotTerms___lambda__1___closed__14; LEAN_EXPORT lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___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*); -uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_Quotation_elabQuot____x40_Lean_Elab_Quotation___hyg_4823__declRange___closed__1; static lean_object* l___private_Init_Meta_0__Lean_quoteList___at_Lean_Elab_Term_Quotation_ArrayStxBuilder_build___spec__1___closed__6; static lean_object* l___private_Lean_Elab_Quotation_0__Lean_Elab_Term_Quotation_getHeadInfo___lambda__23___closed__16; @@ -2931,7 +2931,7 @@ static lean_object* _init_l_Lean_Elab_Term_Quotation_mkTuple___closed__13() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_Quotation_mkTuple___closed__10; x_2 = l_Lean_Elab_Term_Quotation_mkTuple___closed__11; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_Term_Quotation_mkTuple___closed__12; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -25345,7 +25345,7 @@ lean_object* x_12; lean_object* x_13; uint8_t x_14; x_12 = lean_array_get_size(x_3); x_13 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_13, 0, x_12); -x_14 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_8, x_13); +x_14 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_8, x_13); lean_dec(x_13); lean_dec(x_8); if (x_14 == 0) diff --git a/stage0/stdlib/Lean/Elab/Quotation/Util.c b/stage0/stdlib/Lean/Elab/Quotation/Util.c index d593c397244c..250eeea55aae 100644 --- a/stage0/stdlib/Lean/Elab/Quotation/Util.c +++ b/stage0/stdlib/Lean/Elab/Quotation/Util.c @@ -14,6 +14,7 @@ extern "C" { #endif uint8_t l_Lean_Syntax_isQuot(lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); uint8_t l_Lean_Syntax_isTokenAntiquot(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); @@ -38,7 +39,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_initFn____x40_Lean_Elab_Quot LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_getPatternsVars(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_Elab_Term_Quotation_getPatternVars___closed__6; -lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_Quotation_getPatternVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__2___closed__10; static lean_object* l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__2___closed__11; @@ -167,7 +167,7 @@ x_11 = lean_ctor_get(x_7, 5); x_12 = l_Lean_replaceRef(x_1, x_11); lean_dec(x_11); lean_ctor_set(x_7, 5, x_12); -x_13 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_13 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_7); return x_13; } @@ -211,7 +211,7 @@ lean_ctor_set(x_26, 7, x_21); lean_ctor_set(x_26, 8, x_22); lean_ctor_set(x_26, 9, x_23); lean_ctor_set(x_26, 10, x_24); -x_27 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_2, x_3, x_4, x_5, x_6, x_26, x_8, x_9); +x_27 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_2, x_3, x_4, x_5, x_6, x_26, x_8, x_9); lean_dec(x_26); return x_27; } @@ -578,7 +578,7 @@ static lean_object* _init_l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_El lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__2___closed__4; x_2 = l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__2___closed__5; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Syntax_instForInTopDownSyntax_loop___at_Lean_Elab_Term_Quotation_getAntiquotationIds___spec__2___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Elab/StructInst.c b/stage0/stdlib/Lean/Elab/StructInst.c index f8b5ebf9381b..7235fbdda10b 100644 --- a/stage0/stdlib/Lean/Elab/StructInst.c +++ b/stage0/stdlib/Lean/Elab/StructInst.c @@ -81,7 +81,6 @@ lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources___spec__2___rarg(lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__2; LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Elab_Term_StructInst_formatStruct___spec__1(lean_object*, lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__8; lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst___closed__3; @@ -134,6 +133,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructInstExp LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_mkDefaultValueAux_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__20; +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkCtorHeaderAux___closed__1; LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Elab_Term_StructInst_DefaultFields_step___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__2; @@ -376,6 +376,7 @@ LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_StructInst_0__Lean_Ela LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_getFieldName___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_DefaultFields_getHierarchyDepth(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNonAtomicExplicitSources___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_expandNumLitFields___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkSourcesWithSyntax___closed__1; @@ -505,7 +506,6 @@ lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_StructInst_Struct_structName___boxed(lean_object*); static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Term_StructInst_DefaultFields_propagateLoop___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_instInhabitedField___closed__1; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__4; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__2___closed__7; @@ -544,6 +544,7 @@ static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___c LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_elabStructInst___closed__2; static lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabModifyOp___lambda__3___closed__2; +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isModifyOp_x3f___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_StructInst_0__Lean_Elab_Term_StructInst_elabStruct(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstExpectedType___closed__2; @@ -558,7 +559,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_StructInst_expandStructIn lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_throwFailedToElabField___rarg___closed__2; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_StructInst_formatField___closed__1; static lean_object* l_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___lambda__1___closed__10; lean_object* l_List_find_x3f___rarg(lean_object*, lean_object*); @@ -706,6 +706,7 @@ extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; LEAN_EXPORT lean_object* l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_getStructName___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_findField_x3f(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_StructInst_expandStructInstFieldAbbrev___spec__2___closed__4; +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_isModifyOp_x3f___spec__3___closed__5; lean_object* l_ReaderT_instMonadReaderT___rarg(lean_object*); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_elabStructInstAux___spec__5___rarg___closed__2; @@ -3441,7 +3442,7 @@ static lean_object* _init_l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_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_StructInst_0__Lean_Elab_Term_StructInst_mkSourcesWithSyntax___closed__1; x_2 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkSourcesWithSyntax___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_StructInst_0__Lean_Elab_Term_StructInst_mkSourcesWithSyntax___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -17593,7 +17594,7 @@ lean_ctor_set(x_322, 0, x_320); lean_ctor_set(x_322, 1, x_321); lean_ctor_set(x_322, 2, x_319); x_323 = lean_unsigned_to_nat(0u); -x_324 = l_Lean_Expr_getAppNumArgsAux(x_251, x_323); +x_324 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_251, x_323); x_325 = lean_nat_sub(x_324, x_323); lean_dec(x_324); x_326 = lean_unsigned_to_nat(1u); @@ -17966,7 +17967,7 @@ lean_ctor_set(x_432, 0, x_430); lean_ctor_set(x_432, 1, x_431); lean_ctor_set(x_432, 2, x_429); x_433 = lean_unsigned_to_nat(0u); -x_434 = l_Lean_Expr_getAppNumArgsAux(x_251, x_433); +x_434 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_251, x_433); x_435 = lean_nat_sub(x_434, x_433); lean_dec(x_434); x_436 = lean_unsigned_to_nat(1u); @@ -21205,7 +21206,7 @@ if (x_35 == 0) { lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; size_t x_44; size_t x_45; lean_object* x_46; x_36 = lean_unsigned_to_nat(0u); -x_37 = l_Lean_Expr_getAppNumArgsAux(x_2, x_36); +x_37 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_36); x_38 = l_Lean_Elab_Term_StructInst_DefaultFields_reduce___closed__1; lean_inc(x_37); x_39 = lean_mk_array(x_37, x_38); @@ -21273,7 +21274,7 @@ else { lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; x_58 = lean_unsigned_to_nat(0u); -x_59 = l_Lean_Expr_getAppNumArgsAux(x_2, x_58); +x_59 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_58); x_60 = lean_mk_empty_array_with_capacity(x_59); lean_dec(x_59); x_61 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_2, x_60); @@ -21386,248 +21387,373 @@ return x_81; } case 10: { -lean_object* x_82; lean_object* x_83; -x_82 = lean_ctor_get(x_2, 1); +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_2, 0); lean_inc(x_82); -x_83 = l_Lean_Elab_Term_StructInst_DefaultFields_reduce(x_1, x_82, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_83) == 0) +x_83 = lean_ctor_get(x_2, 1); +lean_inc(x_83); +lean_inc(x_83); +x_84 = l_Lean_Elab_Term_StructInst_DefaultFields_reduce(x_1, x_83, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_84) == 0) { -uint8_t x_84; -x_84 = !lean_is_exclusive(x_83); -if (x_84 == 0) +uint8_t x_85; +x_85 = !lean_is_exclusive(x_84); +if (x_85 == 0) { -lean_object* x_85; lean_object* x_86; -x_85 = lean_ctor_get(x_83, 0); -x_86 = l_Lean_Elab_Term_StructInst_defaultMissing_x3f(x_2); -if (lean_obj_tag(x_86) == 0) +lean_object* x_86; lean_object* x_87; +x_86 = lean_ctor_get(x_84, 0); +x_87 = l_Lean_Elab_Term_StructInst_defaultMissing_x3f(x_2); +if (lean_obj_tag(x_87) == 0) { -lean_object* x_87; -x_87 = lean_expr_update_mdata(x_2, x_85); -lean_ctor_set(x_83, 0, x_87); -return x_83; +size_t x_88; size_t x_89; uint8_t x_90; +x_88 = lean_ptr_addr(x_83); +lean_dec(x_83); +x_89 = lean_ptr_addr(x_86); +x_90 = lean_usize_dec_eq(x_88, x_89); +if (x_90 == 0) +{ +lean_object* x_91; +lean_dec(x_2); +x_91 = l_Lean_Expr_mdata___override(x_82, x_86); +lean_ctor_set(x_84, 0, x_91); +return x_84; } else { -uint8_t x_88; lean_dec(x_86); -x_88 = l_Lean_Expr_isMVar(x_85); -if (x_88 == 0) +lean_dec(x_82); +lean_ctor_set(x_84, 0, x_2); +return x_84; +} +} +else { +uint8_t x_92; +lean_dec(x_87); +x_92 = l_Lean_Expr_isMVar(x_86); +if (x_92 == 0) +{ +lean_dec(x_83); +lean_dec(x_82); lean_dec(x_2); -return x_83; +return x_84; } else { -lean_object* x_89; -x_89 = lean_expr_update_mdata(x_2, x_85); -lean_ctor_set(x_83, 0, x_89); -return x_83; +size_t x_93; size_t x_94; uint8_t x_95; +x_93 = lean_ptr_addr(x_83); +lean_dec(x_83); +x_94 = lean_ptr_addr(x_86); +x_95 = lean_usize_dec_eq(x_93, x_94); +if (x_95 == 0) +{ +lean_object* x_96; +lean_dec(x_2); +x_96 = l_Lean_Expr_mdata___override(x_82, x_86); +lean_ctor_set(x_84, 0, x_96); +return x_84; +} +else +{ +lean_dec(x_86); +lean_dec(x_82); +lean_ctor_set(x_84, 0, x_2); +return x_84; +} } } } else { -lean_object* x_90; lean_object* x_91; lean_object* x_92; -x_90 = lean_ctor_get(x_83, 0); -x_91 = lean_ctor_get(x_83, 1); -lean_inc(x_91); -lean_inc(x_90); +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_84, 0); +x_98 = lean_ctor_get(x_84, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_84); +x_99 = l_Lean_Elab_Term_StructInst_defaultMissing_x3f(x_2); +if (lean_obj_tag(x_99) == 0) +{ +size_t x_100; size_t x_101; uint8_t x_102; +x_100 = lean_ptr_addr(x_83); lean_dec(x_83); -x_92 = l_Lean_Elab_Term_StructInst_defaultMissing_x3f(x_2); -if (lean_obj_tag(x_92) == 0) +x_101 = lean_ptr_addr(x_97); +x_102 = lean_usize_dec_eq(x_100, x_101); +if (x_102 == 0) { -lean_object* x_93; lean_object* x_94; -x_93 = lean_expr_update_mdata(x_2, x_90); -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_91); -return x_94; +lean_object* x_103; lean_object* x_104; +lean_dec(x_2); +x_103 = l_Lean_Expr_mdata___override(x_82, x_97); +x_104 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_98); +return x_104; } else { -uint8_t x_95; -lean_dec(x_92); -x_95 = l_Lean_Expr_isMVar(x_90); -if (x_95 == 0) +lean_object* x_105; +lean_dec(x_97); +lean_dec(x_82); +x_105 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_2); +lean_ctor_set(x_105, 1, x_98); +return x_105; +} +} +else { -lean_object* x_96; +uint8_t x_106; +lean_dec(x_99); +x_106 = l_Lean_Expr_isMVar(x_97); +if (x_106 == 0) +{ +lean_object* x_107; +lean_dec(x_83); +lean_dec(x_82); lean_dec(x_2); -x_96 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_96, 0, x_90); -lean_ctor_set(x_96, 1, x_91); -return x_96; +x_107 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_107, 0, x_97); +lean_ctor_set(x_107, 1, x_98); +return x_107; } else { -lean_object* x_97; lean_object* x_98; -x_97 = lean_expr_update_mdata(x_2, x_90); -x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_97); -lean_ctor_set(x_98, 1, x_91); -return x_98; +size_t x_108; size_t x_109; uint8_t x_110; +x_108 = lean_ptr_addr(x_83); +lean_dec(x_83); +x_109 = lean_ptr_addr(x_97); +x_110 = lean_usize_dec_eq(x_108, x_109); +if (x_110 == 0) +{ +lean_object* x_111; lean_object* x_112; +lean_dec(x_2); +x_111 = l_Lean_Expr_mdata___override(x_82, x_97); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_98); +return x_112; +} +else +{ +lean_object* x_113; +lean_dec(x_97); +lean_dec(x_82); +x_113 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_113, 0, x_2); +lean_ctor_set(x_113, 1, x_98); +return x_113; +} } } } } else { -uint8_t x_99; +uint8_t x_114; +lean_dec(x_83); +lean_dec(x_82); lean_dec(x_2); -x_99 = !lean_is_exclusive(x_83); -if (x_99 == 0) +x_114 = !lean_is_exclusive(x_84); +if (x_114 == 0) { -return x_83; +return x_84; } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_100 = lean_ctor_get(x_83, 0); -x_101 = lean_ctor_get(x_83, 1); -lean_inc(x_101); -lean_inc(x_100); -lean_dec(x_83); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_100); -lean_ctor_set(x_102, 1, x_101); -return x_102; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_84, 0); +x_116 = lean_ctor_get(x_84, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_84); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } case 11: { -lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_103 = lean_ctor_get(x_2, 1); -lean_inc(x_103); -x_104 = lean_ctor_get(x_2, 2); -lean_inc(x_104); +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_118 = lean_ctor_get(x_2, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_2, 1); +lean_inc(x_119); +x_120 = lean_ctor_get(x_2, 2); +lean_inc(x_120); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_104); -x_105 = l_Lean_Meta_project_x3f(x_104, x_103, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_103); -if (lean_obj_tag(x_105) == 0) +lean_inc(x_120); +x_121 = l_Lean_Meta_project_x3f(x_120, x_119, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_121) == 0) { -lean_object* x_106; -x_106 = lean_ctor_get(x_105, 0); -lean_inc(x_106); -if (lean_obj_tag(x_106) == 0) +lean_object* x_122; +x_122 = lean_ctor_get(x_121, 0); +lean_inc(x_122); +if (lean_obj_tag(x_122) == 0) { -lean_object* x_107; lean_object* x_108; -x_107 = lean_ctor_get(x_105, 1); -lean_inc(x_107); -lean_dec(x_105); -x_108 = l_Lean_Elab_Term_StructInst_DefaultFields_reduce(x_1, x_104, x_3, x_4, x_5, x_6, x_107); -if (lean_obj_tag(x_108) == 0) +lean_object* x_123; lean_object* x_124; +x_123 = lean_ctor_get(x_121, 1); +lean_inc(x_123); +lean_dec(x_121); +lean_inc(x_120); +x_124 = l_Lean_Elab_Term_StructInst_DefaultFields_reduce(x_1, x_120, x_3, x_4, x_5, x_6, x_123); +if (lean_obj_tag(x_124) == 0) +{ +uint8_t x_125; +x_125 = !lean_is_exclusive(x_124); +if (x_125 == 0) +{ +lean_object* x_126; size_t x_127; size_t x_128; uint8_t x_129; +x_126 = lean_ctor_get(x_124, 0); +x_127 = lean_ptr_addr(x_120); +lean_dec(x_120); +x_128 = lean_ptr_addr(x_126); +x_129 = lean_usize_dec_eq(x_127, x_128); +if (x_129 == 0) +{ +lean_object* x_130; +lean_dec(x_2); +x_130 = l_Lean_Expr_proj___override(x_118, x_119, x_126); +lean_ctor_set(x_124, 0, x_130); +return x_124; +} +else { -uint8_t x_109; -x_109 = !lean_is_exclusive(x_108); -if (x_109 == 0) +lean_dec(x_126); +lean_dec(x_119); +lean_dec(x_118); +lean_ctor_set(x_124, 0, x_2); +return x_124; +} +} +else { -lean_object* x_110; lean_object* x_111; -x_110 = lean_ctor_get(x_108, 0); -x_111 = lean_expr_update_proj(x_2, x_110); -lean_ctor_set(x_108, 0, x_111); -return x_108; +lean_object* x_131; lean_object* x_132; size_t x_133; size_t x_134; uint8_t x_135; +x_131 = lean_ctor_get(x_124, 0); +x_132 = lean_ctor_get(x_124, 1); +lean_inc(x_132); +lean_inc(x_131); +lean_dec(x_124); +x_133 = lean_ptr_addr(x_120); +lean_dec(x_120); +x_134 = lean_ptr_addr(x_131); +x_135 = lean_usize_dec_eq(x_133, x_134); +if (x_135 == 0) +{ +lean_object* x_136; lean_object* x_137; +lean_dec(x_2); +x_136 = l_Lean_Expr_proj___override(x_118, x_119, x_131); +x_137 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set(x_137, 1, x_132); +return x_137; } else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_112 = lean_ctor_get(x_108, 0); -x_113 = lean_ctor_get(x_108, 1); -lean_inc(x_113); -lean_inc(x_112); -lean_dec(x_108); -x_114 = lean_expr_update_proj(x_2, x_112); -x_115 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_115, 0, x_114); -lean_ctor_set(x_115, 1, x_113); -return x_115; +lean_object* x_138; +lean_dec(x_131); +lean_dec(x_119); +lean_dec(x_118); +x_138 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_138, 0, x_2); +lean_ctor_set(x_138, 1, x_132); +return x_138; +} } } else { -uint8_t x_116; +uint8_t x_139; +lean_dec(x_120); +lean_dec(x_119); +lean_dec(x_118); lean_dec(x_2); -x_116 = !lean_is_exclusive(x_108); -if (x_116 == 0) +x_139 = !lean_is_exclusive(x_124); +if (x_139 == 0) { -return x_108; +return x_124; } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_117 = lean_ctor_get(x_108, 0); -x_118 = lean_ctor_get(x_108, 1); -lean_inc(x_118); -lean_inc(x_117); -lean_dec(x_108); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_117); -lean_ctor_set(x_119, 1, x_118); -return x_119; +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_124, 0); +x_141 = lean_ctor_get(x_124, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_124); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } } else { -lean_object* x_120; lean_object* x_121; -lean_dec(x_104); +lean_object* x_143; lean_object* x_144; +lean_dec(x_120); +lean_dec(x_119); +lean_dec(x_118); lean_dec(x_2); -x_120 = lean_ctor_get(x_105, 1); -lean_inc(x_120); -lean_dec(x_105); -x_121 = lean_ctor_get(x_106, 0); -lean_inc(x_121); -lean_dec(x_106); -x_2 = x_121; -x_7 = x_120; +x_143 = lean_ctor_get(x_121, 1); +lean_inc(x_143); +lean_dec(x_121); +x_144 = lean_ctor_get(x_122, 0); +lean_inc(x_144); +lean_dec(x_122); +x_2 = x_144; +x_7 = x_143; goto _start; } } else { -uint8_t x_123; -lean_dec(x_104); +uint8_t x_146; +lean_dec(x_120); +lean_dec(x_119); +lean_dec(x_118); 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_123 = !lean_is_exclusive(x_105); -if (x_123 == 0) +x_146 = !lean_is_exclusive(x_121); +if (x_146 == 0) { -return x_105; +return x_121; } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_124 = lean_ctor_get(x_105, 0); -x_125 = lean_ctor_get(x_105, 1); -lean_inc(x_125); -lean_inc(x_124); -lean_dec(x_105); -x_126 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_126, 0, x_124); -lean_ctor_set(x_126, 1, x_125); -return x_126; +lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_147 = lean_ctor_get(x_121, 0); +x_148 = lean_ctor_get(x_121, 1); +lean_inc(x_148); +lean_inc(x_147); +lean_dec(x_121); +x_149 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_149, 0, x_147); +lean_ctor_set(x_149, 1, x_148); +return x_149; } } } default: { -lean_object* x_127; +lean_object* x_150; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_127 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_127, 0, x_2); -lean_ctor_set(x_127, 1, x_7); -return x_127; +x_150 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_150, 0, x_2); +lean_ctor_set(x_150, 1, x_7); +return x_150; } } } diff --git a/stage0/stdlib/Lean/Elab/Structure.c b/stage0/stdlib/Lean/Elab/Structure.c index ceae4abd4b4b..69dd343de392 100644 --- a/stage0/stdlib/Lean/Elab/Structure.c +++ b/stage0/stdlib/Lean/Elab/Structure.c @@ -22,6 +22,7 @@ LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Structure_ static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addCtorFields___closed__3; static lean_object* l_Lean_Elab_Command_elabStructure___closed__11; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; +lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); 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___private_Lean_Elab_Structure_0__Lean_Elab_Command_findExistingField_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(lean_object*, lean_object*); @@ -54,7 +55,7 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_ lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_FunBinders_elabFunBinderViews___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_checkResultingUniverse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -305,7 +306,6 @@ lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_T lean_object* l_Lean_LocalContext_setBinderInfo(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___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_checkValidFieldModifier___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__3___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_withParents_go___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -390,7 +390,6 @@ static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__5___closed__2; static lean_object* l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkCoercionToCopiedParent_copyFields___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Term_elabTerm(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___spec__1___rarg(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__1___closed__2; static lean_object* l_Lean_Elab_getOptDerivingClasses___at_Lean_Elab_Command_elabStructure___spec__2___closed__4; @@ -445,6 +444,7 @@ static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure lean_object* l_Lean_Meta_mkId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___closed__6; static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_addDefaults___spec__2___closed__1; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_processSubfields_go___rarg___closed__1; lean_object* l_Std_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_elabBinderViews_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -573,6 +573,7 @@ lean_object* l_Lean_addDocString_x27___at_Lean_Elab_Term_expandDeclId___spec__9( static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withFields_go___rarg___closed__9; uint8_t l_Lean_Expr_isForall(lean_object*); uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); +lean_object* l_Lean_Elab_Term_elabTermEnsuringType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_whnf(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_reprStructFieldKind____x40_Lean_Elab_Structure___hyg_327____boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabStructureView___lambda__4___closed__6; @@ -660,7 +661,6 @@ lean_object* l_Lean_Syntax_getSepArgs(lean_object*); uint8_t l_Lean_isAttribute(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabStructure___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_collectLevelParamsInFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); 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*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_toVisibility___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabStructure___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -721,6 +721,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Struc 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___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_522____closed__11; static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___closed__6; +lean_object* l_Lean_Elab_Term_elabTerm___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_mkAuxConstructions___lambda__1(uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabStructure___closed__1; LEAN_EXPORT uint8_t l_Lean_Elab_Command_instDecidableEqStructFieldKind(uint8_t, uint8_t); @@ -759,6 +760,7 @@ lean_object* l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(lean_obj lean_object* l_Array_ofSubarray___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_withUsed___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandFields___spec__5___lambda__3___closed__5; +lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getOptDerivingClasses___at_Lean_Elab_Command_elabStructure___spec__2___closed__2; lean_object* l_Lean_Meta_getLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getStructureCtor(lean_object*, lean_object*); @@ -818,7 +820,7 @@ static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_Structure LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_elabFieldTypeValue___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyDefaultValue_x3f_go_x3f___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Structure_0__Lean_Elab_Command_copyNewFieldsFrom_copyFields_copy___rarg___lambda__5___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_12385_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_12391_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_3275_(lean_object*); uint8_t l_Lean_TagDeclarationExtension_isTagged(lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); @@ -1905,7 +1907,7 @@ lean_ctor_set(x_23, 0, x_22); lean_ctor_set(x_23, 1, x_14); x_24 = lean_ctor_get(x_1, 2); lean_inc(x_24); -x_25 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_24, x_4); +x_25 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_24, x_4); x_26 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_26, 0, x_23); lean_ctor_set(x_26, 1, x_25); @@ -1975,7 +1977,7 @@ x_51 = lean_ctor_get(x_40, 0); lean_inc(x_51); lean_dec(x_40); x_52 = lean_unsigned_to_nat(1024u); -x_53 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_51, x_52); +x_53 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_51, x_52); x_54 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_reprStructFieldInfo____x40_Lean_Elab_Structure___hyg_522____closed__26; x_55 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_55, 0, x_54); @@ -3220,34 +3222,96 @@ return x_13; } else { -lean_object* x_14; lean_object* x_15; +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; x_14 = lean_array_uget(x_1, x_3); +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_9, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_9, 2); +lean_inc(x_17); +x_18 = lean_ctor_get(x_9, 3); +lean_inc(x_18); +x_19 = lean_ctor_get(x_9, 4); +lean_inc(x_19); +x_20 = lean_ctor_get(x_9, 5); +lean_inc(x_20); +x_21 = lean_ctor_get(x_9, 6); +lean_inc(x_21); +x_22 = lean_ctor_get(x_9, 7); +lean_inc(x_22); +x_23 = lean_ctor_get(x_9, 8); +lean_inc(x_23); +x_24 = lean_ctor_get(x_9, 9); +lean_inc(x_24); +x_25 = lean_ctor_get(x_9, 10); +lean_inc(x_25); +x_26 = l_Lean_replaceRef(x_14, x_20); +lean_dec(x_20); +x_27 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_27, 0, x_15); +lean_ctor_set(x_27, 1, x_16); +lean_ctor_set(x_27, 2, x_17); +lean_ctor_set(x_27, 3, x_18); +lean_ctor_set(x_27, 4, x_19); +lean_ctor_set(x_27, 5, x_26); +lean_ctor_set(x_27, 6, x_21); +lean_ctor_set(x_27, 7, x_22); +lean_ctor_set(x_27, 8, x_23); +lean_ctor_set(x_27, 9, x_24); +lean_ctor_set(x_27, 10, x_25); +lean_inc(x_10); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_28 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4(x_14, x_5, x_6, x_7, x_8, x_27, x_10, x_11); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; size_t x_32; size_t x_33; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_array_push(x_4, x_29); +x_32 = 1; +x_33 = lean_usize_add(x_3, x_32); +x_3 = x_33; +x_4 = x_31; +x_11 = x_30; +goto _start; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_28, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_28, 1); +lean_inc(x_36); +lean_dec(x_28); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_15 = l_Lean_Elab_elabAttr___at___private_Lean_Elab_Structure_0__Lean_Elab_Command_expandCtor___spec__4(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_15) == 0) +x_37 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_36); +if (lean_obj_tag(x_37) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_array_push(x_4, x_16); -x_19 = 1; -x_20 = lean_usize_add(x_3, x_19); -x_3 = x_20; -x_4 = x_18; -x_11 = x_17; +lean_object* x_38; size_t x_39; size_t x_40; +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = 1; +x_40 = lean_usize_add(x_3, x_39); +x_3 = x_40; +x_11 = x_38; goto _start; } else { -uint8_t x_22; +uint8_t x_42; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3255,23 +3319,24 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_22 = !lean_is_exclusive(x_15); -if (x_22 == 0) +x_42 = !lean_is_exclusive(x_37); +if (x_42 == 0) { -return x_15; +return x_37; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_15, 0); -x_24 = lean_ctor_get(x_15, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_15); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_37, 0); +x_44 = lean_ctor_get(x_37, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_37); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} } } } @@ -9324,7 +9389,7 @@ x_19 = lean_ctor_get(x_15, 1); lean_inc(x_19); lean_dec(x_15); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_1, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_20); x_22 = lean_unsigned_to_nat(1u); x_23 = lean_nat_add(x_19, x_22); lean_dec(x_19); @@ -9373,7 +9438,7 @@ x_32 = lean_ctor_get(x_15, 1); lean_inc(x_32); lean_dec(x_15); x_33 = lean_unsigned_to_nat(0u); -x_34 = l_Lean_Expr_getAppNumArgsAux(x_1, x_33); +x_34 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_33); x_35 = lean_unsigned_to_nat(1u); x_36 = lean_nat_add(x_32, x_35); lean_dec(x_32); @@ -9543,7 +9608,7 @@ x_19 = lean_ctor_get(x_10, 1); lean_inc(x_19); lean_dec(x_10); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_3, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_20); x_22 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; lean_inc(x_21); x_23 = lean_mk_array(x_21, x_22); @@ -11493,7 +11558,7 @@ x_21 = l_Lean_Elab_elabModifiers___at___private_Lean_Elab_Structure_0__Lean_Elab x_22 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_22, 0, x_20); lean_ctor_set(x_22, 1, x_21); -x_23 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_23 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_13); x_24 = !lean_is_exclusive(x_23); if (x_24 == 0) { @@ -11599,7 +11664,7 @@ lean_inc(x_19); lean_dec(x_18); x_20 = l_Lean_Expr_const___override(x_19, x_16); x_21 = lean_unsigned_to_nat(0u); -x_22 = l_Lean_Expr_getAppNumArgsAux(x_1, x_21); +x_22 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_21); x_23 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; lean_inc(x_22); x_24 = lean_mk_array(x_22, x_23); @@ -13695,7 +13760,7 @@ lean_inc(x_3); x_19 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_18); if (lean_obj_tag(x_19) == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); x_21 = lean_ctor_get(x_19, 1); @@ -13703,114 +13768,121 @@ lean_inc(x_21); lean_dec(x_19); x_22 = lean_box(0); x_23 = 1; +x_24 = lean_box(x_23); +x_25 = lean_box(x_23); +x_26 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_26, 0, x_15); +lean_closure_set(x_26, 1, x_22); +lean_closure_set(x_26, 2, x_24); +lean_closure_set(x_26, 3, x_25); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_24 = l_Lean_Elab_Term_elabTerm(x_15, x_22, x_23, x_23, x_3, x_4, x_5, x_6, x_7, x_8, x_21); -if (lean_obj_tag(x_24) == 0) +x_27 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_21); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = 1; -x_28 = l_Lean_Meta_mkLambdaFVars(x_20, x_25, x_16, x_23, x_27, x_5, x_6, x_7, x_8, x_26); +lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = 1; +x_31 = l_Lean_Meta_mkLambdaFVars(x_20, x_28, x_16, x_23, x_30, x_5, x_6, x_7, x_8, x_29); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_28) == 0) -{ -uint8_t x_29; -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +if (lean_obj_tag(x_31) == 0) { -lean_object* x_30; lean_object* x_31; -x_30 = lean_ctor_get(x_28, 0); -lean_ctor_set(x_11, 0, x_30); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_22); -lean_ctor_set(x_31, 1, x_11); -lean_ctor_set(x_28, 0, x_31); -return x_28; -} -else +uint8_t x_32; +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_32 = lean_ctor_get(x_28, 0); -x_33 = lean_ctor_get(x_28, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_28); -lean_ctor_set(x_11, 0, x_32); +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_31, 0); +lean_ctor_set(x_11, 0, x_33); x_34 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_34, 0, x_22); lean_ctor_set(x_34, 1, x_11); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_33); -return x_35; +lean_ctor_set(x_31, 0, x_34); +return x_31; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_31, 0); +x_36 = lean_ctor_get(x_31, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_31); +lean_ctor_set(x_11, 0, x_35); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_22); +lean_ctor_set(x_37, 1, x_11); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +return x_38; } } else { -uint8_t x_36; +uint8_t x_39; lean_free_object(x_11); -x_36 = !lean_is_exclusive(x_28); -if (x_36 == 0) +x_39 = !lean_is_exclusive(x_31); +if (x_39 == 0) { -return x_28; +return x_31; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_28, 0); -x_38 = lean_ctor_get(x_28, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_28); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_31, 0); +x_41 = lean_ctor_get(x_31, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_31); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; } } } else { -uint8_t x_40; +uint8_t x_43; lean_dec(x_20); lean_free_object(x_11); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_40 = !lean_is_exclusive(x_24); -if (x_40 == 0) +x_43 = !lean_is_exclusive(x_27); +if (x_43 == 0) { -return x_24; +return x_27; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_24, 0); -x_42 = lean_ctor_get(x_24, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_24); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_27, 0); +x_45 = lean_ctor_get(x_27, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_27); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } } } else { -uint8_t x_44; +uint8_t x_47; lean_free_object(x_11); lean_dec(x_15); lean_dec(x_8); @@ -13819,29 +13891,29 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_44 = !lean_is_exclusive(x_19); -if (x_44 == 0) +x_47 = !lean_is_exclusive(x_19); +if (x_47 == 0) { return x_19; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_19, 0); -x_46 = lean_ctor_get(x_19, 1); -lean_inc(x_46); -lean_inc(x_45); +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_19, 0); +x_49 = lean_ctor_get(x_19, 1); +lean_inc(x_49); +lean_inc(x_48); lean_dec(x_19); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; } } } else { -uint8_t x_48; +uint8_t x_51; lean_free_object(x_11); lean_dec(x_15); lean_dec(x_8); @@ -13851,201 +13923,208 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_48 = !lean_is_exclusive(x_17); -if (x_48 == 0) +x_51 = !lean_is_exclusive(x_17); +if (x_51 == 0) { return x_17; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_17, 0); -x_50 = lean_ctor_get(x_17, 1); -lean_inc(x_50); -lean_inc(x_49); +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_17, 0); +x_53 = lean_ctor_get(x_17, 1); +lean_inc(x_53); +lean_inc(x_52); lean_dec(x_17); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; } } } else { -lean_object* x_52; uint8_t x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_11, 0); -lean_inc(x_52); +lean_object* x_55; uint8_t x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_11, 0); +lean_inc(x_55); lean_dec(x_11); -x_53 = 0; +x_56 = 0; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_54 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_53, x_53, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_54) == 0) +x_57 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_56, x_56, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_57) == 0) { -lean_object* x_55; lean_object* x_56; -x_55 = lean_ctor_get(x_54, 1); -lean_inc(x_55); -lean_dec(x_54); +lean_object* x_58; lean_object* x_59; +x_58 = lean_ctor_get(x_57, 1); +lean_inc(x_58); +lean_dec(x_57); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_3); -x_56 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_55); -if (lean_obj_tag(x_56) == 0) +x_59 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_58); +if (lean_obj_tag(x_59) == 0) { -lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = lean_box(0); -x_60 = 1; +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = lean_box(0); +x_63 = 1; +x_64 = lean_box(x_63); +x_65 = lean_box(x_63); +x_66 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_66, 0, x_55); +lean_closure_set(x_66, 1, x_62); +lean_closure_set(x_66, 2, x_64); +lean_closure_set(x_66, 3, x_65); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_61 = l_Lean_Elab_Term_elabTerm(x_52, x_59, x_60, x_60, x_3, x_4, x_5, x_6, x_7, x_8, x_58); -if (lean_obj_tag(x_61) == 0) +x_67 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_66, x_3, x_4, x_5, x_6, x_7, x_8, x_61); +if (lean_obj_tag(x_67) == 0) { -lean_object* x_62; lean_object* x_63; uint8_t x_64; lean_object* x_65; -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 = 1; -x_65 = l_Lean_Meta_mkLambdaFVars(x_57, x_62, x_53, x_60, x_64, x_5, x_6, x_7, x_8, x_63); +lean_object* x_68; lean_object* x_69; uint8_t x_70; lean_object* x_71; +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); +x_70 = 1; +x_71 = l_Lean_Meta_mkLambdaFVars(x_60, x_68, x_56, x_63, x_70, x_5, x_6, x_7, x_8, x_69); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_65) == 0) +if (lean_obj_tag(x_71) == 0) { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -if (lean_is_exclusive(x_65)) { - lean_ctor_release(x_65, 0); - lean_ctor_release(x_65, 1); - x_68 = x_65; +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_74 = x_71; } else { - lean_dec_ref(x_65); - x_68 = lean_box(0); + lean_dec_ref(x_71); + x_74 = lean_box(0); } -x_69 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_69, 0, x_66); -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_59); -lean_ctor_set(x_70, 1, x_69); -if (lean_is_scalar(x_68)) { - x_71 = lean_alloc_ctor(0, 2, 0); +x_75 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_75, 0, x_72); +x_76 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_76, 0, x_62); +lean_ctor_set(x_76, 1, x_75); +if (lean_is_scalar(x_74)) { + x_77 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_68; + x_77 = x_74; } -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_67); -return x_71; +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_73); +return x_77; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_72 = lean_ctor_get(x_65, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_65, 1); -lean_inc(x_73); -if (lean_is_exclusive(x_65)) { - lean_ctor_release(x_65, 0); - lean_ctor_release(x_65, 1); - x_74 = x_65; +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_78 = lean_ctor_get(x_71, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_71, 1); +lean_inc(x_79); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_80 = x_71; } else { - lean_dec_ref(x_65); - x_74 = lean_box(0); + lean_dec_ref(x_71); + x_80 = lean_box(0); } -if (lean_is_scalar(x_74)) { - x_75 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_80)) { + x_81 = lean_alloc_ctor(1, 2, 0); } else { - x_75 = x_74; + x_81 = x_80; } -lean_ctor_set(x_75, 0, x_72); -lean_ctor_set(x_75, 1, x_73); -return x_75; +lean_ctor_set(x_81, 0, x_78); +lean_ctor_set(x_81, 1, x_79); +return x_81; } } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -lean_dec(x_57); +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +lean_dec(x_60); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_76 = lean_ctor_get(x_61, 0); -lean_inc(x_76); -x_77 = lean_ctor_get(x_61, 1); -lean_inc(x_77); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_78 = x_61; +x_82 = lean_ctor_get(x_67, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_67, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_67)) { + lean_ctor_release(x_67, 0); + lean_ctor_release(x_67, 1); + x_84 = x_67; } else { - lean_dec_ref(x_61); - x_78 = lean_box(0); + lean_dec_ref(x_67); + x_84 = lean_box(0); } -if (lean_is_scalar(x_78)) { - x_79 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_84)) { + x_85 = lean_alloc_ctor(1, 2, 0); } else { - x_79 = x_78; + x_85 = x_84; } -lean_ctor_set(x_79, 0, x_76); -lean_ctor_set(x_79, 1, x_77); -return x_79; +lean_ctor_set(x_85, 0, x_82); +lean_ctor_set(x_85, 1, x_83); +return x_85; } } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -lean_dec(x_52); +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_dec(x_55); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_80 = lean_ctor_get(x_56, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_56, 1); -lean_inc(x_81); -if (lean_is_exclusive(x_56)) { - lean_ctor_release(x_56, 0); - lean_ctor_release(x_56, 1); - x_82 = x_56; +x_86 = lean_ctor_get(x_59, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_59, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_88 = x_59; } else { - lean_dec_ref(x_56); - x_82 = lean_box(0); + lean_dec_ref(x_59); + x_88 = lean_box(0); } -if (lean_is_scalar(x_82)) { - x_83 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_88)) { + x_89 = lean_alloc_ctor(1, 2, 0); } else { - x_83 = x_82; + x_89 = x_88; } -lean_ctor_set(x_83, 0, x_80); -lean_ctor_set(x_83, 1, x_81); -return x_83; +lean_ctor_set(x_89, 0, x_86); +lean_ctor_set(x_89, 1, x_87); +return x_89; } } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -lean_dec(x_52); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_dec(x_55); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -14053,342 +14132,350 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_84 = lean_ctor_get(x_54, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_54, 1); -lean_inc(x_85); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_86 = x_54; +x_90 = lean_ctor_get(x_57, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_57, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_92 = x_57; } else { - lean_dec_ref(x_54); - x_86 = lean_box(0); + lean_dec_ref(x_57); + x_92 = lean_box(0); } -if (lean_is_scalar(x_86)) { - x_87 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_92)) { + x_93 = lean_alloc_ctor(1, 2, 0); } else { - x_87 = x_86; + x_93 = x_92; } -lean_ctor_set(x_87, 0, x_84); -lean_ctor_set(x_87, 1, x_85); -return x_87; +lean_ctor_set(x_93, 0, x_90); +lean_ctor_set(x_93, 1, x_91); +return x_93; } } } } else { -uint8_t x_88; -x_88 = !lean_is_exclusive(x_10); -if (x_88 == 0) +uint8_t x_94; +x_94 = !lean_is_exclusive(x_10); +if (x_94 == 0) { -lean_object* x_89; lean_object* x_90; -x_89 = lean_ctor_get(x_10, 0); +lean_object* x_95; lean_object* x_96; +x_95 = lean_ctor_get(x_10, 0); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_90 = l_Lean_Elab_Term_elabType(x_89, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_90) == 0) +x_96 = l_Lean_Elab_Term_elabType(x_95, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_96) == 0) { -lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; -x_91 = lean_ctor_get(x_90, 0); -lean_inc(x_91); -x_92 = lean_ctor_get(x_90, 1); -lean_inc(x_92); -lean_dec(x_90); -x_93 = 0; +lean_object* x_97; lean_object* x_98; uint8_t x_99; lean_object* x_100; +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +lean_dec(x_96); +x_99 = 0; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_94 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_93, x_93, x_3, x_4, x_5, x_6, x_7, x_8, x_92); -if (lean_obj_tag(x_94) == 0) +x_100 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_99, x_99, x_3, x_4, x_5, x_6, x_7, x_8, x_98); +if (lean_obj_tag(x_100) == 0) { -lean_object* x_95; lean_object* x_96; -x_95 = lean_ctor_get(x_94, 1); -lean_inc(x_95); -lean_dec(x_94); +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +lean_dec(x_100); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_3); -x_96 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_95); -if (lean_obj_tag(x_96) == 0) +x_102 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_101); +if (lean_obj_tag(x_102) == 0) { -lean_object* x_97; -x_97 = lean_ctor_get(x_1, 7); -lean_inc(x_97); +lean_object* x_103; +x_103 = lean_ctor_get(x_1, 7); +lean_inc(x_103); lean_dec(x_1); -if (lean_obj_tag(x_97) == 0) +if (lean_obj_tag(x_103) == 0) { -lean_object* x_98; lean_object* x_99; uint8_t x_100; uint8_t x_101; lean_object* x_102; +lean_object* x_104; lean_object* x_105; uint8_t x_106; uint8_t x_107; lean_object* x_108; lean_dec(x_4); lean_dec(x_3); -x_98 = lean_ctor_get(x_96, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_96, 1); -lean_inc(x_99); -lean_dec(x_96); -x_100 = 1; -x_101 = 1; -x_102 = l_Lean_Meta_mkForallFVars(x_98, x_91, x_93, x_100, x_101, x_5, x_6, x_7, x_8, x_99); +x_104 = lean_ctor_get(x_102, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_102, 1); +lean_inc(x_105); +lean_dec(x_102); +x_106 = 1; +x_107 = 1; +x_108 = l_Lean_Meta_mkForallFVars(x_104, x_97, x_99, x_106, x_107, x_5, x_6, x_7, x_8, x_105); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_102) == 0) +if (lean_obj_tag(x_108) == 0) { -uint8_t x_103; -x_103 = !lean_is_exclusive(x_102); -if (x_103 == 0) +uint8_t x_109; +x_109 = !lean_is_exclusive(x_108); +if (x_109 == 0) { -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_102, 0); -lean_ctor_set(x_10, 0, x_104); -x_105 = lean_box(0); -x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_10); -lean_ctor_set(x_106, 1, x_105); -lean_ctor_set(x_102, 0, x_106); -return x_102; +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_108, 0); +lean_ctor_set(x_10, 0, x_110); +x_111 = lean_box(0); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_10); +lean_ctor_set(x_112, 1, x_111); +lean_ctor_set(x_108, 0, x_112); +return x_108; } else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_107 = lean_ctor_get(x_102, 0); -x_108 = lean_ctor_get(x_102, 1); -lean_inc(x_108); -lean_inc(x_107); -lean_dec(x_102); -lean_ctor_set(x_10, 0, x_107); -x_109 = lean_box(0); -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_10); -lean_ctor_set(x_110, 1, x_109); -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_108); -return x_111; +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_113 = lean_ctor_get(x_108, 0); +x_114 = lean_ctor_get(x_108, 1); +lean_inc(x_114); +lean_inc(x_113); +lean_dec(x_108); +lean_ctor_set(x_10, 0, x_113); +x_115 = lean_box(0); +x_116 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_116, 0, x_10); +lean_ctor_set(x_116, 1, x_115); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_114); +return x_117; } } else { -uint8_t x_112; +uint8_t x_118; lean_free_object(x_10); -x_112 = !lean_is_exclusive(x_102); -if (x_112 == 0) +x_118 = !lean_is_exclusive(x_108); +if (x_118 == 0) { -return x_102; +return x_108; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_102, 0); -x_114 = lean_ctor_get(x_102, 1); -lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_102); -x_115 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -return x_115; +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_ctor_get(x_108, 0); +x_120 = lean_ctor_get(x_108, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_108); +x_121 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_121, 0, x_119); +lean_ctor_set(x_121, 1, x_120); +return x_121; } } } else { -lean_object* x_116; lean_object* x_117; uint8_t x_118; -x_116 = lean_ctor_get(x_96, 0); -lean_inc(x_116); -x_117 = lean_ctor_get(x_96, 1); -lean_inc(x_117); -lean_dec(x_96); -x_118 = !lean_is_exclusive(x_97); -if (x_118 == 0) +lean_object* x_122; lean_object* x_123; uint8_t x_124; +x_122 = lean_ctor_get(x_102, 0); +lean_inc(x_122); +x_123 = lean_ctor_get(x_102, 1); +lean_inc(x_123); +lean_dec(x_102); +x_124 = !lean_is_exclusive(x_103); +if (x_124 == 0) { -lean_object* x_119; lean_object* x_120; uint8_t x_121; lean_object* x_122; -x_119 = lean_ctor_get(x_97, 0); -lean_inc(x_91); -lean_ctor_set(x_97, 0, x_91); -x_120 = lean_box(0); -x_121 = 1; +lean_object* x_125; lean_object* x_126; uint8_t x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_125 = lean_ctor_get(x_103, 0); +lean_inc(x_97); +lean_ctor_set(x_103, 0, x_97); +x_126 = lean_box(0); +x_127 = 1; +x_128 = lean_box(x_127); +x_129 = lean_box(x_127); +x_130 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_130, 0, x_125); +lean_closure_set(x_130, 1, x_103); +lean_closure_set(x_130, 2, x_128); +lean_closure_set(x_130, 3, x_129); +lean_closure_set(x_130, 4, x_126); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_122 = l_Lean_Elab_Term_elabTermEnsuringType(x_119, x_97, x_121, x_121, x_120, x_3, x_4, x_5, x_6, x_7, x_8, x_117); -if (lean_obj_tag(x_122) == 0) +x_131 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_130, x_3, x_4, x_5, x_6, x_7, x_8, x_123); +if (lean_obj_tag(x_131) == 0) { -lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_123 = lean_ctor_get(x_122, 0); -lean_inc(x_123); -x_124 = lean_ctor_get(x_122, 1); -lean_inc(x_124); -lean_dec(x_122); +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_131, 0); +lean_inc(x_132); +x_133 = lean_ctor_get(x_131, 1); +lean_inc(x_133); +lean_dec(x_131); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_125 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_93, x_93, x_3, x_4, x_5, x_6, x_7, x_8, x_124); -if (lean_obj_tag(x_125) == 0) +x_134 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_99, x_99, x_3, x_4, x_5, x_6, x_7, x_8, x_133); +if (lean_obj_tag(x_134) == 0) { -lean_object* x_126; uint8_t x_127; lean_object* x_128; -x_126 = lean_ctor_get(x_125, 1); -lean_inc(x_126); -lean_dec(x_125); -x_127 = 1; -lean_inc(x_116); -x_128 = l_Lean_Meta_mkForallFVars(x_116, x_91, x_93, x_121, x_127, x_5, x_6, x_7, x_8, x_126); -if (lean_obj_tag(x_128) == 0) -{ -lean_object* x_129; lean_object* x_130; lean_object* x_131; -x_129 = lean_ctor_get(x_128, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_128, 1); -lean_inc(x_130); -lean_dec(x_128); -x_131 = l_Lean_Meta_mkLambdaFVars(x_116, x_123, x_93, x_121, x_127, x_5, x_6, x_7, x_8, x_130); +lean_object* x_135; uint8_t x_136; lean_object* x_137; +x_135 = lean_ctor_get(x_134, 1); +lean_inc(x_135); +lean_dec(x_134); +x_136 = 1; +lean_inc(x_122); +x_137 = l_Lean_Meta_mkForallFVars(x_122, x_97, x_99, x_127, x_136, x_5, x_6, x_7, x_8, x_135); +if (lean_obj_tag(x_137) == 0) +{ +lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_138 = lean_ctor_get(x_137, 0); +lean_inc(x_138); +x_139 = lean_ctor_get(x_137, 1); +lean_inc(x_139); +lean_dec(x_137); +x_140 = l_Lean_Meta_mkLambdaFVars(x_122, x_132, x_99, x_127, x_136, x_5, x_6, x_7, x_8, x_139); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_131) == 0) +if (lean_obj_tag(x_140) == 0) { -uint8_t x_132; -x_132 = !lean_is_exclusive(x_131); -if (x_132 == 0) +uint8_t x_141; +x_141 = !lean_is_exclusive(x_140); +if (x_141 == 0) { -lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_133 = lean_ctor_get(x_131, 0); -lean_ctor_set(x_10, 0, x_129); -x_134 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_134, 0, x_133); -x_135 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_135, 0, x_10); -lean_ctor_set(x_135, 1, x_134); -lean_ctor_set(x_131, 0, x_135); -return x_131; +lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_142 = lean_ctor_get(x_140, 0); +lean_ctor_set(x_10, 0, x_138); +x_143 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_143, 0, x_142); +x_144 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_144, 0, x_10); +lean_ctor_set(x_144, 1, x_143); +lean_ctor_set(x_140, 0, x_144); +return x_140; } else { -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -x_136 = lean_ctor_get(x_131, 0); -x_137 = lean_ctor_get(x_131, 1); -lean_inc(x_137); -lean_inc(x_136); -lean_dec(x_131); -lean_ctor_set(x_10, 0, x_129); -x_138 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_138, 0, x_136); -x_139 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_139, 0, x_10); -lean_ctor_set(x_139, 1, x_138); -x_140 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_140, 0, x_139); -lean_ctor_set(x_140, 1, x_137); -return x_140; +lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_145 = lean_ctor_get(x_140, 0); +x_146 = lean_ctor_get(x_140, 1); +lean_inc(x_146); +lean_inc(x_145); +lean_dec(x_140); +lean_ctor_set(x_10, 0, x_138); +x_147 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_147, 0, x_145); +x_148 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_148, 0, x_10); +lean_ctor_set(x_148, 1, x_147); +x_149 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_149, 0, x_148); +lean_ctor_set(x_149, 1, x_146); +return x_149; } } else { -uint8_t x_141; -lean_dec(x_129); +uint8_t x_150; +lean_dec(x_138); lean_free_object(x_10); -x_141 = !lean_is_exclusive(x_131); -if (x_141 == 0) +x_150 = !lean_is_exclusive(x_140); +if (x_150 == 0) { -return x_131; +return x_140; } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_142 = lean_ctor_get(x_131, 0); -x_143 = lean_ctor_get(x_131, 1); -lean_inc(x_143); -lean_inc(x_142); -lean_dec(x_131); -x_144 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_144, 0, x_142); -lean_ctor_set(x_144, 1, x_143); -return x_144; +lean_object* x_151; lean_object* x_152; lean_object* x_153; +x_151 = lean_ctor_get(x_140, 0); +x_152 = lean_ctor_get(x_140, 1); +lean_inc(x_152); +lean_inc(x_151); +lean_dec(x_140); +x_153 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_153, 0, x_151); +lean_ctor_set(x_153, 1, x_152); +return x_153; } } } else { -uint8_t x_145; -lean_dec(x_123); -lean_dec(x_116); +uint8_t x_154; +lean_dec(x_132); +lean_dec(x_122); lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_145 = !lean_is_exclusive(x_128); -if (x_145 == 0) +x_154 = !lean_is_exclusive(x_137); +if (x_154 == 0) { -return x_128; +return x_137; } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_146 = lean_ctor_get(x_128, 0); -x_147 = lean_ctor_get(x_128, 1); -lean_inc(x_147); -lean_inc(x_146); -lean_dec(x_128); -x_148 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_148, 0, x_146); -lean_ctor_set(x_148, 1, x_147); -return x_148; +lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_155 = lean_ctor_get(x_137, 0); +x_156 = lean_ctor_get(x_137, 1); +lean_inc(x_156); +lean_inc(x_155); +lean_dec(x_137); +x_157 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_157, 0, x_155); +lean_ctor_set(x_157, 1, x_156); +return x_157; } } } else { -uint8_t x_149; -lean_dec(x_123); -lean_dec(x_116); -lean_dec(x_91); +uint8_t x_158; +lean_dec(x_132); +lean_dec(x_122); +lean_dec(x_97); lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_149 = !lean_is_exclusive(x_125); -if (x_149 == 0) +x_158 = !lean_is_exclusive(x_134); +if (x_158 == 0) { -return x_125; +return x_134; } else { -lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_150 = lean_ctor_get(x_125, 0); -x_151 = lean_ctor_get(x_125, 1); -lean_inc(x_151); -lean_inc(x_150); -lean_dec(x_125); -x_152 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_152, 0, x_150); -lean_ctor_set(x_152, 1, x_151); -return x_152; +lean_object* x_159; lean_object* x_160; lean_object* x_161; +x_159 = lean_ctor_get(x_134, 0); +x_160 = lean_ctor_get(x_134, 1); +lean_inc(x_160); +lean_inc(x_159); +lean_dec(x_134); +x_161 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_161, 0, x_159); +lean_ctor_set(x_161, 1, x_160); +return x_161; } } } else { -uint8_t x_153; -lean_dec(x_116); -lean_dec(x_91); +uint8_t x_162; +lean_dec(x_122); +lean_dec(x_97); lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); @@ -14396,206 +14483,214 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_153 = !lean_is_exclusive(x_122); -if (x_153 == 0) +x_162 = !lean_is_exclusive(x_131); +if (x_162 == 0) { -return x_122; +return x_131; } else { -lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_154 = lean_ctor_get(x_122, 0); -x_155 = lean_ctor_get(x_122, 1); -lean_inc(x_155); -lean_inc(x_154); -lean_dec(x_122); -x_156 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_156, 0, x_154); -lean_ctor_set(x_156, 1, x_155); -return x_156; +lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_163 = lean_ctor_get(x_131, 0); +x_164 = lean_ctor_get(x_131, 1); +lean_inc(x_164); +lean_inc(x_163); +lean_dec(x_131); +x_165 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_165, 0, x_163); +lean_ctor_set(x_165, 1, x_164); +return x_165; } } } else { -lean_object* x_157; lean_object* x_158; lean_object* x_159; uint8_t x_160; lean_object* x_161; -x_157 = lean_ctor_get(x_97, 0); -lean_inc(x_157); -lean_dec(x_97); -lean_inc(x_91); -x_158 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_158, 0, x_91); -x_159 = lean_box(0); -x_160 = 1; +lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_166 = lean_ctor_get(x_103, 0); +lean_inc(x_166); +lean_dec(x_103); +lean_inc(x_97); +x_167 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_167, 0, x_97); +x_168 = lean_box(0); +x_169 = 1; +x_170 = lean_box(x_169); +x_171 = lean_box(x_169); +x_172 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_172, 0, x_166); +lean_closure_set(x_172, 1, x_167); +lean_closure_set(x_172, 2, x_170); +lean_closure_set(x_172, 3, x_171); +lean_closure_set(x_172, 4, x_168); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_161 = l_Lean_Elab_Term_elabTermEnsuringType(x_157, x_158, x_160, x_160, x_159, x_3, x_4, x_5, x_6, x_7, x_8, x_117); -if (lean_obj_tag(x_161) == 0) +x_173 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_172, x_3, x_4, x_5, x_6, x_7, x_8, x_123); +if (lean_obj_tag(x_173) == 0) { -lean_object* x_162; lean_object* x_163; lean_object* x_164; -x_162 = lean_ctor_get(x_161, 0); -lean_inc(x_162); -x_163 = lean_ctor_get(x_161, 1); -lean_inc(x_163); -lean_dec(x_161); +lean_object* x_174; lean_object* x_175; lean_object* x_176; +x_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_173, 1); +lean_inc(x_175); +lean_dec(x_173); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_164 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_93, x_93, x_3, x_4, x_5, x_6, x_7, x_8, x_163); -if (lean_obj_tag(x_164) == 0) -{ -lean_object* x_165; uint8_t x_166; lean_object* x_167; -x_165 = lean_ctor_get(x_164, 1); -lean_inc(x_165); -lean_dec(x_164); -x_166 = 1; -lean_inc(x_116); -x_167 = l_Lean_Meta_mkForallFVars(x_116, x_91, x_93, x_160, x_166, x_5, x_6, x_7, x_8, x_165); -if (lean_obj_tag(x_167) == 0) +x_176 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_99, x_99, x_3, x_4, x_5, x_6, x_7, x_8, x_175); +if (lean_obj_tag(x_176) == 0) { -lean_object* x_168; lean_object* x_169; lean_object* x_170; -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -x_169 = lean_ctor_get(x_167, 1); -lean_inc(x_169); -lean_dec(x_167); -x_170 = l_Lean_Meta_mkLambdaFVars(x_116, x_162, x_93, x_160, x_166, x_5, x_6, x_7, x_8, x_169); +lean_object* x_177; uint8_t x_178; lean_object* x_179; +x_177 = lean_ctor_get(x_176, 1); +lean_inc(x_177); +lean_dec(x_176); +x_178 = 1; +lean_inc(x_122); +x_179 = l_Lean_Meta_mkForallFVars(x_122, x_97, x_99, x_169, x_178, x_5, x_6, x_7, x_8, x_177); +if (lean_obj_tag(x_179) == 0) +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_180 = lean_ctor_get(x_179, 0); +lean_inc(x_180); +x_181 = lean_ctor_get(x_179, 1); +lean_inc(x_181); +lean_dec(x_179); +x_182 = l_Lean_Meta_mkLambdaFVars(x_122, x_174, x_99, x_169, x_178, x_5, x_6, x_7, x_8, x_181); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_170) == 0) +if (lean_obj_tag(x_182) == 0) { -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_171 = lean_ctor_get(x_170, 0); -lean_inc(x_171); -x_172 = lean_ctor_get(x_170, 1); -lean_inc(x_172); -if (lean_is_exclusive(x_170)) { - lean_ctor_release(x_170, 0); - lean_ctor_release(x_170, 1); - x_173 = x_170; +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_183 = lean_ctor_get(x_182, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_182, 1); +lean_inc(x_184); +if (lean_is_exclusive(x_182)) { + lean_ctor_release(x_182, 0); + lean_ctor_release(x_182, 1); + x_185 = x_182; } else { - lean_dec_ref(x_170); - x_173 = lean_box(0); -} -lean_ctor_set(x_10, 0, x_168); -x_174 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_174, 0, x_171); -x_175 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_175, 0, x_10); -lean_ctor_set(x_175, 1, x_174); -if (lean_is_scalar(x_173)) { - x_176 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_182); + x_185 = lean_box(0); +} +lean_ctor_set(x_10, 0, x_180); +x_186 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_186, 0, x_183); +x_187 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_187, 0, x_10); +lean_ctor_set(x_187, 1, x_186); +if (lean_is_scalar(x_185)) { + x_188 = lean_alloc_ctor(0, 2, 0); } else { - x_176 = x_173; + x_188 = x_185; } -lean_ctor_set(x_176, 0, x_175); -lean_ctor_set(x_176, 1, x_172); -return x_176; +lean_ctor_set(x_188, 0, x_187); +lean_ctor_set(x_188, 1, x_184); +return x_188; } else { -lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; -lean_dec(x_168); +lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; +lean_dec(x_180); lean_free_object(x_10); -x_177 = lean_ctor_get(x_170, 0); -lean_inc(x_177); -x_178 = lean_ctor_get(x_170, 1); -lean_inc(x_178); -if (lean_is_exclusive(x_170)) { - lean_ctor_release(x_170, 0); - lean_ctor_release(x_170, 1); - x_179 = x_170; +x_189 = lean_ctor_get(x_182, 0); +lean_inc(x_189); +x_190 = lean_ctor_get(x_182, 1); +lean_inc(x_190); +if (lean_is_exclusive(x_182)) { + lean_ctor_release(x_182, 0); + lean_ctor_release(x_182, 1); + x_191 = x_182; } else { - lean_dec_ref(x_170); - x_179 = lean_box(0); + lean_dec_ref(x_182); + x_191 = lean_box(0); } -if (lean_is_scalar(x_179)) { - x_180 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_191)) { + x_192 = lean_alloc_ctor(1, 2, 0); } else { - x_180 = x_179; + x_192 = x_191; } -lean_ctor_set(x_180, 0, x_177); -lean_ctor_set(x_180, 1, x_178); -return x_180; +lean_ctor_set(x_192, 0, x_189); +lean_ctor_set(x_192, 1, x_190); +return x_192; } } else { -lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; -lean_dec(x_162); -lean_dec(x_116); +lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; +lean_dec(x_174); +lean_dec(x_122); lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_181 = lean_ctor_get(x_167, 0); -lean_inc(x_181); -x_182 = lean_ctor_get(x_167, 1); -lean_inc(x_182); -if (lean_is_exclusive(x_167)) { - lean_ctor_release(x_167, 0); - lean_ctor_release(x_167, 1); - x_183 = x_167; +x_193 = lean_ctor_get(x_179, 0); +lean_inc(x_193); +x_194 = lean_ctor_get(x_179, 1); +lean_inc(x_194); +if (lean_is_exclusive(x_179)) { + lean_ctor_release(x_179, 0); + lean_ctor_release(x_179, 1); + x_195 = x_179; } else { - lean_dec_ref(x_167); - x_183 = lean_box(0); + lean_dec_ref(x_179); + x_195 = lean_box(0); } -if (lean_is_scalar(x_183)) { - x_184 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_195)) { + x_196 = lean_alloc_ctor(1, 2, 0); } else { - x_184 = x_183; + x_196 = x_195; } -lean_ctor_set(x_184, 0, x_181); -lean_ctor_set(x_184, 1, x_182); -return x_184; +lean_ctor_set(x_196, 0, x_193); +lean_ctor_set(x_196, 1, x_194); +return x_196; } } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -lean_dec(x_162); -lean_dec(x_116); -lean_dec(x_91); +lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +lean_dec(x_174); +lean_dec(x_122); +lean_dec(x_97); lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_185 = lean_ctor_get(x_164, 0); -lean_inc(x_185); -x_186 = lean_ctor_get(x_164, 1); -lean_inc(x_186); -if (lean_is_exclusive(x_164)) { - lean_ctor_release(x_164, 0); - lean_ctor_release(x_164, 1); - x_187 = x_164; +x_197 = lean_ctor_get(x_176, 0); +lean_inc(x_197); +x_198 = lean_ctor_get(x_176, 1); +lean_inc(x_198); +if (lean_is_exclusive(x_176)) { + lean_ctor_release(x_176, 0); + lean_ctor_release(x_176, 1); + x_199 = x_176; } else { - lean_dec_ref(x_164); - x_187 = lean_box(0); + lean_dec_ref(x_176); + x_199 = lean_box(0); } -if (lean_is_scalar(x_187)) { - x_188 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_199)) { + x_200 = lean_alloc_ctor(1, 2, 0); } else { - x_188 = x_187; + x_200 = x_199; } -lean_ctor_set(x_188, 0, x_185); -lean_ctor_set(x_188, 1, x_186); -return x_188; +lean_ctor_set(x_200, 0, x_197); +lean_ctor_set(x_200, 1, x_198); +return x_200; } } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -lean_dec(x_116); -lean_dec(x_91); +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; +lean_dec(x_122); +lean_dec(x_97); lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); @@ -14603,34 +14698,34 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_189 = lean_ctor_get(x_161, 0); -lean_inc(x_189); -x_190 = lean_ctor_get(x_161, 1); -lean_inc(x_190); -if (lean_is_exclusive(x_161)) { - lean_ctor_release(x_161, 0); - lean_ctor_release(x_161, 1); - x_191 = x_161; +x_201 = lean_ctor_get(x_173, 0); +lean_inc(x_201); +x_202 = lean_ctor_get(x_173, 1); +lean_inc(x_202); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_203 = x_173; } else { - lean_dec_ref(x_161); - x_191 = lean_box(0); + lean_dec_ref(x_173); + x_203 = lean_box(0); } -if (lean_is_scalar(x_191)) { - x_192 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_203)) { + x_204 = lean_alloc_ctor(1, 2, 0); } else { - x_192 = x_191; + x_204 = x_203; } -lean_ctor_set(x_192, 0, x_189); -lean_ctor_set(x_192, 1, x_190); -return x_192; +lean_ctor_set(x_204, 0, x_201); +lean_ctor_set(x_204, 1, x_202); +return x_204; } } } } else { -uint8_t x_193; -lean_dec(x_91); +uint8_t x_205; +lean_dec(x_97); lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); @@ -14639,30 +14734,30 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_193 = !lean_is_exclusive(x_96); -if (x_193 == 0) +x_205 = !lean_is_exclusive(x_102); +if (x_205 == 0) { -return x_96; +return x_102; } else { -lean_object* x_194; lean_object* x_195; lean_object* x_196; -x_194 = lean_ctor_get(x_96, 0); -x_195 = lean_ctor_get(x_96, 1); -lean_inc(x_195); -lean_inc(x_194); -lean_dec(x_96); -x_196 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_196, 0, x_194); -lean_ctor_set(x_196, 1, x_195); -return x_196; +lean_object* x_206; lean_object* x_207; lean_object* x_208; +x_206 = lean_ctor_get(x_102, 0); +x_207 = lean_ctor_get(x_102, 1); +lean_inc(x_207); +lean_inc(x_206); +lean_dec(x_102); +x_208 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_208, 0, x_206); +lean_ctor_set(x_208, 1, x_207); +return x_208; } } } else { -uint8_t x_197; -lean_dec(x_91); +uint8_t x_209; +lean_dec(x_97); lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); @@ -14672,29 +14767,29 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_197 = !lean_is_exclusive(x_94); -if (x_197 == 0) +x_209 = !lean_is_exclusive(x_100); +if (x_209 == 0) { -return x_94; +return x_100; } else { -lean_object* x_198; lean_object* x_199; lean_object* x_200; -x_198 = lean_ctor_get(x_94, 0); -x_199 = lean_ctor_get(x_94, 1); -lean_inc(x_199); -lean_inc(x_198); -lean_dec(x_94); -x_200 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_200, 0, x_198); -lean_ctor_set(x_200, 1, x_199); -return x_200; +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_100, 0); +x_211 = lean_ctor_get(x_100, 1); +lean_inc(x_211); +lean_inc(x_210); +lean_dec(x_100); +x_212 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_212, 0, x_210); +lean_ctor_set(x_212, 1, x_211); +return x_212; } } } else { -uint8_t x_201; +uint8_t x_213; lean_free_object(x_10); lean_dec(x_8); lean_dec(x_7); @@ -14704,31 +14799,31 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_201 = !lean_is_exclusive(x_90); -if (x_201 == 0) +x_213 = !lean_is_exclusive(x_96); +if (x_213 == 0) { -return x_90; +return x_96; } else { -lean_object* x_202; lean_object* x_203; lean_object* x_204; -x_202 = lean_ctor_get(x_90, 0); -x_203 = lean_ctor_get(x_90, 1); -lean_inc(x_203); -lean_inc(x_202); -lean_dec(x_90); -x_204 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_204, 0, x_202); -lean_ctor_set(x_204, 1, x_203); -return x_204; +lean_object* x_214; lean_object* x_215; lean_object* x_216; +x_214 = lean_ctor_get(x_96, 0); +x_215 = lean_ctor_get(x_96, 1); +lean_inc(x_215); +lean_inc(x_214); +lean_dec(x_96); +x_216 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_216, 0, x_214); +lean_ctor_set(x_216, 1, x_215); +return x_216; } } } else { -lean_object* x_205; lean_object* x_206; -x_205 = lean_ctor_get(x_10, 0); -lean_inc(x_205); +lean_object* x_217; lean_object* x_218; +x_217 = lean_ctor_get(x_10, 0); +lean_inc(x_217); lean_dec(x_10); lean_inc(x_8); lean_inc(x_7); @@ -14736,339 +14831,347 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_206 = l_Lean_Elab_Term_elabType(x_205, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_206) == 0) +x_218 = l_Lean_Elab_Term_elabType(x_217, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_218) == 0) { -lean_object* x_207; lean_object* x_208; uint8_t x_209; lean_object* x_210; -x_207 = lean_ctor_get(x_206, 0); -lean_inc(x_207); -x_208 = lean_ctor_get(x_206, 1); -lean_inc(x_208); -lean_dec(x_206); -x_209 = 0; +lean_object* x_219; lean_object* x_220; uint8_t x_221; lean_object* x_222; +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +x_220 = lean_ctor_get(x_218, 1); +lean_inc(x_220); +lean_dec(x_218); +x_221 = 0; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_210 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_209, x_209, x_3, x_4, x_5, x_6, x_7, x_8, x_208); -if (lean_obj_tag(x_210) == 0) +x_222 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_221, x_221, x_3, x_4, x_5, x_6, x_7, x_8, x_220); +if (lean_obj_tag(x_222) == 0) { -lean_object* x_211; lean_object* x_212; -x_211 = lean_ctor_get(x_210, 1); -lean_inc(x_211); -lean_dec(x_210); +lean_object* x_223; lean_object* x_224; +x_223 = lean_ctor_get(x_222, 1); +lean_inc(x_223); +lean_dec(x_222); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_3); -x_212 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_211); -if (lean_obj_tag(x_212) == 0) +x_224 = l_Lean_Elab_Term_addAutoBoundImplicits(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_223); +if (lean_obj_tag(x_224) == 0) { -lean_object* x_213; -x_213 = lean_ctor_get(x_1, 7); -lean_inc(x_213); +lean_object* x_225; +x_225 = lean_ctor_get(x_1, 7); +lean_inc(x_225); lean_dec(x_1); -if (lean_obj_tag(x_213) == 0) +if (lean_obj_tag(x_225) == 0) { -lean_object* x_214; lean_object* x_215; uint8_t x_216; uint8_t x_217; lean_object* x_218; +lean_object* x_226; lean_object* x_227; uint8_t x_228; uint8_t x_229; lean_object* x_230; lean_dec(x_4); lean_dec(x_3); -x_214 = lean_ctor_get(x_212, 0); -lean_inc(x_214); -x_215 = lean_ctor_get(x_212, 1); -lean_inc(x_215); -lean_dec(x_212); -x_216 = 1; -x_217 = 1; -x_218 = l_Lean_Meta_mkForallFVars(x_214, x_207, x_209, x_216, x_217, x_5, x_6, x_7, x_8, x_215); +x_226 = lean_ctor_get(x_224, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_224, 1); +lean_inc(x_227); +lean_dec(x_224); +x_228 = 1; +x_229 = 1; +x_230 = l_Lean_Meta_mkForallFVars(x_226, x_219, x_221, x_228, x_229, x_5, x_6, x_7, x_8, x_227); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_218) == 0) +if (lean_obj_tag(x_230) == 0) { -lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; -x_219 = lean_ctor_get(x_218, 0); -lean_inc(x_219); -x_220 = lean_ctor_get(x_218, 1); -lean_inc(x_220); -if (lean_is_exclusive(x_218)) { - lean_ctor_release(x_218, 0); - lean_ctor_release(x_218, 1); - x_221 = x_218; +lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; +x_231 = lean_ctor_get(x_230, 0); +lean_inc(x_231); +x_232 = lean_ctor_get(x_230, 1); +lean_inc(x_232); +if (lean_is_exclusive(x_230)) { + lean_ctor_release(x_230, 0); + lean_ctor_release(x_230, 1); + x_233 = x_230; } else { - lean_dec_ref(x_218); - x_221 = lean_box(0); -} -x_222 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_222, 0, x_219); -x_223 = lean_box(0); -x_224 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_224, 0, x_222); -lean_ctor_set(x_224, 1, x_223); -if (lean_is_scalar(x_221)) { - x_225 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_230); + x_233 = lean_box(0); +} +x_234 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_234, 0, x_231); +x_235 = lean_box(0); +x_236 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_236, 0, x_234); +lean_ctor_set(x_236, 1, x_235); +if (lean_is_scalar(x_233)) { + x_237 = lean_alloc_ctor(0, 2, 0); } else { - x_225 = x_221; + x_237 = x_233; } -lean_ctor_set(x_225, 0, x_224); -lean_ctor_set(x_225, 1, x_220); -return x_225; +lean_ctor_set(x_237, 0, x_236); +lean_ctor_set(x_237, 1, x_232); +return x_237; } else { -lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; -x_226 = lean_ctor_get(x_218, 0); -lean_inc(x_226); -x_227 = lean_ctor_get(x_218, 1); -lean_inc(x_227); -if (lean_is_exclusive(x_218)) { - lean_ctor_release(x_218, 0); - lean_ctor_release(x_218, 1); - x_228 = x_218; +lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; +x_238 = lean_ctor_get(x_230, 0); +lean_inc(x_238); +x_239 = lean_ctor_get(x_230, 1); +lean_inc(x_239); +if (lean_is_exclusive(x_230)) { + lean_ctor_release(x_230, 0); + lean_ctor_release(x_230, 1); + x_240 = x_230; } else { - lean_dec_ref(x_218); - x_228 = lean_box(0); + lean_dec_ref(x_230); + x_240 = lean_box(0); } -if (lean_is_scalar(x_228)) { - x_229 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_240)) { + x_241 = lean_alloc_ctor(1, 2, 0); } else { - x_229 = x_228; + x_241 = x_240; } -lean_ctor_set(x_229, 0, x_226); -lean_ctor_set(x_229, 1, x_227); -return x_229; +lean_ctor_set(x_241, 0, x_238); +lean_ctor_set(x_241, 1, x_239); +return x_241; } } else { -lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; uint8_t x_236; lean_object* x_237; -x_230 = lean_ctor_get(x_212, 0); -lean_inc(x_230); -x_231 = lean_ctor_get(x_212, 1); -lean_inc(x_231); -lean_dec(x_212); -x_232 = lean_ctor_get(x_213, 0); -lean_inc(x_232); -if (lean_is_exclusive(x_213)) { - lean_ctor_release(x_213, 0); - x_233 = x_213; +lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; uint8_t x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; +x_242 = lean_ctor_get(x_224, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_224, 1); +lean_inc(x_243); +lean_dec(x_224); +x_244 = lean_ctor_get(x_225, 0); +lean_inc(x_244); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + x_245 = x_225; } else { - lean_dec_ref(x_213); - x_233 = lean_box(0); + lean_dec_ref(x_225); + x_245 = lean_box(0); } -lean_inc(x_207); -if (lean_is_scalar(x_233)) { - x_234 = lean_alloc_ctor(1, 1, 0); +lean_inc(x_219); +if (lean_is_scalar(x_245)) { + x_246 = lean_alloc_ctor(1, 1, 0); } else { - x_234 = x_233; + x_246 = x_245; } -lean_ctor_set(x_234, 0, x_207); -x_235 = lean_box(0); -x_236 = 1; +lean_ctor_set(x_246, 0, x_219); +x_247 = lean_box(0); +x_248 = 1; +x_249 = lean_box(x_248); +x_250 = lean_box(x_248); +x_251 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_251, 0, x_244); +lean_closure_set(x_251, 1, x_246); +lean_closure_set(x_251, 2, x_249); +lean_closure_set(x_251, 3, x_250); +lean_closure_set(x_251, 4, x_247); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_237 = l_Lean_Elab_Term_elabTermEnsuringType(x_232, x_234, x_236, x_236, x_235, x_3, x_4, x_5, x_6, x_7, x_8, x_231); -if (lean_obj_tag(x_237) == 0) +x_252 = l_Lean_Elab_Term_withoutAutoBoundImplicit___rarg(x_251, x_3, x_4, x_5, x_6, x_7, x_8, x_243); +if (lean_obj_tag(x_252) == 0) { -lean_object* x_238; lean_object* x_239; lean_object* x_240; -x_238 = lean_ctor_get(x_237, 0); -lean_inc(x_238); -x_239 = lean_ctor_get(x_237, 1); -lean_inc(x_239); -lean_dec(x_237); +lean_object* x_253; lean_object* x_254; lean_object* x_255; +x_253 = lean_ctor_get(x_252, 0); +lean_inc(x_253); +x_254 = lean_ctor_get(x_252, 1); +lean_inc(x_254); +lean_dec(x_252); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_240 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_209, x_209, x_3, x_4, x_5, x_6, x_7, x_8, x_239); -if (lean_obj_tag(x_240) == 0) -{ -lean_object* x_241; uint8_t x_242; lean_object* x_243; -x_241 = lean_ctor_get(x_240, 1); -lean_inc(x_241); -lean_dec(x_240); -x_242 = 1; -lean_inc(x_230); -x_243 = l_Lean_Meta_mkForallFVars(x_230, x_207, x_209, x_236, x_242, x_5, x_6, x_7, x_8, x_241); -if (lean_obj_tag(x_243) == 0) -{ -lean_object* x_244; lean_object* x_245; lean_object* x_246; -x_244 = lean_ctor_get(x_243, 0); -lean_inc(x_244); -x_245 = lean_ctor_get(x_243, 1); -lean_inc(x_245); -lean_dec(x_243); -x_246 = l_Lean_Meta_mkLambdaFVars(x_230, x_238, x_209, x_236, x_242, x_5, x_6, x_7, x_8, x_245); +x_255 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_221, x_221, x_3, x_4, x_5, x_6, x_7, x_8, x_254); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; uint8_t x_257; lean_object* x_258; +x_256 = lean_ctor_get(x_255, 1); +lean_inc(x_256); +lean_dec(x_255); +x_257 = 1; +lean_inc(x_242); +x_258 = l_Lean_Meta_mkForallFVars(x_242, x_219, x_221, x_248, x_257, x_5, x_6, x_7, x_8, x_256); +if (lean_obj_tag(x_258) == 0) +{ +lean_object* x_259; lean_object* x_260; lean_object* x_261; +x_259 = lean_ctor_get(x_258, 0); +lean_inc(x_259); +x_260 = lean_ctor_get(x_258, 1); +lean_inc(x_260); +lean_dec(x_258); +x_261 = l_Lean_Meta_mkLambdaFVars(x_242, x_253, x_221, x_248, x_257, x_5, x_6, x_7, x_8, x_260); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -if (lean_obj_tag(x_246) == 0) +if (lean_obj_tag(x_261) == 0) { -lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; -x_247 = lean_ctor_get(x_246, 0); -lean_inc(x_247); -x_248 = lean_ctor_get(x_246, 1); -lean_inc(x_248); -if (lean_is_exclusive(x_246)) { - lean_ctor_release(x_246, 0); - lean_ctor_release(x_246, 1); - x_249 = x_246; +lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_262 = lean_ctor_get(x_261, 0); +lean_inc(x_262); +x_263 = lean_ctor_get(x_261, 1); +lean_inc(x_263); +if (lean_is_exclusive(x_261)) { + lean_ctor_release(x_261, 0); + lean_ctor_release(x_261, 1); + x_264 = x_261; } else { - lean_dec_ref(x_246); - x_249 = lean_box(0); -} -x_250 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_250, 0, x_244); -x_251 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_251, 0, x_247); -x_252 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_252, 0, x_250); -lean_ctor_set(x_252, 1, x_251); -if (lean_is_scalar(x_249)) { - x_253 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_261); + x_264 = lean_box(0); +} +x_265 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_265, 0, x_259); +x_266 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_266, 0, x_262); +x_267 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +if (lean_is_scalar(x_264)) { + x_268 = lean_alloc_ctor(0, 2, 0); } else { - x_253 = x_249; + x_268 = x_264; } -lean_ctor_set(x_253, 0, x_252); -lean_ctor_set(x_253, 1, x_248); -return x_253; +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_263); +return x_268; } else { -lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; -lean_dec(x_244); -x_254 = lean_ctor_get(x_246, 0); -lean_inc(x_254); -x_255 = lean_ctor_get(x_246, 1); -lean_inc(x_255); -if (lean_is_exclusive(x_246)) { - lean_ctor_release(x_246, 0); - lean_ctor_release(x_246, 1); - x_256 = x_246; +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; +lean_dec(x_259); +x_269 = lean_ctor_get(x_261, 0); +lean_inc(x_269); +x_270 = lean_ctor_get(x_261, 1); +lean_inc(x_270); +if (lean_is_exclusive(x_261)) { + lean_ctor_release(x_261, 0); + lean_ctor_release(x_261, 1); + x_271 = x_261; } else { - lean_dec_ref(x_246); - x_256 = lean_box(0); + lean_dec_ref(x_261); + x_271 = lean_box(0); } -if (lean_is_scalar(x_256)) { - x_257 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_271)) { + x_272 = lean_alloc_ctor(1, 2, 0); } else { - x_257 = x_256; + x_272 = x_271; } -lean_ctor_set(x_257, 0, x_254); -lean_ctor_set(x_257, 1, x_255); -return x_257; +lean_ctor_set(x_272, 0, x_269); +lean_ctor_set(x_272, 1, x_270); +return x_272; } } else { -lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; -lean_dec(x_238); -lean_dec(x_230); +lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; +lean_dec(x_253); +lean_dec(x_242); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_258 = lean_ctor_get(x_243, 0); -lean_inc(x_258); -x_259 = lean_ctor_get(x_243, 1); -lean_inc(x_259); -if (lean_is_exclusive(x_243)) { - lean_ctor_release(x_243, 0); - lean_ctor_release(x_243, 1); - x_260 = x_243; +x_273 = lean_ctor_get(x_258, 0); +lean_inc(x_273); +x_274 = lean_ctor_get(x_258, 1); +lean_inc(x_274); +if (lean_is_exclusive(x_258)) { + lean_ctor_release(x_258, 0); + lean_ctor_release(x_258, 1); + x_275 = x_258; } else { - lean_dec_ref(x_243); - x_260 = lean_box(0); + lean_dec_ref(x_258); + x_275 = lean_box(0); } -if (lean_is_scalar(x_260)) { - x_261 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_275)) { + x_276 = lean_alloc_ctor(1, 2, 0); } else { - x_261 = x_260; + x_276 = x_275; } -lean_ctor_set(x_261, 0, x_258); -lean_ctor_set(x_261, 1, x_259); -return x_261; +lean_ctor_set(x_276, 0, x_273); +lean_ctor_set(x_276, 1, x_274); +return x_276; } } else { -lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; -lean_dec(x_238); -lean_dec(x_230); -lean_dec(x_207); +lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; +lean_dec(x_253); +lean_dec(x_242); +lean_dec(x_219); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_262 = lean_ctor_get(x_240, 0); -lean_inc(x_262); -x_263 = lean_ctor_get(x_240, 1); -lean_inc(x_263); -if (lean_is_exclusive(x_240)) { - lean_ctor_release(x_240, 0); - lean_ctor_release(x_240, 1); - x_264 = x_240; +x_277 = lean_ctor_get(x_255, 0); +lean_inc(x_277); +x_278 = lean_ctor_get(x_255, 1); +lean_inc(x_278); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_279 = x_255; } else { - lean_dec_ref(x_240); - x_264 = lean_box(0); + lean_dec_ref(x_255); + x_279 = lean_box(0); } -if (lean_is_scalar(x_264)) { - x_265 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_279)) { + x_280 = lean_alloc_ctor(1, 2, 0); } else { - x_265 = x_264; + x_280 = x_279; } -lean_ctor_set(x_265, 0, x_262); -lean_ctor_set(x_265, 1, x_263); -return x_265; +lean_ctor_set(x_280, 0, x_277); +lean_ctor_set(x_280, 1, x_278); +return x_280; } } else { -lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; -lean_dec(x_230); -lean_dec(x_207); +lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; +lean_dec(x_242); +lean_dec(x_219); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_266 = lean_ctor_get(x_237, 0); -lean_inc(x_266); -x_267 = lean_ctor_get(x_237, 1); -lean_inc(x_267); -if (lean_is_exclusive(x_237)) { - lean_ctor_release(x_237, 0); - lean_ctor_release(x_237, 1); - x_268 = x_237; +x_281 = lean_ctor_get(x_252, 0); +lean_inc(x_281); +x_282 = lean_ctor_get(x_252, 1); +lean_inc(x_282); +if (lean_is_exclusive(x_252)) { + lean_ctor_release(x_252, 0); + lean_ctor_release(x_252, 1); + x_283 = x_252; } else { - lean_dec_ref(x_237); - x_268 = lean_box(0); + lean_dec_ref(x_252); + x_283 = lean_box(0); } -if (lean_is_scalar(x_268)) { - x_269 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_283)) { + x_284 = lean_alloc_ctor(1, 2, 0); } else { - x_269 = x_268; + x_284 = x_283; } -lean_ctor_set(x_269, 0, x_266); -lean_ctor_set(x_269, 1, x_267); -return x_269; +lean_ctor_set(x_284, 0, x_281); +lean_ctor_set(x_284, 1, x_282); +return x_284; } } } else { -lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; -lean_dec(x_207); +lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; +lean_dec(x_219); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -15076,32 +15179,32 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_270 = lean_ctor_get(x_212, 0); -lean_inc(x_270); -x_271 = lean_ctor_get(x_212, 1); -lean_inc(x_271); -if (lean_is_exclusive(x_212)) { - lean_ctor_release(x_212, 0); - lean_ctor_release(x_212, 1); - x_272 = x_212; +x_285 = lean_ctor_get(x_224, 0); +lean_inc(x_285); +x_286 = lean_ctor_get(x_224, 1); +lean_inc(x_286); +if (lean_is_exclusive(x_224)) { + lean_ctor_release(x_224, 0); + lean_ctor_release(x_224, 1); + x_287 = x_224; } else { - lean_dec_ref(x_212); - x_272 = lean_box(0); + lean_dec_ref(x_224); + x_287 = lean_box(0); } -if (lean_is_scalar(x_272)) { - x_273 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_287)) { + x_288 = lean_alloc_ctor(1, 2, 0); } else { - x_273 = x_272; + x_288 = x_287; } -lean_ctor_set(x_273, 0, x_270); -lean_ctor_set(x_273, 1, x_271); -return x_273; +lean_ctor_set(x_288, 0, x_285); +lean_ctor_set(x_288, 1, x_286); +return x_288; } } else { -lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; -lean_dec(x_207); +lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; +lean_dec(x_219); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -15110,31 +15213,31 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_274 = lean_ctor_get(x_210, 0); -lean_inc(x_274); -x_275 = lean_ctor_get(x_210, 1); -lean_inc(x_275); -if (lean_is_exclusive(x_210)) { - lean_ctor_release(x_210, 0); - lean_ctor_release(x_210, 1); - x_276 = x_210; +x_289 = lean_ctor_get(x_222, 0); +lean_inc(x_289); +x_290 = lean_ctor_get(x_222, 1); +lean_inc(x_290); +if (lean_is_exclusive(x_222)) { + lean_ctor_release(x_222, 0); + lean_ctor_release(x_222, 1); + x_291 = x_222; } else { - lean_dec_ref(x_210); - x_276 = lean_box(0); + lean_dec_ref(x_222); + x_291 = lean_box(0); } -if (lean_is_scalar(x_276)) { - x_277 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_291)) { + x_292 = lean_alloc_ctor(1, 2, 0); } else { - x_277 = x_276; + x_292 = x_291; } -lean_ctor_set(x_277, 0, x_274); -lean_ctor_set(x_277, 1, x_275); -return x_277; +lean_ctor_set(x_292, 0, x_289); +lean_ctor_set(x_292, 1, x_290); +return x_292; } } else { -lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; +lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -15143,26 +15246,26 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_278 = lean_ctor_get(x_206, 0); -lean_inc(x_278); -x_279 = lean_ctor_get(x_206, 1); -lean_inc(x_279); -if (lean_is_exclusive(x_206)) { - lean_ctor_release(x_206, 0); - lean_ctor_release(x_206, 1); - x_280 = x_206; +x_293 = lean_ctor_get(x_218, 0); +lean_inc(x_293); +x_294 = lean_ctor_get(x_218, 1); +lean_inc(x_294); +if (lean_is_exclusive(x_218)) { + lean_ctor_release(x_218, 0); + lean_ctor_release(x_218, 1); + x_295 = x_218; } else { - lean_dec_ref(x_206); - x_280 = lean_box(0); + lean_dec_ref(x_218); + x_295 = lean_box(0); } -if (lean_is_scalar(x_280)) { - x_281 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_295)) { + x_296 = lean_alloc_ctor(1, 2, 0); } else { - x_281 = x_280; + x_296 = x_295; } -lean_ctor_set(x_281, 0, x_278); -lean_ctor_set(x_281, 1, x_279); -return x_281; +lean_ctor_set(x_296, 0, x_293); +lean_ctor_set(x_296, 1, x_294); +return x_296; } } } @@ -20374,7 +20477,7 @@ static lean_object* _init_l___private_Lean_Elab_Structure_0__Lean_Elab_Command_a 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_addCtorFields___closed__1; x_2 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addCtorFields___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_addCtorFields___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -23486,7 +23589,7 @@ lean_inc(x_15); lean_dec(x_14); x_16 = l_Lean_Expr_const___override(x_15, x_12); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_4, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_17); x_19 = l___private_Lean_Elab_Structure_0__Lean_Elab_Command_getFieldType___lambda__2___closed__3; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -25775,7 +25878,9 @@ lean_inc(x_89); lean_dec(x_64); x_90 = 0; lean_inc(x_15); -lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); lean_inc(x_10); x_91 = l_Lean_Elab_Term_applyAttributesAt(x_58, x_89, x_90, x_10, x_11, x_12, x_13, x_14, x_15, x_88); lean_dec(x_89); @@ -30017,7 +30122,7 @@ lean_dec(x_8); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_12385_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_12391_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -30742,7 +30847,7 @@ l_Lean_Elab_Command_elabStructure___closed__12 = _init_l_Lean_Elab_Command_elabS lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__12); l_Lean_Elab_Command_elabStructure___closed__13 = _init_l_Lean_Elab_Command_elabStructure___closed__13(); lean_mark_persistent(l_Lean_Elab_Command_elabStructure___closed__13); -res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_12385_(lean_io_mk_world()); +res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Structure___hyg_12391_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/Syntax.c b/stage0/stdlib/Lean/Elab/Syntax.c index 4edd9787e5f5..d7abe169c2c3 100644 --- a/stage0/stdlib/Lean/Elab/Syntax.c +++ b/stage0/stdlib/Lean/Elab/Syntax.c @@ -45,6 +45,7 @@ static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyn lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Elab_Command_resolveSyntaxKind___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_toParserDescr_processSeq___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__34; static lean_object* l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__7; lean_object* lean_mk_empty_array_with_capacity(lean_object*); @@ -56,7 +57,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Command_expandNoKindMacroRulesAux(lean_obje LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntaxAbbrev___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Term_toParserDescr_process___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_sequenceMap___at_Lean_Elab_Command_elabSyntax___spec__2___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_filterTRAux___at_Lean_resolveGlobalConstCore___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_checkLeftRec___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_toParserDescr_processAlias___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -130,6 +131,7 @@ uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclareSyntaxCat___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstWithInfos___at_Lean_Elab_Term_toParserDescr_processNullaryOrCat___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Term_toParserDescr_processNullaryOrCat___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__7___boxed(lean_object**); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__18; lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__2(lean_object*); @@ -140,7 +142,7 @@ uint8_t l_Char_isDigit(uint32_t); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Term_checkLeftRec___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__30; static lean_object* l_Lean_Elab_Term_toParserDescr_processSepBy1___lambda__1___closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__78; uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_toParserDescr_process___closed__5; @@ -178,7 +180,7 @@ lean_object* l_Lean_MessageData_ofList(lean_object*); static lean_object* l_panic___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_inferMacroRulesAltKind___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Term_toParserDescr_processNonReserved___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__33; uint8_t l_Char_isWhitespace(uint32_t); LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at_Lean_Elab_Term_toParserDescr_processNullaryOrCat___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -296,6 +298,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Term_checkLeftRec uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_toParserDescr_processNonReserved___closed__8; LEAN_EXPORT lean_object* l_Array_sequenceMap_loop___at_Lean_Elab_Command_elabSyntax___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Syntax_TSepArray_push___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__19; lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); @@ -343,7 +346,7 @@ static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyn lean_object* l_Lean_Unhygienic_run___rarg(lean_object*); lean_object* l_String_capitalize(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ensureUnaryOutput(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9219_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464_(lean_object*); static lean_object* l_Lean_Elab_Term_toParserDescr_process___closed__13; static lean_object* l_Lean_Elab_Term_toParserDescr_processNonReserved___closed__7; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expandNoKindMacroRulesAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -354,7 +357,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveParserName___rarg___lambda__3(l lean_object* l_instInhabited___rarg(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclareSyntaxCat_declRange___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Command_strLitToPattern___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__8; static lean_object* l_Lean_addTrace___at_Lean_Elab_Term_checkLeftRec___spec__3___closed__5; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Command_elabSyntax___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); @@ -374,6 +376,7 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Term_toParserDescr_processAlias_ static lean_object* l_panic___at_Lean_Elab_Term_toParserDescr_processAlias___spec__2___closed__1; static lean_object* l_Lean_Elab_Term_toParserDescr_processAlias___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Term_withNestedParser(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Command_elabSyntax___lambda__5___closed__13; lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__1; lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -469,6 +472,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Command_expand static lean_object* l_Lean_Elab_Term_toParserDescr_processSepBy___lambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSyntaxAbbrev___closed__3; static lean_object* l_Lean_Elab_Term_toParserDescr_process___closed__10; +lean_object* l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Command_elabSyntax___lambda__5___closed__8; static lean_object* l_Lean_Elab_Term_toParserDescr_processParserCategory___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -487,7 +491,7 @@ lean_object* l_Lean_Parser_ensureUnaryParserAlias(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__43; static lean_object* l_Lean_Elab_Command_expandNoKindMacroRulesAux___lambda__1___closed__4; lean_object* l_Lean_mkAtomFrom(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__11(lean_object*, lean_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_elabSyntaxAbbrev___closed__1; static lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__15; lean_object* l_Lean_Syntax_mkNumLit(lean_object*, lean_object*); @@ -552,6 +556,7 @@ static lean_object* l_Lean_Elab_Term_checkLeftRec___lambda__2___closed__4; lean_object* l_Lean_Parser_ensureConstantParserAlias(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Term_checkLeftRec___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1(lean_object*, lean_object*); +lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Command_elabSyntax___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_toParserDescr_processNonReserved___closed__15; static lean_object* l_Lean_Elab_Term_toParserDescr_processNonReserved___closed__3; @@ -599,6 +604,7 @@ static lean_object* l_Lean_addTrace___at_Lean_Elab_Term_checkLeftRec___spec__3__ lean_object* l_Lean_Elab_Command_getMainModule___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_toParserDescr_process___closed__7; lean_object* l_Lean_Parser_isParserAlias(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__5___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Term_checkLeftRec___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSyntax_declRange___closed__1; @@ -641,12 +647,14 @@ LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstWithInfos___at_Lean_Elab_ static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__53; lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__8___rarg(lean_object*); +static lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464____closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSyntaxAbbrev_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntaxAbbrev(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_String_trim(lean_object*); static lean_object* l_Lean_Elab_Term_toParserDescr_processAlias___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Command_elabDeclareSyntaxCat_declRange___closed__3; static lean_object* l_Lean_Elab_Term_toParserDescr_processParserCategory___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__6___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Elab_Term_expandOptPrecedence(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_toParserDescr_isValidAtom___boxed(lean_object*); uint8_t l_Lean_isIdFirst(uint32_t); @@ -661,7 +669,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveParserName(lean_object*); lean_object* l_Lean_Elab_Term_elabBinders___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__3___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_toParserDescr_process___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__55; static lean_object* l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__5; static lean_object* l_Lean_Elab_Command_elabSyntax___lambda__4___closed__1; @@ -683,7 +690,6 @@ static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyn static lean_object* l_Lean_Elab_Term_toParserDescr_process___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__8___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq(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_Syntax___hyg_9219____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__12___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__77; static lean_object* l_Lean_Elab_Command_expandNoKindMacroRulesAux___lambda__1___closed__1; @@ -693,7 +699,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveParserName___at_Lean_Elab_Term_ static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_checkLeftRec___spec__7___closed__2; uint8_t l_List_isEmpty___rarg(lean_object*); static lean_object* l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__13; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_inferMacroRulesAltKind___spec__2___boxed(lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getScope___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Term_checkLeftRec___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -709,7 +715,7 @@ static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyn static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__10; static lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Command_elabSyntaxAbbrev_declRange___closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__73; LEAN_EXPORT lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Term_withNotFirst___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__56; @@ -767,7 +773,7 @@ static lean_object* l_Lean_Elab_Command_expandNoKindMacroRulesAux___lambda__1___ LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_mkUnusedBaseName(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___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_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___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*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_toParserDescr_processNonReserved___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1363,7 +1369,7 @@ static lean_object* _init_l___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParse 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_Syntax_0__Lean_Elab_Term_mkParserSeq___closed__4; x_2 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___closed__5; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9726,7 +9732,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -9771,7 +9777,7 @@ lean_dec(x_24); x_26 = lean_st_ref_take(x_5, x_25); x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -x_28 = lean_ctor_get(x_27, 4); +x_28 = lean_ctor_get(x_27, 5); lean_inc(x_28); x_29 = lean_ctor_get(x_26, 1); lean_inc(x_29); @@ -9780,7 +9786,7 @@ x_30 = !lean_is_exclusive(x_27); if (x_30 == 0) { lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_27, 4); +x_31 = lean_ctor_get(x_27, 5); lean_dec(x_31); x_32 = !lean_is_exclusive(x_28); if (x_32 == 0) @@ -9827,7 +9833,7 @@ x_46 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_46, 0, x_43); lean_ctor_set(x_46, 1, x_45); lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_42); -lean_ctor_set(x_27, 4, x_46); +lean_ctor_set(x_27, 5, x_46); x_47 = lean_st_ref_set(x_5, x_27, x_29); x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); @@ -9852,64 +9858,67 @@ return x_51; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; x_52 = lean_ctor_get(x_27, 0); x_53 = lean_ctor_get(x_27, 1); x_54 = lean_ctor_get(x_27, 2); x_55 = lean_ctor_get(x_27, 3); +x_56 = lean_ctor_get(x_27, 4); +lean_inc(x_56); lean_inc(x_55); lean_inc(x_54); lean_inc(x_53); lean_inc(x_52); lean_dec(x_27); -x_56 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); -x_57 = lean_ctor_get(x_28, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_28, 1); +x_57 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); +x_58 = lean_ctor_get(x_28, 0); lean_inc(x_58); +x_59 = lean_ctor_get(x_28, 1); +lean_inc(x_59); if (lean_is_exclusive(x_28)) { lean_ctor_release(x_28, 0); lean_ctor_release(x_28, 1); - x_59 = x_28; + x_60 = x_28; } else { lean_dec_ref(x_28); - x_59 = lean_box(0); + x_60 = lean_box(0); } -x_60 = l_Std_PersistentArray_push___rarg(x_58, x_1); -if (lean_is_scalar(x_59)) { - x_61 = lean_alloc_ctor(0, 2, 1); +x_61 = l_Std_PersistentArray_push___rarg(x_59, x_1); +if (lean_is_scalar(x_60)) { + x_62 = lean_alloc_ctor(0, 2, 1); } else { - x_61 = x_59; + x_62 = x_60; } -lean_ctor_set(x_61, 0, x_57); -lean_ctor_set(x_61, 1, x_60); -lean_ctor_set_uint8(x_61, sizeof(void*)*2, x_56); -x_62 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_62, 0, x_52); -lean_ctor_set(x_62, 1, x_53); -lean_ctor_set(x_62, 2, x_54); -lean_ctor_set(x_62, 3, x_55); -lean_ctor_set(x_62, 4, x_61); -x_63 = lean_st_ref_set(x_5, x_62, x_29); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; +lean_ctor_set(x_62, 0, x_58); +lean_ctor_set(x_62, 1, x_61); +lean_ctor_set_uint8(x_62, sizeof(void*)*2, x_57); +x_63 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_63, 0, x_52); +lean_ctor_set(x_63, 1, x_53); +lean_ctor_set(x_63, 2, x_54); +lean_ctor_set(x_63, 3, x_55); +lean_ctor_set(x_63, 4, x_56); +lean_ctor_set(x_63, 5, x_62); +x_64 = lean_st_ref_set(x_5, x_63, x_29); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_66 = x_64; } else { - lean_dec_ref(x_63); - x_65 = lean_box(0); + lean_dec_ref(x_64); + x_66 = lean_box(0); } -x_66 = lean_box(0); -if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 0); +x_67 = lean_box(0); +if (lean_is_scalar(x_66)) { + x_68 = lean_alloc_ctor(0, 2, 0); } else { - x_67 = x_65; + x_68 = x_66; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_64); -return x_67; +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_68, 1, x_65); +return x_68; } } } @@ -9961,7 +9970,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -10132,7 +10141,7 @@ lean_dec(x_15); x_17 = lean_st_ref_get(x_6, x_16); x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); -x_19 = lean_ctor_get(x_18, 4); +x_19 = lean_ctor_get(x_18, 5); lean_inc(x_19); lean_dec(x_18); x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*2); @@ -15559,7 +15568,7 @@ x_53 = lean_ctor_get(x_44, 1); lean_inc(x_53); lean_dec(x_44); x_54 = l_List_reverse___rarg(x_53); -x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_54, x_2, x_3, x_52); +x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_54, x_2, x_3, x_52); lean_dec(x_3); lean_dec(x_2); x_56 = !lean_is_exclusive(x_55); @@ -15621,7 +15630,7 @@ x_71 = lean_ctor_get(x_44, 1); lean_inc(x_71); lean_dec(x_44); x_72 = l_List_reverse___rarg(x_71); -x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_2, x_3, x_70); +x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_72, x_2, x_3, x_70); lean_dec(x_3); lean_dec(x_2); x_74 = lean_ctor_get(x_73, 1); @@ -15912,7 +15921,7 @@ x_53 = lean_ctor_get(x_44, 1); lean_inc(x_53); lean_dec(x_44); x_54 = l_List_reverse___rarg(x_53); -x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_54, x_2, x_3, x_52); +x_55 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_54, x_2, x_3, x_52); lean_dec(x_3); lean_dec(x_2); x_56 = !lean_is_exclusive(x_55); @@ -15974,7 +15983,7 @@ x_71 = lean_ctor_get(x_44, 1); lean_inc(x_71); lean_dec(x_44); x_72 = l_List_reverse___rarg(x_71); -x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__5(x_72, x_2, x_3, x_70); +x_73 = l_List_forM___at_Lean_Elab_Command_elabCommand___spec__9(x_72, x_2, x_3, x_70); lean_dec(x_3); lean_dec(x_2); x_74 = lean_ctor_get(x_73, 1); @@ -16324,7 +16333,7 @@ x_17 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_17, 0, x_2); lean_inc(x_4); lean_inc(x_3); -x_18 = l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__15(x_13, x_17, x_3, x_4, x_8); +x_18 = l_Lean_logTrace___at_Lean_Elab_Command_elabCommand___spec__19(x_13, x_17, x_3, x_4, x_8); x_19 = lean_ctor_get(x_18, 1); lean_inc(x_19); lean_dec(x_18); @@ -16340,26 +16349,34 @@ static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__1 _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("ParserDescr.node", 16); +x_1 = lean_mk_string_from_bytes(",", 1); return x_1; } } static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__2() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("ParserDescr.node", 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__3() { +_start: +{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__1; +x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__2; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__1; +x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__2; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__2; +x_3 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__3; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16367,7 +16384,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__4() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -16377,7 +16394,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__5() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__6() { _start: { lean_object* x_1; @@ -16385,22 +16402,22 @@ x_1 = lean_mk_string_from_bytes("Lean.TrailingParserDescr", 24); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__6() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__5; +x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__6; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__7() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__5; +x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__6; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__6; +x_3 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__7; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16408,7 +16425,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__8() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__9() { _start: { lean_object* x_1; @@ -16416,22 +16433,22 @@ x_1 = lean_mk_string_from_bytes("ParserDescr.trailingNode", 24); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__9() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__8; +x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__9; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__10() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__8; +x_1 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__9; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__9; +x_3 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__10; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16439,7 +16456,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__11() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12() { _start: { lean_object* x_1; @@ -16447,1489 +16464,805 @@ x_1 = lean_mk_string_from_bytes("trailingNode", 12); return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__13; -x_2 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__11; +x_2 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -lean_object* x_17; lean_object* x_18; -x_17 = lean_alloc_closure((void*)(l_Lean_evalOptPrio), 3, 1); -lean_closure_set(x_17, 0, x_1); +lean_object* x_18; lean_object* x_19; +x_18 = lean_alloc_closure((void*)(l_Lean_evalOptPrio), 3, 1); +lean_closure_set(x_18, 0, x_1); +lean_inc(x_16); lean_inc(x_15); -lean_inc(x_14); -x_18 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabSyntax___spec__4(x_17, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_19 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabSyntax___spec__4(x_18, x_15, x_16, x_17); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_Elab_Command_getScope___rarg(x_15, x_20); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l_Lean_Elab_Command_getScope___rarg(x_16, x_21); +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_ctor_get(x_22, 2); +x_24 = lean_ctor_get(x_22, 1); lean_inc(x_24); lean_dec(x_22); -lean_inc(x_13); -x_25 = l_Lean_Name_append(x_24, x_13); -lean_dec(x_24); -x_26 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__3; +x_25 = lean_ctor_get(x_23, 2); +lean_inc(x_25); +lean_dec(x_23); +lean_inc(x_14); +x_26 = l_Lean_Name_append(x_25, x_14); +lean_dec(x_25); +x_27 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__3; lean_inc(x_2); -x_27 = lean_name_append_after(x_2, x_26); +x_28 = lean_name_append_after(x_2, x_27); lean_inc(x_3); -x_28 = l_Lean_mkIdentFrom(x_3, x_27); -x_29 = lean_box(0); -x_30 = l_Lean_Elab_Command_getScope___rarg(x_15, x_23); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); +x_29 = l_Lean_mkIdentFrom(x_3, x_28); +x_30 = lean_box(0); +x_31 = l_Lean_Elab_Command_getScope___rarg(x_16, x_24); +x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); -lean_dec(x_30); -x_33 = lean_ctor_get(x_31, 5); +x_33 = lean_ctor_get(x_31, 1); lean_inc(x_33); -x_34 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabSyntax___lambda__3___boxed), 11, 3); -lean_closure_set(x_34, 0, x_31); -lean_closure_set(x_34, 1, x_4); -lean_closure_set(x_34, 2, x_2); -x_35 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); -lean_closure_set(x_35, 0, x_33); -lean_closure_set(x_35, 1, x_34); -x_36 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withAutoBoundImplicit___rarg), 8, 1); -lean_closure_set(x_36, 0, x_35); -lean_inc(x_14); -x_37 = l_Lean_Elab_Command_liftTermElabM___rarg(x_29, x_36, x_14, x_15, x_32); -if (lean_obj_tag(x_37) == 0) +lean_dec(x_31); +x_34 = lean_ctor_get(x_32, 5); +lean_inc(x_34); +x_35 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabSyntax___lambda__3___boxed), 11, 3); +lean_closure_set(x_35, 0, x_32); +lean_closure_set(x_35, 1, x_4); +lean_closure_set(x_35, 2, x_2); +x_36 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); +lean_closure_set(x_36, 0, x_34); +lean_closure_set(x_36, 1, x_35); +x_37 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withAutoBoundImplicit___rarg), 8, 1); +lean_closure_set(x_37, 0, x_36); +lean_inc(x_15); +x_38 = l_Lean_Elab_Command_liftTermElabM___rarg(x_30, x_37, x_15, x_16, x_33); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_38; lean_object* x_39; uint8_t x_40; -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; 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; +x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); -lean_dec(x_37); -x_40 = !lean_is_exclusive(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_38, 0); -x_42 = lean_ctor_get(x_38, 1); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = lean_ctor_get(x_39, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_39, 1); +lean_inc(x_42); +if (lean_is_exclusive(x_39)) { + lean_ctor_release(x_39, 0); + lean_ctor_release(x_39, 1); + x_43 = x_39; +} else { + lean_dec_ref(x_39); + x_43 = lean_box(0); +} lean_inc(x_3); -x_43 = l_Lean_mkIdentFrom(x_3, x_13); -if (lean_obj_tag(x_42) == 0) -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_44 = l_Lean_MonadRef_mkInfoFromRefPos___at___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___spec__1(x_14, x_15, x_39); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); +x_44 = l_Lean_mkIdentFrom(x_3, x_14); +x_45 = l_Lean_MonadRef_mkInfoFromRefPos___at___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___spec__1(x_15, x_16, x_40); +x_46 = lean_ctor_get(x_45, 1); lean_inc(x_46); -lean_dec(x_44); -x_47 = l_Lean_Elab_Command_getCurrMacroScope(x_14, x_15, x_46); -x_48 = lean_ctor_get(x_47, 0); +lean_dec(x_45); +x_47 = l_Lean_Elab_Command_getCurrMacroScope(x_15, x_16, x_46); +x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); -lean_inc(x_49); lean_dec(x_47); -x_50 = l_Lean_Elab_Command_getMainModule___rarg(x_15, x_49); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -lean_dec(x_50); -x_53 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__7; +x_49 = l_Lean_Elab_Command_getMainModule___rarg(x_16, x_48); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +lean_dec(x_49); +x_51 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__15; lean_inc(x_5); -x_54 = l_Lean_Name_str___override(x_5, x_53); -x_55 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__9; +x_52 = l_Lean_Name_str___override(x_5, x_51); +x_53 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__21; +x_54 = l_Lean_Name_str___override(x_6, x_53); +x_55 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__23; +x_56 = l_Lean_Name_str___override(x_54, x_55); +x_57 = l_Nat_repr(x_20); +x_58 = lean_box(2); +x_59 = l_Lean_Syntax_mkNumLit(x_57, x_58); +x_60 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__27; +x_61 = lean_array_push(x_60, x_59); +lean_inc(x_7); +x_62 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_62, 0, x_58); +lean_ctor_set(x_62, 1, x_7); +lean_ctor_set(x_62, 2, x_61); +x_63 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__29; +x_64 = lean_array_push(x_63, x_29); +x_65 = lean_array_push(x_64, x_62); +x_66 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_66, 0, x_58); +lean_ctor_set(x_66, 1, x_56); +lean_ctor_set(x_66, 2, x_65); +x_67 = lean_array_push(x_63, x_8); +x_68 = lean_array_push(x_67, x_66); +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_58); +lean_ctor_set(x_69, 1, x_52); +lean_ctor_set(x_69, 2, x_68); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_369; +x_369 = l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__3; +x_70 = x_369; +goto block_368; +} +else +{ +lean_object* x_370; +x_370 = lean_ctor_get(x_13, 0); +lean_inc(x_370); +lean_dec(x_13); +x_70 = x_370; +goto block_368; +} +block_368: +{ +lean_object* x_71; lean_object* x_72; +x_71 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__1; +x_72 = l_Lean_Syntax_TSepArray_push___rarg(x_71, x_70, x_69); +if (lean_obj_tag(x_42) == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_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; +x_73 = l_Lean_MonadRef_mkInfoFromRefPos___at___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___spec__1(x_15, x_16, x_50); +x_74 = lean_ctor_get(x_73, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_73, 1); +lean_inc(x_75); +lean_dec(x_73); +x_76 = l_Lean_Elab_Command_getCurrMacroScope(x_15, x_16, x_75); +x_77 = lean_ctor_get(x_76, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_76, 1); +lean_inc(x_78); +lean_dec(x_76); +x_79 = l_Lean_Elab_Command_getMainModule___rarg(x_16, x_78); +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +lean_dec(x_79); +x_82 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__7; +lean_inc(x_9); +x_83 = l_Lean_Name_str___override(x_9, x_82); +x_84 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__9; +lean_inc(x_9); +x_85 = l_Lean_Name_str___override(x_9, x_84); +x_86 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; lean_inc(x_5); -x_56 = l_Lean_Name_str___override(x_5, x_55); -x_57 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; -lean_inc(x_6); -x_58 = l_Lean_Name_str___override(x_6, x_57); -x_59 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__14; -lean_inc(x_45); -x_60 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_60, 0, x_45); -lean_ctor_set(x_60, 1, x_59); -x_61 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__15; -lean_inc(x_6); -x_62 = l_Lean_Name_str___override(x_6, x_61); -x_63 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__21; -x_64 = l_Lean_Name_str___override(x_7, x_63); -x_65 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__23; -x_66 = l_Lean_Name_str___override(x_64, x_65); -x_67 = l_Nat_repr(x_19); -x_68 = lean_box(2); -x_69 = l_Lean_Syntax_mkNumLit(x_67, x_68); -x_70 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__27; -x_71 = lean_array_push(x_70, x_69); -lean_inc(x_8); -x_72 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_72, 0, x_68); -lean_ctor_set(x_72, 1, x_8); -lean_ctor_set(x_72, 2, x_71); -x_73 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__29; -x_74 = lean_array_push(x_73, x_28); -x_75 = lean_array_push(x_74, x_72); -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_68); -lean_ctor_set(x_76, 1, x_66); -lean_ctor_set(x_76, 2, x_75); -x_77 = lean_array_push(x_73, x_9); -x_78 = lean_array_push(x_77, x_76); -x_79 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_79, 0, x_68); -lean_ctor_set(x_79, 1, x_62); -lean_ctor_set(x_79, 2, x_78); -x_80 = lean_array_push(x_70, x_79); -lean_inc(x_8); -x_81 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_81, 0, x_68); -lean_ctor_set(x_81, 1, x_8); -lean_ctor_set(x_81, 2, x_80); -x_82 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__30; -lean_inc(x_45); -x_83 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_83, 0, x_45); -lean_ctor_set(x_83, 1, x_82); -x_84 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__28; -x_85 = lean_array_push(x_84, x_60); -x_86 = lean_array_push(x_85, x_81); -x_87 = lean_array_push(x_86, x_83); -x_88 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_88, 0, x_68); -lean_ctor_set(x_88, 1, x_58); -lean_ctor_set(x_88, 2, x_87); -x_89 = lean_array_push(x_70, x_88); -lean_inc(x_8); -x_90 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_90, 0, x_68); -lean_ctor_set(x_90, 1, x_8); -lean_ctor_set(x_90, 2, x_89); -x_91 = l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__3; -lean_inc(x_8); +x_87 = l_Lean_Name_str___override(x_5, x_86); +x_88 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__14; +lean_inc(x_74); +x_89 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_89, 0, x_74); +lean_ctor_set(x_89, 1, x_88); +x_90 = l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__3; +x_91 = l_Array_append___rarg(x_90, x_72); +lean_inc(x_7); x_92 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_92, 0, x_68); -lean_ctor_set(x_92, 1, x_8); +lean_ctor_set(x_92, 0, x_58); +lean_ctor_set(x_92, 1, x_7); lean_ctor_set(x_92, 2, x_91); -x_93 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__33; -lean_inc(x_5); -x_94 = l_Lean_Name_str___override(x_5, x_93); -lean_inc(x_45); -x_95 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_95, 0, x_45); -lean_ctor_set(x_95, 1, x_93); -x_96 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__35; +x_93 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__30; +lean_inc(x_74); +x_94 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_94, 0, x_74); +lean_ctor_set(x_94, 1, x_93); +x_95 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__28; +x_96 = lean_array_push(x_95, x_89); +x_97 = lean_array_push(x_96, x_92); +x_98 = lean_array_push(x_97, x_94); +x_99 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_99, 0, x_58); +lean_ctor_set(x_99, 1, x_87); +lean_ctor_set(x_99, 2, x_98); +x_100 = lean_array_push(x_60, x_99); +lean_inc(x_7); +x_101 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_101, 0, x_58); +lean_ctor_set(x_101, 1, x_7); +lean_ctor_set(x_101, 2, x_100); +lean_inc(x_7); +x_102 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_102, 0, x_58); +lean_ctor_set(x_102, 1, x_7); +lean_ctor_set(x_102, 2, x_90); +x_103 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__33; +lean_inc(x_9); +x_104 = l_Lean_Name_str___override(x_9, x_103); +lean_inc(x_74); +x_105 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_105, 0, x_74); +lean_ctor_set(x_105, 1, x_103); +x_106 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__35; +lean_inc(x_9); +x_107 = l_Lean_Name_str___override(x_9, x_106); +x_108 = lean_array_push(x_63, x_44); +lean_inc(x_102); +x_109 = lean_array_push(x_108, x_102); +x_110 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_110, 0, x_58); +lean_ctor_set(x_110, 1, x_107); +lean_ctor_set(x_110, 2, x_109); +x_111 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__37; +lean_inc(x_9); +x_112 = l_Lean_Name_str___override(x_9, x_111); +x_113 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__39; lean_inc(x_5); -x_97 = l_Lean_Name_str___override(x_5, x_96); -x_98 = lean_array_push(x_73, x_43); -lean_inc(x_92); -x_99 = lean_array_push(x_98, x_92); -x_100 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_100, 0, x_68); -lean_ctor_set(x_100, 1, x_97); -lean_ctor_set(x_100, 2, x_99); -x_101 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__37; +x_114 = l_Lean_Name_str___override(x_5, x_113); +x_115 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__41; +lean_inc(x_74); +x_116 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_116, 0, x_74); +lean_ctor_set(x_116, 1, x_115); +x_117 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__12; +x_118 = l_Lean_Name_str___override(x_10, x_117); +lean_inc(x_77); +lean_inc(x_118); +lean_inc(x_80); +x_119 = l_Lean_addMacroScope(x_80, x_118, x_77); +x_120 = lean_box(0); +lean_inc(x_118); +if (lean_is_scalar(x_43)) { + x_121 = lean_alloc_ctor(0, 2, 0); +} else { + x_121 = x_43; +} +lean_ctor_set(x_121, 0, x_118); +lean_ctor_set(x_121, 1, x_120); +x_122 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_122, 0, x_121); +lean_ctor_set(x_122, 1, x_120); +x_123 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__44; +lean_inc(x_74); +x_124 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_124, 0, x_74); +lean_ctor_set(x_124, 1, x_123); +lean_ctor_set(x_124, 2, x_119); +lean_ctor_set(x_124, 3, x_122); +x_125 = lean_array_push(x_63, x_116); +x_126 = lean_array_push(x_125, x_124); +x_127 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_127, 0, x_58); +lean_ctor_set(x_127, 1, x_114); +lean_ctor_set(x_127, 2, x_126); +x_128 = lean_array_push(x_60, x_127); +lean_inc(x_7); +x_129 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_129, 0, x_58); +lean_ctor_set(x_129, 1, x_7); +lean_ctor_set(x_129, 2, x_128); +lean_inc(x_102); +x_130 = lean_array_push(x_63, x_102); +x_131 = lean_array_push(x_130, x_129); +x_132 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_132, 0, x_58); +lean_ctor_set(x_132, 1, x_112); +lean_ctor_set(x_132, 2, x_131); +x_133 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__48; +x_134 = l_Lean_Name_str___override(x_9, x_133); +x_135 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__50; +lean_inc(x_74); +x_136 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_136, 0, x_74); +lean_ctor_set(x_136, 1, x_135); +x_137 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__7; lean_inc(x_5); -x_102 = l_Lean_Name_str___override(x_5, x_101); -x_103 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__39; -lean_inc(x_6); -x_104 = l_Lean_Name_str___override(x_6, x_103); -x_105 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__41; -lean_inc(x_45); -x_106 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_106, 0, x_45); -lean_ctor_set(x_106, 1, x_105); -x_107 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__12; -x_108 = l_Lean_Name_str___override(x_10, x_107); -lean_inc(x_48); -lean_inc(x_108); -lean_inc(x_51); -x_109 = l_Lean_addMacroScope(x_51, x_108, x_48); -x_110 = lean_box(0); -lean_inc(x_108); -lean_ctor_set(x_38, 1, x_110); -lean_ctor_set(x_38, 0, x_108); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_38); -lean_ctor_set(x_111, 1, x_110); -x_112 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__44; -lean_inc(x_45); -x_113 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_113, 0, x_45); -lean_ctor_set(x_113, 1, x_112); -lean_ctor_set(x_113, 2, x_109); -lean_ctor_set(x_113, 3, x_111); -x_114 = lean_array_push(x_73, x_106); -x_115 = lean_array_push(x_114, x_113); -x_116 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_116, 0, x_68); -lean_ctor_set(x_116, 1, x_104); -lean_ctor_set(x_116, 2, x_115); -x_117 = lean_array_push(x_70, x_116); -lean_inc(x_8); -x_118 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_118, 0, x_68); -lean_ctor_set(x_118, 1, x_8); -lean_ctor_set(x_118, 2, x_117); -lean_inc(x_92); -x_119 = lean_array_push(x_73, x_92); -x_120 = lean_array_push(x_119, x_118); -x_121 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_121, 0, x_68); -lean_ctor_set(x_121, 1, x_102); -lean_ctor_set(x_121, 2, x_120); -x_122 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__48; -x_123 = l_Lean_Name_str___override(x_5, x_122); -x_124 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__50; -lean_inc(x_45); -x_125 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_125, 0, x_45); -lean_ctor_set(x_125, 1, x_124); -x_126 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__7; -lean_inc(x_6); -x_127 = l_Lean_Name_str___override(x_6, x_126); -x_128 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__4; -x_129 = l_Lean_addMacroScope(x_51, x_128, x_48); -x_130 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__54; -x_131 = l_Lean_Name_str___override(x_108, x_130); -x_132 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_132, 0, x_131); -lean_ctor_set(x_132, 1, x_110); -x_133 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_133, 0, x_132); -lean_ctor_set(x_133, 1, x_110); -x_134 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__3; -x_135 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_135, 0, x_45); -lean_ctor_set(x_135, 1, x_134); -lean_ctor_set(x_135, 2, x_129); -lean_ctor_set(x_135, 3, x_133); -lean_inc(x_25); -x_136 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_110, x_25); -x_137 = l_Nat_repr(x_11); -x_138 = l_Lean_Syntax_mkNumLit(x_137, x_68); -x_139 = lean_array_push(x_73, x_135); -x_140 = lean_array_push(x_84, x_125); -x_141 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__85; -x_142 = lean_array_push(x_141, x_95); -x_143 = lean_array_push(x_142, x_100); -x_144 = lean_array_push(x_143, x_121); +x_138 = l_Lean_Name_str___override(x_5, x_137); +x_139 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__5; +x_140 = l_Lean_addMacroScope(x_80, x_139, x_77); +x_141 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__54; +x_142 = l_Lean_Name_str___override(x_118, x_141); +x_143 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_143, 0, x_142); +lean_ctor_set(x_143, 1, x_120); +x_144 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_120); +x_145 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__4; +x_146 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_146, 0, x_74); +lean_ctor_set(x_146, 1, x_145); +lean_ctor_set(x_146, 2, x_140); +lean_ctor_set(x_146, 3, x_144); +lean_inc(x_26); +x_147 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_120, x_26); +x_148 = l_Nat_repr(x_11); +x_149 = l_Lean_Syntax_mkNumLit(x_148, x_58); +x_150 = lean_array_push(x_63, x_146); +x_151 = lean_array_push(x_95, x_136); +x_152 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__85; +x_153 = lean_array_push(x_152, x_105); +x_154 = lean_array_push(x_153, x_110); +x_155 = lean_array_push(x_154, x_132); if (lean_obj_tag(x_12) == 0) { -x_145 = x_91; -goto block_202; +x_156 = x_90; +goto block_213; } else { -lean_object* x_203; lean_object* x_204; -x_203 = lean_ctor_get(x_12, 0); -lean_inc(x_203); +lean_object* x_214; lean_object* x_215; +x_214 = lean_ctor_get(x_12, 0); +lean_inc(x_214); lean_dec(x_12); -x_204 = lean_array_push(x_70, x_203); -x_145 = x_204; -goto block_202; +x_215 = lean_array_push(x_60, x_214); +x_156 = x_215; +goto block_213; } -block_202: +block_213: { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_146 = l_Array_append___rarg(x_91, x_145); -lean_inc(x_8); -x_147 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_147, 0, x_68); -lean_ctor_set(x_147, 1, x_8); -lean_ctor_set(x_147, 2, x_146); -x_148 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__31; -x_149 = lean_array_push(x_148, x_147); -x_150 = lean_array_push(x_149, x_90); -lean_inc(x_92); -x_151 = lean_array_push(x_150, x_92); -lean_inc(x_92); -x_152 = lean_array_push(x_151, x_92); -lean_inc(x_92); -x_153 = lean_array_push(x_152, x_92); -lean_inc(x_92); -x_154 = lean_array_push(x_153, x_92); -x_155 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_155, 0, x_68); -lean_ctor_set(x_155, 1, x_56); -lean_ctor_set(x_155, 2, x_154); -x_156 = lean_array_push(x_73, x_155); -if (lean_obj_tag(x_136) == 0) -{ -lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; 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_dec(x_6); -x_157 = l_Lean_quoteNameMk(x_25); -x_158 = lean_array_push(x_84, x_157); -x_159 = lean_array_push(x_158, x_138); -x_160 = lean_array_push(x_159, x_41); -x_161 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_161, 0, x_68); -lean_ctor_set(x_161, 1, x_8); -lean_ctor_set(x_161, 2, x_160); -x_162 = lean_array_push(x_139, x_161); -x_163 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_163, 0, x_68); -lean_ctor_set(x_163, 1, x_127); -lean_ctor_set(x_163, 2, x_162); -x_164 = lean_array_push(x_140, x_163); -lean_inc(x_92); -x_165 = lean_array_push(x_164, x_92); +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; +x_157 = l_Array_append___rarg(x_90, x_156); +lean_inc(x_7); +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_58); +lean_ctor_set(x_158, 1, x_7); +lean_ctor_set(x_158, 2, x_157); +x_159 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__31; +x_160 = lean_array_push(x_159, x_158); +x_161 = lean_array_push(x_160, x_101); +lean_inc(x_102); +x_162 = lean_array_push(x_161, x_102); +lean_inc(x_102); +x_163 = lean_array_push(x_162, x_102); +lean_inc(x_102); +x_164 = lean_array_push(x_163, x_102); +lean_inc(x_102); +x_165 = lean_array_push(x_164, x_102); x_166 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_166, 0, x_68); -lean_ctor_set(x_166, 1, x_123); +lean_ctor_set(x_166, 0, x_58); +lean_ctor_set(x_166, 1, x_85); lean_ctor_set(x_166, 2, x_165); -x_167 = lean_array_push(x_144, x_166); -lean_inc(x_92); -x_168 = lean_array_push(x_167, x_92); -lean_inc(x_92); -x_169 = lean_array_push(x_168, x_92); -x_170 = lean_array_push(x_169, x_92); -x_171 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_171, 0, x_68); -lean_ctor_set(x_171, 1, x_94); -lean_ctor_set(x_171, 2, x_170); -x_172 = lean_array_push(x_156, x_171); -x_173 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_173, 0, x_68); -lean_ctor_set(x_173, 1, x_54); -lean_ctor_set(x_173, 2, x_172); -x_174 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_173, x_14, x_15, x_52); -return x_174; -} -else +x_167 = lean_array_push(x_63, x_166); +if (lean_obj_tag(x_147) == 0) { -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; -lean_dec(x_25); -x_175 = lean_ctor_get(x_136, 0); -lean_inc(x_175); -lean_dec(x_136); -x_176 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__22; -x_177 = l_Lean_Name_str___override(x_6, x_176); -x_178 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__16; -x_179 = l_String_intercalate(x_178, x_175); -x_180 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__17; -x_181 = lean_string_append(x_180, x_179); -lean_dec(x_179); -x_182 = l_Lean_Syntax_mkNameLit(x_181, x_68); -x_183 = lean_array_push(x_70, x_182); +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_dec(x_5); +x_168 = l_Lean_quoteNameMk(x_26); +x_169 = lean_array_push(x_95, x_168); +x_170 = lean_array_push(x_169, x_149); +x_171 = lean_array_push(x_170, x_41); +x_172 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_172, 0, x_58); +lean_ctor_set(x_172, 1, x_7); +lean_ctor_set(x_172, 2, x_171); +x_173 = lean_array_push(x_150, x_172); +x_174 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_174, 0, x_58); +lean_ctor_set(x_174, 1, x_138); +lean_ctor_set(x_174, 2, x_173); +x_175 = lean_array_push(x_151, x_174); +lean_inc(x_102); +x_176 = lean_array_push(x_175, x_102); +x_177 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_177, 0, x_58); +lean_ctor_set(x_177, 1, x_134); +lean_ctor_set(x_177, 2, x_176); +x_178 = lean_array_push(x_155, x_177); +lean_inc(x_102); +x_179 = lean_array_push(x_178, x_102); +lean_inc(x_102); +x_180 = lean_array_push(x_179, x_102); +x_181 = lean_array_push(x_180, x_102); +x_182 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_182, 0, x_58); +lean_ctor_set(x_182, 1, x_104); +lean_ctor_set(x_182, 2, x_181); +x_183 = lean_array_push(x_167, x_182); x_184 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_184, 0, x_68); -lean_ctor_set(x_184, 1, x_177); +lean_ctor_set(x_184, 0, x_58); +lean_ctor_set(x_184, 1, x_83); lean_ctor_set(x_184, 2, x_183); -x_185 = lean_array_push(x_84, x_184); -x_186 = lean_array_push(x_185, x_138); -x_187 = lean_array_push(x_186, x_41); -x_188 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_188, 0, x_68); -lean_ctor_set(x_188, 1, x_8); -lean_ctor_set(x_188, 2, x_187); -x_189 = lean_array_push(x_139, x_188); -x_190 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_190, 0, x_68); -lean_ctor_set(x_190, 1, x_127); -lean_ctor_set(x_190, 2, x_189); -x_191 = lean_array_push(x_140, x_190); -lean_inc(x_92); -x_192 = lean_array_push(x_191, x_92); -x_193 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_193, 0, x_68); -lean_ctor_set(x_193, 1, x_123); -lean_ctor_set(x_193, 2, x_192); -x_194 = lean_array_push(x_144, x_193); -lean_inc(x_92); -x_195 = lean_array_push(x_194, x_92); -lean_inc(x_92); -x_196 = lean_array_push(x_195, x_92); -x_197 = lean_array_push(x_196, x_92); -x_198 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_198, 0, x_68); -lean_ctor_set(x_198, 1, x_94); -lean_ctor_set(x_198, 2, x_197); -x_199 = lean_array_push(x_156, x_198); -x_200 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_200, 0, x_68); -lean_ctor_set(x_200, 1, x_54); -lean_ctor_set(x_200, 2, x_199); -x_201 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_200, x_14, x_15, x_52); -return x_201; -} -} +x_185 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_184, x_15, x_16, x_81); +return x_185; } else { -lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; -x_205 = lean_ctor_get(x_42, 0); -lean_inc(x_205); -lean_dec(x_42); -x_206 = l_Lean_MonadRef_mkInfoFromRefPos___at___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___spec__1(x_14, x_15, x_39); -x_207 = lean_ctor_get(x_206, 0); -lean_inc(x_207); -x_208 = lean_ctor_get(x_206, 1); -lean_inc(x_208); -lean_dec(x_206); -x_209 = l_Lean_Elab_Command_getCurrMacroScope(x_14, x_15, x_208); -x_210 = lean_ctor_get(x_209, 0); -lean_inc(x_210); -x_211 = lean_ctor_get(x_209, 1); -lean_inc(x_211); -lean_dec(x_209); -x_212 = l_Lean_Elab_Command_getMainModule___rarg(x_15, x_211); -x_213 = lean_ctor_get(x_212, 0); -lean_inc(x_213); -x_214 = lean_ctor_get(x_212, 1); -lean_inc(x_214); -lean_dec(x_212); -x_215 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__7; -lean_inc(x_5); -x_216 = l_Lean_Name_str___override(x_5, x_215); -x_217 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__9; -lean_inc(x_5); -x_218 = l_Lean_Name_str___override(x_5, x_217); -x_219 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; -lean_inc(x_6); -x_220 = l_Lean_Name_str___override(x_6, x_219); -x_221 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__14; -lean_inc(x_207); -x_222 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_222, 0, x_207); -lean_ctor_set(x_222, 1, x_221); -x_223 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__15; -lean_inc(x_6); -x_224 = l_Lean_Name_str___override(x_6, x_223); -x_225 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__21; -x_226 = l_Lean_Name_str___override(x_7, x_225); -x_227 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__23; -x_228 = l_Lean_Name_str___override(x_226, x_227); -x_229 = l_Nat_repr(x_19); -x_230 = lean_box(2); -x_231 = l_Lean_Syntax_mkNumLit(x_229, x_230); -x_232 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__27; -x_233 = lean_array_push(x_232, x_231); -lean_inc(x_8); -x_234 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_234, 0, x_230); -lean_ctor_set(x_234, 1, x_8); -lean_ctor_set(x_234, 2, x_233); -x_235 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__29; -x_236 = lean_array_push(x_235, x_28); -x_237 = lean_array_push(x_236, x_234); -x_238 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_238, 0, x_230); -lean_ctor_set(x_238, 1, x_228); -lean_ctor_set(x_238, 2, x_237); -x_239 = lean_array_push(x_235, x_9); -x_240 = lean_array_push(x_239, x_238); -x_241 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_241, 0, x_230); -lean_ctor_set(x_241, 1, x_224); -lean_ctor_set(x_241, 2, x_240); -x_242 = lean_array_push(x_232, x_241); -lean_inc(x_8); -x_243 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_243, 0, x_230); -lean_ctor_set(x_243, 1, x_8); -lean_ctor_set(x_243, 2, x_242); -x_244 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__30; -lean_inc(x_207); -x_245 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_245, 0, x_207); -lean_ctor_set(x_245, 1, x_244); -x_246 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__28; -x_247 = lean_array_push(x_246, x_222); -x_248 = lean_array_push(x_247, x_243); -x_249 = lean_array_push(x_248, x_245); -x_250 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_250, 0, x_230); -lean_ctor_set(x_250, 1, x_220); -lean_ctor_set(x_250, 2, x_249); -x_251 = lean_array_push(x_232, x_250); -lean_inc(x_8); -x_252 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_252, 0, x_230); -lean_ctor_set(x_252, 1, x_8); -lean_ctor_set(x_252, 2, x_251); -x_253 = l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__3; -lean_inc(x_8); +lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; +lean_dec(x_26); +x_186 = lean_ctor_get(x_147, 0); +lean_inc(x_186); +lean_dec(x_147); +x_187 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__22; +x_188 = l_Lean_Name_str___override(x_5, x_187); +x_189 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__16; +x_190 = l_String_intercalate(x_189, x_186); +x_191 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__17; +x_192 = lean_string_append(x_191, x_190); +lean_dec(x_190); +x_193 = l_Lean_Syntax_mkNameLit(x_192, x_58); +x_194 = lean_array_push(x_60, x_193); +x_195 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_195, 0, x_58); +lean_ctor_set(x_195, 1, x_188); +lean_ctor_set(x_195, 2, x_194); +x_196 = lean_array_push(x_95, x_195); +x_197 = lean_array_push(x_196, x_149); +x_198 = lean_array_push(x_197, x_41); +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_58); +lean_ctor_set(x_199, 1, x_7); +lean_ctor_set(x_199, 2, x_198); +x_200 = lean_array_push(x_150, x_199); +x_201 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_201, 0, x_58); +lean_ctor_set(x_201, 1, x_138); +lean_ctor_set(x_201, 2, x_200); +x_202 = lean_array_push(x_151, x_201); +lean_inc(x_102); +x_203 = lean_array_push(x_202, x_102); +x_204 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_204, 0, x_58); +lean_ctor_set(x_204, 1, x_134); +lean_ctor_set(x_204, 2, x_203); +x_205 = lean_array_push(x_155, x_204); +lean_inc(x_102); +x_206 = lean_array_push(x_205, x_102); +lean_inc(x_102); +x_207 = lean_array_push(x_206, x_102); +x_208 = lean_array_push(x_207, x_102); +x_209 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_209, 0, x_58); +lean_ctor_set(x_209, 1, x_104); +lean_ctor_set(x_209, 2, x_208); +x_210 = lean_array_push(x_167, x_209); +x_211 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_211, 0, x_58); +lean_ctor_set(x_211, 1, x_83); +lean_ctor_set(x_211, 2, x_210); +x_212 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_211, x_15, x_16, x_81); +return x_212; +} +} +} +else +{ +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; +x_216 = lean_ctor_get(x_42, 0); +lean_inc(x_216); +lean_dec(x_42); +x_217 = l_Lean_MonadRef_mkInfoFromRefPos___at___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___spec__1(x_15, x_16, x_50); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +x_219 = lean_ctor_get(x_217, 1); +lean_inc(x_219); +lean_dec(x_217); +x_220 = l_Lean_Elab_Command_getCurrMacroScope(x_15, x_16, x_219); +x_221 = lean_ctor_get(x_220, 0); +lean_inc(x_221); +x_222 = lean_ctor_get(x_220, 1); +lean_inc(x_222); +lean_dec(x_220); +x_223 = l_Lean_Elab_Command_getMainModule___rarg(x_16, x_222); +x_224 = lean_ctor_get(x_223, 0); +lean_inc(x_224); +x_225 = lean_ctor_get(x_223, 1); +lean_inc(x_225); +lean_dec(x_223); +x_226 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__7; +lean_inc(x_9); +x_227 = l_Lean_Name_str___override(x_9, x_226); +x_228 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__9; +lean_inc(x_9); +x_229 = l_Lean_Name_str___override(x_9, x_228); +x_230 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; +lean_inc(x_5); +x_231 = l_Lean_Name_str___override(x_5, x_230); +x_232 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__14; +lean_inc(x_218); +x_233 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_233, 0, x_218); +lean_ctor_set(x_233, 1, x_232); +x_234 = l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__3; +x_235 = l_Array_append___rarg(x_234, x_72); +lean_inc(x_7); +x_236 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_236, 0, x_58); +lean_ctor_set(x_236, 1, x_7); +lean_ctor_set(x_236, 2, x_235); +x_237 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__30; +lean_inc(x_218); +x_238 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_238, 0, x_218); +lean_ctor_set(x_238, 1, x_237); +x_239 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__28; +x_240 = lean_array_push(x_239, x_233); +x_241 = lean_array_push(x_240, x_236); +x_242 = lean_array_push(x_241, x_238); +x_243 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_243, 0, x_58); +lean_ctor_set(x_243, 1, x_231); +lean_ctor_set(x_243, 2, x_242); +x_244 = lean_array_push(x_60, x_243); +lean_inc(x_7); +x_245 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_245, 0, x_58); +lean_ctor_set(x_245, 1, x_7); +lean_ctor_set(x_245, 2, x_244); +lean_inc(x_7); +x_246 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_246, 0, x_58); +lean_ctor_set(x_246, 1, x_7); +lean_ctor_set(x_246, 2, x_234); +x_247 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__33; +lean_inc(x_9); +x_248 = l_Lean_Name_str___override(x_9, x_247); +lean_inc(x_218); +x_249 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_249, 0, x_218); +lean_ctor_set(x_249, 1, x_247); +x_250 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__35; +lean_inc(x_9); +x_251 = l_Lean_Name_str___override(x_9, x_250); +x_252 = lean_array_push(x_63, x_44); +lean_inc(x_246); +x_253 = lean_array_push(x_252, x_246); x_254 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_254, 0, x_230); -lean_ctor_set(x_254, 1, x_8); +lean_ctor_set(x_254, 0, x_58); +lean_ctor_set(x_254, 1, x_251); lean_ctor_set(x_254, 2, x_253); -x_255 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__33; -lean_inc(x_5); -x_256 = l_Lean_Name_str___override(x_5, x_255); -lean_inc(x_207); -x_257 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_257, 0, x_207); -lean_ctor_set(x_257, 1, x_255); -x_258 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__35; -lean_inc(x_5); -x_259 = l_Lean_Name_str___override(x_5, x_258); -x_260 = lean_array_push(x_235, x_43); -lean_inc(x_254); -x_261 = lean_array_push(x_260, x_254); -x_262 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_262, 0, x_230); -lean_ctor_set(x_262, 1, x_259); -lean_ctor_set(x_262, 2, x_261); -x_263 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__37; +x_255 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__37; +lean_inc(x_9); +x_256 = l_Lean_Name_str___override(x_9, x_255); +x_257 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__39; lean_inc(x_5); -x_264 = l_Lean_Name_str___override(x_5, x_263); -x_265 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__39; -lean_inc(x_6); -x_266 = l_Lean_Name_str___override(x_6, x_265); -x_267 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__41; -lean_inc(x_207); -x_268 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_268, 0, x_207); -lean_ctor_set(x_268, 1, x_267); -x_269 = l_List_filterMap___at_Lean_Elab_Term_resolveParserName___spec__1___closed__1; +x_258 = l_Lean_Name_str___override(x_5, x_257); +x_259 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__41; +lean_inc(x_218); +x_260 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_260, 0, x_218); +lean_ctor_set(x_260, 1, x_259); +x_261 = l_List_filterMap___at_Lean_Elab_Term_resolveParserName___spec__1___closed__1; lean_inc(x_10); -x_270 = l_Lean_Name_str___override(x_10, x_269); -lean_inc(x_210); -lean_inc(x_270); -lean_inc(x_213); -x_271 = l_Lean_addMacroScope(x_213, x_270, x_210); -x_272 = lean_box(0); -lean_ctor_set(x_38, 1, x_272); -lean_ctor_set(x_38, 0, x_270); -x_273 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_273, 0, x_38); -lean_ctor_set(x_273, 1, x_272); -x_274 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__7; -lean_inc(x_207); -x_275 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_275, 0, x_207); -lean_ctor_set(x_275, 1, x_274); -lean_ctor_set(x_275, 2, x_271); -lean_ctor_set(x_275, 3, x_273); -x_276 = lean_array_push(x_235, x_268); -x_277 = lean_array_push(x_276, x_275); -x_278 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_278, 0, x_230); -lean_ctor_set(x_278, 1, x_266); -lean_ctor_set(x_278, 2, x_277); -x_279 = lean_array_push(x_232, x_278); -lean_inc(x_8); -x_280 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_280, 0, x_230); -lean_ctor_set(x_280, 1, x_8); -lean_ctor_set(x_280, 2, x_279); -lean_inc(x_254); -x_281 = lean_array_push(x_235, x_254); -x_282 = lean_array_push(x_281, x_280); -x_283 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_283, 0, x_230); -lean_ctor_set(x_283, 1, x_264); -lean_ctor_set(x_283, 2, x_282); -x_284 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__48; -x_285 = l_Lean_Name_str___override(x_5, x_284); -x_286 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__50; -lean_inc(x_207); -x_287 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_287, 0, x_207); -lean_ctor_set(x_287, 1, x_286); -x_288 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__7; -lean_inc(x_6); -x_289 = l_Lean_Name_str___override(x_6, x_288); -x_290 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12; -x_291 = l_Lean_addMacroScope(x_213, x_290, x_210); -x_292 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__12; -x_293 = l_Lean_Name_str___override(x_10, x_292); -x_294 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__11; -x_295 = l_Lean_Name_str___override(x_293, x_294); -x_296 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_296, 0, x_295); -lean_ctor_set(x_296, 1, x_272); -x_297 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_297, 0, x_296); -lean_ctor_set(x_297, 1, x_272); -x_298 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__10; -x_299 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_299, 0, x_207); -lean_ctor_set(x_299, 1, x_298); -lean_ctor_set(x_299, 2, x_291); -lean_ctor_set(x_299, 3, x_297); -lean_inc(x_25); -x_300 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_272, x_25); -x_301 = l_Nat_repr(x_11); -x_302 = l_Lean_Syntax_mkNumLit(x_301, x_230); -x_303 = l_Nat_repr(x_205); -x_304 = l_Lean_Syntax_mkNumLit(x_303, x_230); -x_305 = lean_array_push(x_235, x_299); -x_306 = lean_array_push(x_246, x_287); -x_307 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__85; -x_308 = lean_array_push(x_307, x_257); -x_309 = lean_array_push(x_308, x_262); -x_310 = lean_array_push(x_309, x_283); +x_262 = l_Lean_Name_str___override(x_10, x_261); +lean_inc(x_221); +lean_inc(x_262); +lean_inc(x_224); +x_263 = l_Lean_addMacroScope(x_224, x_262, x_221); +x_264 = lean_box(0); +if (lean_is_scalar(x_43)) { + x_265 = lean_alloc_ctor(0, 2, 0); +} else { + x_265 = x_43; +} +lean_ctor_set(x_265, 0, x_262); +lean_ctor_set(x_265, 1, x_264); +x_266 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_266, 0, x_265); +lean_ctor_set(x_266, 1, x_264); +x_267 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__8; +lean_inc(x_218); +x_268 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_268, 0, x_218); +lean_ctor_set(x_268, 1, x_267); +lean_ctor_set(x_268, 2, x_263); +lean_ctor_set(x_268, 3, x_266); +x_269 = lean_array_push(x_63, x_260); +x_270 = lean_array_push(x_269, x_268); +x_271 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_271, 0, x_58); +lean_ctor_set(x_271, 1, x_258); +lean_ctor_set(x_271, 2, x_270); +x_272 = lean_array_push(x_60, x_271); +lean_inc(x_7); +x_273 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_273, 0, x_58); +lean_ctor_set(x_273, 1, x_7); +lean_ctor_set(x_273, 2, x_272); +lean_inc(x_246); +x_274 = lean_array_push(x_63, x_246); +x_275 = lean_array_push(x_274, x_273); +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_58); +lean_ctor_set(x_276, 1, x_256); +lean_ctor_set(x_276, 2, x_275); +x_277 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__48; +x_278 = l_Lean_Name_str___override(x_9, x_277); +x_279 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__50; +lean_inc(x_218); +x_280 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_280, 0, x_218); +lean_ctor_set(x_280, 1, x_279); +x_281 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__7; +lean_inc(x_5); +x_282 = l_Lean_Name_str___override(x_5, x_281); +x_283 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__13; +x_284 = l_Lean_addMacroScope(x_224, x_283, x_221); +x_285 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__12; +x_286 = l_Lean_Name_str___override(x_10, x_285); +x_287 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12; +x_288 = l_Lean_Name_str___override(x_286, x_287); +x_289 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_289, 0, x_288); +lean_ctor_set(x_289, 1, x_264); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_264); +x_291 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__11; +x_292 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_292, 0, x_218); +lean_ctor_set(x_292, 1, x_291); +lean_ctor_set(x_292, 2, x_284); +lean_ctor_set(x_292, 3, x_290); +lean_inc(x_26); +x_293 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_264, x_26); +x_294 = l_Nat_repr(x_11); +x_295 = l_Lean_Syntax_mkNumLit(x_294, x_58); +x_296 = l_Nat_repr(x_216); +x_297 = l_Lean_Syntax_mkNumLit(x_296, x_58); +x_298 = lean_array_push(x_63, x_292); +x_299 = lean_array_push(x_239, x_280); +x_300 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__85; +x_301 = lean_array_push(x_300, x_249); +x_302 = lean_array_push(x_301, x_254); +x_303 = lean_array_push(x_302, x_276); if (lean_obj_tag(x_12) == 0) { -x_311 = x_253; -goto block_372; +x_304 = x_234; +goto block_365; } else { -lean_object* x_373; lean_object* x_374; -x_373 = lean_ctor_get(x_12, 0); -lean_inc(x_373); +lean_object* x_366; lean_object* x_367; +x_366 = lean_ctor_get(x_12, 0); +lean_inc(x_366); lean_dec(x_12); -x_374 = lean_array_push(x_232, x_373); -x_311 = x_374; -goto block_372; +x_367 = lean_array_push(x_60, x_366); +x_304 = x_367; +goto block_365; } -block_372: +block_365: { -lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; -x_312 = l_Array_append___rarg(x_253, x_311); -lean_inc(x_8); -x_313 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_313, 0, x_230); -lean_ctor_set(x_313, 1, x_8); -lean_ctor_set(x_313, 2, x_312); -x_314 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__31; -x_315 = lean_array_push(x_314, x_313); -x_316 = lean_array_push(x_315, x_252); -lean_inc(x_254); -x_317 = lean_array_push(x_316, x_254); -lean_inc(x_254); -x_318 = lean_array_push(x_317, x_254); -lean_inc(x_254); -x_319 = lean_array_push(x_318, x_254); -lean_inc(x_254); -x_320 = lean_array_push(x_319, x_254); -x_321 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_321, 0, x_230); -lean_ctor_set(x_321, 1, x_218); -lean_ctor_set(x_321, 2, x_320); -x_322 = lean_array_push(x_235, x_321); -if (lean_obj_tag(x_300) == 0) -{ -lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; -lean_dec(x_6); -x_323 = l_Lean_quoteNameMk(x_25); -x_324 = l_Lean_Elab_Term_toParserDescr_processSepBy1___lambda__1___closed__8; -x_325 = lean_array_push(x_324, x_323); -x_326 = lean_array_push(x_325, x_302); -x_327 = lean_array_push(x_326, x_304); -x_328 = lean_array_push(x_327, x_41); -x_329 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_329, 0, x_230); -lean_ctor_set(x_329, 1, x_8); -lean_ctor_set(x_329, 2, x_328); -x_330 = lean_array_push(x_305, x_329); -x_331 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_331, 0, x_230); -lean_ctor_set(x_331, 1, x_289); -lean_ctor_set(x_331, 2, x_330); -x_332 = lean_array_push(x_306, x_331); -lean_inc(x_254); -x_333 = lean_array_push(x_332, x_254); +lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; +x_305 = l_Array_append___rarg(x_234, x_304); +lean_inc(x_7); +x_306 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_306, 0, x_58); +lean_ctor_set(x_306, 1, x_7); +lean_ctor_set(x_306, 2, x_305); +x_307 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__31; +x_308 = lean_array_push(x_307, x_306); +x_309 = lean_array_push(x_308, x_245); +lean_inc(x_246); +x_310 = lean_array_push(x_309, x_246); +lean_inc(x_246); +x_311 = lean_array_push(x_310, x_246); +lean_inc(x_246); +x_312 = lean_array_push(x_311, x_246); +lean_inc(x_246); +x_313 = lean_array_push(x_312, x_246); +x_314 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_314, 0, x_58); +lean_ctor_set(x_314, 1, x_229); +lean_ctor_set(x_314, 2, x_313); +x_315 = lean_array_push(x_63, x_314); +if (lean_obj_tag(x_293) == 0) +{ +lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; +lean_dec(x_5); +x_316 = l_Lean_quoteNameMk(x_26); +x_317 = l_Lean_Elab_Term_toParserDescr_processSepBy1___lambda__1___closed__8; +x_318 = lean_array_push(x_317, x_316); +x_319 = lean_array_push(x_318, x_295); +x_320 = lean_array_push(x_319, x_297); +x_321 = lean_array_push(x_320, x_41); +x_322 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_322, 0, x_58); +lean_ctor_set(x_322, 1, x_7); +lean_ctor_set(x_322, 2, x_321); +x_323 = lean_array_push(x_298, x_322); +x_324 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_324, 0, x_58); +lean_ctor_set(x_324, 1, x_282); +lean_ctor_set(x_324, 2, x_323); +x_325 = lean_array_push(x_299, x_324); +lean_inc(x_246); +x_326 = lean_array_push(x_325, x_246); +x_327 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_327, 0, x_58); +lean_ctor_set(x_327, 1, x_278); +lean_ctor_set(x_327, 2, x_326); +x_328 = lean_array_push(x_303, x_327); +lean_inc(x_246); +x_329 = lean_array_push(x_328, x_246); +lean_inc(x_246); +x_330 = lean_array_push(x_329, x_246); +x_331 = lean_array_push(x_330, x_246); +x_332 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_332, 0, x_58); +lean_ctor_set(x_332, 1, x_248); +lean_ctor_set(x_332, 2, x_331); +x_333 = lean_array_push(x_315, x_332); x_334 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_334, 0, x_230); -lean_ctor_set(x_334, 1, x_285); +lean_ctor_set(x_334, 0, x_58); +lean_ctor_set(x_334, 1, x_227); lean_ctor_set(x_334, 2, x_333); -x_335 = lean_array_push(x_310, x_334); -lean_inc(x_254); -x_336 = lean_array_push(x_335, x_254); -lean_inc(x_254); -x_337 = lean_array_push(x_336, x_254); -x_338 = lean_array_push(x_337, x_254); -x_339 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_339, 0, x_230); -lean_ctor_set(x_339, 1, x_256); -lean_ctor_set(x_339, 2, x_338); -x_340 = lean_array_push(x_322, x_339); -x_341 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_341, 0, x_230); -lean_ctor_set(x_341, 1, x_216); -lean_ctor_set(x_341, 2, x_340); -x_342 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_341, x_14, x_15, x_214); -return x_342; -} -else -{ -lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; -lean_dec(x_25); -x_343 = lean_ctor_get(x_300, 0); -lean_inc(x_343); -lean_dec(x_300); -x_344 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__22; -x_345 = l_Lean_Name_str___override(x_6, x_344); -x_346 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__16; -x_347 = l_String_intercalate(x_346, x_343); -x_348 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__17; -x_349 = lean_string_append(x_348, x_347); -lean_dec(x_347); -x_350 = l_Lean_Syntax_mkNameLit(x_349, x_230); -x_351 = lean_array_push(x_232, x_350); -x_352 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_352, 0, x_230); -lean_ctor_set(x_352, 1, x_345); -lean_ctor_set(x_352, 2, x_351); -x_353 = l_Lean_Elab_Term_toParserDescr_processSepBy1___lambda__1___closed__8; -x_354 = lean_array_push(x_353, x_352); -x_355 = lean_array_push(x_354, x_302); -x_356 = lean_array_push(x_355, x_304); -x_357 = lean_array_push(x_356, x_41); -x_358 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_358, 0, x_230); -lean_ctor_set(x_358, 1, x_8); -lean_ctor_set(x_358, 2, x_357); -x_359 = lean_array_push(x_305, x_358); -x_360 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_360, 0, x_230); -lean_ctor_set(x_360, 1, x_289); -lean_ctor_set(x_360, 2, x_359); -x_361 = lean_array_push(x_306, x_360); -lean_inc(x_254); -x_362 = lean_array_push(x_361, x_254); +x_335 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_334, x_15, x_16, x_225); +return x_335; +} +else +{ +lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; +lean_dec(x_26); +x_336 = lean_ctor_get(x_293, 0); +lean_inc(x_336); +lean_dec(x_293); +x_337 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__22; +x_338 = l_Lean_Name_str___override(x_5, x_337); +x_339 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__16; +x_340 = l_String_intercalate(x_339, x_336); +x_341 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__17; +x_342 = lean_string_append(x_341, x_340); +lean_dec(x_340); +x_343 = l_Lean_Syntax_mkNameLit(x_342, x_58); +x_344 = lean_array_push(x_60, x_343); +x_345 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_345, 0, x_58); +lean_ctor_set(x_345, 1, x_338); +lean_ctor_set(x_345, 2, x_344); +x_346 = l_Lean_Elab_Term_toParserDescr_processSepBy1___lambda__1___closed__8; +x_347 = lean_array_push(x_346, x_345); +x_348 = lean_array_push(x_347, x_295); +x_349 = lean_array_push(x_348, x_297); +x_350 = lean_array_push(x_349, x_41); +x_351 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_351, 0, x_58); +lean_ctor_set(x_351, 1, x_7); +lean_ctor_set(x_351, 2, x_350); +x_352 = lean_array_push(x_298, x_351); +x_353 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_353, 0, x_58); +lean_ctor_set(x_353, 1, x_282); +lean_ctor_set(x_353, 2, x_352); +x_354 = lean_array_push(x_299, x_353); +lean_inc(x_246); +x_355 = lean_array_push(x_354, x_246); +x_356 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_356, 0, x_58); +lean_ctor_set(x_356, 1, x_278); +lean_ctor_set(x_356, 2, x_355); +x_357 = lean_array_push(x_303, x_356); +lean_inc(x_246); +x_358 = lean_array_push(x_357, x_246); +lean_inc(x_246); +x_359 = lean_array_push(x_358, x_246); +x_360 = lean_array_push(x_359, x_246); +x_361 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_361, 0, x_58); +lean_ctor_set(x_361, 1, x_248); +lean_ctor_set(x_361, 2, x_360); +x_362 = lean_array_push(x_315, x_361); x_363 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_363, 0, x_230); -lean_ctor_set(x_363, 1, x_285); +lean_ctor_set(x_363, 0, x_58); +lean_ctor_set(x_363, 1, x_227); lean_ctor_set(x_363, 2, x_362); -x_364 = lean_array_push(x_310, x_363); -lean_inc(x_254); -x_365 = lean_array_push(x_364, x_254); -lean_inc(x_254); -x_366 = lean_array_push(x_365, x_254); -x_367 = lean_array_push(x_366, x_254); -x_368 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_368, 0, x_230); -lean_ctor_set(x_368, 1, x_256); -lean_ctor_set(x_368, 2, x_367); -x_369 = lean_array_push(x_322, x_368); -x_370 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_370, 0, x_230); -lean_ctor_set(x_370, 1, x_216); -lean_ctor_set(x_370, 2, x_369); -x_371 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_370, x_14, x_15, x_214); -return x_371; +x_364 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_363, x_15, x_16, x_225); +return x_364; } } } } -else -{ -lean_object* x_375; lean_object* x_376; lean_object* x_377; -x_375 = lean_ctor_get(x_38, 0); -x_376 = lean_ctor_get(x_38, 1); -lean_inc(x_376); -lean_inc(x_375); -lean_dec(x_38); -lean_inc(x_3); -x_377 = l_Lean_mkIdentFrom(x_3, x_13); -if (lean_obj_tag(x_376) == 0) -{ -lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; -x_378 = l_Lean_MonadRef_mkInfoFromRefPos___at___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___spec__1(x_14, x_15, x_39); -x_379 = lean_ctor_get(x_378, 0); -lean_inc(x_379); -x_380 = lean_ctor_get(x_378, 1); -lean_inc(x_380); -lean_dec(x_378); -x_381 = l_Lean_Elab_Command_getCurrMacroScope(x_14, x_15, x_380); -x_382 = lean_ctor_get(x_381, 0); -lean_inc(x_382); -x_383 = lean_ctor_get(x_381, 1); -lean_inc(x_383); -lean_dec(x_381); -x_384 = l_Lean_Elab_Command_getMainModule___rarg(x_15, x_383); -x_385 = lean_ctor_get(x_384, 0); -lean_inc(x_385); -x_386 = lean_ctor_get(x_384, 1); -lean_inc(x_386); -lean_dec(x_384); -x_387 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__7; -lean_inc(x_5); -x_388 = l_Lean_Name_str___override(x_5, x_387); -x_389 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__9; -lean_inc(x_5); -x_390 = l_Lean_Name_str___override(x_5, x_389); -x_391 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; -lean_inc(x_6); -x_392 = l_Lean_Name_str___override(x_6, x_391); -x_393 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__14; -lean_inc(x_379); -x_394 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_394, 0, x_379); -lean_ctor_set(x_394, 1, x_393); -x_395 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__15; -lean_inc(x_6); -x_396 = l_Lean_Name_str___override(x_6, x_395); -x_397 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__21; -x_398 = l_Lean_Name_str___override(x_7, x_397); -x_399 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__23; -x_400 = l_Lean_Name_str___override(x_398, x_399); -x_401 = l_Nat_repr(x_19); -x_402 = lean_box(2); -x_403 = l_Lean_Syntax_mkNumLit(x_401, x_402); -x_404 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__27; -x_405 = lean_array_push(x_404, x_403); -lean_inc(x_8); -x_406 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_406, 0, x_402); -lean_ctor_set(x_406, 1, x_8); -lean_ctor_set(x_406, 2, x_405); -x_407 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__29; -x_408 = lean_array_push(x_407, x_28); -x_409 = lean_array_push(x_408, x_406); -x_410 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_410, 0, x_402); -lean_ctor_set(x_410, 1, x_400); -lean_ctor_set(x_410, 2, x_409); -x_411 = lean_array_push(x_407, x_9); -x_412 = lean_array_push(x_411, x_410); -x_413 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_413, 0, x_402); -lean_ctor_set(x_413, 1, x_396); -lean_ctor_set(x_413, 2, x_412); -x_414 = lean_array_push(x_404, x_413); -lean_inc(x_8); -x_415 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_415, 0, x_402); -lean_ctor_set(x_415, 1, x_8); -lean_ctor_set(x_415, 2, x_414); -x_416 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__30; -lean_inc(x_379); -x_417 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_417, 0, x_379); -lean_ctor_set(x_417, 1, x_416); -x_418 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__28; -x_419 = lean_array_push(x_418, x_394); -x_420 = lean_array_push(x_419, x_415); -x_421 = lean_array_push(x_420, x_417); -x_422 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_422, 0, x_402); -lean_ctor_set(x_422, 1, x_392); -lean_ctor_set(x_422, 2, x_421); -x_423 = lean_array_push(x_404, x_422); -lean_inc(x_8); -x_424 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_424, 0, x_402); -lean_ctor_set(x_424, 1, x_8); -lean_ctor_set(x_424, 2, x_423); -x_425 = l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__3; -lean_inc(x_8); -x_426 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_426, 0, x_402); -lean_ctor_set(x_426, 1, x_8); -lean_ctor_set(x_426, 2, x_425); -x_427 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__33; -lean_inc(x_5); -x_428 = l_Lean_Name_str___override(x_5, x_427); -lean_inc(x_379); -x_429 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_429, 0, x_379); -lean_ctor_set(x_429, 1, x_427); -x_430 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__35; -lean_inc(x_5); -x_431 = l_Lean_Name_str___override(x_5, x_430); -x_432 = lean_array_push(x_407, x_377); -lean_inc(x_426); -x_433 = lean_array_push(x_432, x_426); -x_434 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_434, 0, x_402); -lean_ctor_set(x_434, 1, x_431); -lean_ctor_set(x_434, 2, x_433); -x_435 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__37; -lean_inc(x_5); -x_436 = l_Lean_Name_str___override(x_5, x_435); -x_437 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__39; -lean_inc(x_6); -x_438 = l_Lean_Name_str___override(x_6, x_437); -x_439 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__41; -lean_inc(x_379); -x_440 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_440, 0, x_379); -lean_ctor_set(x_440, 1, x_439); -x_441 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__12; -x_442 = l_Lean_Name_str___override(x_10, x_441); -lean_inc(x_382); -lean_inc(x_442); -lean_inc(x_385); -x_443 = l_Lean_addMacroScope(x_385, x_442, x_382); -x_444 = lean_box(0); -lean_inc(x_442); -x_445 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_445, 0, x_442); -lean_ctor_set(x_445, 1, x_444); -x_446 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_446, 0, x_445); -lean_ctor_set(x_446, 1, x_444); -x_447 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__44; -lean_inc(x_379); -x_448 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_448, 0, x_379); -lean_ctor_set(x_448, 1, x_447); -lean_ctor_set(x_448, 2, x_443); -lean_ctor_set(x_448, 3, x_446); -x_449 = lean_array_push(x_407, x_440); -x_450 = lean_array_push(x_449, x_448); -x_451 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_451, 0, x_402); -lean_ctor_set(x_451, 1, x_438); -lean_ctor_set(x_451, 2, x_450); -x_452 = lean_array_push(x_404, x_451); -lean_inc(x_8); -x_453 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_453, 0, x_402); -lean_ctor_set(x_453, 1, x_8); -lean_ctor_set(x_453, 2, x_452); -lean_inc(x_426); -x_454 = lean_array_push(x_407, x_426); -x_455 = lean_array_push(x_454, x_453); -x_456 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_456, 0, x_402); -lean_ctor_set(x_456, 1, x_436); -lean_ctor_set(x_456, 2, x_455); -x_457 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__48; -x_458 = l_Lean_Name_str___override(x_5, x_457); -x_459 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__50; -lean_inc(x_379); -x_460 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_460, 0, x_379); -lean_ctor_set(x_460, 1, x_459); -x_461 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__7; -lean_inc(x_6); -x_462 = l_Lean_Name_str___override(x_6, x_461); -x_463 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__4; -x_464 = l_Lean_addMacroScope(x_385, x_463, x_382); -x_465 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__54; -x_466 = l_Lean_Name_str___override(x_442, x_465); -x_467 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_467, 0, x_466); -lean_ctor_set(x_467, 1, x_444); -x_468 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_468, 0, x_467); -lean_ctor_set(x_468, 1, x_444); -x_469 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__3; -x_470 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_470, 0, x_379); -lean_ctor_set(x_470, 1, x_469); -lean_ctor_set(x_470, 2, x_464); -lean_ctor_set(x_470, 3, x_468); -lean_inc(x_25); -x_471 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_444, x_25); -x_472 = l_Nat_repr(x_11); -x_473 = l_Lean_Syntax_mkNumLit(x_472, x_402); -x_474 = lean_array_push(x_407, x_470); -x_475 = lean_array_push(x_418, x_460); -x_476 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__85; -x_477 = lean_array_push(x_476, x_429); -x_478 = lean_array_push(x_477, x_434); -x_479 = lean_array_push(x_478, x_456); -if (lean_obj_tag(x_12) == 0) -{ -x_480 = x_425; -goto block_537; } else { -lean_object* x_538; lean_object* x_539; -x_538 = lean_ctor_get(x_12, 0); -lean_inc(x_538); -lean_dec(x_12); -x_539 = lean_array_push(x_404, x_538); -x_480 = x_539; -goto block_537; -} -block_537: -{ -lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; -x_481 = l_Array_append___rarg(x_425, x_480); -lean_inc(x_8); -x_482 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_482, 0, x_402); -lean_ctor_set(x_482, 1, x_8); -lean_ctor_set(x_482, 2, x_481); -x_483 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__31; -x_484 = lean_array_push(x_483, x_482); -x_485 = lean_array_push(x_484, x_424); -lean_inc(x_426); -x_486 = lean_array_push(x_485, x_426); -lean_inc(x_426); -x_487 = lean_array_push(x_486, x_426); -lean_inc(x_426); -x_488 = lean_array_push(x_487, x_426); -lean_inc(x_426); -x_489 = lean_array_push(x_488, x_426); -x_490 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_490, 0, x_402); -lean_ctor_set(x_490, 1, x_390); -lean_ctor_set(x_490, 2, x_489); -x_491 = lean_array_push(x_407, x_490); -if (lean_obj_tag(x_471) == 0) -{ -lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; -lean_dec(x_6); -x_492 = l_Lean_quoteNameMk(x_25); -x_493 = lean_array_push(x_418, x_492); -x_494 = lean_array_push(x_493, x_473); -x_495 = lean_array_push(x_494, x_375); -x_496 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_496, 0, x_402); -lean_ctor_set(x_496, 1, x_8); -lean_ctor_set(x_496, 2, x_495); -x_497 = lean_array_push(x_474, x_496); -x_498 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_498, 0, x_402); -lean_ctor_set(x_498, 1, x_462); -lean_ctor_set(x_498, 2, x_497); -x_499 = lean_array_push(x_475, x_498); -lean_inc(x_426); -x_500 = lean_array_push(x_499, x_426); -x_501 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_501, 0, x_402); -lean_ctor_set(x_501, 1, x_458); -lean_ctor_set(x_501, 2, x_500); -x_502 = lean_array_push(x_479, x_501); -lean_inc(x_426); -x_503 = lean_array_push(x_502, x_426); -lean_inc(x_426); -x_504 = lean_array_push(x_503, x_426); -x_505 = lean_array_push(x_504, x_426); -x_506 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_506, 0, x_402); -lean_ctor_set(x_506, 1, x_428); -lean_ctor_set(x_506, 2, x_505); -x_507 = lean_array_push(x_491, x_506); -x_508 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_508, 0, x_402); -lean_ctor_set(x_508, 1, x_388); -lean_ctor_set(x_508, 2, x_507); -x_509 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_508, x_14, x_15, x_386); -return x_509; -} -else -{ -lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; -lean_dec(x_25); -x_510 = lean_ctor_get(x_471, 0); -lean_inc(x_510); -lean_dec(x_471); -x_511 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__22; -x_512 = l_Lean_Name_str___override(x_6, x_511); -x_513 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__16; -x_514 = l_String_intercalate(x_513, x_510); -x_515 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__17; -x_516 = lean_string_append(x_515, x_514); -lean_dec(x_514); -x_517 = l_Lean_Syntax_mkNameLit(x_516, x_402); -x_518 = lean_array_push(x_404, x_517); -x_519 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_519, 0, x_402); -lean_ctor_set(x_519, 1, x_512); -lean_ctor_set(x_519, 2, x_518); -x_520 = lean_array_push(x_418, x_519); -x_521 = lean_array_push(x_520, x_473); -x_522 = lean_array_push(x_521, x_375); -x_523 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_523, 0, x_402); -lean_ctor_set(x_523, 1, x_8); -lean_ctor_set(x_523, 2, x_522); -x_524 = lean_array_push(x_474, x_523); -x_525 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_525, 0, x_402); -lean_ctor_set(x_525, 1, x_462); -lean_ctor_set(x_525, 2, x_524); -x_526 = lean_array_push(x_475, x_525); -lean_inc(x_426); -x_527 = lean_array_push(x_526, x_426); -x_528 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_528, 0, x_402); -lean_ctor_set(x_528, 1, x_458); -lean_ctor_set(x_528, 2, x_527); -x_529 = lean_array_push(x_479, x_528); -lean_inc(x_426); -x_530 = lean_array_push(x_529, x_426); -lean_inc(x_426); -x_531 = lean_array_push(x_530, x_426); -x_532 = lean_array_push(x_531, x_426); -x_533 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_533, 0, x_402); -lean_ctor_set(x_533, 1, x_428); -lean_ctor_set(x_533, 2, x_532); -x_534 = lean_array_push(x_491, x_533); -x_535 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_535, 0, x_402); -lean_ctor_set(x_535, 1, x_388); -lean_ctor_set(x_535, 2, x_534); -x_536 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_535, x_14, x_15, x_386); -return x_536; -} -} -} -else -{ -lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; lean_object* x_570; lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; lean_object* x_647; -x_540 = lean_ctor_get(x_376, 0); -lean_inc(x_540); -lean_dec(x_376); -x_541 = l_Lean_MonadRef_mkInfoFromRefPos___at___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___spec__1(x_14, x_15, x_39); -x_542 = lean_ctor_get(x_541, 0); -lean_inc(x_542); -x_543 = lean_ctor_get(x_541, 1); -lean_inc(x_543); -lean_dec(x_541); -x_544 = l_Lean_Elab_Command_getCurrMacroScope(x_14, x_15, x_543); -x_545 = lean_ctor_get(x_544, 0); -lean_inc(x_545); -x_546 = lean_ctor_get(x_544, 1); -lean_inc(x_546); -lean_dec(x_544); -x_547 = l_Lean_Elab_Command_getMainModule___rarg(x_15, x_546); -x_548 = lean_ctor_get(x_547, 0); -lean_inc(x_548); -x_549 = lean_ctor_get(x_547, 1); -lean_inc(x_549); -lean_dec(x_547); -x_550 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__7; -lean_inc(x_5); -x_551 = l_Lean_Name_str___override(x_5, x_550); -x_552 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__9; -lean_inc(x_5); -x_553 = l_Lean_Name_str___override(x_5, x_552); -x_554 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; -lean_inc(x_6); -x_555 = l_Lean_Name_str___override(x_6, x_554); -x_556 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__14; -lean_inc(x_542); -x_557 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_557, 0, x_542); -lean_ctor_set(x_557, 1, x_556); -x_558 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__15; -lean_inc(x_6); -x_559 = l_Lean_Name_str___override(x_6, x_558); -x_560 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__21; -x_561 = l_Lean_Name_str___override(x_7, x_560); -x_562 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__23; -x_563 = l_Lean_Name_str___override(x_561, x_562); -x_564 = l_Nat_repr(x_19); -x_565 = lean_box(2); -x_566 = l_Lean_Syntax_mkNumLit(x_564, x_565); -x_567 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__27; -x_568 = lean_array_push(x_567, x_566); -lean_inc(x_8); -x_569 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_569, 0, x_565); -lean_ctor_set(x_569, 1, x_8); -lean_ctor_set(x_569, 2, x_568); -x_570 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__29; -x_571 = lean_array_push(x_570, x_28); -x_572 = lean_array_push(x_571, x_569); -x_573 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_573, 0, x_565); -lean_ctor_set(x_573, 1, x_563); -lean_ctor_set(x_573, 2, x_572); -x_574 = lean_array_push(x_570, x_9); -x_575 = lean_array_push(x_574, x_573); -x_576 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_576, 0, x_565); -lean_ctor_set(x_576, 1, x_559); -lean_ctor_set(x_576, 2, x_575); -x_577 = lean_array_push(x_567, x_576); -lean_inc(x_8); -x_578 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_578, 0, x_565); -lean_ctor_set(x_578, 1, x_8); -lean_ctor_set(x_578, 2, x_577); -x_579 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__30; -lean_inc(x_542); -x_580 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_580, 0, x_542); -lean_ctor_set(x_580, 1, x_579); -x_581 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__28; -x_582 = lean_array_push(x_581, x_557); -x_583 = lean_array_push(x_582, x_578); -x_584 = lean_array_push(x_583, x_580); -x_585 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_585, 0, x_565); -lean_ctor_set(x_585, 1, x_555); -lean_ctor_set(x_585, 2, x_584); -x_586 = lean_array_push(x_567, x_585); -lean_inc(x_8); -x_587 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_587, 0, x_565); -lean_ctor_set(x_587, 1, x_8); -lean_ctor_set(x_587, 2, x_586); -x_588 = l_Lean_Elab_Term_toParserDescr_processNullaryOrCat___closed__3; -lean_inc(x_8); -x_589 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_589, 0, x_565); -lean_ctor_set(x_589, 1, x_8); -lean_ctor_set(x_589, 2, x_588); -x_590 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__33; -lean_inc(x_5); -x_591 = l_Lean_Name_str___override(x_5, x_590); -lean_inc(x_542); -x_592 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_592, 0, x_542); -lean_ctor_set(x_592, 1, x_590); -x_593 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__35; -lean_inc(x_5); -x_594 = l_Lean_Name_str___override(x_5, x_593); -x_595 = lean_array_push(x_570, x_377); -lean_inc(x_589); -x_596 = lean_array_push(x_595, x_589); -x_597 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_597, 0, x_565); -lean_ctor_set(x_597, 1, x_594); -lean_ctor_set(x_597, 2, x_596); -x_598 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__37; -lean_inc(x_5); -x_599 = l_Lean_Name_str___override(x_5, x_598); -x_600 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__39; -lean_inc(x_6); -x_601 = l_Lean_Name_str___override(x_6, x_600); -x_602 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__41; -lean_inc(x_542); -x_603 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_603, 0, x_542); -lean_ctor_set(x_603, 1, x_602); -x_604 = l_List_filterMap___at_Lean_Elab_Term_resolveParserName___spec__1___closed__1; -lean_inc(x_10); -x_605 = l_Lean_Name_str___override(x_10, x_604); -lean_inc(x_545); -lean_inc(x_605); -lean_inc(x_548); -x_606 = l_Lean_addMacroScope(x_548, x_605, x_545); -x_607 = lean_box(0); -x_608 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_608, 0, x_605); -lean_ctor_set(x_608, 1, x_607); -x_609 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_609, 0, x_608); -lean_ctor_set(x_609, 1, x_607); -x_610 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__7; -lean_inc(x_542); -x_611 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_611, 0, x_542); -lean_ctor_set(x_611, 1, x_610); -lean_ctor_set(x_611, 2, x_606); -lean_ctor_set(x_611, 3, x_609); -x_612 = lean_array_push(x_570, x_603); -x_613 = lean_array_push(x_612, x_611); -x_614 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_614, 0, x_565); -lean_ctor_set(x_614, 1, x_601); -lean_ctor_set(x_614, 2, x_613); -x_615 = lean_array_push(x_567, x_614); -lean_inc(x_8); -x_616 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_616, 0, x_565); -lean_ctor_set(x_616, 1, x_8); -lean_ctor_set(x_616, 2, x_615); -lean_inc(x_589); -x_617 = lean_array_push(x_570, x_589); -x_618 = lean_array_push(x_617, x_616); -x_619 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_619, 0, x_565); -lean_ctor_set(x_619, 1, x_599); -lean_ctor_set(x_619, 2, x_618); -x_620 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__48; -x_621 = l_Lean_Name_str___override(x_5, x_620); -x_622 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__50; -lean_inc(x_542); -x_623 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_623, 0, x_542); -lean_ctor_set(x_623, 1, x_622); -x_624 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__7; -lean_inc(x_6); -x_625 = l_Lean_Name_str___override(x_6, x_624); -x_626 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12; -x_627 = l_Lean_addMacroScope(x_548, x_626, x_545); -x_628 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__12; -x_629 = l_Lean_Name_str___override(x_10, x_628); -x_630 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__11; -x_631 = l_Lean_Name_str___override(x_629, x_630); -x_632 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_632, 0, x_631); -lean_ctor_set(x_632, 1, x_607); -x_633 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_633, 0, x_632); -lean_ctor_set(x_633, 1, x_607); -x_634 = l_Lean_Elab_Command_elabSyntax___lambda__5___closed__10; -x_635 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_635, 0, x_542); -lean_ctor_set(x_635, 1, x_634); -lean_ctor_set(x_635, 2, x_627); -lean_ctor_set(x_635, 3, x_633); -lean_inc(x_25); -x_636 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_607, x_25); -x_637 = l_Nat_repr(x_11); -x_638 = l_Lean_Syntax_mkNumLit(x_637, x_565); -x_639 = l_Nat_repr(x_540); -x_640 = l_Lean_Syntax_mkNumLit(x_639, x_565); -x_641 = lean_array_push(x_570, x_635); -x_642 = lean_array_push(x_581, x_623); -x_643 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__85; -x_644 = lean_array_push(x_643, x_592); -x_645 = lean_array_push(x_644, x_597); -x_646 = lean_array_push(x_645, x_619); -if (lean_obj_tag(x_12) == 0) -{ -x_647 = x_588; -goto block_708; -} -else -{ -lean_object* x_709; lean_object* x_710; -x_709 = lean_ctor_get(x_12, 0); -lean_inc(x_709); -lean_dec(x_12); -x_710 = lean_array_push(x_567, x_709); -x_647 = x_710; -goto block_708; -} -block_708: -{ -lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; lean_object* x_657; lean_object* x_658; -x_648 = l_Array_append___rarg(x_588, x_647); -lean_inc(x_8); -x_649 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_649, 0, x_565); -lean_ctor_set(x_649, 1, x_8); -lean_ctor_set(x_649, 2, x_648); -x_650 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__31; -x_651 = lean_array_push(x_650, x_649); -x_652 = lean_array_push(x_651, x_587); -lean_inc(x_589); -x_653 = lean_array_push(x_652, x_589); -lean_inc(x_589); -x_654 = lean_array_push(x_653, x_589); -lean_inc(x_589); -x_655 = lean_array_push(x_654, x_589); -lean_inc(x_589); -x_656 = lean_array_push(x_655, x_589); -x_657 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_657, 0, x_565); -lean_ctor_set(x_657, 1, x_553); -lean_ctor_set(x_657, 2, x_656); -x_658 = lean_array_push(x_570, x_657); -if (lean_obj_tag(x_636) == 0) -{ -lean_object* x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; lean_object* x_677; lean_object* x_678; -lean_dec(x_6); -x_659 = l_Lean_quoteNameMk(x_25); -x_660 = l_Lean_Elab_Term_toParserDescr_processSepBy1___lambda__1___closed__8; -x_661 = lean_array_push(x_660, x_659); -x_662 = lean_array_push(x_661, x_638); -x_663 = lean_array_push(x_662, x_640); -x_664 = lean_array_push(x_663, x_375); -x_665 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_665, 0, x_565); -lean_ctor_set(x_665, 1, x_8); -lean_ctor_set(x_665, 2, x_664); -x_666 = lean_array_push(x_641, x_665); -x_667 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_667, 0, x_565); -lean_ctor_set(x_667, 1, x_625); -lean_ctor_set(x_667, 2, x_666); -x_668 = lean_array_push(x_642, x_667); -lean_inc(x_589); -x_669 = lean_array_push(x_668, x_589); -x_670 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_670, 0, x_565); -lean_ctor_set(x_670, 1, x_621); -lean_ctor_set(x_670, 2, x_669); -x_671 = lean_array_push(x_646, x_670); -lean_inc(x_589); -x_672 = lean_array_push(x_671, x_589); -lean_inc(x_589); -x_673 = lean_array_push(x_672, x_589); -x_674 = lean_array_push(x_673, x_589); -x_675 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_675, 0, x_565); -lean_ctor_set(x_675, 1, x_591); -lean_ctor_set(x_675, 2, x_674); -x_676 = lean_array_push(x_658, x_675); -x_677 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_677, 0, x_565); -lean_ctor_set(x_677, 1, x_551); -lean_ctor_set(x_677, 2, x_676); -x_678 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_677, x_14, x_15, x_549); -return x_678; -} -else -{ -lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; -lean_dec(x_25); -x_679 = lean_ctor_get(x_636, 0); -lean_inc(x_679); -lean_dec(x_636); -x_680 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__22; -x_681 = l_Lean_Name_str___override(x_6, x_680); -x_682 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__16; -x_683 = l_String_intercalate(x_682, x_679); -x_684 = l_Lean_Elab_Term_ensureUnaryOutput___lambda__1___closed__17; -x_685 = lean_string_append(x_684, x_683); -lean_dec(x_683); -x_686 = l_Lean_Syntax_mkNameLit(x_685, x_565); -x_687 = lean_array_push(x_567, x_686); -x_688 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_688, 0, x_565); -lean_ctor_set(x_688, 1, x_681); -lean_ctor_set(x_688, 2, x_687); -x_689 = l_Lean_Elab_Term_toParserDescr_processSepBy1___lambda__1___closed__8; -x_690 = lean_array_push(x_689, x_688); -x_691 = lean_array_push(x_690, x_638); -x_692 = lean_array_push(x_691, x_640); -x_693 = lean_array_push(x_692, x_375); -x_694 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_694, 0, x_565); -lean_ctor_set(x_694, 1, x_8); -lean_ctor_set(x_694, 2, x_693); -x_695 = lean_array_push(x_641, x_694); -x_696 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_696, 0, x_565); -lean_ctor_set(x_696, 1, x_625); -lean_ctor_set(x_696, 2, x_695); -x_697 = lean_array_push(x_642, x_696); -lean_inc(x_589); -x_698 = lean_array_push(x_697, x_589); -x_699 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_699, 0, x_565); -lean_ctor_set(x_699, 1, x_621); -lean_ctor_set(x_699, 2, x_698); -x_700 = lean_array_push(x_646, x_699); -lean_inc(x_589); -x_701 = lean_array_push(x_700, x_589); -lean_inc(x_589); -x_702 = lean_array_push(x_701, x_589); -x_703 = lean_array_push(x_702, x_589); -x_704 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_704, 0, x_565); -lean_ctor_set(x_704, 1, x_591); -lean_ctor_set(x_704, 2, x_703); -x_705 = lean_array_push(x_658, x_704); -x_706 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_706, 0, x_565); -lean_ctor_set(x_706, 1, x_551); -lean_ctor_set(x_706, 2, x_705); -x_707 = l_Lean_Elab_Command_elabSyntax___lambda__4(x_3, x_706, x_14, x_15, x_549); -return x_707; -} -} -} -} -} -else -{ -uint8_t x_711; -lean_dec(x_28); -lean_dec(x_25); -lean_dec(x_19); +uint8_t x_371; +lean_dec(x_29); +lean_dec(x_26); +lean_dec(x_20); +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -17942,29 +17275,30 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_711 = !lean_is_exclusive(x_37); -if (x_711 == 0) +x_371 = !lean_is_exclusive(x_38); +if (x_371 == 0) { -return x_37; +return x_38; } else { -lean_object* x_712; lean_object* x_713; lean_object* x_714; -x_712 = lean_ctor_get(x_37, 0); -x_713 = lean_ctor_get(x_37, 1); -lean_inc(x_713); -lean_inc(x_712); -lean_dec(x_37); -x_714 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_714, 0, x_712); -lean_ctor_set(x_714, 1, x_713); -return x_714; +lean_object* x_372; lean_object* x_373; lean_object* x_374; +x_372 = lean_ctor_get(x_38, 0); +x_373 = lean_ctor_get(x_38, 1); +lean_inc(x_373); +lean_inc(x_372); +lean_dec(x_38); +x_374 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_374, 0, x_372); +lean_ctor_set(x_374, 1, x_373); +return x_374; } } } else { -uint8_t x_715; +uint8_t x_375; +lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -17979,58 +17313,59 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_715 = !lean_is_exclusive(x_18); -if (x_715 == 0) +x_375 = !lean_is_exclusive(x_19); +if (x_375 == 0) { -return x_18; +return x_19; } else { -lean_object* x_716; lean_object* x_717; lean_object* x_718; -x_716 = lean_ctor_get(x_18, 0); -x_717 = lean_ctor_get(x_18, 1); -lean_inc(x_717); -lean_inc(x_716); -lean_dec(x_18); -x_718 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_718, 0, x_716); -lean_ctor_set(x_718, 1, x_717); -return x_718; +lean_object* x_376; lean_object* x_377; lean_object* x_378; +x_376 = lean_ctor_get(x_19, 0); +x_377 = lean_ctor_get(x_19, 1); +lean_inc(x_377); +lean_inc(x_376); +lean_dec(x_19); +x_378 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_378, 0, x_376); +lean_ctor_set(x_378, 1, x_377); +return x_378; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_13) == 0) { -lean_object* x_17; lean_object* x_18; +lean_object* x_18; lean_object* x_19; lean_inc(x_4); lean_inc(x_2); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkNameFromParserSyntax), 4, 2); -lean_closure_set(x_17, 0, x_2); -lean_closure_set(x_17, 1, x_4); +x_18 = lean_alloc_closure((void*)(l_Lean_Elab_Command_mkNameFromParserSyntax), 4, 2); +lean_closure_set(x_18, 0, x_2); +lean_closure_set(x_18, 1, x_4); +lean_inc(x_16); lean_inc(x_15); -lean_inc(x_14); -x_18 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabSyntax___spec__9(x_17, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_19 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabSyntax___spec__9(x_18, x_15, x_16, x_17); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_Elab_Command_elabSyntax___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_13, x_11, x_19, x_14, x_15, x_20); -return x_21; +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l_Lean_Elab_Command_elabSyntax___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14, x_11, x_12, x_20, x_15, x_16, x_21); +return x_22; } else { -uint8_t x_22; +uint8_t x_23; +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); @@ -18042,89 +17377,90 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) +x_23 = !lean_is_exclusive(x_19); +if (x_23 == 0) { -return x_18; +return x_19; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_18, 0); -x_24 = lean_ctor_get(x_18, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_19, 0); +x_25 = lean_ctor_get(x_19, 1); +lean_inc(x_25); lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_18); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +lean_dec(x_19); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_12, 0); -lean_inc(x_26); -lean_dec(x_12); -x_27 = l_Lean_Syntax_getId(x_26); -lean_dec(x_26); -x_28 = l_Lean_Elab_Command_elabSyntax___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_13, x_11, x_27, x_14, x_15, x_16); -return x_28; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_13, 0); +lean_inc(x_27); +lean_dec(x_13); +x_28 = l_Lean_Syntax_getId(x_27); +lean_dec(x_27); +x_29 = l_Lean_Elab_Command_elabSyntax___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14, x_11, x_12, x_28, x_15, x_16, x_17); +return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -lean_dec(x_13); -x_17 = lean_box(2); -x_18 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__21; -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set(x_19, 2, x_1); -lean_inc(x_19); -x_20 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_isAtomLikeSyntax(x_19); -if (x_20 == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_dec(x_14); +x_18 = lean_box(2); +x_19 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__21; +x_20 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +lean_ctor_set(x_20, 2, x_1); +lean_inc(x_20); +x_21 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_isAtomLikeSyntax(x_20); +if (x_21 == 0) { -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_13) == 0) { -lean_object* x_21; lean_object* x_22; -x_21 = l_Lean_Parser_leadPrec; -x_22 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_2, x_3, x_4, x_19, x_5, x_6, x_7, x_18, x_8, x_9, x_10, x_11, x_21, x_14, x_15, x_16); -return x_22; +lean_object* x_22; lean_object* x_23; +x_22 = l_Lean_Parser_leadPrec; +x_23 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_2, x_3, x_4, x_20, x_5, x_6, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_22, x_15, x_16, x_17); +return x_23; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_12, 0); -lean_inc(x_23); -lean_dec(x_12); -x_24 = lean_alloc_closure((void*)(l_Lean_evalPrec), 3, 1); -lean_closure_set(x_24, 0, x_23); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_13, 0); +lean_inc(x_24); +lean_dec(x_13); +x_25 = lean_alloc_closure((void*)(l_Lean_evalPrec), 3, 1); +lean_closure_set(x_25, 0, x_24); +lean_inc(x_16); lean_inc(x_15); -lean_inc(x_14); -x_25 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabSyntax___spec__4(x_24, x_14, x_15, x_16); -if (lean_obj_tag(x_25) == 0) +x_26 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabSyntax___spec__4(x_25, x_15, x_16, x_17); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -lean_dec(x_25); -x_28 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_2, x_3, x_4, x_19, x_5, x_6, x_7, x_18, x_8, x_9, x_10, x_11, x_26, x_14, x_15, x_27); -return x_28; +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_2, x_3, x_4, x_20, x_5, x_6, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_27, x_15, x_16, x_28); +return x_29; } else { -uint8_t x_29; -lean_dec(x_19); +uint8_t x_30; +lean_dec(x_20); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -18135,64 +17471,65 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_29 = !lean_is_exclusive(x_25); -if (x_29 == 0) +x_30 = !lean_is_exclusive(x_26); +if (x_30 == 0) { -return x_25; +return x_26; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_25, 0); -x_31 = lean_ctor_get(x_25, 1); +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_26, 0); +x_32 = lean_ctor_get(x_26, 1); +lean_inc(x_32); lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_25); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_dec(x_26); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } } } else { -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_13) == 0) { -lean_object* x_33; lean_object* x_34; -x_33 = l_Lean_Parser_maxPrec; -x_34 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_2, x_3, x_4, x_19, x_5, x_6, x_7, x_18, x_8, x_9, x_10, x_11, x_33, x_14, x_15, x_16); -return x_34; +lean_object* x_34; lean_object* x_35; +x_34 = l_Lean_Parser_maxPrec; +x_35 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_2, x_3, x_4, x_20, x_5, x_6, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_34, x_15, x_16, x_17); +return x_35; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_12, 0); -lean_inc(x_35); -lean_dec(x_12); -x_36 = lean_alloc_closure((void*)(l_Lean_evalPrec), 3, 1); -lean_closure_set(x_36, 0, x_35); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_13, 0); +lean_inc(x_36); +lean_dec(x_13); +x_37 = lean_alloc_closure((void*)(l_Lean_evalPrec), 3, 1); +lean_closure_set(x_37, 0, x_36); +lean_inc(x_16); lean_inc(x_15); -lean_inc(x_14); -x_37 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabSyntax___spec__4(x_36, x_14, x_15, x_16); -if (lean_obj_tag(x_37) == 0) +x_38 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Command_elabSyntax___spec__4(x_37, x_15, x_16, x_17); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_37, 1); +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); -lean_dec(x_37); -x_40 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_2, x_3, x_4, x_19, x_5, x_6, x_7, x_18, x_8, x_9, x_10, x_11, x_38, x_14, x_15, x_39); -return x_40; +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_2, x_3, x_4, x_20, x_5, x_6, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_39, x_15, x_16, x_40); +return x_41; } else { -uint8_t x_41; -lean_dec(x_19); +uint8_t x_42; +lean_dec(x_20); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -18203,23 +17540,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_41 = !lean_is_exclusive(x_37); -if (x_41 == 0) +x_42 = !lean_is_exclusive(x_38); +if (x_42 == 0) { -return x_37; +return x_38; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_37, 0); -x_43 = lean_ctor_get(x_37, 1); +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_38, 0); +x_44 = lean_ctor_get(x_38, 1); +lean_inc(x_44); lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_37); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_dec(x_38); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } @@ -18234,38 +17571,162 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Command_elabSyntax___lambda__1), 1, return x_1; } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__8___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("unknown category '", 18); -return x_1; +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__8___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("unknown category '", 18); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__8___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Command_elabSyntax___lambda__8___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_dec(x_12); +x_17 = lean_unsigned_to_nat(7u); +x_18 = l_Lean_Syntax_getArg(x_1, x_17); +x_19 = l_Lean_Syntax_getArgs(x_18); +lean_dec(x_18); +x_20 = l_Lean_Elab_Command_elabSyntax___lambda__8___closed__1; +x_21 = l_Array_sequenceMap___at_Lean_Elab_Command_elabSyntax___spec__2(x_19, x_20); +lean_dec(x_19); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_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_22 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_16); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_unsigned_to_nat(9u); +x_25 = l_Lean_Syntax_getArg(x_1, x_24); +lean_dec(x_1); +x_26 = l_Lean_Syntax_getId(x_25); +x_27 = lean_erase_macro_scopes(x_26); +x_28 = lean_st_ref_get(x_15, x_16); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +lean_dec(x_29); +lean_inc(x_27); +x_32 = l_Lean_Parser_isParserCategory(x_31, x_27); +lean_dec(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +lean_dec(x_23); +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_33 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_33, 0, x_27); +x_34 = l_Lean_Elab_Command_elabSyntax___lambda__8___closed__3; +x_35 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_33); +x_36 = l_Lean_throwUnknownConstant___at_Lean_Elab_Term_toParserDescr_processNullaryOrCat___spec__8___closed__4; +x_37 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +x_38 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabSyntax___spec__13(x_25, x_37, x_14, x_15, x_30); +lean_dec(x_15); +lean_dec(x_25); +x_39 = !lean_is_exclusive(x_38); +if (x_39 == 0) +{ +return x_38; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_38, 0); +x_41 = lean_ctor_get(x_38, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_38); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; +} +} +else +{ +lean_object* x_43; lean_object* x_44; +lean_dec(x_25); +x_43 = lean_box(0); +x_44 = l_Lean_Elab_Command_elabSyntax___lambda__7(x_23, x_13, x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_43, x_14, x_15, x_30); +return x_44; +} +} } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__8___closed__3() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__9___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Command_elabSyntax___lambda__8___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("namedPrio", 9); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_dec(x_11); x_16 = lean_unsigned_to_nat(6u); x_17 = l_Lean_Syntax_getArg(x_1, x_16); -x_18 = l_Lean_Syntax_getArgs(x_17); -lean_dec(x_17); -x_19 = l_Lean_Elab_Command_elabSyntax___lambda__8___closed__1; -x_20 = l_Array_sequenceMap___at_Lean_Elab_Command_elabSyntax___spec__2(x_18, x_19); -lean_dec(x_18); -if (lean_obj_tag(x_20) == 0) +x_18 = l_Lean_Syntax_isNone(x_17); +if (x_18 == 0) +{ +lean_object* x_19; uint8_t x_20; +x_19 = lean_unsigned_to_nat(1u); +lean_inc(x_17); +x_20 = l_Lean_Syntax_matchesNull(x_17, x_19); +if (x_20 == 0) { lean_object* x_21; +lean_dec(x_17); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -18284,31 +17745,22 @@ return x_21; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_22 = lean_ctor_get(x_20, 0); -lean_inc(x_22); -lean_dec(x_20); -x_23 = lean_unsigned_to_nat(8u); -x_24 = l_Lean_Syntax_getArg(x_1, x_23); -lean_dec(x_1); -x_25 = l_Lean_Syntax_getId(x_24); -x_26 = lean_erase_macro_scopes(x_25); -x_27 = lean_st_ref_get(x_14, x_15); -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_ctor_get(x_28, 0); -lean_inc(x_30); -lean_dec(x_28); -lean_inc(x_26); -x_31 = l_Lean_Parser_isParserCategory(x_30, x_26); -lean_dec(x_30); -if (x_31 == 0) +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_22 = lean_unsigned_to_nat(0u); +x_23 = l_Lean_Syntax_getArg(x_17, x_22); +lean_dec(x_17); +x_24 = l_Lean_Elab_Command_elabSyntax___lambda__9___closed__1; +lean_inc(x_6); +x_25 = l_Lean_Name_str___override(x_6, x_24); +lean_inc(x_23); +x_26 = l_Lean_Syntax_isOfKind(x_23, x_25); +lean_dec(x_25); +if (x_26 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -lean_dec(x_22); +lean_object* x_27; +lean_dec(x_23); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_10); lean_dec(x_9); @@ -18319,58 +17771,44 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_32 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_32, 0, x_26); -x_33 = l_Lean_Elab_Command_elabSyntax___lambda__8___closed__3; -x_34 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_32); -x_35 = l_Lean_throwUnknownConstant___at_Lean_Elab_Term_toParserDescr_processNullaryOrCat___spec__8___closed__4; -x_36 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lean_throwErrorAt___at_Lean_Elab_Command_elabSyntax___spec__13(x_24, x_36, x_13, x_14, x_29); -lean_dec(x_14); -lean_dec(x_24); -x_38 = !lean_is_exclusive(x_37); -if (x_38 == 0) -{ -return x_37; +lean_dec(x_1); +x_27 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_15); +return x_27; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_37, 0); -x_40 = lean_ctor_get(x_37, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_37); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_28 = lean_unsigned_to_nat(3u); +x_29 = l_Lean_Syntax_getArg(x_23, x_28); +lean_dec(x_23); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = lean_box(0); +x_32 = l_Lean_Elab_Command_elabSyntax___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_12, x_10, x_31, x_30, x_13, x_14, x_15); +return x_32; +} } } else { -lean_object* x_42; lean_object* x_43; -lean_dec(x_24); -x_42 = lean_box(0); -x_43 = l_Lean_Elab_Command_elabSyntax___lambda__7(x_22, x_12, x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_42, x_13, x_14, x_29); -return x_43; -} +lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_dec(x_17); +x_33 = lean_box(0); +x_34 = lean_box(0); +x_35 = l_Lean_Elab_Command_elabSyntax___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_12, x_10, x_34, x_33, x_13, x_14, x_15); +return x_35; } } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__9___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__10___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("namedPrio", 9); +x_1 = lean_mk_string_from_bytes("namedName", 9); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; lean_object* x_16; uint8_t x_17; @@ -18409,9 +17847,9 @@ lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint x_21 = lean_unsigned_to_nat(0u); x_22 = l_Lean_Syntax_getArg(x_16, x_21); lean_dec(x_16); -x_23 = l_Lean_Elab_Command_elabSyntax___lambda__9___closed__1; -lean_inc(x_3); -x_24 = l_Lean_Name_str___override(x_3, x_23); +x_23 = l_Lean_Elab_Command_elabSyntax___lambda__10___closed__1; +lean_inc(x_6); +x_24 = l_Lean_Name_str___override(x_6, x_23); lean_inc(x_22); x_25 = l_Lean_Syntax_isOfKind(x_22, x_24); lean_dec(x_24); @@ -18443,7 +17881,7 @@ lean_dec(x_22); x_29 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_29, 0, x_28); x_30 = lean_box(0); -x_31 = l_Lean_Elab_Command_elabSyntax___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_11, x_9, x_30, x_29, x_12, x_13, x_14); +x_31 = l_Lean_Elab_Command_elabSyntax___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_11, x_30, x_29, x_12, x_13, x_14); return x_31; } } @@ -18454,134 +17892,153 @@ lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_dec(x_16); x_32 = lean_box(0); x_33 = lean_box(0); -x_34 = l_Lean_Elab_Command_elabSyntax___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_11, x_9, x_33, x_32, x_12, x_13, x_14); +x_34 = l_Lean_Elab_Command_elabSyntax___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_11, x_33, x_32, x_12, x_13, x_14); return x_34; } } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__10___closed__1() { +static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__11___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("namedName", 9); +x_1 = lean_mk_string_from_bytes("precedence", 10); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -lean_dec(x_9); -x_14 = lean_unsigned_to_nat(4u); -x_15 = l_Lean_Syntax_getArg(x_1, x_14); -x_16 = l_Lean_Syntax_isNone(x_15); -if (x_16 == 0) -{ -lean_object* x_17; uint8_t x_18; -x_17 = lean_unsigned_to_nat(1u); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +lean_dec(x_7); +x_12 = lean_unsigned_to_nat(2u); +x_13 = l_Lean_Syntax_getArg(x_1, x_12); +x_14 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__5; +lean_inc(x_2); +x_15 = l_Lean_Name_str___override(x_2, x_14); +x_16 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__17; lean_inc(x_15); -x_18 = l_Lean_Syntax_matchesNull(x_15, x_17); +x_17 = l_Lean_Name_str___override(x_15, x_16); +lean_inc(x_13); +x_18 = l_Lean_Syntax_isOfKind(x_13, x_17); +lean_dec(x_17); if (x_18 == 0) { lean_object* x_19; lean_dec(x_15); -lean_dec(x_12); -lean_dec(x_11); +lean_dec(x_13); lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_19 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_13); +x_19 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_11); return x_19; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Syntax_getArg(x_15, x_20); -lean_dec(x_15); -x_22 = l_Lean_Elab_Command_elabSyntax___lambda__10___closed__1; -lean_inc(x_3); -x_23 = l_Lean_Name_str___override(x_3, x_22); +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_unsigned_to_nat(4u); +x_21 = l_Lean_Syntax_getArg(x_1, x_20); +x_22 = l_Lean_Syntax_isNone(x_21); +if (x_22 == 0) +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_unsigned_to_nat(1u); lean_inc(x_21); -x_24 = l_Lean_Syntax_isOfKind(x_21, x_23); -lean_dec(x_23); +x_24 = l_Lean_Syntax_matchesNull(x_21, x_23); if (x_24 == 0) { lean_object* x_25; lean_dec(x_21); -lean_dec(x_12); -lean_dec(x_11); +lean_dec(x_15); +lean_dec(x_13); lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_25 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_13); +x_25 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_11); return x_25; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_26 = lean_unsigned_to_nat(3u); +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_26 = lean_unsigned_to_nat(0u); x_27 = l_Lean_Syntax_getArg(x_21, x_26); lean_dec(x_21); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = lean_box(0); -x_30 = l_Lean_Elab_Command_elabSyntax___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_10, x_29, x_28, x_11, x_12, x_13); -return x_30; -} -} +x_28 = l_Lean_Elab_Command_elabSyntax___lambda__11___closed__1; +lean_inc(x_2); +x_29 = l_Lean_Name_str___override(x_2, x_28); +lean_inc(x_27); +x_30 = l_Lean_Syntax_isOfKind(x_27, x_29); +lean_dec(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +lean_dec(x_27); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_31 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_11); +return x_31; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -lean_dec(x_15); -x_31 = lean_box(0); -x_32 = lean_box(0); -x_33 = l_Lean_Elab_Command_elabSyntax___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_10, x_32, x_31, x_11, x_12, x_13); -return x_33; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_32 = l_Lean_Syntax_getArg(x_27, x_23); +lean_dec(x_27); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_32); +x_34 = lean_box(0); +x_35 = l_Lean_Elab_Command_elabSyntax___lambda__10(x_1, x_3, x_15, x_2, x_13, x_4, x_5, x_6, x_8, x_34, x_33, x_9, x_10, x_11); +return x_35; } } } -static lean_object* _init_l_Lean_Elab_Command_elabSyntax___lambda__11___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("precedence", 10); -return x_1; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_21); +x_36 = lean_box(0); +x_37 = lean_box(0); +x_38 = l_Lean_Elab_Command_elabSyntax___lambda__10(x_1, x_3, x_15, x_2, x_13, x_4, x_5, x_6, x_8, x_37, x_36, x_9, x_10, x_11); +return x_38; +} } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_dec(x_6); x_11 = lean_unsigned_to_nat(1u); x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__5; -lean_inc(x_2); -x_14 = l_Lean_Name_str___override(x_2, x_13); -x_15 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__17; -lean_inc(x_14); -x_16 = l_Lean_Name_str___override(x_14, x_15); +x_13 = l_Lean_Syntax_isNone(x_12); +if (x_13 == 0) +{ +uint8_t x_14; lean_inc(x_12); -x_17 = l_Lean_Syntax_isOfKind(x_12, x_16); -lean_dec(x_16); -if (x_17 == 0) +x_14 = l_Lean_Syntax_matchesNull(x_12, x_11); +if (x_14 == 0) { -lean_object* x_18; -lean_dec(x_14); +lean_object* x_15; lean_dec(x_12); lean_dec(x_9); lean_dec(x_8); @@ -18591,26 +18048,27 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_18 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_10); -return x_18; +x_15 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_10); +return x_15; } else { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_unsigned_to_nat(3u); -x_20 = l_Lean_Syntax_getArg(x_1, x_19); -x_21 = l_Lean_Syntax_isNone(x_20); -if (x_21 == 0) -{ -uint8_t x_22; -lean_inc(x_20); -x_22 = l_Lean_Syntax_matchesNull(x_20, x_11); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_16 = lean_unsigned_to_nat(0u); +x_17 = l_Lean_Syntax_getArg(x_12, x_16); +lean_dec(x_12); +x_18 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__5; +lean_inc(x_2); +x_19 = l_Lean_Name_str___override(x_2, x_18); +x_20 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotParser___closed__12; +x_21 = l_Lean_Name_str___override(x_19, x_20); +lean_inc(x_17); +x_22 = l_Lean_Syntax_isOfKind(x_17, x_21); +lean_dec(x_21); if (x_22 == 0) { lean_object* x_23; -lean_dec(x_20); -lean_dec(x_14); -lean_dec(x_12); +lean_dec(x_17); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -18624,55 +18082,27 @@ return x_23; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_Syntax_getArg(x_20, x_24); -lean_dec(x_20); -x_26 = l_Lean_Elab_Command_elabSyntax___lambda__11___closed__1; -lean_inc(x_2); -x_27 = l_Lean_Name_str___override(x_2, x_26); -lean_inc(x_25); -x_28 = l_Lean_Syntax_isOfKind(x_25, x_27); -lean_dec(x_27); -if (x_28 == 0) -{ -lean_object* x_29; -lean_dec(x_25); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_29 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Command_elabSyntax___spec__1___rarg(x_10); -return x_29; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_30 = l_Lean_Syntax_getArg(x_25, x_11); -lean_dec(x_25); -x_31 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_31, 0, x_30); -x_32 = lean_box(0); -x_33 = l_Lean_Elab_Command_elabSyntax___lambda__10(x_1, x_3, x_4, x_14, x_2, x_12, x_5, x_7, x_32, x_31, x_8, x_9, x_10); -return x_33; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_24 = l_Lean_Syntax_getArg(x_17, x_11); +lean_dec(x_17); +x_25 = l_Lean_Syntax_getArgs(x_24); +lean_dec(x_24); +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_27 = lean_box(0); +x_28 = l_Lean_Elab_Command_elabSyntax___lambda__11(x_1, x_2, x_3, x_4, x_5, x_7, x_27, x_26, x_8, x_9, x_10); +return x_28; } } } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -lean_dec(x_20); -x_34 = lean_box(0); -x_35 = lean_box(0); -x_36 = l_Lean_Elab_Command_elabSyntax___lambda__10(x_1, x_3, x_4, x_14, x_2, x_12, x_5, x_7, x_35, x_34, x_8, x_9, x_10); -return x_36; -} +lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_12); +x_29 = lean_box(0); +x_30 = lean_box(0); +x_31 = l_Lean_Elab_Command_elabSyntax___lambda__11(x_1, x_2, x_3, x_4, x_5, x_7, x_30, x_29, x_8, x_9, x_10); +return x_31; } } } @@ -18778,7 +18208,7 @@ x_20 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotPar x_21 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__2; x_22 = lean_box(0); lean_inc(x_1); -x_23 = l_Lean_Elab_Command_elabSyntax___lambda__11(x_1, x_19, x_1, x_20, x_21, x_22, x_18, x_2, x_3, x_4); +x_23 = l_Lean_Elab_Command_elabSyntax___lambda__12(x_1, x_19, x_1, x_20, x_21, x_22, x_18, x_2, x_3, x_4); return x_23; } } @@ -18793,7 +18223,7 @@ x_26 = l___private_Lean_Elab_Syntax_0__Lean_Elab_Command_declareSyntaxCatQuotPar x_27 = l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_Syntax_0__Lean_Elab_Term_mkParserSeq___spec__1___closed__2; x_28 = lean_box(0); lean_inc(x_1); -x_29 = l_Lean_Elab_Command_elabSyntax___lambda__11(x_1, x_25, x_1, x_26, x_27, x_28, x_24, x_2, x_3, x_4); +x_29 = l_Lean_Elab_Command_elabSyntax___lambda__12(x_1, x_25, x_1, x_26, x_27, x_28, x_24, x_2, x_3, x_4); return x_29; } } @@ -18915,6 +18345,81 @@ lean_dec(x_1); return x_12; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__5___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +lean_object* x_18; +x_18 = l_Lean_Elab_Command_elabSyntax___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +return x_18; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__6___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +lean_object* x_18; +x_18 = l_Lean_Elab_Command_elabSyntax___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +return x_18; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Command_elabSyntax___lambda__7___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +lean_object* x_18; +x_18 = l_Lean_Elab_Command_elabSyntax___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +return x_18; +} +} static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabSyntax___closed__1() { _start: { @@ -18969,7 +18474,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabSyntax_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(354u); +x_1 = lean_unsigned_to_nat(357u); x_2 = lean_unsigned_to_nat(43u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20160,7 +19665,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabSyntaxAbbrev_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(356u); +x_1 = lean_unsigned_to_nat(359u); x_2 = lean_unsigned_to_nat(37u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20172,7 +19677,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabSyntaxAbbrev_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(362u); +x_1 = lean_unsigned_to_nat(365u); x_2 = lean_unsigned_to_nat(49u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20200,7 +19705,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabSyntaxAbbrev_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(356u); +x_1 = lean_unsigned_to_nat(359u); x_2 = lean_unsigned_to_nat(41u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -20212,7 +19717,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Command_elabSyntaxAbbrev_decl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(356u); +x_1 = lean_unsigned_to_nat(359u); x_2 = lean_unsigned_to_nat(57u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -21370,7 +20875,7 @@ lean_dec(x_2); return x_4; } } -static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9219____closed__1() { +static lean_object* _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -21380,11 +20885,11 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9219_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9219____closed__1; +x_2 = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464____closed__1; x_3 = l_Lean_registerTraceClass(x_2, x_1); return x_3; } @@ -22036,6 +21541,8 @@ l_Lean_Elab_Command_elabSyntax___lambda__5___closed__11 = _init_l_Lean_Elab_Comm lean_mark_persistent(l_Lean_Elab_Command_elabSyntax___lambda__5___closed__11); l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12 = _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12(); lean_mark_persistent(l_Lean_Elab_Command_elabSyntax___lambda__5___closed__12); +l_Lean_Elab_Command_elabSyntax___lambda__5___closed__13 = _init_l_Lean_Elab_Command_elabSyntax___lambda__5___closed__13(); +lean_mark_persistent(l_Lean_Elab_Command_elabSyntax___lambda__5___closed__13); l_Lean_Elab_Command_elabSyntax___lambda__8___closed__1 = _init_l_Lean_Elab_Command_elabSyntax___lambda__8___closed__1(); lean_mark_persistent(l_Lean_Elab_Command_elabSyntax___lambda__8___closed__1); l_Lean_Elab_Command_elabSyntax___lambda__8___closed__2 = _init_l_Lean_Elab_Command_elabSyntax___lambda__8___closed__2(); @@ -22146,9 +21653,9 @@ l_Lean_Elab_Command_expandNoKindMacroRulesAux___lambda__1___closed__5 = _init_l_ lean_mark_persistent(l_Lean_Elab_Command_expandNoKindMacroRulesAux___lambda__1___closed__5); l_Lean_Elab_Command_expandNoKindMacroRulesAux___lambda__1___closed__6 = _init_l_Lean_Elab_Command_expandNoKindMacroRulesAux___lambda__1___closed__6(); lean_mark_persistent(l_Lean_Elab_Command_expandNoKindMacroRulesAux___lambda__1___closed__6); -l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9219____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9219____closed__1(); -lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9219____closed__1); -res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9219_(lean_io_mk_world()); +l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464____closed__1 = _init_l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464____closed__1(); +lean_mark_persistent(l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464____closed__1); +res = l_Lean_Elab_Command_initFn____x40_Lean_Elab_Syntax___hyg_9464_(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/SyntheticMVars.c b/stage0/stdlib/Lean/Elab/SyntheticMVars.c index bace6a06a547..a62b2e7442ff 100644 --- a/stage0/stdlib/Lean/Elab/SyntheticMVars.c +++ b/stage0/stdlib/Lean/Elab/SyntheticMVars.c @@ -22,6 +22,7 @@ LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVa LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefault___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_RBNode_erase___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__2; @@ -33,16 +34,19 @@ lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__7; static lean_object* l_Std_RBNode_forIn_visit___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefault___spec__2___closed__3; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__16; +lean_object* l_Lean_getDelayedMVarRoot___at_Lean_Elab_Term_isLetRecAuxMVar___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_Elab_Term_runTactic___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_occursCheck_visitMVar___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_runPendingTacticsAt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_runTactic___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_getDelayedMVarAssignment_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance(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_SyntheticMVars_0__Lean_Elab_Term_processPostponedUniverseContraints___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -79,10 +83,11 @@ uint64_t l_Lean_Level_hash(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_getMVarDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withSynthesizeLight___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__9; lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isClass_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__5; extern lean_object* l_Lean_Meta_instInhabitedPostponedEntry; lean_object* l_Lean_Meta_isSyntheticMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefault___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -95,16 +100,18 @@ size_t lean_usize_shift_right(size_t, size_t); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefault___closed__2; lean_object* l_Lean_Expr_appArg_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_instInhabitedTermElabM(lean_object*); static lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__1; -uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_101_(uint8_t, uint8_t); static lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__2___closed__1; static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___spec__1___closed__2; LEAN_EXPORT lean_object* l_Lean_occursCheck_visit___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___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_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_occursCheck_visitMVar___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getPostponed___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withSynthesize___rarg___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -123,6 +130,7 @@ static lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2; lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultLoop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___spec__1___closed__1; @@ -132,14 +140,15 @@ static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throw lean_object* l_Std_PersistentHashMap_insert___at_Lean_instantiateMVarDeclMVars___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instantiateLCtxMVars___at_Lean_Elab_Term_runTactic___spec__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___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_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__5; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar___lambda__2___closed__2; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr(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_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_RBNode_setBlack___rarg(lean_object*); lean_object* l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___closed__1; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___closed__1; LEAN_EXPORT lean_object* l_Lean_commitWhen___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizePendingInstMVar_x27___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -150,6 +159,7 @@ lean_object* l_Std_HashSetImp_insert___at_Lean_CollectMVars_visit___spec__3(lean uint8_t l_Lean_Level_normLtAux(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__4; LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingInstancesStep___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSomeUsingDefaultPrio_visit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvar___override(lean_object*); @@ -158,7 +168,8 @@ static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVa lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallMetaTelescopeReducingAux(lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846_(lean_object*); +lean_object* l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_commitWhen___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizePendingInstMVar_x27___spec__1___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizePendingInstMVar_x27___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_assignExprMVar___at_Lean_Elab_Term_exprToSyntax___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -168,16 +179,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__2(l LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentArray_get_x21___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_expandCoe(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_reportStuckSyntheticMVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabTerm(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizePending___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_instantiateLCtxMVars___at_Lean_Elab_Term_runTactic___spec__2___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___lambda__1___boxed(lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__3; -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___closed__1; uint8_t l_Lean_Expr_hasExprMVar(lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); @@ -185,19 +193,23 @@ static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synth static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSomeUsingDefaultPrio___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_replace___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__9(lean_object*, lean_object*, lean_object*); +static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__2; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefault___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__6; +lean_object* l_Std_RBNode_appendTrees___rarg(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio___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___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingInstances(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___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___spec__1___closed__3; +lean_object* l_Std_RBNode_balRight___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___closed__2; +uint8_t l_Std_RBNode_isBlack___rarg(lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__4; +uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVarsNoPostponing___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__7___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__8(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_reportStuckSyntheticMVars(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesizeSyntheticMVars_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -227,13 +239,12 @@ static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synth lean_object* lean_expr_dbg_to_string(lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumeElabTerm___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_logAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_modn(size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizePendingInstMVar_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__2___closed__3; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__17; @@ -246,16 +257,16 @@ lean_object* l_Lean_MetavarContext_getExprAssignmentCore_x3f(lean_object*, lean_ LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__9; -uint8_t l_Lean_MessageData_hasSyntheticSorry(lean_object*); +lean_object* l_Std_RBNode_balLeft___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__1; +LEAN_EXPORT lean_object* l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2___boxed(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); -static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_elem___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_runTactic(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_SyntheticMVars_0__Lean_Elab_Term_resumePostponed(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -268,8 +279,6 @@ LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at___private_Lean_Elab lean_object* l_Lean_SimplePersistentEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_withSynthesizeLight___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__8; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__2; static lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__2; LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -281,18 +290,19 @@ LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesiz static lean_object* l_Lean_markUsedAssignment___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__5___closed__1; lean_object* l_Lean_Elab_Term_withoutPostponing___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__2; +LEAN_EXPORT lean_object* l_Std_RBNode_erase___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__13; static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesizeSyntheticMVars_loop___spec__1___closed__1; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__21; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); extern lean_object* l_Lean_Elab_instInhabitedInfoTree; +lean_object* l_Lean_Meta_getMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSomeUsingDefaultPrio_visit___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_markUsedAssignment___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_List_find_x3f___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_traceAtCmdPos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_postponeExceptionId; -static lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__7; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_getDefaultInstancesPriorities___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefault___spec__1___rarg___boxed(lean_object*, lean_object*); static lean_object* l_Std_RBNode_forIn_visit___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefault___spec__2___closed__1; @@ -318,6 +328,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getDefaultInstancesPriorities___at___privat LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_ensureAtomicBinderName___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_getExprMVarAssignment_x3f___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withSynthesizeLight(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__6; @@ -334,20 +345,22 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVarsNoPostponing(u LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__15(lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_occursCheck_visit___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_runTactic___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withSynthesize___rarg(lean_object*, lean_object*, lean_object*, uint8_t); -static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getDelayedMVarAssignment_x3f___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___closed__1; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__6; lean_object* lean_panic_fn(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getDefaultInstances___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___boxed(lean_object*); lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getMVarDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_reportUnsolvedGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -355,19 +368,19 @@ lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); -lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); lean_object* l_Lean_Elab_Term_throwTypeMismatchError___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashSetImp_expand___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__5(lean_object*, lean_object*); static lean_object* l_Lean_instantiateLCtxMVars___at_Lean_Elab_Term_runTactic___spec__2___closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_runTactic___spec__7(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashSetImp_insert___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_reportStuckSyntheticMVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__1; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__8; lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__2; lean_object* l_ReaderT_pure___at_Lean_Elab_Term_addTermInfo___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___lambda__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___lambda__1(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___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__1; @@ -379,6 +392,7 @@ LEAN_EXPORT lean_object* l_Lean_occursCheck___at___private_Lean_Elab_SyntheticMV LEAN_EXPORT lean_object* l_Std_PersistentArray_foldlM___at_Lean_Elab_Term_runTactic___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashSetImp_moveEntries___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getDefaultInstancesPriorities___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefault___spec__1___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__3; static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__5; LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -396,18 +410,19 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_ lean_object* l_Lean_indentExpr(lean_object*); lean_object* l_Lean_Elab_Term_synthesizeCoeInstMVarCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__5; extern lean_object* l_Lean_Meta_defaultInstanceExtension; +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_processPostponed(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefault___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_RBNode_find___at_Lean_Meta_addDefaultInstanceEntry___spec__3(lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___closed__1; lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_runTactic___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlMAux___at_Lean_Elab_Term_runTactic___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2047,17 +2062,17 @@ lean_ctor_set(x_31, 0, x_29); x_32 = lean_st_ref_get(x_9, x_30); if (x_3 == 0) { -uint8_t x_313; -x_313 = 1; -x_33 = x_313; -goto block_312; +uint8_t x_315; +x_315 = 1; +x_33 = x_315; +goto block_314; } else { -uint8_t x_314; -x_314 = 0; -x_33 = x_314; -goto block_312; +uint8_t x_316; +x_316 = 0; +x_33 = x_316; +goto block_314; } block_23: { @@ -2115,7 +2130,7 @@ return x_22; } } } -block_312: +block_314: { lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; x_34 = lean_ctor_get(x_32, 1); @@ -2124,7 +2139,7 @@ lean_dec(x_32); x_35 = lean_st_ref_get(x_5, x_34); x_36 = lean_ctor_get(x_35, 0); lean_inc(x_36); -x_37 = lean_ctor_get(x_36, 4); +x_37 = lean_ctor_get(x_36, 5); lean_inc(x_37); lean_dec(x_36); x_38 = lean_ctor_get_uint8(x_37, sizeof(void*)*2); @@ -2355,7 +2370,7 @@ return x_88; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; lean_object* x_198; lean_object* x_199; lean_object* x_279; +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; lean_object* x_199; lean_object* x_200; lean_object* x_281; x_89 = lean_ctor_get(x_35, 1); lean_inc(x_89); lean_dec(x_35); @@ -2373,152 +2388,152 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_31); lean_inc(x_2); -x_279 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumeElabTerm(x_2, x_31, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_92); -if (lean_obj_tag(x_279) == 0) -{ -lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; -x_280 = lean_ctor_get(x_279, 0); -lean_inc(x_280); -x_281 = lean_ctor_get(x_279, 1); -lean_inc(x_281); -lean_dec(x_279); -x_282 = lean_box(0); -x_283 = lean_ctor_get(x_8, 0); +x_281 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumeElabTerm(x_2, x_31, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_92); +if (lean_obj_tag(x_281) == 0) +{ +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_282 = lean_ctor_get(x_281, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_281, 1); lean_inc(x_283); -x_284 = lean_ctor_get(x_8, 1); -lean_inc(x_284); -x_285 = lean_ctor_get(x_8, 2); +lean_dec(x_281); +x_284 = lean_box(0); +x_285 = lean_ctor_get(x_8, 0); lean_inc(x_285); -x_286 = lean_ctor_get(x_8, 3); +x_286 = lean_ctor_get(x_8, 1); lean_inc(x_286); -x_287 = lean_ctor_get(x_8, 4); +x_287 = lean_ctor_get(x_8, 2); lean_inc(x_287); -x_288 = lean_ctor_get(x_8, 5); +x_288 = lean_ctor_get(x_8, 3); lean_inc(x_288); -x_289 = lean_ctor_get(x_8, 6); +x_289 = lean_ctor_get(x_8, 4); lean_inc(x_289); -x_290 = lean_ctor_get(x_8, 7); +x_290 = lean_ctor_get(x_8, 5); lean_inc(x_290); -x_291 = lean_ctor_get(x_8, 8); +x_291 = lean_ctor_get(x_8, 6); lean_inc(x_291); -x_292 = lean_ctor_get(x_8, 9); +x_292 = lean_ctor_get(x_8, 7); lean_inc(x_292); -x_293 = lean_ctor_get(x_8, 10); +x_293 = lean_ctor_get(x_8, 8); lean_inc(x_293); -x_294 = l_Lean_replaceRef(x_2, x_288); -lean_dec(x_288); +x_294 = lean_ctor_get(x_8, 9); +lean_inc(x_294); +x_295 = lean_ctor_get(x_8, 10); +lean_inc(x_295); +x_296 = l_Lean_replaceRef(x_2, x_290); +lean_dec(x_290); lean_dec(x_2); -x_295 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_295, 0, x_283); -lean_ctor_set(x_295, 1, x_284); -lean_ctor_set(x_295, 2, x_285); -lean_ctor_set(x_295, 3, x_286); -lean_ctor_set(x_295, 4, x_287); -lean_ctor_set(x_295, 5, x_294); -lean_ctor_set(x_295, 6, x_289); -lean_ctor_set(x_295, 7, x_290); -lean_ctor_set(x_295, 8, x_291); -lean_ctor_set(x_295, 9, x_292); -lean_ctor_set(x_295, 10, x_293); +x_297 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_297, 0, x_285); +lean_ctor_set(x_297, 1, x_286); +lean_ctor_set(x_297, 2, x_287); +lean_ctor_set(x_297, 3, x_288); +lean_ctor_set(x_297, 4, x_289); +lean_ctor_set(x_297, 5, x_296); +lean_ctor_set(x_297, 6, x_291); +lean_ctor_set(x_297, 7, x_292); +lean_ctor_set(x_297, 8, x_293); +lean_ctor_set(x_297, 9, x_294); +lean_ctor_set(x_297, 10, x_295); lean_inc(x_9); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_296 = l_Lean_Elab_Term_ensureHasType(x_31, x_280, x_282, x_4, x_5, x_6, x_7, x_295, x_9, x_281); -if (lean_obj_tag(x_296) == 0) -{ -lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; uint8_t x_301; -x_297 = lean_ctor_get(x_296, 0); -lean_inc(x_297); -x_298 = lean_ctor_get(x_296, 1); -lean_inc(x_298); -lean_dec(x_296); +x_298 = l_Lean_Elab_Term_ensureHasType(x_31, x_282, x_284, x_4, x_5, x_6, x_7, x_297, x_9, x_283); +if (lean_obj_tag(x_298) == 0) +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; uint8_t x_303; +x_299 = lean_ctor_get(x_298, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_298, 1); +lean_inc(x_300); +lean_dec(x_298); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_297); -x_299 = l_Lean_occursCheck___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__1(x_1, x_297, x_4, x_5, x_6, x_7, x_8, x_9, x_298); -x_300 = lean_ctor_get(x_299, 0); -lean_inc(x_300); -x_301 = lean_unbox(x_300); -lean_dec(x_300); -if (x_301 == 0) +lean_inc(x_299); +x_301 = l_Lean_occursCheck___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___spec__1(x_1, x_299, x_4, x_5, x_6, x_7, x_8, x_9, x_300); +x_302 = lean_ctor_get(x_301, 0); +lean_inc(x_302); +x_303 = lean_unbox(x_302); +lean_dec(x_302); +if (x_303 == 0) { -lean_object* x_302; uint8_t x_303; -lean_dec(x_297); +lean_object* x_304; uint8_t x_305; +lean_dec(x_299); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_302 = lean_ctor_get(x_299, 1); -lean_inc(x_302); -lean_dec(x_299); -x_303 = 0; -x_93 = x_303; -x_94 = x_302; -goto block_197; +x_304 = lean_ctor_get(x_301, 1); +lean_inc(x_304); +lean_dec(x_301); +x_305 = 0; +x_93 = x_305; +x_94 = x_304; +goto block_198; } else { -lean_object* x_304; lean_object* x_305; lean_object* x_306; uint8_t x_307; -x_304 = lean_ctor_get(x_299, 1); -lean_inc(x_304); -lean_dec(x_299); +lean_object* x_306; lean_object* x_307; lean_object* x_308; uint8_t x_309; +x_306 = lean_ctor_get(x_301, 1); +lean_inc(x_306); +lean_dec(x_301); lean_inc(x_1); -x_305 = l_Lean_assignExprMVar___at_Lean_Elab_Term_exprToSyntax___spec__2(x_1, x_297, x_4, x_5, x_6, x_7, x_8, x_9, x_304); +x_307 = l_Lean_assignExprMVar___at_Lean_Elab_Term_exprToSyntax___spec__2(x_1, x_299, x_4, x_5, x_6, x_7, x_8, x_9, x_306); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_306 = lean_ctor_get(x_305, 1); -lean_inc(x_306); -lean_dec(x_305); -x_307 = 1; -x_93 = x_307; -x_94 = x_306; -goto block_197; +x_308 = lean_ctor_get(x_307, 1); +lean_inc(x_308); +lean_dec(x_307); +x_309 = 1; +x_93 = x_309; +x_94 = x_308; +goto block_198; } } else { -lean_object* x_308; lean_object* x_309; +lean_object* x_310; lean_object* x_311; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_308 = lean_ctor_get(x_296, 0); -lean_inc(x_308); -x_309 = lean_ctor_get(x_296, 1); -lean_inc(x_309); -lean_dec(x_296); -x_198 = x_308; -x_199 = x_309; -goto block_278; +x_310 = lean_ctor_get(x_298, 0); +lean_inc(x_310); +x_311 = lean_ctor_get(x_298, 1); +lean_inc(x_311); +lean_dec(x_298); +x_199 = x_310; +x_200 = x_311; +goto block_280; } } else { -lean_object* x_310; lean_object* x_311; +lean_object* x_312; lean_object* x_313; lean_dec(x_31); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_2); -x_310 = lean_ctor_get(x_279, 0); -lean_inc(x_310); -x_311 = lean_ctor_get(x_279, 1); -lean_inc(x_311); -lean_dec(x_279); -x_198 = x_310; -x_199 = x_311; -goto block_278; +x_312 = lean_ctor_get(x_281, 0); +lean_inc(x_312); +x_313 = lean_ctor_get(x_281, 1); +lean_inc(x_313); +lean_dec(x_281); +x_199 = x_312; +x_200 = x_313; +goto block_280; } -block_197: +block_198: { lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; uint8_t x_101; x_95 = lean_st_ref_get(x_9, x_94); @@ -2529,7 +2544,7 @@ lean_dec(x_95); x_97 = lean_st_ref_take(x_5, x_96); x_98 = lean_ctor_get(x_97, 0); lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 4); +x_99 = lean_ctor_get(x_98, 5); lean_inc(x_99); x_100 = lean_ctor_get(x_97, 1); lean_inc(x_100); @@ -2538,7 +2553,7 @@ x_101 = !lean_is_exclusive(x_98); if (x_101 == 0) { lean_object* x_102; uint8_t x_103; -x_102 = lean_ctor_get(x_98, 4); +x_102 = lean_ctor_get(x_98, 5); lean_dec(x_102); x_103 = !lean_is_exclusive(x_99); if (x_103 == 0) @@ -2663,7 +2678,7 @@ x_142 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_142, 0, x_137); lean_ctor_set(x_142, 1, x_91); lean_ctor_set_uint8(x_142, sizeof(void*)*2, x_136); -lean_ctor_set(x_98, 4, x_142); +lean_ctor_set(x_98, 5, x_142); x_143 = lean_st_ref_set(x_5, x_98, x_100); lean_dec(x_5); x_144 = lean_ctor_get(x_143, 1); @@ -2705,7 +2720,7 @@ x_155 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_155, 0, x_154); lean_ctor_set(x_155, 1, x_91); lean_ctor_set_uint8(x_155, sizeof(void*)*2, x_136); -lean_ctor_set(x_98, 4, x_155); +lean_ctor_set(x_98, 5, x_155); x_156 = lean_st_ref_set(x_5, x_98, x_100); lean_dec(x_5); x_157 = lean_ctor_get(x_156, 1); @@ -2737,441 +2752,449 @@ goto block_23; } else { -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; uint8_t x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; uint8_t x_173; +lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; uint8_t x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; x_163 = lean_ctor_get(x_98, 0); x_164 = lean_ctor_get(x_98, 1); x_165 = lean_ctor_get(x_98, 2); x_166 = lean_ctor_get(x_98, 3); +x_167 = lean_ctor_get(x_98, 4); +lean_inc(x_167); lean_inc(x_166); lean_inc(x_165); lean_inc(x_164); lean_inc(x_163); lean_dec(x_98); -x_167 = lean_ctor_get_uint8(x_99, sizeof(void*)*2); -x_168 = lean_ctor_get(x_99, 0); -lean_inc(x_168); -x_169 = lean_ctor_get(x_99, 1); +x_168 = lean_ctor_get_uint8(x_99, sizeof(void*)*2); +x_169 = lean_ctor_get(x_99, 0); lean_inc(x_169); +x_170 = lean_ctor_get(x_99, 1); +lean_inc(x_170); if (lean_is_exclusive(x_99)) { lean_ctor_release(x_99, 0); lean_ctor_release(x_99, 1); - x_170 = x_99; + x_171 = x_99; } else { lean_dec_ref(x_99); - x_170 = lean_box(0); + x_171 = lean_box(0); } -x_171 = lean_ctor_get(x_169, 2); -lean_inc(x_171); -x_172 = lean_unsigned_to_nat(0u); -x_173 = lean_nat_dec_lt(x_172, x_171); -if (x_173 == 0) +x_172 = lean_ctor_get(x_170, 2); +lean_inc(x_172); +x_173 = lean_unsigned_to_nat(0u); +x_174 = lean_nat_dec_lt(x_173, x_172); +if (x_174 == 0) { -lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -lean_dec(x_171); -lean_dec(x_169); +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_dec(x_172); +lean_dec(x_170); lean_dec(x_1); -if (lean_is_scalar(x_170)) { - x_174 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_171)) { + x_175 = lean_alloc_ctor(0, 2, 1); } else { - x_174 = x_170; -} -lean_ctor_set(x_174, 0, x_168); -lean_ctor_set(x_174, 1, x_91); -lean_ctor_set_uint8(x_174, sizeof(void*)*2, x_167); -x_175 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_175, 0, x_163); -lean_ctor_set(x_175, 1, x_164); -lean_ctor_set(x_175, 2, x_165); -lean_ctor_set(x_175, 3, x_166); -lean_ctor_set(x_175, 4, x_174); -x_176 = lean_st_ref_set(x_5, x_175, x_100); + x_175 = x_171; +} +lean_ctor_set(x_175, 0, x_169); +lean_ctor_set(x_175, 1, x_91); +lean_ctor_set_uint8(x_175, sizeof(void*)*2, x_168); +x_176 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_176, 0, x_163); +lean_ctor_set(x_176, 1, x_164); +lean_ctor_set(x_176, 2, x_165); +lean_ctor_set(x_176, 3, x_166); +lean_ctor_set(x_176, 4, x_167); +lean_ctor_set(x_176, 5, x_175); +x_177 = lean_st_ref_set(x_5, x_176, x_100); lean_dec(x_5); -x_177 = lean_ctor_get(x_176, 1); -lean_inc(x_177); -if (lean_is_exclusive(x_176)) { - lean_ctor_release(x_176, 0); - lean_ctor_release(x_176, 1); - x_178 = x_176; +x_178 = lean_ctor_get(x_177, 1); +lean_inc(x_178); +if (lean_is_exclusive(x_177)) { + lean_ctor_release(x_177, 0); + lean_ctor_release(x_177, 1); + x_179 = x_177; } else { - lean_dec_ref(x_176); - x_178 = lean_box(0); + lean_dec_ref(x_177); + x_179 = lean_box(0); } -x_179 = lean_box(0); -x_180 = lean_box(x_93); -x_181 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_181, 0, x_180); -lean_ctor_set(x_181, 1, x_179); -if (lean_is_scalar(x_178)) { - x_182 = lean_alloc_ctor(0, 2, 0); +x_180 = lean_box(0); +x_181 = lean_box(x_93); +x_182 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_182, 0, x_181); +lean_ctor_set(x_182, 1, x_180); +if (lean_is_scalar(x_179)) { + x_183 = lean_alloc_ctor(0, 2, 0); } else { - x_182 = x_178; + x_183 = x_179; } -lean_ctor_set(x_182, 0, x_181); -lean_ctor_set(x_182, 1, x_177); -x_11 = x_182; +lean_ctor_set(x_183, 0, x_182); +lean_ctor_set(x_183, 1, x_178); +x_11 = x_183; goto block_23; } else { -lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; -x_183 = lean_unsigned_to_nat(1u); -x_184 = lean_nat_sub(x_171, x_183); -lean_dec(x_171); -x_185 = l_Lean_Elab_instInhabitedInfoTree; -x_186 = l_Std_PersistentArray_get_x21___rarg(x_185, x_169, x_184); -lean_dec(x_184); -x_187 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_168, x_1, x_186); -if (lean_is_scalar(x_170)) { - x_188 = lean_alloc_ctor(0, 2, 1); +lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; +x_184 = lean_unsigned_to_nat(1u); +x_185 = lean_nat_sub(x_172, x_184); +lean_dec(x_172); +x_186 = l_Lean_Elab_instInhabitedInfoTree; +x_187 = l_Std_PersistentArray_get_x21___rarg(x_186, x_170, x_185); +lean_dec(x_185); +x_188 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_169, x_1, x_187); +if (lean_is_scalar(x_171)) { + x_189 = lean_alloc_ctor(0, 2, 1); } else { - x_188 = x_170; -} -lean_ctor_set(x_188, 0, x_187); -lean_ctor_set(x_188, 1, x_91); -lean_ctor_set_uint8(x_188, sizeof(void*)*2, x_167); -x_189 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_189, 0, x_163); -lean_ctor_set(x_189, 1, x_164); -lean_ctor_set(x_189, 2, x_165); -lean_ctor_set(x_189, 3, x_166); -lean_ctor_set(x_189, 4, x_188); -x_190 = lean_st_ref_set(x_5, x_189, x_100); + x_189 = x_171; +} +lean_ctor_set(x_189, 0, x_188); +lean_ctor_set(x_189, 1, x_91); +lean_ctor_set_uint8(x_189, sizeof(void*)*2, x_168); +x_190 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_190, 0, x_163); +lean_ctor_set(x_190, 1, x_164); +lean_ctor_set(x_190, 2, x_165); +lean_ctor_set(x_190, 3, x_166); +lean_ctor_set(x_190, 4, x_167); +lean_ctor_set(x_190, 5, x_189); +x_191 = lean_st_ref_set(x_5, x_190, x_100); lean_dec(x_5); -x_191 = lean_ctor_get(x_190, 1); -lean_inc(x_191); -if (lean_is_exclusive(x_190)) { - lean_ctor_release(x_190, 0); - lean_ctor_release(x_190, 1); - x_192 = x_190; -} else { - lean_dec_ref(x_190); - x_192 = lean_box(0); -} -x_193 = lean_box(0); -x_194 = lean_box(x_93); -x_195 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_195, 0, x_194); -lean_ctor_set(x_195, 1, x_193); -if (lean_is_scalar(x_192)) { - x_196 = lean_alloc_ctor(0, 2, 0); +x_192 = lean_ctor_get(x_191, 1); +lean_inc(x_192); +if (lean_is_exclusive(x_191)) { + lean_ctor_release(x_191, 0); + lean_ctor_release(x_191, 1); + x_193 = x_191; } else { - x_196 = x_192; + lean_dec_ref(x_191); + x_193 = lean_box(0); } +x_194 = lean_box(0); +x_195 = lean_box(x_93); +x_196 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_196, 0, x_195); -lean_ctor_set(x_196, 1, x_191); -x_11 = x_196; +lean_ctor_set(x_196, 1, x_194); +if (lean_is_scalar(x_193)) { + x_197 = lean_alloc_ctor(0, 2, 0); +} else { + x_197 = x_193; +} +lean_ctor_set(x_197, 0, x_196); +lean_ctor_set(x_197, 1, x_192); +x_11 = x_197; goto block_23; } } } -block_278: +block_280: { -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_206; -x_200 = lean_st_ref_get(x_9, x_199); +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; uint8_t x_207; +x_201 = lean_st_ref_get(x_9, x_200); lean_dec(x_9); -x_201 = lean_ctor_get(x_200, 1); -lean_inc(x_201); -lean_dec(x_200); -x_202 = lean_st_ref_take(x_5, x_201); -x_203 = lean_ctor_get(x_202, 0); -lean_inc(x_203); -x_204 = lean_ctor_get(x_203, 4); +x_202 = lean_ctor_get(x_201, 1); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_st_ref_take(x_5, x_202); +x_204 = lean_ctor_get(x_203, 0); lean_inc(x_204); -x_205 = lean_ctor_get(x_202, 1); +x_205 = lean_ctor_get(x_204, 5); lean_inc(x_205); -lean_dec(x_202); -x_206 = !lean_is_exclusive(x_203); -if (x_206 == 0) +x_206 = lean_ctor_get(x_203, 1); +lean_inc(x_206); +lean_dec(x_203); +x_207 = !lean_is_exclusive(x_204); +if (x_207 == 0) { -lean_object* x_207; uint8_t x_208; -x_207 = lean_ctor_get(x_203, 4); -lean_dec(x_207); -x_208 = !lean_is_exclusive(x_204); -if (x_208 == 0) +lean_object* x_208; uint8_t x_209; +x_208 = lean_ctor_get(x_204, 5); +lean_dec(x_208); +x_209 = !lean_is_exclusive(x_205); +if (x_209 == 0) { -lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; uint8_t x_213; -x_209 = lean_ctor_get(x_204, 0); -x_210 = lean_ctor_get(x_204, 1); -x_211 = lean_ctor_get(x_210, 2); -lean_inc(x_211); -x_212 = lean_unsigned_to_nat(0u); -x_213 = lean_nat_dec_lt(x_212, x_211); -if (x_213 == 0) +lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; uint8_t x_214; +x_210 = lean_ctor_get(x_205, 0); +x_211 = lean_ctor_get(x_205, 1); +x_212 = lean_ctor_get(x_211, 2); +lean_inc(x_212); +x_213 = lean_unsigned_to_nat(0u); +x_214 = lean_nat_dec_lt(x_213, x_212); +if (x_214 == 0) { -lean_object* x_214; uint8_t x_215; +lean_object* x_215; uint8_t x_216; +lean_dec(x_212); lean_dec(x_211); -lean_dec(x_210); lean_dec(x_1); -lean_ctor_set(x_204, 1, x_91); -x_214 = lean_st_ref_set(x_5, x_203, x_205); +lean_ctor_set(x_205, 1, x_91); +x_215 = lean_st_ref_set(x_5, x_204, x_206); lean_dec(x_5); -x_215 = !lean_is_exclusive(x_214); -if (x_215 == 0) +x_216 = !lean_is_exclusive(x_215); +if (x_216 == 0) { -lean_object* x_216; -x_216 = lean_ctor_get(x_214, 0); -lean_dec(x_216); -lean_ctor_set_tag(x_214, 1); -lean_ctor_set(x_214, 0, x_198); -x_11 = x_214; +lean_object* x_217; +x_217 = lean_ctor_get(x_215, 0); +lean_dec(x_217); +lean_ctor_set_tag(x_215, 1); +lean_ctor_set(x_215, 0, x_199); +x_11 = x_215; goto block_23; } else { -lean_object* x_217; lean_object* x_218; -x_217 = lean_ctor_get(x_214, 1); -lean_inc(x_217); -lean_dec(x_214); -x_218 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_218, 0, x_198); -lean_ctor_set(x_218, 1, x_217); -x_11 = x_218; +lean_object* x_218; lean_object* x_219; +x_218 = lean_ctor_get(x_215, 1); +lean_inc(x_218); +lean_dec(x_215); +x_219 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_219, 0, x_199); +lean_ctor_set(x_219, 1, x_218); +x_11 = x_219; goto block_23; } } else { -lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; uint8_t x_225; -x_219 = lean_unsigned_to_nat(1u); -x_220 = lean_nat_sub(x_211, x_219); -lean_dec(x_211); -x_221 = l_Lean_Elab_instInhabitedInfoTree; -x_222 = l_Std_PersistentArray_get_x21___rarg(x_221, x_210, x_220); -lean_dec(x_220); -x_223 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_209, x_1, x_222); -lean_ctor_set(x_204, 1, x_91); -lean_ctor_set(x_204, 0, x_223); -x_224 = lean_st_ref_set(x_5, x_203, x_205); +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; uint8_t x_226; +x_220 = lean_unsigned_to_nat(1u); +x_221 = lean_nat_sub(x_212, x_220); +lean_dec(x_212); +x_222 = l_Lean_Elab_instInhabitedInfoTree; +x_223 = l_Std_PersistentArray_get_x21___rarg(x_222, x_211, x_221); +lean_dec(x_221); +x_224 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_210, x_1, x_223); +lean_ctor_set(x_205, 1, x_91); +lean_ctor_set(x_205, 0, x_224); +x_225 = lean_st_ref_set(x_5, x_204, x_206); lean_dec(x_5); -x_225 = !lean_is_exclusive(x_224); -if (x_225 == 0) +x_226 = !lean_is_exclusive(x_225); +if (x_226 == 0) { -lean_object* x_226; -x_226 = lean_ctor_get(x_224, 0); -lean_dec(x_226); -lean_ctor_set_tag(x_224, 1); -lean_ctor_set(x_224, 0, x_198); -x_11 = x_224; +lean_object* x_227; +x_227 = lean_ctor_get(x_225, 0); +lean_dec(x_227); +lean_ctor_set_tag(x_225, 1); +lean_ctor_set(x_225, 0, x_199); +x_11 = x_225; goto block_23; } else { -lean_object* x_227; lean_object* x_228; -x_227 = lean_ctor_get(x_224, 1); -lean_inc(x_227); -lean_dec(x_224); -x_228 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_228, 0, x_198); -lean_ctor_set(x_228, 1, x_227); -x_11 = x_228; +lean_object* x_228; lean_object* x_229; +x_228 = lean_ctor_get(x_225, 1); +lean_inc(x_228); +lean_dec(x_225); +x_229 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_229, 0, x_199); +lean_ctor_set(x_229, 1, x_228); +x_11 = x_229; goto block_23; } } } else { -uint8_t x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; uint8_t x_234; -x_229 = lean_ctor_get_uint8(x_204, sizeof(void*)*2); -x_230 = lean_ctor_get(x_204, 0); -x_231 = lean_ctor_get(x_204, 1); -lean_inc(x_231); -lean_inc(x_230); -lean_dec(x_204); -x_232 = lean_ctor_get(x_231, 2); +uint8_t x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; uint8_t x_235; +x_230 = lean_ctor_get_uint8(x_205, sizeof(void*)*2); +x_231 = lean_ctor_get(x_205, 0); +x_232 = lean_ctor_get(x_205, 1); lean_inc(x_232); -x_233 = lean_unsigned_to_nat(0u); -x_234 = lean_nat_dec_lt(x_233, x_232); -if (x_234 == 0) +lean_inc(x_231); +lean_dec(x_205); +x_233 = lean_ctor_get(x_232, 2); +lean_inc(x_233); +x_234 = lean_unsigned_to_nat(0u); +x_235 = lean_nat_dec_lt(x_234, x_233); +if (x_235 == 0) { -lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; +lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; +lean_dec(x_233); lean_dec(x_232); -lean_dec(x_231); lean_dec(x_1); -x_235 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_235, 0, x_230); -lean_ctor_set(x_235, 1, x_91); -lean_ctor_set_uint8(x_235, sizeof(void*)*2, x_229); -lean_ctor_set(x_203, 4, x_235); -x_236 = lean_st_ref_set(x_5, x_203, x_205); +x_236 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_236, 0, x_231); +lean_ctor_set(x_236, 1, x_91); +lean_ctor_set_uint8(x_236, sizeof(void*)*2, x_230); +lean_ctor_set(x_204, 5, x_236); +x_237 = lean_st_ref_set(x_5, x_204, x_206); lean_dec(x_5); -x_237 = lean_ctor_get(x_236, 1); -lean_inc(x_237); -if (lean_is_exclusive(x_236)) { - lean_ctor_release(x_236, 0); - lean_ctor_release(x_236, 1); - x_238 = x_236; +x_238 = lean_ctor_get(x_237, 1); +lean_inc(x_238); +if (lean_is_exclusive(x_237)) { + lean_ctor_release(x_237, 0); + lean_ctor_release(x_237, 1); + x_239 = x_237; } else { - lean_dec_ref(x_236); - x_238 = lean_box(0); + lean_dec_ref(x_237); + x_239 = lean_box(0); } -if (lean_is_scalar(x_238)) { - x_239 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_239)) { + x_240 = lean_alloc_ctor(1, 2, 0); } else { - x_239 = x_238; - lean_ctor_set_tag(x_239, 1); + x_240 = x_239; + lean_ctor_set_tag(x_240, 1); } -lean_ctor_set(x_239, 0, x_198); -lean_ctor_set(x_239, 1, x_237); -x_11 = x_239; +lean_ctor_set(x_240, 0, x_199); +lean_ctor_set(x_240, 1, x_238); +x_11 = x_240; goto block_23; } else { -lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; -x_240 = lean_unsigned_to_nat(1u); -x_241 = lean_nat_sub(x_232, x_240); -lean_dec(x_232); -x_242 = l_Lean_Elab_instInhabitedInfoTree; -x_243 = l_Std_PersistentArray_get_x21___rarg(x_242, x_231, x_241); -lean_dec(x_241); -x_244 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_230, x_1, x_243); -x_245 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_245, 0, x_244); -lean_ctor_set(x_245, 1, x_91); -lean_ctor_set_uint8(x_245, sizeof(void*)*2, x_229); -lean_ctor_set(x_203, 4, x_245); -x_246 = lean_st_ref_set(x_5, x_203, x_205); +lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; +x_241 = lean_unsigned_to_nat(1u); +x_242 = lean_nat_sub(x_233, x_241); +lean_dec(x_233); +x_243 = l_Lean_Elab_instInhabitedInfoTree; +x_244 = l_Std_PersistentArray_get_x21___rarg(x_243, x_232, x_242); +lean_dec(x_242); +x_245 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_231, x_1, x_244); +x_246 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_246, 0, x_245); +lean_ctor_set(x_246, 1, x_91); +lean_ctor_set_uint8(x_246, sizeof(void*)*2, x_230); +lean_ctor_set(x_204, 5, x_246); +x_247 = lean_st_ref_set(x_5, x_204, x_206); lean_dec(x_5); -x_247 = lean_ctor_get(x_246, 1); -lean_inc(x_247); -if (lean_is_exclusive(x_246)) { - lean_ctor_release(x_246, 0); - lean_ctor_release(x_246, 1); - x_248 = x_246; +x_248 = lean_ctor_get(x_247, 1); +lean_inc(x_248); +if (lean_is_exclusive(x_247)) { + lean_ctor_release(x_247, 0); + lean_ctor_release(x_247, 1); + x_249 = x_247; } else { - lean_dec_ref(x_246); - x_248 = lean_box(0); + lean_dec_ref(x_247); + x_249 = lean_box(0); } -if (lean_is_scalar(x_248)) { - x_249 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_249)) { + x_250 = lean_alloc_ctor(1, 2, 0); } else { - x_249 = x_248; - lean_ctor_set_tag(x_249, 1); + x_250 = x_249; + lean_ctor_set_tag(x_250, 1); } -lean_ctor_set(x_249, 0, x_198); -lean_ctor_set(x_249, 1, x_247); -x_11 = x_249; +lean_ctor_set(x_250, 0, x_199); +lean_ctor_set(x_250, 1, x_248); +x_11 = x_250; goto block_23; } } } else { -lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; uint8_t x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; uint8_t x_260; -x_250 = lean_ctor_get(x_203, 0); -x_251 = lean_ctor_get(x_203, 1); -x_252 = lean_ctor_get(x_203, 2); -x_253 = lean_ctor_get(x_203, 3); +lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; uint8_t x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; uint8_t x_262; +x_251 = lean_ctor_get(x_204, 0); +x_252 = lean_ctor_get(x_204, 1); +x_253 = lean_ctor_get(x_204, 2); +x_254 = lean_ctor_get(x_204, 3); +x_255 = lean_ctor_get(x_204, 4); +lean_inc(x_255); +lean_inc(x_254); lean_inc(x_253); lean_inc(x_252); lean_inc(x_251); -lean_inc(x_250); -lean_dec(x_203); -x_254 = lean_ctor_get_uint8(x_204, sizeof(void*)*2); -x_255 = lean_ctor_get(x_204, 0); -lean_inc(x_255); -x_256 = lean_ctor_get(x_204, 1); -lean_inc(x_256); -if (lean_is_exclusive(x_204)) { - lean_ctor_release(x_204, 0); - lean_ctor_release(x_204, 1); - x_257 = x_204; +lean_dec(x_204); +x_256 = lean_ctor_get_uint8(x_205, sizeof(void*)*2); +x_257 = lean_ctor_get(x_205, 0); +lean_inc(x_257); +x_258 = lean_ctor_get(x_205, 1); +lean_inc(x_258); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + x_259 = x_205; } else { - lean_dec_ref(x_204); - x_257 = lean_box(0); + lean_dec_ref(x_205); + x_259 = lean_box(0); } -x_258 = lean_ctor_get(x_256, 2); -lean_inc(x_258); -x_259 = lean_unsigned_to_nat(0u); -x_260 = lean_nat_dec_lt(x_259, x_258); -if (x_260 == 0) +x_260 = lean_ctor_get(x_258, 2); +lean_inc(x_260); +x_261 = lean_unsigned_to_nat(0u); +x_262 = lean_nat_dec_lt(x_261, x_260); +if (x_262 == 0) { -lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; +lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +lean_dec(x_260); lean_dec(x_258); -lean_dec(x_256); lean_dec(x_1); -if (lean_is_scalar(x_257)) { - x_261 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_259)) { + x_263 = lean_alloc_ctor(0, 2, 1); } else { - x_261 = x_257; -} -lean_ctor_set(x_261, 0, x_255); -lean_ctor_set(x_261, 1, x_91); -lean_ctor_set_uint8(x_261, sizeof(void*)*2, x_254); -x_262 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_262, 0, x_250); -lean_ctor_set(x_262, 1, x_251); -lean_ctor_set(x_262, 2, x_252); -lean_ctor_set(x_262, 3, x_253); -lean_ctor_set(x_262, 4, x_261); -x_263 = lean_st_ref_set(x_5, x_262, x_205); + x_263 = x_259; +} +lean_ctor_set(x_263, 0, x_257); +lean_ctor_set(x_263, 1, x_91); +lean_ctor_set_uint8(x_263, sizeof(void*)*2, x_256); +x_264 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_264, 0, x_251); +lean_ctor_set(x_264, 1, x_252); +lean_ctor_set(x_264, 2, x_253); +lean_ctor_set(x_264, 3, x_254); +lean_ctor_set(x_264, 4, x_255); +lean_ctor_set(x_264, 5, x_263); +x_265 = lean_st_ref_set(x_5, x_264, x_206); lean_dec(x_5); -x_264 = lean_ctor_get(x_263, 1); -lean_inc(x_264); -if (lean_is_exclusive(x_263)) { - lean_ctor_release(x_263, 0); - lean_ctor_release(x_263, 1); - x_265 = x_263; +x_266 = lean_ctor_get(x_265, 1); +lean_inc(x_266); +if (lean_is_exclusive(x_265)) { + lean_ctor_release(x_265, 0); + lean_ctor_release(x_265, 1); + x_267 = x_265; } else { - lean_dec_ref(x_263); - x_265 = lean_box(0); + lean_dec_ref(x_265); + x_267 = lean_box(0); } -if (lean_is_scalar(x_265)) { - x_266 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_267)) { + x_268 = lean_alloc_ctor(1, 2, 0); } else { - x_266 = x_265; - lean_ctor_set_tag(x_266, 1); + x_268 = x_267; + lean_ctor_set_tag(x_268, 1); } -lean_ctor_set(x_266, 0, x_198); -lean_ctor_set(x_266, 1, x_264); -x_11 = x_266; +lean_ctor_set(x_268, 0, x_199); +lean_ctor_set(x_268, 1, x_266); +x_11 = x_268; goto block_23; } else { -lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; -x_267 = lean_unsigned_to_nat(1u); -x_268 = lean_nat_sub(x_258, x_267); -lean_dec(x_258); -x_269 = l_Lean_Elab_instInhabitedInfoTree; -x_270 = l_Std_PersistentArray_get_x21___rarg(x_269, x_256, x_268); -lean_dec(x_268); -x_271 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_255, x_1, x_270); -if (lean_is_scalar(x_257)) { - x_272 = lean_alloc_ctor(0, 2, 1); +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; +x_269 = lean_unsigned_to_nat(1u); +x_270 = lean_nat_sub(x_260, x_269); +lean_dec(x_260); +x_271 = l_Lean_Elab_instInhabitedInfoTree; +x_272 = l_Std_PersistentArray_get_x21___rarg(x_271, x_258, x_270); +lean_dec(x_270); +x_273 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_257, x_1, x_272); +if (lean_is_scalar(x_259)) { + x_274 = lean_alloc_ctor(0, 2, 1); } else { - x_272 = x_257; -} -lean_ctor_set(x_272, 0, x_271); -lean_ctor_set(x_272, 1, x_91); -lean_ctor_set_uint8(x_272, sizeof(void*)*2, x_254); -x_273 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_273, 0, x_250); -lean_ctor_set(x_273, 1, x_251); -lean_ctor_set(x_273, 2, x_252); -lean_ctor_set(x_273, 3, x_253); -lean_ctor_set(x_273, 4, x_272); -x_274 = lean_st_ref_set(x_5, x_273, x_205); + x_274 = x_259; +} +lean_ctor_set(x_274, 0, x_273); +lean_ctor_set(x_274, 1, x_91); +lean_ctor_set_uint8(x_274, sizeof(void*)*2, x_256); +x_275 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_275, 0, x_251); +lean_ctor_set(x_275, 1, x_252); +lean_ctor_set(x_275, 2, x_253); +lean_ctor_set(x_275, 3, x_254); +lean_ctor_set(x_275, 4, x_255); +lean_ctor_set(x_275, 5, x_274); +x_276 = lean_st_ref_set(x_5, x_275, x_206); lean_dec(x_5); -x_275 = lean_ctor_get(x_274, 1); -lean_inc(x_275); -if (lean_is_exclusive(x_274)) { - lean_ctor_release(x_274, 0); - lean_ctor_release(x_274, 1); - x_276 = x_274; +x_277 = lean_ctor_get(x_276, 1); +lean_inc(x_277); +if (lean_is_exclusive(x_276)) { + lean_ctor_release(x_276, 0); + lean_ctor_release(x_276, 1); + x_278 = x_276; } else { - lean_dec_ref(x_274); - x_276 = lean_box(0); + lean_dec_ref(x_276); + x_278 = lean_box(0); } -if (lean_is_scalar(x_276)) { - x_277 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_278)) { + x_279 = lean_alloc_ctor(1, 2, 0); } else { - x_277 = x_276; - lean_ctor_set_tag(x_277, 1); + x_279 = x_278; + lean_ctor_set_tag(x_279, 1); } -lean_ctor_set(x_277, 0, x_198); -lean_ctor_set(x_277, 1, x_275); -x_11 = x_277; +lean_ctor_set(x_279, 0, x_199); +lean_ctor_set(x_279, 1, x_277); +x_11 = x_279; goto block_23; } } @@ -3217,214 +3240,213 @@ return x_1; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_17 = lean_st_ref_get(x_10, x_11); -x_18 = lean_ctor_get(x_17, 1); +lean_object* x_12; lean_object* x_13; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_17 = l_Lean_Elab_Term_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11); +x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); lean_dec(x_17); -x_19 = lean_st_ref_get(x_6, x_18); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_box(x_3); -x_23 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__1___boxed), 10, 3); -lean_closure_set(x_23, 0, x_1); -lean_closure_set(x_23, 1, x_2); -lean_closure_set(x_23, 2, x_22); +x_20 = lean_box(x_3); +x_21 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__1___boxed), 10, 3); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_2); +lean_closure_set(x_21, 2, x_20); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_24 = l_Lean_Elab_Term_withSavedContext___rarg(x_4, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_21); -if (lean_obj_tag(x_24) == 0) +x_22 = l_Lean_Elab_Term_withSavedContext___rarg(x_4, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_19); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -lean_dec(x_20); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_dec(x_18); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_box(0); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_25); -lean_ctor_set(x_28, 1, x_27); -x_12 = x_28; -x_13 = x_26; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_box(0); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_23); +lean_ctor_set(x_26, 1, x_25); +x_12 = x_26; +x_13 = x_24; goto block_16; } else { -lean_object* x_29; -x_29 = lean_ctor_get(x_24, 0); -lean_inc(x_29); -if (lean_obj_tag(x_29) == 0) +lean_object* x_27; +x_27 = lean_ctor_get(x_22, 0); +lean_inc(x_27); +if (lean_obj_tag(x_27) == 0) { if (x_3 == 0) { +lean_object* x_28; lean_object* x_29; +lean_dec(x_18); +x_28 = lean_ctor_get(x_22, 1); +lean_inc(x_28); +lean_dec(x_22); +x_29 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_28); +if (lean_obj_tag(x_29) == 0) +{ lean_object* x_30; lean_object* x_31; -lean_dec(x_20); -x_30 = lean_ctor_get(x_24, 1); +x_30 = lean_ctor_get(x_29, 1); lean_inc(x_30); -lean_dec(x_24); -x_31 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_30); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -lean_dec(x_31); -x_33 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__1; -x_12 = x_33; -x_13 = x_32; +lean_dec(x_29); +x_31 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__1; +x_12 = x_31; +x_13 = x_30; goto block_16; } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_31); -if (x_34 == 0) +uint8_t x_32; +x_32 = !lean_is_exclusive(x_29); +if (x_32 == 0) { -return x_31; +return x_29; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_31, 0); -x_36 = lean_ctor_get(x_31, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_31); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_29, 0); +x_34 = lean_ctor_get(x_29, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_29); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -lean_dec(x_29); +lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +lean_dec(x_27); +x_36 = lean_ctor_get(x_22, 1); +lean_inc(x_36); +lean_dec(x_22); +x_37 = 1; +x_38 = l_Lean_Elab_Term_SavedState_restore(x_18, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_36); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_5); -x_38 = lean_ctor_get(x_24, 1); -lean_inc(x_38); -lean_dec(x_24); -x_39 = lean_st_ref_get(x_10, x_38); -lean_dec(x_10); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -x_41 = lean_st_ref_set(x_6, x_20, x_40); lean_dec(x_6); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -x_43 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__2; -x_12 = x_43; -x_13 = x_42; +lean_dec(x_5); +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +lean_dec(x_38); +x_40 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__2; +x_12 = x_40; +x_13 = x_39; goto block_16; } } else { -uint8_t x_44; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -x_44 = !lean_is_exclusive(x_24); -if (x_44 == 0) +uint8_t x_41; +x_41 = !lean_is_exclusive(x_22); +if (x_41 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; -x_45 = lean_ctor_get(x_24, 1); -x_46 = lean_ctor_get(x_24, 0); -lean_dec(x_46); -x_47 = lean_ctor_get(x_29, 0); -lean_inc(x_47); -x_48 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__3; -x_49 = lean_nat_dec_eq(x_47, x_48); -lean_dec(x_47); -if (x_49 == 0) +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_42 = lean_ctor_get(x_22, 1); +x_43 = lean_ctor_get(x_22, 0); +lean_dec(x_43); +x_44 = lean_ctor_get(x_27, 0); +lean_inc(x_44); +x_45 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__3; +x_46 = lean_nat_dec_eq(x_44, x_45); +lean_dec(x_44); +if (x_46 == 0) { -lean_dec(x_20); +lean_dec(x_18); lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -return x_24; +lean_dec(x_5); +return x_22; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -lean_free_object(x_24); -lean_dec(x_29); -x_50 = lean_st_ref_get(x_10, x_45); +uint8_t x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_free_object(x_22); +lean_dec(x_27); +x_47 = 1; +x_48 = l_Lean_Elab_Term_SavedState_restore(x_18, x_47, x_5, x_6, x_7, x_8, x_9, x_10, x_42); lean_dec(x_10); -x_51 = lean_ctor_get(x_50, 1); -lean_inc(x_51); -lean_dec(x_50); -x_52 = lean_st_ref_set(x_6, x_20, x_51); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -lean_dec(x_52); -x_54 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__2; -x_12 = x_54; -x_13 = x_53; +lean_dec(x_5); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__2; +x_12 = x_50; +x_13 = x_49; goto block_16; } } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_55 = lean_ctor_get(x_24, 1); -lean_inc(x_55); -lean_dec(x_24); -x_56 = lean_ctor_get(x_29, 0); -lean_inc(x_56); -x_57 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__3; -x_58 = lean_nat_dec_eq(x_56, x_57); -lean_dec(x_56); -if (x_58 == 0) +lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_51 = lean_ctor_get(x_22, 1); +lean_inc(x_51); +lean_dec(x_22); +x_52 = lean_ctor_get(x_27, 0); +lean_inc(x_52); +x_53 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__3; +x_54 = lean_nat_dec_eq(x_52, x_53); +lean_dec(x_52); +if (x_54 == 0) { -lean_object* x_59; -lean_dec(x_20); +lean_object* x_55; +lean_dec(x_18); lean_dec(x_10); -lean_dec(x_6); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_29); -lean_ctor_set(x_59, 1, x_55); -return x_59; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_27); +lean_ctor_set(x_55, 1, x_51); +return x_55; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -lean_dec(x_29); -x_60 = lean_st_ref_get(x_10, x_55); +uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +lean_dec(x_27); +x_56 = 1; +x_57 = l_Lean_Elab_Term_SavedState_restore(x_18, x_56, x_5, x_6, x_7, x_8, x_9, x_10, x_51); lean_dec(x_10); -x_61 = lean_ctor_get(x_60, 1); -lean_inc(x_61); -lean_dec(x_60); -x_62 = lean_st_ref_set(x_6, x_20, x_61); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -x_63 = lean_ctor_get(x_62, 1); -lean_inc(x_63); -lean_dec(x_62); -x_64 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__2; -x_12 = x_64; -x_13 = x_63; +lean_dec(x_5); +x_58 = lean_ctor_get(x_57, 1); +lean_inc(x_58); +lean_dec(x_57); +x_59 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed___lambda__2___closed__2; +x_12 = x_59; +x_13 = x_58; goto block_16; } } @@ -3648,7 +3670,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__1; x_2 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__2; x_3 = lean_unsigned_to_nat(66u); -x_4 = lean_unsigned_to_nat(36u); +x_4 = lean_unsigned_to_nat(26u); x_5 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -3852,7 +3874,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__1; x_2 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar___lambda__2___closed__1; x_3 = lean_unsigned_to_nat(99u); -x_4 = lean_unsigned_to_nat(33u); +x_4 = lean_unsigned_to_nat(24u); x_5 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -6469,7 +6491,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Synthe lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -8468,85 +8490,111 @@ return x_13; } else { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_2, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 2); -lean_inc(x_15); -if (lean_obj_tag(x_15) == 0) +uint8_t x_14; +x_14 = !lean_is_exclusive(x_2); +if (x_14 == 0) { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_2); -if (x_16 == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_2, 0); +x_16 = lean_ctor_get(x_2, 1); +x_17 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_17 = lean_ctor_get(x_2, 1); -x_18 = lean_ctor_get(x_2, 0); -lean_dec(x_18); -x_19 = lean_ctor_get(x_14, 1); +lean_object* x_19; +x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); -x_20 = lean_ctor_get(x_14, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_8, 0); -x_22 = lean_ctor_get(x_8, 1); -x_23 = lean_ctor_get(x_8, 2); -x_24 = lean_ctor_get(x_8, 3); -x_25 = lean_ctor_get(x_8, 4); -x_26 = lean_ctor_get(x_8, 5); -x_27 = lean_ctor_get(x_8, 6); -x_28 = lean_ctor_get(x_8, 7); -x_29 = lean_ctor_get(x_8, 8); -x_30 = lean_ctor_get(x_8, 9); -x_31 = lean_ctor_get(x_8, 10); -x_32 = l_Lean_replaceRef(x_19, x_26); -lean_dec(x_19); +lean_dec(x_17); +lean_ctor_set(x_2, 1, x_3); +{ +lean_object* _tmp_1 = x_16; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_9 = x_19; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; +} +goto _start; +} +else +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_18, 0); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_dec(x_17); +x_24 = lean_ctor_get(x_21, 0); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_ctor_get(x_8, 0); +x_26 = lean_ctor_get(x_8, 1); +x_27 = lean_ctor_get(x_8, 2); +x_28 = lean_ctor_get(x_8, 3); +x_29 = lean_ctor_get(x_8, 4); +x_30 = lean_ctor_get(x_8, 5); +x_31 = lean_ctor_get(x_8, 6); +x_32 = lean_ctor_get(x_8, 7); +x_33 = lean_ctor_get(x_8, 8); +x_34 = lean_ctor_get(x_8, 9); +x_35 = lean_ctor_get(x_8, 10); +x_36 = l_Lean_replaceRef(x_24, x_30); +lean_dec(x_24); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); lean_inc(x_31); -lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); lean_inc(x_27); +lean_inc(x_26); lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -x_33 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_33, 0, x_21); -lean_ctor_set(x_33, 1, x_22); -lean_ctor_set(x_33, 2, x_23); -lean_ctor_set(x_33, 3, x_24); -lean_ctor_set(x_33, 4, x_25); -lean_ctor_set(x_33, 5, x_32); -lean_ctor_set(x_33, 6, x_27); -lean_ctor_set(x_33, 7, x_28); -lean_ctor_set(x_33, 8, x_29); -lean_ctor_set(x_33, 9, x_30); -lean_ctor_set(x_33, 10, x_31); +x_37 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_37, 0, x_25); +lean_ctor_set(x_37, 1, x_26); +lean_ctor_set(x_37, 2, x_27); +lean_ctor_set(x_37, 3, x_28); +lean_ctor_set(x_37, 4, x_29); +lean_ctor_set(x_37, 5, x_36); +lean_ctor_set(x_37, 6, x_31); +lean_ctor_set(x_37, 7, x_32); +lean_ctor_set(x_37, 8, x_33); +lean_ctor_set(x_37, 9, x_34); +lean_ctor_set(x_37, 10, x_35); lean_inc(x_9); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_1); -x_34 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio(x_20, x_1, x_4, x_5, x_6, x_7, x_33, x_9, x_10); -if (lean_obj_tag(x_34) == 0) +lean_inc(x_15); +x_38 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio(x_15, x_1, x_4, x_5, x_6, x_7, x_37, x_9, x_23); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_35; uint8_t x_36; -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_unbox(x_35); -lean_dec(x_35); -if (x_36 == 0) +lean_object* x_39; uint8_t x_40; +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_unbox(x_39); +lean_dec(x_39); +if (x_40 == 0) { -lean_object* x_37; -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -lean_dec(x_34); +lean_object* x_41; +x_41 = lean_ctor_get(x_38, 1); +lean_inc(x_41); +lean_dec(x_38); lean_ctor_set(x_2, 1, x_3); { -lean_object* _tmp_1 = x_17; +lean_object* _tmp_1 = x_16; lean_object* _tmp_2 = x_2; -lean_object* _tmp_9 = x_37; +lean_object* _tmp_9 = x_41; x_2 = _tmp_1; x_3 = _tmp_2; x_10 = _tmp_9; @@ -8555,112 +8603,117 @@ goto _start; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_free_object(x_2); -lean_dec(x_14); +lean_dec(x_15); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_1); -x_39 = lean_ctor_get(x_34, 1); -lean_inc(x_39); -lean_dec(x_34); -x_40 = l_List_reverse___rarg(x_17); -x_41 = l_List_appendTR___rarg(x_40, x_3); -x_42 = lean_st_ref_get(x_9, x_39); -lean_dec(x_9); -x_43 = lean_ctor_get(x_42, 1); +x_43 = lean_ctor_get(x_38, 1); lean_inc(x_43); -lean_dec(x_42); -x_44 = lean_st_ref_take(x_5, x_43); -x_45 = lean_ctor_get(x_44, 0); +lean_dec(x_38); +x_44 = lean_st_ref_get(x_9, x_43); +lean_dec(x_9); +x_45 = lean_ctor_get(x_44, 1); lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); lean_dec(x_44); -x_47 = !lean_is_exclusive(x_45); -if (x_47 == 0) +x_46 = lean_st_ref_take(x_5, x_45); +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +lean_dec(x_46); +x_49 = !lean_is_exclusive(x_47); +if (x_49 == 0) { -lean_object* x_48; lean_object* x_49; uint8_t x_50; -x_48 = lean_ctor_get(x_45, 1); -lean_dec(x_48); -lean_ctor_set(x_45, 1, x_41); -x_49 = lean_st_ref_set(x_5, x_45, x_46); +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_50 = lean_ctor_get(x_47, 2); +lean_dec(x_50); +x_51 = l_List_reverse___rarg(x_16); +x_52 = l_List_appendTR___rarg(x_51, x_3); +lean_ctor_set(x_47, 2, x_52); +x_53 = lean_st_ref_set(x_5, x_47, x_48); lean_dec(x_5); -x_50 = !lean_is_exclusive(x_49); -if (x_50 == 0) +x_54 = !lean_is_exclusive(x_53); +if (x_54 == 0) { -lean_object* x_51; uint8_t x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_49, 0); -lean_dec(x_51); -x_52 = 1; -x_53 = lean_box(x_52); -lean_ctor_set(x_49, 0, x_53); -return x_49; +lean_object* x_55; uint8_t x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_53, 0); +lean_dec(x_55); +x_56 = 1; +x_57 = lean_box(x_56); +lean_ctor_set(x_53, 0, x_57); +return x_53; } else { -lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; -x_54 = lean_ctor_get(x_49, 1); -lean_inc(x_54); -lean_dec(x_49); -x_55 = 1; -x_56 = lean_box(x_55); -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_57, 1, x_54); -return x_57; +lean_object* x_58; uint8_t x_59; lean_object* x_60; lean_object* x_61; +x_58 = lean_ctor_get(x_53, 1); +lean_inc(x_58); +lean_dec(x_53); +x_59 = 1; +x_60 = lean_box(x_59); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_58); +return x_61; } } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; -x_58 = lean_ctor_get(x_45, 0); -x_59 = lean_ctor_get(x_45, 2); -x_60 = lean_ctor_get(x_45, 3); -x_61 = lean_ctor_get(x_45, 4); -lean_inc(x_61); -lean_inc(x_60); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_45); -x_62 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_62, 0, x_58); -lean_ctor_set(x_62, 1, x_41); -lean_ctor_set(x_62, 2, x_59); -lean_ctor_set(x_62, 3, x_60); -lean_ctor_set(x_62, 4, x_61); -x_63 = lean_st_ref_set(x_5, x_62, x_46); -lean_dec(x_5); -x_64 = lean_ctor_get(x_63, 1); +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; +x_62 = lean_ctor_get(x_47, 0); +x_63 = lean_ctor_get(x_47, 1); +x_64 = lean_ctor_get(x_47, 3); +x_65 = lean_ctor_get(x_47, 4); +x_66 = lean_ctor_get(x_47, 5); +lean_inc(x_66); +lean_inc(x_65); lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_47); +x_67 = l_List_reverse___rarg(x_16); +x_68 = l_List_appendTR___rarg(x_67, x_3); +x_69 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_69, 0, x_62); +lean_ctor_set(x_69, 1, x_63); +lean_ctor_set(x_69, 2, x_68); +lean_ctor_set(x_69, 3, x_64); +lean_ctor_set(x_69, 4, x_65); +lean_ctor_set(x_69, 5, x_66); +x_70 = lean_st_ref_set(x_5, x_69, x_48); +lean_dec(x_5); +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_72 = x_70; } else { - lean_dec_ref(x_63); - x_65 = lean_box(0); + lean_dec_ref(x_70); + x_72 = lean_box(0); } -x_66 = 1; -x_67 = lean_box(x_66); -if (lean_is_scalar(x_65)) { - x_68 = lean_alloc_ctor(0, 2, 0); +x_73 = 1; +x_74 = lean_box(x_73); +if (lean_is_scalar(x_72)) { + x_75 = lean_alloc_ctor(0, 2, 0); } else { - x_68 = x_65; + x_75 = x_72; } -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_64); -return x_68; +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_71); +return x_75; } } } else { -uint8_t x_69; +uint8_t x_76; lean_free_object(x_2); -lean_dec(x_17); -lean_dec(x_14); +lean_dec(x_16); +lean_dec(x_15); lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); @@ -8668,181 +8721,239 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_34); -if (x_69 == 0) +x_76 = !lean_is_exclusive(x_38); +if (x_76 == 0) { -return x_34; +return x_38; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_34, 0); -x_71 = lean_ctor_get(x_34, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_34); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_38, 0); +x_78 = lean_ctor_get(x_38, 1); +lean_inc(x_78); +lean_inc(x_77); +lean_dec(x_38); +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_73 = lean_ctor_get(x_2, 1); -lean_inc(x_73); -lean_dec(x_2); -x_74 = lean_ctor_get(x_14, 1); -lean_inc(x_74); -x_75 = lean_ctor_get(x_14, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_8, 0); -x_77 = lean_ctor_get(x_8, 1); -x_78 = lean_ctor_get(x_8, 2); -x_79 = lean_ctor_get(x_8, 3); -x_80 = lean_ctor_get(x_8, 4); -x_81 = lean_ctor_get(x_8, 5); -x_82 = lean_ctor_get(x_8, 6); -x_83 = lean_ctor_get(x_8, 7); -x_84 = lean_ctor_get(x_8, 8); -x_85 = lean_ctor_get(x_8, 9); -x_86 = lean_ctor_get(x_8, 10); -x_87 = l_Lean_replaceRef(x_74, x_81); -lean_dec(x_74); -lean_inc(x_86); -lean_inc(x_85); -lean_inc(x_84); +lean_object* x_80; +lean_dec(x_22); +lean_dec(x_21); +x_80 = lean_ctor_get(x_17, 1); +lean_inc(x_80); +lean_dec(x_17); +lean_ctor_set(x_2, 1, x_3); +{ +lean_object* _tmp_1 = x_16; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_9 = x_80; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; +} +goto _start; +} +} +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_82 = lean_ctor_get(x_2, 0); +x_83 = lean_ctor_get(x_2, 1); lean_inc(x_83); lean_inc(x_82); -lean_inc(x_80); -lean_inc(x_79); -lean_inc(x_78); -lean_inc(x_77); -lean_inc(x_76); -x_88 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_88, 0, x_76); -lean_ctor_set(x_88, 1, x_77); -lean_ctor_set(x_88, 2, x_78); -lean_ctor_set(x_88, 3, x_79); -lean_ctor_set(x_88, 4, x_80); -lean_ctor_set(x_88, 5, x_87); -lean_ctor_set(x_88, 6, x_82); -lean_ctor_set(x_88, 7, x_83); -lean_ctor_set(x_88, 8, x_84); -lean_ctor_set(x_88, 9, x_85); -lean_ctor_set(x_88, 10, x_86); +lean_dec(x_2); +x_84 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(x_82, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_85 = lean_ctor_get(x_84, 0); +lean_inc(x_85); +if (lean_obj_tag(x_85) == 0) +{ +lean_object* x_86; lean_object* x_87; +x_86 = lean_ctor_get(x_84, 1); +lean_inc(x_86); +lean_dec(x_84); +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_82); +lean_ctor_set(x_87, 1, x_3); +x_2 = x_83; +x_3 = x_87; +x_10 = x_86; +goto _start; +} +else +{ +lean_object* x_89; lean_object* x_90; +x_89 = lean_ctor_get(x_85, 0); +lean_inc(x_89); +lean_dec(x_85); +x_90 = lean_ctor_get(x_89, 1); +lean_inc(x_90); +if (lean_obj_tag(x_90) == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_91 = lean_ctor_get(x_84, 1); +lean_inc(x_91); +lean_dec(x_84); +x_92 = lean_ctor_get(x_89, 0); +lean_inc(x_92); +lean_dec(x_89); +x_93 = lean_ctor_get(x_8, 0); +x_94 = lean_ctor_get(x_8, 1); +x_95 = lean_ctor_get(x_8, 2); +x_96 = lean_ctor_get(x_8, 3); +x_97 = lean_ctor_get(x_8, 4); +x_98 = lean_ctor_get(x_8, 5); +x_99 = lean_ctor_get(x_8, 6); +x_100 = lean_ctor_get(x_8, 7); +x_101 = lean_ctor_get(x_8, 8); +x_102 = lean_ctor_get(x_8, 9); +x_103 = lean_ctor_get(x_8, 10); +x_104 = l_Lean_replaceRef(x_92, x_98); +lean_dec(x_92); +lean_inc(x_103); +lean_inc(x_102); +lean_inc(x_101); +lean_inc(x_100); +lean_inc(x_99); +lean_inc(x_97); +lean_inc(x_96); +lean_inc(x_95); +lean_inc(x_94); +lean_inc(x_93); +x_105 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_105, 0, x_93); +lean_ctor_set(x_105, 1, x_94); +lean_ctor_set(x_105, 2, x_95); +lean_ctor_set(x_105, 3, x_96); +lean_ctor_set(x_105, 4, x_97); +lean_ctor_set(x_105, 5, x_104); +lean_ctor_set(x_105, 6, x_99); +lean_ctor_set(x_105, 7, x_100); +lean_ctor_set(x_105, 8, x_101); +lean_ctor_set(x_105, 9, x_102); +lean_ctor_set(x_105, 10, x_103); lean_inc(x_9); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_1); -x_89 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio(x_75, x_1, x_4, x_5, x_6, x_7, x_88, x_9, x_10); -if (lean_obj_tag(x_89) == 0) +lean_inc(x_82); +x_106 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio(x_82, x_1, x_4, x_5, x_6, x_7, x_105, x_9, x_91); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_90; uint8_t x_91; -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -x_91 = lean_unbox(x_90); -lean_dec(x_90); -if (x_91 == 0) +lean_object* x_107; uint8_t x_108; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_unbox(x_107); +lean_dec(x_107); +if (x_108 == 0) { -lean_object* x_92; lean_object* x_93; -x_92 = lean_ctor_get(x_89, 1); -lean_inc(x_92); -lean_dec(x_89); -x_93 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_93, 0, x_14); -lean_ctor_set(x_93, 1, x_3); -x_2 = x_73; -x_3 = x_93; -x_10 = x_92; +lean_object* x_109; lean_object* x_110; +x_109 = lean_ctor_get(x_106, 1); +lean_inc(x_109); +lean_dec(x_106); +x_110 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_110, 0, x_82); +lean_ctor_set(x_110, 1, x_3); +x_2 = x_83; +x_3 = x_110; +x_10 = x_109; goto _start; } else { -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; uint8_t x_112; lean_object* x_113; lean_object* x_114; -lean_dec(x_14); +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; uint8_t x_130; lean_object* x_131; lean_object* x_132; +lean_dec(x_82); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_1); -x_95 = lean_ctor_get(x_89, 1); -lean_inc(x_95); -lean_dec(x_89); -x_96 = l_List_reverse___rarg(x_73); -x_97 = l_List_appendTR___rarg(x_96, x_3); -x_98 = lean_st_ref_get(x_9, x_95); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_dec(x_106); +x_113 = lean_st_ref_get(x_9, x_112); lean_dec(x_9); -x_99 = lean_ctor_get(x_98, 1); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_st_ref_take(x_5, x_99); -x_101 = lean_ctor_get(x_100, 0); -lean_inc(x_101); -x_102 = lean_ctor_get(x_100, 1); -lean_inc(x_102); -lean_dec(x_100); -x_103 = lean_ctor_get(x_101, 0); -lean_inc(x_103); -x_104 = lean_ctor_get(x_101, 2); -lean_inc(x_104); -x_105 = lean_ctor_get(x_101, 3); -lean_inc(x_105); -x_106 = lean_ctor_get(x_101, 4); -lean_inc(x_106); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - lean_ctor_release(x_101, 2); - lean_ctor_release(x_101, 3); - lean_ctor_release(x_101, 4); - x_107 = x_101; +x_114 = lean_ctor_get(x_113, 1); +lean_inc(x_114); +lean_dec(x_113); +x_115 = lean_st_ref_take(x_5, x_114); +x_116 = lean_ctor_get(x_115, 0); +lean_inc(x_116); +x_117 = lean_ctor_get(x_115, 1); +lean_inc(x_117); +lean_dec(x_115); +x_118 = lean_ctor_get(x_116, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_116, 1); +lean_inc(x_119); +x_120 = lean_ctor_get(x_116, 3); +lean_inc(x_120); +x_121 = lean_ctor_get(x_116, 4); +lean_inc(x_121); +x_122 = lean_ctor_get(x_116, 5); +lean_inc(x_122); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + lean_ctor_release(x_116, 2); + lean_ctor_release(x_116, 3); + lean_ctor_release(x_116, 4); + lean_ctor_release(x_116, 5); + x_123 = x_116; } else { - lean_dec_ref(x_101); - x_107 = lean_box(0); + lean_dec_ref(x_116); + x_123 = lean_box(0); } -if (lean_is_scalar(x_107)) { - x_108 = lean_alloc_ctor(0, 5, 0); +x_124 = l_List_reverse___rarg(x_83); +x_125 = l_List_appendTR___rarg(x_124, x_3); +if (lean_is_scalar(x_123)) { + x_126 = lean_alloc_ctor(0, 6, 0); } else { - x_108 = x_107; -} -lean_ctor_set(x_108, 0, x_103); -lean_ctor_set(x_108, 1, x_97); -lean_ctor_set(x_108, 2, x_104); -lean_ctor_set(x_108, 3, x_105); -lean_ctor_set(x_108, 4, x_106); -x_109 = lean_st_ref_set(x_5, x_108, x_102); + x_126 = x_123; +} +lean_ctor_set(x_126, 0, x_118); +lean_ctor_set(x_126, 1, x_119); +lean_ctor_set(x_126, 2, x_125); +lean_ctor_set(x_126, 3, x_120); +lean_ctor_set(x_126, 4, x_121); +lean_ctor_set(x_126, 5, x_122); +x_127 = lean_st_ref_set(x_5, x_126, x_117); lean_dec(x_5); -x_110 = lean_ctor_get(x_109, 1); -lean_inc(x_110); -if (lean_is_exclusive(x_109)) { - lean_ctor_release(x_109, 0); - lean_ctor_release(x_109, 1); - x_111 = x_109; +x_128 = lean_ctor_get(x_127, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_129 = x_127; } else { - lean_dec_ref(x_109); - x_111 = lean_box(0); + lean_dec_ref(x_127); + x_129 = lean_box(0); } -x_112 = 1; -x_113 = lean_box(x_112); -if (lean_is_scalar(x_111)) { - x_114 = lean_alloc_ctor(0, 2, 0); +x_130 = 1; +x_131 = lean_box(x_130); +if (lean_is_scalar(x_129)) { + x_132 = lean_alloc_ctor(0, 2, 0); } else { - x_114 = x_111; + x_132 = x_129; } -lean_ctor_set(x_114, 0, x_113); -lean_ctor_set(x_114, 1, x_110); -return x_114; +lean_ctor_set(x_132, 0, x_131); +lean_ctor_set(x_132, 1, x_128); +return x_132; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -lean_dec(x_73); -lean_dec(x_14); +lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; +lean_dec(x_83); +lean_dec(x_82); lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); @@ -8850,61 +8961,44 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_115 = lean_ctor_get(x_89, 0); -lean_inc(x_115); -x_116 = lean_ctor_get(x_89, 1); -lean_inc(x_116); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_117 = x_89; +x_133 = lean_ctor_get(x_106, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_106, 1); +lean_inc(x_134); +if (lean_is_exclusive(x_106)) { + lean_ctor_release(x_106, 0); + lean_ctor_release(x_106, 1); + x_135 = x_106; } else { - lean_dec_ref(x_89); - x_117 = lean_box(0); + lean_dec_ref(x_106); + x_135 = lean_box(0); } -if (lean_is_scalar(x_117)) { - x_118 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_135)) { + x_136 = lean_alloc_ctor(1, 2, 0); } else { - x_118 = x_117; -} -lean_ctor_set(x_118, 0, x_115); -lean_ctor_set(x_118, 1, x_116); -return x_118; + x_136 = x_135; } +lean_ctor_set(x_136, 0, x_133); +lean_ctor_set(x_136, 1, x_134); +return x_136; } } else { -uint8_t x_119; -lean_dec(x_15); -x_119 = !lean_is_exclusive(x_2); -if (x_119 == 0) -{ -lean_object* x_120; lean_object* x_121; -x_120 = lean_ctor_get(x_2, 1); -x_121 = lean_ctor_get(x_2, 0); -lean_dec(x_121); -lean_ctor_set(x_2, 1, x_3); -{ -lean_object* _tmp_1 = x_120; -lean_object* _tmp_2 = x_2; -x_2 = _tmp_1; -x_3 = _tmp_2; -} +lean_object* x_137; lean_object* x_138; +lean_dec(x_90); +lean_dec(x_89); +x_137 = lean_ctor_get(x_84, 1); +lean_inc(x_137); +lean_dec(x_84); +x_138 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_138, 0, x_82); +lean_ctor_set(x_138, 1, x_3); +x_2 = x_83; +x_3 = x_138; +x_10 = x_137; goto _start; } -else -{ -lean_object* x_123; lean_object* x_124; -x_123 = lean_ctor_get(x_2, 1); -lean_inc(x_123); -lean_dec(x_2); -x_124 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_124, 0, x_14); -lean_ctor_set(x_124, 1, x_3); -x_2 = x_123; -x_3 = x_124; -goto _start; } } } @@ -8933,7 +9027,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = lean_ctor_get(x_12, 1); +x_14 = lean_ctor_get(x_12, 2); lean_inc(x_14); lean_dec(x_12); x_15 = l_List_reverse___rarg(x_14); @@ -9469,7 +9563,7 @@ static lean_object* _init_l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2( lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__1; x_2 = l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__1; -x_3 = lean_unsigned_to_nat(251u); +x_3 = lean_unsigned_to_nat(252u); x_4 = lean_unsigned_to_nat(11u); x_5 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9479,38 +9573,86 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar(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) { _start: { -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_1, 1); -lean_inc(x_10); -x_11 = lean_ctor_get(x_1, 2); +lean_object* x_10; lean_object* x_11; +x_10 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); -x_12 = !lean_is_exclusive(x_7); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_12 = !lean_is_exclusive(x_10); if (x_12 == 0) { lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_7, 5); -x_14 = l_Lean_replaceRef(x_10, x_13); +x_13 = lean_ctor_get(x_10, 0); lean_dec(x_13); +x_14 = lean_box(0); +lean_ctor_set(x_10, 0, x_14); +return x_10; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_15); lean_dec(x_10); -lean_ctor_set(x_7, 5, x_14); -switch (lean_obj_tag(x_11)) { +x_16 = lean_box(0); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +return x_17; +} +} +else +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_10); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_19 = lean_ctor_get(x_10, 1); +x_20 = lean_ctor_get(x_10, 0); +lean_dec(x_20); +x_21 = lean_ctor_get(x_11, 0); +lean_inc(x_21); +lean_dec(x_11); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = !lean_is_exclusive(x_7); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_7, 5); +x_26 = l_Lean_replaceRef(x_22, x_25); +lean_dec(x_25); +lean_dec(x_22); +lean_ctor_set(x_7, 5, x_26); +switch (lean_obj_tag(x_23)) { case 0: { if (x_2 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_1, 0); -lean_inc(x_15); -lean_dec(x_1); -lean_inc(x_15); -x_16 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___boxed), 8, 1); -lean_closure_set(x_16, 0, x_15); -x_17 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_15, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_17; +lean_object* x_27; lean_object* x_28; +lean_free_object(x_10); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___boxed), 8, 1); +lean_closure_set(x_27, 0, x_1); +x_28 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_1, x_27, x_3, x_4, x_5, x_6, x_7, x_8, x_19); +return x_28; } else { -lean_object* x_18; lean_object* x_19; +lean_object* x_29; lean_dec(x_7); lean_dec(x_8); lean_dec(x_6); @@ -9518,195 +9660,339 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_18 = lean_box(0); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_9); -return x_19; +x_29 = lean_box(0); +lean_ctor_set(x_10, 0, x_29); +return x_10; } } case 1: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; 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_free_object(x_10); lean_dec(x_1); -x_20 = lean_ctor_get(x_11, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_11, 1); -lean_inc(x_21); -x_22 = lean_ctor_get(x_11, 2); -lean_inc(x_22); -x_23 = lean_ctor_get(x_11, 3); -lean_inc(x_23); -x_24 = lean_ctor_get(x_11, 4); -lean_inc(x_24); -x_25 = lean_ctor_get(x_11, 5); -lean_inc(x_25); -lean_dec(x_11); -x_26 = l_Lean_Expr_appArg_x21(x_21); -lean_dec(x_21); -x_27 = l_Lean_Expr_mvarId_x21(x_26); -lean_dec(x_26); -lean_inc(x_27); -x_28 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__2), 13, 6); -lean_closure_set(x_28, 0, x_27); -lean_closure_set(x_28, 1, x_20); -lean_closure_set(x_28, 2, x_22); -lean_closure_set(x_28, 3, x_23); -lean_closure_set(x_28, 4, x_24); -lean_closure_set(x_28, 5, x_25); -x_29 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_27, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_29; +x_30 = lean_ctor_get(x_23, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_23, 1); +lean_inc(x_31); +x_32 = lean_ctor_get(x_23, 2); +lean_inc(x_32); +x_33 = lean_ctor_get(x_23, 3); +lean_inc(x_33); +x_34 = lean_ctor_get(x_23, 4); +lean_inc(x_34); +x_35 = lean_ctor_get(x_23, 5); +lean_inc(x_35); +lean_dec(x_23); +x_36 = l_Lean_Expr_appArg_x21(x_31); +lean_dec(x_31); +x_37 = l_Lean_Expr_mvarId_x21(x_36); +lean_dec(x_36); +lean_inc(x_37); +x_38 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__2), 13, 6); +lean_closure_set(x_38, 0, x_37); +lean_closure_set(x_38, 1, x_30); +lean_closure_set(x_38, 2, x_32); +lean_closure_set(x_38, 3, x_33); +lean_closure_set(x_38, 4, x_34); +lean_closure_set(x_38, 5, x_35); +x_39 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_37, x_38, x_3, x_4, x_5, x_6, x_7, x_8, x_19); +return x_39; } default: { -lean_object* x_30; lean_object* x_31; -lean_dec(x_11); +lean_object* x_40; lean_object* x_41; +lean_dec(x_23); +lean_free_object(x_10); lean_dec(x_1); -x_30 = l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2; -x_31 = l_panic___at_Lean_Elab_Term_reportStuckSyntheticMVar___spec__1(x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_31; +x_40 = l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2; +x_41 = l_panic___at_Lean_Elab_Term_reportStuckSyntheticMVar___spec__1(x_40, x_3, x_4, x_5, x_6, x_7, x_8, x_19); +return x_41; } } } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_32 = lean_ctor_get(x_7, 0); -x_33 = lean_ctor_get(x_7, 1); -x_34 = lean_ctor_get(x_7, 2); -x_35 = lean_ctor_get(x_7, 3); -x_36 = lean_ctor_get(x_7, 4); -x_37 = lean_ctor_get(x_7, 5); -x_38 = lean_ctor_get(x_7, 6); -x_39 = lean_ctor_get(x_7, 7); -x_40 = lean_ctor_get(x_7, 8); -x_41 = lean_ctor_get(x_7, 9); -x_42 = lean_ctor_get(x_7, 10); +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_42 = lean_ctor_get(x_7, 0); +x_43 = lean_ctor_get(x_7, 1); +x_44 = lean_ctor_get(x_7, 2); +x_45 = lean_ctor_get(x_7, 3); +x_46 = lean_ctor_get(x_7, 4); +x_47 = lean_ctor_get(x_7, 5); +x_48 = lean_ctor_get(x_7, 6); +x_49 = lean_ctor_get(x_7, 7); +x_50 = lean_ctor_get(x_7, 8); +x_51 = lean_ctor_get(x_7, 9); +x_52 = lean_ctor_get(x_7, 10); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); lean_inc(x_42); -lean_inc(x_41); -lean_inc(x_40); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); lean_dec(x_7); -x_43 = l_Lean_replaceRef(x_10, x_37); -lean_dec(x_37); -lean_dec(x_10); -x_44 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_44, 0, x_32); -lean_ctor_set(x_44, 1, x_33); -lean_ctor_set(x_44, 2, x_34); -lean_ctor_set(x_44, 3, x_35); -lean_ctor_set(x_44, 4, x_36); -lean_ctor_set(x_44, 5, x_43); -lean_ctor_set(x_44, 6, x_38); -lean_ctor_set(x_44, 7, x_39); -lean_ctor_set(x_44, 8, x_40); -lean_ctor_set(x_44, 9, x_41); -lean_ctor_set(x_44, 10, x_42); -switch (lean_obj_tag(x_11)) { +x_53 = l_Lean_replaceRef(x_22, x_47); +lean_dec(x_47); +lean_dec(x_22); +x_54 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_54, 0, x_42); +lean_ctor_set(x_54, 1, x_43); +lean_ctor_set(x_54, 2, x_44); +lean_ctor_set(x_54, 3, x_45); +lean_ctor_set(x_54, 4, x_46); +lean_ctor_set(x_54, 5, x_53); +lean_ctor_set(x_54, 6, x_48); +lean_ctor_set(x_54, 7, x_49); +lean_ctor_set(x_54, 8, x_50); +lean_ctor_set(x_54, 9, x_51); +lean_ctor_set(x_54, 10, x_52); +switch (lean_obj_tag(x_23)) { case 0: { if (x_2 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_1, 0); -lean_inc(x_45); -lean_dec(x_1); -lean_inc(x_45); -x_46 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___boxed), 8, 1); -lean_closure_set(x_46, 0, x_45); -x_47 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_45, x_46, x_3, x_4, x_5, x_6, x_44, x_8, x_9); -return x_47; +lean_object* x_55; lean_object* x_56; +lean_free_object(x_10); +lean_inc(x_1); +x_55 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___boxed), 8, 1); +lean_closure_set(x_55, 0, x_1); +x_56 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_1, x_55, x_3, x_4, x_5, x_6, x_54, x_8, x_19); +return x_56; } else { -lean_object* x_48; lean_object* x_49; -lean_dec(x_44); +lean_object* x_57; +lean_dec(x_54); lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_48 = lean_box(0); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_9); -return x_49; +x_57 = lean_box(0); +lean_ctor_set(x_10, 0, x_57); +return x_10; } } case 1: { -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_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_free_object(x_10); lean_dec(x_1); -x_50 = lean_ctor_get(x_11, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_11, 1); -lean_inc(x_51); -x_52 = lean_ctor_get(x_11, 2); -lean_inc(x_52); -x_53 = lean_ctor_get(x_11, 3); -lean_inc(x_53); -x_54 = lean_ctor_get(x_11, 4); -lean_inc(x_54); -x_55 = lean_ctor_get(x_11, 5); -lean_inc(x_55); -lean_dec(x_11); -x_56 = l_Lean_Expr_appArg_x21(x_51); -lean_dec(x_51); -x_57 = l_Lean_Expr_mvarId_x21(x_56); -lean_dec(x_56); -lean_inc(x_57); -x_58 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__2), 13, 6); -lean_closure_set(x_58, 0, x_57); -lean_closure_set(x_58, 1, x_50); -lean_closure_set(x_58, 2, x_52); -lean_closure_set(x_58, 3, x_53); -lean_closure_set(x_58, 4, x_54); -lean_closure_set(x_58, 5, x_55); -x_59 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_57, x_58, x_3, x_4, x_5, x_6, x_44, x_8, x_9); -return x_59; +x_58 = lean_ctor_get(x_23, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_23, 1); +lean_inc(x_59); +x_60 = lean_ctor_get(x_23, 2); +lean_inc(x_60); +x_61 = lean_ctor_get(x_23, 3); +lean_inc(x_61); +x_62 = lean_ctor_get(x_23, 4); +lean_inc(x_62); +x_63 = lean_ctor_get(x_23, 5); +lean_inc(x_63); +lean_dec(x_23); +x_64 = l_Lean_Expr_appArg_x21(x_59); +lean_dec(x_59); +x_65 = l_Lean_Expr_mvarId_x21(x_64); +lean_dec(x_64); +lean_inc(x_65); +x_66 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__2), 13, 6); +lean_closure_set(x_66, 0, x_65); +lean_closure_set(x_66, 1, x_58); +lean_closure_set(x_66, 2, x_60); +lean_closure_set(x_66, 3, x_61); +lean_closure_set(x_66, 4, x_62); +lean_closure_set(x_66, 5, x_63); +x_67 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_65, x_66, x_3, x_4, x_5, x_6, x_54, x_8, x_19); +return x_67; } default: { -lean_object* x_60; lean_object* x_61; -lean_dec(x_11); +lean_object* x_68; lean_object* x_69; +lean_dec(x_23); +lean_free_object(x_10); lean_dec(x_1); -x_60 = l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2; -x_61 = l_panic___at_Lean_Elab_Term_reportStuckSyntheticMVar___spec__1(x_60, x_3, x_4, x_5, x_6, x_44, x_8, x_9); -return x_61; -} -} -} +x_68 = l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2; +x_69 = l_panic___at_Lean_Elab_Term_reportStuckSyntheticMVar___spec__1(x_68, x_3, x_4, x_5, x_6, x_54, x_8, x_19); +return x_69; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -uint8_t x_10; lean_object* x_11; -x_10 = lean_unbox(x_2); -lean_dec(x_2); -x_11 = l_Lean_Elab_Term_reportStuckSyntheticMVar(x_1, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_11; +lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_70 = lean_ctor_get(x_10, 1); +lean_inc(x_70); +lean_dec(x_10); +x_71 = lean_ctor_get(x_11, 0); +lean_inc(x_71); +lean_dec(x_11); +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = lean_ctor_get(x_7, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_7, 1); +lean_inc(x_75); +x_76 = lean_ctor_get(x_7, 2); +lean_inc(x_76); +x_77 = lean_ctor_get(x_7, 3); +lean_inc(x_77); +x_78 = lean_ctor_get(x_7, 4); +lean_inc(x_78); +x_79 = lean_ctor_get(x_7, 5); +lean_inc(x_79); +x_80 = lean_ctor_get(x_7, 6); +lean_inc(x_80); +x_81 = lean_ctor_get(x_7, 7); +lean_inc(x_81); +x_82 = lean_ctor_get(x_7, 8); +lean_inc(x_82); +x_83 = lean_ctor_get(x_7, 9); +lean_inc(x_83); +x_84 = lean_ctor_get(x_7, 10); +lean_inc(x_84); +if (lean_is_exclusive(x_7)) { + lean_ctor_release(x_7, 0); + lean_ctor_release(x_7, 1); + lean_ctor_release(x_7, 2); + lean_ctor_release(x_7, 3); + lean_ctor_release(x_7, 4); + lean_ctor_release(x_7, 5); + lean_ctor_release(x_7, 6); + lean_ctor_release(x_7, 7); + lean_ctor_release(x_7, 8); + lean_ctor_release(x_7, 9); + lean_ctor_release(x_7, 10); + x_85 = x_7; +} else { + lean_dec_ref(x_7); + x_85 = lean_box(0); +} +x_86 = l_Lean_replaceRef(x_72, x_79); +lean_dec(x_79); +lean_dec(x_72); +if (lean_is_scalar(x_85)) { + x_87 = lean_alloc_ctor(0, 11, 0); +} else { + x_87 = x_85; +} +lean_ctor_set(x_87, 0, x_74); +lean_ctor_set(x_87, 1, x_75); +lean_ctor_set(x_87, 2, x_76); +lean_ctor_set(x_87, 3, x_77); +lean_ctor_set(x_87, 4, x_78); +lean_ctor_set(x_87, 5, x_86); +lean_ctor_set(x_87, 6, x_80); +lean_ctor_set(x_87, 7, x_81); +lean_ctor_set(x_87, 8, x_82); +lean_ctor_set(x_87, 9, x_83); +lean_ctor_set(x_87, 10, x_84); +switch (lean_obj_tag(x_73)) { +case 0: +{ +if (x_2 == 0) +{ +lean_object* x_88; lean_object* x_89; +lean_inc(x_1); +x_88 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___boxed), 8, 1); +lean_closure_set(x_88, 0, x_1); +x_89 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_1, x_88, x_3, x_4, x_5, x_6, x_87, x_8, x_70); +return x_89; +} +else +{ +lean_object* x_90; lean_object* x_91; +lean_dec(x_87); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_90 = lean_box(0); +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_70); +return x_91; +} +} +case 1: +{ +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_dec(x_1); +x_92 = lean_ctor_get(x_73, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_73, 1); +lean_inc(x_93); +x_94 = lean_ctor_get(x_73, 2); +lean_inc(x_94); +x_95 = lean_ctor_get(x_73, 3); +lean_inc(x_95); +x_96 = lean_ctor_get(x_73, 4); +lean_inc(x_96); +x_97 = lean_ctor_get(x_73, 5); +lean_inc(x_97); +lean_dec(x_73); +x_98 = l_Lean_Expr_appArg_x21(x_93); +lean_dec(x_93); +x_99 = l_Lean_Expr_mvarId_x21(x_98); +lean_dec(x_98); +lean_inc(x_99); +x_100 = lean_alloc_closure((void*)(l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__2), 13, 6); +lean_closure_set(x_100, 0, x_99); +lean_closure_set(x_100, 1, x_92); +lean_closure_set(x_100, 2, x_94); +lean_closure_set(x_100, 3, x_95); +lean_closure_set(x_100, 4, x_96); +lean_closure_set(x_100, 5, x_97); +x_101 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_99, x_100, x_3, x_4, x_5, x_6, x_87, x_8, x_70); +return x_101; +} +default: +{ +lean_object* x_102; lean_object* x_103; +lean_dec(x_73); +lean_dec(x_1); +x_102 = l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2; +x_103 = l_panic___at_Lean_Elab_Term_reportStuckSyntheticMVar___spec__1(x_102, x_3, x_4, x_5, x_6, x_87, x_8, x_70); +return x_103; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Term_reportStuckSyntheticMVar___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportStuckSyntheticMVar___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; lean_object* x_11; +x_10 = lean_unbox(x_2); +lean_dec(x_2); +x_11 = l_Lean_Elab_Term_reportStuckSyntheticMVar(x_1, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_11; } } LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_reportStuckSyntheticMVars___spec__1(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -9804,9 +10090,9 @@ x_14 = !lean_is_exclusive(x_12); if (x_14 == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_15 = lean_ctor_get(x_12, 1); +x_15 = lean_ctor_get(x_12, 2); x_16 = lean_box(0); -lean_ctor_set(x_12, 1, x_16); +lean_ctor_set(x_12, 2, x_16); x_17 = lean_st_ref_set(x_3, x_12, x_13); x_18 = lean_ctor_get(x_17, 1); lean_inc(x_18); @@ -9862,76 +10148,79 @@ return x_28; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; x_29 = lean_ctor_get(x_12, 0); x_30 = lean_ctor_get(x_12, 1); x_31 = lean_ctor_get(x_12, 2); x_32 = lean_ctor_get(x_12, 3); x_33 = lean_ctor_get(x_12, 4); +x_34 = lean_ctor_get(x_12, 5); +lean_inc(x_34); lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); lean_dec(x_12); -x_34 = lean_box(0); -x_35 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_35, 0, x_29); -lean_ctor_set(x_35, 1, x_34); -lean_ctor_set(x_35, 2, x_31); -lean_ctor_set(x_35, 3, x_32); -lean_ctor_set(x_35, 4, x_33); -x_36 = lean_st_ref_set(x_3, x_35, x_13); -x_37 = lean_ctor_get(x_36, 1); -lean_inc(x_37); -lean_dec(x_36); -x_38 = lean_box(0); -x_39 = l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_reportStuckSyntheticMVars___spec__1(x_1, x_30, x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_37); -if (lean_obj_tag(x_39) == 0) +x_35 = lean_box(0); +x_36 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_36, 0, x_29); +lean_ctor_set(x_36, 1, x_30); +lean_ctor_set(x_36, 2, x_35); +lean_ctor_set(x_36, 3, x_32); +lean_ctor_set(x_36, 4, x_33); +lean_ctor_set(x_36, 5, x_34); +x_37 = lean_st_ref_set(x_3, x_36, x_13); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = lean_box(0); +x_40 = l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_reportStuckSyntheticMVars___spec__1(x_1, x_31, x_39, x_2, x_3, x_4, x_5, x_6, x_7, x_38); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - x_41 = x_39; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_42 = x_40; } else { - lean_dec_ref(x_39); - x_41 = lean_box(0); + lean_dec_ref(x_40); + x_42 = lean_box(0); } -if (lean_is_scalar(x_41)) { - x_42 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_42)) { + x_43 = lean_alloc_ctor(0, 2, 0); } else { - x_42 = x_41; + x_43 = x_42; } -lean_ctor_set(x_42, 0, x_38); -lean_ctor_set(x_42, 1, x_40); -return x_42; +lean_ctor_set(x_43, 0, x_39); +lean_ctor_set(x_43, 1, x_41); +return x_43; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_43 = lean_ctor_get(x_39, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_39, 1); +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_40, 0); lean_inc(x_44); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - x_45 = x_39; +x_45 = lean_ctor_get(x_40, 1); +lean_inc(x_45); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_46 = x_40; } else { - lean_dec_ref(x_39); - x_45 = lean_box(0); + lean_dec_ref(x_40); + x_46 = lean_box(0); } -if (lean_is_scalar(x_45)) { - x_46 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_46)) { + x_47 = lean_alloc_ctor(1, 2, 0); } else { - x_46 = x_45; + x_47 = x_46; } -lean_ctor_set(x_46, 0, x_43); -lean_ctor_set(x_46, 1, x_44); -return x_46; +lean_ctor_set(x_47, 0, x_44); +lean_ctor_set(x_47, 1, x_45); +return x_47; } } } @@ -9956,152 +10245,287 @@ x_10 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_reportStuckSynthet return x_10; } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_2; uint8_t x_3; lean_object* x_4; -x_2 = lean_ctor_get(x_1, 1); -x_3 = 0; -x_4 = l_Lean_Syntax_getPos_x3f(x_2, x_3); -if (lean_obj_tag(x_4) == 0) +if (lean_obj_tag(x_2) == 0) { -uint8_t x_5; -x_5 = 0; -return x_5; +lean_object* x_11; +lean_dec(x_1); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_3); +lean_ctor_set(x_11, 1, x_10); +return x_11; } else { -uint8_t x_6; -lean_dec(x_4); -x_6 = 1; -return x_6; -} -} -} -static lean_object* _init_l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___lambda__1___boxed), 1, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_7 = lean_st_ref_get(x_5, x_6); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_st_ref_get(x_1, x_8); -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___closed__1; -x_14 = l_List_find_x3f___rarg(x_13, x_12); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; -x_15 = lean_box(0); -lean_ctor_set(x_9, 0, x_15); -return x_9; -} -else +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_3); +x_12 = lean_ctor_get(x_2, 0); +x_13 = lean_ctor_get(x_2, 1); +x_14 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_14, 0); +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); lean_dec(x_14); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -lean_ctor_set(x_9, 0, x_17); -return x_9; +lean_inc(x_1); +{ +lean_object* _tmp_1 = x_13; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_9 = x_16; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; } +goto _start; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_9, 1); -lean_inc(x_19); +lean_object* x_18; uint8_t x_19; +x_18 = lean_ctor_get(x_15, 0); lean_inc(x_18); -lean_dec(x_9); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___closed__1; -x_22 = l_List_find_x3f___rarg(x_21, x_20); -if (lean_obj_tag(x_22) == 0) +lean_dec(x_15); +x_19 = !lean_is_exclusive(x_14); +if (x_19 == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_box(0); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_19); -return x_24; -} -else +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; +x_20 = lean_ctor_get(x_14, 1); +x_21 = lean_ctor_get(x_14, 0); +lean_dec(x_21); +x_22 = lean_ctor_get(x_18, 0); +lean_inc(x_22); +lean_dec(x_18); +x_23 = 0; +x_24 = l_Lean_Syntax_getPos_x3f(x_22, x_23); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_22, 0); -lean_inc(x_25); lean_dec(x_22); -x_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_19); -return x_27; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef(lean_object* x_1) { -_start: +lean_free_object(x_14); +lean_inc(x_1); { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___boxed), 6, 0); -return x_2; +lean_object* _tmp_1 = x_13; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_9 = x_20; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; } +goto _start; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___lambda__1___boxed(lean_object* x_1) { -_start: +else { -uint8_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___lambda__1(x_1); +uint8_t x_26; lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; +x_26 = !lean_is_exclusive(x_24); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_24, 0); +lean_dec(x_27); +lean_ctor_set(x_24, 0, x_22); +x_28 = lean_box(0); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_24); +lean_ctor_set(x_29, 1, x_28); +lean_ctor_set(x_14, 0, x_29); +return x_14; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +lean_dec(x_24); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_22); +x_31 = lean_box(0); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +lean_ctor_set(x_14, 0, x_32); +return x_14; +} +} +} +else +{ +lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; +x_33 = lean_ctor_get(x_14, 1); +lean_inc(x_33); +lean_dec(x_14); +x_34 = lean_ctor_get(x_18, 0); +lean_inc(x_34); +lean_dec(x_18); +x_35 = 0; +x_36 = l_Lean_Syntax_getPos_x3f(x_34, x_35); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_34); +lean_inc(x_1); +{ +lean_object* _tmp_1 = x_13; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_9 = x_33; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_10 = _tmp_9; +} +goto _start; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +lean_dec(x_1); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_38 = x_36; +} else { + lean_dec_ref(x_36); + x_38 = lean_box(0); +} +if (lean_is_scalar(x_38)) { + x_39 = lean_alloc_ctor(1, 1, 0); +} else { + x_39 = x_38; +} +lean_ctor_set(x_39, 0, x_34); +x_40 = lean_box(0); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_33); +return x_42; +} +} +} } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_7; -x_7 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg(x_1, x_2, x_3, x_4, x_5, x_6); +lean_object* x_9; lean_object* x_10; +x_9 = lean_box(0); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +} +static lean_object* _init_l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___lambda__1___boxed), 8, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_8 = lean_st_ref_get(x_6, x_7); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_st_ref_get(x_2, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_ctor_get(x_11, 2); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefault___closed__1; +x_15 = l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___spec__1(x_14, x_13, x_14, x_1, x_2, x_3, x_4, x_5, x_6, x_12); +lean_dec(x_13); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +lean_dec(x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +x_19 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___closed__1; +x_20 = lean_box(0); +x_21 = lean_apply_8(x_19, x_20, x_1, x_2, x_3, x_4, x_5, x_6, x_18); +return x_21; +} +else +{ +uint8_t x_22; +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_7; +x_22 = !lean_is_exclusive(x_15); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_15, 0); +lean_dec(x_23); +x_24 = lean_ctor_get(x_17, 0); +lean_inc(x_24); +lean_dec(x_17); +lean_ctor_set(x_15, 0, x_24); +return x_15; } +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_15, 1); +lean_inc(x_25); +lean_dec(x_15); +x_26 = lean_ctor_get(x_17, 0); +lean_inc(x_26); +lean_dec(x_17); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +return x_27; } -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___boxed(lean_object* x_1) { +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_2; -x_2 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef(x_1); +lean_object* x_11; +x_11 = l_List_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -return x_2; +return x_9; } } LEAN_EXPORT lean_object* l_Std_mkHashSet___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__1(lean_object* x_1) { @@ -11520,865 +11944,38 @@ x_39 = lean_ctor_get(x_29, 0); lean_dec(x_39); x_40 = lean_ctor_get(x_31, 0); lean_inc(x_40); -lean_dec(x_31); -lean_ctor_set(x_29, 0, x_40); -return x_29; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_29, 1); -lean_inc(x_41); -lean_dec(x_29); -x_42 = lean_ctor_get(x_31, 0); -lean_inc(x_42); -lean_dec(x_31); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_41); -return x_43; -} -} -} -} -} -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__15(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Meta_instInhabitedPostponedEntry; -x_3 = lean_panic_fn(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; uint8_t x_254; uint8_t x_255; -x_254 = 2; -x_255 = l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_101_(x_3, x_254); -if (x_255 == 0) -{ -lean_object* x_256; -x_256 = lean_box(0); -x_11 = x_256; -goto block_253; -} -else -{ -uint8_t x_257; -lean_inc(x_2); -x_257 = l_Lean_MessageData_hasSyntheticSorry(x_2); -if (x_257 == 0) -{ -lean_object* x_258; -x_258 = lean_box(0); -x_11 = x_258; -goto block_253; -} -else -{ -lean_object* x_259; lean_object* x_260; -lean_dec(x_2); -x_259 = lean_box(0); -x_260 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_260, 0, x_259); -lean_ctor_set(x_260, 1, x_10); -return x_260; -} -} -block_253: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_11); -x_12 = lean_ctor_get(x_8, 0); -x_13 = lean_ctor_get(x_8, 1); -x_14 = lean_ctor_get(x_8, 5); -x_15 = lean_ctor_get(x_8, 6); -x_16 = lean_ctor_get(x_8, 7); -x_17 = l_Lean_replaceRef(x_1, x_14); -x_18 = 0; -x_19 = l_Lean_Syntax_getPos_x3f(x_17, x_18); -x_20 = l_Lean_Syntax_getTailPos_x3f(x_17, x_18); -if (lean_obj_tag(x_19) == 0) -{ -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_21 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_FileMap_toPosition(x_13, x_24); -lean_inc(x_25); -x_26 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_26, 0, x_25); -lean_inc(x_16); -lean_inc(x_15); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_15); -lean_ctor_set(x_27, 1, x_16); -x_28 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_22); -x_29 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__7; -lean_inc(x_12); -x_30 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_30, 0, x_12); -lean_ctor_set(x_30, 1, x_25); -lean_ctor_set(x_30, 2, x_26); -lean_ctor_set(x_30, 3, x_29); -lean_ctor_set(x_30, 4, x_28); -lean_ctor_set_uint8(x_30, sizeof(void*)*5, x_3); -x_31 = lean_st_ref_take(x_9, x_23); -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -x_34 = !lean_is_exclusive(x_32); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_35 = lean_ctor_get(x_32, 5); -x_36 = l_Std_PersistentArray_push___rarg(x_35, x_30); -lean_ctor_set(x_32, 5, x_36); -x_37 = lean_st_ref_set(x_9, x_32, x_33); -x_38 = !lean_is_exclusive(x_37); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_37, 0); -lean_dec(x_39); -x_40 = lean_box(0); -lean_ctor_set(x_37, 0, x_40); -return x_37; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_37, 1); -lean_inc(x_41); -lean_dec(x_37); -x_42 = lean_box(0); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_41); -return x_43; -} -} -else -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_44 = lean_ctor_get(x_32, 0); -x_45 = lean_ctor_get(x_32, 1); -x_46 = lean_ctor_get(x_32, 2); -x_47 = lean_ctor_get(x_32, 3); -x_48 = lean_ctor_get(x_32, 4); -x_49 = lean_ctor_get(x_32, 5); -lean_inc(x_49); -lean_inc(x_48); -lean_inc(x_47); -lean_inc(x_46); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_32); -x_50 = l_Std_PersistentArray_push___rarg(x_49, x_30); -x_51 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_51, 0, x_44); -lean_ctor_set(x_51, 1, x_45); -lean_ctor_set(x_51, 2, x_46); -lean_ctor_set(x_51, 3, x_47); -lean_ctor_set(x_51, 4, x_48); -lean_ctor_set(x_51, 5, x_50); -x_52 = lean_st_ref_set(x_9, x_51, x_33); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -if (lean_is_exclusive(x_52)) { - lean_ctor_release(x_52, 0); - lean_ctor_release(x_52, 1); - x_54 = x_52; -} else { - lean_dec_ref(x_52); - x_54 = lean_box(0); -} -x_55 = lean_box(0); -if (lean_is_scalar(x_54)) { - x_56 = lean_alloc_ctor(0, 2, 0); -} else { - x_56 = x_54; -} -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_53); -return x_56; -} -} -else -{ -uint8_t x_57; -x_57 = !lean_is_exclusive(x_20); -if (x_57 == 0) -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -x_58 = lean_ctor_get(x_20, 0); -x_59 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); -lean_dec(x_59); -x_62 = lean_unsigned_to_nat(0u); -x_63 = l_Lean_FileMap_toPosition(x_13, x_62); -x_64 = l_Lean_FileMap_toPosition(x_13, x_58); -lean_dec(x_58); -lean_ctor_set(x_20, 0, x_64); -lean_inc(x_16); -lean_inc(x_15); -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_15); -lean_ctor_set(x_65, 1, x_16); -x_66 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_60); -x_67 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__7; -lean_inc(x_12); -x_68 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_68, 0, x_12); -lean_ctor_set(x_68, 1, x_63); -lean_ctor_set(x_68, 2, x_20); -lean_ctor_set(x_68, 3, x_67); -lean_ctor_set(x_68, 4, x_66); -lean_ctor_set_uint8(x_68, sizeof(void*)*5, x_3); -x_69 = lean_st_ref_take(x_9, x_61); -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_69, 1); -lean_inc(x_71); -lean_dec(x_69); -x_72 = !lean_is_exclusive(x_70); -if (x_72 == 0) -{ -lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_73 = lean_ctor_get(x_70, 5); -x_74 = l_Std_PersistentArray_push___rarg(x_73, x_68); -lean_ctor_set(x_70, 5, x_74); -x_75 = lean_st_ref_set(x_9, x_70, x_71); -x_76 = !lean_is_exclusive(x_75); -if (x_76 == 0) -{ -lean_object* x_77; lean_object* x_78; -x_77 = lean_ctor_get(x_75, 0); -lean_dec(x_77); -x_78 = lean_box(0); -lean_ctor_set(x_75, 0, x_78); -return x_75; -} -else -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_75, 1); -lean_inc(x_79); -lean_dec(x_75); -x_80 = lean_box(0); -x_81 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_81, 1, x_79); -return x_81; -} -} -else -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_82 = lean_ctor_get(x_70, 0); -x_83 = lean_ctor_get(x_70, 1); -x_84 = lean_ctor_get(x_70, 2); -x_85 = lean_ctor_get(x_70, 3); -x_86 = lean_ctor_get(x_70, 4); -x_87 = lean_ctor_get(x_70, 5); -lean_inc(x_87); -lean_inc(x_86); -lean_inc(x_85); -lean_inc(x_84); -lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_70); -x_88 = l_Std_PersistentArray_push___rarg(x_87, x_68); -x_89 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_89, 0, x_82); -lean_ctor_set(x_89, 1, x_83); -lean_ctor_set(x_89, 2, x_84); -lean_ctor_set(x_89, 3, x_85); -lean_ctor_set(x_89, 4, x_86); -lean_ctor_set(x_89, 5, x_88); -x_90 = lean_st_ref_set(x_9, x_89, x_71); -x_91 = lean_ctor_get(x_90, 1); -lean_inc(x_91); -if (lean_is_exclusive(x_90)) { - lean_ctor_release(x_90, 0); - lean_ctor_release(x_90, 1); - x_92 = x_90; -} else { - lean_dec_ref(x_90); - x_92 = lean_box(0); -} -x_93 = lean_box(0); -if (lean_is_scalar(x_92)) { - x_94 = lean_alloc_ctor(0, 2, 0); -} else { - x_94 = x_92; -} -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_91); -return x_94; -} -} -else -{ -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; -x_95 = lean_ctor_get(x_20, 0); -lean_inc(x_95); -lean_dec(x_20); -x_96 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); -x_97 = lean_ctor_get(x_96, 0); -lean_inc(x_97); -x_98 = lean_ctor_get(x_96, 1); -lean_inc(x_98); -lean_dec(x_96); -x_99 = lean_unsigned_to_nat(0u); -x_100 = l_Lean_FileMap_toPosition(x_13, x_99); -x_101 = l_Lean_FileMap_toPosition(x_13, x_95); -lean_dec(x_95); -x_102 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_102, 0, x_101); -lean_inc(x_16); -lean_inc(x_15); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_15); -lean_ctor_set(x_103, 1, x_16); -x_104 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_97); -x_105 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__7; -lean_inc(x_12); -x_106 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_106, 0, x_12); -lean_ctor_set(x_106, 1, x_100); -lean_ctor_set(x_106, 2, x_102); -lean_ctor_set(x_106, 3, x_105); -lean_ctor_set(x_106, 4, x_104); -lean_ctor_set_uint8(x_106, sizeof(void*)*5, x_3); -x_107 = lean_st_ref_take(x_9, x_98); -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = lean_ctor_get(x_108, 0); -lean_inc(x_110); -x_111 = lean_ctor_get(x_108, 1); -lean_inc(x_111); -x_112 = lean_ctor_get(x_108, 2); -lean_inc(x_112); -x_113 = lean_ctor_get(x_108, 3); -lean_inc(x_113); -x_114 = lean_ctor_get(x_108, 4); -lean_inc(x_114); -x_115 = lean_ctor_get(x_108, 5); -lean_inc(x_115); -if (lean_is_exclusive(x_108)) { - lean_ctor_release(x_108, 0); - lean_ctor_release(x_108, 1); - lean_ctor_release(x_108, 2); - lean_ctor_release(x_108, 3); - lean_ctor_release(x_108, 4); - lean_ctor_release(x_108, 5); - x_116 = x_108; -} else { - lean_dec_ref(x_108); - x_116 = lean_box(0); -} -x_117 = l_Std_PersistentArray_push___rarg(x_115, x_106); -if (lean_is_scalar(x_116)) { - x_118 = lean_alloc_ctor(0, 6, 0); -} else { - x_118 = x_116; -} -lean_ctor_set(x_118, 0, x_110); -lean_ctor_set(x_118, 1, x_111); -lean_ctor_set(x_118, 2, x_112); -lean_ctor_set(x_118, 3, x_113); -lean_ctor_set(x_118, 4, x_114); -lean_ctor_set(x_118, 5, x_117); -x_119 = lean_st_ref_set(x_9, x_118, x_109); -x_120 = lean_ctor_get(x_119, 1); -lean_inc(x_120); -if (lean_is_exclusive(x_119)) { - lean_ctor_release(x_119, 0); - lean_ctor_release(x_119, 1); - x_121 = x_119; -} else { - lean_dec_ref(x_119); - x_121 = lean_box(0); -} -x_122 = lean_box(0); -if (lean_is_scalar(x_121)) { - x_123 = lean_alloc_ctor(0, 2, 0); -} else { - x_123 = x_121; -} -lean_ctor_set(x_123, 0, x_122); -lean_ctor_set(x_123, 1, x_120); -return x_123; -} -} -} -else -{ -if (lean_obj_tag(x_20) == 0) -{ -uint8_t x_124; -x_124 = !lean_is_exclusive(x_19); -if (x_124 == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; uint8_t x_137; -x_125 = lean_ctor_get(x_19, 0); -x_126 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); -x_127 = lean_ctor_get(x_126, 0); -lean_inc(x_127); -x_128 = lean_ctor_get(x_126, 1); -lean_inc(x_128); -lean_dec(x_126); -x_129 = l_Lean_FileMap_toPosition(x_13, x_125); -lean_dec(x_125); -lean_inc(x_129); -lean_ctor_set(x_19, 0, x_129); -lean_inc(x_16); -lean_inc(x_15); -x_130 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_130, 0, x_15); -lean_ctor_set(x_130, 1, x_16); -x_131 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_131, 0, x_130); -lean_ctor_set(x_131, 1, x_127); -x_132 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__7; -lean_inc(x_12); -x_133 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_133, 0, x_12); -lean_ctor_set(x_133, 1, x_129); -lean_ctor_set(x_133, 2, x_19); -lean_ctor_set(x_133, 3, x_132); -lean_ctor_set(x_133, 4, x_131); -lean_ctor_set_uint8(x_133, sizeof(void*)*5, x_3); -x_134 = lean_st_ref_take(x_9, x_128); -x_135 = lean_ctor_get(x_134, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_134, 1); -lean_inc(x_136); -lean_dec(x_134); -x_137 = !lean_is_exclusive(x_135); -if (x_137 == 0) -{ -lean_object* x_138; lean_object* x_139; lean_object* x_140; uint8_t x_141; -x_138 = lean_ctor_get(x_135, 5); -x_139 = l_Std_PersistentArray_push___rarg(x_138, x_133); -lean_ctor_set(x_135, 5, x_139); -x_140 = lean_st_ref_set(x_9, x_135, x_136); -x_141 = !lean_is_exclusive(x_140); -if (x_141 == 0) -{ -lean_object* x_142; lean_object* x_143; -x_142 = lean_ctor_get(x_140, 0); -lean_dec(x_142); -x_143 = lean_box(0); -lean_ctor_set(x_140, 0, x_143); -return x_140; -} -else -{ -lean_object* x_144; lean_object* x_145; lean_object* x_146; -x_144 = lean_ctor_get(x_140, 1); -lean_inc(x_144); -lean_dec(x_140); -x_145 = lean_box(0); -x_146 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_146, 0, x_145); -lean_ctor_set(x_146, 1, x_144); -return x_146; -} -} -else -{ -lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_147 = lean_ctor_get(x_135, 0); -x_148 = lean_ctor_get(x_135, 1); -x_149 = lean_ctor_get(x_135, 2); -x_150 = lean_ctor_get(x_135, 3); -x_151 = lean_ctor_get(x_135, 4); -x_152 = lean_ctor_get(x_135, 5); -lean_inc(x_152); -lean_inc(x_151); -lean_inc(x_150); -lean_inc(x_149); -lean_inc(x_148); -lean_inc(x_147); -lean_dec(x_135); -x_153 = l_Std_PersistentArray_push___rarg(x_152, x_133); -x_154 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_154, 0, x_147); -lean_ctor_set(x_154, 1, x_148); -lean_ctor_set(x_154, 2, x_149); -lean_ctor_set(x_154, 3, x_150); -lean_ctor_set(x_154, 4, x_151); -lean_ctor_set(x_154, 5, x_153); -x_155 = lean_st_ref_set(x_9, x_154, x_136); -x_156 = lean_ctor_get(x_155, 1); -lean_inc(x_156); -if (lean_is_exclusive(x_155)) { - lean_ctor_release(x_155, 0); - lean_ctor_release(x_155, 1); - x_157 = x_155; -} else { - lean_dec_ref(x_155); - x_157 = lean_box(0); -} -x_158 = lean_box(0); -if (lean_is_scalar(x_157)) { - x_159 = lean_alloc_ctor(0, 2, 0); -} else { - x_159 = x_157; -} -lean_ctor_set(x_159, 0, x_158); -lean_ctor_set(x_159, 1, x_156); -return x_159; -} -} -else -{ -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_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; -x_160 = lean_ctor_get(x_19, 0); -lean_inc(x_160); -lean_dec(x_19); -x_161 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); -x_162 = lean_ctor_get(x_161, 0); -lean_inc(x_162); -x_163 = lean_ctor_get(x_161, 1); -lean_inc(x_163); -lean_dec(x_161); -x_164 = l_Lean_FileMap_toPosition(x_13, x_160); -lean_dec(x_160); -lean_inc(x_164); -x_165 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_165, 0, x_164); -lean_inc(x_16); -lean_inc(x_15); -x_166 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_166, 0, x_15); -lean_ctor_set(x_166, 1, x_16); -x_167 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_167, 0, x_166); -lean_ctor_set(x_167, 1, x_162); -x_168 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__7; -lean_inc(x_12); -x_169 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_169, 0, x_12); -lean_ctor_set(x_169, 1, x_164); -lean_ctor_set(x_169, 2, x_165); -lean_ctor_set(x_169, 3, x_168); -lean_ctor_set(x_169, 4, x_167); -lean_ctor_set_uint8(x_169, sizeof(void*)*5, x_3); -x_170 = lean_st_ref_take(x_9, x_163); -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 = lean_ctor_get(x_171, 0); -lean_inc(x_173); -x_174 = lean_ctor_get(x_171, 1); -lean_inc(x_174); -x_175 = lean_ctor_get(x_171, 2); -lean_inc(x_175); -x_176 = lean_ctor_get(x_171, 3); -lean_inc(x_176); -x_177 = lean_ctor_get(x_171, 4); -lean_inc(x_177); -x_178 = lean_ctor_get(x_171, 5); -lean_inc(x_178); -if (lean_is_exclusive(x_171)) { - lean_ctor_release(x_171, 0); - lean_ctor_release(x_171, 1); - lean_ctor_release(x_171, 2); - lean_ctor_release(x_171, 3); - lean_ctor_release(x_171, 4); - lean_ctor_release(x_171, 5); - x_179 = x_171; -} else { - lean_dec_ref(x_171); - x_179 = lean_box(0); -} -x_180 = l_Std_PersistentArray_push___rarg(x_178, x_169); -if (lean_is_scalar(x_179)) { - x_181 = lean_alloc_ctor(0, 6, 0); -} else { - x_181 = x_179; -} -lean_ctor_set(x_181, 0, x_173); -lean_ctor_set(x_181, 1, x_174); -lean_ctor_set(x_181, 2, x_175); -lean_ctor_set(x_181, 3, x_176); -lean_ctor_set(x_181, 4, x_177); -lean_ctor_set(x_181, 5, x_180); -x_182 = lean_st_ref_set(x_9, x_181, x_172); -x_183 = lean_ctor_get(x_182, 1); -lean_inc(x_183); -if (lean_is_exclusive(x_182)) { - lean_ctor_release(x_182, 0); - lean_ctor_release(x_182, 1); - x_184 = x_182; -} else { - lean_dec_ref(x_182); - x_184 = lean_box(0); -} -x_185 = lean_box(0); -if (lean_is_scalar(x_184)) { - x_186 = lean_alloc_ctor(0, 2, 0); -} else { - x_186 = x_184; -} -lean_ctor_set(x_186, 0, x_185); -lean_ctor_set(x_186, 1, x_183); -return x_186; -} -} -else -{ -lean_object* x_187; uint8_t x_188; -x_187 = lean_ctor_get(x_19, 0); -lean_inc(x_187); -lean_dec(x_19); -x_188 = !lean_is_exclusive(x_20); -if (x_188 == 0) -{ -lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; uint8_t x_202; -x_189 = lean_ctor_get(x_20, 0); -x_190 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); -x_191 = lean_ctor_get(x_190, 0); -lean_inc(x_191); -x_192 = lean_ctor_get(x_190, 1); -lean_inc(x_192); -lean_dec(x_190); -x_193 = l_Lean_FileMap_toPosition(x_13, x_187); -lean_dec(x_187); -x_194 = l_Lean_FileMap_toPosition(x_13, x_189); -lean_dec(x_189); -lean_ctor_set(x_20, 0, x_194); -lean_inc(x_16); -lean_inc(x_15); -x_195 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_195, 0, x_15); -lean_ctor_set(x_195, 1, x_16); -x_196 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_196, 0, x_195); -lean_ctor_set(x_196, 1, x_191); -x_197 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__7; -lean_inc(x_12); -x_198 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_198, 0, x_12); -lean_ctor_set(x_198, 1, x_193); -lean_ctor_set(x_198, 2, x_20); -lean_ctor_set(x_198, 3, x_197); -lean_ctor_set(x_198, 4, x_196); -lean_ctor_set_uint8(x_198, sizeof(void*)*5, x_3); -x_199 = lean_st_ref_take(x_9, x_192); -x_200 = lean_ctor_get(x_199, 0); -lean_inc(x_200); -x_201 = lean_ctor_get(x_199, 1); -lean_inc(x_201); -lean_dec(x_199); -x_202 = !lean_is_exclusive(x_200); -if (x_202 == 0) -{ -lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_206; -x_203 = lean_ctor_get(x_200, 5); -x_204 = l_Std_PersistentArray_push___rarg(x_203, x_198); -lean_ctor_set(x_200, 5, x_204); -x_205 = lean_st_ref_set(x_9, x_200, x_201); -x_206 = !lean_is_exclusive(x_205); -if (x_206 == 0) -{ -lean_object* x_207; lean_object* x_208; -x_207 = lean_ctor_get(x_205, 0); -lean_dec(x_207); -x_208 = lean_box(0); -lean_ctor_set(x_205, 0, x_208); -return x_205; -} -else -{ -lean_object* x_209; lean_object* x_210; lean_object* x_211; -x_209 = lean_ctor_get(x_205, 1); -lean_inc(x_209); -lean_dec(x_205); -x_210 = lean_box(0); -x_211 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_211, 0, x_210); -lean_ctor_set(x_211, 1, x_209); -return x_211; -} -} -else -{ -lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; -x_212 = lean_ctor_get(x_200, 0); -x_213 = lean_ctor_get(x_200, 1); -x_214 = lean_ctor_get(x_200, 2); -x_215 = lean_ctor_get(x_200, 3); -x_216 = lean_ctor_get(x_200, 4); -x_217 = lean_ctor_get(x_200, 5); -lean_inc(x_217); -lean_inc(x_216); -lean_inc(x_215); -lean_inc(x_214); -lean_inc(x_213); -lean_inc(x_212); -lean_dec(x_200); -x_218 = l_Std_PersistentArray_push___rarg(x_217, x_198); -x_219 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_219, 0, x_212); -lean_ctor_set(x_219, 1, x_213); -lean_ctor_set(x_219, 2, x_214); -lean_ctor_set(x_219, 3, x_215); -lean_ctor_set(x_219, 4, x_216); -lean_ctor_set(x_219, 5, x_218); -x_220 = lean_st_ref_set(x_9, x_219, x_201); -x_221 = lean_ctor_get(x_220, 1); -lean_inc(x_221); -if (lean_is_exclusive(x_220)) { - lean_ctor_release(x_220, 0); - lean_ctor_release(x_220, 1); - x_222 = x_220; -} else { - lean_dec_ref(x_220); - x_222 = lean_box(0); -} -x_223 = lean_box(0); -if (lean_is_scalar(x_222)) { - x_224 = lean_alloc_ctor(0, 2, 0); -} else { - x_224 = x_222; -} -lean_ctor_set(x_224, 0, x_223); -lean_ctor_set(x_224, 1, x_221); -return x_224; -} +lean_dec(x_31); +lean_ctor_set(x_29, 0, x_40); +return x_29; } else { -lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; -x_225 = lean_ctor_get(x_20, 0); -lean_inc(x_225); -lean_dec(x_20); -x_226 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); -x_227 = lean_ctor_get(x_226, 0); -lean_inc(x_227); -x_228 = lean_ctor_get(x_226, 1); -lean_inc(x_228); -lean_dec(x_226); -x_229 = l_Lean_FileMap_toPosition(x_13, x_187); -lean_dec(x_187); -x_230 = l_Lean_FileMap_toPosition(x_13, x_225); -lean_dec(x_225); -x_231 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_231, 0, x_230); -lean_inc(x_16); -lean_inc(x_15); -x_232 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_232, 0, x_15); -lean_ctor_set(x_232, 1, x_16); -x_233 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_233, 0, x_232); -lean_ctor_set(x_233, 1, x_227); -x_234 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__7; -lean_inc(x_12); -x_235 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_235, 0, x_12); -lean_ctor_set(x_235, 1, x_229); -lean_ctor_set(x_235, 2, x_231); -lean_ctor_set(x_235, 3, x_234); -lean_ctor_set(x_235, 4, x_233); -lean_ctor_set_uint8(x_235, sizeof(void*)*5, x_3); -x_236 = lean_st_ref_take(x_9, x_228); -x_237 = lean_ctor_get(x_236, 0); -lean_inc(x_237); -x_238 = lean_ctor_get(x_236, 1); -lean_inc(x_238); -lean_dec(x_236); -x_239 = lean_ctor_get(x_237, 0); -lean_inc(x_239); -x_240 = lean_ctor_get(x_237, 1); -lean_inc(x_240); -x_241 = lean_ctor_get(x_237, 2); -lean_inc(x_241); -x_242 = lean_ctor_get(x_237, 3); -lean_inc(x_242); -x_243 = lean_ctor_get(x_237, 4); -lean_inc(x_243); -x_244 = lean_ctor_get(x_237, 5); -lean_inc(x_244); -if (lean_is_exclusive(x_237)) { - lean_ctor_release(x_237, 0); - lean_ctor_release(x_237, 1); - lean_ctor_release(x_237, 2); - lean_ctor_release(x_237, 3); - lean_ctor_release(x_237, 4); - lean_ctor_release(x_237, 5); - x_245 = x_237; -} else { - lean_dec_ref(x_237); - x_245 = lean_box(0); -} -x_246 = l_Std_PersistentArray_push___rarg(x_244, x_235); -if (lean_is_scalar(x_245)) { - x_247 = lean_alloc_ctor(0, 6, 0); -} else { - x_247 = x_245; -} -lean_ctor_set(x_247, 0, x_239); -lean_ctor_set(x_247, 1, x_240); -lean_ctor_set(x_247, 2, x_241); -lean_ctor_set(x_247, 3, x_242); -lean_ctor_set(x_247, 4, x_243); -lean_ctor_set(x_247, 5, x_246); -x_248 = lean_st_ref_set(x_9, x_247, x_238); -x_249 = lean_ctor_get(x_248, 1); -lean_inc(x_249); -if (lean_is_exclusive(x_248)) { - lean_ctor_release(x_248, 0); - lean_ctor_release(x_248, 1); - x_250 = x_248; -} else { - lean_dec_ref(x_248); - x_250 = lean_box(0); -} -x_251 = lean_box(0); -if (lean_is_scalar(x_250)) { - x_252 = lean_alloc_ctor(0, 2, 0); -} else { - x_252 = x_250; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_29, 1); +lean_inc(x_41); +lean_dec(x_29); +x_42 = lean_ctor_get(x_31, 0); +lean_inc(x_42); +lean_dec(x_31); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_41); +return x_43; } -lean_ctor_set(x_252, 0, x_251); -lean_ctor_set(x_252, 1, x_249); -return x_252; } } } } +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__15(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Meta_instInhabitedPostponedEntry; +x_3 = lean_panic_fn(x_2, x_1); +return x_3; } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___closed__1() { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___closed__1() { _start: { lean_object* x_1; @@ -12386,7 +11983,7 @@ x_1 = lean_mk_string_from_bytes("stuck at solving universe constraint", 36); return x_1; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_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___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, 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; @@ -12409,7 +12006,7 @@ if (x_20 == 0) lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; x_21 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___spec__1___closed__4; x_22 = l_panic___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__15(x_21); -x_23 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___closed__1; +x_23 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___closed__1; lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -12428,7 +12025,7 @@ x_27 = lean_ctor_get(x_22, 0); lean_inc(x_27); lean_dec(x_22); x_28 = 2; -x_29 = l_Lean_logAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(x_27, x_25, x_28, x_8, x_9, x_10, x_11, x_12, x_13, x_26); +x_29 = l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4(x_27, x_25, x_28, x_8, x_9, x_10, x_11, x_12, x_13, x_26); lean_dec(x_27); x_30 = lean_ctor_get(x_29, 1); lean_inc(x_30); @@ -12476,7 +12073,7 @@ else { lean_object* x_38; lean_object* x_39; lean_object* x_40; x_38 = lean_array_fget(x_1, x_4); -x_39 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___closed__1; +x_39 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___closed__1; lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -12495,7 +12092,7 @@ x_43 = lean_ctor_get(x_38, 0); lean_inc(x_43); lean_dec(x_38); x_44 = 2; -x_45 = l_Lean_logAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(x_43, x_41, x_44, x_8, x_9, x_10, x_11, x_12, x_13, x_42); +x_45 = l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4(x_43, x_41, x_44, x_8, x_9, x_10, x_11, x_12, x_13, x_42); lean_dec(x_43); x_46 = lean_ctor_get(x_45, 1); lean_inc(x_46); @@ -12640,7 +12237,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_21); -x_24 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17(x_20, x_21, x_21, x_22, x_21, x_22, x_23, x_1, x_2, x_3, x_4, x_5, x_6, x_19); +x_24 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(x_20, x_21, x_21, x_22, x_21, x_22, x_23, x_1, x_2, x_3, x_4, x_5, x_6, x_19); if (lean_obj_tag(x_24) == 0) { lean_object* x_25; lean_object* x_26; lean_object* x_38; uint8_t x_39; @@ -12670,7 +12267,7 @@ goto block_37; block_37: { lean_object* x_27; lean_object* x_28; -x_27 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___closed__1; +x_27 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___closed__1; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); @@ -12915,28 +12512,11 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_3); -lean_dec(x_3); -x_12 = l_Lean_logAt___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_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___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); @@ -13002,54 +12582,342 @@ return x_10; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_10, 1); -lean_inc(x_18); -lean_dec(x_10); -x_19 = lean_box(0); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -return x_20; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_10, 1); +lean_inc(x_18); +lean_dec(x_10); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; +} +} +} +else +{ +uint8_t x_21; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_10); +if (x_21 == 0) +{ +return x_10; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_10, 0); +x_23 = lean_ctor_get(x_10, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_10); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_processPostponedUniverseContraints___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_processPostponedUniverseContraints(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_5 = lean_ctor_get(x_2, 0); +x_6 = lean_ctor_get(x_2, 1); +x_7 = lean_ctor_get(x_2, 2); +x_8 = lean_ctor_get(x_2, 3); +x_9 = l_Lean_Name_quickCmp(x_1, x_6); +switch (x_9) { +case 0: +{ +uint8_t x_10; +x_10 = l_Std_RBNode_isBlack___rarg(x_5); +if (x_10 == 0) +{ +lean_object* x_11; uint8_t x_12; +x_11 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_5); +x_12 = 0; +lean_ctor_set(x_2, 0, x_11); +lean_ctor_set_uint8(x_2, sizeof(void*)*4, x_12); +return x_2; +} +else +{ +lean_object* x_13; lean_object* x_14; +lean_free_object(x_2); +x_13 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_5); +x_14 = l_Std_RBNode_balLeft___rarg(x_13, x_6, x_7, x_8); +return x_14; +} +} +case 1: +{ +lean_object* x_15; +lean_free_object(x_2); +lean_dec(x_7); +lean_dec(x_6); +x_15 = l_Std_RBNode_appendTrees___rarg(x_5, x_8); +return x_15; +} +default: +{ +uint8_t x_16; +x_16 = l_Std_RBNode_isBlack___rarg(x_8); +if (x_16 == 0) +{ +lean_object* x_17; uint8_t x_18; +x_17 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_8); +x_18 = 0; +lean_ctor_set(x_2, 3, x_17); +lean_ctor_set_uint8(x_2, sizeof(void*)*4, x_18); +return x_2; +} +else +{ +lean_object* x_19; lean_object* x_20; +lean_free_object(x_2); +x_19 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_8); +x_20 = l_Std_RBNode_balRight___rarg(x_5, x_6, x_7, x_19); +return x_20; +} +} +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_21 = lean_ctor_get(x_2, 0); +x_22 = lean_ctor_get(x_2, 1); +x_23 = lean_ctor_get(x_2, 2); +x_24 = lean_ctor_get(x_2, 3); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_2); +x_25 = l_Lean_Name_quickCmp(x_1, x_22); +switch (x_25) { +case 0: +{ +uint8_t x_26; +x_26 = l_Std_RBNode_isBlack___rarg(x_21); +if (x_26 == 0) +{ +lean_object* x_27; uint8_t x_28; lean_object* x_29; +x_27 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_21); +x_28 = 0; +x_29 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_29, 0, x_27); +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_uint8(x_29, sizeof(void*)*4, x_28); +return x_29; +} +else +{ +lean_object* x_30; lean_object* x_31; +x_30 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_21); +x_31 = l_Std_RBNode_balLeft___rarg(x_30, x_22, x_23, x_24); +return x_31; +} +} +case 1: +{ +lean_object* x_32; +lean_dec(x_23); +lean_dec(x_22); +x_32 = l_Std_RBNode_appendTrees___rarg(x_21, x_24); +return x_32; +} +default: +{ +uint8_t x_33; +x_33 = l_Std_RBNode_isBlack___rarg(x_24); +if (x_33 == 0) +{ +lean_object* x_34; uint8_t x_35; lean_object* x_36; +x_34 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_24); +x_35 = 0; +x_36 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_36, 0, x_21); +lean_ctor_set(x_36, 1, x_22); +lean_ctor_set(x_36, 2, x_23); +lean_ctor_set(x_36, 3, x_34); +lean_ctor_set_uint8(x_36, sizeof(void*)*4, x_35); +return x_36; +} +else +{ +lean_object* x_37; lean_object* x_38; +x_37 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_24); +x_38 = l_Std_RBNode_balRight___rarg(x_21, x_22, x_23, x_37); +return x_38; +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_erase___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_2); +x_4 = l_Std_RBNode_setBlack___rarg(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_9 = lean_st_ref_get(x_7, x_8); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = lean_st_ref_take(x_3, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Std_RBNode_erase___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__1(x_1, x_15); +lean_ctor_set(x_12, 1, x_16); +x_17 = lean_st_ref_set(x_3, x_12, x_13); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_17, 0); +lean_dec(x_19); +x_20 = lean_box(0); +lean_ctor_set(x_17, 0, x_20); +return x_17; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; +} +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_24 = lean_ctor_get(x_12, 0); +x_25 = lean_ctor_get(x_12, 1); +x_26 = lean_ctor_get(x_12, 2); +x_27 = lean_ctor_get(x_12, 3); +x_28 = lean_ctor_get(x_12, 4); +x_29 = lean_ctor_get(x_12, 5); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_12); +x_30 = l_Std_RBNode_erase___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__1(x_1, x_25); +x_31 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_31, 0, x_24); +lean_ctor_set(x_31, 1, x_30); +lean_ctor_set(x_31, 2, x_26); +lean_ctor_set(x_31, 3, x_27); +lean_ctor_set(x_31, 4, x_28); +lean_ctor_set(x_31, 5, x_29); +x_32 = lean_st_ref_set(x_3, x_31, x_13); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +if (lean_is_exclusive(x_32)) { + lean_ctor_release(x_32, 0); + lean_ctor_release(x_32, 1); + x_34 = x_32; +} else { + lean_dec_ref(x_32); + x_34 = lean_box(0); +} +x_35 = lean_box(0); +if (lean_is_scalar(x_34)) { + x_36 = lean_alloc_ctor(0, 2, 0); +} else { + x_36 = x_34; } +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_33); +return x_36; } } -else -{ -uint8_t x_21; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_21 = !lean_is_exclusive(x_10); -if (x_21 == 0) -{ -return x_10; } -else +LEAN_EXPORT lean_object* l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_10, 0); -x_23 = lean_ctor_get(x_10, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_10); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_3; +x_3 = l_Std_RBNode_del___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__2(x_1, x_2); +lean_dec(x_1); +return x_3; } } +LEAN_EXPORT lean_object* l_Std_RBNode_erase___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_RBNode_erase___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___spec__1(x_1, x_2); +lean_dec(x_1); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_processPostponedUniverseContraints___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_8; -x_8 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_processPostponedUniverseContraints(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_object* x_9; +x_9 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -return x_8; +lean_dec(x_1); +return x_9; } } static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesizeSyntheticMVars_loop___spec__1___closed__1() { @@ -13089,9 +12957,18 @@ return x_11; LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars_loop(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +lean_object* x_11; lean_dec(x_3); -x_11 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg(x_5, x_6, x_7, x_8, x_9, x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_11 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef(x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); @@ -13158,7 +13035,7 @@ if (x_34 == 0) lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; x_35 = lean_ctor_get(x_33, 0); x_36 = lean_ctor_get(x_33, 1); -x_37 = lean_ctor_get(x_35, 1); +x_37 = lean_ctor_get(x_35, 2); lean_inc(x_37); lean_dec(x_35); x_38 = l_List_isEmpty___rarg(x_37); @@ -13555,7 +13432,7 @@ x_111 = lean_ctor_get(x_33, 1); lean_inc(x_111); lean_inc(x_110); lean_dec(x_33); -x_112 = lean_ctor_get(x_110, 1); +x_112 = lean_ctor_get(x_110, 2); lean_inc(x_112); lean_dec(x_110); x_113 = l_List_isEmpty___rarg(x_112); @@ -14065,7 +13942,7 @@ if (lean_is_exclusive(x_204)) { lean_dec_ref(x_204); x_207 = lean_box(0); } -x_208 = lean_ctor_get(x_205, 1); +x_208 = lean_ctor_get(x_205, 2); lean_inc(x_208); lean_dec(x_205); x_209 = l_List_isEmpty___rarg(x_208); @@ -14491,33 +14368,223 @@ return x_280; } } } +else +{ +uint8_t x_281; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_281 = !lean_is_exclusive(x_11); +if (x_281 == 0) +{ +return x_11; +} +else +{ +lean_object* x_282; lean_object* x_283; lean_object* x_284; +x_282 = lean_ctor_get(x_11, 0); +x_283 = lean_ctor_get(x_11, 1); +lean_inc(x_283); +lean_inc(x_282); +lean_dec(x_11); +x_284 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_284, 0, x_282); +lean_ctor_set(x_284, 1, x_283); +return x_284; +} +} +} +} +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +if (x_1 == 0) +{ +uint8_t x_10; lean_object* x_11; lean_object* x_12; +x_10 = 1; +x_11 = lean_box(x_10); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_9); +return x_12; +} +else +{ +uint8_t x_13; lean_object* x_14; lean_object* x_15; +x_13 = 0; +x_14 = lean_box(x_13); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_9); +return x_15; +} +} +} +static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("not ready yet", 13); +return x_1; +} +} +static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__1; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__2; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("succeeded", 9); +return x_1; +} +} +static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__4; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__5; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +lean_dec(x_3); +x_26 = lean_st_ref_get(x_9, x_10); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_27, 3); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_ctor_get_uint8(x_28, sizeof(void*)*1); +lean_dec(x_28); +if (x_29 == 0) +{ +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_26, 1); +lean_inc(x_30); +lean_dec(x_26); +x_31 = 0; +x_11 = x_31; +x_12 = x_30; +goto block_25; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_32 = lean_ctor_get(x_26, 1); +lean_inc(x_32); +lean_dec(x_26); +lean_inc(x_1); +x_33 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_32); +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_unbox(x_34); +lean_dec(x_34); +x_11 = x_36; +x_12 = x_35; +goto block_25; +} +block_25: +{ +if (x_11 == 0) +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_1); +x_13 = lean_box(0); +x_14 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1(x_2, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_14; +} +else +{ +if (x_2 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__3; +x_16 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_1, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_12); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1(x_2, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_17); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_20 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__6; +x_21 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_1, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_12); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1(x_2, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_22); +return x_24; } -LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -if (x_1 == 0) -{ -uint8_t x_10; lean_object* x_11; lean_object* x_12; -x_10 = 1; -x_11 = lean_box(x_10); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_9); -return x_12; } -else -{ -uint8_t x_13; lean_object* x_14; lean_object* x_15; -x_13 = 0; -x_14 = lean_box(x_13); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_9); -return x_15; } } } -LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; @@ -14537,7 +14604,7 @@ static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMV _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("not ready yet", 13); +x_1 = lean_mk_string_from_bytes("resuming ", 9); return x_1; } } @@ -14546,62 +14613,6 @@ static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMV { lean_object* x_1; lean_object* x_2; x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__2; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__3; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("succeeded", 9); -return x_1; -} -} -static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__5; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__6; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("resuming ", 9); -return x_1; -} -} -static lean_object* _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__8; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } @@ -14626,7 +14637,7 @@ return x_13; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_23; lean_object* x_24; lean_object* x_25; 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; uint8_t x_60; x_14 = lean_ctor_get(x_4, 0); lean_inc(x_14); x_15 = lean_ctor_get(x_4, 1); @@ -14642,96 +14653,93 @@ if (lean_is_exclusive(x_4)) { x_23 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__1; lean_inc(x_3); x_24 = l_Lean_Name_str___override(x_3, x_23); -x_73 = lean_ctor_get(x_14, 0); -lean_inc(x_73); -lean_inc(x_73); -x_74 = l_Lean_Expr_mvar___override(x_73); -x_75 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_75, 0, x_74); -x_76 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__9; -x_77 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_77, 0, x_76); -lean_ctor_set(x_77, 1, x_75); -x_78 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__8; -x_79 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_79, 0, x_77); -lean_ctor_set(x_79, 1, x_78); -x_80 = lean_alloc_closure((void*)(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___boxed), 8, 1); -lean_closure_set(x_80, 0, x_79); -x_81 = lean_st_ref_get(x_11, x_12); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_82, 3); -lean_inc(x_83); -lean_dec(x_82); -x_84 = lean_ctor_get_uint8(x_83, sizeof(void*)*1); -lean_dec(x_83); -if (x_84 == 0) +lean_inc(x_14); +x_50 = l_Lean_Expr_mvar___override(x_14); +x_51 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_51, 0, x_50); +x_52 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__3; +x_53 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +x_54 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__2___closed__8; +x_55 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +x_56 = lean_alloc_closure((void*)(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__3___boxed), 8, 1); +lean_closure_set(x_56, 0, x_55); +x_57 = lean_st_ref_get(x_11, x_12); +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_58, 3); +lean_inc(x_59); +lean_dec(x_58); +x_60 = lean_ctor_get_uint8(x_59, sizeof(void*)*1); +lean_dec(x_59); +if (x_60 == 0) { -lean_object* x_85; -lean_dec(x_80); -lean_dec(x_73); -x_85 = lean_ctor_get(x_81, 1); -lean_inc(x_85); -lean_dec(x_81); -x_25 = x_85; -goto block_72; +lean_object* x_61; +lean_dec(x_56); +x_61 = lean_ctor_get(x_57, 1); +lean_inc(x_61); +lean_dec(x_57); +x_25 = x_61; +goto block_49; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; -x_86 = lean_ctor_get(x_81, 1); -lean_inc(x_86); -lean_dec(x_81); +lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; +x_62 = lean_ctor_get(x_57, 1); +lean_inc(x_62); +lean_dec(x_57); lean_inc(x_24); -x_87 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_86); -x_88 = lean_ctor_get(x_87, 0); -lean_inc(x_88); -x_89 = lean_unbox(x_88); -lean_dec(x_88); -if (x_89 == 0) +x_63 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_62); +x_64 = lean_ctor_get(x_63, 0); +lean_inc(x_64); +x_65 = lean_unbox(x_64); +lean_dec(x_64); +if (x_65 == 0) { -lean_object* x_90; -lean_dec(x_80); -lean_dec(x_73); -x_90 = lean_ctor_get(x_87, 1); -lean_inc(x_90); -lean_dec(x_87); -x_25 = x_90; -goto block_72; +lean_object* x_66; +lean_dec(x_56); +x_66 = lean_ctor_get(x_63, 1); +lean_inc(x_66); +lean_dec(x_63); +x_25 = x_66; +goto block_49; } else { -lean_object* x_91; lean_object* x_92; -x_91 = lean_ctor_get(x_87, 1); -lean_inc(x_91); -lean_dec(x_87); +lean_object* x_67; lean_object* x_68; +x_67 = lean_ctor_get(x_63, 1); +lean_inc(x_67); +lean_dec(x_63); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_92 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_73, x_80, x_6, x_7, x_8, x_9, x_10, x_11, x_91); -if (lean_obj_tag(x_92) == 0) +lean_inc(x_14); +x_68 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(x_14, x_56, x_6, x_7, x_8, x_9, x_10, x_11, x_67); +if (lean_obj_tag(x_68) == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -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_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); lean_inc(x_24); -x_95 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_24, x_93, x_6, x_7, x_8, x_9, x_10, x_11, x_94); -x_96 = lean_ctor_get(x_95, 1); -lean_inc(x_96); -lean_dec(x_95); -x_25 = x_96; -goto block_72; +x_71 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_24, x_69, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +x_72 = lean_ctor_get(x_71, 1); +lean_inc(x_72); +lean_dec(x_71); +x_25 = x_72; +goto block_49; } else { -uint8_t x_97; +uint8_t x_73; lean_dec(x_24); lean_dec(x_16); lean_dec(x_15); @@ -14744,23 +14752,23 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_97 = !lean_is_exclusive(x_92); -if (x_97 == 0) +x_73 = !lean_is_exclusive(x_68); +if (x_73 == 0) { -return x_92; +return x_68; } else { -lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_98 = lean_ctor_get(x_92, 0); -x_99 = lean_ctor_get(x_92, 1); -lean_inc(x_99); -lean_inc(x_98); -lean_dec(x_92); -x_100 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_100, 0, x_98); -lean_ctor_set(x_100, 1, x_99); -return x_100; +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_68, 0); +x_75 = lean_ctor_get(x_68, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_68); +x_76 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_75); +return x_76; } } } @@ -14791,7 +14799,7 @@ x_12 = x_18; goto _start; } } -block_72: +block_49: { lean_object* x_26; lean_inc(x_11); @@ -14804,131 +14812,73 @@ lean_inc(x_14); x_26 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar(x_14, x_1, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_25); if (lean_obj_tag(x_26) == 0) { -lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; +lean_object* x_27; uint8_t x_28; x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_57 = lean_st_ref_get(x_11, x_28); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_58, 3); -lean_inc(x_59); -lean_dec(x_58); -x_60 = lean_ctor_get_uint8(x_59, sizeof(void*)*1); -lean_dec(x_59); -if (x_60 == 0) -{ -lean_object* x_61; uint8_t x_62; -x_61 = lean_ctor_get(x_57, 1); -lean_inc(x_61); -lean_dec(x_57); -x_62 = 0; -x_29 = x_62; -x_30 = x_61; -goto block_56; -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; -x_63 = lean_ctor_get(x_57, 1); -lean_inc(x_63); -lean_dec(x_57); -lean_inc(x_24); -x_64 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_63); -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_64, 1); -lean_inc(x_66); -lean_dec(x_64); -x_67 = lean_unbox(x_65); -lean_dec(x_65); -x_29 = x_67; -x_30 = x_66; -goto block_56; -} -block_56: -{ -if (x_29 == 0) +x_28 = lean_unbox(x_27); +if (x_28 == 0) { -lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -lean_dec(x_24); -x_31 = lean_box(0); -x_32 = lean_unbox(x_27); +lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_29 = lean_ctor_get(x_26, 1); +lean_inc(x_29); +lean_dec(x_26); +x_30 = lean_box(0); +x_31 = lean_unbox(x_27); lean_dec(x_27); -x_33 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1(x_32, x_31, x_6, x_7, x_8, x_9, x_10, x_11, x_30); -x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_32 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2(x_24, x_31, x_30, x_6, x_7, x_8, x_9, x_10, x_11, x_29); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); +lean_dec(x_32); +x_35 = lean_unbox(x_33); lean_dec(x_33); -x_36 = lean_unbox(x_34); -lean_dec(x_34); -x_17 = x_36; -x_18 = x_35; -goto block_22; -} -else -{ -uint8_t x_37; -x_37 = lean_unbox(x_27); -if (x_37 == 0) -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_38 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__4; -x_39 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_24, x_38, x_6, x_7, x_8, x_9, x_10, x_11, x_30); -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); -lean_inc(x_41); -lean_dec(x_39); -x_42 = lean_unbox(x_27); -lean_dec(x_27); -x_43 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1(x_42, x_40, x_6, x_7, x_8, x_9, x_10, x_11, x_41); -lean_dec(x_40); -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_43, 1); -lean_inc(x_45); -lean_dec(x_43); -x_46 = lean_unbox(x_44); -lean_dec(x_44); -x_17 = x_46; -x_18 = x_45; +x_17 = x_35; +x_18 = x_34; goto block_22; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_47 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__7; -x_48 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_24, x_47, x_6, x_7, x_8, x_9, x_10, x_11, x_30); -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_48, 1); -lean_inc(x_50); -lean_dec(x_48); -x_51 = lean_unbox(x_27); +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; uint8_t x_44; +x_36 = lean_ctor_get(x_26, 1); +lean_inc(x_36); +lean_dec(x_26); +x_37 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved(x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_36); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = lean_unbox(x_27); lean_dec(x_27); -x_52 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__1(x_51, x_49, x_6, x_7, x_8, x_9, x_10, x_11, x_50); -lean_dec(x_49); -x_53 = lean_ctor_get(x_52, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_52, 1); -lean_inc(x_54); -lean_dec(x_52); -x_55 = lean_unbox(x_53); -lean_dec(x_53); -x_17 = x_55; -x_18 = x_54; +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_41 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2(x_24, x_40, x_38, x_6, x_7, x_8, x_9, x_10, x_11, x_39); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +x_44 = lean_unbox(x_42); +lean_dec(x_42); +x_17 = x_44; +x_18 = x_43; goto block_22; } } -} -} else { -uint8_t x_68; +uint8_t x_45; lean_dec(x_24); lean_dec(x_16); lean_dec(x_15); @@ -14941,23 +14891,23 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_68 = !lean_is_exclusive(x_26); -if (x_68 == 0) +x_45 = !lean_is_exclusive(x_26); +if (x_45 == 0) { return x_26; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_26, 0); -x_70 = lean_ctor_get(x_26, 1); -lean_inc(x_70); -lean_inc(x_69); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_26, 0); +x_47 = lean_ctor_get(x_26, 1); +lean_inc(x_47); +lean_inc(x_46); lean_dec(x_26); -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; +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; } } } @@ -15283,7 +15233,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -x_20 = lean_ctor_get(x_18, 1); +x_20 = lean_ctor_get(x_18, 2); lean_inc(x_20); lean_dec(x_18); x_21 = lean_unsigned_to_nat(0u); @@ -15302,10 +15252,10 @@ x_28 = !lean_is_exclusive(x_26); if (x_28 == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_29 = lean_ctor_get(x_26, 1); +x_29 = lean_ctor_get(x_26, 2); lean_dec(x_29); x_30 = lean_box(0); -lean_ctor_set(x_26, 1, x_30); +lean_ctor_set(x_26, 2, x_30); x_31 = lean_st_ref_set(x_4, x_26, x_27); x_32 = lean_ctor_get(x_31, 1); lean_inc(x_32); @@ -15338,10 +15288,10 @@ x_43 = !lean_is_exclusive(x_41); if (x_43 == 0) { lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_44 = lean_ctor_get(x_41, 1); +x_44 = lean_ctor_get(x_41, 2); lean_inc(x_36); x_45 = l_List_appendTR___rarg(x_44, x_36); -lean_ctor_set(x_41, 1, x_45); +lean_ctor_set(x_41, 2, x_45); x_46 = lean_st_ref_set(x_4, x_41, x_42); lean_dec(x_4); x_47 = !lean_is_exclusive(x_46); @@ -15407,12 +15357,14 @@ return x_63; } else { -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; uint8_t x_75; +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; x_64 = lean_ctor_get(x_41, 0); x_65 = lean_ctor_get(x_41, 1); x_66 = lean_ctor_get(x_41, 2); x_67 = lean_ctor_get(x_41, 3); x_68 = lean_ctor_get(x_41, 4); +x_69 = lean_ctor_get(x_41, 5); +lean_inc(x_69); lean_inc(x_68); lean_inc(x_67); lean_inc(x_66); @@ -15420,238 +15372,246 @@ lean_inc(x_65); lean_inc(x_64); lean_dec(x_41); lean_inc(x_36); -x_69 = l_List_appendTR___rarg(x_65, x_36); -x_70 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_70, 0, x_64); -lean_ctor_set(x_70, 1, x_69); -lean_ctor_set(x_70, 2, x_66); -lean_ctor_set(x_70, 3, x_67); -lean_ctor_set(x_70, 4, x_68); -x_71 = lean_st_ref_set(x_4, x_70, x_42); +x_70 = l_List_appendTR___rarg(x_66, x_36); +x_71 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_71, 0, x_64); +lean_ctor_set(x_71, 1, x_65); +lean_ctor_set(x_71, 2, x_70); +lean_ctor_set(x_71, 3, x_67); +lean_ctor_set(x_71, 4, x_68); +lean_ctor_set(x_71, 5, x_69); +x_72 = lean_st_ref_set(x_4, x_71, x_42); lean_dec(x_4); -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_73 = x_71; +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_74 = x_72; } else { - lean_dec_ref(x_71); - x_73 = lean_box(0); + lean_dec_ref(x_72); + x_74 = lean_box(0); } -x_74 = l_List_lengthTRAux___rarg(x_36, x_21); +x_75 = l_List_lengthTRAux___rarg(x_36, x_21); lean_dec(x_36); -x_75 = lean_nat_dec_eq(x_22, x_74); -lean_dec(x_74); +x_76 = lean_nat_dec_eq(x_22, x_75); +lean_dec(x_75); lean_dec(x_22); -if (x_75 == 0) +if (x_76 == 0) { -uint8_t x_76; lean_object* x_77; lean_object* x_78; -x_76 = 1; -x_77 = lean_box(x_76); -if (lean_is_scalar(x_73)) { - x_78 = lean_alloc_ctor(0, 2, 0); +uint8_t x_77; lean_object* x_78; lean_object* x_79; +x_77 = 1; +x_78 = lean_box(x_77); +if (lean_is_scalar(x_74)) { + x_79 = lean_alloc_ctor(0, 2, 0); } else { - x_78 = x_73; + x_79 = x_74; } -lean_ctor_set(x_78, 0, x_77); -lean_ctor_set(x_78, 1, x_72); -return x_78; +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_73); +return x_79; } else { -uint8_t x_79; lean_object* x_80; lean_object* x_81; -x_79 = 0; -x_80 = lean_box(x_79); -if (lean_is_scalar(x_73)) { - x_81 = lean_alloc_ctor(0, 2, 0); +uint8_t x_80; lean_object* x_81; lean_object* x_82; +x_80 = 0; +x_81 = lean_box(x_80); +if (lean_is_scalar(x_74)) { + x_82 = lean_alloc_ctor(0, 2, 0); } else { - x_81 = x_73; + x_82 = x_74; } -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_81, 1, x_72); -return x_81; +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_73); +return x_82; } } } else { -uint8_t x_82; +uint8_t x_83; lean_dec(x_22); lean_dec(x_8); lean_dec(x_4); -x_82 = !lean_is_exclusive(x_35); -if (x_82 == 0) +x_83 = !lean_is_exclusive(x_35); +if (x_83 == 0) { return x_35; } else { -lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_83 = lean_ctor_get(x_35, 0); -x_84 = lean_ctor_get(x_35, 1); +lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_35, 0); +x_85 = lean_ctor_get(x_35, 1); +lean_inc(x_85); lean_inc(x_84); -lean_inc(x_83); lean_dec(x_35); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -return x_85; +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +return x_86; } } } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_86 = lean_ctor_get(x_26, 0); -x_87 = lean_ctor_get(x_26, 2); -x_88 = lean_ctor_get(x_26, 3); -x_89 = lean_ctor_get(x_26, 4); +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; +x_87 = lean_ctor_get(x_26, 0); +x_88 = lean_ctor_get(x_26, 1); +x_89 = lean_ctor_get(x_26, 3); +x_90 = lean_ctor_get(x_26, 4); +x_91 = lean_ctor_get(x_26, 5); +lean_inc(x_91); +lean_inc(x_90); lean_inc(x_89); lean_inc(x_88); lean_inc(x_87); -lean_inc(x_86); lean_dec(x_26); -x_90 = lean_box(0); -x_91 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_91, 0, x_86); -lean_ctor_set(x_91, 1, x_90); -lean_ctor_set(x_91, 2, x_87); -lean_ctor_set(x_91, 3, x_88); -lean_ctor_set(x_91, 4, x_89); -x_92 = lean_st_ref_set(x_4, x_91, x_27); -x_93 = lean_ctor_get(x_92, 1); -lean_inc(x_93); -lean_dec(x_92); -x_94 = l_List_reverse___rarg(x_20); -x_95 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__2; +x_92 = lean_box(0); +x_93 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_93, 0, x_87); +lean_ctor_set(x_93, 1, x_88); +lean_ctor_set(x_93, 2, x_92); +lean_ctor_set(x_93, 3, x_89); +lean_ctor_set(x_93, 4, x_90); +lean_ctor_set(x_93, 5, x_91); +x_94 = lean_st_ref_set(x_4, x_93, x_27); +x_95 = lean_ctor_get(x_94, 1); +lean_inc(x_95); +lean_dec(x_94); +x_96 = l_List_reverse___rarg(x_20); +x_97 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__2; lean_inc(x_8); lean_inc(x_4); -x_96 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1(x_1, x_2, x_95, x_94, x_90, x_3, x_4, x_5, x_6, x_7, x_8, x_93); -if (lean_obj_tag(x_96) == 0) +x_98 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1(x_1, x_2, x_97, x_96, x_92, x_3, x_4, x_5, x_6, x_7, x_8, x_95); +if (lean_obj_tag(x_98) == 0) { -lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; -x_97 = lean_ctor_get(x_96, 0); -lean_inc(x_97); -x_98 = lean_ctor_get(x_96, 1); -lean_inc(x_98); -lean_dec(x_96); -x_99 = lean_st_ref_get(x_8, x_98); -lean_dec(x_8); -x_100 = lean_ctor_get(x_99, 1); +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; uint8_t x_119; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_98, 1); lean_inc(x_100); -lean_dec(x_99); -x_101 = lean_st_ref_take(x_4, x_100); -x_102 = lean_ctor_get(x_101, 0); +lean_dec(x_98); +x_101 = lean_st_ref_get(x_8, x_100); +lean_dec(x_8); +x_102 = lean_ctor_get(x_101, 1); lean_inc(x_102); -x_103 = lean_ctor_get(x_101, 1); -lean_inc(x_103); lean_dec(x_101); -x_104 = lean_ctor_get(x_102, 0); +x_103 = lean_st_ref_take(x_4, x_102); +x_104 = lean_ctor_get(x_103, 0); lean_inc(x_104); -x_105 = lean_ctor_get(x_102, 1); +x_105 = lean_ctor_get(x_103, 1); lean_inc(x_105); -x_106 = lean_ctor_get(x_102, 2); +lean_dec(x_103); +x_106 = lean_ctor_get(x_104, 0); lean_inc(x_106); -x_107 = lean_ctor_get(x_102, 3); +x_107 = lean_ctor_get(x_104, 1); lean_inc(x_107); -x_108 = lean_ctor_get(x_102, 4); +x_108 = lean_ctor_get(x_104, 2); lean_inc(x_108); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - lean_ctor_release(x_102, 2); - lean_ctor_release(x_102, 3); - lean_ctor_release(x_102, 4); - x_109 = x_102; +x_109 = lean_ctor_get(x_104, 3); +lean_inc(x_109); +x_110 = lean_ctor_get(x_104, 4); +lean_inc(x_110); +x_111 = lean_ctor_get(x_104, 5); +lean_inc(x_111); +if (lean_is_exclusive(x_104)) { + lean_ctor_release(x_104, 0); + lean_ctor_release(x_104, 1); + lean_ctor_release(x_104, 2); + lean_ctor_release(x_104, 3); + lean_ctor_release(x_104, 4); + lean_ctor_release(x_104, 5); + x_112 = x_104; } else { - lean_dec_ref(x_102); - x_109 = lean_box(0); + lean_dec_ref(x_104); + x_112 = lean_box(0); } -lean_inc(x_97); -x_110 = l_List_appendTR___rarg(x_105, x_97); -if (lean_is_scalar(x_109)) { - x_111 = lean_alloc_ctor(0, 5, 0); +lean_inc(x_99); +x_113 = l_List_appendTR___rarg(x_108, x_99); +if (lean_is_scalar(x_112)) { + x_114 = lean_alloc_ctor(0, 6, 0); } else { - x_111 = x_109; + x_114 = x_112; } -lean_ctor_set(x_111, 0, x_104); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_111, 2, x_106); -lean_ctor_set(x_111, 3, x_107); -lean_ctor_set(x_111, 4, x_108); -x_112 = lean_st_ref_set(x_4, x_111, x_103); +lean_ctor_set(x_114, 0, x_106); +lean_ctor_set(x_114, 1, x_107); +lean_ctor_set(x_114, 2, x_113); +lean_ctor_set(x_114, 3, x_109); +lean_ctor_set(x_114, 4, x_110); +lean_ctor_set(x_114, 5, x_111); +x_115 = lean_st_ref_set(x_4, x_114, x_105); lean_dec(x_4); -x_113 = lean_ctor_get(x_112, 1); -lean_inc(x_113); -if (lean_is_exclusive(x_112)) { - lean_ctor_release(x_112, 0); - lean_ctor_release(x_112, 1); - x_114 = x_112; +x_116 = lean_ctor_get(x_115, 1); +lean_inc(x_116); +if (lean_is_exclusive(x_115)) { + lean_ctor_release(x_115, 0); + lean_ctor_release(x_115, 1); + x_117 = x_115; } else { - lean_dec_ref(x_112); - x_114 = lean_box(0); + lean_dec_ref(x_115); + x_117 = lean_box(0); } -x_115 = l_List_lengthTRAux___rarg(x_97, x_21); -lean_dec(x_97); -x_116 = lean_nat_dec_eq(x_22, x_115); -lean_dec(x_115); +x_118 = l_List_lengthTRAux___rarg(x_99, x_21); +lean_dec(x_99); +x_119 = lean_nat_dec_eq(x_22, x_118); +lean_dec(x_118); lean_dec(x_22); -if (x_116 == 0) -{ -uint8_t x_117; lean_object* x_118; lean_object* x_119; -x_117 = 1; -x_118 = lean_box(x_117); -if (lean_is_scalar(x_114)) { - x_119 = lean_alloc_ctor(0, 2, 0); -} else { - x_119 = x_114; -} -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_113); -return x_119; -} -else +if (x_119 == 0) { uint8_t x_120; lean_object* x_121; lean_object* x_122; -x_120 = 0; +x_120 = 1; x_121 = lean_box(x_120); -if (lean_is_scalar(x_114)) { +if (lean_is_scalar(x_117)) { x_122 = lean_alloc_ctor(0, 2, 0); } else { - x_122 = x_114; + x_122 = x_117; } lean_ctor_set(x_122, 0, x_121); -lean_ctor_set(x_122, 1, x_113); +lean_ctor_set(x_122, 1, x_116); return x_122; } +else +{ +uint8_t x_123; lean_object* x_124; lean_object* x_125; +x_123 = 0; +x_124 = lean_box(x_123); +if (lean_is_scalar(x_117)) { + x_125 = lean_alloc_ctor(0, 2, 0); +} else { + x_125 = x_117; +} +lean_ctor_set(x_125, 0, x_124); +lean_ctor_set(x_125, 1, x_116); +return x_125; +} } else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_dec(x_22); lean_dec(x_8); lean_dec(x_4); -x_123 = lean_ctor_get(x_96, 0); -lean_inc(x_123); -x_124 = lean_ctor_get(x_96, 1); -lean_inc(x_124); -if (lean_is_exclusive(x_96)) { - lean_ctor_release(x_96, 0); - lean_ctor_release(x_96, 1); - x_125 = x_96; +x_126 = lean_ctor_get(x_98, 0); +lean_inc(x_126); +x_127 = lean_ctor_get(x_98, 1); +lean_inc(x_127); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_128 = x_98; } else { - lean_dec_ref(x_96); - x_125 = lean_box(0); + lean_dec_ref(x_98); + x_128 = lean_box(0); } -if (lean_is_scalar(x_125)) { - x_126 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_128)) { + x_129 = lean_alloc_ctor(1, 2, 0); } else { - x_126 = x_125; + x_129 = x_128; } -lean_ctor_set(x_126, 0, x_123); -lean_ctor_set(x_126, 1, x_124); -return x_126; +lean_ctor_set(x_129, 0, x_126); +lean_ctor_set(x_129, 1, x_127); +return x_129; } } } @@ -15727,216 +15687,241 @@ return x_3; LEAN_EXPORT lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); -x_12 = lean_ctor_get(x_1, 2); +lean_object* x_11; lean_object* x_12; +x_11 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = !lean_is_exclusive(x_8); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); if (x_13 == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_8, 5); -x_15 = l_Lean_replaceRef(x_11, x_14); +lean_object* x_14; uint8_t x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_11, 0); lean_dec(x_14); -lean_ctor_set(x_8, 5, x_15); -switch (lean_obj_tag(x_12)) { -case 0: +x_15 = 1; +x_16 = lean_box(x_15); +lean_ctor_set(x_11, 0, x_16); +return x_11; +} +else { -lean_object* x_16; lean_object* x_17; +lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_11, 1); +lean_inc(x_17); lean_dec(x_11); -x_16 = lean_ctor_get(x_1, 0); -lean_inc(x_16); -lean_dec(x_1); -x_17 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_17; +x_18 = 1; +x_19 = lean_box(x_18); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_17); +return x_20; } -case 1: +} +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_dec(x_11); -x_18 = lean_ctor_get(x_12, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_12, 1); -lean_inc(x_19); -x_20 = lean_ctor_get(x_12, 2); -lean_inc(x_20); -x_21 = lean_ctor_get(x_12, 3); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_21 = lean_ctor_get(x_11, 1); lean_inc(x_21); -x_22 = lean_ctor_get(x_12, 4); +lean_dec(x_11); +x_22 = lean_ctor_get(x_12, 0); lean_inc(x_22); -x_23 = lean_ctor_get(x_12, 5); -lean_inc(x_23); lean_dec(x_12); -x_24 = lean_ctor_get(x_1, 0); +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_1); -x_25 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar(x_24, x_18, x_19, x_20, x_21, x_22, x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_25; -} -case 2: +lean_dec(x_22); +x_25 = !lean_is_exclusive(x_8); +if (x_25 == 0) { -lean_dec(x_11); -if (x_3 == 0) +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_8, 5); +x_27 = l_Lean_replaceRef(x_23, x_26); +lean_dec(x_26); +lean_ctor_set(x_8, 5, x_27); +switch (lean_obj_tag(x_24)) { +case 0: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -lean_dec(x_1); -x_26 = lean_ctor_get(x_12, 1); -lean_inc(x_26); -lean_dec(x_12); -x_27 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___closed__1; -x_28 = l_Lean_Elab_Term_withSavedContext___rarg(x_26, x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_object* x_28; +lean_dec(x_23); +x_28 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_21); return x_28; } -else +case 1: { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_12, 0); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_dec(x_23); +x_29 = lean_ctor_get(x_24, 0); lean_inc(x_29); -x_30 = lean_ctor_get(x_12, 1); +x_30 = lean_ctor_get(x_24, 1); lean_inc(x_30); -lean_dec(x_12); -x_31 = lean_ctor_get(x_1, 0); +x_31 = lean_ctor_get(x_24, 2); lean_inc(x_31); +x_32 = lean_ctor_get(x_24, 3); +lean_inc(x_32); +x_33 = lean_ctor_get(x_24, 4); +lean_inc(x_33); +x_34 = lean_ctor_get(x_24, 5); +lean_inc(x_34); +lean_dec(x_24); +x_35 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar(x_1, x_29, x_30, x_31, x_32, x_33, x_34, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +return x_35; +} +case 2: +{ +lean_dec(x_23); +if (x_3 == 0) +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_dec(x_1); -x_32 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___lambda__1), 9, 2); -lean_closure_set(x_32, 0, x_31); -lean_closure_set(x_32, 1, x_29); -x_33 = l_Lean_Elab_Term_withSavedContext___rarg(x_30, x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_33; +x_36 = lean_ctor_get(x_24, 1); +lean_inc(x_36); +lean_dec(x_24); +x_37 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___closed__1; +x_38 = l_Lean_Elab_Term_withSavedContext___rarg(x_36, x_37, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +return x_38; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_24, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_24, 1); +lean_inc(x_40); +lean_dec(x_24); +x_41 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___lambda__1), 9, 2); +lean_closure_set(x_41, 0, x_1); +lean_closure_set(x_41, 1, x_39); +x_42 = l_Lean_Elab_Term_withSavedContext___rarg(x_40, x_41, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +return x_42; } } default: { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_12, 0); -lean_inc(x_34); -lean_dec(x_12); -x_35 = lean_ctor_get(x_1, 0); -lean_inc(x_35); -lean_dec(x_1); -x_36 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed(x_34, x_11, x_35, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_36; +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_24, 0); +lean_inc(x_43); +lean_dec(x_24); +x_44 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed(x_43, x_23, x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +return x_44; } } } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_37 = lean_ctor_get(x_8, 0); -x_38 = lean_ctor_get(x_8, 1); -x_39 = lean_ctor_get(x_8, 2); -x_40 = lean_ctor_get(x_8, 3); -x_41 = lean_ctor_get(x_8, 4); -x_42 = lean_ctor_get(x_8, 5); -x_43 = lean_ctor_get(x_8, 6); -x_44 = lean_ctor_get(x_8, 7); -x_45 = lean_ctor_get(x_8, 8); -x_46 = lean_ctor_get(x_8, 9); -x_47 = lean_ctor_get(x_8, 10); +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_45 = lean_ctor_get(x_8, 0); +x_46 = lean_ctor_get(x_8, 1); +x_47 = lean_ctor_get(x_8, 2); +x_48 = lean_ctor_get(x_8, 3); +x_49 = lean_ctor_get(x_8, 4); +x_50 = lean_ctor_get(x_8, 5); +x_51 = lean_ctor_get(x_8, 6); +x_52 = lean_ctor_get(x_8, 7); +x_53 = lean_ctor_get(x_8, 8); +x_54 = lean_ctor_get(x_8, 9); +x_55 = lean_ctor_get(x_8, 10); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); -lean_inc(x_44); -lean_inc(x_43); -lean_inc(x_42); -lean_inc(x_41); -lean_inc(x_40); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); lean_dec(x_8); -x_48 = l_Lean_replaceRef(x_11, x_42); -lean_dec(x_42); -x_49 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_49, 0, x_37); -lean_ctor_set(x_49, 1, x_38); -lean_ctor_set(x_49, 2, x_39); -lean_ctor_set(x_49, 3, x_40); -lean_ctor_set(x_49, 4, x_41); -lean_ctor_set(x_49, 5, x_48); -lean_ctor_set(x_49, 6, x_43); -lean_ctor_set(x_49, 7, x_44); -lean_ctor_set(x_49, 8, x_45); -lean_ctor_set(x_49, 9, x_46); -lean_ctor_set(x_49, 10, x_47); -switch (lean_obj_tag(x_12)) { +x_56 = l_Lean_replaceRef(x_23, x_50); +lean_dec(x_50); +x_57 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_57, 0, x_45); +lean_ctor_set(x_57, 1, x_46); +lean_ctor_set(x_57, 2, x_47); +lean_ctor_set(x_57, 3, x_48); +lean_ctor_set(x_57, 4, x_49); +lean_ctor_set(x_57, 5, x_56); +lean_ctor_set(x_57, 6, x_51); +lean_ctor_set(x_57, 7, x_52); +lean_ctor_set(x_57, 8, x_53); +lean_ctor_set(x_57, 9, x_54); +lean_ctor_set(x_57, 10, x_55); +switch (lean_obj_tag(x_24)) { case 0: { -lean_object* x_50; lean_object* x_51; -lean_dec(x_11); -x_50 = lean_ctor_get(x_1, 0); -lean_inc(x_50); -lean_dec(x_1); -x_51 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar(x_50, x_4, x_5, x_6, x_7, x_49, x_9, x_10); -return x_51; -} -case 1: -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -lean_dec(x_11); -x_52 = lean_ctor_get(x_12, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_12, 1); -lean_inc(x_53); -x_54 = lean_ctor_get(x_12, 2); -lean_inc(x_54); -x_55 = lean_ctor_get(x_12, 3); -lean_inc(x_55); -x_56 = lean_ctor_get(x_12, 4); -lean_inc(x_56); -x_57 = lean_ctor_get(x_12, 5); -lean_inc(x_57); -lean_dec(x_12); -x_58 = lean_ctor_get(x_1, 0); -lean_inc(x_58); -lean_dec(x_1); -x_59 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar(x_58, x_52, x_53, x_54, x_55, x_56, x_57, x_4, x_5, x_6, x_7, x_49, x_9, x_10); -return x_59; +lean_object* x_58; +lean_dec(x_23); +x_58 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingInstMVar(x_1, x_4, x_5, x_6, x_7, x_57, x_9, x_21); +return x_58; +} +case 1: +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_23); +x_59 = lean_ctor_get(x_24, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_24, 1); +lean_inc(x_60); +x_61 = lean_ctor_get(x_24, 2); +lean_inc(x_61); +x_62 = lean_ctor_get(x_24, 3); +lean_inc(x_62); +x_63 = lean_ctor_get(x_24, 4); +lean_inc(x_63); +x_64 = lean_ctor_get(x_24, 5); +lean_inc(x_64); +lean_dec(x_24); +x_65 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizePendingCoeInstMVar(x_1, x_59, x_60, x_61, x_62, x_63, x_64, x_4, x_5, x_6, x_7, x_57, x_9, x_21); +return x_65; } case 2: { -lean_dec(x_11); +lean_dec(x_23); if (x_3 == 0) { -lean_object* x_60; lean_object* x_61; lean_object* x_62; +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_dec(x_1); -x_60 = lean_ctor_get(x_12, 1); -lean_inc(x_60); -lean_dec(x_12); -x_61 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___closed__1; -x_62 = l_Lean_Elab_Term_withSavedContext___rarg(x_60, x_61, x_4, x_5, x_6, x_7, x_49, x_9, x_10); -return x_62; +x_66 = lean_ctor_get(x_24, 1); +lean_inc(x_66); +lean_dec(x_24); +x_67 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___closed__1; +x_68 = l_Lean_Elab_Term_withSavedContext___rarg(x_66, x_67, x_4, x_5, x_6, x_7, x_57, x_9, x_21); +return x_68; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_63 = lean_ctor_get(x_12, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_12, 1); -lean_inc(x_64); -lean_dec(x_12); -x_65 = lean_ctor_get(x_1, 0); -lean_inc(x_65); -lean_dec(x_1); -x_66 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___lambda__1), 9, 2); -lean_closure_set(x_66, 0, x_65); -lean_closure_set(x_66, 1, x_63); -x_67 = l_Lean_Elab_Term_withSavedContext___rarg(x_64, x_66, x_4, x_5, x_6, x_7, x_49, x_9, x_10); -return x_67; +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_69 = lean_ctor_get(x_24, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_24, 1); +lean_inc(x_70); +lean_dec(x_24); +x_71 = lean_alloc_closure((void*)(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVar___lambda__1), 9, 2); +lean_closure_set(x_71, 0, x_1); +lean_closure_set(x_71, 1, x_69); +x_72 = l_Lean_Elab_Term_withSavedContext___rarg(x_70, x_71, x_4, x_5, x_6, x_7, x_57, x_9, x_21); +return x_72; } } default: { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_12, 0); -lean_inc(x_68); -lean_dec(x_12); -x_69 = lean_ctor_get(x_1, 0); -lean_inc(x_69); -lean_dec(x_1); -x_70 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed(x_68, x_11, x_69, x_2, x_4, x_5, x_6, x_7, x_49, x_9, x_10); -return x_70; +lean_object* x_73; lean_object* x_74; +x_73 = lean_ctor_get(x_24, 0); +lean_inc(x_73); +lean_dec(x_24); +x_74 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_resumePostponed(x_73, x_23, x_1, x_2, x_4, x_5, x_6, x_7, x_57, x_9, x_21); +return x_74; +} } } } @@ -17291,7 +17276,7 @@ lean_dec(x_12); x_14 = lean_st_ref_get(x_6, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 4); +x_16 = lean_ctor_get(x_15, 5); lean_inc(x_16); lean_dec(x_15); x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); @@ -17345,7 +17330,7 @@ lean_inc(x_30); x_31 = lean_ctor_get(x_29, 1); lean_inc(x_31); lean_dec(x_29); -x_32 = lean_ctor_get(x_30, 4); +x_32 = lean_ctor_get(x_30, 5); lean_inc(x_32); lean_dec(x_30); x_33 = lean_ctor_get(x_32, 1); @@ -17370,7 +17355,7 @@ lean_dec(x_37); x_39 = lean_st_ref_take(x_6, x_38); x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 4); +x_41 = lean_ctor_get(x_40, 5); lean_inc(x_41); x_42 = lean_ctor_get(x_39, 1); lean_inc(x_42); @@ -17379,7 +17364,7 @@ x_43 = !lean_is_exclusive(x_40); if (x_43 == 0) { lean_object* x_44; uint8_t x_45; -x_44 = lean_ctor_get(x_40, 4); +x_44 = lean_ctor_get(x_40, 5); lean_dec(x_44); x_45 = !lean_is_exclusive(x_41); if (x_45 == 0) @@ -17424,7 +17409,7 @@ x_56 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_56, 0, x_54); lean_ctor_set(x_56, 1, x_55); lean_ctor_set_uint8(x_56, sizeof(void*)*2, x_53); -lean_ctor_set(x_40, 4, x_56); +lean_ctor_set(x_40, 5, x_56); x_57 = lean_st_ref_set(x_6, x_40, x_42); lean_dec(x_6); x_58 = lean_ctor_get(x_57, 1); @@ -17449,298 +17434,304 @@ return x_60; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; x_61 = lean_ctor_get(x_40, 0); x_62 = lean_ctor_get(x_40, 1); x_63 = lean_ctor_get(x_40, 2); x_64 = lean_ctor_get(x_40, 3); +x_65 = lean_ctor_get(x_40, 4); +lean_inc(x_65); lean_inc(x_64); lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_dec(x_40); -x_65 = lean_ctor_get_uint8(x_41, sizeof(void*)*2); -x_66 = lean_ctor_get(x_41, 0); -lean_inc(x_66); +x_66 = lean_ctor_get_uint8(x_41, sizeof(void*)*2); +x_67 = lean_ctor_get(x_41, 0); +lean_inc(x_67); if (lean_is_exclusive(x_41)) { lean_ctor_release(x_41, 0); lean_ctor_release(x_41, 1); - x_67 = x_41; + x_68 = x_41; } else { lean_dec_ref(x_41); - x_67 = lean_box(0); + x_68 = lean_box(0); } -x_68 = l_Std_PersistentArray_push___rarg(x_22, x_35); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 1); +x_69 = l_Std_PersistentArray_push___rarg(x_22, x_35); +if (lean_is_scalar(x_68)) { + x_70 = lean_alloc_ctor(0, 2, 1); } else { - x_69 = x_67; + x_70 = x_68; } -lean_ctor_set(x_69, 0, x_66); -lean_ctor_set(x_69, 1, x_68); -lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_65); -x_70 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_70, 0, x_61); -lean_ctor_set(x_70, 1, x_62); -lean_ctor_set(x_70, 2, x_63); -lean_ctor_set(x_70, 3, x_64); -lean_ctor_set(x_70, 4, x_69); -x_71 = lean_st_ref_set(x_6, x_70, x_42); +lean_ctor_set(x_70, 0, x_67); +lean_ctor_set(x_70, 1, x_69); +lean_ctor_set_uint8(x_70, sizeof(void*)*2, x_66); +x_71 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_71, 0, x_61); +lean_ctor_set(x_71, 1, x_62); +lean_ctor_set(x_71, 2, x_63); +lean_ctor_set(x_71, 3, x_64); +lean_ctor_set(x_71, 4, x_65); +lean_ctor_set(x_71, 5, x_70); +x_72 = lean_st_ref_set(x_6, x_71, x_42); lean_dec(x_6); -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_73 = x_71; +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_74 = x_72; } else { - lean_dec_ref(x_71); - x_73 = lean_box(0); + lean_dec_ref(x_72); + x_74 = lean_box(0); } -if (lean_is_scalar(x_73)) { - x_74 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(0, 2, 0); } else { - x_74 = x_73; + x_75 = x_74; } -lean_ctor_set(x_74, 0, x_25); -lean_ctor_set(x_74, 1, x_72); -return x_74; +lean_ctor_set(x_75, 0, x_25); +lean_ctor_set(x_75, 1, x_73); +return x_75; } } else { -uint8_t x_75; +uint8_t x_76; lean_dec(x_25); lean_dec(x_22); lean_dec(x_10); lean_dec(x_6); -x_75 = !lean_is_exclusive(x_34); -if (x_75 == 0) +x_76 = !lean_is_exclusive(x_34); +if (x_76 == 0) { return x_34; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_34, 0); -x_77 = lean_ctor_get(x_34, 1); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_34, 0); +x_78 = lean_ctor_get(x_34, 1); +lean_inc(x_78); lean_inc(x_77); -lean_inc(x_76); lean_dec(x_34); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_79 = lean_ctor_get(x_24, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_24, 1); +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_80 = lean_ctor_get(x_24, 0); lean_inc(x_80); +x_81 = lean_ctor_get(x_24, 1); +lean_inc(x_81); lean_dec(x_24); -x_81 = lean_st_ref_get(x_10, x_80); -x_82 = lean_ctor_get(x_81, 1); -lean_inc(x_82); -lean_dec(x_81); -x_83 = lean_st_ref_get(x_6, x_82); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +x_82 = lean_st_ref_get(x_10, x_81); +x_83 = lean_ctor_get(x_82, 1); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_st_ref_get(x_6, x_83); +x_85 = lean_ctor_get(x_84, 0); lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_ctor_get(x_84, 4); +x_86 = lean_ctor_get(x_84, 1); lean_inc(x_86); lean_dec(x_84); -x_87 = lean_ctor_get(x_86, 1); +x_87 = lean_ctor_get(x_85, 5); lean_inc(x_87); -lean_dec(x_86); +lean_dec(x_85); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); lean_inc(x_10); lean_inc(x_6); -x_88 = lean_apply_10(x_2, x_87, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_85); -if (lean_obj_tag(x_88) == 0) +x_89 = lean_apply_10(x_2, x_88, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_86); +if (lean_obj_tag(x_89) == 0) { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_88, 1); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_90 = lean_ctor_get(x_89, 0); lean_inc(x_90); -lean_dec(x_88); -x_91 = lean_st_ref_get(x_10, x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = lean_st_ref_get(x_10, x_91); lean_dec(x_10); -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); -lean_dec(x_91); -x_93 = lean_st_ref_take(x_6, x_92); -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_94, 4); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +x_94 = lean_st_ref_take(x_6, x_93); +x_95 = lean_ctor_get(x_94, 0); lean_inc(x_95); -x_96 = lean_ctor_get(x_93, 1); +x_96 = lean_ctor_get(x_95, 5); lean_inc(x_96); -lean_dec(x_93); -x_97 = !lean_is_exclusive(x_94); -if (x_97 == 0) +x_97 = lean_ctor_get(x_94, 1); +lean_inc(x_97); +lean_dec(x_94); +x_98 = !lean_is_exclusive(x_95); +if (x_98 == 0) { -lean_object* x_98; uint8_t x_99; -x_98 = lean_ctor_get(x_94, 4); -lean_dec(x_98); -x_99 = !lean_is_exclusive(x_95); -if (x_99 == 0) +lean_object* x_99; uint8_t x_100; +x_99 = lean_ctor_get(x_95, 5); +lean_dec(x_99); +x_100 = !lean_is_exclusive(x_96); +if (x_100 == 0) { -lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; -x_100 = lean_ctor_get(x_95, 1); -lean_dec(x_100); -x_101 = l_Std_PersistentArray_push___rarg(x_22, x_89); -lean_ctor_set(x_95, 1, x_101); -x_102 = lean_st_ref_set(x_6, x_94, x_96); +lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; +x_101 = lean_ctor_get(x_96, 1); +lean_dec(x_101); +x_102 = l_Std_PersistentArray_push___rarg(x_22, x_90); +lean_ctor_set(x_96, 1, x_102); +x_103 = lean_st_ref_set(x_6, x_95, x_97); lean_dec(x_6); -x_103 = !lean_is_exclusive(x_102); -if (x_103 == 0) +x_104 = !lean_is_exclusive(x_103); +if (x_104 == 0) { -lean_object* x_104; -x_104 = lean_ctor_get(x_102, 0); -lean_dec(x_104); -lean_ctor_set_tag(x_102, 1); -lean_ctor_set(x_102, 0, x_79); -return x_102; +lean_object* x_105; +x_105 = lean_ctor_get(x_103, 0); +lean_dec(x_105); +lean_ctor_set_tag(x_103, 1); +lean_ctor_set(x_103, 0, x_80); +return x_103; } else { -lean_object* x_105; lean_object* x_106; -x_105 = lean_ctor_get(x_102, 1); -lean_inc(x_105); -lean_dec(x_102); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_79); -lean_ctor_set(x_106, 1, x_105); -return x_106; +lean_object* x_106; lean_object* x_107; +x_106 = lean_ctor_get(x_103, 1); +lean_inc(x_106); +lean_dec(x_103); +x_107 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_107, 0, x_80); +lean_ctor_set(x_107, 1, x_106); +return x_107; } } else { -uint8_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_107 = lean_ctor_get_uint8(x_95, sizeof(void*)*2); -x_108 = lean_ctor_get(x_95, 0); -lean_inc(x_108); -lean_dec(x_95); -x_109 = l_Std_PersistentArray_push___rarg(x_22, x_89); -x_110 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -lean_ctor_set_uint8(x_110, sizeof(void*)*2, x_107); -lean_ctor_set(x_94, 4, x_110); -x_111 = lean_st_ref_set(x_6, x_94, x_96); +uint8_t x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_108 = lean_ctor_get_uint8(x_96, sizeof(void*)*2); +x_109 = lean_ctor_get(x_96, 0); +lean_inc(x_109); +lean_dec(x_96); +x_110 = l_Std_PersistentArray_push___rarg(x_22, x_90); +x_111 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +lean_ctor_set_uint8(x_111, sizeof(void*)*2, x_108); +lean_ctor_set(x_95, 5, x_111); +x_112 = lean_st_ref_set(x_6, x_95, x_97); lean_dec(x_6); -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_113 = x_111; +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_114 = x_112; } else { - lean_dec_ref(x_111); - x_113 = lean_box(0); + lean_dec_ref(x_112); + x_114 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; - lean_ctor_set_tag(x_114, 1); + x_115 = x_114; + lean_ctor_set_tag(x_115, 1); } -lean_ctor_set(x_114, 0, x_79); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_115, 0, x_80); +lean_ctor_set(x_115, 1, x_113); +return x_115; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_115 = lean_ctor_get(x_94, 0); -x_116 = lean_ctor_get(x_94, 1); -x_117 = lean_ctor_get(x_94, 2); -x_118 = lean_ctor_get(x_94, 3); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; uint8_t x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_116 = lean_ctor_get(x_95, 0); +x_117 = lean_ctor_get(x_95, 1); +x_118 = lean_ctor_get(x_95, 2); +x_119 = lean_ctor_get(x_95, 3); +x_120 = lean_ctor_get(x_95, 4); +lean_inc(x_120); +lean_inc(x_119); lean_inc(x_118); lean_inc(x_117); lean_inc(x_116); -lean_inc(x_115); -lean_dec(x_94); -x_119 = lean_ctor_get_uint8(x_95, sizeof(void*)*2); -x_120 = lean_ctor_get(x_95, 0); -lean_inc(x_120); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_121 = x_95; +lean_dec(x_95); +x_121 = lean_ctor_get_uint8(x_96, sizeof(void*)*2); +x_122 = lean_ctor_get(x_96, 0); +lean_inc(x_122); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_123 = x_96; } else { - lean_dec_ref(x_95); - x_121 = lean_box(0); + lean_dec_ref(x_96); + x_123 = lean_box(0); } -x_122 = l_Std_PersistentArray_push___rarg(x_22, x_89); -if (lean_is_scalar(x_121)) { - x_123 = lean_alloc_ctor(0, 2, 1); +x_124 = l_Std_PersistentArray_push___rarg(x_22, x_90); +if (lean_is_scalar(x_123)) { + x_125 = lean_alloc_ctor(0, 2, 1); } else { - x_123 = x_121; -} -lean_ctor_set(x_123, 0, x_120); -lean_ctor_set(x_123, 1, x_122); -lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_119); -x_124 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_124, 0, x_115); -lean_ctor_set(x_124, 1, x_116); -lean_ctor_set(x_124, 2, x_117); -lean_ctor_set(x_124, 3, x_118); -lean_ctor_set(x_124, 4, x_123); -x_125 = lean_st_ref_set(x_6, x_124, x_96); + x_125 = x_123; +} +lean_ctor_set(x_125, 0, x_122); +lean_ctor_set(x_125, 1, x_124); +lean_ctor_set_uint8(x_125, sizeof(void*)*2, x_121); +x_126 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_126, 0, x_116); +lean_ctor_set(x_126, 1, x_117); +lean_ctor_set(x_126, 2, x_118); +lean_ctor_set(x_126, 3, x_119); +lean_ctor_set(x_126, 4, x_120); +lean_ctor_set(x_126, 5, x_125); +x_127 = lean_st_ref_set(x_6, x_126, x_97); lean_dec(x_6); -x_126 = lean_ctor_get(x_125, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - x_127 = x_125; +x_128 = lean_ctor_get(x_127, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_129 = x_127; } else { - lean_dec_ref(x_125); - x_127 = lean_box(0); + lean_dec_ref(x_127); + x_129 = lean_box(0); } -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(1, 2, 0); } else { - x_128 = x_127; - lean_ctor_set_tag(x_128, 1); + x_130 = x_129; + lean_ctor_set_tag(x_130, 1); } -lean_ctor_set(x_128, 0, x_79); -lean_ctor_set(x_128, 1, x_126); -return x_128; +lean_ctor_set(x_130, 0, x_80); +lean_ctor_set(x_130, 1, x_128); +return x_130; } } else { -uint8_t x_129; -lean_dec(x_79); +uint8_t x_131; +lean_dec(x_80); lean_dec(x_22); lean_dec(x_10); lean_dec(x_6); -x_129 = !lean_is_exclusive(x_88); -if (x_129 == 0) +x_131 = !lean_is_exclusive(x_89); +if (x_131 == 0) { -return x_88; +return x_89; } else { -lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_130 = lean_ctor_get(x_88, 0); -x_131 = lean_ctor_get(x_88, 1); -lean_inc(x_131); -lean_inc(x_130); -lean_dec(x_88); -x_132 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); -return x_132; +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_89, 0); +x_133 = lean_ctor_get(x_89, 1); +lean_inc(x_133); +lean_inc(x_132); +lean_dec(x_89); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; } } } @@ -17896,7 +17887,7 @@ lean_dec(x_47); x_49 = lean_st_ref_get(x_4, x_48); x_50 = lean_ctor_get(x_49, 0); lean_inc(x_50); -x_51 = lean_ctor_get(x_50, 4); +x_51 = lean_ctor_get(x_50, 5); lean_inc(x_51); lean_dec(x_50); x_52 = lean_ctor_get_uint8(x_51, sizeof(void*)*2); @@ -17952,7 +17943,7 @@ lean_dec(x_62); x_64 = lean_st_ref_take(x_4, x_63); x_65 = lean_ctor_get(x_64, 0); lean_inc(x_65); -x_66 = lean_ctor_get(x_65, 4); +x_66 = lean_ctor_get(x_65, 5); lean_inc(x_66); x_67 = lean_ctor_get(x_64, 1); lean_inc(x_67); @@ -17961,7 +17952,7 @@ x_68 = !lean_is_exclusive(x_65); if (x_68 == 0) { lean_object* x_69; uint8_t x_70; -x_69 = lean_ctor_get(x_65, 4); +x_69 = lean_ctor_get(x_65, 5); lean_dec(x_69); x_70 = !lean_is_exclusive(x_66); if (x_70 == 0) @@ -18079,7 +18070,7 @@ x_104 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_104, 0, x_99); lean_ctor_set(x_104, 1, x_57); lean_ctor_set_uint8(x_104, sizeof(void*)*2, x_98); -lean_ctor_set(x_65, 4, x_104); +lean_ctor_set(x_65, 5, x_104); x_105 = lean_st_ref_set(x_4, x_65, x_67); x_106 = lean_ctor_get(x_105, 1); lean_inc(x_106); @@ -18118,7 +18109,7 @@ x_115 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_115, 0, x_114); lean_ctor_set(x_115, 1, x_57); lean_ctor_set_uint8(x_115, sizeof(void*)*2, x_98); -lean_ctor_set(x_65, 4, x_115); +lean_ctor_set(x_65, 5, x_115); x_116 = lean_st_ref_set(x_4, x_65, x_67); x_117 = lean_ctor_get(x_116, 1); lean_inc(x_117); @@ -18148,431 +18139,439 @@ goto block_46; } else { -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; uint8_t x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; uint8_t x_132; +lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; uint8_t x_133; x_122 = lean_ctor_get(x_65, 0); x_123 = lean_ctor_get(x_65, 1); x_124 = lean_ctor_get(x_65, 2); x_125 = lean_ctor_get(x_65, 3); +x_126 = lean_ctor_get(x_65, 4); +lean_inc(x_126); lean_inc(x_125); lean_inc(x_124); lean_inc(x_123); lean_inc(x_122); lean_dec(x_65); -x_126 = lean_ctor_get_uint8(x_66, sizeof(void*)*2); -x_127 = lean_ctor_get(x_66, 0); -lean_inc(x_127); -x_128 = lean_ctor_get(x_66, 1); +x_127 = lean_ctor_get_uint8(x_66, sizeof(void*)*2); +x_128 = lean_ctor_get(x_66, 0); lean_inc(x_128); +x_129 = lean_ctor_get(x_66, 1); +lean_inc(x_129); if (lean_is_exclusive(x_66)) { lean_ctor_release(x_66, 0); lean_ctor_release(x_66, 1); - x_129 = x_66; + x_130 = x_66; } else { lean_dec_ref(x_66); - x_129 = lean_box(0); + x_130 = lean_box(0); } -x_130 = lean_ctor_get(x_128, 2); -lean_inc(x_130); -x_131 = lean_unsigned_to_nat(0u); -x_132 = lean_nat_dec_lt(x_131, x_130); -if (x_132 == 0) +x_131 = lean_ctor_get(x_129, 2); +lean_inc(x_131); +x_132 = lean_unsigned_to_nat(0u); +x_133 = lean_nat_dec_lt(x_132, x_131); +if (x_133 == 0) { -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -lean_dec(x_130); -lean_dec(x_128); +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_dec(x_131); +lean_dec(x_129); lean_dec(x_1); -if (lean_is_scalar(x_129)) { - x_133 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_130)) { + x_134 = lean_alloc_ctor(0, 2, 1); } else { - x_133 = x_129; -} -lean_ctor_set(x_133, 0, x_127); -lean_ctor_set(x_133, 1, x_57); -lean_ctor_set_uint8(x_133, sizeof(void*)*2, x_126); -x_134 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_134, 0, x_122); -lean_ctor_set(x_134, 1, x_123); -lean_ctor_set(x_134, 2, x_124); -lean_ctor_set(x_134, 3, x_125); -lean_ctor_set(x_134, 4, x_133); -x_135 = lean_st_ref_set(x_4, x_134, x_67); -x_136 = lean_ctor_get(x_135, 1); -lean_inc(x_136); -if (lean_is_exclusive(x_135)) { - lean_ctor_release(x_135, 0); - lean_ctor_release(x_135, 1); - x_137 = x_135; + x_134 = x_130; +} +lean_ctor_set(x_134, 0, x_128); +lean_ctor_set(x_134, 1, x_57); +lean_ctor_set_uint8(x_134, sizeof(void*)*2, x_127); +x_135 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_135, 0, x_122); +lean_ctor_set(x_135, 1, x_123); +lean_ctor_set(x_135, 2, x_124); +lean_ctor_set(x_135, 3, x_125); +lean_ctor_set(x_135, 4, x_126); +lean_ctor_set(x_135, 5, x_134); +x_136 = lean_st_ref_set(x_4, x_135, x_67); +x_137 = lean_ctor_get(x_136, 1); +lean_inc(x_137); +if (lean_is_exclusive(x_136)) { + lean_ctor_release(x_136, 0); + lean_ctor_release(x_136, 1); + x_138 = x_136; } else { - lean_dec_ref(x_135); - x_137 = lean_box(0); -} -x_138 = lean_box(0); -x_139 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_139, 0, x_60); -lean_ctor_set(x_139, 1, x_138); -if (lean_is_scalar(x_137)) { - x_140 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_136); + x_138 = lean_box(0); +} +x_139 = lean_box(0); +x_140 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_140, 0, x_60); +lean_ctor_set(x_140, 1, x_139); +if (lean_is_scalar(x_138)) { + x_141 = lean_alloc_ctor(0, 2, 0); } else { - x_140 = x_137; + x_141 = x_138; } -lean_ctor_set(x_140, 0, x_139); -lean_ctor_set(x_140, 1, x_136); -x_34 = x_140; +lean_ctor_set(x_141, 0, x_140); +lean_ctor_set(x_141, 1, x_137); +x_34 = x_141; goto block_46; } else { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_141 = lean_nat_sub(x_130, x_10); -lean_dec(x_130); -x_142 = l_Lean_Elab_instInhabitedInfoTree; -x_143 = l_Std_PersistentArray_get_x21___rarg(x_142, x_128, x_141); -lean_dec(x_141); -x_144 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_127, x_1, x_143); -if (lean_is_scalar(x_129)) { - x_145 = lean_alloc_ctor(0, 2, 1); +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; +x_142 = lean_nat_sub(x_131, x_10); +lean_dec(x_131); +x_143 = l_Lean_Elab_instInhabitedInfoTree; +x_144 = l_Std_PersistentArray_get_x21___rarg(x_143, x_129, x_142); +lean_dec(x_142); +x_145 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_128, x_1, x_144); +if (lean_is_scalar(x_130)) { + x_146 = lean_alloc_ctor(0, 2, 1); } else { - x_145 = x_129; + x_146 = x_130; } -lean_ctor_set(x_145, 0, x_144); -lean_ctor_set(x_145, 1, x_57); -lean_ctor_set_uint8(x_145, sizeof(void*)*2, x_126); -x_146 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_146, 0, x_122); -lean_ctor_set(x_146, 1, x_123); -lean_ctor_set(x_146, 2, x_124); -lean_ctor_set(x_146, 3, x_125); -lean_ctor_set(x_146, 4, x_145); -x_147 = lean_st_ref_set(x_4, x_146, x_67); -x_148 = lean_ctor_get(x_147, 1); -lean_inc(x_148); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_149 = x_147; +lean_ctor_set(x_146, 0, x_145); +lean_ctor_set(x_146, 1, x_57); +lean_ctor_set_uint8(x_146, sizeof(void*)*2, x_127); +x_147 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_147, 0, x_122); +lean_ctor_set(x_147, 1, x_123); +lean_ctor_set(x_147, 2, x_124); +lean_ctor_set(x_147, 3, x_125); +lean_ctor_set(x_147, 4, x_126); +lean_ctor_set(x_147, 5, x_146); +x_148 = lean_st_ref_set(x_4, x_147, x_67); +x_149 = lean_ctor_get(x_148, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_148)) { + lean_ctor_release(x_148, 0); + lean_ctor_release(x_148, 1); + x_150 = x_148; } else { - lean_dec_ref(x_147); - x_149 = lean_box(0); -} -x_150 = lean_box(0); -x_151 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_151, 0, x_60); -lean_ctor_set(x_151, 1, x_150); -if (lean_is_scalar(x_149)) { - x_152 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_148); + x_150 = lean_box(0); +} +x_151 = lean_box(0); +x_152 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_152, 0, x_60); +lean_ctor_set(x_152, 1, x_151); +if (lean_is_scalar(x_150)) { + x_153 = lean_alloc_ctor(0, 2, 0); } else { - x_152 = x_149; + x_153 = x_150; } -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_148); -x_34 = x_152; +lean_ctor_set(x_153, 0, x_152); +lean_ctor_set(x_153, 1, x_149); +x_34 = x_153; goto block_46; } } } else { -lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; uint8_t x_161; -x_153 = lean_ctor_get(x_59, 0); -lean_inc(x_153); -x_154 = lean_ctor_get(x_59, 1); +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; uint8_t x_162; +x_154 = lean_ctor_get(x_59, 0); lean_inc(x_154); +x_155 = lean_ctor_get(x_59, 1); +lean_inc(x_155); lean_dec(x_59); -x_155 = lean_st_ref_get(x_8, x_154); -x_156 = lean_ctor_get(x_155, 1); -lean_inc(x_156); -lean_dec(x_155); -x_157 = lean_st_ref_take(x_4, x_156); -x_158 = lean_ctor_get(x_157, 0); -lean_inc(x_158); -x_159 = lean_ctor_get(x_158, 4); +x_156 = lean_st_ref_get(x_8, x_155); +x_157 = lean_ctor_get(x_156, 1); +lean_inc(x_157); +lean_dec(x_156); +x_158 = lean_st_ref_take(x_4, x_157); +x_159 = lean_ctor_get(x_158, 0); lean_inc(x_159); -x_160 = lean_ctor_get(x_157, 1); +x_160 = lean_ctor_get(x_159, 5); lean_inc(x_160); -lean_dec(x_157); -x_161 = !lean_is_exclusive(x_158); -if (x_161 == 0) -{ -lean_object* x_162; uint8_t x_163; -x_162 = lean_ctor_get(x_158, 4); -lean_dec(x_162); -x_163 = !lean_is_exclusive(x_159); -if (x_163 == 0) -{ -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; uint8_t x_168; -x_164 = lean_ctor_get(x_159, 0); -x_165 = lean_ctor_get(x_159, 1); -x_166 = lean_ctor_get(x_165, 2); -lean_inc(x_166); -x_167 = lean_unsigned_to_nat(0u); -x_168 = lean_nat_dec_lt(x_167, x_166); -if (x_168 == 0) +x_161 = lean_ctor_get(x_158, 1); +lean_inc(x_161); +lean_dec(x_158); +x_162 = !lean_is_exclusive(x_159); +if (x_162 == 0) +{ +lean_object* x_163; uint8_t x_164; +x_163 = lean_ctor_get(x_159, 5); +lean_dec(x_163); +x_164 = !lean_is_exclusive(x_160); +if (x_164 == 0) +{ +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_169; +x_165 = lean_ctor_get(x_160, 0); +x_166 = lean_ctor_get(x_160, 1); +x_167 = lean_ctor_get(x_166, 2); +lean_inc(x_167); +x_168 = lean_unsigned_to_nat(0u); +x_169 = lean_nat_dec_lt(x_168, x_167); +if (x_169 == 0) { -lean_object* x_169; uint8_t x_170; +lean_object* x_170; uint8_t x_171; +lean_dec(x_167); lean_dec(x_166); -lean_dec(x_165); lean_dec(x_1); -lean_ctor_set(x_159, 1, x_57); -x_169 = lean_st_ref_set(x_4, x_158, x_160); -x_170 = !lean_is_exclusive(x_169); -if (x_170 == 0) -{ -lean_object* x_171; -x_171 = lean_ctor_get(x_169, 0); -lean_dec(x_171); -lean_ctor_set_tag(x_169, 1); -lean_ctor_set(x_169, 0, x_153); -x_34 = x_169; +lean_ctor_set(x_160, 1, x_57); +x_170 = lean_st_ref_set(x_4, x_159, x_161); +x_171 = !lean_is_exclusive(x_170); +if (x_171 == 0) +{ +lean_object* x_172; +x_172 = lean_ctor_get(x_170, 0); +lean_dec(x_172); +lean_ctor_set_tag(x_170, 1); +lean_ctor_set(x_170, 0, x_154); +x_34 = x_170; goto block_46; } else { -lean_object* x_172; lean_object* x_173; -x_172 = lean_ctor_get(x_169, 1); -lean_inc(x_172); -lean_dec(x_169); -x_173 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_173, 0, x_153); -lean_ctor_set(x_173, 1, x_172); -x_34 = x_173; +lean_object* x_173; lean_object* x_174; +x_173 = lean_ctor_get(x_170, 1); +lean_inc(x_173); +lean_dec(x_170); +x_174 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_174, 0, x_154); +lean_ctor_set(x_174, 1, x_173); +x_34 = x_174; goto block_46; } } else { -lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; uint8_t x_179; -x_174 = lean_nat_sub(x_166, x_10); -lean_dec(x_166); -x_175 = l_Lean_Elab_instInhabitedInfoTree; -x_176 = l_Std_PersistentArray_get_x21___rarg(x_175, x_165, x_174); -lean_dec(x_174); -x_177 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_164, x_1, x_176); -lean_ctor_set(x_159, 1, x_57); -lean_ctor_set(x_159, 0, x_177); -x_178 = lean_st_ref_set(x_4, x_158, x_160); -x_179 = !lean_is_exclusive(x_178); -if (x_179 == 0) -{ -lean_object* x_180; -x_180 = lean_ctor_get(x_178, 0); -lean_dec(x_180); -lean_ctor_set_tag(x_178, 1); -lean_ctor_set(x_178, 0, x_153); -x_34 = x_178; +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; uint8_t x_180; +x_175 = lean_nat_sub(x_167, x_10); +lean_dec(x_167); +x_176 = l_Lean_Elab_instInhabitedInfoTree; +x_177 = l_Std_PersistentArray_get_x21___rarg(x_176, x_166, x_175); +lean_dec(x_175); +x_178 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_165, x_1, x_177); +lean_ctor_set(x_160, 1, x_57); +lean_ctor_set(x_160, 0, x_178); +x_179 = lean_st_ref_set(x_4, x_159, x_161); +x_180 = !lean_is_exclusive(x_179); +if (x_180 == 0) +{ +lean_object* x_181; +x_181 = lean_ctor_get(x_179, 0); +lean_dec(x_181); +lean_ctor_set_tag(x_179, 1); +lean_ctor_set(x_179, 0, x_154); +x_34 = x_179; goto block_46; } else { -lean_object* x_181; lean_object* x_182; -x_181 = lean_ctor_get(x_178, 1); -lean_inc(x_181); -lean_dec(x_178); -x_182 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_182, 0, x_153); -lean_ctor_set(x_182, 1, x_181); -x_34 = x_182; +lean_object* x_182; lean_object* x_183; +x_182 = lean_ctor_get(x_179, 1); +lean_inc(x_182); +lean_dec(x_179); +x_183 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_183, 0, x_154); +lean_ctor_set(x_183, 1, x_182); +x_34 = x_183; goto block_46; } } } else { -uint8_t x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; uint8_t x_188; -x_183 = lean_ctor_get_uint8(x_159, sizeof(void*)*2); -x_184 = lean_ctor_get(x_159, 0); -x_185 = lean_ctor_get(x_159, 1); -lean_inc(x_185); -lean_inc(x_184); -lean_dec(x_159); -x_186 = lean_ctor_get(x_185, 2); +uint8_t x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; uint8_t x_189; +x_184 = lean_ctor_get_uint8(x_160, sizeof(void*)*2); +x_185 = lean_ctor_get(x_160, 0); +x_186 = lean_ctor_get(x_160, 1); lean_inc(x_186); -x_187 = lean_unsigned_to_nat(0u); -x_188 = lean_nat_dec_lt(x_187, x_186); -if (x_188 == 0) +lean_inc(x_185); +lean_dec(x_160); +x_187 = lean_ctor_get(x_186, 2); +lean_inc(x_187); +x_188 = lean_unsigned_to_nat(0u); +x_189 = lean_nat_dec_lt(x_188, x_187); +if (x_189 == 0) { -lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; +lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; +lean_dec(x_187); lean_dec(x_186); -lean_dec(x_185); lean_dec(x_1); -x_189 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_189, 0, x_184); -lean_ctor_set(x_189, 1, x_57); -lean_ctor_set_uint8(x_189, sizeof(void*)*2, x_183); -lean_ctor_set(x_158, 4, x_189); -x_190 = lean_st_ref_set(x_4, x_158, x_160); -x_191 = lean_ctor_get(x_190, 1); -lean_inc(x_191); -if (lean_is_exclusive(x_190)) { - lean_ctor_release(x_190, 0); - lean_ctor_release(x_190, 1); - x_192 = x_190; +x_190 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_190, 0, x_185); +lean_ctor_set(x_190, 1, x_57); +lean_ctor_set_uint8(x_190, sizeof(void*)*2, x_184); +lean_ctor_set(x_159, 5, x_190); +x_191 = lean_st_ref_set(x_4, x_159, x_161); +x_192 = lean_ctor_get(x_191, 1); +lean_inc(x_192); +if (lean_is_exclusive(x_191)) { + lean_ctor_release(x_191, 0); + lean_ctor_release(x_191, 1); + x_193 = x_191; } else { - lean_dec_ref(x_190); - x_192 = lean_box(0); + lean_dec_ref(x_191); + x_193 = lean_box(0); } -if (lean_is_scalar(x_192)) { - x_193 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_193)) { + x_194 = lean_alloc_ctor(1, 2, 0); } else { - x_193 = x_192; - lean_ctor_set_tag(x_193, 1); + x_194 = x_193; + lean_ctor_set_tag(x_194, 1); } -lean_ctor_set(x_193, 0, x_153); -lean_ctor_set(x_193, 1, x_191); -x_34 = x_193; +lean_ctor_set(x_194, 0, x_154); +lean_ctor_set(x_194, 1, x_192); +x_34 = x_194; goto block_46; } else { -lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; -x_194 = lean_nat_sub(x_186, x_10); -lean_dec(x_186); -x_195 = l_Lean_Elab_instInhabitedInfoTree; -x_196 = l_Std_PersistentArray_get_x21___rarg(x_195, x_185, x_194); -lean_dec(x_194); -x_197 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_184, x_1, x_196); -x_198 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_198, 0, x_197); -lean_ctor_set(x_198, 1, x_57); -lean_ctor_set_uint8(x_198, sizeof(void*)*2, x_183); -lean_ctor_set(x_158, 4, x_198); -x_199 = lean_st_ref_set(x_4, x_158, x_160); -x_200 = lean_ctor_get(x_199, 1); -lean_inc(x_200); -if (lean_is_exclusive(x_199)) { - lean_ctor_release(x_199, 0); - lean_ctor_release(x_199, 1); - x_201 = x_199; +lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +x_195 = lean_nat_sub(x_187, x_10); +lean_dec(x_187); +x_196 = l_Lean_Elab_instInhabitedInfoTree; +x_197 = l_Std_PersistentArray_get_x21___rarg(x_196, x_186, x_195); +lean_dec(x_195); +x_198 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_185, x_1, x_197); +x_199 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_199, 0, x_198); +lean_ctor_set(x_199, 1, x_57); +lean_ctor_set_uint8(x_199, sizeof(void*)*2, x_184); +lean_ctor_set(x_159, 5, x_199); +x_200 = lean_st_ref_set(x_4, x_159, x_161); +x_201 = lean_ctor_get(x_200, 1); +lean_inc(x_201); +if (lean_is_exclusive(x_200)) { + lean_ctor_release(x_200, 0); + lean_ctor_release(x_200, 1); + x_202 = x_200; } else { - lean_dec_ref(x_199); - x_201 = lean_box(0); + lean_dec_ref(x_200); + x_202 = lean_box(0); } -if (lean_is_scalar(x_201)) { - x_202 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_202)) { + x_203 = lean_alloc_ctor(1, 2, 0); } else { - x_202 = x_201; - lean_ctor_set_tag(x_202, 1); + x_203 = x_202; + lean_ctor_set_tag(x_203, 1); } -lean_ctor_set(x_202, 0, x_153); -lean_ctor_set(x_202, 1, x_200); -x_34 = x_202; +lean_ctor_set(x_203, 0, x_154); +lean_ctor_set(x_203, 1, x_201); +x_34 = x_203; goto block_46; } } } else { -lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; uint8_t x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; uint8_t x_213; -x_203 = lean_ctor_get(x_158, 0); -x_204 = lean_ctor_get(x_158, 1); -x_205 = lean_ctor_get(x_158, 2); -x_206 = lean_ctor_get(x_158, 3); +lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; uint8_t x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; uint8_t x_215; +x_204 = lean_ctor_get(x_159, 0); +x_205 = lean_ctor_get(x_159, 1); +x_206 = lean_ctor_get(x_159, 2); +x_207 = lean_ctor_get(x_159, 3); +x_208 = lean_ctor_get(x_159, 4); +lean_inc(x_208); +lean_inc(x_207); lean_inc(x_206); lean_inc(x_205); lean_inc(x_204); -lean_inc(x_203); -lean_dec(x_158); -x_207 = lean_ctor_get_uint8(x_159, sizeof(void*)*2); -x_208 = lean_ctor_get(x_159, 0); -lean_inc(x_208); -x_209 = lean_ctor_get(x_159, 1); -lean_inc(x_209); -if (lean_is_exclusive(x_159)) { - lean_ctor_release(x_159, 0); - lean_ctor_release(x_159, 1); - x_210 = x_159; +lean_dec(x_159); +x_209 = lean_ctor_get_uint8(x_160, sizeof(void*)*2); +x_210 = lean_ctor_get(x_160, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_160, 1); +lean_inc(x_211); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_212 = x_160; } else { - lean_dec_ref(x_159); - x_210 = lean_box(0); + lean_dec_ref(x_160); + x_212 = lean_box(0); } -x_211 = lean_ctor_get(x_209, 2); -lean_inc(x_211); -x_212 = lean_unsigned_to_nat(0u); -x_213 = lean_nat_dec_lt(x_212, x_211); -if (x_213 == 0) +x_213 = lean_ctor_get(x_211, 2); +lean_inc(x_213); +x_214 = lean_unsigned_to_nat(0u); +x_215 = lean_nat_dec_lt(x_214, x_213); +if (x_215 == 0) { -lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; +lean_dec(x_213); lean_dec(x_211); -lean_dec(x_209); lean_dec(x_1); -if (lean_is_scalar(x_210)) { - x_214 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_212)) { + x_216 = lean_alloc_ctor(0, 2, 1); } else { - x_214 = x_210; -} -lean_ctor_set(x_214, 0, x_208); -lean_ctor_set(x_214, 1, x_57); -lean_ctor_set_uint8(x_214, sizeof(void*)*2, x_207); -x_215 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_215, 0, x_203); -lean_ctor_set(x_215, 1, x_204); -lean_ctor_set(x_215, 2, x_205); -lean_ctor_set(x_215, 3, x_206); -lean_ctor_set(x_215, 4, x_214); -x_216 = lean_st_ref_set(x_4, x_215, x_160); -x_217 = lean_ctor_get(x_216, 1); -lean_inc(x_217); -if (lean_is_exclusive(x_216)) { - lean_ctor_release(x_216, 0); - lean_ctor_release(x_216, 1); - x_218 = x_216; + x_216 = x_212; +} +lean_ctor_set(x_216, 0, x_210); +lean_ctor_set(x_216, 1, x_57); +lean_ctor_set_uint8(x_216, sizeof(void*)*2, x_209); +x_217 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_217, 0, x_204); +lean_ctor_set(x_217, 1, x_205); +lean_ctor_set(x_217, 2, x_206); +lean_ctor_set(x_217, 3, x_207); +lean_ctor_set(x_217, 4, x_208); +lean_ctor_set(x_217, 5, x_216); +x_218 = lean_st_ref_set(x_4, x_217, x_161); +x_219 = lean_ctor_get(x_218, 1); +lean_inc(x_219); +if (lean_is_exclusive(x_218)) { + lean_ctor_release(x_218, 0); + lean_ctor_release(x_218, 1); + x_220 = x_218; } else { - lean_dec_ref(x_216); - x_218 = lean_box(0); + lean_dec_ref(x_218); + x_220 = lean_box(0); } -if (lean_is_scalar(x_218)) { - x_219 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_220)) { + x_221 = lean_alloc_ctor(1, 2, 0); } else { - x_219 = x_218; - lean_ctor_set_tag(x_219, 1); + x_221 = x_220; + lean_ctor_set_tag(x_221, 1); } -lean_ctor_set(x_219, 0, x_153); -lean_ctor_set(x_219, 1, x_217); -x_34 = x_219; +lean_ctor_set(x_221, 0, x_154); +lean_ctor_set(x_221, 1, x_219); +x_34 = x_221; goto block_46; } else { -lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; -x_220 = lean_nat_sub(x_211, x_10); -lean_dec(x_211); -x_221 = l_Lean_Elab_instInhabitedInfoTree; -x_222 = l_Std_PersistentArray_get_x21___rarg(x_221, x_209, x_220); -lean_dec(x_220); -x_223 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_208, x_1, x_222); -if (lean_is_scalar(x_210)) { - x_224 = lean_alloc_ctor(0, 2, 1); +lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; +x_222 = lean_nat_sub(x_213, x_10); +lean_dec(x_213); +x_223 = l_Lean_Elab_instInhabitedInfoTree; +x_224 = l_Std_PersistentArray_get_x21___rarg(x_223, x_211, x_222); +lean_dec(x_222); +x_225 = l_Std_PersistentHashMap_insert___at_Lean_Elab_assignInfoHoleId___spec__1(x_210, x_1, x_224); +if (lean_is_scalar(x_212)) { + x_226 = lean_alloc_ctor(0, 2, 1); } else { - x_224 = x_210; -} -lean_ctor_set(x_224, 0, x_223); -lean_ctor_set(x_224, 1, x_57); -lean_ctor_set_uint8(x_224, sizeof(void*)*2, x_207); -x_225 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_225, 0, x_203); -lean_ctor_set(x_225, 1, x_204); -lean_ctor_set(x_225, 2, x_205); -lean_ctor_set(x_225, 3, x_206); -lean_ctor_set(x_225, 4, x_224); -x_226 = lean_st_ref_set(x_4, x_225, x_160); -x_227 = lean_ctor_get(x_226, 1); -lean_inc(x_227); -if (lean_is_exclusive(x_226)) { - lean_ctor_release(x_226, 0); - lean_ctor_release(x_226, 1); - x_228 = x_226; + x_226 = x_212; +} +lean_ctor_set(x_226, 0, x_225); +lean_ctor_set(x_226, 1, x_57); +lean_ctor_set_uint8(x_226, sizeof(void*)*2, x_209); +x_227 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_227, 0, x_204); +lean_ctor_set(x_227, 1, x_205); +lean_ctor_set(x_227, 2, x_206); +lean_ctor_set(x_227, 3, x_207); +lean_ctor_set(x_227, 4, x_208); +lean_ctor_set(x_227, 5, x_226); +x_228 = lean_st_ref_set(x_4, x_227, x_161); +x_229 = lean_ctor_get(x_228, 1); +lean_inc(x_229); +if (lean_is_exclusive(x_228)) { + lean_ctor_release(x_228, 0); + lean_ctor_release(x_228, 1); + x_230 = x_228; } else { - lean_dec_ref(x_226); - x_228 = lean_box(0); + lean_dec_ref(x_228); + x_230 = lean_box(0); } -if (lean_is_scalar(x_228)) { - x_229 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_230)) { + x_231 = lean_alloc_ctor(1, 2, 0); } else { - x_229 = x_228; - lean_ctor_set_tag(x_229, 1); + x_231 = x_230; + lean_ctor_set_tag(x_231, 1); } -lean_ctor_set(x_229, 0, x_153); -lean_ctor_set(x_229, 1, x_227); -x_34 = x_229; +lean_ctor_set(x_231, 0, x_154); +lean_ctor_set(x_231, 1, x_229); +x_34 = x_231; goto block_46; } } @@ -18861,14 +18860,24 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_11; +return x_11; +} +} +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_2); +lean_dec(x_2); +x_12 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2(x_1, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; } } -LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -19215,7 +19224,7 @@ lean_inc(x_14); x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); lean_dec(x_13); -x_16 = lean_ctor_get(x_14, 1); +x_16 = lean_ctor_get(x_14, 2); lean_inc(x_16); lean_dec(x_14); x_17 = lean_st_ref_get(x_9, x_15); @@ -19231,11 +19240,11 @@ lean_dec(x_19); x_22 = !lean_is_exclusive(x_20); if (x_22 == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_57; lean_object* x_58; lean_object* x_84; -x_23 = lean_ctor_get(x_20, 1); +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_58; lean_object* x_59; lean_object* x_86; +x_23 = lean_ctor_get(x_20, 2); lean_dec(x_23); x_24 = lean_box(0); -lean_ctor_set(x_20, 1, x_24); +lean_ctor_set(x_20, 2, x_24); x_25 = lean_st_ref_set(x_5, x_20, x_21); x_26 = lean_ctor_get(x_25, 1); lean_inc(x_26); @@ -19246,160 +19255,160 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_84 = lean_apply_7(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_26); -if (lean_obj_tag(x_84) == 0) +x_86 = lean_apply_7(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_26); +if (lean_obj_tag(x_86) == 0) { -lean_object* x_85; lean_object* x_86; uint8_t x_87; lean_object* x_88; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = 0; +lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +x_89 = 0; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_88 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_2, x_87, x_4, x_5, x_6, x_7, x_8, x_9, x_86); -if (lean_obj_tag(x_88) == 0) +x_90 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_2, x_89, x_4, x_5, x_6, x_7, x_8, x_9, x_88); +if (lean_obj_tag(x_90) == 0) { if (x_2 == 0) { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_89 = lean_ctor_get(x_88, 1); -lean_inc(x_89); -lean_dec(x_88); -x_90 = lean_box(0); -x_91 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_85, x_90, x_4, x_5, x_6, x_7, x_8, x_9, x_89); +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +lean_dec(x_90); +x_92 = lean_box(0); +x_93 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_87, x_92, x_4, x_5, x_6, x_7, x_8, x_9, x_91); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); -lean_dec(x_91); -x_27 = x_92; -x_28 = x_93; -goto block_56; +x_94 = lean_ctor_get(x_93, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_93, 1); +lean_inc(x_95); +lean_dec(x_93); +x_27 = x_94; +x_28 = x_95; +goto block_57; } else { if (x_3 == 0) { -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_94 = lean_ctor_get(x_88, 1); -lean_inc(x_94); -lean_dec(x_88); -x_95 = lean_box(0); -x_96 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_85, x_95, x_4, x_5, x_6, x_7, x_8, x_9, x_94); +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_dec(x_90); +x_97 = lean_box(0); +x_98 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_87, x_97, x_4, x_5, x_6, x_7, x_8, x_9, x_96); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -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_27 = x_97; -x_28 = x_98; -goto block_56; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_98, 1); +lean_inc(x_100); +lean_dec(x_98); +x_27 = x_99; +x_28 = x_100; +goto block_57; } else { -lean_object* x_99; lean_object* x_100; -x_99 = lean_ctor_get(x_88, 1); -lean_inc(x_99); -lean_dec(x_88); +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_90, 1); +lean_inc(x_101); +lean_dec(x_90); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_100 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultLoop(x_4, x_5, x_6, x_7, x_8, x_9, x_99); -if (lean_obj_tag(x_100) == 0) +x_102 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultLoop(x_4, x_5, x_6, x_7, x_8, x_9, x_101); +if (lean_obj_tag(x_102) == 0) { -lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_101 = lean_ctor_get(x_100, 0); -lean_inc(x_101); -x_102 = lean_ctor_get(x_100, 1); -lean_inc(x_102); -lean_dec(x_100); -x_103 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_85, x_101, x_4, x_5, x_6, x_7, x_8, x_9, x_102); +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_103 = lean_ctor_get(x_102, 0); +lean_inc(x_103); +x_104 = lean_ctor_get(x_102, 1); +lean_inc(x_104); +lean_dec(x_102); +x_105 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_87, x_103, x_4, x_5, x_6, x_7, x_8, x_9, x_104); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -lean_dec(x_101); -x_104 = lean_ctor_get(x_103, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_103, 1); -lean_inc(x_105); lean_dec(x_103); -x_27 = x_104; -x_28 = x_105; -goto block_56; +x_106 = lean_ctor_get(x_105, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_105, 1); +lean_inc(x_107); +lean_dec(x_105); +x_27 = x_106; +x_28 = x_107; +goto block_57; } else { -lean_object* x_106; lean_object* x_107; -lean_dec(x_85); +lean_object* x_108; lean_object* x_109; +lean_dec(x_87); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_106 = lean_ctor_get(x_100, 0); -lean_inc(x_106); -x_107 = lean_ctor_get(x_100, 1); -lean_inc(x_107); -lean_dec(x_100); -x_57 = x_106; -x_58 = x_107; -goto block_83; +x_108 = lean_ctor_get(x_102, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_102, 1); +lean_inc(x_109); +lean_dec(x_102); +x_58 = x_108; +x_59 = x_109; +goto block_85; } } } } else { -lean_object* x_108; lean_object* x_109; -lean_dec(x_85); +lean_object* x_110; lean_object* x_111; +lean_dec(x_87); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_108 = lean_ctor_get(x_88, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_88, 1); -lean_inc(x_109); -lean_dec(x_88); -x_57 = x_108; -x_58 = x_109; -goto block_83; +x_110 = lean_ctor_get(x_90, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_90, 1); +lean_inc(x_111); +lean_dec(x_90); +x_58 = x_110; +x_59 = x_111; +goto block_85; } } else { -lean_object* x_110; lean_object* x_111; +lean_object* x_112; lean_object* x_113; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_110 = lean_ctor_get(x_84, 0); -lean_inc(x_110); -x_111 = lean_ctor_get(x_84, 1); -lean_inc(x_111); -lean_dec(x_84); -x_57 = x_110; -x_58 = x_111; -goto block_83; +x_112 = lean_ctor_get(x_86, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_86, 1); +lean_inc(x_113); +lean_dec(x_86); +x_58 = x_112; +x_59 = x_113; +goto block_85; } -block_56: +block_57: { lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; x_29 = lean_st_ref_get(x_9, x_28); @@ -19417,9 +19426,9 @@ x_34 = !lean_is_exclusive(x_32); if (x_34 == 0) { lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_35 = lean_ctor_get(x_32, 1); +x_35 = lean_ctor_get(x_32, 2); x_36 = l_List_appendTR___rarg(x_35, x_16); -lean_ctor_set(x_32, 1, x_36); +lean_ctor_set(x_32, 2, x_36); x_37 = lean_st_ref_set(x_5, x_32, x_33); lean_dec(x_5); x_38 = !lean_is_exclusive(x_37); @@ -19451,219 +19460,205 @@ return x_43; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; x_44 = lean_ctor_get(x_32, 0); x_45 = lean_ctor_get(x_32, 1); x_46 = lean_ctor_get(x_32, 2); x_47 = lean_ctor_get(x_32, 3); x_48 = lean_ctor_get(x_32, 4); +x_49 = lean_ctor_get(x_32, 5); +lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); lean_dec(x_32); -x_49 = l_List_appendTR___rarg(x_45, x_16); -x_50 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_50, 0, x_44); -lean_ctor_set(x_50, 1, x_49); -lean_ctor_set(x_50, 2, x_46); -lean_ctor_set(x_50, 3, x_47); -lean_ctor_set(x_50, 4, x_48); -x_51 = lean_st_ref_set(x_5, x_50, x_33); +x_50 = l_List_appendTR___rarg(x_46, x_16); +x_51 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_51, 0, x_44); +lean_ctor_set(x_51, 1, x_45); +lean_ctor_set(x_51, 2, x_50); +lean_ctor_set(x_51, 3, x_47); +lean_ctor_set(x_51, 4, x_48); +lean_ctor_set(x_51, 5, x_49); +x_52 = lean_st_ref_set(x_5, x_51, x_33); lean_dec(x_5); -x_52 = lean_ctor_get(x_51, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_51)) { - lean_ctor_release(x_51, 0); - lean_ctor_release(x_51, 1); - x_53 = x_51; +x_53 = lean_ctor_get(x_52, 1); +lean_inc(x_53); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + x_54 = x_52; } else { - lean_dec_ref(x_51); - x_53 = lean_box(0); + lean_dec_ref(x_52); + x_54 = lean_box(0); } -x_54 = lean_ctor_get(x_27, 0); -lean_inc(x_54); +x_55 = lean_ctor_get(x_27, 0); +lean_inc(x_55); lean_dec(x_27); -if (lean_is_scalar(x_53)) { - x_55 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_54)) { + x_56 = lean_alloc_ctor(0, 2, 0); } else { - x_55 = x_53; + x_56 = x_54; } -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_52); -return x_55; +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_53); +return x_56; } } -block_83: +block_85: { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; -x_59 = lean_st_ref_get(x_9, x_58); +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; +x_60 = lean_st_ref_get(x_9, x_59); lean_dec(x_9); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_st_ref_take(x_5, x_60); -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); +x_61 = lean_ctor_get(x_60, 1); +lean_inc(x_61); +lean_dec(x_60); +x_62 = lean_st_ref_take(x_5, x_61); +x_63 = lean_ctor_get(x_62, 0); lean_inc(x_63); -lean_dec(x_61); -x_64 = !lean_is_exclusive(x_62); -if (x_64 == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; -x_65 = lean_ctor_get(x_62, 1); -x_66 = l_List_appendTR___rarg(x_65, x_16); -lean_ctor_set(x_62, 1, x_66); -x_67 = lean_st_ref_set(x_5, x_62, x_63); +x_64 = lean_ctor_get(x_62, 1); +lean_inc(x_64); +lean_dec(x_62); +x_65 = !lean_is_exclusive(x_63); +if (x_65 == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; +x_66 = lean_ctor_get(x_63, 2); +x_67 = l_List_appendTR___rarg(x_66, x_16); +lean_ctor_set(x_63, 2, x_67); +x_68 = lean_st_ref_set(x_5, x_63, x_64); lean_dec(x_5); -x_68 = !lean_is_exclusive(x_67); -if (x_68 == 0) +x_69 = !lean_is_exclusive(x_68); +if (x_69 == 0) { -lean_object* x_69; -x_69 = lean_ctor_get(x_67, 0); -lean_dec(x_69); -lean_ctor_set_tag(x_67, 1); -lean_ctor_set(x_67, 0, x_57); -return x_67; +lean_object* x_70; +x_70 = lean_ctor_get(x_68, 0); +lean_dec(x_70); +lean_ctor_set_tag(x_68, 1); +lean_ctor_set(x_68, 0, x_58); +return x_68; } else { -lean_object* x_70; lean_object* x_71; -x_70 = lean_ctor_get(x_67, 1); -lean_inc(x_70); -lean_dec(x_67); -x_71 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_71, 0, x_57); -lean_ctor_set(x_71, 1, x_70); -return x_71; +lean_object* x_71; lean_object* x_72; +x_71 = lean_ctor_get(x_68, 1); +lean_inc(x_71); +lean_dec(x_68); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_58); +lean_ctor_set(x_72, 1, x_71); +return x_72; } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_72 = lean_ctor_get(x_62, 0); -x_73 = lean_ctor_get(x_62, 1); -x_74 = lean_ctor_get(x_62, 2); -x_75 = lean_ctor_get(x_62, 3); -x_76 = lean_ctor_get(x_62, 4); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_73 = lean_ctor_get(x_63, 0); +x_74 = lean_ctor_get(x_63, 1); +x_75 = lean_ctor_get(x_63, 2); +x_76 = lean_ctor_get(x_63, 3); +x_77 = lean_ctor_get(x_63, 4); +x_78 = lean_ctor_get(x_63, 5); +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_dec(x_62); -x_77 = l_List_appendTR___rarg(x_73, x_16); -x_78 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_78, 0, x_72); -lean_ctor_set(x_78, 1, x_77); -lean_ctor_set(x_78, 2, x_74); -lean_ctor_set(x_78, 3, x_75); -lean_ctor_set(x_78, 4, x_76); -x_79 = lean_st_ref_set(x_5, x_78, x_63); +lean_dec(x_63); +x_79 = l_List_appendTR___rarg(x_75, x_16); +x_80 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_80, 0, x_73); +lean_ctor_set(x_80, 1, x_74); +lean_ctor_set(x_80, 2, x_79); +lean_ctor_set(x_80, 3, x_76); +lean_ctor_set(x_80, 4, x_77); +lean_ctor_set(x_80, 5, x_78); +x_81 = lean_st_ref_set(x_5, x_80, x_64); lean_dec(x_5); -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_82 = lean_ctor_get(x_81, 1); +lean_inc(x_82); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_83 = x_81; } else { - lean_dec_ref(x_79); - x_81 = lean_box(0); + lean_dec_ref(x_81); + x_83 = lean_box(0); } -if (lean_is_scalar(x_81)) { - x_82 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_83)) { + x_84 = lean_alloc_ctor(1, 2, 0); } else { - x_82 = x_81; - lean_ctor_set_tag(x_82, 1); + x_84 = x_83; + lean_ctor_set_tag(x_84, 1); } -lean_ctor_set(x_82, 0, x_57); -lean_ctor_set(x_82, 1, x_80); -return x_82; +lean_ctor_set(x_84, 0, x_58); +lean_ctor_set(x_84, 1, x_82); +return x_84; } } } else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_141; lean_object* x_142; lean_object* x_161; -x_112 = lean_ctor_get(x_20, 0); -x_113 = lean_ctor_get(x_20, 2); -x_114 = lean_ctor_get(x_20, 3); -x_115 = lean_ctor_get(x_20, 4); +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_145; lean_object* x_146; lean_object* x_166; +x_114 = lean_ctor_get(x_20, 0); +x_115 = lean_ctor_get(x_20, 1); +x_116 = lean_ctor_get(x_20, 3); +x_117 = lean_ctor_get(x_20, 4); +x_118 = lean_ctor_get(x_20, 5); +lean_inc(x_118); +lean_inc(x_117); +lean_inc(x_116); lean_inc(x_115); lean_inc(x_114); -lean_inc(x_113); -lean_inc(x_112); lean_dec(x_20); -x_116 = lean_box(0); -x_117 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_117, 0, x_112); -lean_ctor_set(x_117, 1, x_116); -lean_ctor_set(x_117, 2, x_113); -lean_ctor_set(x_117, 3, x_114); -lean_ctor_set(x_117, 4, x_115); -x_118 = lean_st_ref_set(x_5, x_117, x_21); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -lean_dec(x_118); +x_119 = lean_box(0); +x_120 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_120, 0, x_114); +lean_ctor_set(x_120, 1, x_115); +lean_ctor_set(x_120, 2, x_119); +lean_ctor_set(x_120, 3, x_116); +lean_ctor_set(x_120, 4, x_117); +lean_ctor_set(x_120, 5, x_118); +x_121 = lean_st_ref_set(x_5, x_120, x_21); +x_122 = lean_ctor_get(x_121, 1); +lean_inc(x_122); +lean_dec(x_121); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_161 = lean_apply_7(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_119); -if (lean_obj_tag(x_161) == 0) +x_166 = lean_apply_7(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_122); +if (lean_obj_tag(x_166) == 0) { -lean_object* x_162; lean_object* x_163; uint8_t x_164; lean_object* x_165; -x_162 = lean_ctor_get(x_161, 0); -lean_inc(x_162); -x_163 = lean_ctor_get(x_161, 1); -lean_inc(x_163); -lean_dec(x_161); -x_164 = 0; +lean_object* x_167; lean_object* x_168; uint8_t x_169; lean_object* x_170; +x_167 = lean_ctor_get(x_166, 0); +lean_inc(x_167); +x_168 = lean_ctor_get(x_166, 1); +lean_inc(x_168); +lean_dec(x_166); +x_169 = 0; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_165 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_2, x_164, x_4, x_5, x_6, x_7, x_8, x_9, x_163); -if (lean_obj_tag(x_165) == 0) +x_170 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_2, x_169, x_4, x_5, x_6, x_7, x_8, x_9, x_168); +if (lean_obj_tag(x_170) == 0) { if (x_2 == 0) { -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; -x_166 = lean_ctor_get(x_165, 1); -lean_inc(x_166); -lean_dec(x_165); -x_167 = lean_box(0); -x_168 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_162, x_167, x_4, x_5, x_6, x_7, x_8, x_9, x_166); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -x_169 = lean_ctor_get(x_168, 0); -lean_inc(x_169); -x_170 = lean_ctor_get(x_168, 1); -lean_inc(x_170); -lean_dec(x_168); -x_120 = x_169; -x_121 = x_170; -goto block_140; -} -else -{ -if (x_3 == 0) -{ lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; -x_171 = lean_ctor_get(x_165, 1); +x_171 = lean_ctor_get(x_170, 1); lean_inc(x_171); -lean_dec(x_165); +lean_dec(x_170); x_172 = lean_box(0); -x_173 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_162, x_172, x_4, x_5, x_6, x_7, x_8, x_9, x_171); +x_173 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_167, x_172, x_4, x_5, x_6, x_7, x_8, x_9, x_171); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -19673,237 +19668,268 @@ lean_inc(x_174); x_175 = lean_ctor_get(x_173, 1); lean_inc(x_175); lean_dec(x_173); -x_120 = x_174; -x_121 = x_175; -goto block_140; +x_123 = x_174; +x_124 = x_175; +goto block_144; } else { -lean_object* x_176; lean_object* x_177; -x_176 = lean_ctor_get(x_165, 1); +if (x_3 == 0) +{ +lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; +x_176 = lean_ctor_get(x_170, 1); lean_inc(x_176); -lean_dec(x_165); +lean_dec(x_170); +x_177 = lean_box(0); +x_178 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_167, x_177, x_4, x_5, x_6, x_7, x_8, x_9, x_176); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +x_179 = lean_ctor_get(x_178, 0); +lean_inc(x_179); +x_180 = lean_ctor_get(x_178, 1); +lean_inc(x_180); +lean_dec(x_178); +x_123 = x_179; +x_124 = x_180; +goto block_144; +} +else +{ +lean_object* x_181; lean_object* x_182; +x_181 = lean_ctor_get(x_170, 1); +lean_inc(x_181); +lean_dec(x_170); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_177 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultLoop(x_4, x_5, x_6, x_7, x_8, x_9, x_176); -if (lean_obj_tag(x_177) == 0) +x_182 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultLoop(x_4, x_5, x_6, x_7, x_8, x_9, x_181); +if (lean_obj_tag(x_182) == 0) { -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_178 = lean_ctor_get(x_177, 0); -lean_inc(x_178); -x_179 = lean_ctor_get(x_177, 1); -lean_inc(x_179); -lean_dec(x_177); -x_180 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_162, x_178, x_4, x_5, x_6, x_7, x_8, x_9, x_179); +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +x_183 = lean_ctor_get(x_182, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_182, 1); +lean_inc(x_184); +lean_dec(x_182); +x_185 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___lambda__1(x_167, x_183, x_4, x_5, x_6, x_7, x_8, x_9, x_184); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -lean_dec(x_178); -x_181 = lean_ctor_get(x_180, 0); -lean_inc(x_181); -x_182 = lean_ctor_get(x_180, 1); -lean_inc(x_182); -lean_dec(x_180); -x_120 = x_181; -x_121 = x_182; -goto block_140; +lean_dec(x_183); +x_186 = lean_ctor_get(x_185, 0); +lean_inc(x_186); +x_187 = lean_ctor_get(x_185, 1); +lean_inc(x_187); +lean_dec(x_185); +x_123 = x_186; +x_124 = x_187; +goto block_144; } else { -lean_object* x_183; lean_object* x_184; -lean_dec(x_162); +lean_object* x_188; lean_object* x_189; +lean_dec(x_167); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_183 = lean_ctor_get(x_177, 0); -lean_inc(x_183); -x_184 = lean_ctor_get(x_177, 1); -lean_inc(x_184); -lean_dec(x_177); -x_141 = x_183; -x_142 = x_184; -goto block_160; +x_188 = lean_ctor_get(x_182, 0); +lean_inc(x_188); +x_189 = lean_ctor_get(x_182, 1); +lean_inc(x_189); +lean_dec(x_182); +x_145 = x_188; +x_146 = x_189; +goto block_165; } } } } else { -lean_object* x_185; lean_object* x_186; -lean_dec(x_162); +lean_object* x_190; lean_object* x_191; +lean_dec(x_167); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_185 = lean_ctor_get(x_165, 0); -lean_inc(x_185); -x_186 = lean_ctor_get(x_165, 1); -lean_inc(x_186); -lean_dec(x_165); -x_141 = x_185; -x_142 = x_186; -goto block_160; +x_190 = lean_ctor_get(x_170, 0); +lean_inc(x_190); +x_191 = lean_ctor_get(x_170, 1); +lean_inc(x_191); +lean_dec(x_170); +x_145 = x_190; +x_146 = x_191; +goto block_165; } } else { -lean_object* x_187; lean_object* x_188; +lean_object* x_192; lean_object* x_193; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_187 = lean_ctor_get(x_161, 0); -lean_inc(x_187); -x_188 = lean_ctor_get(x_161, 1); -lean_inc(x_188); -lean_dec(x_161); -x_141 = x_187; -x_142 = x_188; -goto block_160; +x_192 = lean_ctor_get(x_166, 0); +lean_inc(x_192); +x_193 = lean_ctor_get(x_166, 1); +lean_inc(x_193); +lean_dec(x_166); +x_145 = x_192; +x_146 = x_193; +goto block_165; } -block_140: +block_144: { -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; -x_122 = lean_st_ref_get(x_9, x_121); +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; +x_125 = lean_st_ref_get(x_9, x_124); lean_dec(x_9); -x_123 = lean_ctor_get(x_122, 1); -lean_inc(x_123); -lean_dec(x_122); -x_124 = lean_st_ref_take(x_5, x_123); -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); +x_126 = lean_ctor_get(x_125, 1); lean_inc(x_126); -lean_dec(x_124); -x_127 = lean_ctor_get(x_125, 0); -lean_inc(x_127); -x_128 = lean_ctor_get(x_125, 1); +lean_dec(x_125); +x_127 = lean_st_ref_take(x_5, x_126); +x_128 = lean_ctor_get(x_127, 0); lean_inc(x_128); -x_129 = lean_ctor_get(x_125, 2); +x_129 = lean_ctor_get(x_127, 1); lean_inc(x_129); -x_130 = lean_ctor_get(x_125, 3); +lean_dec(x_127); +x_130 = lean_ctor_get(x_128, 0); lean_inc(x_130); -x_131 = lean_ctor_get(x_125, 4); +x_131 = lean_ctor_get(x_128, 1); lean_inc(x_131); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - lean_ctor_release(x_125, 2); - lean_ctor_release(x_125, 3); - lean_ctor_release(x_125, 4); - x_132 = x_125; +x_132 = lean_ctor_get(x_128, 2); +lean_inc(x_132); +x_133 = lean_ctor_get(x_128, 3); +lean_inc(x_133); +x_134 = lean_ctor_get(x_128, 4); +lean_inc(x_134); +x_135 = lean_ctor_get(x_128, 5); +lean_inc(x_135); +if (lean_is_exclusive(x_128)) { + lean_ctor_release(x_128, 0); + lean_ctor_release(x_128, 1); + lean_ctor_release(x_128, 2); + lean_ctor_release(x_128, 3); + lean_ctor_release(x_128, 4); + lean_ctor_release(x_128, 5); + x_136 = x_128; } else { - lean_dec_ref(x_125); - x_132 = lean_box(0); + lean_dec_ref(x_128); + x_136 = lean_box(0); } -x_133 = l_List_appendTR___rarg(x_128, x_16); -if (lean_is_scalar(x_132)) { - x_134 = lean_alloc_ctor(0, 5, 0); +x_137 = l_List_appendTR___rarg(x_132, x_16); +if (lean_is_scalar(x_136)) { + x_138 = lean_alloc_ctor(0, 6, 0); } else { - x_134 = x_132; -} -lean_ctor_set(x_134, 0, x_127); -lean_ctor_set(x_134, 1, x_133); -lean_ctor_set(x_134, 2, x_129); -lean_ctor_set(x_134, 3, x_130); -lean_ctor_set(x_134, 4, x_131); -x_135 = lean_st_ref_set(x_5, x_134, x_126); + x_138 = x_136; +} +lean_ctor_set(x_138, 0, x_130); +lean_ctor_set(x_138, 1, x_131); +lean_ctor_set(x_138, 2, x_137); +lean_ctor_set(x_138, 3, x_133); +lean_ctor_set(x_138, 4, x_134); +lean_ctor_set(x_138, 5, x_135); +x_139 = lean_st_ref_set(x_5, x_138, x_129); lean_dec(x_5); -x_136 = lean_ctor_get(x_135, 1); -lean_inc(x_136); -if (lean_is_exclusive(x_135)) { - lean_ctor_release(x_135, 0); - lean_ctor_release(x_135, 1); - x_137 = x_135; +x_140 = lean_ctor_get(x_139, 1); +lean_inc(x_140); +if (lean_is_exclusive(x_139)) { + lean_ctor_release(x_139, 0); + lean_ctor_release(x_139, 1); + x_141 = x_139; } else { - lean_dec_ref(x_135); - x_137 = lean_box(0); + lean_dec_ref(x_139); + x_141 = lean_box(0); } -x_138 = lean_ctor_get(x_120, 0); -lean_inc(x_138); -lean_dec(x_120); -if (lean_is_scalar(x_137)) { - x_139 = lean_alloc_ctor(0, 2, 0); +x_142 = lean_ctor_get(x_123, 0); +lean_inc(x_142); +lean_dec(x_123); +if (lean_is_scalar(x_141)) { + x_143 = lean_alloc_ctor(0, 2, 0); } else { - x_139 = x_137; + x_143 = x_141; } -lean_ctor_set(x_139, 0, x_138); -lean_ctor_set(x_139, 1, x_136); -return x_139; +lean_ctor_set(x_143, 0, x_142); +lean_ctor_set(x_143, 1, x_140); +return x_143; } -block_160: +block_165: { -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; -x_143 = lean_st_ref_get(x_9, x_142); +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; +x_147 = lean_st_ref_get(x_9, x_146); lean_dec(x_9); -x_144 = lean_ctor_get(x_143, 1); -lean_inc(x_144); -lean_dec(x_143); -x_145 = lean_st_ref_take(x_5, x_144); -x_146 = lean_ctor_get(x_145, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_145, 1); -lean_inc(x_147); -lean_dec(x_145); -x_148 = lean_ctor_get(x_146, 0); +x_148 = lean_ctor_get(x_147, 1); lean_inc(x_148); -x_149 = lean_ctor_get(x_146, 1); -lean_inc(x_149); -x_150 = lean_ctor_get(x_146, 2); +lean_dec(x_147); +x_149 = lean_st_ref_take(x_5, x_148); +x_150 = lean_ctor_get(x_149, 0); lean_inc(x_150); -x_151 = lean_ctor_get(x_146, 3); +x_151 = lean_ctor_get(x_149, 1); lean_inc(x_151); -x_152 = lean_ctor_get(x_146, 4); +lean_dec(x_149); +x_152 = lean_ctor_get(x_150, 0); lean_inc(x_152); -if (lean_is_exclusive(x_146)) { - lean_ctor_release(x_146, 0); - lean_ctor_release(x_146, 1); - lean_ctor_release(x_146, 2); - lean_ctor_release(x_146, 3); - lean_ctor_release(x_146, 4); - x_153 = x_146; +x_153 = lean_ctor_get(x_150, 1); +lean_inc(x_153); +x_154 = lean_ctor_get(x_150, 2); +lean_inc(x_154); +x_155 = lean_ctor_get(x_150, 3); +lean_inc(x_155); +x_156 = lean_ctor_get(x_150, 4); +lean_inc(x_156); +x_157 = lean_ctor_get(x_150, 5); +lean_inc(x_157); +if (lean_is_exclusive(x_150)) { + lean_ctor_release(x_150, 0); + lean_ctor_release(x_150, 1); + lean_ctor_release(x_150, 2); + lean_ctor_release(x_150, 3); + lean_ctor_release(x_150, 4); + lean_ctor_release(x_150, 5); + x_158 = x_150; } else { - lean_dec_ref(x_146); - x_153 = lean_box(0); + lean_dec_ref(x_150); + x_158 = lean_box(0); } -x_154 = l_List_appendTR___rarg(x_149, x_16); -if (lean_is_scalar(x_153)) { - x_155 = lean_alloc_ctor(0, 5, 0); +x_159 = l_List_appendTR___rarg(x_154, x_16); +if (lean_is_scalar(x_158)) { + x_160 = lean_alloc_ctor(0, 6, 0); } else { - x_155 = x_153; -} -lean_ctor_set(x_155, 0, x_148); -lean_ctor_set(x_155, 1, x_154); -lean_ctor_set(x_155, 2, x_150); -lean_ctor_set(x_155, 3, x_151); -lean_ctor_set(x_155, 4, x_152); -x_156 = lean_st_ref_set(x_5, x_155, x_147); + x_160 = x_158; +} +lean_ctor_set(x_160, 0, x_152); +lean_ctor_set(x_160, 1, x_153); +lean_ctor_set(x_160, 2, x_159); +lean_ctor_set(x_160, 3, x_155); +lean_ctor_set(x_160, 4, x_156); +lean_ctor_set(x_160, 5, x_157); +x_161 = lean_st_ref_set(x_5, x_160, x_151); lean_dec(x_5); -x_157 = lean_ctor_get(x_156, 1); -lean_inc(x_157); -if (lean_is_exclusive(x_156)) { - lean_ctor_release(x_156, 0); - lean_ctor_release(x_156, 1); - x_158 = x_156; +x_162 = lean_ctor_get(x_161, 1); +lean_inc(x_162); +if (lean_is_exclusive(x_161)) { + lean_ctor_release(x_161, 0); + lean_ctor_release(x_161, 1); + x_163 = x_161; } else { - lean_dec_ref(x_156); - x_158 = lean_box(0); + lean_dec_ref(x_161); + x_163 = lean_box(0); } -if (lean_is_scalar(x_158)) { - x_159 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_163)) { + x_164 = lean_alloc_ctor(1, 2, 0); } else { - x_159 = x_158; - lean_ctor_set_tag(x_159, 1); + x_164 = x_163; + lean_ctor_set_tag(x_164, 1); } -lean_ctor_set(x_159, 0, x_141); -lean_ctor_set(x_159, 1, x_157); -return x_159; +lean_ctor_set(x_164, 0, x_145); +lean_ctor_set(x_164, 1, x_162); +return x_164; } } } @@ -20211,7 +20237,299 @@ return x_47; } } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__1() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +x_10 = l_Lean_Elab_Term_runTactic(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; +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_markAsResolved(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_11); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_12; +} +else +{ +uint8_t x_13; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) +{ +return x_10; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_10, 0); +x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_10); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; +} +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_lt(x_3, x_2); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_4); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_dec(x_4); +x_14 = lean_array_uget(x_1, x_3); +x_22 = l_Lean_getDelayedMVarRoot___at_Lean_Elab_Term_isLetRecAuxMVar___spec__1(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_24); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; +lean_dec(x_23); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___closed__1; +x_15 = x_28; +x_16 = x_27; +goto block_21; +} +else +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_26, 0); +lean_inc(x_29); +lean_dec(x_26); +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +if (lean_obj_tag(x_30) == 2) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_31 = lean_ctor_get(x_25, 1); +lean_inc(x_31); +lean_dec(x_25); +x_32 = lean_ctor_get(x_30, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +lean_dec(x_30); +x_34 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___lambda__1), 9, 2); +lean_closure_set(x_34, 0, x_23); +lean_closure_set(x_34, 1, x_32); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_35 = l_Lean_Elab_Term_withSavedContext___rarg(x_33, x_34, x_5, x_6, x_7, x_8, x_9, x_10, x_31); +if (lean_obj_tag(x_35) == 0) +{ +lean_object* x_36; lean_object* x_37; +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +lean_dec(x_35); +x_37 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___closed__1; +x_15 = x_37; +x_16 = x_36; +goto block_21; +} +else +{ +uint8_t x_38; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_38 = !lean_is_exclusive(x_35); +if (x_38 == 0) +{ +return x_35; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_35, 0); +x_40 = lean_ctor_get(x_35, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_35); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} +} +} +else +{ +lean_object* x_42; lean_object* x_43; +lean_dec(x_30); +lean_dec(x_23); +x_42 = lean_ctor_get(x_25, 1); +lean_inc(x_42); +lean_dec(x_25); +x_43 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___closed__1; +x_15 = x_43; +x_16 = x_42; +goto block_21; +} +} +block_21: +{ +lean_object* x_17; size_t x_18; size_t x_19; +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +x_18 = 1; +x_19 = lean_usize_add(x_3, x_18); +x_3 = x_19; +x_4 = x_17; +x_11 = x_16; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_runPendingTacticsAt(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; +x_9 = l_Lean_Meta_getMVars(x_1, x_4, x_5, x_6, x_7, x_8); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_array_get_size(x_10); +x_13 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_14 = 0; +x_15 = lean_box(0); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1(x_10, x_13, x_14, x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_11); +lean_dec(x_10); +if (lean_obj_tag(x_16) == 0) +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_16, 0); +lean_dec(x_18); +lean_ctor_set(x_16, 0, x_15); +return x_16; +} +else +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +lean_dec(x_16); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_15); +lean_ctor_set(x_20, 1, x_19); +return x_20; +} +} +else +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_16); +if (x_21 == 0) +{ +return x_16; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_16, 0); +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_16); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_1); +return x_14; +} +} +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__1() { _start: { lean_object* x_1; @@ -20219,21 +20537,21 @@ x_1 = lean_mk_string_from_bytes("resume", 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeUsingDefaultPrio_synthesizeUsingDefaultInstance___lambda__3___closed__2; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__2; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__2; x_3 = l_Lean_registerTraceClass(x_2, x_1); return x_3; } @@ -20349,10 +20667,10 @@ l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__1 = _init_l_Lean_Elab_Term_r lean_mark_persistent(l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__1); l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2 = _init_l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2(); lean_mark_persistent(l_Lean_Elab_Term_reportStuckSyntheticMVar___closed__2); -l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___closed__1 = _init_l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___rarg___closed__1); -l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___closed__1(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__17___closed__1); +l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___closed__1 = _init_l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___closed__1(); +lean_mark_persistent(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_getSomeSynthethicMVarsRef___closed__1); +l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___spec__16___closed__1); l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___closed__1 = _init_l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___closed__1(); lean_mark_persistent(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___closed__1); l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___closed__2 = _init_l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_throwStuckAtUniverseCnstr___closed__2(); @@ -20363,24 +20681,24 @@ l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesizeSyntheticMVars_loop___sp lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesizeSyntheticMVars_loop___spec__1___closed__1); l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesizeSyntheticMVars_loop___spec__1___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesizeSyntheticMVars_loop___spec__1___closed__2(); lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_synthesizeSyntheticMVars_loop___spec__1___closed__2); +l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__1 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__1(); +lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__1); +l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__2 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__2(); +lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__2); +l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__3 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__3(); +lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__3); +l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__4 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__4(); +lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__4); +l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__5 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__5(); +lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__5); +l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__6 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__6(); +lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___lambda__2___closed__6); l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__1 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__1(); lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__1); l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__2 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__2(); lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__2); l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__3 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__3(); lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__3); -l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__4 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__4(); -lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__4); -l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__5 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__5(); -lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__5); -l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__6 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__6(); -lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__6); -l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__7 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__7(); -lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__7); -l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__8 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__8(); -lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__8); -l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__9 = _init_l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__9(); -lean_mark_persistent(l_List_filterAuxM___at___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___spec__1___closed__9); l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__1 = _init_l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__1(); lean_mark_persistent(l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__1); l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__2 = _init_l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_synthesizeSyntheticMVarsStep___lambda__1___closed__2(); @@ -20449,11 +20767,13 @@ l_Lean_instantiateLCtxMVars___at_Lean_Elab_Term_runTactic___spec__2___closed__7 lean_mark_persistent(l_Lean_instantiateLCtxMVars___at_Lean_Elab_Term_runTactic___spec__2___closed__7); l_Lean_Elab_Term_withSynthesizeLight___rarg___closed__1 = _init_l_Lean_Elab_Term_withSynthesizeLight___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_withSynthesizeLight___rarg___closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267____closed__2); -res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5267_(lean_io_mk_world()); +l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_runPendingTacticsAt___spec__1___closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846____closed__2); +res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_SyntheticMVars___hyg_5846_(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/Basic.c b/stage0/stdlib/Lean/Elab/Tactic/Basic.c index 2461f8eee109..5384b8026c7a 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Basic.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Basic.c @@ -16,68 +16,68 @@ extern "C" { lean_object* l_List_reverse___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___closed__3; static lean_object* l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_getNameOfIdent_x27___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withCaseRef(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___boxed__const__1; -static lean_object* l_Lean_Elab_Tactic_evalTacticAux___closed__8; -static lean_object* l_Lean_Elab_Tactic_evalTacticAux___closed__4; -static lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); +static lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM; -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__2; static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__8; lean_object* l_Lean_registerTraceClass(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getMainTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___closed__1; -static lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__1; lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__5; static lean_object* l_Lean_Elab_Tactic_instMonadTacticM___closed__7; LEAN_EXPORT lean_object* l_Lean_isExprMVarAssigned___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__5; lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__15; -static lean_object* l_Lean_Elab_Tactic_evalTacticAux___closed__1; static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__3; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_throwNoGoalsToBeSolved___spec__1(lean_object*); uint8_t l_Std_PersistentHashMap_contains___at_Lean_isExprMVarAssigned___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withCaseRef___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_adaptExpander___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkTacticAttribute(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SavedState_restore(lean_object*, 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_SavedState_restore(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_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_admitGoal___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4(lean_object*, lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); uint8_t l_Lean_Elab_isAbortExceptionId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadTacticM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_pruneSolvedGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_tagUntaggedGoals___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg___closed__1; static lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getCurrMacroScope___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___closed__7; +lean_object* l_Lean_toMessageList(lean_object*); extern lean_object* l_Lean_maxRecDepthErrorMessage; +lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_appendGoals___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_pruneSolvedGoals___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_instantiateMVars___at_Lean_Elab_Tactic_getMainTarget___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_focus(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_focusAndDone(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Tactic_adaptExpander___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux(lean_object*, 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_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg(lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_done(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_mkInitialTacticInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_expandEval(lean_object*, lean_object*, lean_object*, lean_object*, lean_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_withCaseRef___rarg___closed__1; lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_run___lambda__1___closed__1; @@ -87,7 +87,7 @@ uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_TacticM_runCore_x27(lean_object*); static lean_object* l_Lean_Elab_goalsToMessageData___closed__1; -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__1; +static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__4; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_tagUntaggedGoals___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__9; static lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___closed__5; @@ -97,99 +97,113 @@ lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Tactic_withMacroExpansion___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tryCatch(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_setGoals___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_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___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_List_forIn_loop___at_Lean_Elab_Tactic_tagUntaggedGoals___spec__2___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__3; static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__14; lean_object* l_Lean_MetavarContext_setMVarUserName(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withMainContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getGoals___boxed(lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_getEntries___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__4; -static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__3; static lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___closed__3; +static lean_object* l_Lean_Elab_Tactic_evalTactic___closed__3; LEAN_EXPORT lean_object* l_Lean_assignExprMVar___at_Lean_Elab_Tactic_closeMainGoal___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__4; lean_object* l_Std_PersistentHashMap_insert___at_Lean_assignExprMVar___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_saveTacticInfoForToken___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_joinSep(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__5(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getCurrMacroScope___rarg(lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_101_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_done___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_liftExcept___at_Lean_Elab_liftMacroM___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__1; +static lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_assignExprMVar___at_Lean_Elab_Tactic_closeMainGoal___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withPPInaccessibleNames___at_Lean_Elab_Term_reportUnsolvedGoals___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaMAtMain(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadExceptExceptionTacticM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withTacticInfoContext___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_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaTacticAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaTacticAux___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_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadExceptExceptionTacticM___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_saveState(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tryCatch___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withoutRecover(lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_closeMainGoal___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getMainGoal_loop(lean_object*, 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_tagUntaggedGoals___boxed(lean_object*, 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_assignExprMVar___at_Lean_Meta_getLevel___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_withFreshMacroScope___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_instAlternativeTacticM___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ensureHasNoMVars___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_goalsToMessageData___closed__2; +static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__3; lean_object* l_Lean_Meta_withMVarContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadTacticM___closed__5; +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkSorry(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvar___override(lean_object*); lean_object* l_Lean_Elab_expandMacroImpl_x3f(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_withTacticInfoContext___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_closeMainGoal___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_eval(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadTacticM___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_focus___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkInitialTacticInfo___elambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs(lean_object*, lean_object*, 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_mkInitialTacticInfo(lean_object*, 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_instMonadExceptExceptionTacticM; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadTacticM; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withTacticInfoContext(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withCaseRef___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTacticAux___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__1; +static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_closeUsingOrAdmit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkTacticInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_orElse___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withTacticInfoContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_log___at_Lean_Elab_Term_traceAtCmdPos___spec__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_focusAndDone___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__6; -static lean_object* l_Lean_Elab_Tactic_evalTacticAux___closed__3; uint8_t l_Lean_Expr_hasExprMVar(lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaMAtMain___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instOrElseTacticM___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadTacticM___closed__8; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_abortTacticExceptionId; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getGoals___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_name_append_index_after(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getUnsolvedGoals(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_getMainTarget(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_Elab_Tactic_evalTactic_expandEval___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getGoals___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__4; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTacticAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Term_reportUnsolvedGoals___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_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___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_st_mk_ref(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_withMacroExpansion___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_saveTacticInfoForToken(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -199,92 +213,96 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_closeMainGoal___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_withMainContext___spec__1(lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalTacticAux___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadTacticM___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadExceptExceptionTacticM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaMAtMain___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getNameOfIdent_x27(lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Tactic_withMacroExpansion___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withCaseRef___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadTacticM___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getMainModule___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT 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_mkInitialTacticInfo___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getMainModule___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__2; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_tagUntaggedGoals___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437____closed__1; -static lean_object* l_Lean_Elab_Tactic_expandTacticMacro___closed__1; +uint8_t l_Array_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_run(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_instAlternativeMetaM; lean_object* l_Lean_Elab_mkElabAttribute___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_MessageData_hasSyntheticSorry(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadTacticM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___closed__1; +static lean_object* l_Lean_Elab_Tactic_evalTactic___closed__2; extern lean_object* l_Lean_Meta_instMonadMetaM; lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_Context_recover___default; static lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___closed__1; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic___closed__1; static lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_TacticM_runCore(lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__2___closed__1; size_t lean_usize_of_nat(lean_object*); lean_object* l_Lean_InternalExceptionId_getName(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__3; lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceOptions(lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadExceptExceptionTacticM___closed__3; lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadExceptExceptionTacticM___closed__1; LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_saveTacticInfoForToken___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_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*); LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_withMacroExpansion___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaTactic___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalTacticAux___closed__7; -static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__10(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getNameOfIdent_x27___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaTactic1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___closed__1; static lean_object* l_Lean_Elab_Tactic_getNameOfIdent_x27___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_appendGoals(lean_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_evalTactic___closed__4; LEAN_EXPORT 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_Lean_Elab_Tactic_instMonadTacticM___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___lambda__1(lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tryTactic_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTacticAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Tactic_withMacroExpansion___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withMainContext(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withPPInaccessibleNames___at_Lean_Elab_Term_reportUnsolvedGoals___spec__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_goalsToMessageData(lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* l_Lean_Meta_getMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_focusAndDone___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_MetavarContext_isAnonymousMVar(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__1; static lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___lambda__1___closed__2; -static lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__3; +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__9(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Term_instMonadTermElabM; extern lean_object* l_Lean_Elab_macroAttribute; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaTactic(lean_object*, 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_expandTacticMacroFns_loop___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_environment_main_module(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___closed__2; static lean_object* l_Lean_Elab_Tactic_instMonadTacticM___closed__2; uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ensureHasNoMVars___closed__2; -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTacticAux___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadTacticM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasMVar(lean_object*); @@ -293,98 +311,116 @@ lean_object* l_Lean_Elab_Term_SavedState_restore(lean_object*, uint8_t, lean_obj lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__11; -static lean_object* l_Lean_Elab_Tactic_evalTacticAux___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); static lean_object* l_Lean_Elab_Tactic_ensureHasNoMVars___closed__1; static lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___lambda__1___closed__1; +static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_setGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withPPInaccessibleNamesImp___rarg(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__10; +static lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tagUntaggedGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Exception_getRef(lean_object*); +LEAN_EXPORT 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*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__13; +static lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withMacroExpansion___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_EXPORT lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___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_st_ref_set(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1; +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__1; +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterAuxM___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isExprMVarAssigned___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_instAlternativeTacticM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ensureHasNoMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_tagUntaggedGoals___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getMainDecl(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_instMonadTacticM___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaTacticAux(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_adaptExpander(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_closeMainGoal(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tryTactic___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621_(lean_object*); lean_object* l_Lean_Meta_getMVarDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_throwNoGoalsToBeSolved___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withMacroExpansion___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportUnsolvedGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_logUnassignedUsingErrorInfos(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_evalTactic___boxed__const__1; static lean_object* l_Lean_Elab_Tactic_instAlternativeTacticM___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic___closed__8; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tryTactic_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_throwNoGoalsToBeSolved___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_replaceMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___closed__6; lean_object* l_Lean_indentD(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; +LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonadReaderT___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___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_withoutRecover___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tryTactic(lean_object*); +static lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_liftMetaTactic1(lean_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_evalTacticAux___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_saveTacticInfoForToken___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_withMainContext___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_saveState___boxed(lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instOrElseTacticM(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_saveState___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_throwNoGoalsToBeSolved(lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_withMacroExpansion(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__2; uint8_t l_List_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__1; uint8_t l_Lean_Elab_isAbortTacticException(lean_object*); +static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__2; static lean_object* l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Elab_goalsToMessageData___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getCurrMacroScope(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM; LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___at_Lean_Elab_Tactic_run___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_tagUntaggedGoals___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getMainModule(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_instAlternativeTacticM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getMainModule___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg(lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadExceptExceptionTacticM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__12; -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_orElse(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getCurrMacroScope___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkTacticAttribute___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getGoals(lean_object*); @@ -394,25 +430,31 @@ lean_object* l_Lean_Elab_Term_saveState___rarg(lean_object*, lean_object*, lean_ static lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkTacticInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_run___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_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg___closed__1; LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Term_reportUnsolvedGoals___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacro(lean_object*, lean_object*, 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_evalTactic_handleEx(lean_object*, lean_object*, lean_object*, lean_object*, 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_evalTactic_expandEval___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_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___closed__2; LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; +static lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getUnsolvedGoals___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_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SavedState_restore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SavedState_restore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1___closed__1; lean_object* l_ReaderT_instAlternativeReaderT___rarg(lean_object*, lean_object*); +lean_object* l_Lean_Exception_toMessageData(lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_tagUntaggedGoals___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Tactic_withMacroExpansion___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg(lean_object*); uint8_t l_Lean_Syntax_isIdent(lean_object*); +static lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___closed__4; +static lean_object* l_Lean_Elab_Tactic_evalTactic___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_admitGoal___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { @@ -1920,7 +1962,7 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_run___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; 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_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; +lean_object* x_10; 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_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; x_23 = lean_st_ref_get(x_8, x_9); x_24 = lean_ctor_get(x_23, 1); lean_inc(x_24); @@ -1931,401 +1973,411 @@ lean_inc(x_26); x_27 = lean_ctor_get(x_25, 1); lean_inc(x_27); lean_dec(x_25); -x_28 = lean_ctor_get(x_26, 1); +x_28 = lean_ctor_get(x_26, 2); lean_inc(x_28); lean_dec(x_26); -x_53 = lean_st_ref_get(x_8, x_27); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_st_ref_take(x_4, x_54); -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); +x_54 = lean_st_ref_get(x_8, x_27); +x_55 = lean_ctor_get(x_54, 1); +lean_inc(x_55); +lean_dec(x_54); +x_56 = lean_st_ref_take(x_4, x_55); +x_57 = lean_ctor_get(x_56, 0); lean_inc(x_57); -lean_dec(x_55); -x_58 = !lean_is_exclusive(x_56); -if (x_58 == 0) +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +x_59 = !lean_is_exclusive(x_57); +if (x_59 == 0) { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_103; lean_object* x_104; -x_59 = lean_ctor_get(x_56, 1); -lean_dec(x_59); -x_60 = lean_box(0); -lean_ctor_set(x_56, 1, x_60); -x_61 = lean_st_ref_set(x_4, x_56, x_57); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_63, 0, x_1); -lean_ctor_set(x_63, 1, x_60); -x_64 = lean_st_ref_get(x_8, x_62); -x_65 = lean_ctor_get(x_64, 1); -lean_inc(x_65); -lean_dec(x_64); -x_66 = lean_st_mk_ref(x_63, x_65); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); +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_105; lean_object* x_106; +x_60 = lean_ctor_get(x_57, 2); +lean_dec(x_60); +x_61 = lean_box(0); +lean_ctor_set(x_57, 2, x_61); +x_62 = lean_st_ref_set(x_4, x_57, x_58); +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +lean_dec(x_62); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_1); +lean_ctor_set(x_64, 1, x_61); +x_65 = lean_st_ref_get(x_8, x_63); +x_66 = lean_ctor_get(x_65, 1); +lean_inc(x_66); +lean_dec(x_65); +x_67 = lean_st_mk_ref(x_64, x_66); +x_68 = lean_ctor_get(x_67, 0); lean_inc(x_68); -lean_dec(x_66); -x_103 = l_Lean_Elab_Tactic_run___lambda__1___closed__1; +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); +x_105 = l_Lean_Elab_Tactic_run___lambda__1___closed__1; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_67); -x_104 = lean_apply_9(x_2, x_103, x_67, x_3, x_4, x_5, x_6, x_7, x_8, x_68); -if (lean_obj_tag(x_104) == 0) +lean_inc(x_68); +x_106 = lean_apply_9(x_2, x_105, x_68, x_3, x_4, x_5, x_6, x_7, x_8, x_69); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -lean_dec(x_104); -x_106 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_103, x_67, x_3, x_4, x_5, x_6, x_7, x_8, x_105); +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_107 = lean_ctor_get(x_106, 1); +lean_inc(x_107); +lean_dec(x_106); +x_108 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_105, x_68, x_3, x_4, x_5, x_6, x_7, x_8, x_107); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_107 = lean_ctor_get(x_106, 0); -lean_inc(x_107); -x_108 = lean_ctor_get(x_106, 1); -lean_inc(x_108); -lean_dec(x_106); -x_69 = x_107; -x_70 = x_108; -goto block_102; +x_109 = lean_ctor_get(x_108, 0); +lean_inc(x_109); +x_110 = lean_ctor_get(x_108, 1); +lean_inc(x_110); +lean_dec(x_108); +x_70 = x_109; +x_71 = x_110; +goto block_104; } else { -lean_object* x_109; lean_object* x_110; uint8_t x_111; -x_109 = lean_ctor_get(x_104, 0); -lean_inc(x_109); -x_110 = lean_ctor_get(x_104, 1); -lean_inc(x_110); -lean_dec(x_104); -x_111 = l_Lean_Elab_isAbortTacticException(x_109); -if (x_111 == 0) +lean_object* x_111; lean_object* x_112; uint8_t x_113; +x_111 = lean_ctor_get(x_106, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_dec(x_106); +x_113 = l_Lean_Elab_isAbortTacticException(x_111); +if (x_113 == 0) { -lean_dec(x_67); +lean_dec(x_68); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_29 = x_109; -x_30 = x_110; -goto block_52; +x_29 = x_111; +x_30 = x_112; +goto block_53; } else { -lean_object* x_112; lean_object* x_113; lean_object* x_114; -lean_dec(x_109); -x_112 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_103, x_67, x_3, x_4, x_5, x_6, x_7, x_8, x_110); +lean_object* x_114; lean_object* x_115; lean_object* x_116; +lean_dec(x_111); +x_114 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_105, x_68, x_3, x_4, x_5, x_6, x_7, x_8, x_112); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_113 = lean_ctor_get(x_112, 0); -lean_inc(x_113); -x_114 = lean_ctor_get(x_112, 1); -lean_inc(x_114); -lean_dec(x_112); -x_69 = x_113; -x_70 = x_114; -goto block_102; +x_115 = lean_ctor_get(x_114, 0); +lean_inc(x_115); +x_116 = lean_ctor_get(x_114, 1); +lean_inc(x_116); +lean_dec(x_114); +x_70 = x_115; +x_71 = x_116; +goto block_104; } } -block_102: +block_104: { -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; uint8_t x_80; -x_71 = lean_st_ref_get(x_8, x_70); -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -lean_dec(x_71); -x_73 = lean_st_ref_get(x_67, x_72); -lean_dec(x_67); -x_74 = lean_ctor_get(x_73, 1); -lean_inc(x_74); -lean_dec(x_73); -x_75 = lean_st_ref_get(x_8, x_74); +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; +x_72 = lean_st_ref_get(x_8, x_71); +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +lean_dec(x_72); +x_74 = lean_st_ref_get(x_68, x_73); +lean_dec(x_68); +x_75 = lean_ctor_get(x_74, 1); +lean_inc(x_75); +lean_dec(x_74); +x_76 = lean_st_ref_get(x_8, x_75); lean_dec(x_8); -x_76 = lean_ctor_get(x_75, 1); -lean_inc(x_76); -lean_dec(x_75); -x_77 = lean_st_ref_take(x_4, x_76); -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); +x_78 = lean_st_ref_take(x_4, x_77); +x_79 = lean_ctor_get(x_78, 0); lean_inc(x_79); -lean_dec(x_77); -x_80 = !lean_is_exclusive(x_78); -if (x_80 == 0) +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +lean_dec(x_78); +x_81 = !lean_is_exclusive(x_79); +if (x_81 == 0) { -lean_object* x_81; lean_object* x_82; uint8_t x_83; -x_81 = lean_ctor_get(x_78, 1); -lean_dec(x_81); -lean_ctor_set(x_78, 1, x_28); -x_82 = lean_st_ref_set(x_4, x_78, x_79); +lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_82 = lean_ctor_get(x_79, 2); +lean_dec(x_82); +lean_ctor_set(x_79, 2, x_28); +x_83 = lean_st_ref_set(x_4, x_79, x_80); lean_dec(x_4); -x_83 = !lean_is_exclusive(x_82); -if (x_83 == 0) +x_84 = !lean_is_exclusive(x_83); +if (x_84 == 0) { -lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_84 = lean_ctor_get(x_82, 0); -lean_dec(x_84); -x_85 = lean_box(0); -x_86 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_86, 0, x_69); -lean_ctor_set(x_86, 1, x_85); -lean_ctor_set(x_82, 0, x_86); -x_10 = x_82; +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_83, 0); +lean_dec(x_85); +x_86 = lean_box(0); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_70); +lean_ctor_set(x_87, 1, x_86); +lean_ctor_set(x_83, 0, x_87); +x_10 = x_83; goto block_22; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_87 = lean_ctor_get(x_82, 1); -lean_inc(x_87); -lean_dec(x_82); -x_88 = lean_box(0); -x_89 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_89, 0, x_69); -lean_ctor_set(x_89, 1, x_88); +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_88 = lean_ctor_get(x_83, 1); +lean_inc(x_88); +lean_dec(x_83); +x_89 = lean_box(0); x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_87); -x_10 = x_90; +lean_ctor_set(x_90, 0, x_70); +lean_ctor_set(x_90, 1, x_89); +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_88); +x_10 = x_91; goto block_22; } } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_91 = lean_ctor_get(x_78, 0); -x_92 = lean_ctor_get(x_78, 2); -x_93 = lean_ctor_get(x_78, 3); -x_94 = lean_ctor_get(x_78, 4); +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_92 = lean_ctor_get(x_79, 0); +x_93 = lean_ctor_get(x_79, 1); +x_94 = lean_ctor_get(x_79, 3); +x_95 = lean_ctor_get(x_79, 4); +x_96 = lean_ctor_get(x_79, 5); +lean_inc(x_96); +lean_inc(x_95); lean_inc(x_94); lean_inc(x_93); lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_78); -x_95 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_95, 0, x_91); -lean_ctor_set(x_95, 1, x_28); -lean_ctor_set(x_95, 2, x_92); -lean_ctor_set(x_95, 3, x_93); -lean_ctor_set(x_95, 4, x_94); -x_96 = lean_st_ref_set(x_4, x_95, x_79); -lean_dec(x_4); -x_97 = lean_ctor_get(x_96, 1); -lean_inc(x_97); -if (lean_is_exclusive(x_96)) { - lean_ctor_release(x_96, 0); - lean_ctor_release(x_96, 1); - x_98 = x_96; +lean_dec(x_79); +x_97 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_97, 0, x_92); +lean_ctor_set(x_97, 1, x_93); +lean_ctor_set(x_97, 2, x_28); +lean_ctor_set(x_97, 3, x_94); +lean_ctor_set(x_97, 4, x_95); +lean_ctor_set(x_97, 5, x_96); +x_98 = lean_st_ref_set(x_4, x_97, x_80); +lean_dec(x_4); +x_99 = lean_ctor_get(x_98, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_100 = x_98; } else { - lean_dec_ref(x_96); - x_98 = lean_box(0); -} -x_99 = lean_box(0); -x_100 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_100, 0, x_69); -lean_ctor_set(x_100, 1, x_99); -if (lean_is_scalar(x_98)) { - x_101 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_98); + x_100 = lean_box(0); +} +x_101 = lean_box(0); +x_102 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_102, 0, x_70); +lean_ctor_set(x_102, 1, x_101); +if (lean_is_scalar(x_100)) { + x_103 = lean_alloc_ctor(0, 2, 0); } else { - x_101 = x_98; + x_103 = x_100; } -lean_ctor_set(x_101, 0, x_100); -lean_ctor_set(x_101, 1, x_97); -x_10 = x_101; +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_99); +x_10 = x_103; goto block_22; } } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; 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_153; lean_object* x_154; -x_115 = lean_ctor_get(x_56, 0); -x_116 = lean_ctor_get(x_56, 2); -x_117 = lean_ctor_get(x_56, 3); -x_118 = lean_ctor_get(x_56, 4); +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_157; lean_object* x_158; +x_117 = lean_ctor_get(x_57, 0); +x_118 = lean_ctor_get(x_57, 1); +x_119 = lean_ctor_get(x_57, 3); +x_120 = lean_ctor_get(x_57, 4); +x_121 = lean_ctor_get(x_57, 5); +lean_inc(x_121); +lean_inc(x_120); +lean_inc(x_119); lean_inc(x_118); lean_inc(x_117); -lean_inc(x_116); -lean_inc(x_115); -lean_dec(x_56); -x_119 = lean_box(0); -x_120 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_120, 0, x_115); -lean_ctor_set(x_120, 1, x_119); -lean_ctor_set(x_120, 2, x_116); -lean_ctor_set(x_120, 3, x_117); -lean_ctor_set(x_120, 4, x_118); -x_121 = lean_st_ref_set(x_4, x_120, x_57); -x_122 = lean_ctor_get(x_121, 1); -lean_inc(x_122); -lean_dec(x_121); -x_123 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_123, 0, x_1); -lean_ctor_set(x_123, 1, x_119); -x_124 = lean_st_ref_get(x_8, x_122); +lean_dec(x_57); +x_122 = lean_box(0); +x_123 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_123, 0, x_117); +lean_ctor_set(x_123, 1, x_118); +lean_ctor_set(x_123, 2, x_122); +lean_ctor_set(x_123, 3, x_119); +lean_ctor_set(x_123, 4, x_120); +lean_ctor_set(x_123, 5, x_121); +x_124 = lean_st_ref_set(x_4, x_123, x_58); x_125 = lean_ctor_get(x_124, 1); lean_inc(x_125); lean_dec(x_124); -x_126 = lean_st_mk_ref(x_123, x_125); -x_127 = lean_ctor_get(x_126, 0); -lean_inc(x_127); -x_128 = lean_ctor_get(x_126, 1); +x_126 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_126, 0, x_1); +lean_ctor_set(x_126, 1, x_122); +x_127 = lean_st_ref_get(x_8, x_125); +x_128 = lean_ctor_get(x_127, 1); lean_inc(x_128); -lean_dec(x_126); -x_153 = l_Lean_Elab_Tactic_run___lambda__1___closed__1; +lean_dec(x_127); +x_129 = lean_st_mk_ref(x_126, 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); +x_157 = l_Lean_Elab_Tactic_run___lambda__1___closed__1; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -lean_inc(x_127); -x_154 = lean_apply_9(x_2, x_153, x_127, x_3, x_4, x_5, x_6, x_7, x_8, x_128); -if (lean_obj_tag(x_154) == 0) +lean_inc(x_130); +x_158 = lean_apply_9(x_2, x_157, x_130, x_3, x_4, x_5, x_6, x_7, x_8, x_131); +if (lean_obj_tag(x_158) == 0) { -lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -x_155 = lean_ctor_get(x_154, 1); -lean_inc(x_155); -lean_dec(x_154); -x_156 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_153, x_127, x_3, x_4, x_5, x_6, x_7, x_8, x_155); +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_159 = lean_ctor_get(x_158, 1); +lean_inc(x_159); +lean_dec(x_158); +x_160 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_157, x_130, x_3, x_4, x_5, x_6, x_7, x_8, x_159); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -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_129 = x_157; -x_130 = x_158; -goto block_152; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_132 = x_161; +x_133 = x_162; +goto block_156; } else { -lean_object* x_159; lean_object* x_160; uint8_t x_161; -x_159 = lean_ctor_get(x_154, 0); -lean_inc(x_159); -x_160 = lean_ctor_get(x_154, 1); -lean_inc(x_160); -lean_dec(x_154); -x_161 = l_Lean_Elab_isAbortTacticException(x_159); -if (x_161 == 0) +lean_object* x_163; lean_object* x_164; uint8_t x_165; +x_163 = lean_ctor_get(x_158, 0); +lean_inc(x_163); +x_164 = lean_ctor_get(x_158, 1); +lean_inc(x_164); +lean_dec(x_158); +x_165 = l_Lean_Elab_isAbortTacticException(x_163); +if (x_165 == 0) { -lean_dec(x_127); +lean_dec(x_130); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_29 = x_159; -x_30 = x_160; -goto block_52; +x_29 = x_163; +x_30 = x_164; +goto block_53; } else { -lean_object* x_162; lean_object* x_163; lean_object* x_164; -lean_dec(x_159); -x_162 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_153, x_127, x_3, x_4, x_5, x_6, x_7, x_8, x_160); +lean_object* x_166; lean_object* x_167; lean_object* x_168; +lean_dec(x_163); +x_166 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_157, x_130, x_3, x_4, x_5, x_6, x_7, x_8, x_164); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_163 = lean_ctor_get(x_162, 0); -lean_inc(x_163); -x_164 = lean_ctor_get(x_162, 1); -lean_inc(x_164); -lean_dec(x_162); -x_129 = x_163; -x_130 = x_164; -goto block_152; -} -} -block_152: -{ -lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; -x_131 = lean_st_ref_get(x_8, x_130); -x_132 = lean_ctor_get(x_131, 1); -lean_inc(x_132); -lean_dec(x_131); -x_133 = lean_st_ref_get(x_127, x_132); -lean_dec(x_127); -x_134 = lean_ctor_get(x_133, 1); -lean_inc(x_134); -lean_dec(x_133); -x_135 = lean_st_ref_get(x_8, x_134); +x_167 = lean_ctor_get(x_166, 0); +lean_inc(x_167); +x_168 = lean_ctor_get(x_166, 1); +lean_inc(x_168); +lean_dec(x_166); +x_132 = x_167; +x_133 = x_168; +goto block_156; +} +} +block_156: +{ +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; +x_134 = lean_st_ref_get(x_8, x_133); +x_135 = lean_ctor_get(x_134, 1); +lean_inc(x_135); +lean_dec(x_134); +x_136 = lean_st_ref_get(x_130, x_135); +lean_dec(x_130); +x_137 = lean_ctor_get(x_136, 1); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_st_ref_get(x_8, x_137); lean_dec(x_8); -x_136 = lean_ctor_get(x_135, 1); -lean_inc(x_136); -lean_dec(x_135); -x_137 = lean_st_ref_take(x_4, x_136); -x_138 = lean_ctor_get(x_137, 0); -lean_inc(x_138); -x_139 = lean_ctor_get(x_137, 1); +x_139 = lean_ctor_get(x_138, 1); lean_inc(x_139); -lean_dec(x_137); -x_140 = lean_ctor_get(x_138, 0); -lean_inc(x_140); -x_141 = lean_ctor_get(x_138, 2); +lean_dec(x_138); +x_140 = lean_st_ref_take(x_4, x_139); +x_141 = lean_ctor_get(x_140, 0); lean_inc(x_141); -x_142 = lean_ctor_get(x_138, 3); +x_142 = lean_ctor_get(x_140, 1); lean_inc(x_142); -x_143 = lean_ctor_get(x_138, 4); +lean_dec(x_140); +x_143 = lean_ctor_get(x_141, 0); lean_inc(x_143); -if (lean_is_exclusive(x_138)) { - lean_ctor_release(x_138, 0); - lean_ctor_release(x_138, 1); - lean_ctor_release(x_138, 2); - lean_ctor_release(x_138, 3); - lean_ctor_release(x_138, 4); - x_144 = x_138; +x_144 = lean_ctor_get(x_141, 1); +lean_inc(x_144); +x_145 = lean_ctor_get(x_141, 3); +lean_inc(x_145); +x_146 = lean_ctor_get(x_141, 4); +lean_inc(x_146); +x_147 = lean_ctor_get(x_141, 5); +lean_inc(x_147); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + lean_ctor_release(x_141, 2); + lean_ctor_release(x_141, 3); + lean_ctor_release(x_141, 4); + lean_ctor_release(x_141, 5); + x_148 = x_141; } else { - lean_dec_ref(x_138); - x_144 = lean_box(0); + lean_dec_ref(x_141); + x_148 = lean_box(0); } -if (lean_is_scalar(x_144)) { - x_145 = lean_alloc_ctor(0, 5, 0); +if (lean_is_scalar(x_148)) { + x_149 = lean_alloc_ctor(0, 6, 0); } else { - x_145 = x_144; + x_149 = x_148; } -lean_ctor_set(x_145, 0, x_140); -lean_ctor_set(x_145, 1, x_28); -lean_ctor_set(x_145, 2, x_141); -lean_ctor_set(x_145, 3, x_142); -lean_ctor_set(x_145, 4, x_143); -x_146 = lean_st_ref_set(x_4, x_145, x_139); +lean_ctor_set(x_149, 0, x_143); +lean_ctor_set(x_149, 1, x_144); +lean_ctor_set(x_149, 2, x_28); +lean_ctor_set(x_149, 3, x_145); +lean_ctor_set(x_149, 4, x_146); +lean_ctor_set(x_149, 5, x_147); +x_150 = lean_st_ref_set(x_4, x_149, x_142); lean_dec(x_4); -x_147 = lean_ctor_get(x_146, 1); -lean_inc(x_147); -if (lean_is_exclusive(x_146)) { - lean_ctor_release(x_146, 0); - lean_ctor_release(x_146, 1); - x_148 = x_146; +x_151 = lean_ctor_get(x_150, 1); +lean_inc(x_151); +if (lean_is_exclusive(x_150)) { + lean_ctor_release(x_150, 0); + lean_ctor_release(x_150, 1); + x_152 = x_150; } else { - lean_dec_ref(x_146); - x_148 = lean_box(0); -} -x_149 = lean_box(0); -x_150 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_150, 0, x_129); -lean_ctor_set(x_150, 1, x_149); -if (lean_is_scalar(x_148)) { - x_151 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_150); + x_152 = lean_box(0); +} +x_153 = lean_box(0); +x_154 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_154, 0, x_132); +lean_ctor_set(x_154, 1, x_153); +if (lean_is_scalar(x_152)) { + x_155 = lean_alloc_ctor(0, 2, 0); } else { - x_151 = x_148; + x_155 = x_152; } -lean_ctor_set(x_151, 0, x_150); -lean_ctor_set(x_151, 1, x_147); -x_10 = x_151; +lean_ctor_set(x_155, 0, x_154); +lean_ctor_set(x_155, 1, x_151); +x_10 = x_155; goto block_22; } } @@ -2385,7 +2437,7 @@ return x_21; } } } -block_52: +block_53: { lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; x_31 = lean_st_ref_get(x_8, x_30); @@ -2403,9 +2455,9 @@ x_36 = !lean_is_exclusive(x_34); if (x_36 == 0) { lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_37 = lean_ctor_get(x_34, 1); +x_37 = lean_ctor_get(x_34, 2); lean_dec(x_37); -lean_ctor_set(x_34, 1, x_28); +lean_ctor_set(x_34, 2, x_28); x_38 = lean_st_ref_set(x_4, x_34, x_35); lean_dec(x_4); x_39 = !lean_is_exclusive(x_38); @@ -2434,43 +2486,46 @@ goto block_22; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; x_43 = lean_ctor_get(x_34, 0); -x_44 = lean_ctor_get(x_34, 2); +x_44 = lean_ctor_get(x_34, 1); x_45 = lean_ctor_get(x_34, 3); x_46 = lean_ctor_get(x_34, 4); +x_47 = lean_ctor_get(x_34, 5); +lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); lean_dec(x_34); -x_47 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_47, 0, x_43); -lean_ctor_set(x_47, 1, x_28); -lean_ctor_set(x_47, 2, x_44); -lean_ctor_set(x_47, 3, x_45); -lean_ctor_set(x_47, 4, x_46); -x_48 = lean_st_ref_set(x_4, x_47, x_35); -lean_dec(x_4); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; +x_48 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_48, 0, x_43); +lean_ctor_set(x_48, 1, x_44); +lean_ctor_set(x_48, 2, x_28); +lean_ctor_set(x_48, 3, x_45); +lean_ctor_set(x_48, 4, x_46); +lean_ctor_set(x_48, 5, x_47); +x_49 = lean_st_ref_set(x_4, x_48, x_35); +lean_dec(x_4); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_51 = x_49; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_49); + x_51 = lean_box(0); } -if (lean_is_scalar(x_50)) { - x_51 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_51)) { + x_52 = lean_alloc_ctor(1, 2, 0); } else { - x_51 = x_50; - lean_ctor_set_tag(x_51, 1); + x_52 = x_51; + lean_ctor_set_tag(x_52, 1); } -lean_ctor_set(x_51, 0, x_29); -lean_ctor_set(x_51, 1, x_49); -x_10 = x_51; +lean_ctor_set(x_52, 0, x_29); +lean_ctor_set(x_52, 1, x_50); +x_10 = x_52; goto block_22; } } @@ -2564,25 +2619,24 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SavedState_restore(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SavedState_restore(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) { _start: { -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -x_12 = 0; -x_13 = l_Lean_Elab_Term_SavedState_restore(x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +x_13 = l_Lean_Elab_Term_SavedState_restore(x_12, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11); x_14 = lean_ctor_get(x_13, 1); lean_inc(x_14); lean_dec(x_13); x_15 = lean_ctor_get(x_1, 1); lean_inc(x_15); lean_dec(x_1); -x_16 = lean_st_ref_get(x_9, x_14); +x_16 = lean_st_ref_get(x_10, x_14); x_17 = lean_ctor_get(x_16, 1); lean_inc(x_17); lean_dec(x_16); -x_18 = lean_st_ref_set(x_3, x_15, x_17); +x_18 = lean_st_ref_set(x_4, x_15, x_17); x_19 = !lean_is_exclusive(x_18); if (x_19 == 0) { @@ -2603,11 +2657,14 @@ return x_22; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SavedState_restore___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SavedState_restore___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_11; -x_11 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_2); +lean_dec(x_2); +x_13 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -2615,8 +2672,7 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -return x_11; +return x_13; } } LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_getCurrMacroScope___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { @@ -3105,7 +3161,7 @@ lean_inc(x_10); x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); -x_12 = lean_ctor_get(x_10, 4); +x_12 = lean_ctor_get(x_10, 5); lean_inc(x_12); lean_dec(x_10); x_13 = lean_ctor_get(x_12, 1); @@ -3118,7 +3174,7 @@ lean_dec(x_14); x_16 = lean_st_ref_take(x_1, x_15); x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 4); +x_18 = lean_ctor_get(x_17, 5); lean_inc(x_18); x_19 = lean_ctor_get(x_16, 1); lean_inc(x_19); @@ -3127,7 +3183,7 @@ x_20 = !lean_is_exclusive(x_17); if (x_20 == 0) { lean_object* x_21; uint8_t x_22; -x_21 = lean_ctor_get(x_17, 4); +x_21 = lean_ctor_get(x_17, 5); lean_dec(x_21); x_22 = !lean_is_exclusive(x_18); if (x_22 == 0) @@ -3171,7 +3227,7 @@ x_33 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_33, 0, x_31); lean_ctor_set(x_33, 1, x_32); lean_ctor_set_uint8(x_33, sizeof(void*)*2, x_30); -lean_ctor_set(x_17, 4, x_33); +lean_ctor_set(x_17, 5, x_33); x_34 = lean_st_ref_set(x_1, x_17, x_19); x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); @@ -3195,61 +3251,64 @@ return x_37; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_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_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; x_38 = lean_ctor_get(x_17, 0); x_39 = lean_ctor_get(x_17, 1); x_40 = lean_ctor_get(x_17, 2); x_41 = lean_ctor_get(x_17, 3); +x_42 = lean_ctor_get(x_17, 4); +lean_inc(x_42); lean_inc(x_41); lean_inc(x_40); lean_inc(x_39); lean_inc(x_38); lean_dec(x_17); -x_42 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); -x_43 = lean_ctor_get(x_18, 0); -lean_inc(x_43); +x_43 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); +x_44 = lean_ctor_get(x_18, 0); +lean_inc(x_44); if (lean_is_exclusive(x_18)) { lean_ctor_release(x_18, 0); lean_ctor_release(x_18, 1); - x_44 = x_18; + x_45 = x_18; } else { lean_dec_ref(x_18); - x_44 = lean_box(0); + x_45 = lean_box(0); } -x_45 = l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___closed__3; -if (lean_is_scalar(x_44)) { - x_46 = lean_alloc_ctor(0, 2, 1); +x_46 = l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___closed__3; +if (lean_is_scalar(x_45)) { + x_47 = lean_alloc_ctor(0, 2, 1); } else { - x_46 = x_44; -} -lean_ctor_set(x_46, 0, x_43); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_42); -x_47 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_47, 0, x_38); -lean_ctor_set(x_47, 1, x_39); -lean_ctor_set(x_47, 2, x_40); -lean_ctor_set(x_47, 3, x_41); -lean_ctor_set(x_47, 4, x_46); -x_48 = lean_st_ref_set(x_1, x_47, x_19); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; + x_47 = x_45; +} +lean_ctor_set(x_47, 0, x_44); +lean_ctor_set(x_47, 1, x_46); +lean_ctor_set_uint8(x_47, sizeof(void*)*2, x_43); +x_48 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_48, 0, x_38); +lean_ctor_set(x_48, 1, x_39); +lean_ctor_set(x_48, 2, x_40); +lean_ctor_set(x_48, 3, x_41); +lean_ctor_set(x_48, 4, x_42); +lean_ctor_set(x_48, 5, x_47); +x_49 = lean_st_ref_set(x_1, x_48, x_19); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_51 = x_49; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_49); + x_51 = lean_box(0); } -if (lean_is_scalar(x_50)) { - x_51 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_51)) { + x_52 = lean_alloc_ctor(0, 2, 0); } else { - x_51 = x_50; + x_52 = x_51; } -lean_ctor_set(x_51, 0, x_13); -lean_ctor_set(x_51, 1, x_49); -return x_51; +lean_ctor_set(x_52, 0, x_13); +lean_ctor_set(x_52, 1, x_50); +return x_52; } } } @@ -3272,7 +3331,7 @@ lean_dec(x_12); x_14 = lean_st_ref_get(x_6, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 4); +x_16 = lean_ctor_get(x_15, 5); lean_inc(x_16); lean_dec(x_15); x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); @@ -3326,7 +3385,7 @@ lean_inc(x_30); x_31 = lean_ctor_get(x_29, 1); lean_inc(x_31); lean_dec(x_29); -x_32 = lean_ctor_get(x_30, 4); +x_32 = lean_ctor_get(x_30, 5); lean_inc(x_32); lean_dec(x_30); x_33 = lean_ctor_get(x_32, 1); @@ -3351,7 +3410,7 @@ lean_dec(x_37); x_39 = lean_st_ref_take(x_6, x_38); x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 4); +x_41 = lean_ctor_get(x_40, 5); lean_inc(x_41); x_42 = lean_ctor_get(x_39, 1); lean_inc(x_42); @@ -3360,7 +3419,7 @@ x_43 = !lean_is_exclusive(x_40); if (x_43 == 0) { lean_object* x_44; uint8_t x_45; -x_44 = lean_ctor_get(x_40, 4); +x_44 = lean_ctor_get(x_40, 5); lean_dec(x_44); x_45 = !lean_is_exclusive(x_41); if (x_45 == 0) @@ -3405,7 +3464,7 @@ x_56 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_56, 0, x_54); lean_ctor_set(x_56, 1, x_55); lean_ctor_set_uint8(x_56, sizeof(void*)*2, x_53); -lean_ctor_set(x_40, 4, x_56); +lean_ctor_set(x_40, 5, x_56); x_57 = lean_st_ref_set(x_6, x_40, x_42); lean_dec(x_6); x_58 = lean_ctor_get(x_57, 1); @@ -3430,298 +3489,304 @@ return x_60; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; x_61 = lean_ctor_get(x_40, 0); x_62 = lean_ctor_get(x_40, 1); x_63 = lean_ctor_get(x_40, 2); x_64 = lean_ctor_get(x_40, 3); +x_65 = lean_ctor_get(x_40, 4); +lean_inc(x_65); lean_inc(x_64); lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_dec(x_40); -x_65 = lean_ctor_get_uint8(x_41, sizeof(void*)*2); -x_66 = lean_ctor_get(x_41, 0); -lean_inc(x_66); +x_66 = lean_ctor_get_uint8(x_41, sizeof(void*)*2); +x_67 = lean_ctor_get(x_41, 0); +lean_inc(x_67); if (lean_is_exclusive(x_41)) { lean_ctor_release(x_41, 0); lean_ctor_release(x_41, 1); - x_67 = x_41; + x_68 = x_41; } else { lean_dec_ref(x_41); - x_67 = lean_box(0); + x_68 = lean_box(0); } -x_68 = l_Std_PersistentArray_push___rarg(x_22, x_35); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 1); +x_69 = l_Std_PersistentArray_push___rarg(x_22, x_35); +if (lean_is_scalar(x_68)) { + x_70 = lean_alloc_ctor(0, 2, 1); } else { - x_69 = x_67; -} -lean_ctor_set(x_69, 0, x_66); -lean_ctor_set(x_69, 1, x_68); -lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_65); -x_70 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_70, 0, x_61); -lean_ctor_set(x_70, 1, x_62); -lean_ctor_set(x_70, 2, x_63); -lean_ctor_set(x_70, 3, x_64); -lean_ctor_set(x_70, 4, x_69); -x_71 = lean_st_ref_set(x_6, x_70, x_42); -lean_dec(x_6); -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_73 = x_71; + x_70 = x_68; +} +lean_ctor_set(x_70, 0, x_67); +lean_ctor_set(x_70, 1, x_69); +lean_ctor_set_uint8(x_70, sizeof(void*)*2, x_66); +x_71 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_71, 0, x_61); +lean_ctor_set(x_71, 1, x_62); +lean_ctor_set(x_71, 2, x_63); +lean_ctor_set(x_71, 3, x_64); +lean_ctor_set(x_71, 4, x_65); +lean_ctor_set(x_71, 5, x_70); +x_72 = lean_st_ref_set(x_6, x_71, x_42); +lean_dec(x_6); +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_74 = x_72; } else { - lean_dec_ref(x_71); - x_73 = lean_box(0); + lean_dec_ref(x_72); + x_74 = lean_box(0); } -if (lean_is_scalar(x_73)) { - x_74 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(0, 2, 0); } else { - x_74 = x_73; + x_75 = x_74; } -lean_ctor_set(x_74, 0, x_25); -lean_ctor_set(x_74, 1, x_72); -return x_74; +lean_ctor_set(x_75, 0, x_25); +lean_ctor_set(x_75, 1, x_73); +return x_75; } } else { -uint8_t x_75; +uint8_t x_76; lean_dec(x_25); lean_dec(x_22); lean_dec(x_10); lean_dec(x_6); -x_75 = !lean_is_exclusive(x_34); -if (x_75 == 0) +x_76 = !lean_is_exclusive(x_34); +if (x_76 == 0) { return x_34; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_34, 0); -x_77 = lean_ctor_get(x_34, 1); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_34, 0); +x_78 = lean_ctor_get(x_34, 1); +lean_inc(x_78); lean_inc(x_77); -lean_inc(x_76); lean_dec(x_34); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_79 = lean_ctor_get(x_24, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_24, 1); +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_80 = lean_ctor_get(x_24, 0); lean_inc(x_80); +x_81 = lean_ctor_get(x_24, 1); +lean_inc(x_81); lean_dec(x_24); -x_81 = lean_st_ref_get(x_10, x_80); -x_82 = lean_ctor_get(x_81, 1); -lean_inc(x_82); -lean_dec(x_81); -x_83 = lean_st_ref_get(x_6, x_82); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +x_82 = lean_st_ref_get(x_10, x_81); +x_83 = lean_ctor_get(x_82, 1); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_st_ref_get(x_6, x_83); +x_85 = lean_ctor_get(x_84, 0); lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_ctor_get(x_84, 4); +x_86 = lean_ctor_get(x_84, 1); lean_inc(x_86); lean_dec(x_84); -x_87 = lean_ctor_get(x_86, 1); +x_87 = lean_ctor_get(x_85, 5); lean_inc(x_87); -lean_dec(x_86); +lean_dec(x_85); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); lean_inc(x_10); lean_inc(x_6); -x_88 = lean_apply_10(x_2, x_87, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_85); -if (lean_obj_tag(x_88) == 0) +x_89 = lean_apply_10(x_2, x_88, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_86); +if (lean_obj_tag(x_89) == 0) { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_88, 1); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_90 = lean_ctor_get(x_89, 0); lean_inc(x_90); -lean_dec(x_88); -x_91 = lean_st_ref_get(x_10, x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = lean_st_ref_get(x_10, x_91); lean_dec(x_10); -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); -lean_dec(x_91); -x_93 = lean_st_ref_take(x_6, x_92); -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_94, 4); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +x_94 = lean_st_ref_take(x_6, x_93); +x_95 = lean_ctor_get(x_94, 0); lean_inc(x_95); -x_96 = lean_ctor_get(x_93, 1); +x_96 = lean_ctor_get(x_95, 5); lean_inc(x_96); -lean_dec(x_93); -x_97 = !lean_is_exclusive(x_94); -if (x_97 == 0) -{ -lean_object* x_98; uint8_t x_99; -x_98 = lean_ctor_get(x_94, 4); -lean_dec(x_98); -x_99 = !lean_is_exclusive(x_95); -if (x_99 == 0) -{ -lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; -x_100 = lean_ctor_get(x_95, 1); -lean_dec(x_100); -x_101 = l_Std_PersistentArray_push___rarg(x_22, x_89); -lean_ctor_set(x_95, 1, x_101); -x_102 = lean_st_ref_set(x_6, x_94, x_96); -lean_dec(x_6); -x_103 = !lean_is_exclusive(x_102); -if (x_103 == 0) -{ -lean_object* x_104; -x_104 = lean_ctor_get(x_102, 0); -lean_dec(x_104); -lean_ctor_set_tag(x_102, 1); -lean_ctor_set(x_102, 0, x_79); -return x_102; -} -else -{ -lean_object* x_105; lean_object* x_106; -x_105 = lean_ctor_get(x_102, 1); -lean_inc(x_105); -lean_dec(x_102); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_79); -lean_ctor_set(x_106, 1, x_105); -return x_106; +x_97 = lean_ctor_get(x_94, 1); +lean_inc(x_97); +lean_dec(x_94); +x_98 = !lean_is_exclusive(x_95); +if (x_98 == 0) +{ +lean_object* x_99; uint8_t x_100; +x_99 = lean_ctor_get(x_95, 5); +lean_dec(x_99); +x_100 = !lean_is_exclusive(x_96); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; +x_101 = lean_ctor_get(x_96, 1); +lean_dec(x_101); +x_102 = l_Std_PersistentArray_push___rarg(x_22, x_90); +lean_ctor_set(x_96, 1, x_102); +x_103 = lean_st_ref_set(x_6, x_95, x_97); +lean_dec(x_6); +x_104 = !lean_is_exclusive(x_103); +if (x_104 == 0) +{ +lean_object* x_105; +x_105 = lean_ctor_get(x_103, 0); +lean_dec(x_105); +lean_ctor_set_tag(x_103, 1); +lean_ctor_set(x_103, 0, x_80); +return x_103; +} +else +{ +lean_object* x_106; lean_object* x_107; +x_106 = lean_ctor_get(x_103, 1); +lean_inc(x_106); +lean_dec(x_103); +x_107 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_107, 0, x_80); +lean_ctor_set(x_107, 1, x_106); +return x_107; } } else { -uint8_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_107 = lean_ctor_get_uint8(x_95, sizeof(void*)*2); -x_108 = lean_ctor_get(x_95, 0); -lean_inc(x_108); -lean_dec(x_95); -x_109 = l_Std_PersistentArray_push___rarg(x_22, x_89); -x_110 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -lean_ctor_set_uint8(x_110, sizeof(void*)*2, x_107); -lean_ctor_set(x_94, 4, x_110); -x_111 = lean_st_ref_set(x_6, x_94, x_96); -lean_dec(x_6); -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_113 = x_111; +uint8_t x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_108 = lean_ctor_get_uint8(x_96, sizeof(void*)*2); +x_109 = lean_ctor_get(x_96, 0); +lean_inc(x_109); +lean_dec(x_96); +x_110 = l_Std_PersistentArray_push___rarg(x_22, x_90); +x_111 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +lean_ctor_set_uint8(x_111, sizeof(void*)*2, x_108); +lean_ctor_set(x_95, 5, x_111); +x_112 = lean_st_ref_set(x_6, x_95, x_97); +lean_dec(x_6); +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_114 = x_112; } else { - lean_dec_ref(x_111); - x_113 = lean_box(0); + lean_dec_ref(x_112); + x_114 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; - lean_ctor_set_tag(x_114, 1); + x_115 = x_114; + lean_ctor_set_tag(x_115, 1); } -lean_ctor_set(x_114, 0, x_79); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_115, 0, x_80); +lean_ctor_set(x_115, 1, x_113); +return x_115; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_115 = lean_ctor_get(x_94, 0); -x_116 = lean_ctor_get(x_94, 1); -x_117 = lean_ctor_get(x_94, 2); -x_118 = lean_ctor_get(x_94, 3); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; uint8_t x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_116 = lean_ctor_get(x_95, 0); +x_117 = lean_ctor_get(x_95, 1); +x_118 = lean_ctor_get(x_95, 2); +x_119 = lean_ctor_get(x_95, 3); +x_120 = lean_ctor_get(x_95, 4); +lean_inc(x_120); +lean_inc(x_119); lean_inc(x_118); lean_inc(x_117); lean_inc(x_116); -lean_inc(x_115); -lean_dec(x_94); -x_119 = lean_ctor_get_uint8(x_95, sizeof(void*)*2); -x_120 = lean_ctor_get(x_95, 0); -lean_inc(x_120); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_121 = x_95; +lean_dec(x_95); +x_121 = lean_ctor_get_uint8(x_96, sizeof(void*)*2); +x_122 = lean_ctor_get(x_96, 0); +lean_inc(x_122); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_123 = x_96; } else { - lean_dec_ref(x_95); - x_121 = lean_box(0); + lean_dec_ref(x_96); + x_123 = lean_box(0); } -x_122 = l_Std_PersistentArray_push___rarg(x_22, x_89); -if (lean_is_scalar(x_121)) { - x_123 = lean_alloc_ctor(0, 2, 1); +x_124 = l_Std_PersistentArray_push___rarg(x_22, x_90); +if (lean_is_scalar(x_123)) { + x_125 = lean_alloc_ctor(0, 2, 1); } else { - x_123 = x_121; + x_125 = x_123; } -lean_ctor_set(x_123, 0, x_120); -lean_ctor_set(x_123, 1, x_122); -lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_119); -x_124 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_124, 0, x_115); -lean_ctor_set(x_124, 1, x_116); -lean_ctor_set(x_124, 2, x_117); -lean_ctor_set(x_124, 3, x_118); -lean_ctor_set(x_124, 4, x_123); -x_125 = lean_st_ref_set(x_6, x_124, x_96); -lean_dec(x_6); -x_126 = lean_ctor_get(x_125, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - x_127 = x_125; +lean_ctor_set(x_125, 0, x_122); +lean_ctor_set(x_125, 1, x_124); +lean_ctor_set_uint8(x_125, sizeof(void*)*2, x_121); +x_126 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_126, 0, x_116); +lean_ctor_set(x_126, 1, x_117); +lean_ctor_set(x_126, 2, x_118); +lean_ctor_set(x_126, 3, x_119); +lean_ctor_set(x_126, 4, x_120); +lean_ctor_set(x_126, 5, x_125); +x_127 = lean_st_ref_set(x_6, x_126, x_97); +lean_dec(x_6); +x_128 = lean_ctor_get(x_127, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_129 = x_127; } else { - lean_dec_ref(x_125); - x_127 = lean_box(0); + lean_dec_ref(x_127); + x_129 = lean_box(0); } -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(1, 2, 0); } else { - x_128 = x_127; - lean_ctor_set_tag(x_128, 1); + x_130 = x_129; + lean_ctor_set_tag(x_130, 1); } -lean_ctor_set(x_128, 0, x_79); -lean_ctor_set(x_128, 1, x_126); -return x_128; +lean_ctor_set(x_130, 0, x_80); +lean_ctor_set(x_130, 1, x_128); +return x_130; } } else { -uint8_t x_129; -lean_dec(x_79); +uint8_t x_131; +lean_dec(x_80); lean_dec(x_22); lean_dec(x_10); lean_dec(x_6); -x_129 = !lean_is_exclusive(x_88); -if (x_129 == 0) +x_131 = !lean_is_exclusive(x_89); +if (x_131 == 0) { -return x_88; +return x_89; } else { -lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_130 = lean_ctor_get(x_88, 0); -x_131 = lean_ctor_get(x_88, 1); -lean_inc(x_131); -lean_inc(x_130); -lean_dec(x_88); -x_132 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); -return x_132; +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_89, 0); +x_133 = lean_ctor_get(x_89, 1); +lean_inc(x_133); +lean_inc(x_132); +lean_dec(x_89); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; } } } @@ -3845,7 +3910,7 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -3883,7 +3948,7 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; @@ -3896,7 +3961,7 @@ x_14 = l_Lean_replaceRef(x_1, x_13); lean_dec(x_13); lean_dec(x_1); lean_ctor_set(x_9, 5, x_14); -x_15 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3948,7 +4013,7 @@ lean_ctor_set(x_28, 7, x_23); lean_ctor_set(x_28, 8, x_24); lean_ctor_set(x_28, 9, x_25); lean_ctor_set(x_28, 10, x_26); -x_29 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); +x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); lean_dec(x_10); lean_dec(x_28); lean_dec(x_8); @@ -3961,46 +4026,1094 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +static lean_object* _init_l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1() { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_12 = lean_st_ref_get(x_10, x_11); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = lean_st_ref_get(x_6, x_13); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 4); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); -lean_dec(x_16); -if (x_17 == 0) +lean_object* x_1; +x_1 = l_Lean_Elab_abortTacticExceptionId; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__2() { +_start: { -lean_object* x_18; lean_object* x_19; -lean_dec(x_2); -x_18 = lean_ctor_get(x_14, 1); -lean_inc(x_18); -lean_dec(x_14); -x_19 = lean_apply_9(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); -return x_19; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg(lean_object* x_1) { +_start: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); -lean_dec(x_14); -x_21 = l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg(x_6, x_7, x_8, x_9, x_10, x_20); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -lean_inc(x_10); -lean_inc(x_9); +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__2; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg), 1, 0); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__5(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) +{ +lean_object* x_6; size_t x_7; size_t x_8; +x_6 = lean_array_uget(x_1, x_2); +x_7 = 1; +x_8 = lean_usize_add(x_2, x_7); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_6, 0); +lean_inc(x_9); +lean_dec(x_6); +x_10 = lean_array_push(x_4, x_9); +x_2 = x_8; +x_4 = x_10; +goto _start; +} +else +{ +lean_dec(x_6); +x_2 = x_8; +goto _start; +} +} +else +{ +return x_4; +} +} +} +static lean_object* _init_l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_nat_dec_lt(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; +lean_dec(x_3); +lean_dec(x_2); +x_5 = l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1; +return x_5; +} +else +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_get_size(x_1); +x_7 = lean_nat_dec_le(x_3, x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +lean_object* x_8; +lean_dec(x_3); +lean_dec(x_2); +x_8 = l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1; +return x_8; +} +else +{ +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_usize_of_nat(x_2); +lean_dec(x_2); +x_10 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_11 = l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1; +x_12 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__5(x_1, x_9, x_10, x_11); +return x_12; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; lean_object* x_6; +x_4 = lean_ctor_get(x_1, 5); +x_5 = 0; +x_6 = l_Lean_Syntax_getPos_x3f(x_4, x_5); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_3); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_6, 0); +lean_inc(x_9); +lean_dec(x_6); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_3); +return x_10; +} +} +} +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = lean_alloc_closure((void*)(l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___rarg___boxed), 3, 0); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(":", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(" ", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; +x_11 = l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___rarg(x_8, x_9, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_11, 0); +x_14 = l_Lean_Exception_getRef(x_1); +x_15 = 0; +x_16 = l_Lean_Syntax_getPos_x3f(x_14, x_15); +lean_dec(x_14); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; +lean_dec(x_13); +x_17 = l_Lean_Exception_toMessageData(x_1); +lean_ctor_set(x_11, 0, x_17); +return x_11; +} +else +{ +lean_object* x_18; uint8_t x_19; +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_nat_dec_eq(x_13, x_18); +lean_dec(x_13); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_20 = lean_ctor_get(x_8, 1); +x_21 = l_Lean_FileMap_toPosition(x_20, x_18); +lean_dec(x_18); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = l_Nat_repr(x_22); +x_24 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_24, 0, x_23); +x_25 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; +x_27 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +x_28 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__2; +x_29 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +x_30 = lean_ctor_get(x_21, 1); +lean_inc(x_30); +lean_dec(x_21); +x_31 = l_Nat_repr(x_30); +x_32 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_32, 0, x_31); +x_33 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_33, 0, x_32); +x_34 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_34, 0, x_29); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__4; +x_36 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +x_37 = l_Lean_Exception_toMessageData(x_1); +x_38 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_26); +lean_ctor_set(x_11, 0, x_39); +return x_11; +} +else +{ +lean_object* x_40; +lean_dec(x_18); +x_40 = l_Lean_Exception_toMessageData(x_1); +lean_ctor_set(x_11, 0, x_40); +return x_11; +} +} +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; +x_41 = lean_ctor_get(x_11, 0); +x_42 = lean_ctor_get(x_11, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_11); +x_43 = l_Lean_Exception_getRef(x_1); +x_44 = 0; +x_45 = l_Lean_Syntax_getPos_x3f(x_43, x_44); +lean_dec(x_43); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; lean_object* x_47; +lean_dec(x_41); +x_46 = l_Lean_Exception_toMessageData(x_1); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_42); +return x_47; +} +else +{ +lean_object* x_48; uint8_t x_49; +x_48 = lean_ctor_get(x_45, 0); +lean_inc(x_48); +lean_dec(x_45); +x_49 = lean_nat_dec_eq(x_41, x_48); +lean_dec(x_41); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_50 = lean_ctor_get(x_8, 1); +x_51 = l_Lean_FileMap_toPosition(x_50, x_48); +lean_dec(x_48); +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +x_53 = l_Nat_repr(x_52); +x_54 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_54, 0, x_53); +x_55 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_55, 0, x_54); +x_56 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; +x_57 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_55); +x_58 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__2; +x_59 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +x_60 = lean_ctor_get(x_51, 1); +lean_inc(x_60); +lean_dec(x_51); +x_61 = l_Nat_repr(x_60); +x_62 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_62, 0, x_61); +x_63 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_63, 0, x_62); +x_64 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_64, 0, x_59); +lean_ctor_set(x_64, 1, x_63); +x_65 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__4; +x_66 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = l_Lean_Exception_toMessageData(x_1); +x_68 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +x_69 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_56); +x_70 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_42); +return x_70; +} +else +{ +lean_object* x_71; lean_object* x_72; +lean_dec(x_48); +x_71 = l_Lean_Exception_toMessageData(x_1); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_42); +return x_72; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__9(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_2, x_1); +if (x_13 == 0) +{ +lean_object* x_14; +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_3); +lean_ctor_set(x_14, 1, x_12); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; +x_15 = lean_array_uget(x_3, x_2); +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_array_uset(x_3, x_2, x_16); +x_18 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7(x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = 1; +x_22 = lean_usize_add(x_2, x_21); +x_23 = lean_array_uset(x_17, x_2, x_19); +x_2 = x_22; +x_3 = x_23; +x_12 = x_20; +goto _start; +} +} +} +static lean_object* _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(", errors ", 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_12 = lean_array_get_size(x_2); +x_13 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_14 = 0; +x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__9(x_13, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; +x_19 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_1); +x_20 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__2; +x_21 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = l_Lean_toMessageList(x_16); +x_23 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_18); +x_25 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_25; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__10(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_inc(x_5); +return x_5; +} +else +{ +lean_object* x_7; +x_7 = lean_array_uget(x_2, x_4); +if (lean_obj_tag(x_7) == 0) +{ +size_t x_8; size_t x_9; +lean_dec(x_7); +x_8 = 1; +x_9 = lean_usize_add(x_4, x_8); +{ +size_t _tmp_3 = x_9; +lean_object* _tmp_4 = x_1; +x_4 = _tmp_3; +x_5 = _tmp_4; +} +goto _start; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_7); +x_12 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_12, 0, x_11); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___lambda__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_box(0); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("unexpected syntax ", 18); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("tactic failed", 13); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__3; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__4; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = lean_box(0); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic_throwExs___lambda__1___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__7; +x_2 = lean_box(0); +x_3 = lean_apply_1(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_21; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_35 = lean_array_get_size(x_2); +x_36 = lean_unsigned_to_nat(0u); +lean_inc(x_35); +x_37 = l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4(x_2, x_36, x_35); +x_38 = l_Array_isEmpty___rarg(x_37); +if (x_38 == 0) +{ +lean_object* x_39; uint8_t x_40; +lean_dec(x_35); +lean_dec(x_2); +x_39 = lean_array_get_size(x_37); +x_40 = lean_nat_dec_lt(x_36, x_39); +lean_dec(x_39); +if (x_40 == 0) +{ +uint8_t x_41; +x_41 = !lean_is_exclusive(x_9); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_42 = lean_ctor_get(x_9, 5); +x_43 = l_Lean_replaceRef(x_1, x_42); +lean_dec(x_42); +lean_dec(x_1); +lean_ctor_set(x_9, 5, x_43); +x_44 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__5; +x_45 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6(x_44, x_37, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_45; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_46 = lean_ctor_get(x_9, 0); +x_47 = lean_ctor_get(x_9, 1); +x_48 = lean_ctor_get(x_9, 2); +x_49 = lean_ctor_get(x_9, 3); +x_50 = lean_ctor_get(x_9, 4); +x_51 = lean_ctor_get(x_9, 5); +x_52 = lean_ctor_get(x_9, 6); +x_53 = lean_ctor_get(x_9, 7); +x_54 = lean_ctor_get(x_9, 8); +x_55 = lean_ctor_get(x_9, 9); +x_56 = lean_ctor_get(x_9, 10); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_9); +x_57 = l_Lean_replaceRef(x_1, x_51); +lean_dec(x_51); +lean_dec(x_1); +x_58 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_58, 0, x_46); +lean_ctor_set(x_58, 1, x_47); +lean_ctor_set(x_58, 2, x_48); +lean_ctor_set(x_58, 3, x_49); +lean_ctor_set(x_58, 4, x_50); +lean_ctor_set(x_58, 5, x_57); +lean_ctor_set(x_58, 6, x_52); +lean_ctor_set(x_58, 7, x_53); +lean_ctor_set(x_58, 8, x_54); +lean_ctor_set(x_58, 9, x_55); +lean_ctor_set(x_58, 10, x_56); +x_59 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__5; +x_60 = l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6(x_59, x_37, x_3, x_4, x_5, x_6, x_7, x_8, x_58, x_10, x_11); +return x_60; +} +} +else +{ +lean_object* x_61; lean_object* x_62; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_61 = lean_array_fget(x_37, x_36); +lean_dec(x_37); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_11); +return x_62; +} +} +else +{ +size_t x_63; size_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_dec(x_37); +x_63 = lean_usize_of_nat(x_35); +lean_dec(x_35); +x_64 = 0; +x_65 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__6; +x_66 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__10(x_65, x_2, x_63, x_64, x_65); +lean_dec(x_2); +x_67 = lean_ctor_get(x_66, 0); +lean_inc(x_67); +lean_dec(x_66); +if (lean_obj_tag(x_67) == 0) +{ +lean_object* x_68; +x_68 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__8; +if (lean_obj_tag(x_68) == 0) +{ +lean_object* x_69; +x_69 = lean_box(0); +x_12 = x_69; +goto block_20; +} +else +{ +lean_object* x_70; +x_70 = lean_ctor_get(x_68, 0); +lean_inc(x_70); +x_21 = x_70; +goto block_34; +} +} +else +{ +lean_object* x_71; +x_71 = lean_ctor_get(x_67, 0); +lean_inc(x_71); +lean_dec(x_67); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; +x_72 = lean_box(0); +x_12 = x_72; +goto block_20; +} +else +{ +lean_object* x_73; +x_73 = lean_ctor_get(x_71, 0); +lean_inc(x_73); +lean_dec(x_71); +x_21 = x_73; +goto block_34; +} +} +} +block_20: +{ +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_dec(x_12); +lean_inc(x_1); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_1); +x_14 = l_Lean_indentD(x_13); +x_15 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__2; +x_16 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +x_17 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; +x_18 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__1(x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_19; +} +block_34: +{ +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_dec(x_21); +lean_inc(x_1); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_1); +x_23 = l_Lean_indentD(x_22); +x_24 = l_Lean_Elab_Tactic_evalTactic_throwExs___closed__2; +x_25 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +x_26 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; +x_27 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__1(x_1, x_27, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_28; +} +else +{ +lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_1); +x_29 = lean_ctor_get(x_21, 0); +lean_inc(x_29); +lean_dec(x_21); +x_30 = 1; +x_31 = l_Lean_Elab_Tactic_SavedState_restore(x_29, x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +lean_dec(x_31); +x_33 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg(x_32); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__5(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___rarg(x_1, x_2, x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_getRefPos___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__8(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_14 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_15 = l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__9(x_13, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__10(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_throwExs___lambda__1___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Elab_Tactic_evalTactic_throwExs___lambda__1(x_1); +lean_dec(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_unsupportedSyntaxExceptionId; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_handleEx(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = 1; +x_15 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_17, 0, x_3); +x_18 = lean_array_push(x_2, x_17); +x_19 = lean_apply_10(x_4, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_ctor_get(x_3, 0); +lean_inc(x_20); +x_21 = l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1; +x_22 = lean_nat_dec_eq(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; uint8_t x_24; +x_23 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1; +x_24 = lean_nat_dec_eq(x_20, x_23); +lean_dec(x_20); +if (x_24 == 0) +{ +lean_object* x_25; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_3); +lean_ctor_set(x_25, 1, x_13); +return x_25; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_3); +x_26 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_27); +x_30 = lean_array_push(x_2, x_29); +x_31 = 1; +x_32 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_28); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = lean_apply_10(x_4, x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_33); +return x_34; +} +} +else +{ +uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_20); +lean_dec(x_3); +x_35 = 1; +x_36 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_37 = lean_ctor_get(x_36, 1); +lean_inc(x_37); +lean_dec(x_36); +x_38 = lean_apply_10(x_4, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_37); +return x_38; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_12 = lean_st_ref_get(x_10, x_11); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_st_ref_get(x_6, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 5); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_2); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +x_19 = lean_apply_9(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_20 = lean_ctor_get(x_14, 1); +lean_inc(x_20); +lean_dec(x_14); +x_21 = l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg(x_6, x_7, x_8, x_9, x_10, x_20); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +lean_inc(x_10); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); @@ -4026,7 +5139,7 @@ lean_inc(x_30); x_31 = lean_ctor_get(x_29, 1); lean_inc(x_31); lean_dec(x_29); -x_32 = lean_ctor_get(x_30, 4); +x_32 = lean_ctor_get(x_30, 5); lean_inc(x_32); lean_dec(x_30); x_33 = lean_ctor_get(x_32, 1); @@ -4051,7 +5164,7 @@ lean_dec(x_37); x_39 = lean_st_ref_take(x_6, x_38); x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 4); +x_41 = lean_ctor_get(x_40, 5); lean_inc(x_41); x_42 = lean_ctor_get(x_39, 1); lean_inc(x_42); @@ -4060,7 +5173,7 @@ x_43 = !lean_is_exclusive(x_40); if (x_43 == 0) { lean_object* x_44; uint8_t x_45; -x_44 = lean_ctor_get(x_40, 4); +x_44 = lean_ctor_get(x_40, 5); lean_dec(x_44); x_45 = !lean_is_exclusive(x_41); if (x_45 == 0) @@ -4105,7 +5218,7 @@ x_56 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_56, 0, x_54); lean_ctor_set(x_56, 1, x_55); lean_ctor_set_uint8(x_56, sizeof(void*)*2, x_53); -lean_ctor_set(x_40, 4, x_56); +lean_ctor_set(x_40, 5, x_56); x_57 = lean_st_ref_set(x_6, x_40, x_42); lean_dec(x_6); x_58 = lean_ctor_get(x_57, 1); @@ -4130,415 +5243,363 @@ return x_60; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; x_61 = lean_ctor_get(x_40, 0); x_62 = lean_ctor_get(x_40, 1); x_63 = lean_ctor_get(x_40, 2); x_64 = lean_ctor_get(x_40, 3); +x_65 = lean_ctor_get(x_40, 4); +lean_inc(x_65); lean_inc(x_64); lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_dec(x_40); -x_65 = lean_ctor_get_uint8(x_41, sizeof(void*)*2); -x_66 = lean_ctor_get(x_41, 0); -lean_inc(x_66); +x_66 = lean_ctor_get_uint8(x_41, sizeof(void*)*2); +x_67 = lean_ctor_get(x_41, 0); +lean_inc(x_67); if (lean_is_exclusive(x_41)) { lean_ctor_release(x_41, 0); lean_ctor_release(x_41, 1); - x_67 = x_41; + x_68 = x_41; } else { lean_dec_ref(x_41); - x_67 = lean_box(0); + x_68 = lean_box(0); } -x_68 = l_Std_PersistentArray_push___rarg(x_22, x_35); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 1); +x_69 = l_Std_PersistentArray_push___rarg(x_22, x_35); +if (lean_is_scalar(x_68)) { + x_70 = lean_alloc_ctor(0, 2, 1); } else { - x_69 = x_67; -} -lean_ctor_set(x_69, 0, x_66); -lean_ctor_set(x_69, 1, x_68); -lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_65); -x_70 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_70, 0, x_61); -lean_ctor_set(x_70, 1, x_62); -lean_ctor_set(x_70, 2, x_63); -lean_ctor_set(x_70, 3, x_64); -lean_ctor_set(x_70, 4, x_69); -x_71 = lean_st_ref_set(x_6, x_70, x_42); -lean_dec(x_6); -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_73 = x_71; + x_70 = x_68; +} +lean_ctor_set(x_70, 0, x_67); +lean_ctor_set(x_70, 1, x_69); +lean_ctor_set_uint8(x_70, sizeof(void*)*2, x_66); +x_71 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_71, 0, x_61); +lean_ctor_set(x_71, 1, x_62); +lean_ctor_set(x_71, 2, x_63); +lean_ctor_set(x_71, 3, x_64); +lean_ctor_set(x_71, 4, x_65); +lean_ctor_set(x_71, 5, x_70); +x_72 = lean_st_ref_set(x_6, x_71, x_42); +lean_dec(x_6); +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_74 = x_72; } else { - lean_dec_ref(x_71); - x_73 = lean_box(0); + lean_dec_ref(x_72); + x_74 = lean_box(0); } -if (lean_is_scalar(x_73)) { - x_74 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(0, 2, 0); } else { - x_74 = x_73; + x_75 = x_74; } -lean_ctor_set(x_74, 0, x_25); -lean_ctor_set(x_74, 1, x_72); -return x_74; +lean_ctor_set(x_75, 0, x_25); +lean_ctor_set(x_75, 1, x_73); +return x_75; } } else { -uint8_t x_75; +uint8_t x_76; lean_dec(x_25); lean_dec(x_22); lean_dec(x_10); lean_dec(x_6); -x_75 = !lean_is_exclusive(x_34); -if (x_75 == 0) +x_76 = !lean_is_exclusive(x_34); +if (x_76 == 0) { return x_34; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_34, 0); -x_77 = lean_ctor_get(x_34, 1); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_34, 0); +x_78 = lean_ctor_get(x_34, 1); +lean_inc(x_78); lean_inc(x_77); -lean_inc(x_76); lean_dec(x_34); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_79 = lean_ctor_get(x_24, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_24, 1); +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_80 = lean_ctor_get(x_24, 0); lean_inc(x_80); +x_81 = lean_ctor_get(x_24, 1); +lean_inc(x_81); lean_dec(x_24); -x_81 = lean_st_ref_get(x_10, x_80); -x_82 = lean_ctor_get(x_81, 1); -lean_inc(x_82); -lean_dec(x_81); -x_83 = lean_st_ref_get(x_6, x_82); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +x_82 = lean_st_ref_get(x_10, x_81); +x_83 = lean_ctor_get(x_82, 1); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_st_ref_get(x_6, x_83); +x_85 = lean_ctor_get(x_84, 0); lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_ctor_get(x_84, 4); +x_86 = lean_ctor_get(x_84, 1); lean_inc(x_86); lean_dec(x_84); -x_87 = lean_ctor_get(x_86, 1); +x_87 = lean_ctor_get(x_85, 5); lean_inc(x_87); -lean_dec(x_86); +lean_dec(x_85); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); lean_inc(x_10); lean_inc(x_6); -x_88 = lean_apply_10(x_2, x_87, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_85); -if (lean_obj_tag(x_88) == 0) +x_89 = lean_apply_10(x_2, x_88, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_86); +if (lean_obj_tag(x_89) == 0) { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_88, 1); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_90 = lean_ctor_get(x_89, 0); lean_inc(x_90); -lean_dec(x_88); -x_91 = lean_st_ref_get(x_10, x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = lean_st_ref_get(x_10, x_91); lean_dec(x_10); -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); -lean_dec(x_91); -x_93 = lean_st_ref_take(x_6, x_92); -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_94, 4); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +x_94 = lean_st_ref_take(x_6, x_93); +x_95 = lean_ctor_get(x_94, 0); lean_inc(x_95); -x_96 = lean_ctor_get(x_93, 1); +x_96 = lean_ctor_get(x_95, 5); lean_inc(x_96); -lean_dec(x_93); -x_97 = !lean_is_exclusive(x_94); -if (x_97 == 0) -{ -lean_object* x_98; uint8_t x_99; -x_98 = lean_ctor_get(x_94, 4); -lean_dec(x_98); -x_99 = !lean_is_exclusive(x_95); -if (x_99 == 0) -{ -lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; -x_100 = lean_ctor_get(x_95, 1); -lean_dec(x_100); -x_101 = l_Std_PersistentArray_push___rarg(x_22, x_89); -lean_ctor_set(x_95, 1, x_101); -x_102 = lean_st_ref_set(x_6, x_94, x_96); -lean_dec(x_6); -x_103 = !lean_is_exclusive(x_102); -if (x_103 == 0) -{ -lean_object* x_104; -x_104 = lean_ctor_get(x_102, 0); -lean_dec(x_104); -lean_ctor_set_tag(x_102, 1); -lean_ctor_set(x_102, 0, x_79); -return x_102; -} -else -{ -lean_object* x_105; lean_object* x_106; -x_105 = lean_ctor_get(x_102, 1); -lean_inc(x_105); -lean_dec(x_102); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_79); -lean_ctor_set(x_106, 1, x_105); -return x_106; +x_97 = lean_ctor_get(x_94, 1); +lean_inc(x_97); +lean_dec(x_94); +x_98 = !lean_is_exclusive(x_95); +if (x_98 == 0) +{ +lean_object* x_99; uint8_t x_100; +x_99 = lean_ctor_get(x_95, 5); +lean_dec(x_99); +x_100 = !lean_is_exclusive(x_96); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; +x_101 = lean_ctor_get(x_96, 1); +lean_dec(x_101); +x_102 = l_Std_PersistentArray_push___rarg(x_22, x_90); +lean_ctor_set(x_96, 1, x_102); +x_103 = lean_st_ref_set(x_6, x_95, x_97); +lean_dec(x_6); +x_104 = !lean_is_exclusive(x_103); +if (x_104 == 0) +{ +lean_object* x_105; +x_105 = lean_ctor_get(x_103, 0); +lean_dec(x_105); +lean_ctor_set_tag(x_103, 1); +lean_ctor_set(x_103, 0, x_80); +return x_103; +} +else +{ +lean_object* x_106; lean_object* x_107; +x_106 = lean_ctor_get(x_103, 1); +lean_inc(x_106); +lean_dec(x_103); +x_107 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_107, 0, x_80); +lean_ctor_set(x_107, 1, x_106); +return x_107; } } else { -uint8_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_107 = lean_ctor_get_uint8(x_95, sizeof(void*)*2); -x_108 = lean_ctor_get(x_95, 0); -lean_inc(x_108); -lean_dec(x_95); -x_109 = l_Std_PersistentArray_push___rarg(x_22, x_89); -x_110 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -lean_ctor_set_uint8(x_110, sizeof(void*)*2, x_107); -lean_ctor_set(x_94, 4, x_110); -x_111 = lean_st_ref_set(x_6, x_94, x_96); -lean_dec(x_6); -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_113 = x_111; +uint8_t x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_108 = lean_ctor_get_uint8(x_96, sizeof(void*)*2); +x_109 = lean_ctor_get(x_96, 0); +lean_inc(x_109); +lean_dec(x_96); +x_110 = l_Std_PersistentArray_push___rarg(x_22, x_90); +x_111 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +lean_ctor_set_uint8(x_111, sizeof(void*)*2, x_108); +lean_ctor_set(x_95, 5, x_111); +x_112 = lean_st_ref_set(x_6, x_95, x_97); +lean_dec(x_6); +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_114 = x_112; } else { - lean_dec_ref(x_111); - x_113 = lean_box(0); + lean_dec_ref(x_112); + x_114 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; - lean_ctor_set_tag(x_114, 1); + x_115 = x_114; + lean_ctor_set_tag(x_115, 1); } -lean_ctor_set(x_114, 0, x_79); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_115, 0, x_80); +lean_ctor_set(x_115, 1, x_113); +return x_115; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_115 = lean_ctor_get(x_94, 0); -x_116 = lean_ctor_get(x_94, 1); -x_117 = lean_ctor_get(x_94, 2); -x_118 = lean_ctor_get(x_94, 3); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; uint8_t x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_116 = lean_ctor_get(x_95, 0); +x_117 = lean_ctor_get(x_95, 1); +x_118 = lean_ctor_get(x_95, 2); +x_119 = lean_ctor_get(x_95, 3); +x_120 = lean_ctor_get(x_95, 4); +lean_inc(x_120); +lean_inc(x_119); lean_inc(x_118); lean_inc(x_117); lean_inc(x_116); -lean_inc(x_115); -lean_dec(x_94); -x_119 = lean_ctor_get_uint8(x_95, sizeof(void*)*2); -x_120 = lean_ctor_get(x_95, 0); -lean_inc(x_120); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_121 = x_95; +lean_dec(x_95); +x_121 = lean_ctor_get_uint8(x_96, sizeof(void*)*2); +x_122 = lean_ctor_get(x_96, 0); +lean_inc(x_122); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_123 = x_96; } else { - lean_dec_ref(x_95); - x_121 = lean_box(0); + lean_dec_ref(x_96); + x_123 = lean_box(0); } -x_122 = l_Std_PersistentArray_push___rarg(x_22, x_89); -if (lean_is_scalar(x_121)) { - x_123 = lean_alloc_ctor(0, 2, 1); +x_124 = l_Std_PersistentArray_push___rarg(x_22, x_90); +if (lean_is_scalar(x_123)) { + x_125 = lean_alloc_ctor(0, 2, 1); } else { - x_123 = x_121; + x_125 = x_123; } -lean_ctor_set(x_123, 0, x_120); -lean_ctor_set(x_123, 1, x_122); -lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_119); -x_124 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_124, 0, x_115); -lean_ctor_set(x_124, 1, x_116); -lean_ctor_set(x_124, 2, x_117); -lean_ctor_set(x_124, 3, x_118); -lean_ctor_set(x_124, 4, x_123); -x_125 = lean_st_ref_set(x_6, x_124, x_96); -lean_dec(x_6); -x_126 = lean_ctor_get(x_125, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - x_127 = x_125; +lean_ctor_set(x_125, 0, x_122); +lean_ctor_set(x_125, 1, x_124); +lean_ctor_set_uint8(x_125, sizeof(void*)*2, x_121); +x_126 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_126, 0, x_116); +lean_ctor_set(x_126, 1, x_117); +lean_ctor_set(x_126, 2, x_118); +lean_ctor_set(x_126, 3, x_119); +lean_ctor_set(x_126, 4, x_120); +lean_ctor_set(x_126, 5, x_125); +x_127 = lean_st_ref_set(x_6, x_126, x_97); +lean_dec(x_6); +x_128 = lean_ctor_get(x_127, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_129 = x_127; } else { - lean_dec_ref(x_125); - x_127 = lean_box(0); + lean_dec_ref(x_127); + x_129 = lean_box(0); } -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(1, 2, 0); } else { - x_128 = x_127; - lean_ctor_set_tag(x_128, 1); + x_130 = x_129; + lean_ctor_set_tag(x_130, 1); } -lean_ctor_set(x_128, 0, x_79); -lean_ctor_set(x_128, 1, x_126); -return x_128; +lean_ctor_set(x_130, 0, x_80); +lean_ctor_set(x_130, 1, x_128); +return x_130; } } else { -uint8_t x_129; -lean_dec(x_79); +uint8_t x_131; +lean_dec(x_80); lean_dec(x_22); lean_dec(x_10); lean_dec(x_6); -x_129 = !lean_is_exclusive(x_88); -if (x_129 == 0) +x_131 = !lean_is_exclusive(x_89); +if (x_131 == 0) { -return x_88; +return x_89; } else { -lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_130 = lean_ctor_get(x_88, 0); -x_131 = lean_ctor_get(x_88, 1); -lean_inc(x_131); -lean_inc(x_130); -lean_dec(x_88); -x_132 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); -return x_132; -} -} -} -} -} -} -static lean_object* _init_l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("unexpected syntax ", 18); -return x_1; +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_89, 0); +x_133 = lean_ctor_get(x_89, 1); +lean_inc(x_133); +lean_inc(x_132); +lean_dec(x_89); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_unsupportedSyntaxExceptionId; -return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_eval(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { if (lean_obj_tag(x_3) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -lean_dec(x_1); -lean_inc(x_2); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_2); -x_14 = l_Lean_indentD(x_13); -x_15 = l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__2; -x_16 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -x_17 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; -x_18 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__1(x_2, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_19; +lean_object* x_14; +lean_dec(x_2); +x_14 = l_Lean_Elab_Tactic_evalTactic_throwExs(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_14; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_20 = lean_ctor_get(x_3, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_3, 1); -lean_inc(x_21); +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_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_3, 1); +lean_inc(x_16); lean_dec(x_3); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_inc(x_2); -x_23 = lean_apply_1(x_22, x_2); -x_24 = lean_ctor_get(x_20, 0); -lean_inc(x_24); -lean_dec(x_20); -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = lean_ctor_get_uint8(x_4, sizeof(void*)*1); -x_27 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set_uint8(x_27, sizeof(void*)*1, x_26); -lean_inc(x_2); -x_28 = l_Lean_Elab_Tactic_mkInitialTacticInfo(x_2, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg___lambda__1), 11, 1); -lean_closure_set(x_31, 0, x_29); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_inc(x_1); +x_18 = lean_apply_1(x_17, x_1); +x_47 = lean_ctor_get(x_15, 0); +lean_inc(x_47); +lean_dec(x_15); +x_48 = lean_ctor_get(x_47, 1); +lean_inc(x_48); +lean_dec(x_47); +x_49 = lean_ctor_get_uint8(x_5, sizeof(void*)*1); +x_50 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*1, x_49); +lean_inc(x_1); +x_51 = l_Lean_Elab_Tactic_mkInitialTacticInfo(x_1, x_50, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); +x_54 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg___lambda__1), 11, 1); +lean_closure_set(x_54, 0, x_52); +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_32 = l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(x_23, x_31, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); -if (lean_obj_tag(x_32) == 0) -{ -lean_dec(x_21); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_32; -} -else -{ -lean_object* x_33; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -if (lean_obj_tag(x_33) == 0) -{ -if (lean_obj_tag(x_21) == 0) +x_55 = l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(x_18, x_54, x_50, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_53); +if (lean_obj_tag(x_55) == 0) { -uint8_t x_34; +lean_dec(x_16); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4549,103 +5610,57 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_34 = !lean_is_exclusive(x_32); -if (x_34 == 0) -{ -lean_object* x_35; -x_35 = lean_ctor_get(x_32, 0); -lean_dec(x_35); -return x_32; -} -else -{ -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_32, 1); -lean_inc(x_36); -lean_dec(x_32); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_33); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -lean_dec(x_33); -x_38 = lean_ctor_get(x_32, 1); -lean_inc(x_38); -lean_dec(x_32); -lean_inc(x_1); -x_39 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_38); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -lean_dec(x_39); -x_3 = x_21; -x_12 = x_40; -goto _start; -} +return x_55; } else { -uint8_t x_42; -x_42 = !lean_is_exclusive(x_32); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_43 = lean_ctor_get(x_32, 1); -x_44 = lean_ctor_get(x_32, 0); -lean_dec(x_44); -x_45 = lean_ctor_get(x_33, 0); -lean_inc(x_45); -x_46 = l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__3; -x_47 = lean_nat_dec_eq(x_45, x_46); -lean_dec(x_45); -if (x_47 == 0) -{ -lean_dec(x_21); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_32; +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +lean_dec(x_55); +x_19 = x_56; +x_20 = x_57; +goto block_46; } -else +block_46: { -lean_object* x_48; lean_object* x_49; -lean_free_object(x_32); -lean_dec(x_33); -lean_inc(x_1); -x_48 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_43); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -lean_dec(x_48); -x_3 = x_21; -x_12 = x_49; +if (lean_obj_tag(x_19) == 0) +{ +uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_21 = 1; +lean_inc(x_2); +x_22 = l_Lean_Elab_Tactic_SavedState_restore(x_2, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_24, 0, x_19); +x_25 = lean_array_push(x_4, x_24); +x_3 = x_16; +x_4 = x_25; +x_13 = x_23; goto _start; } -} else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_51 = lean_ctor_get(x_32, 1); -lean_inc(x_51); -lean_dec(x_32); -x_52 = lean_ctor_get(x_33, 0); -lean_inc(x_52); -x_53 = l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__3; -x_54 = lean_nat_dec_eq(x_52, x_53); -lean_dec(x_52); -if (x_54 == 0) +lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_27 = lean_ctor_get(x_19, 0); +lean_inc(x_27); +x_28 = l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1; +x_29 = lean_nat_dec_eq(x_27, x_28); +if (x_29 == 0) { -lean_object* x_55; -lean_dec(x_21); +lean_object* x_30; uint8_t x_31; +x_30 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1; +x_31 = lean_nat_dec_eq(x_27, x_30); +lean_dec(x_27); +if (x_31 == 0) +{ +lean_object* x_32; +lean_dec(x_16); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4656,55 +5671,57 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_33); -lean_ctor_set(x_55, 1, x_51); -return x_55; +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_19); +lean_ctor_set(x_32, 1, x_20); +return x_32; } else { -lean_object* x_56; lean_object* x_57; +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; +lean_dec(x_19); +x_33 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); lean_dec(x_33); -lean_inc(x_1); -x_56 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_51); -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); -x_3 = x_21; -x_12 = x_57; +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_34); +x_37 = lean_array_push(x_4, x_36); +x_38 = 1; +lean_inc(x_2); +x_39 = l_Lean_Elab_Tactic_SavedState_restore(x_2, x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_35); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_3 = x_16; +x_4 = x_37; +x_13 = x_40; goto _start; } } +else +{ +uint8_t x_42; lean_object* x_43; lean_object* x_44; +lean_dec(x_27); +lean_dec(x_19); +x_42 = 1; +lean_inc(x_2); +x_43 = l_Lean_Elab_Tactic_SavedState_restore(x_2, x_42, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +x_3 = x_16; +x_13 = x_44; +goto _start; } } } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_11; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; -x_13 = l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_13; -} } -LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; @@ -4717,7 +5734,7 @@ lean_ctor_set(x_14, 1, x_10); return x_14; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__1() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__1() { _start: { lean_object* x_1; @@ -4725,17 +5742,17 @@ x_1 = lean_mk_string_from_bytes("_traceMsg", 9); return x_1; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__2() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__1; +x_2 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__3() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__3() { _start: { lean_object* x_1; @@ -4743,16 +5760,16 @@ x_1 = lean_mk_string_from_bytes("[", 1); return x_1; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__4() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__3; +x_1 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__5() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__5() { _start: { lean_object* x_1; @@ -4760,16 +5777,16 @@ x_1 = lean_mk_string_from_bytes("] ", 2); return x_1; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__6() { +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__5; +x_1 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; @@ -4800,15 +5817,15 @@ if (x_23 == 0) { lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; x_24 = lean_ctor_get(x_19, 0); -x_25 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__2; +x_25 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__2; x_26 = l_Lean_Name_append(x_1, x_25); x_27 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_27, 0, x_1); -x_28 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__4; +x_28 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__4; x_29 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_29, 0, x_28); lean_ctor_set(x_29, 1, x_27); -x_30 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__6; +x_30 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__6; x_31 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); @@ -4859,15 +5876,15 @@ x_45 = lean_ctor_get_uint8(x_19, sizeof(void*)*1); x_46 = lean_ctor_get(x_19, 0); lean_inc(x_46); lean_dec(x_19); -x_47 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__2; +x_47 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__2; x_48 = l_Lean_Name_append(x_1, x_47); x_49 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_49, 0, x_1); -x_50 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__4; +x_50 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__4; x_51 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_51, 0, x_50); lean_ctor_set(x_51, 1, x_49); -x_52 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__6; +x_52 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__6; x_53 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); @@ -4936,15 +5953,15 @@ if (lean_is_exclusive(x_19)) { lean_dec_ref(x_19); x_73 = lean_box(0); } -x_74 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__2; +x_74 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__2; x_75 = l_Lean_Name_append(x_1, x_74); x_76 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_76, 0, x_1); -x_77 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__4; +x_77 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__4; x_78 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_78, 0, x_77); lean_ctor_set(x_78, 1, x_76); -x_79 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__6; +x_79 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__6; x_80 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_80, 0, x_78); lean_ctor_set(x_80, 1, x_79); @@ -5000,7 +6017,7 @@ return x_93; } } } -LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { if (lean_obj_tag(x_1) == 0) @@ -5052,7 +6069,7 @@ x_23 = lean_ctor_get(x_17, 1); lean_inc(x_23); lean_dec(x_17); lean_inc(x_15); -x_24 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +x_24 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); x_26 = lean_unbox(x_25); @@ -5079,7 +6096,7 @@ x_30 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_30, 0, x_16); x_31 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_31, 0, x_30); -x_32 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3(x_15, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +x_32 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3(x_15, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); x_33 = lean_ctor_get(x_32, 1); lean_inc(x_33); lean_dec(x_32); @@ -5091,7 +6108,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -5129,7 +6146,7 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; @@ -5142,7 +6159,7 @@ x_14 = l_Lean_replaceRef(x_1, x_13); lean_dec(x_13); lean_dec(x_1); lean_ctor_set(x_9, 5, x_14); -x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -5194,7 +6211,7 @@ lean_ctor_set(x_28, 7, x_23); lean_ctor_set(x_28, 8, x_24); lean_ctor_set(x_28, 9, x_25); lean_ctor_set(x_28, 10, x_26); -x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); +x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); lean_dec(x_10); lean_dec(x_28); lean_dec(x_8); @@ -5207,7 +6224,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__1() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -5217,21 +6234,21 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__2() { +static lean_object* _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__1; +x_1 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__1; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__2; +x_11 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__2; x_12 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_12, 0, x_1); lean_ctor_set(x_12, 1, x_11); @@ -5241,38 +6258,38 @@ lean_ctor_set(x_13, 1, x_10); return x_13; } } -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg___closed__1() { +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__3; +x_2 = l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg___closed__1; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg___closed__1; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg), 1, 0); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg), 1, 0); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; @@ -5441,7 +6458,7 @@ return x_41; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; lean_object* x_7; @@ -5453,7 +6470,7 @@ lean_ctor_set(x_7, 1, x_4); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; @@ -5464,7 +6481,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; @@ -5475,7 +6492,7 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; lean_object* x_13; 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; @@ -5501,23 +6518,23 @@ lean_inc(x_19); x_20 = lean_ctor_get(x_8, 10); lean_inc(x_20); lean_inc(x_14); -x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__1___boxed), 4, 1); +x_21 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__1___boxed), 4, 1); lean_closure_set(x_21, 0, x_14); lean_inc(x_18); x_22 = lean_alloc_closure((void*)(l_ReaderT_pure___at_Lean_Elab_liftMacroM___spec__2___rarg___boxed), 3, 1); lean_closure_set(x_22, 0, x_18); lean_inc(x_14); -x_23 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__2___boxed), 4, 1); +x_23 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__2___boxed), 4, 1); lean_closure_set(x_23, 0, x_14); lean_inc(x_19); lean_inc(x_18); lean_inc(x_14); -x_24 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__3___boxed), 6, 3); +x_24 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__3___boxed), 6, 3); lean_closure_set(x_24, 0, x_14); lean_closure_set(x_24, 1, x_18); lean_closure_set(x_24, 2, x_19); lean_inc(x_14); -x_25 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__4___boxed), 6, 3); +x_25 = lean_alloc_closure((void*)(l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__4___boxed), 6, 3); lean_closure_set(x_25, 0, x_14); lean_closure_set(x_25, 1, x_18); lean_closure_set(x_25, 2, x_19); @@ -5580,7 +6597,7 @@ x_46 = lean_ctor_get(x_37, 1); lean_inc(x_46); lean_dec(x_37); x_47 = l_List_reverse___rarg(x_46); -x_48 = l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4(x_47, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); +x_48 = l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4(x_47, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -5639,7 +6656,7 @@ x_61 = lean_ctor_get(x_37, 1); lean_inc(x_61); lean_dec(x_37); x_62 = l_List_reverse___rarg(x_61); -x_63 = l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4(x_62, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_60); +x_63 = l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4(x_62, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_60); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -5691,14 +6708,14 @@ x_72 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_72, 0, x_69); x_73 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_73, 0, x_72); -x_74 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__5(x_68, x_73, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +x_74 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__5(x_68, x_73, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); return x_74; } else { lean_object* x_75; lean_dec(x_69); -x_75 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7(x_68, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +x_75 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7(x_68, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -5721,13 +6738,13 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_76 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg(x_29); +x_76 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg(x_29); return x_76; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_expandEval___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; @@ -5739,7 +6756,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_11 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; lean_object* x_14; @@ -5748,7 +6765,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_14 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_14; } else @@ -5783,120 +6800,123 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic_expandEval(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_4); -lean_inc(x_1); -x_14 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -x_16 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_15); -return x_16; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__1() { -_start: +if (lean_obj_tag(x_3) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("tactic '", 8); -return x_1; -} +lean_object* x_15; +x_15 = l_Lean_Elab_Tactic_evalTactic_eval(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_15; } -static lean_object* _init_l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__3() { -_start: +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_16 = lean_ctor_get(x_3, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_3, 1); +lean_inc(x_17); +lean_dec(x_3); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_inc(x_1); +x_19 = lean_apply_1(x_18, x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic_expandEval___lambda__1), 10, 1); +lean_closure_set(x_20, 0, x_19); +x_49 = lean_ctor_get(x_16, 0); +lean_inc(x_49); +lean_dec(x_16); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +lean_dec(x_49); +x_51 = lean_ctor_get_uint8(x_6, sizeof(void*)*1); +x_52 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set_uint8(x_52, sizeof(void*)*1, x_51); +lean_inc(x_1); +x_53 = l_Lean_Elab_Tactic_mkInitialTacticInfo(x_1, x_52, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +lean_dec(x_53); +x_56 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg___lambda__1), 11, 1); +lean_closure_set(x_56, 0, x_54); +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_57 = l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(x_20, x_56, x_52, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_55); +if (lean_obj_tag(x_57) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("' has not been implemented", 26); -return x_1; -} +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_57; } -static lean_object* _init_l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_58; lean_object* x_59; +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_57, 1); +lean_inc(x_59); +lean_dec(x_57); +x_21 = x_58; +x_22 = x_59; +goto block_48; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns_loop(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +block_48: { -if (lean_obj_tag(x_3) == 0) +if (lean_obj_tag(x_21) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -lean_dec(x_1); +uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = 1; lean_inc(x_2); -x_13 = l_Lean_Syntax_getKind(x_2); -x_14 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__2; -x_16 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -x_17 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__4; -x_18 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -x_19 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__1(x_2, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_19; +x_24 = l_Lean_Elab_Tactic_SavedState_restore(x_2, x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_26, 0, x_21); +x_27 = lean_array_push(x_5, x_26); +x_3 = x_17; +x_5 = x_27; +x_14 = x_25; +goto _start; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_20 = lean_ctor_get(x_3, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_3, 1); -lean_inc(x_21); -lean_dec(x_3); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_inc(x_2); -x_23 = lean_apply_1(x_22, x_2); -x_24 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_expandTacticMacroFns_loop___lambda__1), 10, 1); -lean_closure_set(x_24, 0, x_23); -x_25 = lean_ctor_get(x_20, 0); -lean_inc(x_25); -lean_dec(x_20); -x_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -x_27 = lean_ctor_get_uint8(x_4, sizeof(void*)*1); -x_28 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set_uint8(x_28, sizeof(void*)*1, x_27); -lean_inc(x_2); -x_29 = l_Lean_Elab_Tactic_mkInitialTacticInfo(x_2, x_28, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); +lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_29 = lean_ctor_get(x_21, 0); +lean_inc(x_29); +x_30 = l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1; +x_31 = lean_nat_dec_eq(x_29, x_30); +if (x_31 == 0) +{ +lean_object* x_32; uint8_t x_33; +x_32 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1; +x_33 = lean_nat_dec_eq(x_29, x_32); lean_dec(x_29); -x_32 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg___lambda__1), 11, 1); -lean_closure_set(x_32, 0, x_30); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_33 = l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(x_24, x_32, x_28, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_31); -if (lean_obj_tag(x_33) == 0) +if (x_33 == 0) { -lean_dec(x_21); +lean_object* x_34; +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -5907,31 +6927,108 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -return x_33; +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_21); +lean_ctor_set(x_34, 1, x_22); +return x_34; +} +else +{ +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_dec(x_21); +x_35 = l_Lean_Elab_Tactic_saveState___rarg(x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_36); +x_39 = lean_array_push(x_5, x_38); +x_40 = 1; +lean_inc(x_2); +x_41 = l_Lean_Elab_Tactic_SavedState_restore(x_2, x_40, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_37); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_3 = x_17; +x_5 = x_39; +x_14 = x_42; +goto _start; +} +} +else +{ +uint8_t x_44; lean_object* x_45; lean_object* x_46; +lean_dec(x_29); +lean_dec(x_21); +x_44 = 1; +lean_inc(x_2); +x_45 = l_Lean_Elab_Tactic_SavedState_restore(x_2, x_44, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +x_46 = lean_ctor_get(x_45, 1); +lean_inc(x_46); +lean_dec(x_45); +x_3 = x_17; +x_14 = x_46; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_8, 5); +x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_6, x_7, x_8, x_9, x_10); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_11); +lean_ctor_set(x_15, 1, x_14); +lean_ctor_set_tag(x_12, 1); +lean_ctor_set(x_12, 0, x_15); +return x_12; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_12, 0); +x_17 = lean_ctor_get(x_12, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_12); +lean_inc(x_11); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_11); +lean_ctor_set(x_18, 1, x_16); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; } -else -{ -uint8_t x_34; -x_34 = !lean_is_exclusive(x_33); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_35 = lean_ctor_get(x_33, 0); -x_36 = lean_ctor_get(x_33, 1); -x_37 = l_List_isEmpty___rarg(x_21); -if (x_37 == 0) -{ -lean_object* x_38; lean_object* x_39; -lean_free_object(x_33); -lean_dec(x_35); -x_38 = lean_box(0); -x_39 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop___lambda__2(x_1, x_2, x_21, x_38, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_36); -return x_39; } -else +} +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_dec(x_21); -lean_dec(x_11); +uint8_t x_12; +x_12 = !lean_is_exclusive(x_9); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 5); +x_14 = l_Lean_replaceRef(x_1, x_13); +lean_dec(x_13); +lean_dec(x_1); +lean_ctor_set(x_9, 5, x_14); +x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -5939,61 +7036,64 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_33; -} -} -else -{ -lean_object* x_40; lean_object* x_41; uint8_t x_42; -x_40 = lean_ctor_get(x_33, 0); -x_41 = lean_ctor_get(x_33, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_33); -x_42 = l_List_isEmpty___rarg(x_21); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; -lean_dec(x_40); -x_43 = lean_box(0); -x_44 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop___lambda__2(x_1, x_2, x_21, x_43, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_41); -return x_44; +lean_dec(x_3); +return x_15; } else { -lean_object* x_45; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_16 = lean_ctor_get(x_9, 0); +x_17 = lean_ctor_get(x_9, 1); +x_18 = lean_ctor_get(x_9, 2); +x_19 = lean_ctor_get(x_9, 3); +x_20 = lean_ctor_get(x_9, 4); +x_21 = lean_ctor_get(x_9, 5); +x_22 = lean_ctor_get(x_9, 6); +x_23 = lean_ctor_get(x_9, 7); +x_24 = lean_ctor_get(x_9, 8); +x_25 = lean_ctor_get(x_9, 9); +x_26 = lean_ctor_get(x_9, 10); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_9); +x_27 = l_Lean_replaceRef(x_1, x_21); lean_dec(x_21); -lean_dec(x_11); +lean_dec(x_1); +x_28 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_28, 0, x_16); +lean_ctor_set(x_28, 1, x_17); +lean_ctor_set(x_28, 2, x_18); +lean_ctor_set(x_28, 3, x_19); +lean_ctor_set(x_28, 4, x_20); +lean_ctor_set(x_28, 5, x_27); +lean_ctor_set(x_28, 6, x_22); +lean_ctor_set(x_28, 7, x_23); +lean_ctor_set(x_28, 8, x_24); +lean_ctor_set(x_28, 9, x_25); +lean_ctor_set(x_28, 10, x_26); +x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_28); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_40); -lean_ctor_set(x_45, 1, x_41); -return x_45; -} -} -} -} -} +lean_dec(x_3); +return x_29; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_evalTacticAux(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_11; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTacticAux___spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic___spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { uint8_t x_14; @@ -6011,7 +7111,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_16 = l_Lean_Elab_Tactic_evalTacticAux(x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_16 = l_Lean_Elab_Tactic_evalTactic(x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_16) == 0) { lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; @@ -6076,11 +7176,11 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTacticAux___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__2; +x_11 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__2; x_12 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_12, 0, x_1); lean_ctor_set(x_12, 1, x_11); @@ -6090,7 +7190,7 @@ lean_ctor_set(x_13, 1, x_10); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; @@ -6101,7 +7201,23 @@ lean_ctor_set(x_5, 1, x_3); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___lambda__2___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_4); +x_14 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1; +x_18 = l_Lean_Elab_Tactic_evalTactic_expandEval(x_1, x_15, x_2, x_3, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_18; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__1() { _start: { lean_object* x_1; @@ -6109,45 +7225,139 @@ x_1 = l_Lean_Elab_Tactic_tacticElabAttribute; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_macroAttribute; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("tactic '", 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__4() { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("' has not been implemented", 26); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_dec(x_2); -x_12 = l_Lean_Elab_Tactic_saveState___rarg(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = lean_st_ref_get(x_10, x_11); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); lean_inc(x_14); lean_dec(x_12); -x_15 = lean_st_ref_get(x_10, x_14); -x_16 = lean_ctor_get(x_15, 0); +x_15 = lean_ctor_get(x_13, 0); +lean_inc(x_15); +lean_dec(x_13); +lean_inc(x_1); +x_16 = l_Lean_Syntax_getKind(x_1); +x_17 = l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__1; lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); +x_18 = l_Lean_KeyedDeclsAttribute_getEntries___rarg(x_17, x_15, x_16); +x_19 = lean_st_ref_get(x_10, x_14); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +x_23 = l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__2; +lean_inc(x_16); +x_24 = l_Lean_KeyedDeclsAttribute_getEntries___rarg(x_23, x_22, x_16); +x_25 = l_List_isEmpty___rarg(x_18); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_dec(x_16); -lean_inc(x_1); -x_19 = l_Lean_Syntax_getKind(x_1); -x_20 = l_Lean_Elab_Tactic_evalTacticAux___lambda__2___closed__1; -x_21 = l_Lean_KeyedDeclsAttribute_getEntries___rarg(x_20, x_18, x_19); -if (lean_obj_tag(x_21) == 0) +x_26 = lean_box(0); +x_27 = l_Lean_Elab_Tactic_evalTactic___lambda__2(x_1, x_24, x_18, x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +return x_27; +} +else { -lean_object* x_22; -x_22 = l_Lean_Elab_Tactic_expandTacticMacro(x_13, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); -return x_22; +uint8_t x_28; +x_28 = l_List_isEmpty___rarg(x_24); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_16); +x_29 = lean_box(0); +x_30 = l_Lean_Elab_Tactic_evalTactic___lambda__2(x_1, x_24, x_18, x_29, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +return x_30; } else { -lean_object* x_23; -x_23 = l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop(x_13, x_1, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); -return x_23; +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_dec(x_24); +lean_dec(x_18); +x_31 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_31, 0, x_16); +x_32 = l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__4; +x_33 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +x_34 = l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__6; +x_35 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_36 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___spec__1(x_1, x_35, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +x_37 = !lean_is_exclusive(x_36); +if (x_37 == 0) +{ +return x_36; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_36, 0); +x_39 = lean_ctor_get(x_36, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_36); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; lean_object* x_13; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; @@ -6177,7 +7387,7 @@ x_31 = lean_ctor_get(x_25, 1); lean_inc(x_31); lean_dec(x_25); lean_inc(x_8); -x_32 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(x_8, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_10, x_31); +x_32 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(x_8, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_10, x_31); x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); x_34 = lean_ctor_get(x_32, 1); @@ -6196,7 +7406,7 @@ if (x_12 == 0) lean_object* x_14; lean_object* x_15; lean_dec(x_8); x_14 = lean_box(0); -x_15 = l_Lean_Elab_Tactic_evalTacticAux___lambda__2(x_1, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_10, x_13); +x_15 = l_Lean_Elab_Tactic_evalTactic___lambda__3(x_1, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_10, x_13); return x_15; } else @@ -6212,27 +7422,27 @@ lean_ctor_set(x_18, 1, x_16); x_19 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_19, 0, x_18); lean_ctor_set(x_19, 1, x_17); -x_20 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3(x_8, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_10, x_13); +x_20 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3(x_8, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_10, x_13); x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); x_22 = lean_ctor_get(x_20, 1); lean_inc(x_22); lean_dec(x_20); -x_23 = l_Lean_Elab_Tactic_evalTacticAux___lambda__2(x_1, x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_10, x_22); +x_23 = l_Lean_Elab_Tactic_evalTactic___lambda__3(x_1, x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_10, x_22); return x_23; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTacticAux___lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic___lambda__1___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___closed__2() { _start: { lean_object* x_1; @@ -6240,17 +7450,17 @@ x_1 = lean_mk_string_from_bytes("null", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_evalTacticAux___closed__2; +x_2 = l_Lean_Elab_Tactic_evalTactic___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -6260,7 +7470,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___closed__5() { _start: { lean_object* x_1; @@ -6268,17 +7478,17 @@ x_1 = lean_mk_string_from_bytes("step", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_evalTacticAux___closed__4; -x_2 = l_Lean_Elab_Tactic_evalTacticAux___closed__5; +x_1 = l_Lean_Elab_Tactic_evalTactic___closed__4; +x_2 = l_Lean_Elab_Tactic_evalTactic___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___closed__7() { _start: { lean_object* x_1; @@ -6286,16 +7496,16 @@ x_1 = lean_mk_string_from_bytes("unexpected tactic", 17); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_evalTacticAux___closed__7; +x_1 = l_Lean_Elab_Tactic_evalTactic___closed__7; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalTacticAux___boxed__const__1() { +static lean_object* _init_l_Lean_Elab_Tactic_evalTactic___boxed__const__1() { _start: { size_t x_1; lean_object* x_2; @@ -6304,7 +7514,7 @@ x_2 = lean_box_usize(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -6367,7 +7577,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_28 = l_Lean_Elab_Tactic_evalTacticAux___closed__1; +x_28 = l_Lean_Elab_Tactic_evalTactic___closed__1; x_29 = l_Lean_Core_withFreshMacroScope___rarg(x_28, x_27, x_9, x_10); return x_29; } @@ -6376,14 +7586,14 @@ case 1: lean_object* x_30; lean_object* x_31; uint8_t x_32; x_30 = lean_ctor_get(x_1, 1); lean_inc(x_30); -x_31 = l_Lean_Elab_Tactic_evalTacticAux___closed__3; +x_31 = l_Lean_Elab_Tactic_evalTactic___closed__3; x_32 = lean_name_eq(x_30, x_31); lean_dec(x_30); if (x_32 == 0) { lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = l_Lean_Elab_Tactic_evalTacticAux___closed__6; -x_34 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTacticAux___lambda__3), 11, 8); +x_33 = l_Lean_Elab_Tactic_evalTactic___closed__6; +x_34 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic___lambda__4), 11, 8); lean_closure_set(x_34, 0, x_1); lean_closure_set(x_34, 1, x_2); lean_closure_set(x_34, 2, x_3); @@ -6414,7 +7624,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_40 = l_Lean_Elab_Tactic_evalTacticAux___closed__1; +x_40 = l_Lean_Elab_Tactic_evalTactic___closed__1; x_41 = l_Lean_Core_withFreshMacroScope___rarg(x_40, x_27, x_9, x_10); return x_41; } @@ -6433,7 +7643,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_43 = l_Lean_Elab_Tactic_evalTacticAux___closed__1; +x_43 = l_Lean_Elab_Tactic_evalTactic___closed__1; x_44 = l_Lean_Core_withFreshMacroScope___rarg(x_43, x_27, x_9, x_10); return x_44; } @@ -6443,9 +7653,9 @@ size_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_objec x_45 = lean_usize_of_nat(x_37); lean_dec(x_37); x_46 = lean_box(0); -x_47 = l_Lean_Elab_Tactic_evalTacticAux___boxed__const__1; +x_47 = l_Lean_Elab_Tactic_evalTactic___boxed__const__1; x_48 = lean_box_usize(x_45); -x_49 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTacticAux___spec__1___boxed), 13, 10); +x_49 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic___spec__3___boxed), 13, 10); lean_closure_set(x_49, 0, x_36); lean_closure_set(x_49, 1, x_47); lean_closure_set(x_49, 2, x_48); @@ -6468,7 +7678,7 @@ lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean x_51 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_51, 0, x_1); x_52 = l_Lean_indentD(x_51); -x_53 = l_Lean_Elab_Tactic_evalTacticAux___closed__8; +x_53 = l_Lean_Elab_Tactic_evalTactic___closed__8; x_54 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_54, 0, x_53); lean_ctor_set(x_54, 1, x_52); @@ -6476,7 +7686,7 @@ x_55 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; x_56 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_56, 0, x_54); lean_ctor_set(x_56, 1, x_55); -x_57 = lean_alloc_closure((void*)(l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2___boxed), 10, 7); +x_57 = lean_alloc_closure((void*)(l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2___boxed), 10, 7); lean_closure_set(x_57, 0, x_56); lean_closure_set(x_57, 1, x_2); lean_closure_set(x_57, 2, x_3); @@ -6503,7 +7713,7 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_1); -x_59 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTacticAux___spec__2(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_59 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic___spec__4(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6596,7 +7806,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_77 = l_Lean_Elab_Tactic_evalTacticAux___closed__1; +x_77 = l_Lean_Elab_Tactic_evalTactic___closed__1; x_78 = l_Lean_Core_withFreshMacroScope___rarg(x_77, x_76, x_9, x_10); return x_78; } @@ -6605,14 +7815,14 @@ case 1: lean_object* x_79; lean_object* x_80; uint8_t x_81; x_79 = lean_ctor_get(x_1, 1); lean_inc(x_79); -x_80 = l_Lean_Elab_Tactic_evalTacticAux___closed__3; +x_80 = l_Lean_Elab_Tactic_evalTactic___closed__3; x_81 = lean_name_eq(x_79, x_80); lean_dec(x_79); if (x_81 == 0) { lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_82 = l_Lean_Elab_Tactic_evalTacticAux___closed__6; -x_83 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTacticAux___lambda__3), 11, 8); +x_82 = l_Lean_Elab_Tactic_evalTactic___closed__6; +x_83 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic___lambda__4), 11, 8); lean_closure_set(x_83, 0, x_1); lean_closure_set(x_83, 1, x_2); lean_closure_set(x_83, 2, x_3); @@ -6643,7 +7853,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_89 = l_Lean_Elab_Tactic_evalTacticAux___closed__1; +x_89 = l_Lean_Elab_Tactic_evalTactic___closed__1; x_90 = l_Lean_Core_withFreshMacroScope___rarg(x_89, x_76, x_9, x_10); return x_90; } @@ -6662,7 +7872,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_92 = l_Lean_Elab_Tactic_evalTacticAux___closed__1; +x_92 = l_Lean_Elab_Tactic_evalTactic___closed__1; x_93 = l_Lean_Core_withFreshMacroScope___rarg(x_92, x_76, x_9, x_10); return x_93; } @@ -6672,9 +7882,9 @@ size_t x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_objec x_94 = lean_usize_of_nat(x_86); lean_dec(x_86); x_95 = lean_box(0); -x_96 = l_Lean_Elab_Tactic_evalTacticAux___boxed__const__1; +x_96 = l_Lean_Elab_Tactic_evalTactic___boxed__const__1; x_97 = lean_box_usize(x_94); -x_98 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTacticAux___spec__1___boxed), 13, 10); +x_98 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic___spec__3___boxed), 13, 10); lean_closure_set(x_98, 0, x_85); lean_closure_set(x_98, 1, x_96); lean_closure_set(x_98, 2, x_97); @@ -6697,7 +7907,7 @@ lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; x_100 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_100, 0, x_1); x_101 = l_Lean_indentD(x_100); -x_102 = l_Lean_Elab_Tactic_evalTacticAux___closed__8; +x_102 = l_Lean_Elab_Tactic_evalTactic___closed__8; x_103 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_103, 0, x_102); lean_ctor_set(x_103, 1, x_101); @@ -6705,7 +7915,7 @@ x_104 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; x_105 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_105, 0, x_103); lean_ctor_set(x_105, 1, x_104); -x_106 = lean_alloc_closure((void*)(l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2___boxed), 10, 7); +x_106 = lean_alloc_closure((void*)(l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2___boxed), 10, 7); lean_closure_set(x_106, 0, x_105); lean_closure_set(x_106, 1, x_2); lean_closure_set(x_106, 2, x_3); @@ -6724,70 +7934,33 @@ lean_object* x_108; lean_dec(x_70); lean_dec(x_69); lean_dec(x_68); -lean_dec(x_67); -lean_dec(x_66); -lean_dec(x_64); -lean_dec(x_63); -lean_dec(x_62); -lean_dec(x_61); -lean_dec(x_60); -lean_dec(x_1); -x_108 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTacticAux___spec__2(x_71, x_2, x_3, x_4, x_5, x_6, x_7, x_72, x_9, x_10); -lean_dec(x_9); -lean_dec(x_72); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_108; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_expandTacticMacro___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_macroAttribute; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacro(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_12 = lean_st_ref_get(x_10, x_11); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_ctor_get(x_13, 0); -lean_inc(x_15); -lean_dec(x_13); -lean_inc(x_2); -x_16 = l_Lean_Syntax_getKind(x_2); -x_17 = l_Lean_Elab_Tactic_expandTacticMacro___closed__1; -x_18 = l_Lean_KeyedDeclsAttribute_getEntries___rarg(x_17, x_15, x_16); -x_19 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop(x_1, x_2, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); -return x_19; +lean_dec(x_67); +lean_dec(x_66); +lean_dec(x_64); +lean_dec(x_63); +lean_dec(x_62); +lean_dec(x_61); +lean_dec(x_60); +lean_dec(x_1); +x_108 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic___spec__4(x_71, x_2, x_3, x_4, x_5, x_6, x_7, x_72, x_9, x_10); +lean_dec(x_9); +lean_dec(x_72); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_108; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_expandTacticMacroFns(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; -x_13 = l_Lean_Elab_Tactic_expandTacticMacroFns_loop(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_13; } } -LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6799,11 +7972,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6815,11 +7988,11 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6831,11 +8004,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6847,11 +8020,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6863,11 +8036,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -6879,44 +8052,60 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__2(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTacticAux___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { size_t x_14; size_t x_15; lean_object* x_16; @@ -6924,16 +8113,16 @@ x_14 = lean_unbox_usize(x_2); lean_dec(x_2); x_15 = lean_unbox_usize(x_3); lean_dec(x_3); -x_16 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTacticAux___spec__1(x_1, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_16 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_evalTactic___spec__3(x_1, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_1); return x_16; } } -LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTacticAux___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTacticAux___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6945,11 +8134,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticAux___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTactic___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Elab_Tactic_evalTacticAux___lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_Elab_Tactic_evalTactic___lambda__1(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; @@ -7059,51 +8248,11 @@ lean_dec(x_2); return x_11; } } -static lean_object* _init_l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_abortTacticExceptionId; -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__1; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__2; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = lean_alloc_closure((void*)(l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg), 1, 0); -return x_9; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_done(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; x_10 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_1); x_11 = !lean_is_exclusive(x_10); if (x_11 == 0) { @@ -7122,7 +8271,7 @@ lean_object* x_16; lean_object* x_17; x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); lean_dec(x_15); -x_17 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg(x_16); +x_17 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg(x_16); return x_17; } else @@ -7182,7 +8331,7 @@ lean_object* x_27; lean_object* x_28; x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); lean_dec(x_26); -x_28 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg(x_27); +x_28 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg(x_27); return x_28; } else @@ -7229,28 +8378,13 @@ return x_34; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_9; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_done___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; x_10 = l_Lean_Elab_Tactic_done(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_2); +lean_dec(x_1); return x_10; } } @@ -7510,6 +8644,7 @@ lean_inc(x_13); lean_dec(x_11); x_14 = l_Lean_Elab_Tactic_done(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); lean_dec(x_3); +lean_dec(x_2); if (lean_obj_tag(x_14) == 0) { uint8_t x_15; @@ -8945,6 +10080,15 @@ x_13 = l_Lean_log___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__3(x_1, x_12, x return x_13; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = 0; +x_12 = l_Lean_Elab_Tactic_SavedState_restore(x_1, x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; +} +} static lean_object* _init_l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___closed__1() { _start: { @@ -8957,7 +10101,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_SavedState_restore___boxed), 10, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___lambda__1___boxed), 10, 0); return x_1; } } @@ -8981,6 +10125,22 @@ x_1 = l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___closed__3; return x_1; } } +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_instMonadBacktrackSavedStateTacticM___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tryCatch___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { @@ -9016,18 +10176,19 @@ return x_15; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); -x_18 = l_Lean_Elab_Tactic_SavedState_restore(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_apply_10(x_2, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_19); -return x_20; +x_18 = 0; +x_19 = l_Lean_Elab_Tactic_SavedState_restore(x_13, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_apply_10(x_2, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_20); +return x_21; } } } @@ -9084,18 +10245,19 @@ return x_16; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); -x_19 = l_Lean_Elab_Tactic_SavedState_restore(x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_apply_10(x_3, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_20); -return x_21; +x_19 = 0; +x_20 = l_Lean_Elab_Tactic_SavedState_restore(x_14, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_apply_10(x_3, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_21); +return x_22; } } } @@ -9222,17 +10384,18 @@ return x_15; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); lean_dec(x_15); -x_17 = l_Lean_Elab_Tactic_SavedState_restore(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_16); -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -x_19 = lean_box(0); -x_20 = lean_apply_10(x_2, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); -return x_20; +x_17 = 0; +x_18 = l_Lean_Elab_Tactic_SavedState_restore(x_13, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_16); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_box(0); +x_21 = lean_apply_10(x_2, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_19); +return x_21; } } } @@ -9367,17 +10530,18 @@ return x_16; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; x_17 = lean_ctor_get(x_16, 1); lean_inc(x_17); lean_dec(x_16); -x_18 = l_Lean_Elab_Tactic_SavedState_restore(x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_box(0); -x_21 = lean_apply_10(x_3, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_19); -return x_21; +x_18 = 0; +x_19 = l_Lean_Elab_Tactic_SavedState_restore(x_14, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_box(0); +x_22 = lean_apply_10(x_3, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_20); +return x_22; } } } @@ -9539,7 +10703,7 @@ lean_inc(x_19); lean_dec(x_17); x_20 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withTacticInfoContext___rarg___lambda__1), 11, 1); lean_closure_set(x_20, 0, x_18); -x_21 = l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(x_16, x_20, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +x_21 = l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(x_16, x_20, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); return x_21; } } @@ -9571,7 +10735,7 @@ lean_dec(x_12); x_14 = lean_st_ref_get(x_6, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 4); +x_16 = lean_ctor_get(x_15, 5); lean_inc(x_16); lean_dec(x_15); x_17 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); @@ -9625,7 +10789,7 @@ lean_inc(x_30); x_31 = lean_ctor_get(x_29, 1); lean_inc(x_31); lean_dec(x_29); -x_32 = lean_ctor_get(x_30, 4); +x_32 = lean_ctor_get(x_30, 5); lean_inc(x_32); lean_dec(x_30); x_33 = lean_ctor_get(x_32, 1); @@ -9650,7 +10814,7 @@ lean_dec(x_37); x_39 = lean_st_ref_take(x_6, x_38); x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 4); +x_41 = lean_ctor_get(x_40, 5); lean_inc(x_41); x_42 = lean_ctor_get(x_39, 1); lean_inc(x_42); @@ -9659,7 +10823,7 @@ x_43 = !lean_is_exclusive(x_40); if (x_43 == 0) { lean_object* x_44; uint8_t x_45; -x_44 = lean_ctor_get(x_40, 4); +x_44 = lean_ctor_get(x_40, 5); lean_dec(x_44); x_45 = !lean_is_exclusive(x_41); if (x_45 == 0) @@ -9704,7 +10868,7 @@ x_56 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_56, 0, x_54); lean_ctor_set(x_56, 1, x_55); lean_ctor_set_uint8(x_56, sizeof(void*)*2, x_53); -lean_ctor_set(x_40, 4, x_56); +lean_ctor_set(x_40, 5, x_56); x_57 = lean_st_ref_set(x_6, x_40, x_42); lean_dec(x_6); x_58 = lean_ctor_get(x_57, 1); @@ -9729,298 +10893,304 @@ return x_60; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; x_61 = lean_ctor_get(x_40, 0); x_62 = lean_ctor_get(x_40, 1); x_63 = lean_ctor_get(x_40, 2); x_64 = lean_ctor_get(x_40, 3); +x_65 = lean_ctor_get(x_40, 4); +lean_inc(x_65); lean_inc(x_64); lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_dec(x_40); -x_65 = lean_ctor_get_uint8(x_41, sizeof(void*)*2); -x_66 = lean_ctor_get(x_41, 0); -lean_inc(x_66); +x_66 = lean_ctor_get_uint8(x_41, sizeof(void*)*2); +x_67 = lean_ctor_get(x_41, 0); +lean_inc(x_67); if (lean_is_exclusive(x_41)) { lean_ctor_release(x_41, 0); lean_ctor_release(x_41, 1); - x_67 = x_41; + x_68 = x_41; } else { lean_dec_ref(x_41); - x_67 = lean_box(0); + x_68 = lean_box(0); } -x_68 = l_Std_PersistentArray_push___rarg(x_22, x_35); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 1); +x_69 = l_Std_PersistentArray_push___rarg(x_22, x_35); +if (lean_is_scalar(x_68)) { + x_70 = lean_alloc_ctor(0, 2, 1); } else { - x_69 = x_67; -} -lean_ctor_set(x_69, 0, x_66); -lean_ctor_set(x_69, 1, x_68); -lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_65); -x_70 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_70, 0, x_61); -lean_ctor_set(x_70, 1, x_62); -lean_ctor_set(x_70, 2, x_63); -lean_ctor_set(x_70, 3, x_64); -lean_ctor_set(x_70, 4, x_69); -x_71 = lean_st_ref_set(x_6, x_70, x_42); -lean_dec(x_6); -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_73 = x_71; + x_70 = x_68; +} +lean_ctor_set(x_70, 0, x_67); +lean_ctor_set(x_70, 1, x_69); +lean_ctor_set_uint8(x_70, sizeof(void*)*2, x_66); +x_71 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_71, 0, x_61); +lean_ctor_set(x_71, 1, x_62); +lean_ctor_set(x_71, 2, x_63); +lean_ctor_set(x_71, 3, x_64); +lean_ctor_set(x_71, 4, x_65); +lean_ctor_set(x_71, 5, x_70); +x_72 = lean_st_ref_set(x_6, x_71, x_42); +lean_dec(x_6); +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_74 = x_72; } else { - lean_dec_ref(x_71); - x_73 = lean_box(0); + lean_dec_ref(x_72); + x_74 = lean_box(0); } -if (lean_is_scalar(x_73)) { - x_74 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(0, 2, 0); } else { - x_74 = x_73; + x_75 = x_74; } -lean_ctor_set(x_74, 0, x_25); -lean_ctor_set(x_74, 1, x_72); -return x_74; +lean_ctor_set(x_75, 0, x_25); +lean_ctor_set(x_75, 1, x_73); +return x_75; } } else { -uint8_t x_75; +uint8_t x_76; lean_dec(x_25); lean_dec(x_22); lean_dec(x_10); lean_dec(x_6); -x_75 = !lean_is_exclusive(x_34); -if (x_75 == 0) +x_76 = !lean_is_exclusive(x_34); +if (x_76 == 0) { return x_34; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_34, 0); -x_77 = lean_ctor_get(x_34, 1); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_34, 0); +x_78 = lean_ctor_get(x_34, 1); +lean_inc(x_78); lean_inc(x_77); -lean_inc(x_76); lean_dec(x_34); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_79 = lean_ctor_get(x_24, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_24, 1); +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_80 = lean_ctor_get(x_24, 0); lean_inc(x_80); +x_81 = lean_ctor_get(x_24, 1); +lean_inc(x_81); lean_dec(x_24); -x_81 = lean_st_ref_get(x_10, x_80); -x_82 = lean_ctor_get(x_81, 1); -lean_inc(x_82); -lean_dec(x_81); -x_83 = lean_st_ref_get(x_6, x_82); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +x_82 = lean_st_ref_get(x_10, x_81); +x_83 = lean_ctor_get(x_82, 1); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_st_ref_get(x_6, x_83); +x_85 = lean_ctor_get(x_84, 0); lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_ctor_get(x_84, 4); +x_86 = lean_ctor_get(x_84, 1); lean_inc(x_86); lean_dec(x_84); -x_87 = lean_ctor_get(x_86, 1); +x_87 = lean_ctor_get(x_85, 5); lean_inc(x_87); -lean_dec(x_86); +lean_dec(x_85); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); lean_inc(x_10); lean_inc(x_6); -x_88 = lean_apply_10(x_2, x_87, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_85); -if (lean_obj_tag(x_88) == 0) +x_89 = lean_apply_10(x_2, x_88, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_86); +if (lean_obj_tag(x_89) == 0) { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_88, 1); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_90 = lean_ctor_get(x_89, 0); lean_inc(x_90); -lean_dec(x_88); -x_91 = lean_st_ref_get(x_10, x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = lean_st_ref_get(x_10, x_91); lean_dec(x_10); -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); -lean_dec(x_91); -x_93 = lean_st_ref_take(x_6, x_92); -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_94, 4); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +x_94 = lean_st_ref_take(x_6, x_93); +x_95 = lean_ctor_get(x_94, 0); lean_inc(x_95); -x_96 = lean_ctor_get(x_93, 1); +x_96 = lean_ctor_get(x_95, 5); lean_inc(x_96); -lean_dec(x_93); -x_97 = !lean_is_exclusive(x_94); -if (x_97 == 0) -{ -lean_object* x_98; uint8_t x_99; -x_98 = lean_ctor_get(x_94, 4); -lean_dec(x_98); -x_99 = !lean_is_exclusive(x_95); -if (x_99 == 0) -{ -lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; -x_100 = lean_ctor_get(x_95, 1); -lean_dec(x_100); -x_101 = l_Std_PersistentArray_push___rarg(x_22, x_89); -lean_ctor_set(x_95, 1, x_101); -x_102 = lean_st_ref_set(x_6, x_94, x_96); -lean_dec(x_6); -x_103 = !lean_is_exclusive(x_102); -if (x_103 == 0) -{ -lean_object* x_104; -x_104 = lean_ctor_get(x_102, 0); -lean_dec(x_104); -lean_ctor_set_tag(x_102, 1); -lean_ctor_set(x_102, 0, x_79); -return x_102; -} -else -{ -lean_object* x_105; lean_object* x_106; -x_105 = lean_ctor_get(x_102, 1); -lean_inc(x_105); -lean_dec(x_102); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_79); -lean_ctor_set(x_106, 1, x_105); -return x_106; +x_97 = lean_ctor_get(x_94, 1); +lean_inc(x_97); +lean_dec(x_94); +x_98 = !lean_is_exclusive(x_95); +if (x_98 == 0) +{ +lean_object* x_99; uint8_t x_100; +x_99 = lean_ctor_get(x_95, 5); +lean_dec(x_99); +x_100 = !lean_is_exclusive(x_96); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; +x_101 = lean_ctor_get(x_96, 1); +lean_dec(x_101); +x_102 = l_Std_PersistentArray_push___rarg(x_22, x_90); +lean_ctor_set(x_96, 1, x_102); +x_103 = lean_st_ref_set(x_6, x_95, x_97); +lean_dec(x_6); +x_104 = !lean_is_exclusive(x_103); +if (x_104 == 0) +{ +lean_object* x_105; +x_105 = lean_ctor_get(x_103, 0); +lean_dec(x_105); +lean_ctor_set_tag(x_103, 1); +lean_ctor_set(x_103, 0, x_80); +return x_103; +} +else +{ +lean_object* x_106; lean_object* x_107; +x_106 = lean_ctor_get(x_103, 1); +lean_inc(x_106); +lean_dec(x_103); +x_107 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_107, 0, x_80); +lean_ctor_set(x_107, 1, x_106); +return x_107; } } else { -uint8_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_107 = lean_ctor_get_uint8(x_95, sizeof(void*)*2); -x_108 = lean_ctor_get(x_95, 0); -lean_inc(x_108); -lean_dec(x_95); -x_109 = l_Std_PersistentArray_push___rarg(x_22, x_89); -x_110 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -lean_ctor_set_uint8(x_110, sizeof(void*)*2, x_107); -lean_ctor_set(x_94, 4, x_110); -x_111 = lean_st_ref_set(x_6, x_94, x_96); -lean_dec(x_6); -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_113 = x_111; +uint8_t x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_108 = lean_ctor_get_uint8(x_96, sizeof(void*)*2); +x_109 = lean_ctor_get(x_96, 0); +lean_inc(x_109); +lean_dec(x_96); +x_110 = l_Std_PersistentArray_push___rarg(x_22, x_90); +x_111 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +lean_ctor_set_uint8(x_111, sizeof(void*)*2, x_108); +lean_ctor_set(x_95, 5, x_111); +x_112 = lean_st_ref_set(x_6, x_95, x_97); +lean_dec(x_6); +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_114 = x_112; } else { - lean_dec_ref(x_111); - x_113 = lean_box(0); + lean_dec_ref(x_112); + x_114 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; - lean_ctor_set_tag(x_114, 1); + x_115 = x_114; + lean_ctor_set_tag(x_115, 1); } -lean_ctor_set(x_114, 0, x_79); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_115, 0, x_80); +lean_ctor_set(x_115, 1, x_113); +return x_115; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_115 = lean_ctor_get(x_94, 0); -x_116 = lean_ctor_get(x_94, 1); -x_117 = lean_ctor_get(x_94, 2); -x_118 = lean_ctor_get(x_94, 3); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; uint8_t x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_116 = lean_ctor_get(x_95, 0); +x_117 = lean_ctor_get(x_95, 1); +x_118 = lean_ctor_get(x_95, 2); +x_119 = lean_ctor_get(x_95, 3); +x_120 = lean_ctor_get(x_95, 4); +lean_inc(x_120); +lean_inc(x_119); lean_inc(x_118); lean_inc(x_117); lean_inc(x_116); -lean_inc(x_115); -lean_dec(x_94); -x_119 = lean_ctor_get_uint8(x_95, sizeof(void*)*2); -x_120 = lean_ctor_get(x_95, 0); -lean_inc(x_120); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_121 = x_95; +lean_dec(x_95); +x_121 = lean_ctor_get_uint8(x_96, sizeof(void*)*2); +x_122 = lean_ctor_get(x_96, 0); +lean_inc(x_122); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_123 = x_96; } else { - lean_dec_ref(x_95); - x_121 = lean_box(0); + lean_dec_ref(x_96); + x_123 = lean_box(0); } -x_122 = l_Std_PersistentArray_push___rarg(x_22, x_89); -if (lean_is_scalar(x_121)) { - x_123 = lean_alloc_ctor(0, 2, 1); +x_124 = l_Std_PersistentArray_push___rarg(x_22, x_90); +if (lean_is_scalar(x_123)) { + x_125 = lean_alloc_ctor(0, 2, 1); } else { - x_123 = x_121; + x_125 = x_123; } -lean_ctor_set(x_123, 0, x_120); -lean_ctor_set(x_123, 1, x_122); -lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_119); -x_124 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_124, 0, x_115); -lean_ctor_set(x_124, 1, x_116); -lean_ctor_set(x_124, 2, x_117); -lean_ctor_set(x_124, 3, x_118); -lean_ctor_set(x_124, 4, x_123); -x_125 = lean_st_ref_set(x_6, x_124, x_96); -lean_dec(x_6); -x_126 = lean_ctor_get(x_125, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - x_127 = x_125; +lean_ctor_set(x_125, 0, x_122); +lean_ctor_set(x_125, 1, x_124); +lean_ctor_set_uint8(x_125, sizeof(void*)*2, x_121); +x_126 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_126, 0, x_116); +lean_ctor_set(x_126, 1, x_117); +lean_ctor_set(x_126, 2, x_118); +lean_ctor_set(x_126, 3, x_119); +lean_ctor_set(x_126, 4, x_120); +lean_ctor_set(x_126, 5, x_125); +x_127 = lean_st_ref_set(x_6, x_126, x_97); +lean_dec(x_6); +x_128 = lean_ctor_get(x_127, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_129 = x_127; } else { - lean_dec_ref(x_125); - x_127 = lean_box(0); + lean_dec_ref(x_127); + x_129 = lean_box(0); } -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(1, 2, 0); } else { - x_128 = x_127; - lean_ctor_set_tag(x_128, 1); + x_130 = x_129; + lean_ctor_set_tag(x_130, 1); } -lean_ctor_set(x_128, 0, x_79); -lean_ctor_set(x_128, 1, x_126); -return x_128; +lean_ctor_set(x_130, 0, x_80); +lean_ctor_set(x_130, 1, x_128); +return x_130; } } else { -uint8_t x_129; -lean_dec(x_79); +uint8_t x_131; +lean_dec(x_80); lean_dec(x_22); lean_dec(x_10); lean_dec(x_6); -x_129 = !lean_is_exclusive(x_88); -if (x_129 == 0) +x_131 = !lean_is_exclusive(x_89); +if (x_131 == 0) { -return x_88; +return x_89; } else { -lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_130 = lean_ctor_get(x_88, 0); -x_131 = lean_ctor_get(x_88, 1); -lean_inc(x_131); -lean_inc(x_130); -lean_dec(x_88); -x_132 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); -return x_132; +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_89, 0); +x_133 = lean_ctor_get(x_89, 1); +lean_inc(x_133); +lean_inc(x_132); +lean_dec(x_89); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; } } } @@ -10195,7 +11365,7 @@ lean_object* x_13; lean_object* x_14; x_13 = lean_alloc_closure((void*)(l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Tactic_withMacroExpansion___spec__1___rarg___lambda__1___boxed), 12, 2); lean_closure_set(x_13, 0, x_1); lean_closure_set(x_13, 1, x_2); -x_14 = l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(x_3, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(x_3, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_14; } } @@ -10216,7 +11386,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); lean_ctor_set(x_5, 2, x_15); -x_16 = l_Lean_Elab_Tactic_evalTacticAux(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_16 = l_Lean_Elab_Tactic_evalTactic(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); return x_16; } else @@ -10271,7 +11441,7 @@ lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 4, x_28); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 5, x_29); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 6, x_30); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 7, x_32); -x_36 = l_Lean_Elab_Tactic_evalTacticAux(x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11); +x_36 = l_Lean_Elab_Tactic_evalTactic(x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11); return x_36; } } @@ -11077,7 +12247,7 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_19 = l_Lean_Elab_Tactic_evalTacticAux(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +x_19 = l_Lean_Elab_Tactic_evalTactic(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; @@ -11246,7 +12416,7 @@ x_27 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; x_28 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_28, 0, x_26); lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -11291,7 +12461,7 @@ x_37 = l_Lean_Elab_Term_reportUnsolvedGoals___closed__8; x_38 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_38, 0, x_36); lean_ctor_set(x_38, 1, x_37); -x_39 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_30); +x_39 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_30); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -12287,11 +13457,12 @@ return x_21; } else { -lean_object* x_22; lean_object* x_23; uint8_t x_24; +lean_object* x_22; uint8_t x_23; lean_object* x_24; uint8_t x_25; x_22 = lean_ctor_get(x_14, 1); lean_inc(x_22); lean_dec(x_14); -x_23 = l_Lean_Elab_Tactic_SavedState_restore(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_22); +x_23 = 0; +x_24 = l_Lean_Elab_Tactic_SavedState_restore(x_12, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_22); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -12300,27 +13471,27 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_23, 0); -lean_dec(x_25); -x_26 = lean_box(0); -lean_ctor_set(x_23, 0, x_26); -return x_23; +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_24, 0); +lean_dec(x_26); +x_27 = lean_box(0); +lean_ctor_set(x_24, 0, x_27); +return x_24; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_23, 1); -lean_inc(x_27); -lean_dec(x_23); -x_28 = lean_box(0); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_27); -return x_29; +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_24, 1); +lean_inc(x_28); +lean_dec(x_24); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +return x_30; } } } @@ -12391,11 +13562,12 @@ return x_22; } else { -lean_object* x_23; lean_object* x_24; uint8_t x_25; +lean_object* x_23; uint8_t x_24; lean_object* x_25; uint8_t x_26; x_23 = lean_ctor_get(x_14, 1); lean_inc(x_23); lean_dec(x_14); -x_24 = l_Lean_Elab_Tactic_SavedState_restore(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +x_24 = 0; +x_25 = l_Lean_Elab_Tactic_SavedState_restore(x_12, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -12404,29 +13576,27 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -lean_object* x_26; uint8_t x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_24, 0); -lean_dec(x_26); -x_27 = 0; -x_28 = lean_box(x_27); -lean_ctor_set(x_24, 0, x_28); -return x_24; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +x_28 = lean_box(x_24); +lean_ctor_set(x_25, 0, x_28); +return x_25; } else { -lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; -x_29 = lean_ctor_get(x_24, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_25, 1); lean_inc(x_29); -lean_dec(x_24); -x_30 = 0; -x_31 = lean_box(x_30); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_29); -return x_32; +lean_dec(x_25); +x_30 = lean_box(x_24); +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; } } } @@ -12946,7 +14116,7 @@ x_6 = l_Lean_Elab_Tactic_withCaseRef___rarg___closed__1; x_7 = lean_array_push(x_6, x_3); x_8 = lean_array_push(x_7, x_4); x_9 = lean_box(2); -x_10 = l_Lean_Elab_Tactic_evalTacticAux___closed__3; +x_10 = l_Lean_Elab_Tactic_evalTactic___closed__3; x_11 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_11, 0, x_9); lean_ctor_set(x_11, 1, x_10); @@ -12982,21 +14152,21 @@ lean_dec(x_1); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_evalTacticAux___closed__4; +x_1 = l_Lean_Elab_Tactic_evalTactic___closed__4; x_2 = l_Lean_Elab_Tactic_mkTacticAttribute___closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437____closed__1; +x_2 = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621____closed__1; x_3 = l_Lean_registerTraceClass(x_2, x_1); return x_3; } @@ -13142,68 +14312,94 @@ l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec lean_mark_persistent(l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___closed__2); l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___closed__3 = _init_l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___closed__3(); lean_mark_persistent(l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Tactic_withTacticInfoContext___spec__2___rarg___closed__3); -l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__1 = _init_l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__1); -l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__2 = _init_l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__2); -l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__3 = _init_l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___closed__3); -l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__1 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__1(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__1); -l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__2 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__2(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__2); -l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__3 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__3(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__3); -l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__4 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__4(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__4); -l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__5 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__5(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__5); -l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__6 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__6(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3___closed__6); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__1(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__1); -l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__2(); -lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__7___closed__2); -l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__8___rarg___closed__1); -l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__1 = _init_l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__1); -l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__2 = _init_l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__2); -l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__3 = _init_l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__3); -l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__4 = _init_l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_expandTacticMacroFns_loop___closed__4); -l_Lean_Elab_Tactic_evalTacticAux___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_evalTacticAux___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___lambda__2___closed__1); -l_Lean_Elab_Tactic_evalTacticAux___closed__1 = _init_l_Lean_Elab_Tactic_evalTacticAux___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___closed__1); -l_Lean_Elab_Tactic_evalTacticAux___closed__2 = _init_l_Lean_Elab_Tactic_evalTacticAux___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___closed__2); -l_Lean_Elab_Tactic_evalTacticAux___closed__3 = _init_l_Lean_Elab_Tactic_evalTacticAux___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___closed__3); -l_Lean_Elab_Tactic_evalTacticAux___closed__4 = _init_l_Lean_Elab_Tactic_evalTacticAux___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___closed__4); -l_Lean_Elab_Tactic_evalTacticAux___closed__5 = _init_l_Lean_Elab_Tactic_evalTacticAux___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___closed__5); -l_Lean_Elab_Tactic_evalTacticAux___closed__6 = _init_l_Lean_Elab_Tactic_evalTacticAux___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___closed__6); -l_Lean_Elab_Tactic_evalTacticAux___closed__7 = _init_l_Lean_Elab_Tactic_evalTacticAux___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___closed__7); -l_Lean_Elab_Tactic_evalTacticAux___closed__8 = _init_l_Lean_Elab_Tactic_evalTacticAux___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___closed__8); -l_Lean_Elab_Tactic_evalTacticAux___boxed__const__1 = _init_l_Lean_Elab_Tactic_evalTacticAux___boxed__const__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalTacticAux___boxed__const__1); -l_Lean_Elab_Tactic_expandTacticMacro___closed__1 = _init_l_Lean_Elab_Tactic_expandTacticMacro___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_expandTacticMacro___closed__1); +l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1 = _init_l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__1); +l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__2 = _init_l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__3___rarg___closed__2); +l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1 = _init_l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1(); +lean_mark_persistent(l_Array_filterMapM___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__4___closed__1); +l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__1 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__1(); +lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__1); +l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__2 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__2(); +lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__2); +l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__3 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__3(); +lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__3); +l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__4 = _init_l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__4(); +lean_mark_persistent(l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__7___closed__4); +l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__1 = _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__1); +l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__2 = _init_l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__2(); +lean_mark_persistent(l_Lean_Elab_throwErrorWithNestedErrors___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__6___closed__2); +l_Lean_Elab_Tactic_evalTactic_throwExs___closed__1 = _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_throwExs___closed__1); +l_Lean_Elab_Tactic_evalTactic_throwExs___closed__2 = _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_throwExs___closed__2); +l_Lean_Elab_Tactic_evalTactic_throwExs___closed__3 = _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_throwExs___closed__3); +l_Lean_Elab_Tactic_evalTactic_throwExs___closed__4 = _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_throwExs___closed__4); +l_Lean_Elab_Tactic_evalTactic_throwExs___closed__5 = _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_throwExs___closed__5); +l_Lean_Elab_Tactic_evalTactic_throwExs___closed__6 = _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_throwExs___closed__6); +l_Lean_Elab_Tactic_evalTactic_throwExs___closed__7 = _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_throwExs___closed__7); +l_Lean_Elab_Tactic_evalTactic_throwExs___closed__8 = _init_l_Lean_Elab_Tactic_evalTactic_throwExs___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_throwExs___closed__8); +l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1 = _init_l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic_handleEx___closed__1); +l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__1 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__1(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__1); +l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__2 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__2(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__2); +l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__3 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__3(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__3); +l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__4 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__4(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__4); +l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__5 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__5(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__5); +l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__6 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__6(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3___closed__6); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__1(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__1); +l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__2 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__2(); +lean_mark_persistent(l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__7___closed__2); +l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__8___rarg___closed__1); +l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__1); +l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__2); +l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__3 = _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__3); +l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__4 = _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__4); +l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__5 = _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__5); +l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__6 = _init_l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___lambda__3___closed__6); +l_Lean_Elab_Tactic_evalTactic___closed__1 = _init_l_Lean_Elab_Tactic_evalTactic___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___closed__1); +l_Lean_Elab_Tactic_evalTactic___closed__2 = _init_l_Lean_Elab_Tactic_evalTactic___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___closed__2); +l_Lean_Elab_Tactic_evalTactic___closed__3 = _init_l_Lean_Elab_Tactic_evalTactic___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___closed__3); +l_Lean_Elab_Tactic_evalTactic___closed__4 = _init_l_Lean_Elab_Tactic_evalTactic___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___closed__4); +l_Lean_Elab_Tactic_evalTactic___closed__5 = _init_l_Lean_Elab_Tactic_evalTactic___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___closed__5); +l_Lean_Elab_Tactic_evalTactic___closed__6 = _init_l_Lean_Elab_Tactic_evalTactic___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___closed__6); +l_Lean_Elab_Tactic_evalTactic___closed__7 = _init_l_Lean_Elab_Tactic_evalTactic___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___closed__7); +l_Lean_Elab_Tactic_evalTactic___closed__8 = _init_l_Lean_Elab_Tactic_evalTactic___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___closed__8); +l_Lean_Elab_Tactic_evalTactic___boxed__const__1 = _init_l_Lean_Elab_Tactic_evalTactic___boxed__const__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_evalTactic___boxed__const__1); l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg___closed__1 = _init_l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg___closed__1); l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg___closed__2 = _init_l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg___closed__2(); lean_mark_persistent(l_Lean_Elab_Tactic_throwNoGoalsToBeSolved___rarg___closed__2); -l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__1 = _init_l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__1); -l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__2 = _init_l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__2(); -lean_mark_persistent(l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_done___spec__1___rarg___closed__2); l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1___closed__1 = _init_l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1___closed__1(); lean_mark_persistent(l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1___closed__1); l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1___closed__2 = _init_l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1___closed__2(); @@ -13252,9 +14448,9 @@ l_Lean_Elab_Tactic_getNameOfIdent_x27___closed__2 = _init_l_Lean_Elab_Tactic_get lean_mark_persistent(l_Lean_Elab_Tactic_getNameOfIdent_x27___closed__2); l_Lean_Elab_Tactic_withCaseRef___rarg___closed__1 = _init_l_Lean_Elab_Tactic_withCaseRef___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_withCaseRef___rarg___closed__1); -l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437____closed__1); -res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_3437_(lean_io_mk_world()); +l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621____closed__1 = _init_l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621____closed__1); +res = l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Basic___hyg_4621_(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 85b352d57221..f654104a8906 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BuiltinTactic.c @@ -66,7 +66,6 @@ static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_evalOpen__ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalIntros_declRange___closed__2; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRotateRight(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_RBNode_insert___at_Lean_NameSet_insert___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Tactic_renameInaccessibles___spec__5___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticSeq1Indented(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -92,7 +91,7 @@ static lean_object* l_Lean_Elab_Tactic_evalIntro___closed__10; static lean_object* l_Lean_Elab_Tactic_evalIntro___closed__32; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSkip___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_evalSubstVars_declRange___closed__5; -lean_object* l_Lean_Elab_Tactic_SavedState_restore(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_SavedState_restore(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalChoiceAux___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSeq1_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRefl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -160,7 +159,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDbgTrace(lean_objec static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDone___closed__5; static lean_object* l_Lean_Elab_Tactic_evalCase___closed__1; static lean_object* l___private_Lean_Elab_Open_0__Lean_Elab_OpenDecl_resolveNameUsingNamespacesCore___at_Lean_Elab_Tactic_evalOpen___spec__22___closed__3; -lean_object* l_Lean_Elab_Tactic_evalTacticAux(lean_object*, lean_object*, 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_evalOpen___spec__11___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_done(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalOpen___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -508,7 +506,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDone(lean_object*); static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalOpen___spec__25___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalFocus___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalFailIfSuccess_declRange___closed__2; -lean_object* l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getUnsolvedGoals(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_Open_0__Lean_Elab_OpenDecl_elabOpenScoped___at_Lean_Elab_Tactic_evalOpen___spec__29(lean_object*, 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_evalOpen_declRange___closed__4; @@ -550,7 +547,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalAssumption___closed__1; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalOpen___spec__2___closed__7; lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSubstVars___closed__3; -lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Term_runTactic___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDone___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalTraceState_declRange___closed__2; @@ -575,7 +571,6 @@ lean_object* l_Array_back___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Tactic_renameInaccessibles___spec__5___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSleep(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_evalRefl___closed__1; -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___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_evalRenameInaccessibles_declRange___closed__3; static lean_object* l_Lean_Elab_Tactic_evalIntro___closed__26; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Tactic_addCheckpoints___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -726,8 +721,10 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAssumption___boxed(lean_object*) LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalFirst_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_elabSetOption___at_Lean_Elab_Tactic_elabSetOption___spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_forEachVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_addCheckpoints_push___closed__10; lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_saveTacticInfoForToken___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* 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*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRevert(lean_object*, 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_evalFocus(lean_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_evalWithAnnotateState___closed__1; @@ -825,6 +822,7 @@ lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRotateLeft(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalParen_declRange(lean_object*); +lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_renameInaccessibles___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalFail___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSubstVars___closed__1; @@ -883,6 +881,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalFail(lean_object*, lean_object*, static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithAnnotateState_declRange___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_renameInaccessibles___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalIntro___closed__9; +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*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalFailIfSuccess(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_evalOpen___spec__35___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalWithAnnotateState___closed__7; @@ -1332,7 +1331,7 @@ lean_inc(x_21); lean_dec(x_19); x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalWithAnnotateState___lambda__1), 11, 1); lean_closure_set(x_22, 0, x_20); -x_23 = l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(x_18, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +x_23 = l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(x_18, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_21); return x_23; } } @@ -1535,6 +1534,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalDone___rarg___boxed(lean_object* lean_object* x_10; x_10 = l_Lean_Elab_Tactic_evalDone___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_2); +lean_dec(x_1); return x_10; } } @@ -1735,7 +1735,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_evalSeq1_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_evalSeq1___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_evalSeq1___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_evalSeq1___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1910,7 +1910,7 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_52 = l_Lean_Elab_Tactic_evalTacticAux(x_51, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_52 = l_Lean_Elab_Tactic_evalTactic(x_51, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); if (lean_obj_tag(x_52) == 0) { lean_object* x_53; lean_object* x_54; @@ -1967,7 +1967,7 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_60 = l_Lean_Elab_Tactic_evalTacticAux(x_59, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_60 = l_Lean_Elab_Tactic_evalTactic(x_59, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); if (lean_obj_tag(x_60) == 0) { lean_object* x_61; lean_object* x_62; @@ -2314,7 +2314,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalParen(lean_object* x_1, lean_obj lean_object* x_11; lean_object* x_12; lean_object* x_13; x_11 = lean_unsigned_to_nat(1u); x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_13; } } @@ -3056,7 +3056,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_19 = l_Lean_Elab_Tactic_evalTacticAux(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_19 = l_Lean_Elab_Tactic_evalTactic(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_19) == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; @@ -3736,7 +3736,7 @@ lean_inc(x_14); lean_dec(x_13); x_15 = lean_unsigned_to_nat(1u); x_16 = l_Lean_Syntax_getArg(x_3, x_15); -x_17 = l_Lean_Elab_Tactic_evalTacticAux(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_14); +x_17 = l_Lean_Elab_Tactic_evalTactic(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_14); return x_17; } else @@ -9192,7 +9192,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_31 = l_Lean_Elab_Tactic_evalTacticAux(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_30, x_9, x_17); +x_31 = l_Lean_Elab_Tactic_evalTactic(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_30, x_9, x_17); if (lean_obj_tag(x_31) == 0) { lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; @@ -10023,7 +10023,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -10068,7 +10068,7 @@ lean_dec(x_24); x_26 = lean_st_ref_take(x_5, x_25); x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -x_28 = lean_ctor_get(x_27, 4); +x_28 = lean_ctor_get(x_27, 5); lean_inc(x_28); x_29 = lean_ctor_get(x_26, 1); lean_inc(x_29); @@ -10077,7 +10077,7 @@ x_30 = !lean_is_exclusive(x_27); if (x_30 == 0) { lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_27, 4); +x_31 = lean_ctor_get(x_27, 5); lean_dec(x_31); x_32 = !lean_is_exclusive(x_28); if (x_32 == 0) @@ -10124,7 +10124,7 @@ x_46 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_46, 0, x_43); lean_ctor_set(x_46, 1, x_45); lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_42); -lean_ctor_set(x_27, 4, x_46); +lean_ctor_set(x_27, 5, x_46); x_47 = lean_st_ref_set(x_5, x_27, x_29); x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); @@ -10149,64 +10149,67 @@ return x_51; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; x_52 = lean_ctor_get(x_27, 0); x_53 = lean_ctor_get(x_27, 1); x_54 = lean_ctor_get(x_27, 2); x_55 = lean_ctor_get(x_27, 3); +x_56 = lean_ctor_get(x_27, 4); +lean_inc(x_56); lean_inc(x_55); lean_inc(x_54); lean_inc(x_53); lean_inc(x_52); lean_dec(x_27); -x_56 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); -x_57 = lean_ctor_get(x_28, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_28, 1); +x_57 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); +x_58 = lean_ctor_get(x_28, 0); lean_inc(x_58); +x_59 = lean_ctor_get(x_28, 1); +lean_inc(x_59); if (lean_is_exclusive(x_28)) { lean_ctor_release(x_28, 0); lean_ctor_release(x_28, 1); - x_59 = x_28; + x_60 = x_28; } else { lean_dec_ref(x_28); - x_59 = lean_box(0); + x_60 = lean_box(0); } -x_60 = l_Std_PersistentArray_push___rarg(x_58, x_1); -if (lean_is_scalar(x_59)) { - x_61 = lean_alloc_ctor(0, 2, 1); +x_61 = l_Std_PersistentArray_push___rarg(x_59, x_1); +if (lean_is_scalar(x_60)) { + x_62 = lean_alloc_ctor(0, 2, 1); } else { - x_61 = x_59; -} -lean_ctor_set(x_61, 0, x_57); -lean_ctor_set(x_61, 1, x_60); -lean_ctor_set_uint8(x_61, sizeof(void*)*2, x_56); -x_62 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_62, 0, x_52); -lean_ctor_set(x_62, 1, x_53); -lean_ctor_set(x_62, 2, x_54); -lean_ctor_set(x_62, 3, x_55); -lean_ctor_set(x_62, 4, x_61); -x_63 = lean_st_ref_set(x_5, x_62, x_29); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; + x_62 = x_60; +} +lean_ctor_set(x_62, 0, x_58); +lean_ctor_set(x_62, 1, x_61); +lean_ctor_set_uint8(x_62, sizeof(void*)*2, x_57); +x_63 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_63, 0, x_52); +lean_ctor_set(x_63, 1, x_53); +lean_ctor_set(x_63, 2, x_54); +lean_ctor_set(x_63, 3, x_55); +lean_ctor_set(x_63, 4, x_56); +lean_ctor_set(x_63, 5, x_62); +x_64 = lean_st_ref_set(x_5, x_63, x_29); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_66 = x_64; } else { - lean_dec_ref(x_63); - x_65 = lean_box(0); + lean_dec_ref(x_64); + x_66 = lean_box(0); } -x_66 = lean_box(0); -if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 0); +x_67 = lean_box(0); +if (lean_is_scalar(x_66)) { + x_68 = lean_alloc_ctor(0, 2, 0); } else { - x_67 = x_65; + x_68 = x_66; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_64); -return x_67; +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_68, 1, x_65); +return x_68; } } } @@ -10258,7 +10261,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -10412,7 +10415,7 @@ lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_dec(x_2); lean_dec(x_1); x_18 = l_Lean_Elab_elabSetOption_setOption___at_Lean_Elab_Tactic_elabSetOption___spec__6___closed__2; -x_19 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +x_19 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -10746,7 +10749,7 @@ x_23 = l_Lean_Elab_Tactic_elabSetOption___closed__1; x_24 = l_Lean_Option_get___at_Std_Format_pretty_x27___spec__1(x_16, x_23); lean_ctor_set(x_8, 4, x_24); lean_ctor_set(x_8, 2, x_16); -x_25 = l_Lean_Elab_Tactic_evalTacticAux(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +x_25 = l_Lean_Elab_Tactic_evalTactic(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); return x_25; } else @@ -10785,7 +10788,7 @@ lean_ctor_set(x_37, 7, x_31); lean_ctor_set(x_37, 8, x_32); lean_ctor_set(x_37, 9, x_33); lean_ctor_set(x_37, 10, x_34); -x_38 = l_Lean_Elab_Tactic_evalTacticAux(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_37, x_9, x_17); +x_38 = l_Lean_Elab_Tactic_evalTactic(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_37, x_9, x_17); return x_38; } } @@ -11105,7 +11108,7 @@ x_20 = lean_unbox(x_19); lean_dec(x_19); if (x_20 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_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_47; +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_48; x_21 = lean_ctor_get(x_18, 1); lean_inc(x_21); lean_dec(x_18); @@ -11132,47 +11135,48 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_47 = l_Lean_Elab_Tactic_evalTacticAux(x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_28); -if (lean_obj_tag(x_47) == 0) +x_48 = l_Lean_Elab_Tactic_evalTactic(x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_28); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_dec(x_27); lean_dec(x_16); -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -lean_dec(x_47); -x_49 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_48); -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_49); +x_51 = lean_ctor_get(x_50, 0); lean_inc(x_51); -lean_dec(x_49); -x_52 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_4, x_50); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_53 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_4, x_51); x_3 = x_17; -x_4 = x_52; -x_13 = x_51; +x_4 = x_53; +x_13 = x_52; goto _start; } else { -lean_object* x_54; lean_object* x_55; -x_54 = lean_ctor_get(x_47, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_47, 1); +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_48, 0); lean_inc(x_55); -lean_dec(x_47); -x_29 = x_54; -x_30 = x_55; -goto block_46; +x_56 = lean_ctor_get(x_48, 1); +lean_inc(x_56); +lean_dec(x_48); +x_29 = x_55; +x_30 = x_56; +goto block_47; } -block_46: +block_47: { -lean_object* x_31; uint8_t x_32; -x_31 = l_Lean_Elab_Tactic_SavedState_restore(x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_30); -x_32 = lean_ctor_get_uint8(x_5, sizeof(void*)*1); -if (x_32 == 0) +uint8_t x_31; lean_object* x_32; uint8_t x_33; +x_31 = 0; +x_32 = l_Lean_Elab_Tactic_SavedState_restore(x_27, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_30); +x_33 = lean_ctor_get_uint8(x_5, sizeof(void*)*1); +if (x_33 == 0) { -uint8_t x_33; +uint8_t x_34; lean_dec(x_17); lean_dec(x_16); lean_dec(x_12); @@ -11185,34 +11189,34 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_33 = !lean_is_exclusive(x_31); -if (x_33 == 0) +x_34 = !lean_is_exclusive(x_32); +if (x_34 == 0) { -lean_object* x_34; -x_34 = lean_ctor_get(x_31, 0); -lean_dec(x_34); -lean_ctor_set_tag(x_31, 1); -lean_ctor_set(x_31, 0, x_29); -return x_31; +lean_object* x_35; +x_35 = lean_ctor_get(x_32, 0); +lean_dec(x_35); +lean_ctor_set_tag(x_32, 1); +lean_ctor_set(x_32, 0, x_29); +return x_32; } else { -lean_object* x_35; lean_object* x_36; -x_35 = lean_ctor_get(x_31, 1); -lean_inc(x_35); -lean_dec(x_31); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_29); -lean_ctor_set(x_36, 1, x_35); -return x_36; +lean_object* x_36; lean_object* x_37; +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); +lean_dec(x_32); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_29); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } else { -lean_object* x_37; lean_object* x_38; -x_37 = lean_ctor_get(x_31, 1); -lean_inc(x_37); -lean_dec(x_31); +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_32, 1); +lean_inc(x_38); +lean_dec(x_32); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -11221,22 +11225,22 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_38 = l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1(x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_37); -if (lean_obj_tag(x_38) == 0) +x_39 = l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1(x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_38); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_38, 1); -lean_inc(x_39); -lean_dec(x_38); -x_40 = lean_array_push(x_4, x_16); +lean_object* x_40; lean_object* x_41; +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_41 = lean_array_push(x_4, x_16); x_3 = x_17; -x_4 = x_40; -x_13 = x_39; +x_4 = x_41; +x_13 = x_40; goto _start; } else { -uint8_t x_42; +uint8_t x_43; lean_dec(x_17); lean_dec(x_16); lean_dec(x_12); @@ -11249,23 +11253,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_42 = !lean_is_exclusive(x_38); -if (x_42 == 0) +x_43 = !lean_is_exclusive(x_39); +if (x_43 == 0) { -return x_38; +return x_39; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_38, 0); -x_44 = lean_ctor_get(x_38, 1); +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_39, 0); +x_45 = lean_ctor_get(x_39, 1); +lean_inc(x_45); lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_38); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -return x_45; +lean_dec(x_39); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } } } @@ -11273,54 +11277,54 @@ return x_45; } else { -lean_object* x_56; +lean_object* x_57; lean_free_object(x_3); lean_dec(x_16); -x_56 = lean_ctor_get(x_18, 1); -lean_inc(x_56); +x_57 = lean_ctor_get(x_18, 1); +lean_inc(x_57); lean_dec(x_18); x_3 = x_17; -x_13 = x_56; +x_13 = x_57; goto _start; } } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_58 = lean_ctor_get(x_3, 0); -x_59 = lean_ctor_get(x_3, 1); +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_59 = lean_ctor_get(x_3, 0); +x_60 = lean_ctor_get(x_3, 1); +lean_inc(x_60); lean_inc(x_59); -lean_inc(x_58); lean_dec(x_3); -lean_inc(x_58); -x_60 = l_Lean_isExprMVarAssigned___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__1(x_58, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_unbox(x_61); -lean_dec(x_61); -if (x_62 == 0) +lean_inc(x_59); +x_61 = l_Lean_isExprMVarAssigned___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__1(x_59, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = lean_unbox(x_62); +lean_dec(x_62); +if (x_63 == 0) { -lean_object* x_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_89; -x_63 = lean_ctor_get(x_60, 1); -lean_inc(x_63); -lean_dec(x_60); +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_91; +x_64 = lean_ctor_get(x_61, 1); +lean_inc(x_64); +lean_dec(x_61); lean_inc(x_2); -lean_inc(x_58); -x_64 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_64, 0, x_58); -lean_ctor_set(x_64, 1, x_2); -x_65 = l_Lean_Elab_Tactic_setGoals(x_64, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_63); -x_66 = lean_ctor_get(x_65, 1); -lean_inc(x_66); -lean_dec(x_65); -x_67 = lean_unsigned_to_nat(1u); -x_68 = l_Lean_Syntax_getArg(x_1, x_67); -x_69 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_66); -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_59); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_59); +lean_ctor_set(x_65, 1, x_2); +x_66 = l_Lean_Elab_Tactic_setGoals(x_65, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_64); +x_67 = lean_ctor_get(x_66, 1); +lean_inc(x_67); +lean_dec(x_66); +x_68 = lean_unsigned_to_nat(1u); +x_69 = l_Lean_Syntax_getArg(x_1, x_68); +x_70 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_67); +x_71 = lean_ctor_get(x_70, 0); lean_inc(x_71); -lean_dec(x_69); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -11329,49 +11333,50 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_89 = l_Lean_Elab_Tactic_evalTacticAux(x_68, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_71); -if (lean_obj_tag(x_89) == 0) +x_91 = l_Lean_Elab_Tactic_evalTactic(x_69, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_72); +if (lean_obj_tag(x_91) == 0) { -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -lean_dec(x_70); -lean_dec(x_58); -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); -lean_dec(x_89); -x_91 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_90); -x_92 = lean_ctor_get(x_91, 0); +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +lean_dec(x_71); +lean_dec(x_59); +x_92 = lean_ctor_get(x_91, 1); lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); lean_dec(x_91); -x_94 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_4, x_92); -x_3 = x_59; -x_4 = x_94; -x_13 = x_93; +x_93 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_92); +x_94 = lean_ctor_get(x_93, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_93, 1); +lean_inc(x_95); +lean_dec(x_93); +x_96 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_4, x_94); +x_3 = x_60; +x_4 = x_96; +x_13 = x_95; goto _start; } else { -lean_object* x_96; lean_object* x_97; -x_96 = lean_ctor_get(x_89, 0); -lean_inc(x_96); -x_97 = lean_ctor_get(x_89, 1); -lean_inc(x_97); -lean_dec(x_89); -x_72 = x_96; -x_73 = x_97; -goto block_88; +lean_object* x_98; lean_object* x_99; +x_98 = lean_ctor_get(x_91, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_91, 1); +lean_inc(x_99); +lean_dec(x_91); +x_73 = x_98; +x_74 = x_99; +goto block_90; } -block_88: +block_90: { -lean_object* x_74; uint8_t x_75; -x_74 = l_Lean_Elab_Tactic_SavedState_restore(x_70, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_73); -x_75 = lean_ctor_get_uint8(x_5, sizeof(void*)*1); -if (x_75 == 0) +uint8_t x_75; lean_object* x_76; uint8_t x_77; +x_75 = 0; +x_76 = l_Lean_Elab_Tactic_SavedState_restore(x_71, x_75, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_74); +x_77 = lean_ctor_get_uint8(x_5, sizeof(void*)*1); +if (x_77 == 0) { -lean_object* x_76; lean_object* x_77; lean_object* x_78; +lean_object* x_78; lean_object* x_79; lean_object* x_80; +lean_dec(x_60); lean_dec(x_59); -lean_dec(x_58); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -11382,32 +11387,32 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -if (lean_is_exclusive(x_74)) { - lean_ctor_release(x_74, 0); - lean_ctor_release(x_74, 1); - x_77 = x_74; +x_78 = lean_ctor_get(x_76, 1); +lean_inc(x_78); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + x_79 = x_76; } else { - lean_dec_ref(x_74); - x_77 = lean_box(0); + lean_dec_ref(x_76); + x_79 = lean_box(0); } -if (lean_is_scalar(x_77)) { - x_78 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_79)) { + x_80 = lean_alloc_ctor(1, 2, 0); } else { - x_78 = x_77; - lean_ctor_set_tag(x_78, 1); + x_80 = x_79; + lean_ctor_set_tag(x_80, 1); } -lean_ctor_set(x_78, 0, x_72); -lean_ctor_set(x_78, 1, x_76); -return x_78; +lean_ctor_set(x_80, 0, x_73); +lean_ctor_set(x_80, 1, x_78); +return x_80; } else { -lean_object* x_79; lean_object* x_80; -x_79 = lean_ctor_get(x_74, 1); -lean_inc(x_79); -lean_dec(x_74); +lean_object* x_81; lean_object* x_82; +x_81 = lean_ctor_get(x_76, 1); +lean_inc(x_81); +lean_dec(x_76); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -11416,24 +11421,24 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_80 = l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1(x_72, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_79); -if (lean_obj_tag(x_80) == 0) -{ -lean_object* x_81; lean_object* x_82; -x_81 = lean_ctor_get(x_80, 1); -lean_inc(x_81); -lean_dec(x_80); -x_82 = lean_array_push(x_4, x_58); -x_3 = x_59; -x_4 = x_82; -x_13 = x_81; +x_82 = l_Lean_Elab_logException___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__1(x_73, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_81); +if (lean_obj_tag(x_82) == 0) +{ +lean_object* x_83; lean_object* x_84; +x_83 = lean_ctor_get(x_82, 1); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_array_push(x_4, x_59); +x_3 = x_60; +x_4 = x_84; +x_13 = x_83; goto _start; } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_dec(x_60); lean_dec(x_59); -lean_dec(x_58); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -11444,39 +11449,39 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_84 = lean_ctor_get(x_80, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_80, 1); -lean_inc(x_85); -if (lean_is_exclusive(x_80)) { - lean_ctor_release(x_80, 0); - lean_ctor_release(x_80, 1); - x_86 = x_80; +x_86 = lean_ctor_get(x_82, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_82, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_82)) { + lean_ctor_release(x_82, 0); + lean_ctor_release(x_82, 1); + x_88 = x_82; } else { - lean_dec_ref(x_80); - x_86 = lean_box(0); + lean_dec_ref(x_82); + x_88 = lean_box(0); } -if (lean_is_scalar(x_86)) { - x_87 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_88)) { + x_89 = lean_alloc_ctor(1, 2, 0); } else { - x_87 = x_86; + x_89 = x_88; } -lean_ctor_set(x_87, 0, x_84); -lean_ctor_set(x_87, 1, x_85); -return x_87; +lean_ctor_set(x_89, 0, x_86); +lean_ctor_set(x_89, 1, x_87); +return x_89; } } } } else { -lean_object* x_98; -lean_dec(x_58); -x_98 = lean_ctor_get(x_60, 1); -lean_inc(x_98); -lean_dec(x_60); -x_3 = x_59; -x_13 = x_98; +lean_object* x_100; +lean_dec(x_59); +x_100 = lean_ctor_get(x_61, 1); +lean_inc(x_100); +lean_dec(x_61); +x_3 = x_60; +x_13 = x_100; goto _start; } } @@ -11802,7 +11807,7 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_42 = l_Lean_Elab_Tactic_evalTacticAux(x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_41); +x_42 = l_Lean_Elab_Tactic_evalTactic(x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_41); if (lean_obj_tag(x_42) == 0) { lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; @@ -11833,73 +11838,74 @@ goto block_27; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +lean_object* x_52; uint8_t x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; x_52 = lean_ctor_get(x_42, 1); lean_inc(x_52); lean_dec(x_42); -x_53 = l_Lean_Elab_Tactic_SavedState_restore(x_40, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_52); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_array_push(x_29, x_16); -lean_ctor_set(x_4, 0, x_55); -x_56 = lean_box(0); -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_57, 1, x_4); -x_18 = x_57; -x_19 = x_54; +x_53 = 0; +x_54 = l_Lean_Elab_Tactic_SavedState_restore(x_40, x_53, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_52); +x_55 = lean_ctor_get(x_54, 1); +lean_inc(x_55); +lean_dec(x_54); +x_56 = lean_array_push(x_29, x_16); +lean_ctor_set(x_4, 0, x_56); +x_57 = lean_box(0); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_4); +x_18 = x_58; +x_19 = x_55; goto block_27; } } else { -lean_object* x_58; +lean_object* x_59; lean_free_object(x_3); lean_dec(x_16); -x_58 = lean_ctor_get(x_31, 1); -lean_inc(x_58); +x_59 = lean_ctor_get(x_31, 1); +lean_inc(x_59); lean_dec(x_31); x_3 = x_17; -x_13 = x_58; +x_13 = x_59; goto _start; } } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; -x_60 = lean_ctor_get(x_4, 0); -x_61 = lean_ctor_get(x_4, 1); +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; +x_61 = lean_ctor_get(x_4, 0); +x_62 = lean_ctor_get(x_4, 1); +lean_inc(x_62); lean_inc(x_61); -lean_inc(x_60); lean_dec(x_4); lean_inc(x_16); -x_62 = l_Lean_isExprMVarAssigned___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__1(x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_63 = lean_ctor_get(x_62, 0); -lean_inc(x_63); -x_64 = lean_unbox(x_63); -lean_dec(x_63); -if (x_64 == 0) +x_63 = l_Lean_isExprMVarAssigned___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__1(x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_64 = lean_ctor_get(x_63, 0); +lean_inc(x_64); +x_65 = lean_unbox(x_64); +lean_dec(x_64); +if (x_65 == 0) { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_65 = lean_ctor_get(x_62, 1); -lean_inc(x_65); -lean_dec(x_62); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_66 = lean_ctor_get(x_63, 1); +lean_inc(x_66); +lean_dec(x_63); lean_inc(x_2); lean_inc(x_16); lean_ctor_set(x_3, 1, x_2); -x_66 = l_Lean_Elab_Tactic_setGoals(x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_65); -x_67 = lean_ctor_get(x_66, 1); -lean_inc(x_67); -lean_dec(x_66); -x_68 = lean_unsigned_to_nat(1u); -x_69 = l_Lean_Syntax_getArg(x_1, x_68); -x_70 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_67); -x_71 = lean_ctor_get(x_70, 0); -lean_inc(x_71); -x_72 = lean_ctor_get(x_70, 1); +x_67 = l_Lean_Elab_Tactic_setGoals(x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_66); +x_68 = lean_ctor_get(x_67, 1); +lean_inc(x_68); +lean_dec(x_67); +x_69 = lean_unsigned_to_nat(1u); +x_70 = l_Lean_Syntax_getArg(x_1, x_69); +x_71 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_68); +x_72 = lean_ctor_get(x_71, 0); lean_inc(x_72); -lean_dec(x_70); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -11908,73 +11914,74 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_73 = l_Lean_Elab_Tactic_evalTacticAux(x_69, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_72); -if (lean_obj_tag(x_73) == 0) +x_74 = l_Lean_Elab_Tactic_evalTactic(x_70, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_73); +if (lean_obj_tag(x_74) == 0) { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -lean_dec(x_71); -lean_dec(x_61); +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +lean_dec(x_72); +lean_dec(x_62); lean_dec(x_16); -x_74 = lean_ctor_get(x_73, 1); -lean_inc(x_74); -lean_dec(x_73); -x_75 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_74); -x_76 = lean_ctor_get(x_75, 0); -lean_inc(x_76); -x_77 = lean_ctor_get(x_75, 1); +x_75 = lean_ctor_get(x_74, 1); +lean_inc(x_75); +lean_dec(x_74); +x_76 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_75); +x_77 = lean_ctor_get(x_76, 0); lean_inc(x_77); -lean_dec(x_75); -x_78 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_60, x_76); -x_79 = 1; -x_80 = lean_box(x_79); -x_81 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_81, 0, x_78); -lean_ctor_set(x_81, 1, x_80); -x_82 = lean_box(0); -x_83 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_81); -x_18 = x_83; -x_19 = x_77; +x_78 = lean_ctor_get(x_76, 1); +lean_inc(x_78); +lean_dec(x_76); +x_79 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_61, x_77); +x_80 = 1; +x_81 = lean_box(x_80); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_79); +lean_ctor_set(x_82, 1, x_81); +x_83 = lean_box(0); +x_84 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_82); +x_18 = x_84; +x_19 = x_78; goto block_27; } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_84 = lean_ctor_get(x_73, 1); -lean_inc(x_84); -lean_dec(x_73); -x_85 = l_Lean_Elab_Tactic_SavedState_restore(x_71, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_84); -x_86 = lean_ctor_get(x_85, 1); -lean_inc(x_86); -lean_dec(x_85); -x_87 = lean_array_push(x_60, x_16); -x_88 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_88, 0, x_87); -lean_ctor_set(x_88, 1, x_61); -x_89 = lean_box(0); +lean_object* x_85; uint8_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_85 = lean_ctor_get(x_74, 1); +lean_inc(x_85); +lean_dec(x_74); +x_86 = 0; +x_87 = l_Lean_Elab_Tactic_SavedState_restore(x_72, x_86, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_85); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); +x_89 = lean_array_push(x_61, x_16); x_90 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_88); -x_18 = x_90; -x_19 = x_86; +lean_ctor_set(x_90, 1, x_62); +x_91 = lean_box(0); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_90); +x_18 = x_92; +x_19 = x_88; goto block_27; } } else { -lean_object* x_91; lean_object* x_92; +lean_object* x_93; lean_object* x_94; lean_free_object(x_3); lean_dec(x_16); -x_91 = lean_ctor_get(x_62, 1); -lean_inc(x_91); -lean_dec(x_62); -x_92 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_92, 0, x_60); -lean_ctor_set(x_92, 1, x_61); +x_93 = lean_ctor_get(x_63, 1); +lean_inc(x_93); +lean_dec(x_63); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_61); +lean_ctor_set(x_94, 1, x_62); x_3 = x_17; -x_4 = x_92; -x_13 = x_91; +x_4 = x_94; +x_13 = x_93; goto _start; } } @@ -12012,53 +12019,53 @@ goto _start; } else { -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; -x_94 = lean_ctor_get(x_3, 0); -x_95 = lean_ctor_get(x_3, 1); -lean_inc(x_95); -lean_inc(x_94); +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; +x_96 = lean_ctor_get(x_3, 0); +x_97 = lean_ctor_get(x_3, 1); +lean_inc(x_97); +lean_inc(x_96); lean_dec(x_3); -x_105 = lean_ctor_get(x_4, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_4, 1); -lean_inc(x_106); +x_107 = lean_ctor_get(x_4, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_4, 1); +lean_inc(x_108); if (lean_is_exclusive(x_4)) { lean_ctor_release(x_4, 0); lean_ctor_release(x_4, 1); - x_107 = x_4; + x_109 = x_4; } else { lean_dec_ref(x_4); - x_107 = lean_box(0); + x_109 = lean_box(0); } -lean_inc(x_94); -x_108 = l_Lean_isExprMVarAssigned___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__1(x_94, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_109 = lean_ctor_get(x_108, 0); -lean_inc(x_109); -x_110 = lean_unbox(x_109); -lean_dec(x_109); -if (x_110 == 0) -{ -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_111 = lean_ctor_get(x_108, 1); +lean_inc(x_96); +x_110 = l_Lean_isExprMVarAssigned___at_Lean_Elab_Tactic_pruneSolvedGoals___spec__1(x_96, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_111 = lean_ctor_get(x_110, 0); lean_inc(x_111); -lean_dec(x_108); +x_112 = lean_unbox(x_111); +lean_dec(x_111); +if (x_112 == 0) +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_113 = lean_ctor_get(x_110, 1); +lean_inc(x_113); +lean_dec(x_110); lean_inc(x_2); -lean_inc(x_94); -x_112 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_112, 0, x_94); -lean_ctor_set(x_112, 1, x_2); -x_113 = l_Lean_Elab_Tactic_setGoals(x_112, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_111); -x_114 = lean_ctor_get(x_113, 1); -lean_inc(x_114); -lean_dec(x_113); -x_115 = lean_unsigned_to_nat(1u); -x_116 = l_Lean_Syntax_getArg(x_1, x_115); -x_117 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_114); -x_118 = lean_ctor_get(x_117, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_117, 1); -lean_inc(x_119); -lean_dec(x_117); +lean_inc(x_96); +x_114 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_114, 0, x_96); +lean_ctor_set(x_114, 1, x_2); +x_115 = l_Lean_Elab_Tactic_setGoals(x_114, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_113); +x_116 = lean_ctor_get(x_115, 1); +lean_inc(x_116); +lean_dec(x_115); +x_117 = lean_unsigned_to_nat(1u); +x_118 = l_Lean_Syntax_getArg(x_1, x_117); +x_119 = l_Lean_Elab_Tactic_saveState___rarg(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_116); +x_120 = lean_ctor_get(x_119, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_119, 1); +lean_inc(x_121); +lean_dec(x_119); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -12067,114 +12074,115 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_120 = l_Lean_Elab_Tactic_evalTacticAux(x_116, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_119); -if (lean_obj_tag(x_120) == 0) +x_122 = l_Lean_Elab_Tactic_evalTactic(x_118, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_121); +if (lean_obj_tag(x_122) == 0) { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; uint8_t x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; -lean_dec(x_118); -lean_dec(x_106); -lean_dec(x_94); -x_121 = lean_ctor_get(x_120, 1); -lean_inc(x_121); +lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_dec(x_120); -x_122 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_121); -x_123 = lean_ctor_get(x_122, 0); +lean_dec(x_108); +lean_dec(x_96); +x_123 = lean_ctor_get(x_122, 1); lean_inc(x_123); -x_124 = lean_ctor_get(x_122, 1); -lean_inc(x_124); lean_dec(x_122); -x_125 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_105, x_123); -x_126 = 1; -x_127 = lean_box(x_126); -if (lean_is_scalar(x_107)) { - x_128 = lean_alloc_ctor(0, 2, 0); +x_124 = l_Lean_Elab_Tactic_getUnsolvedGoals(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_123); +x_125 = lean_ctor_get(x_124, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_124, 1); +lean_inc(x_126); +lean_dec(x_124); +x_127 = l_List_foldl___at_Array_appendList___spec__1___rarg(x_107, x_125); +x_128 = 1; +x_129 = lean_box(x_128); +if (lean_is_scalar(x_109)) { + x_130 = lean_alloc_ctor(0, 2, 0); } else { - x_128 = x_107; + x_130 = x_109; } -lean_ctor_set(x_128, 0, x_125); -lean_ctor_set(x_128, 1, x_127); -x_129 = lean_box(0); -x_130 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_130, 0, x_129); -lean_ctor_set(x_130, 1, x_128); -x_96 = x_130; -x_97 = x_124; -goto block_104; +lean_ctor_set(x_130, 0, x_127); +lean_ctor_set(x_130, 1, x_129); +x_131 = lean_box(0); +x_132 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_132, 0, x_131); +lean_ctor_set(x_132, 1, x_130); +x_98 = x_132; +x_99 = x_126; +goto block_106; } else { -lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_131 = lean_ctor_get(x_120, 1); -lean_inc(x_131); -lean_dec(x_120); -x_132 = l_Lean_Elab_Tactic_SavedState_restore(x_118, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_131); -x_133 = lean_ctor_get(x_132, 1); +lean_object* x_133; uint8_t x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_133 = lean_ctor_get(x_122, 1); lean_inc(x_133); -lean_dec(x_132); -x_134 = lean_array_push(x_105, x_94); -if (lean_is_scalar(x_107)) { - x_135 = lean_alloc_ctor(0, 2, 0); +lean_dec(x_122); +x_134 = 0; +x_135 = l_Lean_Elab_Tactic_SavedState_restore(x_120, x_134, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_133); +x_136 = lean_ctor_get(x_135, 1); +lean_inc(x_136); +lean_dec(x_135); +x_137 = lean_array_push(x_107, x_96); +if (lean_is_scalar(x_109)) { + x_138 = lean_alloc_ctor(0, 2, 0); } else { - x_135 = x_107; + x_138 = x_109; } -lean_ctor_set(x_135, 0, x_134); -lean_ctor_set(x_135, 1, x_106); -x_136 = lean_box(0); -x_137 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set(x_137, 1, x_135); -x_96 = x_137; -x_97 = x_133; -goto block_104; +lean_ctor_set(x_138, 0, x_137); +lean_ctor_set(x_138, 1, x_108); +x_139 = lean_box(0); +x_140 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_140, 0, x_139); +lean_ctor_set(x_140, 1, x_138); +x_98 = x_140; +x_99 = x_136; +goto block_106; } } else { -lean_object* x_138; lean_object* x_139; -lean_dec(x_94); -x_138 = lean_ctor_get(x_108, 1); -lean_inc(x_138); -lean_dec(x_108); -if (lean_is_scalar(x_107)) { - x_139 = lean_alloc_ctor(0, 2, 0); +lean_object* x_141; lean_object* x_142; +lean_dec(x_96); +x_141 = lean_ctor_get(x_110, 1); +lean_inc(x_141); +lean_dec(x_110); +if (lean_is_scalar(x_109)) { + x_142 = lean_alloc_ctor(0, 2, 0); } else { - x_139 = x_107; + x_142 = x_109; } -lean_ctor_set(x_139, 0, x_105); -lean_ctor_set(x_139, 1, x_106); -x_3 = x_95; -x_4 = x_139; -x_13 = x_138; +lean_ctor_set(x_142, 0, x_107); +lean_ctor_set(x_142, 1, x_108); +x_3 = x_97; +x_4 = x_142; +x_13 = x_141; goto _start; } -block_104: +block_106: { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_98 = lean_ctor_get(x_96, 1); -lean_inc(x_98); -lean_dec(x_96); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; x_100 = lean_ctor_get(x_98, 1); lean_inc(x_100); -if (lean_is_exclusive(x_98)) { - lean_ctor_release(x_98, 0); - lean_ctor_release(x_98, 1); - x_101 = x_98; +lean_dec(x_98); +x_101 = lean_ctor_get(x_100, 0); +lean_inc(x_101); +x_102 = lean_ctor_get(x_100, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + x_103 = x_100; } else { - lean_dec_ref(x_98); - x_101 = lean_box(0); + lean_dec_ref(x_100); + x_103 = lean_box(0); } -if (lean_is_scalar(x_101)) { - x_102 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_103)) { + x_104 = lean_alloc_ctor(0, 2, 0); } else { - x_102 = x_101; + x_104 = x_103; } -lean_ctor_set(x_102, 0, x_99); -lean_ctor_set(x_102, 1, x_100); -x_3 = x_95; -x_4 = x_102; -x_13 = x_97; +lean_ctor_set(x_104, 0, x_101); +lean_ctor_set(x_104, 1, x_102); +x_3 = x_97; +x_4 = x_104; +x_13 = x_99; goto _start; } } @@ -12256,7 +12264,7 @@ x_20 = lean_ctor_get(x_16, 1); lean_inc(x_20); lean_dec(x_16); x_21 = l_Lean_Elab_Tactic_evalAnyGoals___closed__3; -x_22 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +x_22 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -12497,7 +12505,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalTacticSeq(lean_object* x_1, lean lean_object* x_11; lean_object* x_12; lean_object* x_13; x_11 = lean_unsigned_to_nat(0u); x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_13; } } @@ -12716,7 +12724,7 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_19 = l_Lean_Elab_Tactic_evalTacticAux(x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +x_19 = l_Lean_Elab_Tactic_evalTactic(x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); if (lean_obj_tag(x_19) == 0) { lean_dec(x_17); @@ -12733,16 +12741,17 @@ return x_19; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; +lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); lean_dec(x_19); -x_22 = l_Lean_Elab_Tactic_SavedState_restore(x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +x_22 = 0; +x_23 = l_Lean_Elab_Tactic_SavedState_restore(x_17, x_22, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); if (lean_obj_tag(x_20) == 0) { -uint8_t x_23; +uint8_t x_24; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -12752,44 +12761,44 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_22, 0); -lean_dec(x_24); -lean_ctor_set_tag(x_22, 1); -lean_ctor_set(x_22, 0, x_20); -return x_22; +lean_object* x_25; +x_25 = lean_ctor_get(x_23, 0); +lean_dec(x_25); +lean_ctor_set_tag(x_23, 1); +lean_ctor_set(x_23, 0, x_20); +return x_23; } else { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_20); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_20); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } else { -uint8_t x_27; -x_27 = !lean_is_exclusive(x_22); -if (x_27 == 0) +uint8_t x_28; +x_28 = !lean_is_exclusive(x_23); +if (x_28 == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_28 = lean_ctor_get(x_22, 1); -x_29 = lean_ctor_get(x_22, 0); -lean_dec(x_29); -x_30 = lean_ctor_get(x_20, 0); -lean_inc(x_30); -x_31 = l_Lean_Elab_Tactic_evalChoiceAux___closed__1; -x_32 = lean_nat_dec_eq(x_31, x_30); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_29 = lean_ctor_get(x_23, 1); +x_30 = lean_ctor_get(x_23, 0); lean_dec(x_30); -if (x_32 == 0) +x_31 = lean_ctor_get(x_20, 0); +lean_inc(x_31); +x_32 = l_Lean_Elab_Tactic_evalChoiceAux___closed__1; +x_33 = lean_nat_dec_eq(x_32, x_31); +lean_dec(x_31); +if (x_33 == 0) { lean_dec(x_10); lean_dec(x_9); @@ -12800,37 +12809,37 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_ctor_set_tag(x_22, 1); -lean_ctor_set(x_22, 0, x_20); -return x_22; +lean_ctor_set_tag(x_23, 1); +lean_ctor_set(x_23, 0, x_20); +return x_23; } else { -lean_object* x_33; lean_object* x_34; -lean_free_object(x_22); +lean_object* x_34; lean_object* x_35; +lean_free_object(x_23); lean_dec(x_20); -x_33 = lean_unsigned_to_nat(1u); -x_34 = lean_nat_add(x_2, x_33); +x_34 = lean_unsigned_to_nat(1u); +x_35 = lean_nat_add(x_2, x_34); lean_dec(x_2); -x_2 = x_34; -x_11 = x_28; +x_2 = x_35; +x_11 = x_29; goto _start; } } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_36 = lean_ctor_get(x_22, 1); -lean_inc(x_36); -lean_dec(x_22); -x_37 = lean_ctor_get(x_20, 0); +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_37 = lean_ctor_get(x_23, 1); lean_inc(x_37); -x_38 = l_Lean_Elab_Tactic_evalChoiceAux___closed__1; -x_39 = lean_nat_dec_eq(x_38, x_37); -lean_dec(x_37); -if (x_39 == 0) +lean_dec(x_23); +x_38 = lean_ctor_get(x_20, 0); +lean_inc(x_38); +x_39 = l_Lean_Elab_Tactic_evalChoiceAux___closed__1; +x_40 = lean_nat_dec_eq(x_39, x_38); +lean_dec(x_38); +if (x_40 == 0) { -lean_object* x_40; +lean_object* x_41; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -12840,20 +12849,20 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_20); -lean_ctor_set(x_40, 1, x_36); -return x_40; +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_20); +lean_ctor_set(x_41, 1, x_37); +return x_41; } else { -lean_object* x_41; lean_object* x_42; +lean_object* x_42; lean_object* x_43; lean_dec(x_20); -x_41 = lean_unsigned_to_nat(1u); -x_42 = lean_nat_add(x_2, x_41); +x_42 = lean_unsigned_to_nat(1u); +x_43 = lean_nat_add(x_2, x_42); lean_dec(x_2); -x_2 = x_42; -x_11 = x_36; +x_2 = x_43; +x_11 = x_37; goto _start; } } @@ -13471,7 +13480,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_23 = l_Lean_Elab_Tactic_evalTacticAux(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_22); +x_23 = l_Lean_Elab_Tactic_evalTactic(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_22); if (lean_obj_tag(x_23) == 0) { lean_object* x_24; uint8_t x_25; @@ -13486,17 +13495,17 @@ goto block_17; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; x_26 = lean_ctor_get(x_23, 1); lean_inc(x_26); lean_dec(x_23); -x_27 = l_Lean_Elab_Tactic_SavedState_restore(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_26); -x_28 = lean_ctor_get(x_27, 1); -lean_inc(x_28); -lean_dec(x_27); -x_29 = 0; -x_11 = x_29; -x_12 = x_28; +x_27 = 0; +x_28 = l_Lean_Elab_Tactic_SavedState_restore(x_21, x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_26); +x_29 = lean_ctor_get(x_28, 1); +lean_inc(x_29); +lean_dec(x_28); +x_11 = x_27; +x_12 = x_29; goto block_17; } block_17: @@ -13522,7 +13531,7 @@ else { lean_object* x_15; lean_object* x_16; x_15 = l_Lean_Elab_Tactic_evalFailIfSuccess___closed__2; -x_16 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_12); +x_16 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_12); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -14104,7 +14113,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_throwIllFormedSyntax___at_Lean_Elab_Tactic_ { lean_object* x_10; lean_object* x_11; x_10 = l_Lean_Elab_throwIllFormedSyntax___at_Lean_Elab_Tactic_evalTraceMessage___spec__1___closed__2; -x_11 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); return x_11; } } @@ -16206,7 +16215,7 @@ x_58 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_58, 0, x_26); lean_ctor_set(x_58, 1, x_57); lean_ctor_set(x_58, 2, x_56); -x_59 = l_Lean_Elab_Tactic_evalTacticAux(x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_34); +x_59 = l_Lean_Elab_Tactic_evalTactic(x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_34); return x_59; } } @@ -16445,7 +16454,7 @@ x_175 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_175, 0, x_83); lean_ctor_set(x_175, 1, x_174); lean_ctor_set(x_175, 2, x_173); -x_176 = l_Lean_Elab_Tactic_evalTacticAux(x_175, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_71); +x_176 = l_Lean_Elab_Tactic_evalTactic(x_175, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_71); return x_176; } else @@ -16665,7 +16674,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); lean_ctor_set(x_5, 2, x_15); -x_16 = l_Lean_Elab_Tactic_evalTacticAux(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_16 = l_Lean_Elab_Tactic_evalTactic(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); return x_16; } else @@ -16720,7 +16729,7 @@ lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 4, x_28); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 5, x_29); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 6, x_30); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 7, x_32); -x_36 = l_Lean_Elab_Tactic_evalTacticAux(x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11); +x_36 = l_Lean_Elab_Tactic_evalTactic(x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11); return x_36; } } @@ -16743,7 +16752,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_14 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__1(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_14 = l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__1(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_14) == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; @@ -23234,7 +23243,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -23287,7 +23296,7 @@ lean_inc(x_29); x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); lean_dec(x_28); -x_31 = lean_ctor_get(x_29, 4); +x_31 = lean_ctor_get(x_29, 5); lean_inc(x_31); lean_dec(x_29); x_32 = lean_ctor_get(x_31, 1); @@ -23312,7 +23321,7 @@ lean_dec(x_36); x_38 = lean_st_ref_take(x_5, x_37); x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); -x_40 = lean_ctor_get(x_39, 4); +x_40 = lean_ctor_get(x_39, 5); lean_inc(x_40); x_41 = lean_ctor_get(x_38, 1); lean_inc(x_41); @@ -23321,7 +23330,7 @@ x_42 = !lean_is_exclusive(x_39); if (x_42 == 0) { lean_object* x_43; uint8_t x_44; -x_43 = lean_ctor_get(x_39, 4); +x_43 = lean_ctor_get(x_39, 5); lean_dec(x_43); x_44 = !lean_is_exclusive(x_40); if (x_44 == 0) @@ -23366,7 +23375,7 @@ x_55 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_55, 0, x_53); lean_ctor_set(x_55, 1, x_54); lean_ctor_set_uint8(x_55, sizeof(void*)*2, x_52); -lean_ctor_set(x_39, 4, x_55); +lean_ctor_set(x_39, 5, x_55); x_56 = lean_st_ref_set(x_5, x_39, x_41); lean_dec(x_5); x_57 = lean_ctor_get(x_56, 1); @@ -23391,245 +23400,251 @@ return x_59; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; x_60 = lean_ctor_get(x_39, 0); x_61 = lean_ctor_get(x_39, 1); x_62 = lean_ctor_get(x_39, 2); x_63 = lean_ctor_get(x_39, 3); +x_64 = lean_ctor_get(x_39, 4); +lean_inc(x_64); lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_dec(x_39); -x_64 = lean_ctor_get_uint8(x_40, sizeof(void*)*2); -x_65 = lean_ctor_get(x_40, 0); -lean_inc(x_65); +x_65 = lean_ctor_get_uint8(x_40, sizeof(void*)*2); +x_66 = lean_ctor_get(x_40, 0); +lean_inc(x_66); if (lean_is_exclusive(x_40)) { lean_ctor_release(x_40, 0); lean_ctor_release(x_40, 1); - x_66 = x_40; + x_67 = x_40; } else { lean_dec_ref(x_40); - x_66 = lean_box(0); + x_67 = lean_box(0); } -x_67 = l_Std_PersistentArray_append___rarg(x_21, x_34); -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 2, 1); +x_68 = l_Std_PersistentArray_append___rarg(x_21, x_34); +if (lean_is_scalar(x_67)) { + x_69 = lean_alloc_ctor(0, 2, 1); } else { - x_68 = x_66; + x_69 = x_67; } -lean_ctor_set(x_68, 0, x_65); -lean_ctor_set(x_68, 1, x_67); -lean_ctor_set_uint8(x_68, sizeof(void*)*2, x_64); -x_69 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_69, 0, x_60); -lean_ctor_set(x_69, 1, x_61); -lean_ctor_set(x_69, 2, x_62); -lean_ctor_set(x_69, 3, x_63); -lean_ctor_set(x_69, 4, x_68); -x_70 = lean_st_ref_set(x_5, x_69, x_41); +lean_ctor_set(x_69, 0, x_66); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_65); +x_70 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_70, 0, x_60); +lean_ctor_set(x_70, 1, x_61); +lean_ctor_set(x_70, 2, x_62); +lean_ctor_set(x_70, 3, x_63); +lean_ctor_set(x_70, 4, x_64); +lean_ctor_set(x_70, 5, x_69); +x_71 = lean_st_ref_set(x_5, x_70, x_41); lean_dec(x_5); -x_71 = lean_ctor_get(x_70, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - x_72 = x_70; +x_72 = lean_ctor_get(x_71, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_73 = x_71; } else { - lean_dec_ref(x_70); - x_72 = lean_box(0); + lean_dec_ref(x_71); + x_73 = lean_box(0); } -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_73)) { + x_74 = lean_alloc_ctor(0, 2, 0); } else { - x_73 = x_72; + x_74 = x_73; } -lean_ctor_set(x_73, 0, x_24); -lean_ctor_set(x_73, 1, x_71); -return x_73; +lean_ctor_set(x_74, 0, x_24); +lean_ctor_set(x_74, 1, x_72); +return x_74; } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; -x_74 = lean_ctor_get(x_23, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_23, 1); +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; uint8_t x_93; +x_75 = lean_ctor_get(x_23, 0); lean_inc(x_75); +x_76 = lean_ctor_get(x_23, 1); +lean_inc(x_76); lean_dec(x_23); -x_76 = lean_st_ref_get(x_9, x_75); -x_77 = lean_ctor_get(x_76, 1); -lean_inc(x_77); -lean_dec(x_76); -x_78 = lean_st_ref_get(x_5, x_77); -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); +x_77 = lean_st_ref_get(x_9, x_76); +x_78 = lean_ctor_get(x_77, 1); +lean_inc(x_78); +lean_dec(x_77); +x_79 = lean_st_ref_get(x_5, x_78); +x_80 = lean_ctor_get(x_79, 0); lean_inc(x_80); -lean_dec(x_78); -x_81 = lean_ctor_get(x_79, 4); +x_81 = lean_ctor_get(x_79, 1); lean_inc(x_81); lean_dec(x_79); -x_82 = lean_ctor_get(x_81, 1); +x_82 = lean_ctor_get(x_80, 5); lean_inc(x_82); -x_83 = l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_renameInaccessibles___spec__11(x_81, x_82, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_80); +lean_dec(x_80); +x_83 = lean_ctor_get(x_82, 1); +lean_inc(x_83); +x_84 = l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_renameInaccessibles___spec__11(x_82, x_83, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_81); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +x_85 = lean_ctor_get(x_84, 0); lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_st_ref_get(x_9, x_85); +x_86 = lean_ctor_get(x_84, 1); +lean_inc(x_86); +lean_dec(x_84); +x_87 = lean_st_ref_get(x_9, x_86); lean_dec(x_9); -x_87 = lean_ctor_get(x_86, 1); -lean_inc(x_87); -lean_dec(x_86); -x_88 = lean_st_ref_take(x_5, x_87); -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_89, 4); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); +x_89 = lean_st_ref_take(x_5, x_88); +x_90 = lean_ctor_get(x_89, 0); lean_inc(x_90); -x_91 = lean_ctor_get(x_88, 1); +x_91 = lean_ctor_get(x_90, 5); lean_inc(x_91); -lean_dec(x_88); -x_92 = !lean_is_exclusive(x_89); -if (x_92 == 0) +x_92 = lean_ctor_get(x_89, 1); +lean_inc(x_92); +lean_dec(x_89); +x_93 = !lean_is_exclusive(x_90); +if (x_93 == 0) { -lean_object* x_93; uint8_t x_94; -x_93 = lean_ctor_get(x_89, 4); -lean_dec(x_93); -x_94 = !lean_is_exclusive(x_90); -if (x_94 == 0) -{ -lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; -x_95 = lean_ctor_get(x_90, 1); -lean_dec(x_95); -x_96 = l_Std_PersistentArray_append___rarg(x_21, x_84); -lean_ctor_set(x_90, 1, x_96); -x_97 = lean_st_ref_set(x_5, x_89, x_91); +lean_object* x_94; uint8_t x_95; +x_94 = lean_ctor_get(x_90, 5); +lean_dec(x_94); +x_95 = !lean_is_exclusive(x_91); +if (x_95 == 0) +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; +x_96 = lean_ctor_get(x_91, 1); +lean_dec(x_96); +x_97 = l_Std_PersistentArray_append___rarg(x_21, x_85); +lean_ctor_set(x_91, 1, x_97); +x_98 = lean_st_ref_set(x_5, x_90, x_92); lean_dec(x_5); -x_98 = !lean_is_exclusive(x_97); -if (x_98 == 0) +x_99 = !lean_is_exclusive(x_98); +if (x_99 == 0) { -lean_object* x_99; -x_99 = lean_ctor_get(x_97, 0); -lean_dec(x_99); -lean_ctor_set_tag(x_97, 1); -lean_ctor_set(x_97, 0, x_74); -return x_97; +lean_object* x_100; +x_100 = lean_ctor_get(x_98, 0); +lean_dec(x_100); +lean_ctor_set_tag(x_98, 1); +lean_ctor_set(x_98, 0, x_75); +return x_98; } else { -lean_object* x_100; lean_object* x_101; -x_100 = lean_ctor_get(x_97, 1); -lean_inc(x_100); -lean_dec(x_97); -x_101 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_101, 0, x_74); -lean_ctor_set(x_101, 1, x_100); -return x_101; +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_98, 1); +lean_inc(x_101); +lean_dec(x_98); +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_75); +lean_ctor_set(x_102, 1, x_101); +return x_102; } } else { -uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_102 = lean_ctor_get_uint8(x_90, sizeof(void*)*2); -x_103 = lean_ctor_get(x_90, 0); -lean_inc(x_103); -lean_dec(x_90); -x_104 = l_Std_PersistentArray_append___rarg(x_21, x_84); -x_105 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set_uint8(x_105, sizeof(void*)*2, x_102); -lean_ctor_set(x_89, 4, x_105); -x_106 = lean_st_ref_set(x_5, x_89, x_91); +uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_103 = lean_ctor_get_uint8(x_91, sizeof(void*)*2); +x_104 = lean_ctor_get(x_91, 0); +lean_inc(x_104); +lean_dec(x_91); +x_105 = l_Std_PersistentArray_append___rarg(x_21, x_85); +x_106 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_106, 0, x_104); +lean_ctor_set(x_106, 1, x_105); +lean_ctor_set_uint8(x_106, sizeof(void*)*2, x_103); +lean_ctor_set(x_90, 5, x_106); +x_107 = lean_st_ref_set(x_5, x_90, x_92); lean_dec(x_5); -x_107 = lean_ctor_get(x_106, 1); -lean_inc(x_107); -if (lean_is_exclusive(x_106)) { - lean_ctor_release(x_106, 0); - lean_ctor_release(x_106, 1); - x_108 = x_106; +x_108 = lean_ctor_get(x_107, 1); +lean_inc(x_108); +if (lean_is_exclusive(x_107)) { + lean_ctor_release(x_107, 0); + lean_ctor_release(x_107, 1); + x_109 = x_107; } else { - lean_dec_ref(x_106); - x_108 = lean_box(0); + lean_dec_ref(x_107); + x_109 = lean_box(0); } -if (lean_is_scalar(x_108)) { - x_109 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_109)) { + x_110 = lean_alloc_ctor(1, 2, 0); } else { - x_109 = x_108; - lean_ctor_set_tag(x_109, 1); + x_110 = x_109; + lean_ctor_set_tag(x_110, 1); } -lean_ctor_set(x_109, 0, x_74); -lean_ctor_set(x_109, 1, x_107); -return x_109; +lean_ctor_set(x_110, 0, x_75); +lean_ctor_set(x_110, 1, x_108); +return x_110; } } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_110 = lean_ctor_get(x_89, 0); -x_111 = lean_ctor_get(x_89, 1); -x_112 = lean_ctor_get(x_89, 2); -x_113 = lean_ctor_get(x_89, 3); +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_111 = lean_ctor_get(x_90, 0); +x_112 = lean_ctor_get(x_90, 1); +x_113 = lean_ctor_get(x_90, 2); +x_114 = lean_ctor_get(x_90, 3); +x_115 = lean_ctor_get(x_90, 4); +lean_inc(x_115); +lean_inc(x_114); lean_inc(x_113); lean_inc(x_112); lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_89); -x_114 = lean_ctor_get_uint8(x_90, sizeof(void*)*2); -x_115 = lean_ctor_get(x_90, 0); -lean_inc(x_115); -if (lean_is_exclusive(x_90)) { - lean_ctor_release(x_90, 0); - lean_ctor_release(x_90, 1); - x_116 = x_90; +lean_dec(x_90); +x_116 = lean_ctor_get_uint8(x_91, sizeof(void*)*2); +x_117 = lean_ctor_get(x_91, 0); +lean_inc(x_117); +if (lean_is_exclusive(x_91)) { + lean_ctor_release(x_91, 0); + lean_ctor_release(x_91, 1); + x_118 = x_91; } else { - lean_dec_ref(x_90); - x_116 = lean_box(0); + lean_dec_ref(x_91); + x_118 = lean_box(0); } -x_117 = l_Std_PersistentArray_append___rarg(x_21, x_84); -if (lean_is_scalar(x_116)) { - x_118 = lean_alloc_ctor(0, 2, 1); +x_119 = l_Std_PersistentArray_append___rarg(x_21, x_85); +if (lean_is_scalar(x_118)) { + x_120 = lean_alloc_ctor(0, 2, 1); } else { - x_118 = x_116; -} -lean_ctor_set(x_118, 0, x_115); -lean_ctor_set(x_118, 1, x_117); -lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); -x_119 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_119, 0, x_110); -lean_ctor_set(x_119, 1, x_111); -lean_ctor_set(x_119, 2, x_112); -lean_ctor_set(x_119, 3, x_113); -lean_ctor_set(x_119, 4, x_118); -x_120 = lean_st_ref_set(x_5, x_119, x_91); + x_120 = x_118; +} +lean_ctor_set(x_120, 0, x_117); +lean_ctor_set(x_120, 1, x_119); +lean_ctor_set_uint8(x_120, sizeof(void*)*2, x_116); +x_121 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_121, 0, x_111); +lean_ctor_set(x_121, 1, x_112); +lean_ctor_set(x_121, 2, x_113); +lean_ctor_set(x_121, 3, x_114); +lean_ctor_set(x_121, 4, x_115); +lean_ctor_set(x_121, 5, x_120); +x_122 = lean_st_ref_set(x_5, x_121, x_92); lean_dec(x_5); -x_121 = lean_ctor_get(x_120, 1); -lean_inc(x_121); -if (lean_is_exclusive(x_120)) { - lean_ctor_release(x_120, 0); - lean_ctor_release(x_120, 1); - x_122 = x_120; +x_123 = lean_ctor_get(x_122, 1); +lean_inc(x_123); +if (lean_is_exclusive(x_122)) { + lean_ctor_release(x_122, 0); + lean_ctor_release(x_122, 1); + x_124 = x_122; } else { - lean_dec_ref(x_120); - x_122 = lean_box(0); + lean_dec_ref(x_122); + x_124 = lean_box(0); } -if (lean_is_scalar(x_122)) { - x_123 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_124)) { + x_125 = lean_alloc_ctor(1, 2, 0); } else { - x_123 = x_122; - lean_ctor_set_tag(x_123, 1); + x_125 = x_124; + lean_ctor_set_tag(x_125, 1); } -lean_ctor_set(x_123, 0, x_74); -lean_ctor_set(x_123, 1, x_121); -return x_123; +lean_ctor_set(x_125, 0, x_75); +lean_ctor_set(x_125, 1, x_123); +return x_125; } } } @@ -26102,34 +26117,35 @@ return x_24; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); lean_dec(x_24); -x_26 = l_Lean_Elab_Tactic_SavedState_restore(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_25); -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -x_28 = lean_nat_add(x_2, x_13); +x_26 = 0; +x_27 = l_Lean_Elab_Tactic_SavedState_restore(x_18, x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_25); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_nat_add(x_2, x_13); lean_dec(x_2); -x_2 = x_28; -x_11 = x_27; +x_2 = x_29; +x_11 = x_28; goto _start; } } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_30 = lean_ctor_get(x_17, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_17, 1); +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_31 = lean_ctor_get(x_17, 0); lean_inc(x_31); +x_32 = lean_ctor_get(x_17, 1); +lean_inc(x_32); lean_dec(x_17); -x_32 = lean_array_fget(x_1, x_2); -x_33 = l_Lean_Syntax_getArg(x_32, x_13); -lean_dec(x_32); -x_34 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); -lean_closure_set(x_34, 0, x_33); +x_33 = lean_array_fget(x_1, x_2); +x_34 = l_Lean_Syntax_getArg(x_33, x_13); +lean_dec(x_33); +x_35 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalTactic), 10, 1); +lean_closure_set(x_35, 0, x_34); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); @@ -26138,10 +26154,10 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_35 = l_Lean_Elab_Tactic_withoutRecover___rarg(x_34, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_31); -if (lean_obj_tag(x_35) == 0) +x_36 = l_Lean_Elab_Tactic_withoutRecover___rarg(x_35, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_32); +if (lean_obj_tag(x_36) == 0) { -lean_dec(x_30); +lean_dec(x_31); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -26151,51 +26167,52 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_35; +return x_36; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_35, 1); -lean_inc(x_36); -lean_dec(x_35); -x_37 = l_Lean_Elab_Tactic_SavedState_restore(x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_36); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -lean_dec(x_37); -x_39 = lean_nat_add(x_2, x_13); +lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_37 = lean_ctor_get(x_36, 1); +lean_inc(x_37); +lean_dec(x_36); +x_38 = 0; +x_39 = l_Lean_Elab_Tactic_SavedState_restore(x_31, x_38, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_37); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_41 = lean_nat_add(x_2, x_13); lean_dec(x_2); -x_2 = x_39; -x_11 = x_38; +x_2 = x_41; +x_11 = x_40; goto _start; } } } else { -uint8_t x_41; -x_41 = lean_nat_dec_lt(x_2, x_12); +uint8_t x_43; +x_43 = lean_nat_dec_lt(x_2, x_12); lean_dec(x_12); -if (x_41 == 0) +if (x_43 == 0) { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_dec(x_2); -x_42 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_evalSeq1___spec__1___closed__4; -x_43 = l_panic___at_Lean_expandExplicitBindersAux_loop___spec__1(x_42); -x_44 = l_Lean_Syntax_getArg(x_43, x_13); -lean_dec(x_43); -x_45 = l_Lean_Elab_Tactic_evalTacticAux(x_44, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_45; +x_44 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_evalSeq1___spec__1___closed__4; +x_45 = l_panic___at_Lean_expandExplicitBindersAux_loop___spec__1(x_44); +x_46 = l_Lean_Syntax_getArg(x_45, x_13); +lean_dec(x_45); +x_47 = l_Lean_Elab_Tactic_evalTactic(x_46, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_47; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_array_fget(x_1, x_2); +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_array_fget(x_1, x_2); lean_dec(x_2); -x_47 = l_Lean_Syntax_getArg(x_46, x_13); -lean_dec(x_46); -x_48 = l_Lean_Elab_Tactic_evalTacticAux(x_47, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_48; +x_49 = l_Lean_Syntax_getArg(x_48, x_13); +lean_dec(x_48); +x_50 = l_Lean_Elab_Tactic_evalTactic(x_49, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_50; } } } @@ -26664,7 +26681,7 @@ lean_ctor_set(x_37, 1, x_17); x_38 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_38, 0, x_37); lean_ctor_set(x_38, 1, x_33); -x_39 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_39 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_39; } } @@ -26681,7 +26698,7 @@ x_42 = l_Lean_Elab_nestedExceptionToMessageData___at_Lean_Elab_Tactic_evalOpen__ x_43 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_43, 0, x_41); lean_ctor_set(x_43, 1, x_42); -x_44 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_43, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_44 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_43, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_44; } } diff --git a/stage0/stdlib/Lean/Elab/Tactic/Cache.c b/stage0/stdlib/Lean/Elab/Tactic/Cache.c index 973af46f8e98..5eb8e4436a8f 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Cache.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Cache.c @@ -24,7 +24,6 @@ static lean_object* l___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_dbg__ static lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Cache___hyg_16____closed__6; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_Elab_Tactic_evalCheckpoint___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_structEq(lean_object*, lean_object*); -lean_object* l_Lean_Elab_Tactic_evalTacticAux(lean_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_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_evalCheckpoint___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCheckpoint___closed__14; @@ -32,6 +31,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCheckpoint_declRange___c lean_object* lean_dbg_trace(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_dbg__cache(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_evalTactic(lean_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_PersistentHashMap_findAtAux___at___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_dbg__cache_x27___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_dbg__cache___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCheckpoint___closed__5; @@ -91,9 +91,9 @@ size_t lean_usize_land(size_t, size_t); static lean_object* l___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_findCache_x3f___closed__3; lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCheckpoint___closed__11; -uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(lean_object*, lean_object*); +uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); -uint64_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694_(lean_object*); +uint64_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698_(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_dbg__cache_x27___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_dbg__cache_x27___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_dbg__cache_x27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -317,7 +317,7 @@ else { lean_object* x_9; uint8_t x_10; x_9 = lean_array_fget(x_1, x_4); -x_10 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(x_5, x_9); +x_10 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(x_5, x_9); lean_dec(x_9); if (x_10 == 0) { @@ -387,7 +387,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_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(x_3, x_11); +x_13 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(x_3, x_11); lean_dec(x_11); if (x_13 == 0) { @@ -446,7 +446,7 @@ lean_object* x_3; uint64_t x_4; size_t x_5; lean_object* x_6; x_3 = lean_ctor_get(x_1, 0); lean_inc(x_3); lean_dec(x_1); -x_4 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694_(x_2); +x_4 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698_(x_2); x_5 = lean_uint64_to_usize(x_4); x_6 = l_Std_PersistentHashMap_findAux___at___private_Lean_Elab_Tactic_Cache_0__Lean_Elab_Tactic_dbg__cache_x27___spec__2(x_3, x_5, x_2); lean_dec(x_2); @@ -1350,7 +1350,7 @@ else lean_object* x_9; lean_object* x_10; uint64_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_9 = lean_array_fget(x_2, x_5); x_10 = lean_array_fget(x_3, x_5); -x_11 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694_(x_9); +x_11 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698_(x_9); x_12 = lean_uint64_to_usize(x_11); x_13 = 1; x_14 = lean_usize_sub(x_1, x_13); @@ -1413,7 +1413,7 @@ else { lean_object* x_17; uint8_t x_18; x_17 = lean_array_fget(x_5, x_2); -x_18 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(x_3, x_17); +x_18 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(x_3, x_17); lean_dec(x_17); if (x_18 == 0) { @@ -1510,7 +1510,7 @@ if (x_18 == 0) lean_object* x_19; lean_object* x_20; uint8_t x_21; x_19 = lean_ctor_get(x_15, 0); x_20 = lean_ctor_get(x_15, 1); -x_21 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(x_4, x_19); +x_21 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(x_4, x_19); if (x_21 == 0) { lean_object* x_22; lean_object* x_23; lean_object* x_24; @@ -1544,7 +1544,7 @@ x_27 = lean_ctor_get(x_15, 1); lean_inc(x_27); lean_inc(x_26); lean_dec(x_15); -x_28 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(x_4, x_26); +x_28 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(x_4, x_26); if (x_28 == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; @@ -1665,7 +1665,7 @@ if (lean_is_exclusive(x_57)) { lean_dec_ref(x_57); x_62 = lean_box(0); } -x_63 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(x_4, x_60); +x_63 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(x_4, x_60); if (x_63 == 0) { lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; @@ -1842,7 +1842,7 @@ if (x_4 == 0) lean_object* x_5; lean_object* x_6; uint64_t x_7; size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; x_5 = lean_ctor_get(x_1, 0); x_6 = lean_ctor_get(x_1, 1); -x_7 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694_(x_2); +x_7 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698_(x_2); x_8 = lean_uint64_to_usize(x_7); x_9 = 1; x_10 = l_Std_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_evalCheckpoint___spec__2(x_5, x_8, x_9, x_2, x_3); @@ -1861,7 +1861,7 @@ x_14 = lean_ctor_get(x_1, 1); lean_inc(x_14); lean_inc(x_13); lean_dec(x_1); -x_15 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694_(x_2); +x_15 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698_(x_2); x_16 = lean_uint64_to_usize(x_15); x_17 = 1; x_18 = l_Std_PersistentHashMap_insertAux___at_Lean_Elab_Tactic_evalCheckpoint___spec__2(x_13, x_16, x_17, x_2, x_3); @@ -1917,7 +1917,7 @@ lean_inc(x_13); lean_dec(x_11); x_14 = lean_unsigned_to_nat(1u); x_15 = l_Lean_Syntax_getArg(x_1, x_14); -x_16 = l_Lean_Elab_Tactic_evalTacticAux(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_16 = l_Lean_Elab_Tactic_evalTactic(x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_16; } else @@ -1940,7 +1940,7 @@ lean_dec(x_19); lean_dec(x_17); x_22 = lean_unsigned_to_nat(1u); x_23 = l_Lean_Syntax_getArg(x_1, x_22); -x_24 = l_Lean_Elab_Tactic_evalTacticAux(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +x_24 = l_Lean_Elab_Tactic_evalTactic(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_18); return x_24; } else @@ -1983,7 +1983,7 @@ lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_27); -x_31 = l_Lean_Elab_Tactic_evalTacticAux(x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_30); +x_31 = l_Lean_Elab_Tactic_evalTactic(x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_30); if (lean_obj_tag(x_31) == 0) { lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_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; diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Basic.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Basic.c index bf33ef2e29dd..0af474be2af7 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Basic.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Basic.c @@ -41,7 +41,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedConv_declRang static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalWhnf___closed__14; lean_object* l_Lean_Elab_Tactic_evalTacticSeq1Indented(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq_declRange(lean_object*); -lean_object* l_Lean_Elab_Tactic_SavedState_restore(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_SavedState_restore(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Elab_Tactic_Conv_remarkAsConvGoal___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalReduce___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalReduce___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -70,7 +70,6 @@ lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact_ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalZeta___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalReduce_declRange___closed__3; lean_object* l_Lean_mkLHSGoal(lean_object*); -lean_object* l_Lean_Elab_Tactic_evalTacticAux(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_Conv_evalNestedTactic___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTacticCore_declRange___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalParen___closed__3; @@ -202,7 +201,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedConv___closed LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_markAsConvGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalWhnf___closed__9; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalZeta___closed__1; -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_evalConvSeqBracketed___lambda__2___closed__3; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeqBracketed_declRange___closed__5; @@ -251,6 +249,7 @@ lean_object* l_Lean_LocalDecl_fvarId(lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Elab_Tactic_Conv_convert___spec__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Conv_Basic_0__Lean_Elab_Tactic_Conv_convLocalDecl___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalConvSeqBracketed___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_evalConvSeqBracketed___lambda__2___closed__25; lean_object* l_ReaderT_pure___at_Lean_Elab_Tactic_saveTacticInfoForToken___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalWhnf_declRange___closed__2; @@ -763,18 +762,19 @@ goto _start; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_23 = lean_ctor_get(x_19, 1); lean_inc(x_23); lean_dec(x_19); -x_24 = l_Lean_Elab_Tactic_SavedState_restore(x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_23); -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = lean_box(0); +x_24 = 0; +x_25 = l_Lean_Elab_Tactic_SavedState_restore(x_16, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_23); +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = lean_box(0); x_1 = x_14; -x_2 = x_26; -x_11 = x_25; +x_2 = x_27; +x_11 = x_26; goto _start; } } @@ -941,7 +941,7 @@ x_71 = l_Lean_Elab_Tactic_Conv_convert___closed__5; x_72 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_72, 0, x_70); lean_ctor_set(x_72, 1, x_71); -x_73 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_72, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_67); +x_73 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_72, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_67); x_74 = lean_ctor_get(x_73, 0); lean_inc(x_74); x_75 = lean_ctor_get(x_73, 1); @@ -2316,7 +2316,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalWhnf_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(74u); +x_1 = lean_unsigned_to_nat(79u); x_2 = lean_unsigned_to_nat(46u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2328,7 +2328,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalWhnf_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(76u); +x_1 = lean_unsigned_to_nat(81u); x_2 = lean_unsigned_to_nat(34u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2356,7 +2356,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalWhnf_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(74u); +x_1 = lean_unsigned_to_nat(79u); x_2 = lean_unsigned_to_nat(50u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2368,7 +2368,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalWhnf_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(74u); +x_1 = lean_unsigned_to_nat(79u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2609,7 +2609,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalReduce_declRa _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(78u); +x_1 = lean_unsigned_to_nat(83u); x_2 = lean_unsigned_to_nat(48u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2621,7 +2621,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalReduce_declRa _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(80u); +x_1 = lean_unsigned_to_nat(85u); x_2 = lean_unsigned_to_nat(36u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2649,7 +2649,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalReduce_declRa _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(78u); +x_1 = lean_unsigned_to_nat(83u); x_2 = lean_unsigned_to_nat(52u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2661,7 +2661,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalReduce_declRa _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(78u); +x_1 = lean_unsigned_to_nat(83u); x_2 = lean_unsigned_to_nat(62u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2920,7 +2920,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalZeta_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(82u); +x_1 = lean_unsigned_to_nat(87u); x_2 = lean_unsigned_to_nat(46u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2932,7 +2932,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalZeta_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(84u); +x_1 = lean_unsigned_to_nat(89u); x_2 = lean_unsigned_to_nat(40u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2960,7 +2960,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalZeta_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(82u); +x_1 = lean_unsigned_to_nat(87u); x_2 = lean_unsigned_to_nat(50u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -2972,7 +2972,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalZeta_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(82u); +x_1 = lean_unsigned_to_nat(87u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3095,7 +3095,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq1Inden _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(86u); +x_1 = lean_unsigned_to_nat(91u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3107,7 +3107,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq1Inden _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(87u); +x_1 = lean_unsigned_to_nat(92u); x_2 = lean_unsigned_to_nat(28u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3135,7 +3135,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq1Inden _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(86u); +x_1 = lean_unsigned_to_nat(91u); x_2 = lean_unsigned_to_nat(62u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3147,7 +3147,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq1Inden _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(86u); +x_1 = lean_unsigned_to_nat(91u); x_2 = lean_unsigned_to_nat(82u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3660,7 +3660,7 @@ x_85 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_85, 0, x_34); lean_ctor_set(x_85, 1, x_84); lean_ctor_set(x_85, 2, x_83); -x_86 = l_Lean_Elab_Tactic_evalTacticAux(x_85, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23); +x_86 = l_Lean_Elab_Tactic_evalTactic(x_85, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23); return x_86; } else @@ -3884,7 +3884,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeqBracke _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(89u); +x_1 = lean_unsigned_to_nat(94u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3896,7 +3896,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeqBracke _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(95u); +x_1 = lean_unsigned_to_nat(100u); x_2 = lean_unsigned_to_nat(49u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3924,7 +3924,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeqBracke _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(89u); +x_1 = lean_unsigned_to_nat(94u); x_2 = lean_unsigned_to_nat(62u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -3936,7 +3936,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeqBracke _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(89u); +x_1 = lean_unsigned_to_nat(94u); x_2 = lean_unsigned_to_nat(82u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4061,7 +4061,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedConv_de _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(97u); +x_1 = lean_unsigned_to_nat(102u); x_2 = lean_unsigned_to_nat(52u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4073,7 +4073,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedConv_de _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(98u); +x_1 = lean_unsigned_to_nat(103u); x_2 = lean_unsigned_to_nat(29u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4101,7 +4101,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedConv_de _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(97u); +x_1 = lean_unsigned_to_nat(102u); x_2 = lean_unsigned_to_nat(56u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4113,7 +4113,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedConv_de _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(97u); +x_1 = lean_unsigned_to_nat(102u); x_2 = lean_unsigned_to_nat(70u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4165,7 +4165,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalConvSeq(lean_object* x_1, l lean_object* x_11; lean_object* x_12; lean_object* x_13; x_11 = lean_unsigned_to_nat(0u); x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_13; } } @@ -4238,7 +4238,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(100u); +x_1 = lean_unsigned_to_nat(105u); x_2 = lean_unsigned_to_nat(49u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4250,7 +4250,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(101u); +x_1 = lean_unsigned_to_nat(106u); x_2 = lean_unsigned_to_nat(19u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4278,7 +4278,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(100u); +x_1 = lean_unsigned_to_nat(105u); x_2 = lean_unsigned_to_nat(53u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4290,7 +4290,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvSeq_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(100u); +x_1 = lean_unsigned_to_nat(105u); x_2 = lean_unsigned_to_nat(64u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4531,7 +4531,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvConvSeq_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(103u); +x_1 = lean_unsigned_to_nat(108u); x_2 = lean_unsigned_to_nat(53u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4543,7 +4543,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvConvSeq_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(106u); +x_1 = lean_unsigned_to_nat(111u); x_2 = lean_unsigned_to_nat(26u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4571,7 +4571,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvConvSeq_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(103u); +x_1 = lean_unsigned_to_nat(108u); x_2 = lean_unsigned_to_nat(57u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4583,7 +4583,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConvConvSeq_d _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(103u); +x_1 = lean_unsigned_to_nat(108u); x_2 = lean_unsigned_to_nat(72u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4635,7 +4635,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalParen(lean_object* x_1, lea lean_object* x_11; lean_object* x_12; lean_object* x_13; x_11 = lean_unsigned_to_nat(1u); x_12 = l_Lean_Syntax_getArg(x_1, x_11); -x_13 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_13; } } @@ -4700,7 +4700,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalParen_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(108u); +x_1 = lean_unsigned_to_nat(113u); x_2 = lean_unsigned_to_nat(47u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4712,7 +4712,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalParen_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(109u); +x_1 = lean_unsigned_to_nat(114u); x_2 = lean_unsigned_to_nat(19u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4740,7 +4740,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalParen_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(108u); +x_1 = lean_unsigned_to_nat(113u); x_2 = lean_unsigned_to_nat(51u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -4752,7 +4752,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalParen_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(108u); +x_1 = lean_unsigned_to_nat(113u); x_2 = lean_unsigned_to_nat(60u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5340,7 +5340,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_13 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_13) == 0) { lean_object* x_14; lean_object* x_15; @@ -5451,7 +5451,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTacticC _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(124u); +x_1 = lean_unsigned_to_nat(129u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5463,7 +5463,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTacticC _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(126u); +x_1 = lean_unsigned_to_nat(131u); x_2 = lean_unsigned_to_nat(34u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5491,7 +5491,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTacticC _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(124u); +x_1 = lean_unsigned_to_nat(129u); x_2 = lean_unsigned_to_nat(62u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5503,7 +5503,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTacticC _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(124u); +x_1 = lean_unsigned_to_nat(129u); x_2 = lean_unsigned_to_nat(82u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5561,7 +5561,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_11 = l_Lean_Elab_Tactic_evalTacticAux(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_Tactic_evalTactic(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; @@ -5922,7 +5922,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTactic_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(128u); +x_1 = lean_unsigned_to_nat(133u); x_2 = lean_unsigned_to_nat(54u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5934,7 +5934,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTactic_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(134u); +x_1 = lean_unsigned_to_nat(139u); x_2 = lean_unsigned_to_nat(43u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5962,7 +5962,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTactic_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(128u); +x_1 = lean_unsigned_to_nat(133u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5974,7 +5974,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalNestedTactic_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(128u); +x_1 = lean_unsigned_to_nat(133u); x_2 = lean_unsigned_to_nat(74u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -6256,7 +6256,7 @@ x_57 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_57, 0, x_36); lean_ctor_set(x_57, 1, x_56); lean_ctor_set(x_57, 2, x_55); -x_58 = l_Lean_Elab_Tactic_evalTacticAux(x_57, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +x_58 = l_Lean_Elab_Tactic_evalTactic(x_57, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); return x_58; } else @@ -6968,7 +6968,7 @@ x_125 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_125, 0, x_79); lean_ctor_set(x_125, 1, x_4); lean_ctor_set(x_125, 2, x_124); -x_126 = l_Lean_Elab_Tactic_evalTacticAux(x_125, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); +x_126 = l_Lean_Elab_Tactic_evalTactic(x_125, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); return x_126; } else @@ -6988,7 +6988,7 @@ x_132 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_132, 0, x_79); lean_ctor_set(x_132, 1, x_4); lean_ctor_set(x_132, 2, x_131); -x_133 = l_Lean_Elab_Tactic_evalTacticAux(x_132, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); +x_133 = l_Lean_Elab_Tactic_evalTactic(x_132, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); return x_133; } } @@ -7026,7 +7026,7 @@ x_148 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_148, 0, x_79); lean_ctor_set(x_148, 1, x_4); lean_ctor_set(x_148, 2, x_147); -x_149 = l_Lean_Elab_Tactic_evalTacticAux(x_148, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); +x_149 = l_Lean_Elab_Tactic_evalTactic(x_148, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); return x_149; } else @@ -7046,7 +7046,7 @@ x_155 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_155, 0, x_79); lean_ctor_set(x_155, 1, x_4); lean_ctor_set(x_155, 2, x_154); -x_156 = l_Lean_Elab_Tactic_evalTacticAux(x_155, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); +x_156 = l_Lean_Elab_Tactic_evalTactic(x_155, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_68); return x_156; } } @@ -7197,7 +7197,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConv_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(148u); +x_1 = lean_unsigned_to_nat(153u); x_2 = lean_unsigned_to_nat(46u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7209,7 +7209,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConv_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(159u); +x_1 = lean_unsigned_to_nat(164u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7237,7 +7237,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConv_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(148u); +x_1 = lean_unsigned_to_nat(153u); x_2 = lean_unsigned_to_nat(50u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7249,7 +7249,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalConv_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(148u); +x_1 = lean_unsigned_to_nat(153u); x_2 = lean_unsigned_to_nat(58u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7372,7 +7372,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalFirst_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(161u); +x_1 = lean_unsigned_to_nat(166u); x_2 = lean_unsigned_to_nat(55u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7384,7 +7384,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalFirst_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(162u); +x_1 = lean_unsigned_to_nat(167u); x_2 = lean_unsigned_to_nat(18u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7412,7 +7412,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalFirst_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(161u); +x_1 = lean_unsigned_to_nat(166u); x_2 = lean_unsigned_to_nat(59u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -7424,7 +7424,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_Conv_evalFirst_declRan _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(161u); +x_1 = lean_unsigned_to_nat(166u); x_2 = lean_unsigned_to_nat(68u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Change.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Change.c index 64eb27894ad7..a29968cb360b 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Change.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Change.c @@ -35,7 +35,6 @@ lean_object* l_Lean_Elab_Tactic_filterOldMVars(lean_object*, lean_object*, lean_ static lean_object* l_Lean_Elab_Tactic_Conv_evalChange___closed__12; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalChange_declRange___closed__3; lean_object* l_Lean_Meta_isExprDefEqGuarded(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalChange_declRange___closed__5; static lean_object* l_Lean_Elab_Tactic_Conv_evalChange___closed__1; @@ -43,6 +42,7 @@ static lean_object* l_Lean_Elab_Tactic_Conv_evalChange___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalChange___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_Conv_getLhs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___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___regBuiltin_Lean_Elab_Tactic_Conv_evalChange___closed__6; lean_object* l_Lean_Elab_Tactic_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalChange_declRange___closed__7; @@ -372,7 +372,7 @@ x_53 = l_Lean_Elab_Tactic_Conv_evalChange___closed__16; x_54 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_54, 0, x_52); lean_ctor_set(x_54, 1, x_53); -x_55 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_54, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); +x_55 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_54, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Congr.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Congr.c index 5edf23ed2618..387f88cdaeeb 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Congr.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Congr.c @@ -143,9 +143,9 @@ static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Elab_Tactic_Conv_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Tactic_Conv_selectIdx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_evalLhs___rarg___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalLhs_declRange___closed__4; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalLhs___boxed(lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_extLetBodyCongr_x3f___lambda__3___closed__6; lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -156,7 +156,6 @@ static lean_object* l___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Tactic_ lean_object* l_Lean_Expr_sort___override(lean_object*); lean_object* l_Lean_Elab_Tactic_Conv_markAsConvGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_extLetBodyCongr_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*); -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_extLetBodyCongr_x3f___lambda__3___closed__3; lean_object* lean_array_to_list(lean_object*, lean_object*); @@ -189,8 +188,10 @@ extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_extLetBodyCongr_x3f___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Tactic_Conv_extCore___lambda__2___closed__3; lean_object* l_Int_toNat(lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___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___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Tactic_Conv_extCore___lambda__2___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalLhs_declRange___closed__5; +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*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Tactic_Conv_selectIdx___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalExt(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalRhs___closed__2; @@ -200,7 +201,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_extLetBodyCongr_x3f___lambda__3 static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalCongr___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalCongr___boxed(lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalExt_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalArg_declRange___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalArg_declRange___closed__2; @@ -1417,7 +1417,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Ta { lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_2, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_10); x_12 = l___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Tactic_Conv_congrApp___closed__1; lean_inc(x_11); x_13 = lean_mk_array(x_11, x_12); @@ -3459,7 +3459,7 @@ x_24 = l___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Tactic_Conv_selectId x_25 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_24); -x_26 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_26 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); return x_26; } } @@ -3584,7 +3584,7 @@ if (lean_obj_tag(x_28) == 0) { lean_object* x_29; lean_object* x_30; uint8_t x_31; x_29 = l___private_Lean_Elab_Tactic_Conv_Congr_0__Lean_Elab_Tactic_Conv_selectIdx___closed__4; -x_30 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_26); +x_30 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_26); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4612,7 +4612,7 @@ lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_dec(x_18); lean_dec(x_3); x_23 = l_Lean_Elab_Tactic_Conv_evalArg___lambda__2___closed__4; -x_24 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_24 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c index e846884f3f4b..23e5f309abc2 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Pattern.c @@ -57,7 +57,6 @@ static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___lambda__3___closed__4; lean_object* l_Lean_Elab_Tactic_Conv_mkConvGoalFor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern_declRange___closed__7; lean_object* lean_st_mk_ref(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___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___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalPattern___closed__4; lean_object* l_Lean_Meta_isExprDefEqGuarded(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -69,6 +68,7 @@ lean_object* l_Lean_Expr_toHeadIndex(lean_object*); lean_object* l_Lean_Elab_Tactic_Conv_getLhs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; +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*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Conv_Pattern_0__Lean_Elab_Tactic_Conv_findPattern_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Conv_Pattern_0__Lean_Elab_Tactic_Conv_findPattern_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_Conv_evalPattern___closed__3; @@ -1749,7 +1749,7 @@ x_41 = l_Lean_Elab_Tactic_Conv_evalPattern___lambda__3___closed__4; x_42 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_42, 0, x_40); lean_ctor_set(x_42, 1, x_41); -x_43 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_42, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_36); +x_43 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_42, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_36); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Conv/Unfold.c b/stage0/stdlib/Lean/Elab/Tactic/Conv/Unfold.c index 7c76f472f3dc..b5fc33bf8b4f 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Conv/Unfold.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Conv/Unfold.c @@ -16,6 +16,7 @@ extern "C" { static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold___closed__16; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold___closed__10; +lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_withMainContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold_declRange___closed__7; lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -34,7 +35,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold___closed__13 static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold_declRange___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_Conv_evalUnfold___closed__5; -lean_object* l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_unfold(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Conv_evalUnfold___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_Conv_evalUnfold_declRange___closed__4; @@ -65,7 +65,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_11 = l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; lean_object* x_14; diff --git a/stage0/stdlib/Lean/Elab/Tactic/Delta.c b/stage0/stdlib/Lean/Elab/Tactic/Delta.c index b6b0d62be6b1..3e17c407b991 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Delta.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Delta.c @@ -63,7 +63,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDelta_declRange___closed static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDelta___closed__10; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDelta___closed__3; lean_object* lean_format_pretty(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_deltaLocalDecl___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*); @@ -73,6 +72,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalDelta___spe extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_evalDelta___spec__7___closed__1; static lean_object* l_Lean_Elab_Tactic_deltaLocalDecl___closed__8; +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___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___regBuiltin_Lean_Elab_Tactic_evalDelta_declRange___closed__6; static lean_object* l_Lean_Elab_Tactic_deltaLocalDecl___closed__6; LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_evalDelta___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -953,7 +953,7 @@ x_16 = l_Lean_Elab_Tactic_deltaLocalDecl___closed__8; x_17 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_18; } } diff --git a/stage0/stdlib/Lean/Elab/Tactic/ElabTerm.c b/stage0/stdlib/Lean/Elab/Tactic/ElabTerm.c index c669a479a3f0..089dd50246f3 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/ElabTerm.c +++ b/stage0/stdlib/Lean/Elab/Tactic/ElabTerm.c @@ -17,7 +17,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducibleAndInstance lean_object* l_Lean_Meta_assert(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_findSomeRevM_x3f___at_Lean_Elab_Tactic_evalRename___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalApplyLikeTactic(lean_object*, lean_object*, 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_evalRename___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalApplyLikeTactic___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSpecialize_declRange___closed__2; size_t lean_usize_add(size_t, size_t); @@ -38,19 +37,18 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_elabAsFVar___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRename_declRange___closed__1; LEAN_EXPORT lean_object* l_Std_PersistentArray_findSomeRevM_x3f___at_Lean_Elab_Tactic_evalRename___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide___closed__2; lean_object* l_Lean_addDecl___at_Lean_Elab_Term_declareTacticSyntax___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_elabTermWithHoles___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithUnfoldingAll___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalApply_declRange___closed__6; +lean_object* l_Lean_Elab_Tactic_SavedState_restore(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalExact(lean_object*); lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithUnfoldingAll_declRange___closed__4; -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_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalWithReducible(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -61,6 +59,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_closeMainGoalUsing___lambda__1(lean_ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducible___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducibleAndInstances___closed__3; uint8_t l_Lean_MetavarKind_isNatural(uint8_t); +LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___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_array_uset(lean_object*, size_t, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalExact___closed__6; lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_getMainTarget___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -69,11 +68,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide(lean_object* LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefine_x27(lean_object*); static lean_object* l_Lean_Elab_Tactic_refineCore___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_refineCore___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefine_x27_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_closeMainGoalUsing(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Tactic_evalTacticAux(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_evalRename_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefine___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabTermForApply___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -84,6 +81,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide_declRange__ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSpecialize(lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalDecide___boxed(lean_object*); +lean_object* l_Lean_Elab_Tactic_evalTactic(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_evalDecide_declRange___closed__6; static lean_object* l_Lean_Elab_Tactic_refineCore___lambda__4___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -109,16 +107,14 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange___close LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalNativeDecide___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_filterOldMVars___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabAsFVar___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalApply(lean_object*, 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_withoutModifyingStateWithInfoAndMessages___at_Lean_Elab_Tactic_evalRename___spec__8(lean_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_evalNativeDecide___rarg___lambda__1___closed__2; static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg___closed__1; lean_object* l_Lean_Elab_Term_mkAuxName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide___closed__5; lean_object* l_Lean_assignExprMVar___at_Lean_Elab_Tactic_closeMainGoal___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalDecide___rarg___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(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*); lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -129,7 +125,6 @@ lean_object* l_Lean_Meta_zetaReduce___lambda__2___boxed(lean_object*, lean_objec static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalConstructor___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_getFVarId___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalDecide___rarg___lambda__1___closed__3; -static lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1___closed__2; static lean_object* l_Lean_Elab_Tactic_evalDecide___rarg___lambda__1___closed__5; lean_object* l_Lean_Meta_mkDecide(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalConstructor___closed__5; @@ -138,6 +133,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSpecialize_declRange___c lean_object* l_Lean_Meta_mkEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_apply(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_getFVarId___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Tactic_evalRename___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalExact_declRange___closed__7; @@ -147,12 +143,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_refineCore___lambda__4(lean_object*, static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefine_x27_declRange___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_filterOldMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalSpecialize___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducible_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefine_declRange___closed__1; lean_object* l_Lean_Meta_intro1Core(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithUnfoldingAll_declRange___closed__2; static lean_object* l_Lean_Elab_Tactic_evalNativeDecide___rarg___lambda__1___closed__7; +static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabTermWithHoles(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_array_fget(lean_object*, lean_object*); @@ -163,6 +160,7 @@ static lean_object* l_Lean_Elab_Tactic_evalNativeDecide___rarg___closed__1; lean_object* l_Lean_Meta_rename(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvar___override(lean_object*); static lean_object* l_Lean_Elab_Tactic_evalSpecialize___closed__2; +LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getMVarsNoDelayed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalRename___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide___closed__4; @@ -187,7 +185,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tacti lean_object* l_Lean_Elab_Term_elabTerm(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalExact___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalConstructor___boxed(lean_object*); -static lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4; static lean_object* l_Lean_Elab_Tactic_evalExact___closed__8; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducibleAndInstances___closed__2; @@ -199,6 +196,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange___close static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducible___closed__1; 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*); static lean_object* l_Lean_Elab_Tactic_evalExact___closed__1; +static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__2; static lean_object* l_Lean_Elab_Tactic_evalDecide___rarg___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalApply___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducibleAndInstances___closed__1; @@ -206,7 +204,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSpecialize_declRange___c static lean_object* l_Lean_Elab_Tactic_evalSpecialize___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_logUnassignedAndAbort___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___regBuiltin_Lean_Elab_Tactic_evalRefine_declRange(lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabTermForApply___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabTerm_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -216,7 +213,6 @@ static lean_object* l_Lean_Elab_Tactic_evalExact___closed__6; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefine_x27_declRange___closed__4; lean_object* l_Lean_Elab_Term_isLetRecAuxMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRename(lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___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_evalWithReducibleAndInstances_declRange___closed__3; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide_declRange(lean_object*); @@ -263,18 +259,22 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefine_x27___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducible_declRange___closed__2; lean_object* l_Lean_LocalDecl_fvarId(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSpecialize___closed__1; +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___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___regBuiltin_Lean_Elab_Tactic_evalRename_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_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___regBuiltin_Lean_Elab_Tactic_evalWithReducible_declRange___closed__1; static lean_object* l___private_Lean_Elab_Tactic_ElabTerm_0__Lean_Elab_Tactic_preprocessPropToDecide___closed__2; lean_object* l_Lean_LocalDecl_type(lean_object*); static lean_object* l_Lean_Elab_Tactic_evalNativeDecide___rarg___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_Tactic_ElabTerm_0__Lean_Elab_Tactic_preprocessPropToDecide___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalExact___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalNativeDecide___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_refineCore___lambda__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_filterOldMVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabTermEnsuringType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_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_evalWithReducibleAndInstances_declRange___closed__7; static lean_object* l_Lean_Elab_Tactic_evalRefine___closed__1; static lean_object* l_Lean_Elab_throwAbortTactic___at_Lean_Elab_Tactic_logUnassignedAndAbort___spec__1___rarg___closed__1; @@ -286,6 +286,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithUnfoldingAll___close static lean_object* l_Lean_Elab_Tactic_filterOldMVars___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalExact___closed__1; +static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__3; static lean_object* l_Lean_Elab_Tactic_evalApply___closed__3; static lean_object* l_Lean_Elab_Tactic_evalNativeDecide___rarg___lambda__1___closed__4; static lean_object* l_Lean_Elab_Tactic_evalRefine___closed__2; @@ -387,6 +388,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalExact___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRefine___closed__1; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_findDeclRevM_x3f___at_Lean_Elab_Tactic_evalRename___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_getFVarId___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducibleAndInstances(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_refineCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -428,7 +430,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_closeMainGoalUsing___lambda__1___box static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange___closed__2; static lean_object* l_Lean_Elab_Tactic_getFVarId___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_refineCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithUnfoldingAll___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalExact(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_evalRefine_x27_declRange___closed__7; @@ -451,7 +452,7 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDecide___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalConstructor___closed__4; static lean_object* l_Lean_Elab_Tactic_evalDecide___rarg___lambda__1___closed__2; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -lean_object* l_Lean_Meta_constructor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_constructor(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithUnfoldingAll___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalExact_declRange___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalWithReducibleAndInstances_declRange(lean_object*); @@ -3016,44 +3017,6 @@ x_15 = l_Lean_Elab_Tactic_elabTermWithHoles(x_1, x_2, x_3, x_14, x_5, x_6, x_7, return x_15; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_ctor_get(x_8, 5); -x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_6, x_7, x_8, x_9, x_10); -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_12, 0); -lean_inc(x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_11); -lean_ctor_set(x_15, 1, x_14); -lean_ctor_set_tag(x_12, 1); -lean_ctor_set(x_12, 0, x_15); -return x_12; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_12, 0); -x_17 = lean_ctor_get(x_12, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_12); -lean_inc(x_11); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_11); -lean_ctor_set(x_18, 1, x_16); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -return x_19; -} -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_refineCore___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { @@ -3251,7 +3214,7 @@ x_43 = l_Lean_Elab_Tactic_refineCore___lambda__4___closed__6; x_44 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_44, 0, x_42); lean_ctor_set(x_44, 1, x_43); -x_45 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_44, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_27); +x_45 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_44, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_27); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -3402,22 +3365,6 @@ x_15 = l_Lean_Elab_Tactic_withMainContext___rarg(x_14, x_4, x_5, x_6, x_7, x_8, return x_15; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_11; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_refineCore___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { @@ -3926,7 +3873,7 @@ lean_dec(x_19); lean_dec(x_18); lean_dec(x_17); x_21 = l_Lean_Elab_Tactic_evalSpecialize___lambda__1___closed__2; -x_22 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +x_22 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -5561,46 +5508,47 @@ 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; +lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); +x_13 = 0; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_13 = l_Lean_Meta_constructor(x_11, x_5, x_6, x_7, x_8, x_12); -if (lean_obj_tag(x_13) == 0) +x_14 = l_Lean_Meta_constructor(x_11, x_13, x_5, x_6, x_7, x_8, x_12); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -lean_dec(x_13); -x_16 = 0; +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = 0; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_17 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_16, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_15); -if (lean_obj_tag(x_17) == 0) +x_18 = l_Lean_Elab_Term_synthesizeSyntheticMVars(x_17, x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -x_19 = l_Lean_Elab_Tactic_replaceMainGoal(x_14, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -return x_19; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = l_Lean_Elab_Tactic_replaceMainGoal(x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_19); +return x_20; } else { -uint8_t x_20; -lean_dec(x_14); +uint8_t x_21; +lean_dec(x_15); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -5609,29 +5557,29 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_20 = !lean_is_exclusive(x_17); -if (x_20 == 0) +x_21 = !lean_is_exclusive(x_18); +if (x_21 == 0) { -return x_17; +return x_18; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_17, 0); -x_22 = lean_ctor_get(x_17, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_18, 0); +x_23 = lean_ctor_get(x_18, 1); +lean_inc(x_23); lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_17); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +lean_dec(x_18); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } } else { -uint8_t x_24; +uint8_t x_25; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -5640,29 +5588,29 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_24 = !lean_is_exclusive(x_13); -if (x_24 == 0) +x_25 = !lean_is_exclusive(x_14); +if (x_25 == 0) { -return x_13; +return x_14; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_13, 0); -x_26 = lean_ctor_get(x_13, 1); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_14, 0); +x_27 = lean_ctor_get(x_14, 1); +lean_inc(x_27); lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_13); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_dec(x_14); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } } else { -uint8_t x_28; +uint8_t x_29; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -5671,23 +5619,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_28 = !lean_is_exclusive(x_10); -if (x_28 == 0) +x_29 = !lean_is_exclusive(x_10); +if (x_29 == 0) { return x_10; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_10, 0); -x_30 = lean_ctor_get(x_10, 1); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_10, 0); +x_31 = lean_ctor_get(x_10, 1); +lean_inc(x_31); lean_inc(x_30); -lean_inc(x_29); lean_dec(x_10); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } } @@ -5901,7 +5849,7 @@ if (x_15 == 0) uint8_t x_16; lean_object* x_17; x_16 = 2; lean_ctor_set_uint8(x_14, 5, x_16); -x_17 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_17 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_17) == 0) { uint8_t x_18; @@ -5981,7 +5929,7 @@ lean_ctor_set_uint8(x_40, 11, x_36); lean_ctor_set_uint8(x_40, 12, x_37); lean_ctor_set_uint8(x_40, 13, x_38); lean_ctor_set(x_6, 0, x_40); -x_41 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_41 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_41) == 0) { lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; @@ -6094,7 +6042,7 @@ lean_ctor_set(x_72, 2, x_52); lean_ctor_set(x_72, 3, x_53); lean_ctor_set(x_72, 4, x_54); lean_ctor_set(x_72, 5, x_55); -x_73 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_72, x_7, x_8, x_9, x_10); +x_73 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_72, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_73) == 0) { lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; @@ -6330,7 +6278,7 @@ if (x_15 == 0) uint8_t x_16; lean_object* x_17; x_16 = 3; lean_ctor_set_uint8(x_14, 5, x_16); -x_17 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_17 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_17) == 0) { uint8_t x_18; @@ -6410,7 +6358,7 @@ lean_ctor_set_uint8(x_40, 11, x_36); lean_ctor_set_uint8(x_40, 12, x_37); lean_ctor_set_uint8(x_40, 13, x_38); lean_ctor_set(x_6, 0, x_40); -x_41 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_41 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_41) == 0) { lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; @@ -6523,7 +6471,7 @@ lean_ctor_set(x_72, 2, x_52); lean_ctor_set(x_72, 3, x_53); lean_ctor_set(x_72, 4, x_54); lean_ctor_set(x_72, 5, x_55); -x_73 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_72, x_7, x_8, x_9, x_10); +x_73 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_72, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_73) == 0) { lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; @@ -6759,7 +6707,7 @@ if (x_15 == 0) uint8_t x_16; lean_object* x_17; x_16 = 0; lean_ctor_set_uint8(x_14, 5, x_16); -x_17 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_17 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_17) == 0) { uint8_t x_18; @@ -6839,7 +6787,7 @@ lean_ctor_set_uint8(x_40, 11, x_36); lean_ctor_set_uint8(x_40, 12, x_37); lean_ctor_set_uint8(x_40, 13, x_38); lean_ctor_set(x_6, 0, x_40); -x_41 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_41 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_41) == 0) { lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; @@ -6952,7 +6900,7 @@ lean_ctor_set(x_72, 2, x_52); lean_ctor_set(x_72, 3, x_53); lean_ctor_set(x_72, 4, x_54); lean_ctor_set(x_72, 5, x_55); -x_73 = l_Lean_Elab_Tactic_evalTacticAux(x_12, x_2, x_3, x_4, x_5, x_72, x_7, x_8, x_9, x_10); +x_73 = l_Lean_Elab_Tactic_evalTactic(x_12, x_2, x_3, x_4, x_5, x_72, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_73) == 0) { lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; @@ -8574,59 +8522,107 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withNewMCtxDepth___at_Lean_Elab_Tac return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_withoutModifyingStateWithInfoAndMessages___at_Lean_Elab_Tactic_evalRename___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_apply_2(x_1, x_2, x_3); -x_12 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___rarg(x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = l_Lean_Elab_Tactic_saveState___rarg(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_14 = lean_apply_9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; uint8_t x_19; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = 0; +x_18 = l_Lean_Elab_Tactic_SavedState_restore(x_12, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_16); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -return x_12; +lean_object* x_20; +x_20 = lean_ctor_get(x_18, 0); +lean_dec(x_20); +lean_ctor_set(x_18, 0, x_15); +return x_18; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_inc(x_14); -lean_dec(x_12); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -return x_16; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_15); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } else { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_12); -if (x_17 == 0) +lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; uint8_t x_27; +x_23 = lean_ctor_get(x_14, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_14, 1); +lean_inc(x_24); +lean_dec(x_14); +x_25 = 0; +x_26 = l_Lean_Elab_Tactic_SavedState_restore(x_12, x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_24); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) { -return x_12; +lean_object* x_28; +x_28 = lean_ctor_get(x_26, 0); +lean_dec(x_28); +lean_ctor_set_tag(x_26, 1); +lean_ctor_set(x_26, 0, x_23); +return x_26; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_12, 0); -x_19 = lean_ctor_get(x_12, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_12); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_26, 1); +lean_inc(x_29); +lean_dec(x_26); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_23); +lean_ctor_set(x_30, 1, x_29); +return x_30; } } } } -static lean_object* _init_l_Lean_Elab_Tactic_evalRename___lambda__1___closed__1() { +static lean_object* _init_l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -8634,16 +8630,16 @@ x_1 = lean_mk_string_from_bytes("failed to find a hypothesis with type", 37); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalRename___lambda__1___closed__2() { +static lean_object* _init_l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_evalRename___lambda__1___closed__1; +x_1 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalRename___lambda__1___closed__3() { +static lean_object* _init_l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__3() { _start: { lean_object* x_1; @@ -8651,16 +8647,16 @@ x_1 = lean_mk_string_from_bytes("", 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4() { +static lean_object* _init_l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_evalRename___lambda__1___closed__3; +x_1 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; lean_object* x_13; @@ -8702,11 +8698,11 @@ x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); x_20 = l_Lean_indentExpr(x_14); -x_21 = l_Lean_Elab_Tactic_evalRename___lambda__1___closed__2; +x_21 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__2; x_22 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_22, 0, x_21); lean_ctor_set(x_22, 1, x_20); -x_23 = l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4; +x_23 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4; x_24 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_24, 0, x_22); lean_ctor_set(x_24, 1, x_23); @@ -8821,10 +8817,21 @@ return x_39; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_12 = lean_alloc_closure((void*)(l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___boxed), 11, 2); +lean_closure_set(x_12, 0, x_1); +lean_closure_set(x_12, 1, x_2); +x_13 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_withoutRecover___rarg), 10, 1); +lean_closure_set(x_13, 0, x_12); +x_14 = l_Lean_Elab_Tactic_saveState___rarg(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); @@ -8833,15 +8840,110 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_12 = l_Lean_Elab_withoutModifyingStateWithInfoAndMessages___at_Lean_Elab_Tactic_evalRename___spec__8(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_12) == 0) +x_17 = l_Lean_Meta_withNewMCtxDepth___at_Lean_Elab_Tactic_evalRename___spec__7___rarg(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); +lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; uint8_t x_22; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = 0; +x_21 = l_Lean_Elab_Tactic_SavedState_restore(x_15, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_19); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +lean_ctor_set(x_21, 0, x_18); +return x_21; +} +else +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_18); +lean_ctor_set(x_25, 1, x_24); +return x_25; +} +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; uint8_t x_30; +x_26 = lean_ctor_get(x_17, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_17, 1); +lean_inc(x_27); +lean_dec(x_17); +x_28 = 0; +x_29 = l_Lean_Elab_Tactic_SavedState_restore(x_15, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_29, 0); +lean_dec(x_31); +lean_ctor_set_tag(x_29, 1); +lean_ctor_set(x_29, 0, x_26); +return x_29; +} +else +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +lean_dec(x_29); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_26); +lean_ctor_set(x_33, 1, x_32); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_13 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -lean_dec(x_12); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); @@ -8849,40 +8951,40 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_3); -x_15 = l_Lean_Elab_Tactic_getMainGoal(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); -if (lean_obj_tag(x_15) == 0) +x_16 = l_Lean_Elab_Tactic_getMainGoal(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -lean_dec(x_15); -x_18 = l_Lean_Syntax_getId(x_2); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Lean_Syntax_getId(x_3); +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -x_19 = l_Lean_Meta_rename(x_16, x_13, x_18, x_7, x_8, x_9, x_10, x_17); -if (lean_obj_tag(x_19) == 0) +x_20 = l_Lean_Meta_rename(x_17, x_14, x_19, x_8, x_9, x_10, x_11, x_18); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_box(0); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_20); -lean_ctor_set(x_23, 1, x_22); -x_24 = l_Lean_Elab_Tactic_replaceMainGoal(x_23, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); -return x_24; +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_box(0); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_21); +lean_ctor_set(x_24, 1, x_23); +x_25 = l_Lean_Elab_Tactic_replaceMainGoal(x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +return x_25; } else { -uint8_t x_25; +uint8_t x_26; +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -8890,31 +8992,31 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -x_25 = !lean_is_exclusive(x_19); -if (x_25 == 0) +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) { -return x_19; +return x_20; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_19, 0); -x_27 = lean_ctor_get(x_19, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_20, 0); +x_28 = lean_ctor_get(x_20, 1); +lean_inc(x_28); lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_19); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; +lean_dec(x_20); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } else { -uint8_t x_29; -lean_dec(x_13); +uint8_t x_30; +lean_dec(x_14); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -8922,30 +9024,30 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -x_29 = !lean_is_exclusive(x_15); -if (x_29 == 0) +x_30 = !lean_is_exclusive(x_16); +if (x_30 == 0) { -return x_15; +return x_16; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_15, 0); -x_31 = lean_ctor_get(x_15, 1); +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_16, 0); +x_32 = lean_ctor_get(x_16, 1); +lean_inc(x_32); lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_15); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_dec(x_16); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } } else { -uint8_t x_33; +uint8_t x_34; +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -8953,24 +9055,23 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -x_33 = !lean_is_exclusive(x_12); -if (x_33 == 0) +x_34 = !lean_is_exclusive(x_13); +if (x_34 == 0) { -return x_12; +return x_13; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_12, 0); -x_35 = lean_ctor_get(x_12, 1); +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_13, 0); +x_36 = lean_ctor_get(x_13, 1); +lean_inc(x_36); lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_12); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; +lean_dec(x_13); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } @@ -9062,18 +9163,14 @@ return x_20; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* x_21; lean_object* x_22; lean_object* x_23; x_21 = lean_box(0); -x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalRename___lambda__1___boxed), 11, 2); +x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalRename___lambda__1___boxed), 12, 3); lean_closure_set(x_22, 0, x_15); lean_closure_set(x_22, 1, x_21); -x_23 = lean_alloc_closure((void*)(l_Lean_Meta_withNewMCtxDepth___at_Lean_Elab_Tactic_evalRename___spec__7___rarg), 10, 1); -lean_closure_set(x_23, 0, x_22); -x_24 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_evalRename___lambda__2___boxed), 11, 2); -lean_closure_set(x_24, 0, x_23); -lean_closure_set(x_24, 1, x_17); -x_25 = l_Lean_Elab_Tactic_withMainContext___rarg(x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_25; +lean_closure_set(x_22, 2, x_17); +x_23 = l_Lean_Elab_Tactic_withMainContext___rarg(x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_23; } } } @@ -9145,22 +9242,22 @@ lean_dec(x_4); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Lean_Elab_Tactic_evalRename___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 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_4); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRename___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_12; -x_12 = l_Lean_Elab_Tactic_evalRename___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_2); -return x_12; +lean_object* x_13; +x_13 = l_Lean_Elab_Tactic_evalRename___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_3); +return x_13; } } static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRename___closed__1() { @@ -9217,7 +9314,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalRename_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(260u); +x_1 = lean_unsigned_to_nat(256u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -9372,7 +9469,7 @@ x_12 = l___private_Lean_Elab_Tactic_ElabTerm_0__Lean_Elab_Tactic_preprocessPropT x_13 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_13, 0, x_12); lean_ctor_set(x_13, 1, x_11); -x_14 = l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4; +x_14 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4; x_15 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_15, 0, x_13); lean_ctor_set(x_15, 1, x_14); @@ -9766,11 +9863,11 @@ x_35 = l_Lean_Elab_Tactic_evalDecide___rarg___lambda__2___closed__2; x_36 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_36, 0, x_35); lean_ctor_set(x_36, 1, x_34); -x_37 = l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4; +x_37 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4; x_38 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_38, 0, x_36); lean_ctor_set(x_38, 1, x_37); -x_39 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_31); +x_39 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_31); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -9910,11 +10007,11 @@ x_72 = l_Lean_Elab_Tactic_evalDecide___rarg___lambda__2___closed__2; x_73 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_73, 0, x_72); lean_ctor_set(x_73, 1, x_71); -x_74 = l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4; +x_74 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4; x_75 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_75, 0, x_73); lean_ctor_set(x_75, 1, x_74); -x_76 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_75, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_68); +x_76 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_75, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_68); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -10167,7 +10264,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange__ _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(270u); x_2 = lean_unsigned_to_nat(43u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10179,7 +10276,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(284u); +x_1 = lean_unsigned_to_nat(280u); x_2 = lean_unsigned_to_nat(74u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10207,7 +10304,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange__ _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(270u); x_2 = lean_unsigned_to_nat(47u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10219,7 +10316,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalDecide_declRange__ _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(270u); x_2 = lean_unsigned_to_nat(57u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10807,7 +10904,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide_declR _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(293u); x_2 = lean_unsigned_to_nat(49u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10819,7 +10916,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide_declR _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(304u); +x_1 = lean_unsigned_to_nat(300u); x_2 = lean_unsigned_to_nat(160u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10847,7 +10944,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide_declR _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(293u); x_2 = lean_unsigned_to_nat(53u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -10859,7 +10956,7 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_evalNativeDecide_declR _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(293u); x_2 = lean_unsigned_to_nat(69u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -11288,14 +11385,14 @@ l_Lean_Elab_Tactic_elabAsFVar___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic lean_mark_persistent(l_Lean_Elab_Tactic_elabAsFVar___lambda__1___closed__1); l_Lean_Elab_Tactic_elabAsFVar___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_elabAsFVar___lambda__1___closed__2(); lean_mark_persistent(l_Lean_Elab_Tactic_elabAsFVar___lambda__1___closed__2); -l_Lean_Elab_Tactic_evalRename___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_evalRename___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalRename___lambda__1___closed__1); -l_Lean_Elab_Tactic_evalRename___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_evalRename___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalRename___lambda__1___closed__2); -l_Lean_Elab_Tactic_evalRename___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_evalRename___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalRename___lambda__1___closed__3); -l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_evalRename___lambda__1___closed__4); +l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__1 = _init_l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__1); +l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__2 = _init_l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__2); +l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__3 = _init_l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__3); +l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4 = _init_l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_evalRename___spec__8___at_Lean_Elab_Tactic_evalRename___spec__9___lambda__1___closed__4); l_Lean_Elab_Tactic_evalRename___closed__1 = _init_l_Lean_Elab_Tactic_evalRename___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_evalRename___closed__1); l_Lean_Elab_Tactic_evalRename___closed__2 = _init_l_Lean_Elab_Tactic_evalRename___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Induction.c b/stage0/stdlib/Lean/Elab/Tactic/Induction.c index c09dbda2d51a..d10bbe175860 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Induction.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Induction.c @@ -14,6 +14,7 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__1; static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___closed__3; static lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_go___lambda__2___closed__1; static lean_object* l_Lean_Elab_Tactic_isHoleRHS___closed__6; @@ -37,6 +38,7 @@ lean_object* l_Lean_registerTraceClass(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___lambda__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_erase_macro_scopes(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_evalInduction___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_initFn____x40_Lean_Elab_Tactic_Induction___hyg_8482_(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); @@ -58,7 +60,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts___lambda__1(lean_ob lean_object* l_Lean_Meta_whnfForall(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_filterTRAux___at_Lean_resolveGlobalConstCore___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__5___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_applyPreTac___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange___closed__6; @@ -69,7 +70,6 @@ uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getOptPreTacOfOptInductionAlts___closed__1; lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___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* l_Lean_Expr_bindingDomain_x21(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); @@ -83,20 +83,18 @@ extern lean_object* l_Std_Format_defWidth; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabCasesTargets___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltsOfOptInductionAlts(lean_object*); -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__2; lean_object* l_Lean_log___at_Lean_Elab_Tactic_closeUsingOrAdmit___spec__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getBindingName___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___lambda__2___closed__3; lean_object* l_Lean_Meta_getElimInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_filterMap___at_Lean_resolveGlobalConst___spec__1(lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__2; lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Tactic_getMainTarget___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__1; lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Tactic_adaptExpander___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__2(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_evalCases___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_Tactic_evalTacticAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__5___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -136,7 +134,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getBindingName___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases___closed__3; -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__2; lean_object* l_Lean_Elab_InfoTree_substitute(lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_withMainContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__2___closed__2; @@ -146,7 +143,6 @@ static lean_object* l_Lean_Elab_Tactic_getInductiveValFromMajor___lambda__1___cl static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___lambda__2___closed__2; lean_object* l_Lean_assignExprMVar___at_Lean_Elab_Tactic_closeMainGoal___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__5___lambda__1___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___closed__2; static lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__2___closed__2; @@ -204,7 +200,6 @@ static lean_object* l_panic___at_Lean_Elab_Tactic_ElimApp_reorderAlts___spec__1_ lean_object* l_Lean_assignExprMVar___at_Lean_Meta_getLevel___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandCases_x3f(lean_object*); -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltRHS___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__5___lambda__2___boxed(lean_object**); @@ -245,7 +240,6 @@ static lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Tactic_Ind static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__8___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2(lean_object*, lean_object*, size_t, size_t); static lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__14___closed__2; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -268,6 +262,7 @@ LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at___private_Lean_Elab_ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__1___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeVars___spec__2___boxed(lean_object*, lean_object*, lean_object*, 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_replaceRef(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkGeneralizationForbiddenSet(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___closed__1; @@ -276,7 +271,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getUserGeneralizingFVarIds___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_addNewArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getUnsolvedGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_State_targetPos___default; @@ -287,8 +281,9 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalA LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__5___boxed(lean_object**); static lean_object* l_Lean_Elab_Tactic_ElimApp_State_alts___default___closed__1; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___lambda__1___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_Tactic_expandTacticMacroFns_loop___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_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getFType___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -305,6 +300,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__1___boxed(le lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__5___lambda__2___closed__8; lean_object* l_Std_RBNode_insert___at_Lean_Meta_ToHide_moveToHiddeProp___spec__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandInductionAlts_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalAlt___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -323,10 +319,11 @@ lean_object* l_Lean_Meta_isExprDefEqGuarded(lean_object*, lean_object*, lean_obj lean_object* l_Lean_Meta_setMVarKind(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction_declRange___closed__3; lean_object* l_Lean_Expr_sort___override(lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalCases_declRange(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getUserGeneralizingFVarIds___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltRHS(lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_reorderAlts(lean_object*, lean_object*); @@ -350,6 +347,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__2___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandMultiAlt_x3f(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getUserGeneralizingFVarIds___closed__2; @@ -378,13 +376,13 @@ size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getFirstAltLhs(lean_object*); extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___closed__1; -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getBindingName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalInduction___lambda__3___boxed(lean_object**); lean_object* l_Lean_Elab_Term_mkConst(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_reorderAlts___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_isHoleRHS___closed__3; @@ -411,14 +409,11 @@ lean_object* l_List_redLength___rarg(lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedMVarId; -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__3; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_Meta_getFVarSetToGeneralize(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getNumArgs(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabCasesTargets___lambda__1(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -431,6 +426,7 @@ static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltVars___boxed(lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__1; uint8_t l_Lean_Syntax_hasArgs(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltsOfOptInductionAlts___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -466,6 +462,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac lean_object* l_Lean_Meta_getCustomEliminator_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_expandInduction_x3f(lean_object*); +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*); lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_generalizeTargets___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -485,7 +482,6 @@ lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMe LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_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_object* l_Lean_Expr_app___override(lean_object*, lean_object*); @@ -521,10 +517,10 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Tactic_ static lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_elabCasesTargets___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabCasesTargets___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___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_evalInduction___closed__8; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalCases___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_ElimApp_mkElimApp___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_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_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_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalInduction_checkTargets___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_generalizeTargetsEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -547,7 +543,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ContextInfo_save___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_isHoleRHS___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getAltsOfInductionAlts(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction___closed__1; @@ -580,6 +575,9 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_ElimApp_evalAlts_go___spec__5___lambda__1___closed__2; lean_object* l_List_toString___at_Lean_resolveGlobalConstNoOverloadCore___spec__2(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalInduction___closed__2; +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__2; +lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___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___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__2___closed__3; static lean_object* l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___spec__3___closed__2; @@ -2175,7 +2173,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__2_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__2___closed__1; x_2 = l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___lambda__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4015,69 +4013,7 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; -x_12 = !lean_is_exclusive(x_9); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_9, 5); -x_14 = l_Lean_replaceRef(x_1, x_13); -lean_dec(x_13); -lean_ctor_set(x_9, 5, x_14); -x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_16 = lean_ctor_get(x_9, 0); -x_17 = lean_ctor_get(x_9, 1); -x_18 = lean_ctor_get(x_9, 2); -x_19 = lean_ctor_get(x_9, 3); -x_20 = lean_ctor_get(x_9, 4); -x_21 = lean_ctor_get(x_9, 5); -x_22 = lean_ctor_get(x_9, 6); -x_23 = lean_ctor_get(x_9, 7); -x_24 = lean_ctor_get(x_9, 8); -x_25 = lean_ctor_get(x_9, 9); -x_26 = lean_ctor_get(x_9, 10); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -lean_inc(x_20); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_9); -x_27 = l_Lean_replaceRef(x_1, x_21); -lean_dec(x_21); -x_28 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_28, 0, x_16); -lean_ctor_set(x_28, 1, x_17); -lean_ctor_set(x_28, 2, x_18); -lean_ctor_set(x_28, 3, x_19); -lean_ctor_set(x_28, 4, x_20); -lean_ctor_set(x_28, 5, x_27); -lean_ctor_set(x_28, 6, x_22); -lean_ctor_set(x_28, 7, x_23); -lean_ctor_set(x_28, 8, x_24); -lean_ctor_set(x_28, 9, x_25); -lean_ctor_set(x_28, 10, x_26); -x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); -lean_dec(x_28); -return x_29; -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { _start: { uint8_t x_5; @@ -4114,7 +4050,7 @@ return x_13; } } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__1() { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -4122,16 +4058,16 @@ x_1 = lean_mk_string_from_bytes("invalid alternative name '", 26); return x_1; } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__2() { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__1; +x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__3() { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -4141,7 +4077,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; lean_object* x_15; uint8_t x_27; @@ -4179,7 +4115,7 @@ size_t x_34; size_t x_35; uint8_t x_36; x_34 = 0; x_35 = lean_usize_of_nat(x_28); lean_dec(x_28); -x_36 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2(x_14, x_3, x_34, x_35); +x_36 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(x_14, x_3, x_34, x_35); if (x_36 == 0) { lean_object* x_37; @@ -4191,8 +4127,16 @@ else { lean_object* x_38; lean_object* x_39; lean_dec(x_14); +lean_dec(x_12); lean_dec(x_11); -x_38 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__3; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_38 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__3; x_39 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_39, 0, x_38); lean_ctor_set(x_39, 1, x_13); @@ -4205,8 +4149,16 @@ else { lean_object* x_40; lean_object* x_41; lean_dec(x_14); +lean_dec(x_12); lean_dec(x_11); -x_40 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__3; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_40 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__3; x_41 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_41, 0, x_40); lean_ctor_set(x_41, 1, x_13); @@ -4218,7 +4170,7 @@ lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean lean_dec(x_15); x_16 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_16, 0, x_14); -x_17 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__2; +x_17 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__2; x_18 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_18, 0, x_17); lean_ctor_set(x_18, 1, x_16); @@ -4226,7 +4178,7 @@ x_19 = l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___closed__4; x_20 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(x_1, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_21 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___spec__1(x_1, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); x_22 = !lean_is_exclusive(x_21); if (x_22 == 0) { @@ -4248,7 +4200,7 @@ return x_25; } } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__1() { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__1() { _start: { lean_object* x_1; @@ -4256,16 +4208,16 @@ x_1 = lean_mk_string_from_bytes("invalid occurrence of wildcard alternative, it return x_1; } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__2() { +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__1; +x_1 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { uint8_t x_18; @@ -4309,9 +4261,15 @@ if (x_27 == 0) { lean_object* x_28; lean_object* x_29; x_28 = lean_box(0); +lean_inc(x_16); lean_inc(x_15); -x_29 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1(x_24, x_26, x_1, x_28, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_24); +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_29 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1(x_24, x_26, x_1, x_28, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); if (lean_obj_tag(x_29) == 0) { lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; @@ -4335,7 +4293,14 @@ else { uint8_t x_35; lean_dec(x_22); +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_5); x_35 = !lean_is_exclusive(x_29); if (x_35 == 0) @@ -4377,9 +4342,16 @@ x_43 = l_Lean_replaceRef(x_24, x_42); lean_dec(x_42); lean_dec(x_24); lean_ctor_set(x_15, 5, x_43); -x_44 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__2; -x_45 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_44, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_44 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__2; +x_45 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_44, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_16); lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); x_46 = !lean_is_exclusive(x_45); if (x_46 == 0) { @@ -4440,9 +4412,16 @@ lean_ctor_set(x_62, 7, x_57); lean_ctor_set(x_62, 8, x_58); lean_ctor_set(x_62, 9, x_59); lean_ctor_set(x_62, 10, x_60); -x_63 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__2; -x_64 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_63, x_9, x_10, x_11, x_12, x_13, x_14, x_62, x_16, x_17); +x_63 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__2; +x_64 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_63, x_9, x_10, x_11, x_12, x_13, x_14, x_62, x_16, x_17); +lean_dec(x_16); lean_dec(x_62); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); x_65 = lean_ctor_get(x_64, 0); lean_inc(x_65); x_66 = lean_ctor_get(x_64, 1); @@ -4469,9 +4448,15 @@ else { lean_object* x_69; lean_object* x_70; x_69 = lean_box(0); +lean_inc(x_16); lean_inc(x_15); -x_70 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1(x_24, x_26, x_1, x_69, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_24); +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_70 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1(x_24, x_26, x_1, x_69, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); if (lean_obj_tag(x_70) == 0) { lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; @@ -4495,7 +4480,14 @@ else { uint8_t x_76; lean_dec(x_22); +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_5); x_76 = !lean_is_exclusive(x_70); if (x_76 == 0) @@ -4523,7 +4515,14 @@ return x_79; else { lean_object* x_84; +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_5); lean_dec(x_4); x_84 = lean_alloc_ctor(0, 2, 0); @@ -4535,7 +4534,14 @@ return x_84; else { lean_object* x_85; +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_5); lean_dec(x_4); x_85 = lean_alloc_ctor(0, 2, 0); @@ -4554,7 +4560,7 @@ x_13 = lean_unsigned_to_nat(0u); x_14 = lean_unsigned_to_nat(1u); x_15 = lean_box(0); lean_inc(x_12); -x_16 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3(x_1, x_2, x_12, x_12, x_13, x_12, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_16 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2(x_1, x_2, x_12, x_12, x_13, x_12, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_12); if (lean_obj_tag(x_16) == 0) { @@ -4604,23 +4610,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; @@ -4628,33 +4618,25 @@ x_5 = lean_unbox_usize(x_3); lean_dec(x_3); x_6 = lean_unbox_usize(x_4); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2(x_1, x_2, x_5, x_6); +x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(x_1, x_2, x_5, x_6); lean_dec(x_2); lean_dec(x_1); x_8 = lean_box(x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; -x_14 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +x_14 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); return x_14; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -4675,14 +4657,7 @@ lean_object* x_17 = _args[16]; _start: { lean_object* x_18; -x_18 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_16); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +x_18 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); @@ -4696,13 +4671,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tac { lean_object* x_12; x_12 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_12; @@ -6284,7 +6252,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -6337,7 +6305,7 @@ lean_inc(x_29); x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); lean_dec(x_28); -x_31 = lean_ctor_get(x_29, 4); +x_31 = lean_ctor_get(x_29, 5); lean_inc(x_31); lean_dec(x_29); x_32 = lean_ctor_get(x_31, 1); @@ -6362,7 +6330,7 @@ lean_dec(x_36); x_38 = lean_st_ref_take(x_5, x_37); x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); -x_40 = lean_ctor_get(x_39, 4); +x_40 = lean_ctor_get(x_39, 5); lean_inc(x_40); x_41 = lean_ctor_get(x_38, 1); lean_inc(x_41); @@ -6371,7 +6339,7 @@ x_42 = !lean_is_exclusive(x_39); if (x_42 == 0) { lean_object* x_43; uint8_t x_44; -x_43 = lean_ctor_get(x_39, 4); +x_43 = lean_ctor_get(x_39, 5); lean_dec(x_43); x_44 = !lean_is_exclusive(x_40); if (x_44 == 0) @@ -6416,7 +6384,7 @@ x_55 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_55, 0, x_53); lean_ctor_set(x_55, 1, x_54); lean_ctor_set_uint8(x_55, sizeof(void*)*2, x_52); -lean_ctor_set(x_39, 4, x_55); +lean_ctor_set(x_39, 5, x_55); x_56 = lean_st_ref_set(x_5, x_39, x_41); lean_dec(x_5); x_57 = lean_ctor_get(x_56, 1); @@ -6441,245 +6409,251 @@ return x_59; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; x_60 = lean_ctor_get(x_39, 0); x_61 = lean_ctor_get(x_39, 1); x_62 = lean_ctor_get(x_39, 2); x_63 = lean_ctor_get(x_39, 3); +x_64 = lean_ctor_get(x_39, 4); +lean_inc(x_64); lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_dec(x_39); -x_64 = lean_ctor_get_uint8(x_40, sizeof(void*)*2); -x_65 = lean_ctor_get(x_40, 0); -lean_inc(x_65); +x_65 = lean_ctor_get_uint8(x_40, sizeof(void*)*2); +x_66 = lean_ctor_get(x_40, 0); +lean_inc(x_66); if (lean_is_exclusive(x_40)) { lean_ctor_release(x_40, 0); lean_ctor_release(x_40, 1); - x_66 = x_40; + x_67 = x_40; } else { lean_dec_ref(x_40); - x_66 = lean_box(0); + x_67 = lean_box(0); } -x_67 = l_Std_PersistentArray_append___rarg(x_21, x_34); -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 2, 1); +x_68 = l_Std_PersistentArray_append___rarg(x_21, x_34); +if (lean_is_scalar(x_67)) { + x_69 = lean_alloc_ctor(0, 2, 1); } else { - x_68 = x_66; + x_69 = x_67; } -lean_ctor_set(x_68, 0, x_65); -lean_ctor_set(x_68, 1, x_67); -lean_ctor_set_uint8(x_68, sizeof(void*)*2, x_64); -x_69 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_69, 0, x_60); -lean_ctor_set(x_69, 1, x_61); -lean_ctor_set(x_69, 2, x_62); -lean_ctor_set(x_69, 3, x_63); -lean_ctor_set(x_69, 4, x_68); -x_70 = lean_st_ref_set(x_5, x_69, x_41); +lean_ctor_set(x_69, 0, x_66); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_65); +x_70 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_70, 0, x_60); +lean_ctor_set(x_70, 1, x_61); +lean_ctor_set(x_70, 2, x_62); +lean_ctor_set(x_70, 3, x_63); +lean_ctor_set(x_70, 4, x_64); +lean_ctor_set(x_70, 5, x_69); +x_71 = lean_st_ref_set(x_5, x_70, x_41); lean_dec(x_5); -x_71 = lean_ctor_get(x_70, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - x_72 = x_70; +x_72 = lean_ctor_get(x_71, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_73 = x_71; } else { - lean_dec_ref(x_70); - x_72 = lean_box(0); + lean_dec_ref(x_71); + x_73 = lean_box(0); } -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_73)) { + x_74 = lean_alloc_ctor(0, 2, 0); } else { - x_73 = x_72; + x_74 = x_73; } -lean_ctor_set(x_73, 0, x_24); -lean_ctor_set(x_73, 1, x_71); -return x_73; +lean_ctor_set(x_74, 0, x_24); +lean_ctor_set(x_74, 1, x_72); +return x_74; } } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; -x_74 = lean_ctor_get(x_23, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_23, 1); +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; uint8_t x_93; +x_75 = lean_ctor_get(x_23, 0); lean_inc(x_75); +x_76 = lean_ctor_get(x_23, 1); +lean_inc(x_76); lean_dec(x_23); -x_76 = lean_st_ref_get(x_9, x_75); -x_77 = lean_ctor_get(x_76, 1); -lean_inc(x_77); -lean_dec(x_76); -x_78 = lean_st_ref_get(x_5, x_77); -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); +x_77 = lean_st_ref_get(x_9, x_76); +x_78 = lean_ctor_get(x_77, 1); +lean_inc(x_78); +lean_dec(x_77); +x_79 = lean_st_ref_get(x_5, x_78); +x_80 = lean_ctor_get(x_79, 0); lean_inc(x_80); -lean_dec(x_78); -x_81 = lean_ctor_get(x_79, 4); +x_81 = lean_ctor_get(x_79, 1); lean_inc(x_81); lean_dec(x_79); -x_82 = lean_ctor_get(x_81, 1); +x_82 = lean_ctor_get(x_80, 5); lean_inc(x_82); -x_83 = l_Std_PersistentArray_mapM___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__10(x_81, x_82, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_80); +lean_dec(x_80); +x_83 = lean_ctor_get(x_82, 1); +lean_inc(x_83); +x_84 = l_Std_PersistentArray_mapM___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__10(x_82, x_83, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_81); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); +x_85 = lean_ctor_get(x_84, 0); lean_inc(x_85); -lean_dec(x_83); -x_86 = lean_st_ref_get(x_9, x_85); +x_86 = lean_ctor_get(x_84, 1); +lean_inc(x_86); +lean_dec(x_84); +x_87 = lean_st_ref_get(x_9, x_86); lean_dec(x_9); -x_87 = lean_ctor_get(x_86, 1); -lean_inc(x_87); -lean_dec(x_86); -x_88 = lean_st_ref_take(x_5, x_87); -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_89, 4); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); +x_89 = lean_st_ref_take(x_5, x_88); +x_90 = lean_ctor_get(x_89, 0); lean_inc(x_90); -x_91 = lean_ctor_get(x_88, 1); +x_91 = lean_ctor_get(x_90, 5); lean_inc(x_91); -lean_dec(x_88); -x_92 = !lean_is_exclusive(x_89); -if (x_92 == 0) -{ -lean_object* x_93; uint8_t x_94; -x_93 = lean_ctor_get(x_89, 4); -lean_dec(x_93); -x_94 = !lean_is_exclusive(x_90); -if (x_94 == 0) -{ -lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; -x_95 = lean_ctor_get(x_90, 1); -lean_dec(x_95); -x_96 = l_Std_PersistentArray_append___rarg(x_21, x_84); -lean_ctor_set(x_90, 1, x_96); -x_97 = lean_st_ref_set(x_5, x_89, x_91); +x_92 = lean_ctor_get(x_89, 1); +lean_inc(x_92); +lean_dec(x_89); +x_93 = !lean_is_exclusive(x_90); +if (x_93 == 0) +{ +lean_object* x_94; uint8_t x_95; +x_94 = lean_ctor_get(x_90, 5); +lean_dec(x_94); +x_95 = !lean_is_exclusive(x_91); +if (x_95 == 0) +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; +x_96 = lean_ctor_get(x_91, 1); +lean_dec(x_96); +x_97 = l_Std_PersistentArray_append___rarg(x_21, x_85); +lean_ctor_set(x_91, 1, x_97); +x_98 = lean_st_ref_set(x_5, x_90, x_92); lean_dec(x_5); -x_98 = !lean_is_exclusive(x_97); -if (x_98 == 0) +x_99 = !lean_is_exclusive(x_98); +if (x_99 == 0) { -lean_object* x_99; -x_99 = lean_ctor_get(x_97, 0); -lean_dec(x_99); -lean_ctor_set_tag(x_97, 1); -lean_ctor_set(x_97, 0, x_74); -return x_97; +lean_object* x_100; +x_100 = lean_ctor_get(x_98, 0); +lean_dec(x_100); +lean_ctor_set_tag(x_98, 1); +lean_ctor_set(x_98, 0, x_75); +return x_98; } else { -lean_object* x_100; lean_object* x_101; -x_100 = lean_ctor_get(x_97, 1); -lean_inc(x_100); -lean_dec(x_97); -x_101 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_101, 0, x_74); -lean_ctor_set(x_101, 1, x_100); -return x_101; +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_98, 1); +lean_inc(x_101); +lean_dec(x_98); +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_75); +lean_ctor_set(x_102, 1, x_101); +return x_102; } } else { -uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_102 = lean_ctor_get_uint8(x_90, sizeof(void*)*2); -x_103 = lean_ctor_get(x_90, 0); -lean_inc(x_103); -lean_dec(x_90); -x_104 = l_Std_PersistentArray_append___rarg(x_21, x_84); -x_105 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set_uint8(x_105, sizeof(void*)*2, x_102); -lean_ctor_set(x_89, 4, x_105); -x_106 = lean_st_ref_set(x_5, x_89, x_91); +uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_103 = lean_ctor_get_uint8(x_91, sizeof(void*)*2); +x_104 = lean_ctor_get(x_91, 0); +lean_inc(x_104); +lean_dec(x_91); +x_105 = l_Std_PersistentArray_append___rarg(x_21, x_85); +x_106 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_106, 0, x_104); +lean_ctor_set(x_106, 1, x_105); +lean_ctor_set_uint8(x_106, sizeof(void*)*2, x_103); +lean_ctor_set(x_90, 5, x_106); +x_107 = lean_st_ref_set(x_5, x_90, x_92); lean_dec(x_5); -x_107 = lean_ctor_get(x_106, 1); -lean_inc(x_107); -if (lean_is_exclusive(x_106)) { - lean_ctor_release(x_106, 0); - lean_ctor_release(x_106, 1); - x_108 = x_106; +x_108 = lean_ctor_get(x_107, 1); +lean_inc(x_108); +if (lean_is_exclusive(x_107)) { + lean_ctor_release(x_107, 0); + lean_ctor_release(x_107, 1); + x_109 = x_107; } else { - lean_dec_ref(x_106); - x_108 = lean_box(0); + lean_dec_ref(x_107); + x_109 = lean_box(0); } -if (lean_is_scalar(x_108)) { - x_109 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_109)) { + x_110 = lean_alloc_ctor(1, 2, 0); } else { - x_109 = x_108; - lean_ctor_set_tag(x_109, 1); + x_110 = x_109; + lean_ctor_set_tag(x_110, 1); } -lean_ctor_set(x_109, 0, x_74); -lean_ctor_set(x_109, 1, x_107); -return x_109; +lean_ctor_set(x_110, 0, x_75); +lean_ctor_set(x_110, 1, x_108); +return x_110; } } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_110 = lean_ctor_get(x_89, 0); -x_111 = lean_ctor_get(x_89, 1); -x_112 = lean_ctor_get(x_89, 2); -x_113 = lean_ctor_get(x_89, 3); +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_111 = lean_ctor_get(x_90, 0); +x_112 = lean_ctor_get(x_90, 1); +x_113 = lean_ctor_get(x_90, 2); +x_114 = lean_ctor_get(x_90, 3); +x_115 = lean_ctor_get(x_90, 4); +lean_inc(x_115); +lean_inc(x_114); lean_inc(x_113); lean_inc(x_112); lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_89); -x_114 = lean_ctor_get_uint8(x_90, sizeof(void*)*2); -x_115 = lean_ctor_get(x_90, 0); -lean_inc(x_115); -if (lean_is_exclusive(x_90)) { - lean_ctor_release(x_90, 0); - lean_ctor_release(x_90, 1); - x_116 = x_90; +lean_dec(x_90); +x_116 = lean_ctor_get_uint8(x_91, sizeof(void*)*2); +x_117 = lean_ctor_get(x_91, 0); +lean_inc(x_117); +if (lean_is_exclusive(x_91)) { + lean_ctor_release(x_91, 0); + lean_ctor_release(x_91, 1); + x_118 = x_91; } else { - lean_dec_ref(x_90); - x_116 = lean_box(0); + lean_dec_ref(x_91); + x_118 = lean_box(0); } -x_117 = l_Std_PersistentArray_append___rarg(x_21, x_84); -if (lean_is_scalar(x_116)) { - x_118 = lean_alloc_ctor(0, 2, 1); +x_119 = l_Std_PersistentArray_append___rarg(x_21, x_85); +if (lean_is_scalar(x_118)) { + x_120 = lean_alloc_ctor(0, 2, 1); } else { - x_118 = x_116; -} -lean_ctor_set(x_118, 0, x_115); -lean_ctor_set(x_118, 1, x_117); -lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); -x_119 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_119, 0, x_110); -lean_ctor_set(x_119, 1, x_111); -lean_ctor_set(x_119, 2, x_112); -lean_ctor_set(x_119, 3, x_113); -lean_ctor_set(x_119, 4, x_118); -x_120 = lean_st_ref_set(x_5, x_119, x_91); + x_120 = x_118; +} +lean_ctor_set(x_120, 0, x_117); +lean_ctor_set(x_120, 1, x_119); +lean_ctor_set_uint8(x_120, sizeof(void*)*2, x_116); +x_121 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_121, 0, x_111); +lean_ctor_set(x_121, 1, x_112); +lean_ctor_set(x_121, 2, x_113); +lean_ctor_set(x_121, 3, x_114); +lean_ctor_set(x_121, 4, x_115); +lean_ctor_set(x_121, 5, x_120); +x_122 = lean_st_ref_set(x_5, x_121, x_92); lean_dec(x_5); -x_121 = lean_ctor_get(x_120, 1); -lean_inc(x_121); -if (lean_is_exclusive(x_120)) { - lean_ctor_release(x_120, 0); - lean_ctor_release(x_120, 1); - x_122 = x_120; +x_123 = lean_ctor_get(x_122, 1); +lean_inc(x_123); +if (lean_is_exclusive(x_122)) { + lean_ctor_release(x_122, 0); + lean_ctor_release(x_122, 1); + x_124 = x_122; } else { - lean_dec_ref(x_120); - x_122 = lean_box(0); + lean_dec_ref(x_122); + x_124 = lean_box(0); } -if (lean_is_scalar(x_122)) { - x_123 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_124)) { + x_125 = lean_alloc_ctor(1, 2, 0); } else { - x_123 = x_122; - lean_ctor_set_tag(x_123, 1); + x_125 = x_124; + lean_ctor_set_tag(x_125, 1); } -lean_ctor_set(x_123, 0, x_74); -lean_ctor_set(x_123, 1, x_121); -return x_123; +lean_ctor_set(x_125, 0, x_75); +lean_ctor_set(x_125, 1, x_123); +return x_125; } } } @@ -12034,7 +12008,14 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_ElimApp_evalAlts(lean_object* x_1, l _start: { lean_object* x_18; +lean_inc(x_16); lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); x_18 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames(x_2, x_4, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); if (lean_obj_tag(x_18) == 0) { @@ -12066,7 +12047,7 @@ lean_closure_set(x_24, 5, x_7); lean_closure_set(x_24, 6, x_8); x_25 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_ElimApp_evalAlts___lambda__1___boxed), 11, 1); lean_closure_set(x_25, 0, x_5); -x_26 = l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(x_24, x_25, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_19); +x_26 = l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(x_24, x_25, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_19); return x_26; } } @@ -12236,7 +12217,7 @@ lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint x_37 = lean_ctor_get(x_31, 1); lean_inc(x_37); lean_dec(x_31); -x_38 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_37); +x_38 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_37); x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); x_40 = lean_ctor_get(x_38, 1); @@ -12271,7 +12252,7 @@ lean_ctor_set(x_24, 1, x_22); x_25 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_23); -x_26 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3(x_17, x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +x_26 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3(x_17, x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_19); x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); @@ -12351,7 +12332,7 @@ lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint x_75 = lean_ctor_get(x_69, 1); lean_inc(x_75); lean_dec(x_69); -x_76 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(x_55, x_2, x_3, x_4, x_5, x_6, x_7, x_54, x_9, x_75); +x_76 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(x_55, x_2, x_3, x_4, x_5, x_6, x_7, x_54, x_9, x_75); x_77 = lean_ctor_get(x_76, 0); lean_inc(x_77); x_78 = lean_ctor_get(x_76, 1); @@ -12386,7 +12367,7 @@ lean_ctor_set(x_62, 1, x_60); x_63 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_63, 0, x_62); lean_ctor_set(x_63, 1, x_61); -x_64 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3(x_55, x_63, x_2, x_3, x_4, x_5, x_6, x_7, x_54, x_9, x_57); +x_64 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3(x_55, x_63, x_2, x_3, x_4, x_5, x_6, x_7, x_54, x_9, x_57); x_65 = lean_ctor_get(x_64, 0); lean_inc(x_65); x_66 = lean_ctor_get(x_64, 1); @@ -12508,7 +12489,7 @@ x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lea x_21 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_21, 0, x_19); lean_ctor_set(x_21, 1, x_20); -x_22 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_22 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); x_23 = !lean_is_exclusive(x_22); if (x_23 == 0) { @@ -12626,7 +12607,7 @@ x_36 = l_Lean_Elab_Tactic_ElimApp_setMotiveArg___closed__6; x_37 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_37, 0, x_35); lean_ctor_set(x_37, 1, x_36); -x_38 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_37, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_38 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_37, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); x_39 = !lean_is_exclusive(x_38); if (x_39 == 0) { @@ -12728,7 +12709,7 @@ x_35 = l_Lean_Elab_Tactic_ElimApp_setMotiveArg___closed__6; x_36 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_36, 0, x_34); lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_36, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_37 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_36, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); x_38 = !lean_is_exclusive(x_37); if (x_38 == 0) { @@ -13686,6 +13667,7 @@ x_13 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lea if (x_2 == 0) { lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_1); x_14 = lean_box(0); x_15 = lean_box(x_2); x_16 = lean_apply_11(x_13, x_15, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); @@ -13695,14 +13677,7 @@ else { lean_object* x_17; lean_object* x_18; uint8_t x_19; x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___lambda__2___closed__3; -x_18 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +x_18 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___spec__1(x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); x_19 = !lean_is_exclusive(x_18); if (x_19 == 0) { @@ -13791,15 +13766,7 @@ if (x_25 == 0) { lean_object* x_26; lean_object* x_27; uint8_t x_28; x_26 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___closed__2; -x_27 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__1(x_17, x_26, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_17); +x_27 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___spec__1(x_17, x_26, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); x_28 = !lean_is_exclusive(x_27); if (x_28 == 0) { @@ -13832,7 +13799,6 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___lambda__2(x_17, x_4, x_32, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_17); if (lean_obj_tag(x_33) == 0) { lean_object* x_34; @@ -14044,7 +14010,6 @@ x_13 = lean_unbox(x_2); lean_dec(x_2); x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_checkAltsOfOptInductionAlts___spec__1___lambda__2(x_1, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_3); -lean_dec(x_1); return x_14; } } @@ -14597,7 +14562,7 @@ x_16 = l_Lean_Elab_Tactic_ElimApp_mkElimApp_loop___closed__4; x_17 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_18; } } @@ -15308,7 +15273,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -15353,7 +15318,7 @@ lean_dec(x_24); x_26 = lean_st_ref_take(x_5, x_25); x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -x_28 = lean_ctor_get(x_27, 4); +x_28 = lean_ctor_get(x_27, 5); lean_inc(x_28); x_29 = lean_ctor_get(x_26, 1); lean_inc(x_29); @@ -15362,7 +15327,7 @@ x_30 = !lean_is_exclusive(x_27); if (x_30 == 0) { lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_27, 4); +x_31 = lean_ctor_get(x_27, 5); lean_dec(x_31); x_32 = !lean_is_exclusive(x_28); if (x_32 == 0) @@ -15409,7 +15374,7 @@ x_46 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_46, 0, x_43); lean_ctor_set(x_46, 1, x_45); lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_42); -lean_ctor_set(x_27, 4, x_46); +lean_ctor_set(x_27, 5, x_46); x_47 = lean_st_ref_set(x_5, x_27, x_29); x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); @@ -15434,64 +15399,67 @@ return x_51; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; x_52 = lean_ctor_get(x_27, 0); x_53 = lean_ctor_get(x_27, 1); x_54 = lean_ctor_get(x_27, 2); x_55 = lean_ctor_get(x_27, 3); +x_56 = lean_ctor_get(x_27, 4); +lean_inc(x_56); lean_inc(x_55); lean_inc(x_54); lean_inc(x_53); lean_inc(x_52); lean_dec(x_27); -x_56 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); -x_57 = lean_ctor_get(x_28, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_28, 1); +x_57 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); +x_58 = lean_ctor_get(x_28, 0); lean_inc(x_58); +x_59 = lean_ctor_get(x_28, 1); +lean_inc(x_59); if (lean_is_exclusive(x_28)) { lean_ctor_release(x_28, 0); lean_ctor_release(x_28, 1); - x_59 = x_28; + x_60 = x_28; } else { lean_dec_ref(x_28); - x_59 = lean_box(0); + x_60 = lean_box(0); } -x_60 = l_Std_PersistentArray_push___rarg(x_58, x_1); -if (lean_is_scalar(x_59)) { - x_61 = lean_alloc_ctor(0, 2, 1); +x_61 = l_Std_PersistentArray_push___rarg(x_59, x_1); +if (lean_is_scalar(x_60)) { + x_62 = lean_alloc_ctor(0, 2, 1); } else { - x_61 = x_59; + x_62 = x_60; } -lean_ctor_set(x_61, 0, x_57); -lean_ctor_set(x_61, 1, x_60); -lean_ctor_set_uint8(x_61, sizeof(void*)*2, x_56); -x_62 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_62, 0, x_52); -lean_ctor_set(x_62, 1, x_53); -lean_ctor_set(x_62, 2, x_54); -lean_ctor_set(x_62, 3, x_55); -lean_ctor_set(x_62, 4, x_61); -x_63 = lean_st_ref_set(x_5, x_62, x_29); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; +lean_ctor_set(x_62, 0, x_58); +lean_ctor_set(x_62, 1, x_61); +lean_ctor_set_uint8(x_62, sizeof(void*)*2, x_57); +x_63 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_63, 0, x_52); +lean_ctor_set(x_63, 1, x_53); +lean_ctor_set(x_63, 2, x_54); +lean_ctor_set(x_63, 3, x_55); +lean_ctor_set(x_63, 4, x_56); +lean_ctor_set(x_63, 5, x_62); +x_64 = lean_st_ref_set(x_5, x_63, x_29); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_66 = x_64; } else { - lean_dec_ref(x_63); - x_65 = lean_box(0); + lean_dec_ref(x_64); + x_66 = lean_box(0); } -x_66 = lean_box(0); -if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 0); +x_67 = lean_box(0); +if (lean_is_scalar(x_66)) { + x_68 = lean_alloc_ctor(0, 2, 0); } else { - x_67 = x_65; + x_68 = x_66; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_64); -return x_67; +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_68, 1, x_65); +return x_68; } } } @@ -15543,7 +15511,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -15629,7 +15597,7 @@ lean_dec(x_15); x_17 = lean_st_ref_get(x_6, x_16); x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); -x_19 = lean_ctor_get(x_18, 4); +x_19 = lean_ctor_get(x_18, 5); lean_inc(x_19); lean_dec(x_18); x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*2); @@ -15915,7 +15883,7 @@ x_25 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInf x_26 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_26, 0, x_24); lean_ctor_set(x_26, 1, x_25); -x_27 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_27 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -16052,7 +16020,7 @@ x_33 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInf x_34 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_34, 0, x_32); lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_34, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_20); +x_35 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_34, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_20); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -16157,7 +16125,7 @@ if (x_15 == 0) lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_dec(x_2); x_16 = l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_getElimNameInfo___lambda__4___closed__2; -x_17 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_17 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -17305,7 +17273,7 @@ if (lean_obj_tag(x_10) == 0) { lean_object* x_11; lean_object* x_12; lean_dec(x_1); -x_11 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__3; +x_11 = l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__3; x_12 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_12, 0, x_11); lean_ctor_set(x_12, 1, x_8); @@ -17690,7 +17658,7 @@ lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean x_19 = lean_ctor_get(x_1, 0); lean_inc(x_19); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_19, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_19, x_20); x_22 = l_Lean_Elab_Tactic_evalInduction___lambda__1___closed__1; lean_inc(x_21); x_23 = lean_mk_array(x_21, x_22); @@ -18064,7 +18032,7 @@ lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint x_58 = lean_ctor_get(x_52, 1); lean_inc(x_58); lean_dec(x_52); -x_59 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__2(x_36, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_58); +x_59 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__2(x_36, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_58); x_60 = lean_ctor_get(x_59, 0); lean_inc(x_60); x_61 = lean_ctor_get(x_59, 1); @@ -18101,7 +18069,7 @@ x_45 = l_Lean_Elab_Tactic_ElimApp_setMotiveArg___closed__6; x_46 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_46, 0, x_44); lean_ctor_set(x_46, 1, x_45); -x_47 = l_Lean_addTrace___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__3(x_36, x_46, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_38); +x_47 = l_Lean_addTrace___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__3(x_36, x_46, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_38); x_48 = lean_ctor_get(x_47, 0); lean_inc(x_48); x_49 = lean_ctor_get(x_47, 1); @@ -18674,7 +18642,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); lean_ctor_set(x_5, 2, x_15); -x_16 = l_Lean_Elab_Tactic_evalTacticAux(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_16 = l_Lean_Elab_Tactic_evalTactic(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); return x_16; } else @@ -18729,7 +18697,7 @@ lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 4, x_28); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 5, x_29); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 6, x_30); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 7, x_32); -x_36 = l_Lean_Elab_Tactic_evalTacticAux(x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11); +x_36 = l_Lean_Elab_Tactic_evalTactic(x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11); return x_36; } } @@ -20486,7 +20454,7 @@ lean_dec(x_34); x_37 = lean_ctor_get(x_35, 0); lean_inc(x_37); x_38 = lean_unsigned_to_nat(0u); -x_39 = l_Lean_Expr_getAppNumArgsAux(x_37, x_38); +x_39 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_37, x_38); x_40 = l_Lean_Elab_Tactic_evalInduction___lambda__1___closed__1; lean_inc(x_39); x_41 = lean_mk_array(x_39, x_40); @@ -21517,16 +21485,16 @@ l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFiel lean_mark_persistent(l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___lambda__1___closed__2); l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___closed__1 = _init_l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_getAltNumFields___closed__1); -l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__1(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__1); -l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__2(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__2); -l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__3 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__3(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___lambda__1___closed__3); -l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__1(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__1); -l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__2(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__3___closed__2); +l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__1); +l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__2); +l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__3 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__3(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___lambda__1___closed__3); +l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__1); +l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_checkAltNames___spec__2___closed__2); l_Lean_Elab_ContextInfo_saveNoFileMap___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__4___rarg___closed__1 = _init_l_Lean_Elab_ContextInfo_saveNoFileMap___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__4___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_ContextInfo_saveNoFileMap___at___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___spec__4___rarg___closed__1); l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___boxed__const__1 = _init_l___private_Lean_Elab_Tactic_Induction_0__Lean_Elab_Tactic_ElimApp_saveAltVarsInfo___boxed__const__1(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Match.c b/stage0/stdlib/Lean/Elab/Tactic/Match.c index 18ec014417b2..3881b60dfdea 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Match.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Match.c @@ -40,12 +40,12 @@ extern lean_object* l_Lean_maxRecDepthErrorMessage; lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Tactic_adaptExpander___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Match_0__Lean_Elab_Tactic_mkAuxiliaryMatchTerm___spec__2___closed__8; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Match_0__Lean_Elab_Tactic_mkAuxiliaryMatchTerm___spec__2___closed__4; -lean_object* l_Lean_Elab_Tactic_evalTacticAux(lean_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_evalMatch___closed__4; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Match_0__Lean_Elab_Tactic_mkAuxiliaryMatchTerm___spec__1___closed__1; lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Match_0__Lean_Elab_Tactic_mkAuxiliaryMatchTerm___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Match_0__Lean_Elab_Tactic_mkAuxiliaryMatchTerm___spec__2___closed__6; +lean_object* l_Lean_Elab_Tactic_evalTactic(lean_object*, 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*); lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Tactic_evalMatch___spec__4___closed__1; @@ -100,12 +100,12 @@ uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Match_0__Lean_Elab_Tactic_mkAuxiliaryMatchTerm___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalMatch___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalMatch___closed__7; +lean_object* l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Match_0__Lean_Elab_Tactic_mkAuxiliaryMatchTerm___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalMatch___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Tactic_evalMatch___spec__6___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Match_0__Lean_Elab_Tactic_mkAuxiliaryMatchTerm___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalMatch___closed__1; -lean_object* l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at_Lean_Elab_Tactic_evalMatch___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalMatch___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_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); @@ -2516,7 +2516,7 @@ x_46 = lean_ctor_get(x_37, 1); lean_inc(x_46); lean_dec(x_37); x_47 = l_List_reverse___rarg(x_46); -x_48 = l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4(x_47, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); +x_48 = l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4(x_47, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -2575,7 +2575,7 @@ x_61 = lean_ctor_get(x_37, 1); lean_inc(x_61); lean_dec(x_37); x_62 = l_List_reverse___rarg(x_61); -x_63 = l_List_forM___at_Lean_Elab_Tactic_expandTacticMacroFns_loop___spec__4(x_62, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_60); +x_63 = l_List_forM___at_Lean_Elab_Tactic_evalTactic_expandEval___spec__4(x_62, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_60); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -2702,7 +2702,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); lean_ctor_set(x_5, 2, x_15); -x_16 = l_Lean_Elab_Tactic_evalTacticAux(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_16 = l_Lean_Elab_Tactic_evalTactic(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); return x_16; } else @@ -2757,7 +2757,7 @@ lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 4, x_28); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 5, x_29); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 6, x_30); lean_ctor_set_uint8(x_35, sizeof(void*)*8 + 7, x_32); -x_36 = l_Lean_Elab_Tactic_evalTacticAux(x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11); +x_36 = l_Lean_Elab_Tactic_evalTactic(x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11); return x_36; } } diff --git a/stage0/stdlib/Lean/Elab/Tactic/Meta.c b/stage0/stdlib/Lean/Elab/Tactic/Meta.c index 97000a441752..9205b9069f00 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Meta.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Meta.c @@ -25,10 +25,10 @@ lean_object* l_Lean_Elab_Tactic_pruneSolvedGoals(lean_object*, lean_object*, lea lean_object* lean_local_ctx_mk_let_decl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_Elab_runTactic___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___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_Elab_runTactic___spec__5___closed__1; -lean_object* l_Lean_Elab_Tactic_evalTacticAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_instantiateLCtxMVars___at_Lean_Elab_runTactic___spec__2___closed__3; +lean_object* l_Lean_Elab_Tactic_evalTactic(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_foldlM___at_Lean_Elab_runTactic___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_TermElabM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1344,7 +1344,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_11 = l_Lean_Elab_Tactic_evalTacticAux(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_Tactic_evalTactic(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; lean_object* x_13; diff --git a/stage0/stdlib/Lean/Elab/Tactic/Rewrite.c b/stage0/stdlib/Lean/Elab/Tactic/Rewrite.c index e705a24d3a4f..a660227340dd 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Rewrite.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Rewrite.c @@ -36,7 +36,7 @@ static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq_ 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*); lean_object* l_List_filterTRAux___at_Lean_resolveGlobalConstCore___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_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_SavedState_restore(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_SavedState_restore(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__1; lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___closed__2; @@ -112,7 +112,6 @@ static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq_ lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__2___closed__1; static lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_withRWRulesSeq___spec__2___closed__1; -lean_object* l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getMainTarget(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__2___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabRewriteConfig___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -120,7 +119,6 @@ static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabRewri 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___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Rewrite___hyg_956_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Term_runTactic___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_evalExpr_x27___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_withRWRulesSeq___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -129,7 +127,6 @@ LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at_Lean_Elab_Tactic_ela lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__11; -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabRewriteConfig___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabRewriteConfig___spec__12___at_Lean_Elab_Tactic_elabRewriteConfig___spec__13___closed__1; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); @@ -154,8 +151,10 @@ extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; static lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___lambda__2___closed__4; 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*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___closed__4; +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_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_object* l_ReaderT_pure___at_Lean_Elab_Tactic_saveTacticInfoForToken___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* 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*); 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_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___closed__8; lean_object* l_Lean_LocalDecl_type(lean_object*); @@ -185,6 +184,7 @@ static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabRewri lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, uint8_t, 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__2___closed__5; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq___closed__9; +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*); lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalRewriteSeq___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___regBuiltin_Lean_Elab_Tactic_evalRewriteSeq(lean_object*); @@ -990,7 +990,7 @@ x_18 = l_Lean_Elab_Tactic_withRWRulesSeq_go___closed__4; x_19 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); -x_20 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__2(x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_20 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic_throwExs___spec__2(x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -1048,16 +1048,17 @@ return x_29; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; +lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; x_30 = lean_ctor_get(x_29, 1); lean_inc(x_30); lean_dec(x_29); -x_31 = l_Lean_Elab_Tactic_SavedState_restore(x_27, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_30); -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -lean_dec(x_31); +x_31 = 0; +x_32 = l_Lean_Elab_Tactic_SavedState_restore(x_27, x_31, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_30); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); x_5 = x_22; -x_14 = x_32; +x_14 = x_33; goto _start; } } @@ -1268,7 +1269,7 @@ x_16 = l_Lean_Elab_Tactic_withRWRulesSeq_go___closed__4; x_17 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_18; } } @@ -2009,59 +2010,60 @@ return x_35; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_dec(x_25); x_36 = lean_ctor_get(x_32, 1); lean_inc(x_36); lean_dec(x_32); -x_37 = l_Lean_Elab_Tactic_SavedState_restore(x_30, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_36); -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_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_38); -if (lean_obj_tag(x_40) == 0) +x_37 = 0; +x_38 = l_Lean_Elab_Tactic_SavedState_restore(x_30, x_37, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_36); +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +lean_dec(x_38); +x_40 = lean_box(x_5); +x_41 = lean_apply_11(x_4, x_40, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_39); +if (lean_obj_tag(x_41) == 0) { -uint8_t x_41; -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) +uint8_t x_42; +x_42 = !lean_is_exclusive(x_41); +if (x_42 == 0) { -return x_40; +return x_41; } 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_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_41, 0); +x_44 = lean_ctor_get(x_41, 1); +lean_inc(x_44); lean_inc(x_43); -lean_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_dec(x_41); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } else { -uint8_t x_45; -x_45 = !lean_is_exclusive(x_40); -if (x_45 == 0) +uint8_t x_46; +x_46 = !lean_is_exclusive(x_41); +if (x_46 == 0) { -return x_40; +return x_41; } 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_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_41, 0); +x_48 = lean_ctor_get(x_41, 1); +lean_inc(x_48); lean_inc(x_47); -lean_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_dec(x_41); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; } } } @@ -2070,14 +2072,14 @@ return x_48; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_dec(x_7); -x_49 = l_Lean_Elab_Tactic_saveState___rarg(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); +x_50 = l_Lean_Elab_Tactic_saveState___rarg(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_51 = lean_ctor_get(x_50, 0); lean_inc(x_51); -lean_dec(x_49); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -2087,74 +2089,75 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_3); -x_52 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_3, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_51); -if (lean_obj_tag(x_52) == 0) +x_53 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_3, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_52); +if (lean_obj_tag(x_53) == 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_object* x_54; lean_object* x_55; lean_object* x_56; +lean_dec(x_51); +x_54 = lean_ctor_get(x_53, 0); lean_inc(x_54); -lean_dec(x_52); -x_55 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_4, x_5, x_6, x_3, x_53, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_54); -return x_55; +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +lean_dec(x_53); +x_56 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_4, x_5, x_6, x_3, x_54, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_55); +return x_56; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_dec(x_3); -x_56 = lean_ctor_get(x_52, 1); -lean_inc(x_56); -lean_dec(x_52); -x_57 = l_Lean_Elab_Tactic_SavedState_restore(x_50, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_56); -x_58 = lean_ctor_get(x_57, 1); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_box(x_5); -x_60 = lean_apply_11(x_4, x_59, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_58); -if (lean_obj_tag(x_60) == 0) +x_57 = lean_ctor_get(x_53, 1); +lean_inc(x_57); +lean_dec(x_53); +x_58 = 0; +x_59 = l_Lean_Elab_Tactic_SavedState_restore(x_51, x_58, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_57); +x_60 = lean_ctor_get(x_59, 1); +lean_inc(x_60); +lean_dec(x_59); +x_61 = lean_box(x_5); +x_62 = lean_apply_11(x_4, x_61, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_60); +if (lean_obj_tag(x_62) == 0) { -uint8_t x_61; -x_61 = !lean_is_exclusive(x_60); -if (x_61 == 0) +uint8_t x_63; +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) { -return x_60; +return x_62; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_60, 0); -x_63 = lean_ctor_get(x_60, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_60); -x_64 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set(x_64, 1, x_63); -return x_64; +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_62, 0); +x_65 = lean_ctor_get(x_62, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_62); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +return x_66; } } else { -uint8_t x_65; -x_65 = !lean_is_exclusive(x_60); -if (x_65 == 0) +uint8_t x_67; +x_67 = !lean_is_exclusive(x_62); +if (x_67 == 0) { -return x_60; +return x_62; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_60, 0); -x_67 = lean_ctor_get(x_60, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_60); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_62, 0); +x_69 = lean_ctor_get(x_62, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_62); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; } } } @@ -2162,18 +2165,20 @@ return x_68; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_69 = lean_ctor_get(x_14, 0); -x_70 = lean_ctor_get(x_14, 1); -x_71 = lean_ctor_get(x_14, 2); -x_72 = lean_ctor_get(x_14, 3); -x_73 = lean_ctor_get(x_14, 4); -x_74 = lean_ctor_get(x_14, 5); -x_75 = lean_ctor_get(x_14, 6); -x_76 = lean_ctor_get(x_14, 7); -x_77 = lean_ctor_get(x_14, 8); -x_78 = lean_ctor_get(x_14, 9); -x_79 = lean_ctor_get(x_14, 10); +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_71 = lean_ctor_get(x_14, 0); +x_72 = lean_ctor_get(x_14, 1); +x_73 = lean_ctor_get(x_14, 2); +x_74 = lean_ctor_get(x_14, 3); +x_75 = lean_ctor_get(x_14, 4); +x_76 = lean_ctor_get(x_14, 5); +x_77 = lean_ctor_get(x_14, 6); +x_78 = lean_ctor_get(x_14, 7); +x_79 = lean_ctor_get(x_14, 8); +x_80 = lean_ctor_get(x_14, 9); +x_81 = lean_ctor_get(x_14, 10); +lean_inc(x_81); +lean_inc(x_80); lean_inc(x_79); lean_inc(x_78); lean_inc(x_77); @@ -2183,147 +2188,146 @@ lean_inc(x_74); lean_inc(x_73); lean_inc(x_72); lean_inc(x_71); -lean_inc(x_70); -lean_inc(x_69); lean_dec(x_14); -x_80 = l_Lean_replaceRef(x_1, x_74); -lean_dec(x_74); +x_82 = l_Lean_replaceRef(x_1, x_76); +lean_dec(x_76); lean_dec(x_1); -x_81 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_81, 0, x_69); -lean_ctor_set(x_81, 1, x_70); -lean_ctor_set(x_81, 2, x_71); -lean_ctor_set(x_81, 3, x_72); -lean_ctor_set(x_81, 4, x_73); -lean_ctor_set(x_81, 5, x_80); -lean_ctor_set(x_81, 6, x_75); -lean_ctor_set(x_81, 7, x_76); -lean_ctor_set(x_81, 8, x_77); -lean_ctor_set(x_81, 9, x_78); -lean_ctor_set(x_81, 10, x_79); +x_83 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_83, 0, x_71); +lean_ctor_set(x_83, 1, x_72); +lean_ctor_set(x_83, 2, x_73); +lean_ctor_set(x_83, 3, x_74); +lean_ctor_set(x_83, 4, x_75); +lean_ctor_set(x_83, 5, x_82); +lean_ctor_set(x_83, 6, x_77); +lean_ctor_set(x_83, 7, x_78); +lean_ctor_set(x_83, 8, x_79); +lean_ctor_set(x_83, 9, x_80); +lean_ctor_set(x_83, 10, x_81); if (x_2 == 0) { -lean_object* x_82; uint8_t x_83; -x_82 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___closed__8; +lean_object* x_84; uint8_t x_85; +x_84 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__2___closed__8; lean_inc(x_3); -x_83 = l_Lean_Syntax_isOfKind(x_3, x_82); -if (x_83 == 0) +x_85 = l_Lean_Syntax_isOfKind(x_3, x_84); +if (x_85 == 0) { -lean_object* x_84; lean_object* x_85; +lean_object* x_86; lean_object* x_87; lean_dec(x_7); lean_dec(x_3); -x_84 = lean_box(x_5); -x_85 = lean_apply_11(x_4, x_84, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_16); -return x_85; +x_86 = lean_box(x_5); +x_87 = lean_apply_11(x_4, x_86, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_16); +return x_87; } else { -lean_object* x_86; lean_object* x_87; uint8_t x_88; -x_86 = lean_unsigned_to_nat(1u); -x_87 = l_Lean_Syntax_getArg(x_3, x_86); +lean_object* x_88; lean_object* x_89; uint8_t x_90; +x_88 = lean_unsigned_to_nat(1u); +x_89 = l_Lean_Syntax_getArg(x_3, x_88); lean_dec(x_3); -lean_inc(x_87); -x_88 = l_Lean_Syntax_isOfKind(x_87, x_7); +lean_inc(x_89); +x_90 = l_Lean_Syntax_isOfKind(x_89, x_7); lean_dec(x_7); -if (x_88 == 0) +if (x_90 == 0) { -lean_object* x_89; lean_object* x_90; -lean_dec(x_87); -x_89 = lean_box(x_5); -x_90 = lean_apply_11(x_4, x_89, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_16); -return x_90; +lean_object* x_91; lean_object* x_92; +lean_dec(x_89); +x_91 = lean_box(x_5); +x_92 = lean_apply_11(x_4, x_91, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_16); +return x_92; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_91 = l_Lean_Elab_Tactic_saveState___rarg(x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_16); -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); -lean_dec(x_91); +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_93 = l_Lean_Elab_Tactic_saveState___rarg(x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_16); +x_94 = lean_ctor_get(x_93, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_93, 1); +lean_inc(x_95); +lean_dec(x_93); lean_inc(x_15); -lean_inc(x_81); +lean_inc(x_83); 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_87); -x_94 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_87, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_93); -if (lean_obj_tag(x_94) == 0) +lean_inc(x_89); +x_96 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_89, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_95); +if (lean_obj_tag(x_96) == 0) { -lean_object* x_95; lean_object* x_96; lean_object* x_97; -lean_dec(x_92); -x_95 = lean_ctor_get(x_94, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_94, 1); -lean_inc(x_96); +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_dec(x_94); -x_97 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_4, x_5, x_6, x_87, x_95, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_96); -return x_97; +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +lean_dec(x_96); +x_99 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_4, x_5, x_6, x_89, x_97, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_98); +return x_99; } else { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -lean_dec(x_87); -x_98 = lean_ctor_get(x_94, 1); -lean_inc(x_98); -lean_dec(x_94); -x_99 = l_Lean_Elab_Tactic_SavedState_restore(x_92, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_98); -x_100 = lean_ctor_get(x_99, 1); +lean_object* x_100; uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_89); +x_100 = lean_ctor_get(x_96, 1); lean_inc(x_100); -lean_dec(x_99); -x_101 = lean_box(x_5); -x_102 = lean_apply_11(x_4, x_101, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_100); -if (lean_obj_tag(x_102) == 0) -{ -lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_103 = lean_ctor_get(x_102, 0); +lean_dec(x_96); +x_101 = 0; +x_102 = l_Lean_Elab_Tactic_SavedState_restore(x_94, x_101, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_100); +x_103 = lean_ctor_get(x_102, 1); lean_inc(x_103); -x_104 = lean_ctor_get(x_102, 1); -lean_inc(x_104); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - x_105 = x_102; +lean_dec(x_102); +x_104 = lean_box(x_5); +x_105 = lean_apply_11(x_4, x_104, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_103); +if (lean_obj_tag(x_105) == 0) +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_106 = lean_ctor_get(x_105, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_105, 1); +lean_inc(x_107); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_108 = x_105; } else { - lean_dec_ref(x_102); - x_105 = lean_box(0); + lean_dec_ref(x_105); + x_108 = lean_box(0); } -if (lean_is_scalar(x_105)) { - x_106 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_108)) { + x_109 = lean_alloc_ctor(0, 2, 0); } else { - x_106 = x_105; + x_109 = x_108; } -lean_ctor_set(x_106, 0, x_103); -lean_ctor_set(x_106, 1, x_104); -return x_106; +lean_ctor_set(x_109, 0, x_106); +lean_ctor_set(x_109, 1, x_107); +return x_109; } else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_107 = lean_ctor_get(x_102, 0); -lean_inc(x_107); -x_108 = lean_ctor_get(x_102, 1); -lean_inc(x_108); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - x_109 = x_102; +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_110 = lean_ctor_get(x_105, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_105, 1); +lean_inc(x_111); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_112 = x_105; } else { - lean_dec_ref(x_102); - x_109 = lean_box(0); + lean_dec_ref(x_105); + x_112 = lean_box(0); } -if (lean_is_scalar(x_109)) { - x_110 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_112)) { + x_113 = lean_alloc_ctor(1, 2, 0); } else { - x_110 = x_109; + x_113 = x_112; } -lean_ctor_set(x_110, 0, x_107); -lean_ctor_set(x_110, 1, x_108); -return x_110; +lean_ctor_set(x_113, 0, x_110); +lean_ctor_set(x_113, 1, x_111); +return x_113; } } } @@ -2331,16 +2335,16 @@ return x_110; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_dec(x_7); -x_111 = l_Lean_Elab_Tactic_saveState___rarg(x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_16); -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -x_113 = lean_ctor_get(x_111, 1); -lean_inc(x_113); -lean_dec(x_111); +x_114 = l_Lean_Elab_Tactic_saveState___rarg(x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_16); +x_115 = lean_ctor_get(x_114, 0); +lean_inc(x_115); +x_116 = lean_ctor_get(x_114, 1); +lean_inc(x_116); +lean_dec(x_114); lean_inc(x_15); -lean_inc(x_81); +lean_inc(x_83); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -2348,73 +2352,50 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_3); -x_114 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_3, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_113); -if (lean_obj_tag(x_114) == 0) +x_117 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_withRWRulesSeq___spec__1(x_3, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_116); +if (lean_obj_tag(x_117) == 0) { -lean_object* x_115; lean_object* x_116; lean_object* x_117; -lean_dec(x_112); -x_115 = lean_ctor_get(x_114, 0); -lean_inc(x_115); -x_116 = lean_ctor_get(x_114, 1); -lean_inc(x_116); -lean_dec(x_114); -x_117 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_4, x_5, x_6, x_3, x_115, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_116); -return x_117; +lean_object* x_118; lean_object* x_119; lean_object* x_120; +lean_dec(x_115); +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_117, 1); +lean_inc(x_119); +lean_dec(x_117); +x_120 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___lambda__1(x_4, x_5, x_6, x_3, x_118, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_119); +return x_120; } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_dec(x_3); -x_118 = lean_ctor_get(x_114, 1); -lean_inc(x_118); -lean_dec(x_114); -x_119 = l_Lean_Elab_Tactic_SavedState_restore(x_112, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_118); -x_120 = lean_ctor_get(x_119, 1); -lean_inc(x_120); -lean_dec(x_119); -x_121 = lean_box(x_5); -x_122 = lean_apply_11(x_4, x_121, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_81, x_15, x_120); -if (lean_obj_tag(x_122) == 0) -{ -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_123 = lean_ctor_get(x_122, 0); -lean_inc(x_123); -x_124 = lean_ctor_get(x_122, 1); +x_121 = lean_ctor_get(x_117, 1); +lean_inc(x_121); +lean_dec(x_117); +x_122 = 0; +x_123 = l_Lean_Elab_Tactic_SavedState_restore(x_115, x_122, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_121); +x_124 = lean_ctor_get(x_123, 1); lean_inc(x_124); -if (lean_is_exclusive(x_122)) { - lean_ctor_release(x_122, 0); - lean_ctor_release(x_122, 1); - x_125 = x_122; -} else { - lean_dec_ref(x_122); - x_125 = lean_box(0); -} -if (lean_is_scalar(x_125)) { - x_126 = lean_alloc_ctor(0, 2, 0); -} else { - x_126 = x_125; -} -lean_ctor_set(x_126, 0, x_123); -lean_ctor_set(x_126, 1, x_124); -return x_126; -} -else +lean_dec(x_123); +x_125 = lean_box(x_5); +x_126 = lean_apply_11(x_4, x_125, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_83, x_15, x_124); +if (lean_obj_tag(x_126) == 0) { lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; -x_127 = lean_ctor_get(x_122, 0); +x_127 = lean_ctor_get(x_126, 0); lean_inc(x_127); -x_128 = lean_ctor_get(x_122, 1); +x_128 = lean_ctor_get(x_126, 1); lean_inc(x_128); -if (lean_is_exclusive(x_122)) { - lean_ctor_release(x_122, 0); - lean_ctor_release(x_122, 1); - x_129 = x_122; +if (lean_is_exclusive(x_126)) { + lean_ctor_release(x_126, 0); + lean_ctor_release(x_126, 1); + x_129 = x_126; } else { - lean_dec_ref(x_122); + lean_dec_ref(x_126); x_129 = lean_box(0); } if (lean_is_scalar(x_129)) { - x_130 = lean_alloc_ctor(1, 2, 0); + x_130 = lean_alloc_ctor(0, 2, 0); } else { x_130 = x_129; } @@ -2422,6 +2403,30 @@ lean_ctor_set(x_130, 0, x_127); lean_ctor_set(x_130, 1, x_128); return x_130; } +else +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_131 = lean_ctor_get(x_126, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_126, 1); +lean_inc(x_132); +if (lean_is_exclusive(x_126)) { + lean_ctor_release(x_126, 0); + lean_ctor_release(x_126, 1); + x_133 = x_126; +} else { + lean_dec_ref(x_126); + x_133 = lean_box(0); +} +if (lean_is_scalar(x_133)) { + x_134 = lean_alloc_ctor(1, 2, 0); +} else { + x_134 = x_133; +} +lean_ctor_set(x_134, 0, x_131); +lean_ctor_set(x_134, 1, x_132); +return x_134; +} } } } @@ -2536,7 +2541,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRul lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__3; x_2 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Elab_Tactic_withRWRulesSeq___spec__10___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2666,7 +2671,7 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -x_49 = l_Lean_Elab_withInfoTreeContext___at___private_Lean_Elab_Tactic_Basic_0__Lean_Elab_Tactic_evalTacticUsing_loop___spec__3(x_47, x_48, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_44); +x_49 = l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Tactic_evalTactic_eval___spec__1(x_47, x_48, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_44); if (lean_obj_tag(x_49) == 0) { lean_object* x_50; lean_object* x_51; lean_object* x_52; @@ -3909,7 +3914,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -3960,7 +3965,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 4); +x_29 = lean_ctor_get(x_27, 5); lean_inc(x_29); lean_dec(x_27); x_30 = lean_ctor_get(x_29, 1); @@ -3983,7 +3988,7 @@ lean_dec(x_34); x_36 = lean_st_ref_take(x_3, x_35); x_37 = lean_ctor_get(x_36, 0); lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 4); +x_38 = lean_ctor_get(x_37, 5); lean_inc(x_38); x_39 = lean_ctor_get(x_36, 1); lean_inc(x_39); @@ -3992,7 +3997,7 @@ x_40 = !lean_is_exclusive(x_37); if (x_40 == 0) { lean_object* x_41; uint8_t x_42; -x_41 = lean_ctor_get(x_37, 4); +x_41 = lean_ctor_get(x_37, 5); lean_dec(x_41); x_42 = !lean_is_exclusive(x_38); if (x_42 == 0) @@ -4037,7 +4042,7 @@ x_53 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_50); -lean_ctor_set(x_37, 4, x_53); +lean_ctor_set(x_37, 5, x_53); x_54 = lean_st_ref_set(x_3, x_37, x_39); lean_dec(x_3); x_55 = lean_ctor_get(x_54, 1); @@ -4062,243 +4067,249 @@ return x_57; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_58 = lean_ctor_get(x_37, 0); x_59 = lean_ctor_get(x_37, 1); x_60 = lean_ctor_get(x_37, 2); x_61 = lean_ctor_get(x_37, 3); +x_62 = lean_ctor_get(x_37, 4); +lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); lean_inc(x_58); lean_dec(x_37); -x_62 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); +x_63 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); +x_64 = lean_ctor_get(x_38, 0); +lean_inc(x_64); if (lean_is_exclusive(x_38)) { lean_ctor_release(x_38, 0); lean_ctor_release(x_38, 1); - x_64 = x_38; + x_65 = x_38; } else { lean_dec_ref(x_38); - x_64 = lean_box(0); + x_65 = lean_box(0); } -x_65 = l_Std_PersistentArray_append___rarg(x_19, x_32); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(0, 2, 1); +x_66 = l_Std_PersistentArray_append___rarg(x_19, x_32); +if (lean_is_scalar(x_65)) { + x_67 = lean_alloc_ctor(0, 2, 1); } else { - x_66 = x_64; -} -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_65); -lean_ctor_set_uint8(x_66, sizeof(void*)*2, x_62); -x_67 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_67, 0, x_58); -lean_ctor_set(x_67, 1, x_59); -lean_ctor_set(x_67, 2, x_60); -lean_ctor_set(x_67, 3, x_61); -lean_ctor_set(x_67, 4, x_66); -x_68 = lean_st_ref_set(x_3, x_67, x_39); + x_67 = x_65; +} +lean_ctor_set(x_67, 0, x_64); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_63); +x_68 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_68, 0, x_58); +lean_ctor_set(x_68, 1, x_59); +lean_ctor_set(x_68, 2, x_60); +lean_ctor_set(x_68, 3, x_61); +lean_ctor_set(x_68, 4, x_62); +lean_ctor_set(x_68, 5, x_67); +x_69 = lean_st_ref_set(x_3, x_68, x_39); lean_dec(x_3); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_70 = x_68; +x_70 = lean_ctor_get(x_69, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_71 = x_69; } else { - lean_dec_ref(x_68); - x_70 = lean_box(0); + lean_dec_ref(x_69); + x_71 = lean_box(0); } -if (lean_is_scalar(x_70)) { - x_71 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_70; + x_72 = x_71; } -lean_ctor_set(x_71, 0, x_22); -lean_ctor_set(x_71, 1, x_69); -return x_71; +lean_ctor_set(x_72, 0, x_22); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_72 = lean_ctor_get(x_21, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_21, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_73 = lean_ctor_get(x_21, 0); lean_inc(x_73); +x_74 = lean_ctor_get(x_21, 1); +lean_inc(x_74); lean_dec(x_21); -x_74 = lean_st_ref_get(x_7, x_73); -x_75 = lean_ctor_get(x_74, 1); -lean_inc(x_75); -lean_dec(x_74); -x_76 = lean_st_ref_get(x_3, x_75); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); +x_75 = lean_st_ref_get(x_7, x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_st_ref_get(x_3, x_76); +x_78 = lean_ctor_get(x_77, 0); lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_ctor_get(x_77, 4); +x_79 = lean_ctor_get(x_77, 1); lean_inc(x_79); lean_dec(x_77); -x_80 = lean_ctor_get(x_79, 1); +x_80 = lean_ctor_get(x_78, 5); lean_inc(x_80); -x_81 = l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabRewriteConfig___spec__7(x_79, x_80, x_2, x_3, x_4, x_5, x_6, x_7, x_78); +lean_dec(x_78); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +x_82 = l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabRewriteConfig___spec__7(x_80, x_81, x_2, x_3, x_4, x_5, x_6, x_7, x_79); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_st_ref_get(x_7, x_83); +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +lean_dec(x_82); +x_85 = lean_st_ref_get(x_7, x_84); lean_dec(x_7); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_3, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_87, 4); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_st_ref_take(x_3, x_86); +x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 1); +x_89 = lean_ctor_get(x_88, 5); lean_inc(x_89); -lean_dec(x_86); -x_90 = !lean_is_exclusive(x_87); -if (x_90 == 0) +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = !lean_is_exclusive(x_88); +if (x_91 == 0) { -lean_object* x_91; uint8_t x_92; -x_91 = lean_ctor_get(x_87, 4); -lean_dec(x_91); -x_92 = !lean_is_exclusive(x_88); -if (x_92 == 0) +lean_object* x_92; uint8_t x_93; +x_92 = lean_ctor_get(x_88, 5); +lean_dec(x_92); +x_93 = !lean_is_exclusive(x_89); +if (x_93 == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; -x_93 = lean_ctor_get(x_88, 1); -lean_dec(x_93); -x_94 = l_Std_PersistentArray_append___rarg(x_19, x_82); -lean_ctor_set(x_88, 1, x_94); -x_95 = lean_st_ref_set(x_3, x_87, x_89); +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_89, 1); +lean_dec(x_94); +x_95 = l_Std_PersistentArray_append___rarg(x_19, x_83); +lean_ctor_set(x_89, 1, x_95); +x_96 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) { -lean_object* x_97; -x_97 = lean_ctor_get(x_95, 0); -lean_dec(x_97); -lean_ctor_set_tag(x_95, 1); -lean_ctor_set(x_95, 0, x_72); -return x_95; +lean_object* x_98; +x_98 = lean_ctor_get(x_96, 0); +lean_dec(x_98); +lean_ctor_set_tag(x_96, 1); +lean_ctor_set(x_96, 0, x_73); +return x_96; } else { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_95, 1); -lean_inc(x_98); -lean_dec(x_95); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_72); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_dec(x_96); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_73); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_100 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_101 = lean_ctor_get(x_88, 0); -lean_inc(x_101); -lean_dec(x_88); -x_102 = l_Std_PersistentArray_append___rarg(x_19, x_82); -x_103 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_100); -lean_ctor_set(x_87, 4, x_103); -x_104 = lean_st_ref_set(x_3, x_87, x_89); +uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_101 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +lean_dec(x_89); +x_103 = l_Std_PersistentArray_append___rarg(x_19, x_83); +x_104 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set_uint8(x_104, sizeof(void*)*2, x_101); +lean_ctor_set(x_88, 5, x_104); +x_105 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_106 = x_104; +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; - lean_ctor_set_tag(x_107, 1); + x_108 = x_107; + lean_ctor_set_tag(x_108, 1); } -lean_ctor_set(x_107, 0, x_72); -lean_ctor_set(x_107, 1, x_105); -return x_107; +lean_ctor_set(x_108, 0, x_73); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_108 = lean_ctor_get(x_87, 0); -x_109 = lean_ctor_get(x_87, 1); -x_110 = lean_ctor_get(x_87, 2); -x_111 = lean_ctor_get(x_87, 3); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_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; +x_109 = lean_ctor_get(x_88, 0); +x_110 = lean_ctor_get(x_88, 1); +x_111 = lean_ctor_get(x_88, 2); +x_112 = lean_ctor_get(x_88, 3); +x_113 = lean_ctor_get(x_88, 4); +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_dec(x_87); -x_112 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_113 = lean_ctor_get(x_88, 0); -lean_inc(x_113); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_114 = x_88; +lean_dec(x_88); +x_114 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_115 = lean_ctor_get(x_89, 0); +lean_inc(x_115); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_116 = x_89; } else { - lean_dec_ref(x_88); - x_114 = lean_box(0); + lean_dec_ref(x_89); + x_116 = lean_box(0); } -x_115 = l_Std_PersistentArray_append___rarg(x_19, x_82); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 1); +x_117 = l_Std_PersistentArray_append___rarg(x_19, x_83); +if (lean_is_scalar(x_116)) { + x_118 = lean_alloc_ctor(0, 2, 1); } else { - x_116 = x_114; -} -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_115); -lean_ctor_set_uint8(x_116, sizeof(void*)*2, x_112); -x_117 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_117, 0, x_108); -lean_ctor_set(x_117, 1, x_109); -lean_ctor_set(x_117, 2, x_110); -lean_ctor_set(x_117, 3, x_111); -lean_ctor_set(x_117, 4, x_116); -x_118 = lean_st_ref_set(x_3, x_117, x_89); + x_118 = x_116; +} +lean_ctor_set(x_118, 0, x_115); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); +x_119 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_119, 0, x_109); +lean_ctor_set(x_119, 1, x_110); +lean_ctor_set(x_119, 2, x_111); +lean_ctor_set(x_119, 3, x_112); +lean_ctor_set(x_119, 4, x_113); +lean_ctor_set(x_119, 5, x_118); +x_120 = lean_st_ref_set(x_3, x_119, x_90); lean_dec(x_3); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_122 = x_120; } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + lean_dec_ref(x_120); + x_122 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); } else { - x_121 = x_120; - lean_ctor_set_tag(x_121, 1); + x_123 = x_122; + lean_ctor_set_tag(x_123, 1); } -lean_ctor_set(x_121, 0, x_72); -lean_ctor_set(x_121, 1, x_119); -return x_121; +lean_ctor_set(x_123, 0, x_73); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } diff --git a/stage0/stdlib/Lean/Elab/Tactic/Simp.c b/stage0/stdlib/Lean/Elab/Tactic/Simp.c index 02f653ce6407..7b76c4c13435 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Simp.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Simp.c @@ -19,61 +19,66 @@ LEAN_EXPORT lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Tactic_ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSimp___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__1(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Std_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_ExtensionState_declNames___default___spec__1; size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__11(lean_object*, lean_object*, 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_elabSimpArgs___spec__9___closed__3; lean_object* l_Lean_Expr_mvarId_x21(lean_object*); lean_object* lean_erase_macro_scopes(lean_object*); static lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__2___closed__6; lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_FunBinders_elabFunBinderViews___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabCDotFunctionAlias_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__6(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__2___closed__3; lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__9; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpConfig___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_throwErrorAt___at_Lean_Elab_Tactic_elabSimpArgs___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_mkDischargeWrapper(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5; lean_object* l_Lean_LocalDecl_userName(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp_declRange___closed__5; LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3; lean_object* l_List_filterTRAux___at_Lean_resolveGlobalConstCore___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___closed__5; -lean_object* l_Lean_Elab_Tactic_SavedState_restore(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_SavedState_restore(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_elabSimpConfigCore___closed__2; static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__8; lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SimpKind_toCtorIdx(uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tacticToDischarge___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SimpExtension_getTheorems(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__4; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_beqSimpKind____x40_Lean_Elab_Tactic_Simp___hyg_536_(uint8_t, uint8_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_EXPORT lean_object* l_panic___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__18(lean_object*); +static lean_object* l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1; lean_object* l_List_mapTRAux___at_Lean_resolveGlobalConstCore___spec__2(lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__1; extern lean_object* l_Std_Format_defWidth; static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__23; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__10(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__2; lean_object* l_Lean_SourceInfo_fromRef(lean_object*); +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__13(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_evalSimpAll___closed__3; lean_object* l_List_filterMap___at_Lean_resolveGlobalConst___spec__1(lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__18; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_mkDischargeWrapper___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__5; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_simpLocation_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___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__2; +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__14; LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at_Lean_Elab_Tactic_elabSimpConfigCore___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_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Tactic_elabSimpArgs___spec__16(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_evalDSimp_declRange___closed__3; lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__9(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -88,32 +93,34 @@ lean_object* l_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___rarg(lean_ static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___lambda__3___closed__1; uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp_declRange___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___closed__7; -static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll_declRange___closed__1; static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SimpTheorems_add(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_352____boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_RBNode_insert___at_Lean_Elab_Term_withAuxDecl___spec__1(lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__20(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_352____closed__2; lean_object* lean_string_append(lean_object*, lean_object*); -static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll_declRange___closed__4; -static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__3; lean_object* l_Lean_Elab_InfoTree_substitute(lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_withMainContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_TermElabM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_simpLocation_go(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*); -static lean_object* l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___lambda__1(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tacticToDischarge___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SimpTheorems_addDeclToUnfold(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__4; lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp_declRange(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp_declRange(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___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_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_simpLocation___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 lean_usize_dec_lt(size_t, size_t); @@ -131,12 +138,12 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__2(lean_objec static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__1; static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__20; static lean_object* l_Lean_Elab_Tactic_mkSimpContext___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__16(lean_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_elabSimpArgs___spec__4___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkSimpContext___boxed(lean_object*, lean_object*, lean_object*, lean_object*, 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_Simp___hyg_6____boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__2___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_LocalContext_empty; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSimpAll(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -145,102 +152,103 @@ lean_object* l_List_mapTRAux___at_Lean_resolveGlobalConstNoOverload___spec__1(le static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_352____closed__3; LEAN_EXPORT lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_PersistentHashMap_contains___at_Lean_Meta_SimpTheorems_erase___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2; static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_179____closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll___closed__1; LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___closed__3; lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_ElabSimpArgsResult_starArg___default; -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__4(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Tactic_tacticToDischarge___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___lambda__2(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_beqSimpKind____x40_Lean_Elab_Tactic_Simp___hyg_536____boxed(lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabTermEnsuringType(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__4; -static lean_object* l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3; +static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___closed__2; +static lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3; static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__3; -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_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_Meta_abstractMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__15; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSimp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_mkSimpContext___spec__1___at_Lean_Elab_Tactic_mkSimpContext___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*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpConfigCtxCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__8; +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1; lean_object* l_Lean_Elab_Tactic_expandOptLocation(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addSimpTheorem___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Meta_SimpTheorems_isLemma(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_dsimpLocation___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8; extern lean_object* l_Lean_Meta_simpExtension; static lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__3___closed__1; -static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1; static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___closed__4; lean_object* l_Lean_Elab_Term_elabTerm(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Tactic_instInhabitedSimpKind; +LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__10; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___lambda__1___boxed(lean_object**); static lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__3___closed__2; uint8_t l_Lean_Expr_hasExprMVar(lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* l_Lean_throwError___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getMajorPosDepElim___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll___closed__4; lean_object* l_Lean_Meta_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4; static lean_object* l_Lean_Elab_Tactic_elabDSimpConfigCore___closed__3; static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp_declRange___closed__7; static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___closed__8; static lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__2___closed__5; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__1___boxed(lean_object**); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4; +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpConfig(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___lambda__3___closed__2; static lean_object* l_Lean_Elab_Tactic_instBEqSimpKind___closed__1; -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Tactic_elabSimpArgs___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_Lean_Meta_evalExpr_x27___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_179____boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSimp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabDSimpConfigCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_format_pretty(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_simpLocation(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___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* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_simpLocation___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__7; static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_179____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_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_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___lambda__2___boxed(lean_object**); static lean_object* l_Lean_Elab_Tactic_elabDSimpConfigCore___closed__2; lean_object* l_Lean_Elab_Term_resolveId_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_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_Elab_Tactic_tacticToDischarge___closed__19; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp_declRange___closed__4; static lean_object* l_Lean_Elab_Tactic_elabSimpConfigCtxCore___closed__3; static lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___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___regBuiltin_Lean_Elab_Tactic_evalDSimp___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -248,20 +256,21 @@ lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_ uint8_t l_Lean_Expr_isConst(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__11(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SimpKind_noConfusion(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_dsimpLocation___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__1(lean_object*, uint8_t, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_elabSimpConfigCore___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5; lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpConfigCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Tactic_elabSimpArgs___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ResolveName_resolveGlobalName(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_elabSimpArgs___closed__3; lean_object* l_Lean_Meta_SimpTheorems_eraseCore(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tacticToDischarge___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_instInhabitedSimpTheorems; static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Simp_DischargeWrapper_with___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp___closed__2; size_t lean_usize_of_nat(lean_object*); @@ -269,129 +278,119 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp_declRange___closed_ extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_dsimpLocation___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_ConstantInfo_type(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_runTactic(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_fvarId(lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SimpKind_noConfusion___rarg___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_withoutModifyingStateWithInfoAndMessages___at_Lean_Elab_Tactic_tacticToDischarge___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp___closed__3; -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__3(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tacticToDischarge___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp_declRange___closed__1; static lean_object* l_Lean_Elab_Tactic_elabDSimpConfigCore___closed__1; -static lean_object* l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__11; -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__16___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_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Tactic_tacticToDischarge___spec__1___rarg___boxed(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_evalSimp___closed__2; -static lean_object* l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2; +LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Tactic_elabSimpArgs___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addSimpTheorem___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getSepArgs(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_Simp_DischargeWrapper_with___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___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_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___closed__1; +static lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2; lean_object* l_Lean_Expr_eta(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp_declRange___closed__6; lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp___closed__1; -LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__13___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_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Tactic_tacticToDischarge___spec__1___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_SavedState_restore(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3; lean_object* l_Lean_Meta_dsimpGoal(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_simpAll(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6; +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_elabSimpArgs___spec__10(lean_object*, 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_evalSimp___closed__4; static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__16; -static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3; +static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2; +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__13___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_evalSimp___closed__8; -static lean_object* l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__2(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll_declRange___closed__7; static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__12; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalDSimp(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_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___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_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__3; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll___closed__2; lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1; +static lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1; lean_object* l_Lean_Meta_getSimpExtension_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___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_st_ref_set(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2; static lean_object* l_Lean_Elab_Tactic_elabSimpConfigCore___closed__3; static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___lambda__3___closed__3; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_Meta_simpGoal(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__12___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__13___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_elabSimpArgs___closed__2; uint8_t l_Lean_Syntax_isNone(lean_object*); lean_object* l_Lean_Elab_Tactic_getFVarIds(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_mkSimpContext___spec__1___closed__2; lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__13; -LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__12(lean_object*, 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_pushInfoLeaf___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_elabSimpConfigCtxCore___closed__2; lean_object* l_Lean_Meta_getPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_dsimpLocation_go(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Tactic_elabSimpArgs___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tacticToDischarge(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_evalSimpAll_declRange___closed__3; LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2; lean_object* l_Lean_Elab_Term_withoutErrToSorry___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_dsimpLocation(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_replaceMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_352____closed__1; extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___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_Lean_Elab_Tactic_tacticToDischarge___closed__21; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SimpKind_toCtorIdx___boxed(lean_object*); +static lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Tactic_elabSimpArgs___spec__12(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_evalSimpAll_declRange___closed__5; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkSimpContext___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__2; lean_object* l_Lean_Meta_SimpTheoremsArray_addTheorem(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_elabSimpArgs___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SimpTheorems_addConst(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp___closed__5; -static lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4; static lean_object* l_Lean_Elab_Tactic_mkSimpContext___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addSimpTheorem(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_elabSimpArgs___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp_declRange___closed__4; lean_object* l_Lean_Meta_mkFreshExprSyntheticOpaqueMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__17; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp___closed__6; -static lean_object* l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_elabSimpArgs___spec__18(lean_object*); static lean_object* l_Lean_Elab_Tactic_elabSimpConfigCtxCore___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_179_(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_Simp___hyg_352_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -401,44 +400,45 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_a LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_dsimpLocation_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabDSimpConfigCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpConfigCtxCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Tactic_elabSimpArgs___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SimpKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); lean_object* l_List_toString___at_Lean_resolveGlobalConstNoOverloadCore___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SimpKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Meta_SimpTheoremsArray_isErased(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Tactic_elabSimpArgs___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isProp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_elabSimpArgs___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_tacticToDischarge___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_tacticToDischarge___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instBEqSimpKind; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_mkSimpContext(lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__7; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimp_declRange___closed__2; static lean_object* l_Lean_Elab_Tactic_SimpKind_noConfusion___rarg___closed__1; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__20(lean_object*, uint8_t, uint8_t, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_isLocalIdent_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_constName_x21(lean_object*); +static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1; lean_object* l_Lean_Elab_Term_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_Simp_defaultMaxSteps; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalDSimp_declRange___closed__2; lean_object* l_Lean_Syntax_formatStxAux(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll_declRange___closed__6; -LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___boxed__const__1; lean_object* l_Lean_Meta_DiscrTree_empty(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSimpAll_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_SimpKind_noConfusion___rarg___lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getSimpCongrTheorems___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2; lean_object* l___private_Lean_Elab_SyntheticMVars_0__Lean_Elab_Term_withSynthesizeImp___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addSimpTheorem___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2; static lean_object* _init_l_Lean_Elab_Tactic_evalUnsafe____x40_Lean_Elab_Tactic_Simp___hyg_6____closed__1() { _start: { @@ -1286,7 +1286,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -1337,7 +1337,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 4); +x_29 = lean_ctor_get(x_27, 5); lean_inc(x_29); lean_dec(x_27); x_30 = lean_ctor_get(x_29, 1); @@ -1360,7 +1360,7 @@ lean_dec(x_34); x_36 = lean_st_ref_take(x_3, x_35); x_37 = lean_ctor_get(x_36, 0); lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 4); +x_38 = lean_ctor_get(x_37, 5); lean_inc(x_38); x_39 = lean_ctor_get(x_36, 1); lean_inc(x_39); @@ -1369,7 +1369,7 @@ x_40 = !lean_is_exclusive(x_37); if (x_40 == 0) { lean_object* x_41; uint8_t x_42; -x_41 = lean_ctor_get(x_37, 4); +x_41 = lean_ctor_get(x_37, 5); lean_dec(x_41); x_42 = !lean_is_exclusive(x_38); if (x_42 == 0) @@ -1414,7 +1414,7 @@ x_53 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_50); -lean_ctor_set(x_37, 4, x_53); +lean_ctor_set(x_37, 5, x_53); x_54 = lean_st_ref_set(x_3, x_37, x_39); lean_dec(x_3); x_55 = lean_ctor_get(x_54, 1); @@ -1439,243 +1439,249 @@ return x_57; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_58 = lean_ctor_get(x_37, 0); x_59 = lean_ctor_get(x_37, 1); x_60 = lean_ctor_get(x_37, 2); x_61 = lean_ctor_get(x_37, 3); +x_62 = lean_ctor_get(x_37, 4); +lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); lean_inc(x_58); lean_dec(x_37); -x_62 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); +x_63 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); +x_64 = lean_ctor_get(x_38, 0); +lean_inc(x_64); if (lean_is_exclusive(x_38)) { lean_ctor_release(x_38, 0); lean_ctor_release(x_38, 1); - x_64 = x_38; + x_65 = x_38; } else { lean_dec_ref(x_38); - x_64 = lean_box(0); + x_65 = lean_box(0); } -x_65 = l_Std_PersistentArray_append___rarg(x_19, x_32); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(0, 2, 1); +x_66 = l_Std_PersistentArray_append___rarg(x_19, x_32); +if (lean_is_scalar(x_65)) { + x_67 = lean_alloc_ctor(0, 2, 1); } else { - x_66 = x_64; + x_67 = x_65; } -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_65); -lean_ctor_set_uint8(x_66, sizeof(void*)*2, x_62); -x_67 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_67, 0, x_58); -lean_ctor_set(x_67, 1, x_59); -lean_ctor_set(x_67, 2, x_60); -lean_ctor_set(x_67, 3, x_61); -lean_ctor_set(x_67, 4, x_66); -x_68 = lean_st_ref_set(x_3, x_67, x_39); +lean_ctor_set(x_67, 0, x_64); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_63); +x_68 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_68, 0, x_58); +lean_ctor_set(x_68, 1, x_59); +lean_ctor_set(x_68, 2, x_60); +lean_ctor_set(x_68, 3, x_61); +lean_ctor_set(x_68, 4, x_62); +lean_ctor_set(x_68, 5, x_67); +x_69 = lean_st_ref_set(x_3, x_68, x_39); lean_dec(x_3); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_70 = x_68; +x_70 = lean_ctor_get(x_69, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_71 = x_69; } else { - lean_dec_ref(x_68); - x_70 = lean_box(0); + lean_dec_ref(x_69); + x_71 = lean_box(0); } -if (lean_is_scalar(x_70)) { - x_71 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_70; + x_72 = x_71; } -lean_ctor_set(x_71, 0, x_22); -lean_ctor_set(x_71, 1, x_69); -return x_71; +lean_ctor_set(x_72, 0, x_22); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_72 = lean_ctor_get(x_21, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_21, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_73 = lean_ctor_get(x_21, 0); lean_inc(x_73); +x_74 = lean_ctor_get(x_21, 1); +lean_inc(x_74); lean_dec(x_21); -x_74 = lean_st_ref_get(x_7, x_73); -x_75 = lean_ctor_get(x_74, 1); -lean_inc(x_75); -lean_dec(x_74); -x_76 = lean_st_ref_get(x_3, x_75); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); +x_75 = lean_st_ref_get(x_7, x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_st_ref_get(x_3, x_76); +x_78 = lean_ctor_get(x_77, 0); lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_ctor_get(x_77, 4); +x_79 = lean_ctor_get(x_77, 1); lean_inc(x_79); lean_dec(x_77); -x_80 = lean_ctor_get(x_79, 1); +x_80 = lean_ctor_get(x_78, 5); lean_inc(x_80); -x_81 = l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__7(x_79, x_80, x_2, x_3, x_4, x_5, x_6, x_7, x_78); +lean_dec(x_78); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +x_82 = l_Std_PersistentArray_mapM___at_Lean_Elab_Tactic_elabSimpConfigCore___spec__7(x_80, x_81, x_2, x_3, x_4, x_5, x_6, x_7, x_79); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_st_ref_get(x_7, x_83); +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +lean_dec(x_82); +x_85 = lean_st_ref_get(x_7, x_84); lean_dec(x_7); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_3, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_87, 4); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_st_ref_take(x_3, x_86); +x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 1); +x_89 = lean_ctor_get(x_88, 5); lean_inc(x_89); -lean_dec(x_86); -x_90 = !lean_is_exclusive(x_87); -if (x_90 == 0) -{ -lean_object* x_91; uint8_t x_92; -x_91 = lean_ctor_get(x_87, 4); -lean_dec(x_91); -x_92 = !lean_is_exclusive(x_88); -if (x_92 == 0) -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; -x_93 = lean_ctor_get(x_88, 1); -lean_dec(x_93); -x_94 = l_Std_PersistentArray_append___rarg(x_19, x_82); -lean_ctor_set(x_88, 1, x_94); -x_95 = lean_st_ref_set(x_3, x_87, x_89); +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = !lean_is_exclusive(x_88); +if (x_91 == 0) +{ +lean_object* x_92; uint8_t x_93; +x_92 = lean_ctor_get(x_88, 5); +lean_dec(x_92); +x_93 = !lean_is_exclusive(x_89); +if (x_93 == 0) +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_89, 1); +lean_dec(x_94); +x_95 = l_Std_PersistentArray_append___rarg(x_19, x_83); +lean_ctor_set(x_89, 1, x_95); +x_96 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) { -lean_object* x_97; -x_97 = lean_ctor_get(x_95, 0); -lean_dec(x_97); -lean_ctor_set_tag(x_95, 1); -lean_ctor_set(x_95, 0, x_72); -return x_95; +lean_object* x_98; +x_98 = lean_ctor_get(x_96, 0); +lean_dec(x_98); +lean_ctor_set_tag(x_96, 1); +lean_ctor_set(x_96, 0, x_73); +return x_96; } else { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_95, 1); -lean_inc(x_98); -lean_dec(x_95); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_72); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_dec(x_96); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_73); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_100 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_101 = lean_ctor_get(x_88, 0); -lean_inc(x_101); -lean_dec(x_88); -x_102 = l_Std_PersistentArray_append___rarg(x_19, x_82); -x_103 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_100); -lean_ctor_set(x_87, 4, x_103); -x_104 = lean_st_ref_set(x_3, x_87, x_89); +uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_101 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +lean_dec(x_89); +x_103 = l_Std_PersistentArray_append___rarg(x_19, x_83); +x_104 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set_uint8(x_104, sizeof(void*)*2, x_101); +lean_ctor_set(x_88, 5, x_104); +x_105 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_106 = x_104; +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; - lean_ctor_set_tag(x_107, 1); + x_108 = x_107; + lean_ctor_set_tag(x_108, 1); } -lean_ctor_set(x_107, 0, x_72); -lean_ctor_set(x_107, 1, x_105); -return x_107; +lean_ctor_set(x_108, 0, x_73); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_108 = lean_ctor_get(x_87, 0); -x_109 = lean_ctor_get(x_87, 1); -x_110 = lean_ctor_get(x_87, 2); -x_111 = lean_ctor_get(x_87, 3); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_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; +x_109 = lean_ctor_get(x_88, 0); +x_110 = lean_ctor_get(x_88, 1); +x_111 = lean_ctor_get(x_88, 2); +x_112 = lean_ctor_get(x_88, 3); +x_113 = lean_ctor_get(x_88, 4); +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_dec(x_87); -x_112 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_113 = lean_ctor_get(x_88, 0); -lean_inc(x_113); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_114 = x_88; +lean_dec(x_88); +x_114 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_115 = lean_ctor_get(x_89, 0); +lean_inc(x_115); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_116 = x_89; } else { - lean_dec_ref(x_88); - x_114 = lean_box(0); + lean_dec_ref(x_89); + x_116 = lean_box(0); } -x_115 = l_Std_PersistentArray_append___rarg(x_19, x_82); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 1); +x_117 = l_Std_PersistentArray_append___rarg(x_19, x_83); +if (lean_is_scalar(x_116)) { + x_118 = lean_alloc_ctor(0, 2, 1); } else { - x_116 = x_114; -} -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_115); -lean_ctor_set_uint8(x_116, sizeof(void*)*2, x_112); -x_117 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_117, 0, x_108); -lean_ctor_set(x_117, 1, x_109); -lean_ctor_set(x_117, 2, x_110); -lean_ctor_set(x_117, 3, x_111); -lean_ctor_set(x_117, 4, x_116); -x_118 = lean_st_ref_set(x_3, x_117, x_89); + x_118 = x_116; +} +lean_ctor_set(x_118, 0, x_115); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); +x_119 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_119, 0, x_109); +lean_ctor_set(x_119, 1, x_110); +lean_ctor_set(x_119, 2, x_111); +lean_ctor_set(x_119, 3, x_112); +lean_ctor_set(x_119, 4, x_113); +lean_ctor_set(x_119, 5, x_118); +x_120 = lean_st_ref_set(x_3, x_119, x_90); lean_dec(x_3); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_122 = x_120; } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + lean_dec_ref(x_120); + x_122 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); } else { - x_121 = x_120; - lean_ctor_set_tag(x_121, 1); + x_123 = x_122; + lean_ctor_set_tag(x_123, 1); } -lean_ctor_set(x_121, 0, x_72); -lean_ctor_set(x_121, 1, x_119); -return x_121; +lean_ctor_set(x_123, 0, x_73); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } @@ -4783,7 +4789,7 @@ x_1 = 0; return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1() { _start: { lean_object* x_1; @@ -4791,17 +4797,17 @@ x_1 = lean_mk_string_from_bytes("ident", 5); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1; +x_2 = l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -4813,7 +4819,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4() { _start: { lean_object* x_1; @@ -4821,11 +4827,11 @@ x_1 = lean_mk_string_from_bytes("term", 4); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; lean_object* x_16; uint8_t x_17; -x_16 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2; +x_16 = l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2; lean_inc(x_1); x_17 = l_Lean_Syntax_isOfKind(x_1, x_16); if (x_17 == 0) @@ -4923,15 +4929,15 @@ return x_37; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_58; uint8_t x_59; lean_object* x_60; +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_59; uint8_t x_60; lean_object* x_61; x_38 = l_Lean_Elab_Tactic_saveState___rarg(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); 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_58 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4; -x_59 = 1; +x_59 = l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4; +x_60 = 1; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); @@ -4939,148 +4945,149 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_1); -x_60 = l_Lean_Elab_Term_resolveId_x3f(x_1, x_58, x_59, x_4, x_5, x_6, x_7, x_8, x_9, x_40); -if (lean_obj_tag(x_60) == 0) +x_61 = l_Lean_Elab_Term_resolveId_x3f(x_1, x_59, x_60, x_4, x_5, x_6, x_7, x_8, x_9, x_40); +if (lean_obj_tag(x_61) == 0) { -lean_object* x_61; +lean_object* x_62; lean_dec(x_39); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -if (lean_obj_tag(x_61) == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_62 = lean_ctor_get(x_60, 1); +x_62 = lean_ctor_get(x_61, 0); lean_inc(x_62); -lean_dec(x_60); -x_63 = l_Lean_Syntax_getId(x_1); +if (lean_obj_tag(x_62) == 0) +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_63 = lean_ctor_get(x_61, 1); +lean_inc(x_63); +lean_dec(x_61); +x_64 = l_Lean_Syntax_getId(x_1); lean_dec(x_1); -x_64 = lean_erase_macro_scopes(x_63); -x_65 = lean_st_ref_get(x_9, x_62); +x_65 = lean_erase_macro_scopes(x_64); +x_66 = lean_st_ref_get(x_9, x_63); lean_dec(x_9); -x_66 = lean_ctor_get(x_65, 1); -lean_inc(x_66); -lean_dec(x_65); -x_67 = l_Lean_Meta_getSimpExtension_x3f(x_64, x_66); -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -if (lean_obj_tag(x_68) == 0) -{ -lean_object* x_69; lean_object* x_70; -x_69 = lean_ctor_get(x_67, 1); +x_67 = lean_ctor_get(x_66, 1); +lean_inc(x_67); +lean_dec(x_66); +x_68 = l_Lean_Meta_getSimpExtension_x3f(x_65, x_67); +x_69 = lean_ctor_get(x_68, 0); lean_inc(x_69); -lean_dec(x_67); -x_70 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3; -x_11 = x_70; -x_12 = x_69; +if (lean_obj_tag(x_69) == 0) +{ +lean_object* x_70; lean_object* x_71; +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3; +x_11 = x_71; +x_12 = x_70; goto block_15; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_71 = lean_ctor_get(x_67, 1); -lean_inc(x_71); -lean_dec(x_67); -x_72 = lean_ctor_get(x_68, 0); +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_72 = lean_ctor_get(x_68, 1); lean_inc(x_72); lean_dec(x_68); -x_73 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_73, 0, x_72); -x_74 = lean_box(0); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -x_11 = x_75; -x_12 = x_71; +x_73 = lean_ctor_get(x_69, 0); +lean_inc(x_73); +lean_dec(x_69); +x_74 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_74, 0, x_73); +x_75 = lean_box(0); +x_76 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_75); +x_11 = x_76; +x_12 = x_72; goto block_15; } } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_dec(x_9); lean_dec(x_1); -x_76 = lean_ctor_get(x_60, 1); -lean_inc(x_76); -lean_dec(x_60); -x_77 = lean_ctor_get(x_61, 0); +x_77 = lean_ctor_get(x_61, 1); lean_inc(x_77); lean_dec(x_61); -x_78 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_78, 0, x_77); -x_79 = lean_box(0); -x_80 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_80, 0, x_78); -lean_ctor_set(x_80, 1, x_79); -x_11 = x_80; -x_12 = x_76; +x_78 = lean_ctor_get(x_62, 0); +lean_inc(x_78); +lean_dec(x_62); +x_79 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_79, 0, x_78); +x_80 = lean_box(0); +x_81 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +x_11 = x_81; +x_12 = x_77; goto block_15; } } else { -lean_object* x_81; -x_81 = lean_ctor_get(x_60, 1); -lean_inc(x_81); -lean_dec(x_60); -x_41 = x_81; -goto block_57; +lean_object* x_82; +x_82 = lean_ctor_get(x_61, 1); +lean_inc(x_82); +lean_dec(x_61); +x_41 = x_82; +goto block_58; } -block_57: +block_58: { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_42 = l_Lean_Elab_Tactic_SavedState_restore(x_39, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_41); +uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_42 = 0; +x_43 = l_Lean_Elab_Tactic_SavedState_restore(x_39, x_42, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_41); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -x_44 = l_Lean_Syntax_getId(x_1); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +x_45 = l_Lean_Syntax_getId(x_1); lean_dec(x_1); -x_45 = lean_erase_macro_scopes(x_44); -x_46 = lean_st_ref_get(x_9, x_43); +x_46 = lean_erase_macro_scopes(x_45); +x_47 = lean_st_ref_get(x_9, x_44); lean_dec(x_9); -x_47 = lean_ctor_get(x_46, 1); -lean_inc(x_47); -lean_dec(x_46); -x_48 = l_Lean_Meta_getSimpExtension_x3f(x_45, x_47); -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -if (lean_obj_tag(x_49) == 0) -{ -lean_object* x_50; lean_object* x_51; -x_50 = lean_ctor_get(x_48, 1); +x_48 = lean_ctor_get(x_47, 1); +lean_inc(x_48); +lean_dec(x_47); +x_49 = l_Lean_Meta_getSimpExtension_x3f(x_46, x_48); +x_50 = lean_ctor_get(x_49, 0); lean_inc(x_50); -lean_dec(x_48); -x_51 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3; -x_11 = x_51; -x_12 = x_50; +if (lean_obj_tag(x_50) == 0) +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3; +x_11 = x_52; +x_12 = x_51; goto block_15; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_52 = lean_ctor_get(x_48, 1); -lean_inc(x_52); -lean_dec(x_48); -x_53 = lean_ctor_get(x_49, 0); +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_53 = lean_ctor_get(x_49, 1); lean_inc(x_53); lean_dec(x_49); -x_54 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_54, 0, x_53); -x_55 = lean_box(0); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -x_11 = x_56; -x_12 = x_52; +x_54 = lean_ctor_get(x_50, 0); +lean_inc(x_54); +lean_dec(x_50); +x_55 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_55, 0, x_54); +x_56 = lean_box(0); +x_57 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +x_11 = x_57; +x_12 = x_53; goto block_15; } } @@ -5098,17 +5105,17 @@ return x_14; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_3); lean_dec(x_2); return x_11; } } -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1() { +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1() { _start: { lean_object* x_1; @@ -5116,38 +5123,38 @@ x_1 = l_Lean_Elab_unsupportedSyntaxExceptionId; return x_1; } } -static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2() { +static lean_object* _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2; +x_2 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg), 1, 0); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg), 1, 0); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -5185,7 +5192,7 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_elabSimpArgs___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; @@ -5198,7 +5205,7 @@ x_14 = l_Lean_replaceRef(x_1, x_13); lean_dec(x_13); lean_dec(x_1); lean_ctor_set(x_9, 5, x_14); -x_15 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -5250,7 +5257,7 @@ lean_ctor_set(x_28, 7, x_23); lean_ctor_set(x_28, 8, x_24); lean_ctor_set(x_28, 9, x_25); lean_ctor_set(x_28, 10, x_26); -x_29 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); +x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); lean_dec(x_10); lean_dec(x_28); lean_dec(x_8); @@ -5263,7 +5270,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Tactic_elabSimpArgs___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -5309,7 +5316,7 @@ return x_24; } } } -static lean_object* _init_l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1() { _start: { lean_object* x_1; @@ -5317,16 +5324,16 @@ x_1 = lean_mk_string_from_bytes("unknown constant '", 18); return x_1; } } -static lean_object* _init_l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1; +x_1 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3() { _start: { lean_object* x_1; @@ -5334,16 +5341,16 @@ x_1 = lean_mk_string_from_bytes("'", 1); return x_1; } } -static lean_object* _init_l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4() { +static lean_object* _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3; +x_1 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; 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; @@ -5351,19 +5358,19 @@ x_11 = lean_box(0); x_12 = l_Lean_Expr_const___override(x_1, x_11); x_13 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_13, 0, x_12); -x_14 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2; +x_14 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2; x_15 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_13); -x_16 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; +x_16 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; x_17 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_18; } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -5374,13 +5381,13 @@ lean_ctor_set(x_14, 1, x_12); return x_14; } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_inc(x_8); lean_inc(x_1); -x_11 = l_Lean_resolveGlobalName___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_resolveGlobalName___at_Lean_Elab_Tactic_elabSimpArgs___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); @@ -5394,7 +5401,7 @@ if (x_16 == 0) lean_object* x_17; lean_object* x_18; lean_dec(x_1); x_17 = lean_box(0); -x_18 = l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1(x_15, x_14, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_18 = l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1(x_15, x_14, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -5409,7 +5416,7 @@ else { lean_object* x_19; uint8_t x_20; lean_dec(x_15); -x_19 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_19 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -5439,7 +5446,7 @@ return x_23; } } } -static lean_object* _init_l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1() { +static lean_object* _init_l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1() { _start: { lean_object* x_1; @@ -5447,27 +5454,27 @@ x_1 = lean_mk_string_from_bytes("expected identifier", 19); return x_1; } } -static lean_object* _init_l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2() { +static lean_object* _init_l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1; +x_1 = l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3() { +static lean_object* _init_l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2; +x_1 = l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { if (lean_obj_tag(x_1) == 3) @@ -5510,7 +5517,7 @@ x_18 = l_Lean_replaceRef(x_1, x_17); lean_dec(x_17); lean_dec(x_1); lean_ctor_set(x_8, 5, x_18); -x_19 = l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_19 = l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_19; } else @@ -5554,7 +5561,7 @@ lean_ctor_set(x_32, 7, x_27); lean_ctor_set(x_32, 8, x_28); lean_ctor_set(x_32, 9, x_29); lean_ctor_set(x_32, 10, x_30); -x_33 = l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_32, x_9, x_10); +x_33 = l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_32, x_9, x_10); return x_33; } } @@ -5562,13 +5569,13 @@ return x_33; else { lean_object* x_34; lean_object* x_35; -x_34 = l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3; -x_35 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__5(x_1, x_34, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_34 = l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3; +x_35 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_elabSimpArgs___spec__5(x_1, x_34, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_35; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -5606,7 +5613,7 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_elabSimpArgs___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; @@ -5619,7 +5626,7 @@ x_14 = l_Lean_replaceRef(x_1, x_13); lean_dec(x_13); lean_dec(x_1); lean_ctor_set(x_9, 5, x_14); -x_15 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__11(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__11(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -5671,7 +5678,7 @@ lean_ctor_set(x_28, 7, x_23); lean_ctor_set(x_28, 8, x_24); lean_ctor_set(x_28, 9, x_25); lean_ctor_set(x_28, 10, x_26); -x_29 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__11(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); +x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__11(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); lean_dec(x_10); lean_dec(x_28); lean_dec(x_8); @@ -5684,7 +5691,7 @@ return x_29; } } } -static lean_object* _init_l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1() { +static lean_object* _init_l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1() { _start: { lean_object* x_1; @@ -5692,7 +5699,7 @@ x_1 = lean_mk_string_from_bytes("ambiguous identifier '", 22); return x_1; } } -static lean_object* _init_l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2() { +static lean_object* _init_l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2() { _start: { lean_object* x_1; @@ -5700,7 +5707,7 @@ x_1 = lean_mk_string_from_bytes("', possible interpretations: ", 29); return x_1; } } -static lean_object* _init_l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3() { +static lean_object* _init_l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3() { _start: { lean_object* x_1; @@ -5708,7 +5715,7 @@ x_1 = lean_mk_string_from_bytes("", 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; @@ -5721,7 +5728,7 @@ lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_11 = l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; @@ -5740,23 +5747,23 @@ lean_inc(x_1); x_17 = l_Lean_Syntax_formatStxAux(x_14, x_15, x_16, x_1); x_18 = l_Std_Format_defWidth; x_19 = lean_format_pretty(x_17, x_18); -x_20 = l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1; +x_20 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1; x_21 = lean_string_append(x_20, x_19); lean_dec(x_19); -x_22 = l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2; +x_22 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2; x_23 = lean_string_append(x_21, x_22); x_24 = lean_box(0); x_25 = l_List_mapTRAux___at_Lean_resolveGlobalConstNoOverload___spec__1(x_12, x_24); x_26 = l_List_toString___at_Lean_resolveGlobalConstNoOverloadCore___spec__2(x_25); x_27 = lean_string_append(x_23, x_26); lean_dec(x_26); -x_28 = l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3; +x_28 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3; x_29 = lean_string_append(x_27, x_28); x_30 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_30, 0, x_29); x_31 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_31, 0, x_30); -x_32 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__10(x_1, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_32 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_elabSimpArgs___spec__10(x_1, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_32; } else @@ -5817,23 +5824,23 @@ lean_inc(x_1); x_44 = l_Lean_Syntax_formatStxAux(x_41, x_42, x_43, x_1); x_45 = l_Std_Format_defWidth; x_46 = lean_format_pretty(x_44, x_45); -x_47 = l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1; +x_47 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1; x_48 = lean_string_append(x_47, x_46); lean_dec(x_46); -x_49 = l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2; +x_49 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2; x_50 = lean_string_append(x_48, x_49); x_51 = lean_box(0); x_52 = l_List_mapTRAux___at_Lean_resolveGlobalConstNoOverload___spec__1(x_12, x_51); x_53 = l_List_toString___at_Lean_resolveGlobalConstNoOverloadCore___spec__2(x_52); x_54 = lean_string_append(x_50, x_53); lean_dec(x_53); -x_55 = l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3; +x_55 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3; x_56 = lean_string_append(x_54, x_55); x_57 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_57, 0, x_56); x_58 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_58, 0, x_57); -x_59 = l_Lean_throwErrorAt___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__10(x_1, x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_40); +x_59 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_elabSimpArgs___spec__10(x_1, x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_40); return x_59; } } @@ -5871,7 +5878,7 @@ return x_63; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -5909,7 +5916,7 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; uint8_t x_12; @@ -5933,15 +5940,15 @@ x_17 = lean_box(0); x_18 = l_Lean_Expr_const___override(x_1, x_17); x_19 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_19, 0, x_18); -x_20 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2; +x_20 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2; x_21 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_21, 0, x_20); lean_ctor_set(x_21, 1, x_19); -x_22 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; +x_22 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; x_23 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_23, 0, x_21); lean_ctor_set(x_23, 1, x_22); -x_24 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__14(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +x_24 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__14(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); return x_24; } else @@ -5975,15 +5982,15 @@ x_30 = lean_box(0); x_31 = l_Lean_Expr_const___override(x_1, x_30); x_32 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_32, 0, x_31); -x_33 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2; +x_33 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2; x_34 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_34, 0, x_33); lean_ctor_set(x_34, 1, x_32); -x_35 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; +x_35 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; x_36 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_36, 0, x_34); lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__14(x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +x_37 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__14(x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_27); return x_37; } else @@ -6001,12 +6008,12 @@ return x_39; } } } -LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Tactic_elabSimpArgs___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_inc(x_1); -x_11 = l_Lean_getConstInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__13(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_getConstInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__13(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; @@ -6067,7 +6074,7 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Tactic_elabSimpArgs___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; @@ -6078,7 +6085,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -6123,7 +6130,7 @@ lean_dec(x_24); x_26 = lean_st_ref_take(x_5, x_25); x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -x_28 = lean_ctor_get(x_27, 4); +x_28 = lean_ctor_get(x_27, 5); lean_inc(x_28); x_29 = lean_ctor_get(x_26, 1); lean_inc(x_29); @@ -6132,7 +6139,7 @@ x_30 = !lean_is_exclusive(x_27); if (x_30 == 0) { lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_27, 4); +x_31 = lean_ctor_get(x_27, 5); lean_dec(x_31); x_32 = !lean_is_exclusive(x_28); if (x_32 == 0) @@ -6179,7 +6186,7 @@ x_46 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_46, 0, x_43); lean_ctor_set(x_46, 1, x_45); lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_42); -lean_ctor_set(x_27, 4, x_46); +lean_ctor_set(x_27, 5, x_46); x_47 = lean_st_ref_set(x_5, x_27, x_29); x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); @@ -6204,69 +6211,72 @@ return x_51; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; x_52 = lean_ctor_get(x_27, 0); x_53 = lean_ctor_get(x_27, 1); x_54 = lean_ctor_get(x_27, 2); x_55 = lean_ctor_get(x_27, 3); +x_56 = lean_ctor_get(x_27, 4); +lean_inc(x_56); lean_inc(x_55); lean_inc(x_54); lean_inc(x_53); lean_inc(x_52); lean_dec(x_27); -x_56 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); -x_57 = lean_ctor_get(x_28, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_28, 1); +x_57 = lean_ctor_get_uint8(x_28, sizeof(void*)*2); +x_58 = lean_ctor_get(x_28, 0); lean_inc(x_58); +x_59 = lean_ctor_get(x_28, 1); +lean_inc(x_59); if (lean_is_exclusive(x_28)) { lean_ctor_release(x_28, 0); lean_ctor_release(x_28, 1); - x_59 = x_28; + x_60 = x_28; } else { lean_dec_ref(x_28); - x_59 = lean_box(0); + x_60 = lean_box(0); } -x_60 = l_Std_PersistentArray_push___rarg(x_58, x_1); -if (lean_is_scalar(x_59)) { - x_61 = lean_alloc_ctor(0, 2, 1); +x_61 = l_Std_PersistentArray_push___rarg(x_59, x_1); +if (lean_is_scalar(x_60)) { + x_62 = lean_alloc_ctor(0, 2, 1); } else { - x_61 = x_59; -} -lean_ctor_set(x_61, 0, x_57); -lean_ctor_set(x_61, 1, x_60); -lean_ctor_set_uint8(x_61, sizeof(void*)*2, x_56); -x_62 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_62, 0, x_52); -lean_ctor_set(x_62, 1, x_53); -lean_ctor_set(x_62, 2, x_54); -lean_ctor_set(x_62, 3, x_55); -lean_ctor_set(x_62, 4, x_61); -x_63 = lean_st_ref_set(x_5, x_62, x_29); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; + x_62 = x_60; +} +lean_ctor_set(x_62, 0, x_58); +lean_ctor_set(x_62, 1, x_61); +lean_ctor_set_uint8(x_62, sizeof(void*)*2, x_57); +x_63 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_63, 0, x_52); +lean_ctor_set(x_63, 1, x_53); +lean_ctor_set(x_63, 2, x_54); +lean_ctor_set(x_63, 3, x_55); +lean_ctor_set(x_63, 4, x_56); +lean_ctor_set(x_63, 5, x_62); +x_64 = lean_st_ref_set(x_5, x_63, x_29); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_66 = x_64; } else { - lean_dec_ref(x_63); - x_65 = lean_box(0); + lean_dec_ref(x_64); + x_66 = lean_box(0); } -x_66 = lean_box(0); -if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 0); +x_67 = lean_box(0); +if (lean_is_scalar(x_66)) { + x_68 = lean_alloc_ctor(0, 2, 0); } else { - x_67 = x_65; + x_68 = x_66; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_64); -return x_67; +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_68, 1, x_65); +return x_68; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Tactic_elabSimpArgs___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; @@ -6277,7 +6287,7 @@ lean_dec(x_11); x_13 = lean_st_ref_get(x_5, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 4); +x_15 = lean_ctor_get(x_14, 5); lean_inc(x_15); lean_dec(x_14); x_16 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); @@ -6319,12 +6329,12 @@ x_24 = l_Lean_withoutModifyingState___at_Lean_Elab_Tactic_elabSimpConfigCore___s x_25 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_25, 0, x_1); lean_ctor_set(x_25, 1, x_24); -x_26 = l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__16(x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +x_26 = l_Lean_Elab_pushInfoTree___at_Lean_Elab_Tactic_elabSimpArgs___spec__16(x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); return x_26; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; @@ -6334,7 +6344,7 @@ lean_ctor_set(x_12, 1, x_11); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; @@ -6347,7 +6357,7 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_1); -x_12 = l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_12) == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; @@ -6363,7 +6373,7 @@ lean_dec(x_15); x_17 = lean_st_ref_get(x_6, x_16); x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); -x_19 = lean_ctor_get(x_18, 4); +x_19 = lean_ctor_get(x_18, 5); lean_inc(x_19); lean_dec(x_18); x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*2); @@ -6409,7 +6419,7 @@ x_25 = lean_ctor_get(x_17, 1); lean_inc(x_25); lean_dec(x_17); lean_inc(x_13); -x_26 = l_Lean_mkConstWithLevelParams___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__12(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_25); +x_26 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Tactic_elabSimpArgs___spec__12(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_25); if (lean_obj_tag(x_26) == 0) { lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; @@ -6432,7 +6442,7 @@ lean_ctor_set(x_33, 3, x_27); lean_ctor_set_uint8(x_33, sizeof(void*)*4, x_32); x_34 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_34, 0, x_33); -x_35 = l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__15(x_34, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_28); +x_35 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Tactic_elabSimpArgs___spec__15(x_34, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_28); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6531,7 +6541,7 @@ return x_47; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -6542,7 +6552,7 @@ lean_ctor_set(x_14, 1, x_12); return x_14; } } -static lean_object* _init_l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1() { +static lean_object* _init_l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1() { _start: { lean_object* x_1; @@ -6550,16 +6560,16 @@ x_1 = lean_mk_string_from_bytes("' does not have [simp] attribute", 32); return x_1; } } -static lean_object* _init_l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2() { +static lean_object* _init_l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1; +x_1 = l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { uint8_t x_12; @@ -6585,15 +6595,15 @@ lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean lean_dec(x_1); x_16 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_16, 0, x_2); -x_17 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; +x_17 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4; x_18 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_18, 0, x_17); lean_ctor_set(x_18, 1, x_16); -x_19 = l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2; +x_19 = l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2; x_20 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_20, 0, x_18); lean_ctor_set(x_20, 1, x_19); -x_21 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_21 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6625,7 +6635,7 @@ else { lean_object* x_26; lean_object* x_27; x_26 = lean_box(0); -x_27 = l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(x_1, x_2, x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_27 = l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(x_1, x_2, x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6641,7 +6651,7 @@ else { lean_object* x_28; lean_object* x_29; x_28 = lean_box(0); -x_29 = l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(x_1, x_2, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_29 = l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(x_1, x_2, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6657,7 +6667,7 @@ else { lean_object* x_30; lean_object* x_31; x_30 = lean_box(0); -x_31 = l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(x_1, x_2, x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_31 = l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(x_1, x_2, x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6670,7 +6680,7 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__18(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Tactic_elabSimpArgs___spec__18(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -6679,7 +6689,7 @@ x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1() { _start: { lean_object* x_1; @@ -6687,17 +6697,17 @@ x_1 = lean_mk_string_from_bytes("simpErase", 9); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_tacticToDischarge___closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1; +x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3() { _start: { lean_object* x_1; @@ -6705,17 +6715,17 @@ x_1 = lean_mk_string_from_bytes("simpLemma", 9); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_tacticToDischarge___closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3; +x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5() { _start: { lean_object* x_1; @@ -6723,17 +6733,17 @@ x_1 = lean_mk_string_from_bytes("simpStar", 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_tacticToDischarge___closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5; +x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7() { _start: { lean_object* x_1; @@ -6741,17 +6751,17 @@ x_1 = lean_mk_string_from_bytes("simpPost", 8); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_tacticToDischarge___closed__4; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7; +x_2 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; @@ -6802,19 +6812,19 @@ if (lean_is_exclusive(x_27)) { } lean_inc(x_19); x_33 = l_Lean_Syntax_getKind(x_19); -x_34 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2; +x_34 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2; x_35 = lean_name_eq(x_33, x_34); if (x_35 == 0) { lean_object* x_36; uint8_t x_37; -x_36 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4; +x_36 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4; x_37 = lean_name_eq(x_33, x_36); if (x_37 == 0) { lean_object* x_38; uint8_t x_39; lean_dec(x_28); lean_dec(x_19); -x_38 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6; +x_38 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6; x_39 = lean_name_eq(x_33, x_38); lean_dec(x_33); if (x_39 == 0) @@ -6832,7 +6842,7 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -x_40 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg(x_16); +x_40 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg(x_16); x_41 = !lean_is_exclusive(x_40); if (x_41 == 0) { @@ -6898,7 +6908,7 @@ lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; x_102 = l_Lean_Syntax_getArg(x_51, x_50); lean_dec(x_51); x_103 = l_Lean_Syntax_getKind(x_102); -x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8; +x_104 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8; x_105 = lean_name_eq(x_103, x_104); lean_dec(x_103); x_58 = x_105; @@ -6939,7 +6949,7 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_57); -x_60 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(x_57, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_60 = l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(x_57, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); if (lean_obj_tag(x_60) == 0) { lean_object* x_61; @@ -7249,7 +7259,7 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_114 = l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2(x_108, x_113, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_111); +x_114 = l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__2(x_108, x_113, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_111); if (lean_obj_tag(x_114) == 0) { lean_object* x_115; uint8_t x_116; @@ -7271,7 +7281,7 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_119 = l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17(x_30, x_117, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_118); +x_119 = l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17(x_30, x_117, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_118); if (lean_obj_tag(x_119) == 0) { lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; @@ -7418,7 +7428,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__20(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__20(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; @@ -7469,19 +7479,19 @@ if (lean_is_exclusive(x_27)) { } lean_inc(x_19); x_33 = l_Lean_Syntax_getKind(x_19); -x_34 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2; +x_34 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2; x_35 = lean_name_eq(x_33, x_34); if (x_35 == 0) { lean_object* x_36; uint8_t x_37; -x_36 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4; +x_36 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4; x_37 = lean_name_eq(x_33, x_36); if (x_37 == 0) { lean_object* x_38; uint8_t x_39; lean_dec(x_28); lean_dec(x_19); -x_38 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6; +x_38 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6; x_39 = lean_name_eq(x_33, x_38); lean_dec(x_33); if (x_39 == 0) @@ -7499,7 +7509,7 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -x_40 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg(x_16); +x_40 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg(x_16); x_41 = !lean_is_exclusive(x_40); if (x_41 == 0) { @@ -7565,7 +7575,7 @@ lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; x_102 = l_Lean_Syntax_getArg(x_51, x_50); lean_dec(x_51); x_103 = l_Lean_Syntax_getKind(x_102); -x_104 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8; +x_104 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8; x_105 = lean_name_eq(x_103, x_104); lean_dec(x_103); x_58 = x_105; @@ -7606,7 +7616,7 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_57); -x_60 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(x_57, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_60 = l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f(x_57, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); if (lean_obj_tag(x_60) == 0) { lean_object* x_61; @@ -7916,7 +7926,7 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_114 = l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2(x_108, x_113, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_111); +x_114 = l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__2(x_108, x_113, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_111); if (lean_obj_tag(x_114) == 0) { lean_object* x_115; uint8_t x_116; @@ -7938,7 +7948,7 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_119 = l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17(x_30, x_117, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_118); +x_119 = l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17(x_30, x_117, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_118); if (lean_obj_tag(x_119) == 0) { lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; @@ -8085,11 +8095,11 @@ goto _start; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__1(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___lambda__1(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { _start: { lean_object* x_21; -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +x_21 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); if (lean_obj_tag(x_21) == 0) { lean_object* x_22; lean_object* x_23; uint8_t x_24; @@ -8188,11 +8198,11 @@ return x_47; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__2(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___lambda__2(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { _start: { lean_object* x_21; -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__20(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +x_21 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__20(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); if (lean_obj_tag(x_21) == 0) { lean_object* x_22; lean_object* x_23; uint8_t x_24; @@ -8291,7 +8301,7 @@ return x_47; } } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs___closed__1() { _start: { lean_object* x_1; @@ -8299,7 +8309,7 @@ x_1 = lean_mk_string_from_bytes("Init.Util", 9); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs___closed__2() { _start: { lean_object* x_1; @@ -8307,7 +8317,7 @@ x_1 = lean_mk_string_from_bytes("getElem!", 8); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs___closed__3() { _start: { lean_object* x_1; @@ -8315,20 +8325,20 @@ x_1 = lean_mk_string_from_bytes("index out of bounds", 19); return x_1; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__1; -x_2 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_1 = l_Lean_Elab_Tactic_elabSimpArgs___closed__1; +x_2 = l_Lean_Elab_Tactic_elabSimpArgs___closed__2; +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); -x_5 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__3; +x_5 = l_Lean_Elab_Tactic_elabSimpArgs___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -static lean_object* _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed__const__1() { +static lean_object* _init_l_Lean_Elab_Tactic_elabSimpArgs___boxed__const__1() { _start: { size_t x_1; lean_object* x_2; @@ -8337,7 +8347,7 @@ x_2 = lean_box_usize(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { uint8_t x_14; @@ -8369,8 +8379,8 @@ lean_dec(x_26); if (x_22 == 0) { lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_28 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__4; -x_29 = l_panic___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__18(x_28); +x_28 = l_Lean_Elab_Tactic_elabSimpArgs___closed__4; +x_29 = l_panic___at_Lean_Elab_Tactic_elabSimpArgs___spec__18(x_28); x_30 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_30, 0, x_29); lean_ctor_set(x_30, 1, x_16); @@ -8382,8 +8392,8 @@ lean_ctor_set(x_33, 1, x_30); x_34 = lean_box(x_3); x_35 = lean_box(x_4); x_36 = lean_box_usize(x_27); -x_37 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed__const__1; -x_38 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__1___boxed), 20, 11); +x_37 = l_Lean_Elab_Tactic_elabSimpArgs___boxed__const__1; +x_38 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_elabSimpArgs___lambda__1___boxed), 20, 11); lean_closure_set(x_38, 0, x_2); lean_closure_set(x_38, 1, x_34); lean_closure_set(x_38, 2, x_35); @@ -8413,8 +8423,8 @@ lean_ctor_set(x_44, 1, x_41); x_45 = lean_box(x_3); x_46 = lean_box(x_4); x_47 = lean_box_usize(x_27); -x_48 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed__const__1; -x_49 = lean_alloc_closure((void*)(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__2___boxed), 20, 11); +x_48 = l_Lean_Elab_Tactic_elabSimpArgs___boxed__const__1; +x_49 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_elabSimpArgs___lambda__2___boxed), 20, 11); lean_closure_set(x_49, 0, x_2); lean_closure_set(x_49, 1, x_45); lean_closure_set(x_49, 2, x_46); @@ -8452,11 +8462,11 @@ return x_53; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -8468,11 +8478,11 @@ lean_dec(x_1); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8484,11 +8494,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_resolveGlobalName___at_Lean_Elab_Tactic_elabSimpArgs___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_resolveGlobalName___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_resolveGlobalName___at_Lean_Elab_Tactic_elabSimpArgs___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); @@ -8499,11 +8509,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8515,11 +8525,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Lean_resolveGlobalConstCore___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Lean_resolveGlobalConstCore___at_Lean_Elab_Tactic_elabSimpArgs___spec__7___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -8532,11 +8542,11 @@ lean_dec(x_3); return x_13; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8548,11 +8558,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_throwError___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__14(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_throwError___at_Lean_Elab_Tactic_elabSimpArgs___spec__14(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8564,11 +8574,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_getConstInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_getConstInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__13(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_getConstInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__13(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8580,11 +8590,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Elab_Tactic_elabSimpArgs___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_mkConstWithLevelParams___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_mkConstWithLevelParams___at_Lean_Elab_Tactic_elabSimpArgs___spec__12(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8596,11 +8606,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Tactic_elabSimpArgs___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_Elab_pushInfoTree___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__16(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_pushInfoTree___at_Lean_Elab_Tactic_elabSimpArgs___spec__16(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8612,11 +8622,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Tactic_elabSimpArgs___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_Elab_pushInfoLeaf___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__15(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_Elab_pushInfoLeaf___at_Lean_Elab_Tactic_elabSimpArgs___spec__15(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8628,11 +8638,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l_Lean_Elab_resolveGlobalConstNoOverloadWithInfo___at_Lean_Elab_Tactic_elabSimpArgs___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -8645,11 +8655,11 @@ lean_dec(x_2); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; -x_13 = l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -8662,7 +8672,7 @@ lean_dec(x_3); return x_13; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; size_t x_19; size_t x_20; lean_object* x_21; @@ -8674,13 +8684,13 @@ x_19 = lean_unbox_usize(x_5); lean_dec(x_5); x_20 = lean_unbox_usize(x_6); lean_dec(x_6); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19(x_1, x_17, x_18, x_4, x_19, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_21 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19(x_1, x_17, x_18, x_4, x_19, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_4); lean_dec(x_1); return x_21; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; size_t x_19; size_t x_20; lean_object* x_21; @@ -8692,13 +8702,13 @@ x_19 = lean_unbox_usize(x_5); lean_dec(x_5); x_20 = lean_unbox_usize(x_6); lean_dec(x_6); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__20(x_1, x_17, x_18, x_4, x_19, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_21 = l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__20(x_1, x_17, x_18, x_4, x_19, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_4); lean_dec(x_1); return x_21; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__1___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___lambda__1___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -8730,13 +8740,13 @@ x_23 = lean_unbox_usize(x_5); lean_dec(x_5); x_24 = lean_unbox_usize(x_6); lean_dec(x_6); -x_25 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__1(x_1, x_21, x_22, x_4, x_23, x_24, 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_25 = l_Lean_Elab_Tactic_elabSimpArgs___lambda__1(x_1, x_21, x_22, x_4, x_23, x_24, 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); lean_dec(x_4); lean_dec(x_1); return x_25; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__2___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___lambda__2___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -8768,13 +8778,13 @@ x_23 = lean_unbox_usize(x_5); lean_dec(x_5); x_24 = lean_unbox_usize(x_6); lean_dec(x_6); -x_25 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___lambda__2(x_1, x_21, x_22, x_4, x_23, x_24, 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_25 = l_Lean_Elab_Tactic_elabSimpArgs___lambda__2(x_1, x_21, x_22, x_4, x_23, x_24, 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); lean_dec(x_4); lean_dec(x_1); return x_25; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabSimpArgs___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { uint8_t x_14; uint8_t x_15; lean_object* x_16; @@ -8782,7 +8792,7 @@ x_14 = lean_unbox(x_3); lean_dec(x_3); x_15 = lean_unbox(x_4); lean_dec(x_4); -x_16 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs(x_1, x_2, x_14, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_16 = l_Lean_Elab_Tactic_elabSimpArgs(x_1, x_2, x_14, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_1); return x_16; } @@ -9437,7 +9447,7 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_31 = l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs(x_25, x_30, x_3, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_23); +x_31 = l_Lean_Elab_Tactic_elabSimpArgs(x_25, x_30, x_3, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_23); lean_dec(x_25); if (lean_obj_tag(x_31) == 0) { @@ -10108,7 +10118,7 @@ else lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_dec(x_2); x_17 = l_Lean_Elab_Tactic_mkSimpContext___lambda__3___closed__2; -x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -10190,7 +10200,7 @@ else lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_dec(x_17); x_25 = l_Lean_Elab_Tactic_mkSimpContext___closed__2; -x_26 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_26 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -12018,68 +12028,68 @@ lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDe l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___closed__4 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___closed__4(); lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_addDeclToUnfoldOrTheorem___closed__4); l_Lean_Elab_Tactic_ElabSimpArgsResult_starArg___default = _init_l_Lean_Elab_Tactic_ElabSimpArgsResult_starArg___default(); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4); -l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1); -l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2(); -lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2); -l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1 = _init_l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1(); -lean_mark_persistent(l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1); -l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2 = _init_l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2(); -lean_mark_persistent(l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2); -l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3 = _init_l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3(); -lean_mark_persistent(l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3); -l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4 = _init_l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4(); -lean_mark_persistent(l_Lean_throwUnknownConstant___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4); -l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1 = _init_l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1(); -lean_mark_persistent(l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1); -l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2 = _init_l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2(); -lean_mark_persistent(l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2); -l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3 = _init_l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3(); -lean_mark_persistent(l_Lean_resolveGlobalConst___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3); -l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1 = _init_l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1(); -lean_mark_persistent(l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1); -l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2 = _init_l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2(); -lean_mark_persistent(l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2); -l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3 = _init_l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3(); -lean_mark_persistent(l_Lean_resolveGlobalConstNoOverload___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3); -l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1 = _init_l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1(); -lean_mark_persistent(l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1); -l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2 = _init_l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2(); -lean_mark_persistent(l_Lean_Meta_SimpTheorems_erase___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__1 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__1(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__1); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__2 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__2(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__2); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__3 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__3(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__3); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__4 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__4(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___closed__4); -l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed__const__1 = _init_l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed__const__1(); -lean_mark_persistent(l___private_Lean_Elab_Tactic_Simp_0__Lean_Elab_Tactic_elabSimpArgs___boxed__const__1); +l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1 = _init_l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__1); +l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2 = _init_l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__2); +l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3 = _init_l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__3); +l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4 = _init_l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs_resolveSimpIdTheorem_x3f___closed__4); +l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__1); +l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2 = _init_l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2(); +lean_mark_persistent(l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_elabSimpArgs___spec__1___rarg___closed__2); +l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1(); +lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__1); +l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2(); +lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__2); +l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3(); +lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__3); +l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4 = _init_l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4(); +lean_mark_persistent(l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabSimpArgs___spec__9___closed__4); +l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1 = _init_l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1(); +lean_mark_persistent(l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__1); +l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2 = _init_l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2(); +lean_mark_persistent(l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__2); +l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3 = _init_l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3(); +lean_mark_persistent(l_Lean_resolveGlobalConst___at_Lean_Elab_Tactic_elabSimpArgs___spec__4___closed__3); +l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1 = _init_l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1(); +lean_mark_persistent(l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__1); +l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2 = _init_l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2(); +lean_mark_persistent(l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__2); +l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3 = _init_l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3(); +lean_mark_persistent(l_Lean_resolveGlobalConstNoOverload___at_Lean_Elab_Tactic_elabSimpArgs___spec__3___closed__3); +l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1 = _init_l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1(); +lean_mark_persistent(l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__1); +l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2 = _init_l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2(); +lean_mark_persistent(l_Lean_Meta_SimpTheorems_erase___at_Lean_Elab_Tactic_elabSimpArgs___spec__17___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__5); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__6); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__7); +l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_elabSimpArgs___spec__19___closed__8); +l_Lean_Elab_Tactic_elabSimpArgs___closed__1 = _init_l_Lean_Elab_Tactic_elabSimpArgs___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs___closed__1); +l_Lean_Elab_Tactic_elabSimpArgs___closed__2 = _init_l_Lean_Elab_Tactic_elabSimpArgs___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs___closed__2); +l_Lean_Elab_Tactic_elabSimpArgs___closed__3 = _init_l_Lean_Elab_Tactic_elabSimpArgs___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs___closed__3); +l_Lean_Elab_Tactic_elabSimpArgs___closed__4 = _init_l_Lean_Elab_Tactic_elabSimpArgs___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs___closed__4); +l_Lean_Elab_Tactic_elabSimpArgs___boxed__const__1 = _init_l_Lean_Elab_Tactic_elabSimpArgs___boxed__const__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_elabSimpArgs___boxed__const__1); l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_mkSimpContext___spec__1___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_mkSimpContext___spec__1___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_mkSimpContext___spec__1___closed__1); l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_mkSimpContext___spec__1___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_mkSimpContext___spec__1___closed__2(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/Split.c b/stage0/stdlib/Lean/Elab/Tactic/Split.c index 2331f6d62867..c46692f23046 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Split.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Split.c @@ -37,20 +37,16 @@ static lean_object* l_Lean_Elab_Tactic_evalSplit___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSplit_declRange___closed__5; lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__6___closed__3; -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalSplit___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSplit___closed__14; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Tactic_evalSplit___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* l_Lean_Elab_Tactic_expandOptLocation(lean_object*); static lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__5___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSplit___closed__7; -lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* l_Lean_Meta_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSplit_declRange___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSplit_declRange(lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalSplit___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalSplit___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSplit_declRange___closed__2; -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -61,6 +57,7 @@ lean_object* l_Lean_Meta_splitLocalDecl_x3f(lean_object*, lean_object*, lean_obj extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSplit___closed__1; +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___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___regBuiltin_Lean_Elab_Tactic_evalSplit___closed__13; static lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__5___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSplit___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*); @@ -78,6 +75,7 @@ static lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__1___closed__2; uint8_t l_Lean_Syntax_isNone(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalSplit_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__1___closed__3; lean_object* l_Lean_Elab_Tactic_replaceMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__5___closed__5; @@ -251,68 +249,6 @@ return x_40; } } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalSplit___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; -x_12 = !lean_is_exclusive(x_9); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_9, 5); -x_14 = l_Lean_replaceRef(x_1, x_13); -lean_dec(x_13); -lean_ctor_set(x_9, 5, x_14); -x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_16 = lean_ctor_get(x_9, 0); -x_17 = lean_ctor_get(x_9, 1); -x_18 = lean_ctor_get(x_9, 2); -x_19 = lean_ctor_get(x_9, 3); -x_20 = lean_ctor_get(x_9, 4); -x_21 = lean_ctor_get(x_9, 5); -x_22 = lean_ctor_get(x_9, 6); -x_23 = lean_ctor_get(x_9, 7); -x_24 = lean_ctor_get(x_9, 8); -x_25 = lean_ctor_get(x_9, 9); -x_26 = lean_ctor_get(x_9, 10); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -lean_inc(x_20); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_9); -x_27 = l_Lean_replaceRef(x_1, x_21); -lean_dec(x_21); -x_28 = lean_alloc_ctor(0, 11, 0); -lean_ctor_set(x_28, 0, x_16); -lean_ctor_set(x_28, 1, x_17); -lean_ctor_set(x_28, 2, x_18); -lean_ctor_set(x_28, 3, x_19); -lean_ctor_set(x_28, 4, x_20); -lean_ctor_set(x_28, 5, x_27); -lean_ctor_set(x_28, 6, x_22); -lean_ctor_set(x_28, 7, x_23); -lean_ctor_set(x_28, 8, x_24); -lean_ctor_set(x_28, 9, x_25); -lean_ctor_set(x_28, 10, x_26); -x_29 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_28, x_10, x_11); -lean_dec(x_28); -return x_29; -} -} -} static lean_object* _init_l_Lean_Elab_Tactic_evalSplit___lambda__1___closed__1() { _start: { @@ -1190,7 +1126,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_evalSplit___lambda__5___closed__4() lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Tactic_evalSplit___lambda__5___closed__1; x_2 = l_Lean_Elab_Tactic_evalSplit___lambda__5___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Elab_Tactic_evalSplit___lambda__5___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1414,15 +1350,7 @@ goto block_26; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_dec(x_19); x_20 = l_Lean_Elab_Tactic_evalSplit___lambda__6___closed__3; -x_21 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalSplit___spec__2(x_13, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_13); +x_21 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalTactic___spec__1(x_13, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); x_22 = !lean_is_exclusive(x_21); if (x_22 == 0) { @@ -1475,7 +1403,7 @@ if (x_13 == 0) lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_dec(x_1); x_14 = l_Lean_Elab_Tactic_evalSplit___closed__2; -x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_15 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -1525,22 +1453,6 @@ lean_dec(x_3); return x_14; } } -LEAN_EXPORT lean_object* l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalSplit___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l_Lean_throwErrorAt___at_Lean_Elab_Tactic_evalSplit___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_12; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_evalSplit___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { diff --git a/stage0/stdlib/Lean/Elab/Tactic/Unfold.c b/stage0/stdlib/Lean/Elab/Tactic/Unfold.c index d38fc28a5037..707f74b54e31 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Unfold.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Unfold.c @@ -58,7 +58,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange___close lean_object* lean_format_pretty(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold_declRange___closed__7; -lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_unfoldTarget(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_evalUnfold___closed__6; @@ -75,6 +74,7 @@ static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__3; size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_Elab_Tactic_evalUnfold_go___lambda__1___closed__4; extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; +lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_throwTacticEx___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_unfoldLocalDecl(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_evalUnfold_go___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -536,7 +536,7 @@ x_16 = l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_evalUnfold_go___spec__7 x_17 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_refineCore___spec__1(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_18 = l_Lean_throwError___at_Lean_Elab_Tactic_evalTactic___spec__2(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_18; } } diff --git a/stage0/stdlib/Lean/Elab/Term.c b/stage0/stdlib/Lean/Elab/Term.c index d9a8cced7dab..2458ffe74bdd 100644 --- a/stage0/stdlib/Lean/Elab/Term.c +++ b/stage0/stdlib/Lean/Elab/Term.c @@ -31,8 +31,10 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImpli static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFns___closed__5; LEAN_EXPORT lean_object* l_Lean_addDocString___at_Lean_Elab_Term_expandDeclId___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___lambda__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__10; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__4; LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__6___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___closed__1; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__5___closed__4; @@ -44,6 +46,7 @@ lean_object* l_Lean_extractMacroScopes(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutAutoBoundImplicit(lean_object*); static lean_object* l_Lean_Elab_Term_instToStringMVarErrorKind___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_instMetaEvalTermElabM___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_RBNode_insert___at_Lean_Elab_Term_registerSyntheticMVar___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -67,6 +70,7 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBound LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicitApp___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_commitIfNoErrors_x3f(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__2; LEAN_EXPORT lean_object* l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_tryCoeThunk_x3f___closed__3; static lean_object* l_Lean_logTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__1___closed__1; @@ -105,7 +109,6 @@ static lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___closed__16; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__9; lean_object* l_Lean_LocalDecl_userName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_autoLift; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutPending(lean_object*); static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instAddErrorMessageContextTermElabM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_State_infoState___default___closed__3; @@ -176,6 +179,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName_loop___boxed(lean_obj static lean_object* l_Lean_localDeclDependsOn___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFnsAux___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__5(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SourceInfo_fromRef(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_commitIfDidNotPostpone___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -193,11 +197,13 @@ static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMe static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__48___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_addTermInfo___boxed(lean_object*, lean_object*, lean_object*, lean_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_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__1; static lean_object* l_Lean_Elab_Term_instInhabitedLetRecToLift___closed__7; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_synthesizeInst___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedTermElabResult___rarg(lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__1; static lean_object* l_Lean_Elab_Term_instMonadTermElabM___closed__5; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkCoe___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isMonadApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg(lean_object*); @@ -218,7 +224,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isLambdaWithImplicit(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicit(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__12(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__2; static lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_throwAutoBoundImplicitLocal___at_Lean_Elab_Term_resolveName_process___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__4; @@ -251,7 +256,6 @@ lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkCoe___closed__1; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__36___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_expandDeclId___spec__13(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_throwErrorIfErrors___closed__2; @@ -293,7 +297,6 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLam static lean_object* l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_getMVarDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__22(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__4; static lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___closed__12; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_collectUnassignedMVars_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTerm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -314,7 +317,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_synthesize LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ensureType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -373,6 +375,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___rarg(lean_object*, lean LEAN_EXPORT lean_object* l_Lean_Elab_Term_withLevelNames___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_expandDeclId___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedTermElabM(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_State_pendingMVars___default; LEAN_EXPORT lean_object* l_Lean_Elab_Term_collectUnassignedMVars_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_101_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -394,6 +397,7 @@ LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Elab_Term_resolveId_x3f___spe static lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__13; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwTypeMismatchError___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabUsingElabFns(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Elab_Term_getSyntheticMVarDecl_x3f___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkCoe___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkAppOptM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___closed__6; @@ -418,6 +422,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAuxDecl___rarg(lean_object*, lean_ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicit___closed__1; lean_object* l_Std_PersistentArray_foldlM___at___private_Lean_Util_Trace_0__Lean_withNestedTracesFinalizer___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwTypeMismatchError___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__1; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___lambda__1___closed__6; LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -432,7 +437,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDecl LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwErrorIfErrors___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_isLetRecAuxMVar___closed__4; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__16; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_expandDeclId___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1___closed__2; @@ -440,11 +445,12 @@ extern lean_object* l_Lean_maxRecDepth; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isTacticOrPostponedHole_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4___closed__2; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__5___closed__2; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__2; lean_object* l_Lean_mkAppN(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambda_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instToStringMVarErrorKind___boxed(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__3; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_decorateErrorMessageWithLambdaImplicitVars___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_LVal_getRef___boxed(lean_object*); static lean_object* l_Lean_Elab_Term_instInhabitedTermElabM___closed__1; @@ -470,7 +476,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_expandDeclId___at_Lean_Elab_Term_expandDecl static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isExplicitApp___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveName___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_expandDeclId___spec__4___closed__1; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__4; LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_mkConsts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadTermElabM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__4(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -491,6 +496,7 @@ LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__5___closed__1; lean_object* l_Std_RBNode_setBlack___rarg(lean_object*); static lean_object* l_Lean_Elab_Term_instMonadTermElabM___closed__4; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__1; LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Lean_Elab_Term_resolveLocalName___spec__6(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2(lean_object*); @@ -528,6 +534,7 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isNoImplicitLam LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Elab_Term_getFVarLocalDecl_x21___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_observing___rarg___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__52(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withMacroExpansionInfo___at_Lean_Elab_Term_withMacroExpansion___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedTermElabM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -559,13 +566,12 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(lean_object*, LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedCache; lean_object* l_Lean_MetavarContext_levelMVarToParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerCustomErrorIfMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__4; lean_object* l_Lean_Option_get___at_Std_Format_pretty_x27___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__14; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLocalIdent_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___closed__3; +LEAN_EXPORT lean_object* l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkConst___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_markUsedAssignment___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -655,7 +661,6 @@ LEAN_EXPORT lean_object* l_Lean_MessageLog_forM___at_Lean_Elab_Term_instMetaEval LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___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* l_Std_mkHashMapImp___rarg(lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__29(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam_x27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkCoe___closed__3; static lean_object* l_Lean_Elab_Term_instMonadBacktrackSavedStateTermElabM___closed__2; @@ -663,10 +668,9 @@ static lean_object* l_Lean_Elab_Term_mkTypeMismatchError___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_blockImplicitLambda___boxed(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___closed__1; static lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___closed__7; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_blockImplicitLambda(lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_exceptionToSorry(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -700,10 +704,10 @@ lean_object* l_Lean_Core_getMessageLog___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__28(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_commitIfDidNotPostpone(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_2191_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_2187_(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkAuxName___at_Lean_Elab_Term_mkAuxName___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_setElabConfig(lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__14; @@ -719,6 +723,7 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___la LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__1; static lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__22; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___lambda__1___closed__9; extern lean_object* l_Lean_Expr_instHashableExpr; @@ -729,6 +734,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkTypeMismatchError(lean_object*, lean LEAN_EXPORT lean_object* l_Lean_Elab_throwPostpone___at_Lean_Elab_Term_tryPostpone___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__33___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_State_levelNames___default; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadBacktrackSavedStateTermElabM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___lambda__1___closed__4; lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); @@ -742,6 +748,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_collectUn LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLetRecAuxMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__3; lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_Context_errToSorry___default; LEAN_EXPORT lean_object* l_Lean_getDelayedMVarRoot___at_Lean_Elab_Term_isLetRecAuxMVar___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -752,7 +759,8 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___closed LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadMacroAdapterTermElabM___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_abortTermExceptionId; LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__4; +LEAN_EXPORT lean_object* l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*, lean_object*); lean_object* l_Lean_Meta_throwAppTypeMismatch___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_expandDeclId___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -767,6 +775,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkInstMVar___lambda__1(lean_object*, l lean_object* l_Lean_printTraces___at_Lean_Core_instMetaEvalCoreM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___lambda__1___closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isHole___closed__4; @@ -806,8 +815,6 @@ extern lean_object* l_Lean_firstFrontendMacroScope; static uint8_t l_Lean_Elab_Term_collectUnassignedMVars_go___closed__1; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__8(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withAutoBoundImplicitForbiddenPred(lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__2; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__3; extern lean_object* l_Lean_Meta_instAlternativeMetaM; lean_object* l_Lean_Elab_mkElabAttribute___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_getResetInfoTrees___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -822,6 +829,7 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___la LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___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_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__42___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_withLogging___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_checkMaxHeartbeats(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_isTacticOrPostponedHole_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -843,7 +851,6 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Term_Context_isNoncomputableSection___default; static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_Context_implicitLambda___default; -LEAN_EXPORT uint8_t l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___lambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_resolveName_process___closed__1; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__1___closed__1; static lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___closed__13; @@ -879,9 +886,11 @@ LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0_ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTerm___closed__4; LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__3; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__47___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_BinderInfo_isImplicit(uint8_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkConst(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_dropTermParens___closed__2; lean_object* l_Lean_LocalDecl_fvarId(lean_object*); @@ -901,12 +910,14 @@ static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__13; LEAN_EXPORT lean_object* l_Lean_mkAuxName___at_Lean_Elab_Term_mkAuxName___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__12; +LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedSyntheticMVarKind; LEAN_EXPORT lean_object* l_Lean_Elab_Term_termElabAttribute; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__1(lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_Term_Context_sectionVars___default; static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__2; static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__3; lean_object* l_Std_PersistentArray_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__7___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_getDeclName_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -918,6 +929,7 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBound LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedCacheKey; LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_instMetaEvalTermElabM___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveLocalName___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_applyVisibility___at_Lean_Elab_Term_expandDeclId___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___private_Lean_Elab_Term_0__Lean_Elab_Term_dropTermParens___closed__1; @@ -932,6 +944,7 @@ static lean_object* l_Lean_Elab_Term_isLetRecAuxMVar___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__17; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_DocString_0__Lean_removeLeadingSpaces(lean_object*); static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__10; static lean_object* l_List_foldl___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__2___closed__2; static lean_object* l_Lean_Elab_Term_getFVarLocalDecl_x21___closed__4; @@ -943,11 +956,12 @@ lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_isAutoBoundImplicitLocalException_x3f(lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__4; lean_object* l_Lean_Meta_getMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Elab_pushInfoTree___at_Lean_Elab_Term_addDotCompletionInfo___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698____boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_findSomeRevMAux___at_Lean_Elab_Term_resolveLocalName___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__40(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_instMetaEvalTermElabM___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -964,7 +978,6 @@ static lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__18; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind___boxed(lean_object*); extern lean_object* l_Lean_instInhabitedTraceElem; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__3; -lean_object* l_List_find_x3f___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMonadBacktrackSavedStateTermElabM; LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -982,7 +995,6 @@ LEAN_EXPORT uint8_t l_Lean_Elab_Term_LVal_isFieldName(lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___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_Elab_Term_withoutSavingRecAppSyntax___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694____boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_traceAtCmdPos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_postponeExceptionId; @@ -990,7 +1002,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_throwPostpone___at_Lean_Elab_Term_tryPostpo lean_object* lean_environment_main_module(lean_object*); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__9; uint8_t lean_expr_eqv(lean_object*, lean_object*); -LEAN_EXPORT uint64_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694_(lean_object*); +LEAN_EXPORT uint64_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Elab_Term_addAutoBoundImplicits_x27___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambda_loop(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___lambda__3(lean_object*); @@ -1003,6 +1015,7 @@ uint8_t l_Lean_Expr_isMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_logUnassignedUsingErrorInfos___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__6(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__15; static lean_object* l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__1; @@ -1023,6 +1036,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_withMacroExpansion___rarg___lambda__1( LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_SavedState_restore(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__4; +static lean_object* l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl___closed__1; static lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Term_0__Lean_Elab_Term_isLambdaWithImplicit___spec__1___closed__1; static lean_object* l_Lean_Elab_Term_instInhabitedTermElabM___closed__2; extern lean_object* l_Lean_KVMap_empty; @@ -1043,7 +1058,7 @@ static lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Term_0__Lean LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_State_infoState___default___closed__2; static lean_object* l_Lean_Elab_Term_resolveName_x27___closed__2; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambda___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_applyAttributes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveId_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1056,7 +1071,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorCustomInfo(lean_objec LEAN_EXPORT lean_object* l_Lean_Elab_Term_isTypeApp_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__10; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambda_loop___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabTerm___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__32(lean_object*, lean_object*, size_t, size_t); @@ -1108,11 +1123,11 @@ LEAN_EXPORT lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_ex LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_withSavedContext___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore(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_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___closed__1; static lean_object* l_Lean_Elab_Term_mkTypeMismatchError___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_adaptExpander(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_logTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_tryPostponeIfMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1159,12 +1174,14 @@ lean_object* l_Std_HashMap_insert___at_Lean_Meta_ToHide_visitVisibleExpr_visit__ static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__9; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__18___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); +LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instBEqCacheKey; lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___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*); static lean_object* l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__3; +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Elab_Term_getSyntheticMVarDecl_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapMAux___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__3___closed__2; LEAN_EXPORT uint8_t l_Lean_Elab_Term_Context_ignoreTCFailures___default; @@ -1177,26 +1194,25 @@ static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term_0__L LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_resolveName_x27___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_mkDeclName___at_Lean_Elab_Term_expandDeclId___spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_addAutoBoundImplicits_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static uint32_t l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__4; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_collectUnassignedMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Elab_Term_0__Lean_Elab_Term_isLambdaWithImplicit___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__1; static lean_object* l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_checkNotAlreadyDeclared___at_Lean_Elab_Term_expandDeclId___spec__6___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFreshLevelMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isLambdaWithImplicit___closed__3; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__25(lean_object*, lean_object*, size_t, size_t); -static lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__2; static lean_object* l_Lean_Elab_Term_mkExplicitBinder___closed__1; uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabImplicitLambdaAux(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_logUnassignedUsingErrorInfos(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_Term_0__Lean_Elab_Term_mkSyntheticSorryFor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_instInhabitedState; @@ -1241,8 +1257,8 @@ LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_ContainsPen lean_object* l_Lean_indentD(lean_object*); extern lean_object* l_Lean_Elab_unsupportedSyntaxExceptionId; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_resolveId_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___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorImplicitArgInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock___closed__6; lean_object* l_Lean_Meta_mkFreshTypeMVar(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1265,14 +1281,13 @@ LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Elab_Term_addTermInfo___spec__ LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwErrorIfErrors(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_logTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__1___closed__5; LEAN_EXPORT lean_object* l_Lean_getDelayedMVarAssignment_x3f___at_Lean_Elab_Term_isLetRecAuxMVar___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920_(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_addAutoBoundImplicits(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Term_exprToSyntax(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623____boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_instMetaEvalTermElabM___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_withoutModifyingStateWithInfoAndMessages___rarg(lean_object*, lean_object*, lean_object*); @@ -1310,8 +1325,6 @@ lean_object* l_Lean_MetavarContext_getDecl(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__2; uint8_t l_Std_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__2___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_resetMessageLog(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1332,6 +1345,7 @@ lean_object* lean_local_ctx_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_resolveId_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__13; LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Elab_Term_ContainsPendingMVar_visit___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__52___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe(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_Elab_isFreshInstanceName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError(lean_object*); @@ -1345,7 +1359,6 @@ LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at_Lean_Elab_Term_addAutoB static lean_object* l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___closed__9; static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__14; static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoeSort___closed__4; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_withInfoTreeContext___at_Lean_Elab_Term_withMacroExpansion___spec__2(lean_object*); lean_object* l_Lean_TagDeclarationExtension_tag(lean_object*, lean_object*, lean_object*); lean_object* l_panic___at___private_Lean_Util_Trace_0__Lean_withNestedTracesFinalizer___spec__6(lean_object*); @@ -1376,7 +1389,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeCoeInstMVarCore(lean_object* LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__16(lean_object*, lean_object*, size_t, size_t); static lean_object* l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__12; LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__38(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutPending___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorCustomInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_tryCoeThunk_x3f___closed__4; LEAN_EXPORT lean_object* l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1___boxed(lean_object*, lean_object*); @@ -1390,6 +1402,7 @@ static lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMe static lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__4; static lean_object* l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLocalIdent_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_isTacticBlock___closed__4; lean_object* l_Lean_mkSimpleThunk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1480,13 +1493,20 @@ static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTer LEAN_EXPORT lean_object* l_Lean_localDeclDependsOn___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_expandDeclId___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_postponeElabTerm___closed__5; -static lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_Context_mayPostpone___default; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__33(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeInstMVarCore___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* _init_l_Lean_Elab_Term_instInhabitedSyntheticMVarKind() { +_start: +{ +lean_object* x_1; +x_1 = lean_box(0); +return x_1; +} +} static lean_object* _init_l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__1() { _start: { @@ -1559,6 +1579,26 @@ lean_dec(x_1); return x_2; } } +static lean_object* _init_l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = lean_box(0); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl___closed__1; +return x_1; +} +} static lean_object* _init_l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__1() { _start: { @@ -1810,6 +1850,14 @@ x_1 = lean_box(0); return x_1; } } +static lean_object* _init_l_Lean_Elab_Term_State_pendingMVars___default() { +_start: +{ +lean_object* x_1; +x_1 = lean_box(0); +return x_1; +} +} static lean_object* _init_l_Lean_Elab_Term_State_mvarErrorInfos___default() { _start: { @@ -1917,12 +1965,13 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(0); x_2 = lean_box(0); x_3 = l_Lean_Elab_Term_instInhabitedState___closed__1; -x_4 = lean_alloc_ctor(0, 5, 0); +x_4 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_1); -lean_ctor_set(x_4, 2, x_2); -lean_ctor_set(x_4, 3, x_1); -lean_ctor_set(x_4, 4, x_3); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_1); +lean_ctor_set(x_4, 3, x_2); +lean_ctor_set(x_4, 4, x_1); +lean_ctor_set(x_4, 5, x_3); return x_4; } } @@ -2231,12 +2280,13 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(0); x_2 = lean_box(0); x_3 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__21; -x_4 = lean_alloc_ctor(0, 5, 0); +x_4 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_1); -lean_ctor_set(x_4, 3, x_2); -lean_ctor_set(x_4, 4, x_3); +lean_ctor_set(x_4, 1, x_1); +lean_ctor_set(x_4, 2, x_2); +lean_ctor_set(x_4, 3, x_1); +lean_ctor_set(x_4, 4, x_2); +lean_ctor_set(x_4, 5, x_3); return x_4; } } @@ -2266,7 +2316,7 @@ x_1 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__23; return x_1; } } -LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(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; @@ -2289,11 +2339,11 @@ return x_9; } } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623_(x_1, x_2); +x_3 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -2304,7 +2354,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_instBEqCacheKey___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_623____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_beqCacheKey____x40_Lean_Elab_Term___hyg_627____boxed), 2, 0); return x_1; } } @@ -2316,7 +2366,7 @@ x_1 = l_Lean_Elab_Tactic_instBEqCacheKey___closed__1; return x_1; } } -LEAN_EXPORT uint64_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694_(lean_object* x_1) { +LEAN_EXPORT uint64_t l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint64_t x_4; uint64_t x_5; uint64_t x_6; uint64_t x_7; uint64_t x_8; @@ -2330,11 +2380,11 @@ x_8 = lean_uint64_mix_hash(x_6, x_7); return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694____boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698____boxed(lean_object* x_1) { _start: { uint64_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694_(x_1); +x_2 = l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698_(x_1); lean_dec(x_1); x_3 = lean_box_uint64(x_2); return x_3; @@ -2344,7 +2394,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_instHashableCacheKey___closed__1() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_694____boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Elab_Term_0__Lean_Elab_Tactic_hashCacheKey____x40_Lean_Elab_Term___hyg_698____boxed), 1, 0); return x_1; } } @@ -2924,7 +2974,7 @@ lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 4); +x_19 = lean_ctor_get(x_17, 5); lean_inc(x_19); lean_dec(x_17); x_20 = lean_ctor_get(x_1, 0); @@ -2978,9 +3028,9 @@ x_40 = !lean_is_exclusive(x_38); if (x_40 == 0) { lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_41 = lean_ctor_get(x_38, 4); +x_41 = lean_ctor_get(x_38, 5); lean_dec(x_41); -lean_ctor_set(x_38, 4, x_19); +lean_ctor_set(x_38, 5, x_19); x_42 = lean_st_ref_set(x_4, x_38, x_39); x_43 = !lean_is_exclusive(x_42); if (x_43 == 0) @@ -3007,183 +3057,190 @@ return x_48; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; x_49 = lean_ctor_get(x_38, 0); x_50 = lean_ctor_get(x_38, 1); x_51 = lean_ctor_get(x_38, 2); x_52 = lean_ctor_get(x_38, 3); +x_53 = lean_ctor_get(x_38, 4); +lean_inc(x_53); lean_inc(x_52); lean_inc(x_51); lean_inc(x_50); lean_inc(x_49); lean_dec(x_38); -x_53 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_53, 0, x_49); -lean_ctor_set(x_53, 1, x_50); -lean_ctor_set(x_53, 2, x_51); -lean_ctor_set(x_53, 3, x_52); -lean_ctor_set(x_53, 4, x_19); -x_54 = lean_st_ref_set(x_4, x_53, x_39); -x_55 = lean_ctor_get(x_54, 1); -lean_inc(x_55); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_56 = x_54; +x_54 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_54, 0, x_49); +lean_ctor_set(x_54, 1, x_50); +lean_ctor_set(x_54, 2, x_51); +lean_ctor_set(x_54, 3, x_52); +lean_ctor_set(x_54, 4, x_53); +lean_ctor_set(x_54, 5, x_19); +x_55 = lean_st_ref_set(x_4, x_54, x_39); +x_56 = lean_ctor_get(x_55, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_57 = x_55; } else { - lean_dec_ref(x_54); - x_56 = lean_box(0); + lean_dec_ref(x_55); + x_57 = lean_box(0); } -x_57 = lean_box(0); -if (lean_is_scalar(x_56)) { - x_58 = lean_alloc_ctor(0, 2, 0); +x_58 = lean_box(0); +if (lean_is_scalar(x_57)) { + x_59 = lean_alloc_ctor(0, 2, 0); } else { - x_58 = x_56; + x_59 = x_57; } -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_55); -return x_58; +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_56); +return x_59; } } else { -uint8_t x_59; +uint8_t x_60; lean_dec(x_19); -x_59 = !lean_is_exclusive(x_33); -if (x_59 == 0) +x_60 = !lean_is_exclusive(x_33); +if (x_60 == 0) { -lean_object* x_60; lean_object* x_61; -x_60 = lean_ctor_get(x_33, 0); -lean_dec(x_60); -x_61 = lean_box(0); -lean_ctor_set(x_33, 0, x_61); +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_33, 0); +lean_dec(x_61); +x_62 = lean_box(0); +lean_ctor_set(x_33, 0, x_62); return x_33; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_33, 1); -lean_inc(x_62); +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_33, 1); +lean_inc(x_63); lean_dec(x_33); -x_63 = lean_box(0); -x_64 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_62); -return x_64; +x_64 = lean_box(0); +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_63); +return x_65; } } } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_65 = lean_ctor_get(x_29, 0); -x_66 = lean_ctor_get(x_29, 1); -x_67 = lean_ctor_get(x_29, 2); -x_68 = lean_ctor_get(x_29, 4); -x_69 = lean_ctor_get(x_29, 5); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_66 = lean_ctor_get(x_29, 0); +x_67 = lean_ctor_get(x_29, 1); +x_68 = lean_ctor_get(x_29, 2); +x_69 = lean_ctor_get(x_29, 4); +x_70 = lean_ctor_get(x_29, 5); +lean_inc(x_70); lean_inc(x_69); lean_inc(x_68); lean_inc(x_67); lean_inc(x_66); -lean_inc(x_65); lean_dec(x_29); -x_70 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_70, 0, x_65); -lean_ctor_set(x_70, 1, x_66); -lean_ctor_set(x_70, 2, x_67); -lean_ctor_set(x_70, 3, x_13); -lean_ctor_set(x_70, 4, x_68); -lean_ctor_set(x_70, 5, x_69); -x_71 = lean_st_ref_set(x_8, x_70, x_30); +x_71 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_71, 0, x_66); +lean_ctor_set(x_71, 1, x_67); +lean_ctor_set(x_71, 2, x_68); +lean_ctor_set(x_71, 3, x_13); +lean_ctor_set(x_71, 4, x_69); +lean_ctor_set(x_71, 5, x_70); +x_72 = lean_st_ref_set(x_8, x_71, x_30); if (x_2 == 0) { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -lean_dec(x_71); -x_73 = lean_st_ref_get(x_8, x_72); -x_74 = lean_ctor_get(x_73, 1); -lean_inc(x_74); -lean_dec(x_73); -x_75 = lean_st_ref_take(x_4, x_74); -x_76 = lean_ctor_get(x_75, 0); -lean_inc(x_76); -x_77 = lean_ctor_get(x_75, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +lean_dec(x_72); +x_74 = lean_st_ref_get(x_8, x_73); +x_75 = lean_ctor_get(x_74, 1); +lean_inc(x_75); +lean_dec(x_74); +x_76 = lean_st_ref_take(x_4, x_75); +x_77 = lean_ctor_get(x_76, 0); lean_inc(x_77); -lean_dec(x_75); -x_78 = lean_ctor_get(x_76, 0); +x_78 = lean_ctor_get(x_76, 1); lean_inc(x_78); -x_79 = lean_ctor_get(x_76, 1); +lean_dec(x_76); +x_79 = lean_ctor_get(x_77, 0); lean_inc(x_79); -x_80 = lean_ctor_get(x_76, 2); +x_80 = lean_ctor_get(x_77, 1); lean_inc(x_80); -x_81 = lean_ctor_get(x_76, 3); +x_81 = lean_ctor_get(x_77, 2); lean_inc(x_81); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - lean_ctor_release(x_76, 2); - lean_ctor_release(x_76, 3); - lean_ctor_release(x_76, 4); - x_82 = x_76; -} else { - lean_dec_ref(x_76); - x_82 = lean_box(0); -} -if (lean_is_scalar(x_82)) { - x_83 = lean_alloc_ctor(0, 5, 0); -} else { - x_83 = x_82; -} -lean_ctor_set(x_83, 0, x_78); -lean_ctor_set(x_83, 1, x_79); -lean_ctor_set(x_83, 2, x_80); -lean_ctor_set(x_83, 3, x_81); -lean_ctor_set(x_83, 4, x_19); -x_84 = lean_st_ref_set(x_4, x_83, x_77); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_86 = x_84; +x_82 = lean_ctor_get(x_77, 3); +lean_inc(x_82); +x_83 = lean_ctor_get(x_77, 4); +lean_inc(x_83); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + lean_ctor_release(x_77, 2); + lean_ctor_release(x_77, 3); + lean_ctor_release(x_77, 4); + lean_ctor_release(x_77, 5); + x_84 = x_77; } else { - lean_dec_ref(x_84); - x_86 = lean_box(0); + lean_dec_ref(x_77); + x_84 = lean_box(0); } -x_87 = lean_box(0); -if (lean_is_scalar(x_86)) { - x_88 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_84)) { + x_85 = lean_alloc_ctor(0, 6, 0); } else { + x_85 = x_84; +} +lean_ctor_set(x_85, 0, x_79); +lean_ctor_set(x_85, 1, x_80); +lean_ctor_set(x_85, 2, x_81); +lean_ctor_set(x_85, 3, x_82); +lean_ctor_set(x_85, 4, x_83); +lean_ctor_set(x_85, 5, x_19); +x_86 = lean_st_ref_set(x_4, x_85, x_78); +x_87 = lean_ctor_get(x_86, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); x_88 = x_86; +} else { + lean_dec_ref(x_86); + x_88 = lean_box(0); +} +x_89 = lean_box(0); +if (lean_is_scalar(x_88)) { + x_90 = lean_alloc_ctor(0, 2, 0); +} else { + x_90 = x_88; } -lean_ctor_set(x_88, 0, x_87); -lean_ctor_set(x_88, 1, x_85); -return x_88; +lean_ctor_set(x_90, 0, x_89); +lean_ctor_set(x_90, 1, x_87); +return x_90; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_dec(x_19); -x_89 = lean_ctor_get(x_71, 1); -lean_inc(x_89); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_90 = x_71; +x_91 = lean_ctor_get(x_72, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_92 = x_72; } else { - lean_dec_ref(x_71); - x_90 = lean_box(0); + lean_dec_ref(x_72); + x_92 = lean_box(0); } -x_91 = lean_box(0); -if (lean_is_scalar(x_90)) { - x_92 = lean_alloc_ctor(0, 2, 0); +x_93 = lean_box(0); +if (lean_is_scalar(x_92)) { + x_94 = lean_alloc_ctor(0, 2, 0); } else { - x_92 = x_90; + x_94 = x_92; } -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_89); -return x_92; +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_91); +return x_94; } } } @@ -3876,7 +3933,7 @@ static lean_object* _init_l_Lean_Elab_Term_getFVarLocalDecl_x21___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_getFVarLocalDecl_x21___closed__1; x_2 = l_Lean_Elab_Term_getFVarLocalDecl_x21___closed__2; -x_3 = lean_unsigned_to_nat(320u); +x_3 = lean_unsigned_to_nat(322u); x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_Elab_Term_getFVarLocalDecl_x21___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4178,7 +4235,7 @@ if (x_11 == 0) { lean_object* x_12; lean_object* x_13; x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); lean_ctor_set(x_10, 0, x_13); @@ -4192,7 +4249,7 @@ x_15 = lean_ctor_get(x_10, 1); lean_inc(x_15); lean_inc(x_14); lean_dec(x_10); -x_16 = lean_ctor_get(x_14, 4); +x_16 = lean_ctor_get(x_14, 5); lean_inc(x_16); lean_dec(x_14); x_17 = lean_alloc_ctor(0, 2, 0); @@ -4220,9 +4277,9 @@ x_14 = !lean_is_exclusive(x_12); if (x_14 == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_15 = lean_ctor_get(x_12, 4); +x_15 = lean_ctor_get(x_12, 5); x_16 = lean_apply_1(x_1, x_15); -lean_ctor_set(x_12, 4, x_16); +lean_ctor_set(x_12, 5, x_16); x_17 = lean_st_ref_set(x_3, x_12, x_13); x_18 = !lean_is_exclusive(x_17); if (x_18 == 0) @@ -4249,45 +4306,48 @@ return x_23; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; x_24 = lean_ctor_get(x_12, 0); x_25 = lean_ctor_get(x_12, 1); x_26 = lean_ctor_get(x_12, 2); x_27 = lean_ctor_get(x_12, 3); x_28 = lean_ctor_get(x_12, 4); +x_29 = lean_ctor_get(x_12, 5); +lean_inc(x_29); lean_inc(x_28); lean_inc(x_27); lean_inc(x_26); lean_inc(x_25); lean_inc(x_24); lean_dec(x_12); -x_29 = lean_apply_1(x_1, x_28); -x_30 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_30, 0, x_24); -lean_ctor_set(x_30, 1, x_25); -lean_ctor_set(x_30, 2, x_26); -lean_ctor_set(x_30, 3, x_27); -lean_ctor_set(x_30, 4, x_29); -x_31 = lean_st_ref_set(x_3, x_30, x_13); -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -if (lean_is_exclusive(x_31)) { - lean_ctor_release(x_31, 0); - lean_ctor_release(x_31, 1); - x_33 = x_31; +x_30 = lean_apply_1(x_1, x_29); +x_31 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_31, 0, x_24); +lean_ctor_set(x_31, 1, x_25); +lean_ctor_set(x_31, 2, x_26); +lean_ctor_set(x_31, 3, x_27); +lean_ctor_set(x_31, 4, x_28); +lean_ctor_set(x_31, 5, x_30); +x_32 = lean_st_ref_set(x_3, x_31, x_13); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +if (lean_is_exclusive(x_32)) { + lean_ctor_release(x_32, 0); + lean_ctor_release(x_32, 1); + x_34 = x_32; } else { - lean_dec_ref(x_31); - x_33 = lean_box(0); + lean_dec_ref(x_32); + x_34 = lean_box(0); } -x_34 = lean_box(0); -if (lean_is_scalar(x_33)) { - x_35 = lean_alloc_ctor(0, 2, 0); +x_35 = lean_box(0); +if (lean_is_scalar(x_34)) { + x_36 = lean_alloc_ctor(0, 2, 0); } else { - x_35 = x_33; + x_36 = x_34; } -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_32); -return x_35; +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_33); +return x_36; } } } @@ -4369,7 +4429,7 @@ lean_inc(x_10); x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); -x_12 = lean_ctor_get(x_10, 4); +x_12 = lean_ctor_get(x_10, 5); lean_inc(x_12); lean_dec(x_10); x_13 = lean_ctor_get(x_12, 1); @@ -4382,7 +4442,7 @@ lean_dec(x_14); x_16 = lean_st_ref_take(x_1, x_15); x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 4); +x_18 = lean_ctor_get(x_17, 5); lean_inc(x_18); x_19 = lean_ctor_get(x_16, 1); lean_inc(x_19); @@ -4391,7 +4451,7 @@ x_20 = !lean_is_exclusive(x_17); if (x_20 == 0) { lean_object* x_21; uint8_t x_22; -x_21 = lean_ctor_get(x_17, 4); +x_21 = lean_ctor_get(x_17, 5); lean_dec(x_21); x_22 = !lean_is_exclusive(x_18); if (x_22 == 0) @@ -4435,7 +4495,7 @@ x_33 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_33, 0, x_31); lean_ctor_set(x_33, 1, x_32); lean_ctor_set_uint8(x_33, sizeof(void*)*2, x_30); -lean_ctor_set(x_17, 4, x_33); +lean_ctor_set(x_17, 5, x_33); x_34 = lean_st_ref_set(x_1, x_17, x_19); x_35 = lean_ctor_get(x_34, 1); lean_inc(x_35); @@ -4459,61 +4519,64 @@ return x_37; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_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_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; x_38 = lean_ctor_get(x_17, 0); x_39 = lean_ctor_get(x_17, 1); x_40 = lean_ctor_get(x_17, 2); x_41 = lean_ctor_get(x_17, 3); +x_42 = lean_ctor_get(x_17, 4); +lean_inc(x_42); lean_inc(x_41); lean_inc(x_40); lean_inc(x_39); lean_inc(x_38); lean_dec(x_17); -x_42 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); -x_43 = lean_ctor_get(x_18, 0); -lean_inc(x_43); +x_43 = lean_ctor_get_uint8(x_18, sizeof(void*)*2); +x_44 = lean_ctor_get(x_18, 0); +lean_inc(x_44); if (lean_is_exclusive(x_18)) { lean_ctor_release(x_18, 0); lean_ctor_release(x_18, 1); - x_44 = x_18; + x_45 = x_18; } else { lean_dec_ref(x_18); - x_44 = lean_box(0); + x_45 = lean_box(0); } -x_45 = l_Lean_Elab_Term_State_infoState___default___closed__4; -if (lean_is_scalar(x_44)) { - x_46 = lean_alloc_ctor(0, 2, 1); +x_46 = l_Lean_Elab_Term_State_infoState___default___closed__4; +if (lean_is_scalar(x_45)) { + x_47 = lean_alloc_ctor(0, 2, 1); } else { - x_46 = x_44; + x_47 = x_45; } -lean_ctor_set(x_46, 0, x_43); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_42); -x_47 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_47, 0, x_38); -lean_ctor_set(x_47, 1, x_39); -lean_ctor_set(x_47, 2, x_40); -lean_ctor_set(x_47, 3, x_41); -lean_ctor_set(x_47, 4, x_46); -x_48 = lean_st_ref_set(x_1, x_47, x_19); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; +lean_ctor_set(x_47, 0, x_44); +lean_ctor_set(x_47, 1, x_46); +lean_ctor_set_uint8(x_47, sizeof(void*)*2, x_43); +x_48 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_48, 0, x_38); +lean_ctor_set(x_48, 1, x_39); +lean_ctor_set(x_48, 2, x_40); +lean_ctor_set(x_48, 3, x_41); +lean_ctor_set(x_48, 4, x_42); +lean_ctor_set(x_48, 5, x_47); +x_49 = lean_st_ref_set(x_1, x_48, x_19); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_51 = x_49; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_49); + x_51 = lean_box(0); } -if (lean_is_scalar(x_50)) { - x_51 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_51)) { + x_52 = lean_alloc_ctor(0, 2, 0); } else { - x_51 = x_50; + x_52 = x_51; } -lean_ctor_set(x_51, 0, x_13); -lean_ctor_set(x_51, 1, x_49); -return x_51; +lean_ctor_set(x_52, 0, x_13); +lean_ctor_set(x_52, 1, x_50); +return x_52; } } } @@ -5497,7 +5560,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -5548,7 +5611,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 4); +x_29 = lean_ctor_get(x_27, 5); lean_inc(x_29); lean_dec(x_27); x_30 = lean_ctor_get(x_29, 1); @@ -5571,7 +5634,7 @@ lean_dec(x_34); x_36 = lean_st_ref_take(x_3, x_35); x_37 = lean_ctor_get(x_36, 0); lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 4); +x_38 = lean_ctor_get(x_37, 5); lean_inc(x_38); x_39 = lean_ctor_get(x_36, 1); lean_inc(x_39); @@ -5580,7 +5643,7 @@ x_40 = !lean_is_exclusive(x_37); if (x_40 == 0) { lean_object* x_41; uint8_t x_42; -x_41 = lean_ctor_get(x_37, 4); +x_41 = lean_ctor_get(x_37, 5); lean_dec(x_41); x_42 = !lean_is_exclusive(x_38); if (x_42 == 0) @@ -5625,7 +5688,7 @@ x_53 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_50); -lean_ctor_set(x_37, 4, x_53); +lean_ctor_set(x_37, 5, x_53); x_54 = lean_st_ref_set(x_3, x_37, x_39); lean_dec(x_3); x_55 = lean_ctor_get(x_54, 1); @@ -5650,243 +5713,249 @@ return x_57; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_58 = lean_ctor_get(x_37, 0); x_59 = lean_ctor_get(x_37, 1); x_60 = lean_ctor_get(x_37, 2); x_61 = lean_ctor_get(x_37, 3); +x_62 = lean_ctor_get(x_37, 4); +lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); lean_inc(x_58); lean_dec(x_37); -x_62 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); +x_63 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); +x_64 = lean_ctor_get(x_38, 0); +lean_inc(x_64); if (lean_is_exclusive(x_38)) { lean_ctor_release(x_38, 0); lean_ctor_release(x_38, 1); - x_64 = x_38; + x_65 = x_38; } else { lean_dec_ref(x_38); - x_64 = lean_box(0); + x_65 = lean_box(0); } -x_65 = l_Std_PersistentArray_append___rarg(x_19, x_32); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(0, 2, 1); +x_66 = l_Std_PersistentArray_append___rarg(x_19, x_32); +if (lean_is_scalar(x_65)) { + x_67 = lean_alloc_ctor(0, 2, 1); } else { - x_66 = x_64; + x_67 = x_65; } -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_65); -lean_ctor_set_uint8(x_66, sizeof(void*)*2, x_62); -x_67 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_67, 0, x_58); -lean_ctor_set(x_67, 1, x_59); -lean_ctor_set(x_67, 2, x_60); -lean_ctor_set(x_67, 3, x_61); -lean_ctor_set(x_67, 4, x_66); -x_68 = lean_st_ref_set(x_3, x_67, x_39); +lean_ctor_set(x_67, 0, x_64); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_63); +x_68 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_68, 0, x_58); +lean_ctor_set(x_68, 1, x_59); +lean_ctor_set(x_68, 2, x_60); +lean_ctor_set(x_68, 3, x_61); +lean_ctor_set(x_68, 4, x_62); +lean_ctor_set(x_68, 5, x_67); +x_69 = lean_st_ref_set(x_3, x_68, x_39); lean_dec(x_3); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_70 = x_68; +x_70 = lean_ctor_get(x_69, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_71 = x_69; } else { - lean_dec_ref(x_68); - x_70 = lean_box(0); + lean_dec_ref(x_69); + x_71 = lean_box(0); } -if (lean_is_scalar(x_70)) { - x_71 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_70; + x_72 = x_71; } -lean_ctor_set(x_71, 0, x_22); -lean_ctor_set(x_71, 1, x_69); -return x_71; +lean_ctor_set(x_72, 0, x_22); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_72 = lean_ctor_get(x_21, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_21, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_73 = lean_ctor_get(x_21, 0); lean_inc(x_73); +x_74 = lean_ctor_get(x_21, 1); +lean_inc(x_74); lean_dec(x_21); -x_74 = lean_st_ref_get(x_7, x_73); -x_75 = lean_ctor_get(x_74, 1); -lean_inc(x_75); -lean_dec(x_74); -x_76 = lean_st_ref_get(x_3, x_75); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); +x_75 = lean_st_ref_get(x_7, x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_st_ref_get(x_3, x_76); +x_78 = lean_ctor_get(x_77, 0); lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_ctor_get(x_77, 4); +x_79 = lean_ctor_get(x_77, 1); lean_inc(x_79); lean_dec(x_77); -x_80 = lean_ctor_get(x_79, 1); +x_80 = lean_ctor_get(x_78, 5); lean_inc(x_80); -x_81 = l_Std_PersistentArray_mapM___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__10(x_79, x_80, x_2, x_3, x_4, x_5, x_6, x_7, x_78); +lean_dec(x_78); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +x_82 = l_Std_PersistentArray_mapM___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__10(x_80, x_81, x_2, x_3, x_4, x_5, x_6, x_7, x_79); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_st_ref_get(x_7, x_83); +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +lean_dec(x_82); +x_85 = lean_st_ref_get(x_7, x_84); lean_dec(x_7); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_3, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_87, 4); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_st_ref_take(x_3, x_86); +x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 1); +x_89 = lean_ctor_get(x_88, 5); lean_inc(x_89); -lean_dec(x_86); -x_90 = !lean_is_exclusive(x_87); -if (x_90 == 0) +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = !lean_is_exclusive(x_88); +if (x_91 == 0) { -lean_object* x_91; uint8_t x_92; -x_91 = lean_ctor_get(x_87, 4); -lean_dec(x_91); -x_92 = !lean_is_exclusive(x_88); -if (x_92 == 0) +lean_object* x_92; uint8_t x_93; +x_92 = lean_ctor_get(x_88, 5); +lean_dec(x_92); +x_93 = !lean_is_exclusive(x_89); +if (x_93 == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; -x_93 = lean_ctor_get(x_88, 1); -lean_dec(x_93); -x_94 = l_Std_PersistentArray_append___rarg(x_19, x_82); -lean_ctor_set(x_88, 1, x_94); -x_95 = lean_st_ref_set(x_3, x_87, x_89); +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_89, 1); +lean_dec(x_94); +x_95 = l_Std_PersistentArray_append___rarg(x_19, x_83); +lean_ctor_set(x_89, 1, x_95); +x_96 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) { -lean_object* x_97; -x_97 = lean_ctor_get(x_95, 0); -lean_dec(x_97); -lean_ctor_set_tag(x_95, 1); -lean_ctor_set(x_95, 0, x_72); -return x_95; +lean_object* x_98; +x_98 = lean_ctor_get(x_96, 0); +lean_dec(x_98); +lean_ctor_set_tag(x_96, 1); +lean_ctor_set(x_96, 0, x_73); +return x_96; } else { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_95, 1); -lean_inc(x_98); -lean_dec(x_95); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_72); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_dec(x_96); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_73); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_100 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_101 = lean_ctor_get(x_88, 0); -lean_inc(x_101); -lean_dec(x_88); -x_102 = l_Std_PersistentArray_append___rarg(x_19, x_82); -x_103 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_100); -lean_ctor_set(x_87, 4, x_103); -x_104 = lean_st_ref_set(x_3, x_87, x_89); +uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_101 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +lean_dec(x_89); +x_103 = l_Std_PersistentArray_append___rarg(x_19, x_83); +x_104 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set_uint8(x_104, sizeof(void*)*2, x_101); +lean_ctor_set(x_88, 5, x_104); +x_105 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_106 = x_104; +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; - lean_ctor_set_tag(x_107, 1); + x_108 = x_107; + lean_ctor_set_tag(x_108, 1); } -lean_ctor_set(x_107, 0, x_72); -lean_ctor_set(x_107, 1, x_105); -return x_107; +lean_ctor_set(x_108, 0, x_73); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_108 = lean_ctor_get(x_87, 0); -x_109 = lean_ctor_get(x_87, 1); -x_110 = lean_ctor_get(x_87, 2); -x_111 = lean_ctor_get(x_87, 3); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_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; +x_109 = lean_ctor_get(x_88, 0); +x_110 = lean_ctor_get(x_88, 1); +x_111 = lean_ctor_get(x_88, 2); +x_112 = lean_ctor_get(x_88, 3); +x_113 = lean_ctor_get(x_88, 4); +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_dec(x_87); -x_112 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_113 = lean_ctor_get(x_88, 0); -lean_inc(x_113); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_114 = x_88; +lean_dec(x_88); +x_114 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_115 = lean_ctor_get(x_89, 0); +lean_inc(x_115); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_116 = x_89; } else { - lean_dec_ref(x_88); - x_114 = lean_box(0); + lean_dec_ref(x_89); + x_116 = lean_box(0); } -x_115 = l_Std_PersistentArray_append___rarg(x_19, x_82); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 1); -} else { - x_116 = x_114; -} -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_115); -lean_ctor_set_uint8(x_116, sizeof(void*)*2, x_112); -x_117 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_117, 0, x_108); -lean_ctor_set(x_117, 1, x_109); -lean_ctor_set(x_117, 2, x_110); -lean_ctor_set(x_117, 3, x_111); -lean_ctor_set(x_117, 4, x_116); -x_118 = lean_st_ref_set(x_3, x_117, x_89); -lean_dec(x_3); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; +x_117 = l_Std_PersistentArray_append___rarg(x_19, x_83); +if (lean_is_scalar(x_116)) { + x_118 = lean_alloc_ctor(0, 2, 1); } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + x_118 = x_116; +} +lean_ctor_set(x_118, 0, x_115); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); +x_119 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_119, 0, x_109); +lean_ctor_set(x_119, 1, x_110); +lean_ctor_set(x_119, 2, x_111); +lean_ctor_set(x_119, 3, x_112); +lean_ctor_set(x_119, 4, x_113); +lean_ctor_set(x_119, 5, x_118); +x_120 = lean_st_ref_set(x_3, x_119, x_90); +lean_dec(x_3); +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_122 = x_120; +} else { + lean_dec_ref(x_120); + x_122 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); } else { - x_121 = x_120; - lean_ctor_set_tag(x_121, 1); + x_123 = x_122; + lean_ctor_set_tag(x_123, 1); } -lean_ctor_set(x_121, 0, x_72); -lean_ctor_set(x_121, 1, x_119); -return x_121; +lean_ctor_set(x_123, 0, x_73); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } @@ -5930,7 +5999,7 @@ lean_inc(x_3); x_32 = l_Lean_Elab_withSaveInfoContext___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_31); if (lean_obj_tag(x_32) == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +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; uint8_t x_45; x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); x_34 = lean_ctor_get(x_32, 1); @@ -5954,237 +6023,249 @@ x_42 = lean_ctor_get(x_25, 2); lean_inc(x_42); x_43 = lean_ctor_get(x_25, 3); lean_inc(x_43); +x_44 = lean_ctor_get(x_25, 4); +lean_inc(x_44); lean_dec(x_25); -x_44 = !lean_is_exclusive(x_38); -if (x_44 == 0) +x_45 = !lean_is_exclusive(x_38); +if (x_45 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_45 = lean_ctor_get(x_38, 3); -lean_dec(x_45); -x_46 = lean_ctor_get(x_38, 2); +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; uint8_t x_56; +x_46 = lean_ctor_get(x_38, 4); lean_dec(x_46); -x_47 = lean_ctor_get(x_38, 1); +x_47 = lean_ctor_get(x_38, 3); lean_dec(x_47); -x_48 = lean_ctor_get(x_38, 0); +x_48 = lean_ctor_get(x_38, 2); lean_dec(x_48); +x_49 = lean_ctor_get(x_38, 1); +lean_dec(x_49); +x_50 = lean_ctor_get(x_38, 0); +lean_dec(x_50); +lean_ctor_set(x_38, 4, x_44); lean_ctor_set(x_38, 3, x_43); lean_ctor_set(x_38, 2, x_42); lean_ctor_set(x_38, 1, x_41); lean_ctor_set(x_38, 0, x_40); -x_49 = lean_st_ref_set(x_3, x_38, x_39); +x_51 = lean_st_ref_set(x_3, x_38, x_39); lean_dec(x_3); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -lean_dec(x_49); -x_51 = lean_st_ref_get(x_7, x_50); -lean_dec(x_7); x_52 = lean_ctor_get(x_51, 1); lean_inc(x_52); lean_dec(x_51); -x_53 = lean_st_ref_set(x_5, x_30, x_52); +x_53 = lean_st_ref_get(x_7, x_52); +lean_dec(x_7); +x_54 = lean_ctor_get(x_53, 1); +lean_inc(x_54); +lean_dec(x_53); +x_55 = lean_st_ref_set(x_5, x_30, x_54); lean_dec(x_5); -x_54 = !lean_is_exclusive(x_53); -if (x_54 == 0) +x_56 = !lean_is_exclusive(x_55); +if (x_56 == 0) { -lean_object* x_55; lean_object* x_56; -x_55 = lean_ctor_get(x_53, 0); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_33); -lean_ctor_set(x_56, 1, x_55); -lean_ctor_set(x_53, 0, x_56); -x_9 = x_53; +lean_object* x_57; lean_object* x_58; +x_57 = lean_ctor_get(x_55, 0); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_33); +lean_ctor_set(x_58, 1, x_57); +lean_ctor_set(x_55, 0, x_58); +x_9 = x_55; goto block_21; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_57 = lean_ctor_get(x_53, 0); -x_58 = lean_ctor_get(x_53, 1); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_53); -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_33); -lean_ctor_set(x_59, 1, x_57); -x_60 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_58); -x_9 = x_60; +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_59 = lean_ctor_get(x_55, 0); +x_60 = lean_ctor_get(x_55, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_55); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_33); +lean_ctor_set(x_61, 1, x_59); +x_62 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_60); +x_9 = x_62; goto block_21; } } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_61 = lean_ctor_get(x_38, 4); -lean_inc(x_61); +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_63 = lean_ctor_get(x_38, 5); +lean_inc(x_63); lean_dec(x_38); -x_62 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_62, 0, x_40); -lean_ctor_set(x_62, 1, x_41); -lean_ctor_set(x_62, 2, x_42); -lean_ctor_set(x_62, 3, x_43); -lean_ctor_set(x_62, 4, x_61); -x_63 = lean_st_ref_set(x_3, x_62, x_39); +x_64 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_64, 0, x_40); +lean_ctor_set(x_64, 1, x_41); +lean_ctor_set(x_64, 2, x_42); +lean_ctor_set(x_64, 3, x_43); +lean_ctor_set(x_64, 4, x_44); +lean_ctor_set(x_64, 5, x_63); +x_65 = lean_st_ref_set(x_3, x_64, x_39); lean_dec(x_3); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -lean_dec(x_63); -x_65 = lean_st_ref_get(x_7, x_64); -lean_dec(x_7); x_66 = lean_ctor_get(x_65, 1); lean_inc(x_66); lean_dec(x_65); -x_67 = lean_st_ref_set(x_5, x_30, x_66); -lean_dec(x_5); -x_68 = lean_ctor_get(x_67, 0); +x_67 = lean_st_ref_get(x_7, x_66); +lean_dec(x_7); +x_68 = lean_ctor_get(x_67, 1); lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_67)) { - lean_ctor_release(x_67, 0); - lean_ctor_release(x_67, 1); - x_70 = x_67; +lean_dec(x_67); +x_69 = lean_st_ref_set(x_5, x_30, x_68); +lean_dec(x_5); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_72 = x_69; } else { - lean_dec_ref(x_67); - x_70 = lean_box(0); + lean_dec_ref(x_69); + x_72 = lean_box(0); } -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_33); -lean_ctor_set(x_71, 1, x_68); -if (lean_is_scalar(x_70)) { - x_72 = lean_alloc_ctor(0, 2, 0); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_33); +lean_ctor_set(x_73, 1, x_70); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(0, 2, 0); } else { - x_72 = x_70; + x_74 = x_72; } -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_69); -x_9 = x_72; +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_71); +x_9 = x_74; goto block_21; } } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; -x_73 = lean_ctor_get(x_32, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_32, 1); -lean_inc(x_74); -lean_dec(x_32); -x_75 = lean_st_ref_get(x_7, x_74); -x_76 = lean_ctor_get(x_75, 1); +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; uint8_t x_87; +x_75 = lean_ctor_get(x_32, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_32, 1); lean_inc(x_76); -lean_dec(x_75); -x_77 = lean_st_ref_take(x_3, x_76); -x_78 = lean_ctor_get(x_77, 0); +lean_dec(x_32); +x_77 = lean_st_ref_get(x_7, x_76); +x_78 = lean_ctor_get(x_77, 1); lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); -lean_inc(x_79); lean_dec(x_77); -x_80 = lean_ctor_get(x_25, 0); +x_79 = lean_st_ref_take(x_3, x_78); +x_80 = lean_ctor_get(x_79, 0); lean_inc(x_80); -x_81 = lean_ctor_get(x_25, 1); +x_81 = lean_ctor_get(x_79, 1); lean_inc(x_81); -x_82 = lean_ctor_get(x_25, 2); +lean_dec(x_79); +x_82 = lean_ctor_get(x_25, 0); lean_inc(x_82); -x_83 = lean_ctor_get(x_25, 3); +x_83 = lean_ctor_get(x_25, 1); lean_inc(x_83); +x_84 = lean_ctor_get(x_25, 2); +lean_inc(x_84); +x_85 = lean_ctor_get(x_25, 3); +lean_inc(x_85); +x_86 = lean_ctor_get(x_25, 4); +lean_inc(x_86); lean_dec(x_25); -x_84 = !lean_is_exclusive(x_78); -if (x_84 == 0) +x_87 = !lean_is_exclusive(x_80); +if (x_87 == 0) { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; -x_85 = lean_ctor_get(x_78, 3); -lean_dec(x_85); -x_86 = lean_ctor_get(x_78, 2); -lean_dec(x_86); -x_87 = lean_ctor_get(x_78, 1); -lean_dec(x_87); -x_88 = lean_ctor_get(x_78, 0); +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; +x_88 = lean_ctor_get(x_80, 4); lean_dec(x_88); -lean_ctor_set(x_78, 3, x_83); -lean_ctor_set(x_78, 2, x_82); -lean_ctor_set(x_78, 1, x_81); -lean_ctor_set(x_78, 0, x_80); -x_89 = lean_st_ref_set(x_3, x_78, x_79); -lean_dec(x_3); -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); +x_89 = lean_ctor_get(x_80, 3); lean_dec(x_89); -x_91 = lean_st_ref_get(x_7, x_90); -lean_dec(x_7); -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); +x_90 = lean_ctor_get(x_80, 2); +lean_dec(x_90); +x_91 = lean_ctor_get(x_80, 1); lean_dec(x_91); -x_93 = lean_st_ref_set(x_5, x_30, x_92); +x_92 = lean_ctor_get(x_80, 0); +lean_dec(x_92); +lean_ctor_set(x_80, 4, x_86); +lean_ctor_set(x_80, 3, x_85); +lean_ctor_set(x_80, 2, x_84); +lean_ctor_set(x_80, 1, x_83); +lean_ctor_set(x_80, 0, x_82); +x_93 = lean_st_ref_set(x_3, x_80, x_81); +lean_dec(x_3); +x_94 = lean_ctor_get(x_93, 1); +lean_inc(x_94); +lean_dec(x_93); +x_95 = lean_st_ref_get(x_7, x_94); +lean_dec(x_7); +x_96 = lean_ctor_get(x_95, 1); +lean_inc(x_96); +lean_dec(x_95); +x_97 = lean_st_ref_set(x_5, x_30, x_96); lean_dec(x_5); -x_94 = !lean_is_exclusive(x_93); -if (x_94 == 0) +x_98 = !lean_is_exclusive(x_97); +if (x_98 == 0) { -lean_object* x_95; -x_95 = lean_ctor_get(x_93, 0); -lean_dec(x_95); -lean_ctor_set_tag(x_93, 1); -lean_ctor_set(x_93, 0, x_73); -x_9 = x_93; +lean_object* x_99; +x_99 = lean_ctor_get(x_97, 0); +lean_dec(x_99); +lean_ctor_set_tag(x_97, 1); +lean_ctor_set(x_97, 0, x_75); +x_9 = x_97; goto block_21; } else { -lean_object* x_96; lean_object* x_97; -x_96 = lean_ctor_get(x_93, 1); -lean_inc(x_96); -lean_dec(x_93); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_73); -lean_ctor_set(x_97, 1, x_96); -x_9 = x_97; +lean_object* x_100; lean_object* x_101; +x_100 = lean_ctor_get(x_97, 1); +lean_inc(x_100); +lean_dec(x_97); +x_101 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_101, 0, x_75); +lean_ctor_set(x_101, 1, x_100); +x_9 = x_101; goto block_21; } } else { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_78, 4); -lean_inc(x_98); -lean_dec(x_78); -x_99 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_99, 0, x_80); -lean_ctor_set(x_99, 1, x_81); -lean_ctor_set(x_99, 2, x_82); -lean_ctor_set(x_99, 3, x_83); -lean_ctor_set(x_99, 4, x_98); -x_100 = lean_st_ref_set(x_3, x_99, x_79); -lean_dec(x_3); -x_101 = lean_ctor_get(x_100, 1); -lean_inc(x_101); -lean_dec(x_100); -x_102 = lean_st_ref_get(x_7, x_101); -lean_dec(x_7); -x_103 = lean_ctor_get(x_102, 1); -lean_inc(x_103); -lean_dec(x_102); -x_104 = lean_st_ref_set(x_5, x_30, x_103); -lean_dec(x_5); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_102 = lean_ctor_get(x_80, 5); +lean_inc(x_102); +lean_dec(x_80); +x_103 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_103, 0, x_82); +lean_ctor_set(x_103, 1, x_83); +lean_ctor_set(x_103, 2, x_84); +lean_ctor_set(x_103, 3, x_85); +lean_ctor_set(x_103, 4, x_86); +lean_ctor_set(x_103, 5, x_102); +x_104 = lean_st_ref_set(x_3, x_103, x_81); +lean_dec(x_3); x_105 = lean_ctor_get(x_104, 1); lean_inc(x_105); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_106 = x_104; +lean_dec(x_104); +x_106 = lean_st_ref_get(x_7, x_105); +lean_dec(x_7); +x_107 = lean_ctor_get(x_106, 1); +lean_inc(x_107); +lean_dec(x_106); +x_108 = lean_st_ref_set(x_5, x_30, x_107); +lean_dec(x_5); +x_109 = lean_ctor_get(x_108, 1); +lean_inc(x_109); +if (lean_is_exclusive(x_108)) { + lean_ctor_release(x_108, 0); + lean_ctor_release(x_108, 1); + x_110 = x_108; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_108); + x_110 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_110)) { + x_111 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; - lean_ctor_set_tag(x_107, 1); + x_111 = x_110; + lean_ctor_set_tag(x_111, 1); } -lean_ctor_set(x_107, 0, x_73); -lean_ctor_set(x_107, 1, x_105); -x_9 = x_107; +lean_ctor_set(x_111, 0, x_75); +lean_ctor_set(x_111, 1, x_109); +x_9 = x_111; goto block_21; } } @@ -7231,7 +7312,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -7282,7 +7363,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 4); +x_29 = lean_ctor_get(x_27, 5); lean_inc(x_29); lean_dec(x_27); x_30 = lean_ctor_get(x_29, 1); @@ -7305,7 +7386,7 @@ lean_dec(x_34); x_36 = lean_st_ref_take(x_3, x_35); x_37 = lean_ctor_get(x_36, 0); lean_inc(x_37); -x_38 = lean_ctor_get(x_37, 4); +x_38 = lean_ctor_get(x_37, 5); lean_inc(x_38); x_39 = lean_ctor_get(x_36, 1); lean_inc(x_39); @@ -7314,7 +7395,7 @@ x_40 = !lean_is_exclusive(x_37); if (x_40 == 0) { lean_object* x_41; uint8_t x_42; -x_41 = lean_ctor_get(x_37, 4); +x_41 = lean_ctor_get(x_37, 5); lean_dec(x_41); x_42 = !lean_is_exclusive(x_38); if (x_42 == 0) @@ -7359,7 +7440,7 @@ x_53 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_53, 0, x_51); lean_ctor_set(x_53, 1, x_52); lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_50); -lean_ctor_set(x_37, 4, x_53); +lean_ctor_set(x_37, 5, x_53); x_54 = lean_st_ref_set(x_3, x_37, x_39); lean_dec(x_3); x_55 = lean_ctor_get(x_54, 1); @@ -7384,243 +7465,249 @@ return x_57; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_58 = lean_ctor_get(x_37, 0); x_59 = lean_ctor_get(x_37, 1); x_60 = lean_ctor_get(x_37, 2); x_61 = lean_ctor_get(x_37, 3); +x_62 = lean_ctor_get(x_37, 4); +lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); lean_inc(x_58); lean_dec(x_37); -x_62 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); +x_63 = lean_ctor_get_uint8(x_38, sizeof(void*)*2); +x_64 = lean_ctor_get(x_38, 0); +lean_inc(x_64); if (lean_is_exclusive(x_38)) { lean_ctor_release(x_38, 0); lean_ctor_release(x_38, 1); - x_64 = x_38; + x_65 = x_38; } else { lean_dec_ref(x_38); - x_64 = lean_box(0); + x_65 = lean_box(0); } -x_65 = l_Std_PersistentArray_append___rarg(x_19, x_32); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(0, 2, 1); +x_66 = l_Std_PersistentArray_append___rarg(x_19, x_32); +if (lean_is_scalar(x_65)) { + x_67 = lean_alloc_ctor(0, 2, 1); } else { - x_66 = x_64; + x_67 = x_65; } -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_65); -lean_ctor_set_uint8(x_66, sizeof(void*)*2, x_62); -x_67 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_67, 0, x_58); -lean_ctor_set(x_67, 1, x_59); -lean_ctor_set(x_67, 2, x_60); -lean_ctor_set(x_67, 3, x_61); -lean_ctor_set(x_67, 4, x_66); -x_68 = lean_st_ref_set(x_3, x_67, x_39); +lean_ctor_set(x_67, 0, x_64); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_63); +x_68 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_68, 0, x_58); +lean_ctor_set(x_68, 1, x_59); +lean_ctor_set(x_68, 2, x_60); +lean_ctor_set(x_68, 3, x_61); +lean_ctor_set(x_68, 4, x_62); +lean_ctor_set(x_68, 5, x_67); +x_69 = lean_st_ref_set(x_3, x_68, x_39); lean_dec(x_3); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_70 = x_68; +x_70 = lean_ctor_get(x_69, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + x_71 = x_69; } else { - lean_dec_ref(x_68); - x_70 = lean_box(0); + lean_dec_ref(x_69); + x_71 = lean_box(0); } -if (lean_is_scalar(x_70)) { - x_71 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_70; + x_72 = x_71; } -lean_ctor_set(x_71, 0, x_22); -lean_ctor_set(x_71, 1, x_69); -return x_71; +lean_ctor_set(x_72, 0, x_22); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_72 = lean_ctor_get(x_21, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_21, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_73 = lean_ctor_get(x_21, 0); lean_inc(x_73); +x_74 = lean_ctor_get(x_21, 1); +lean_inc(x_74); lean_dec(x_21); -x_74 = lean_st_ref_get(x_7, x_73); -x_75 = lean_ctor_get(x_74, 1); -lean_inc(x_75); -lean_dec(x_74); -x_76 = lean_st_ref_get(x_3, x_75); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); +x_75 = lean_st_ref_get(x_7, x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_st_ref_get(x_3, x_76); +x_78 = lean_ctor_get(x_77, 0); lean_inc(x_78); -lean_dec(x_76); -x_79 = lean_ctor_get(x_77, 4); +x_79 = lean_ctor_get(x_77, 1); lean_inc(x_79); lean_dec(x_77); -x_80 = lean_ctor_get(x_79, 1); +x_80 = lean_ctor_get(x_78, 5); lean_inc(x_80); -x_81 = l_Std_PersistentArray_mapM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__7(x_79, x_80, x_2, x_3, x_4, x_5, x_6, x_7, x_78); +lean_dec(x_78); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +x_82 = l_Std_PersistentArray_mapM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_withoutModifyingStateWithInfoAndMessagesImpl___spec__7(x_80, x_81, x_2, x_3, x_4, x_5, x_6, x_7, x_79); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_st_ref_get(x_7, x_83); +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +lean_dec(x_82); +x_85 = lean_st_ref_get(x_7, x_84); lean_dec(x_7); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -x_86 = lean_st_ref_take(x_3, x_85); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_87, 4); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_st_ref_take(x_3, x_86); +x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); -x_89 = lean_ctor_get(x_86, 1); +x_89 = lean_ctor_get(x_88, 5); lean_inc(x_89); -lean_dec(x_86); -x_90 = !lean_is_exclusive(x_87); -if (x_90 == 0) +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = !lean_is_exclusive(x_88); +if (x_91 == 0) { -lean_object* x_91; uint8_t x_92; -x_91 = lean_ctor_get(x_87, 4); -lean_dec(x_91); -x_92 = !lean_is_exclusive(x_88); -if (x_92 == 0) +lean_object* x_92; uint8_t x_93; +x_92 = lean_ctor_get(x_88, 5); +lean_dec(x_92); +x_93 = !lean_is_exclusive(x_89); +if (x_93 == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; -x_93 = lean_ctor_get(x_88, 1); -lean_dec(x_93); -x_94 = l_Std_PersistentArray_append___rarg(x_19, x_82); -lean_ctor_set(x_88, 1, x_94); -x_95 = lean_st_ref_set(x_3, x_87, x_89); +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_89, 1); +lean_dec(x_94); +x_95 = l_Std_PersistentArray_append___rarg(x_19, x_83); +lean_ctor_set(x_89, 1, x_95); +x_96 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_96 = !lean_is_exclusive(x_95); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_96); +if (x_97 == 0) { -lean_object* x_97; -x_97 = lean_ctor_get(x_95, 0); -lean_dec(x_97); -lean_ctor_set_tag(x_95, 1); -lean_ctor_set(x_95, 0, x_72); -return x_95; +lean_object* x_98; +x_98 = lean_ctor_get(x_96, 0); +lean_dec(x_98); +lean_ctor_set_tag(x_96, 1); +lean_ctor_set(x_96, 0, x_73); +return x_96; } else { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_95, 1); -lean_inc(x_98); -lean_dec(x_95); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_72); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_99; lean_object* x_100; +x_99 = lean_ctor_get(x_96, 1); +lean_inc(x_99); +lean_dec(x_96); +x_100 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_100, 0, x_73); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -uint8_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_100 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_101 = lean_ctor_get(x_88, 0); -lean_inc(x_101); -lean_dec(x_88); -x_102 = l_Std_PersistentArray_append___rarg(x_19, x_82); -x_103 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_100); -lean_ctor_set(x_87, 4, x_103); -x_104 = lean_st_ref_set(x_3, x_87, x_89); +uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_101 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_102 = lean_ctor_get(x_89, 0); +lean_inc(x_102); +lean_dec(x_89); +x_103 = l_Std_PersistentArray_append___rarg(x_19, x_83); +x_104 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set_uint8(x_104, sizeof(void*)*2, x_101); +lean_ctor_set(x_88, 5, x_104); +x_105 = lean_st_ref_set(x_3, x_88, x_90); lean_dec(x_3); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_106 = x_104; +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; } else { - lean_dec_ref(x_104); - x_106 = lean_box(0); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -if (lean_is_scalar(x_106)) { - x_107 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); } else { - x_107 = x_106; - lean_ctor_set_tag(x_107, 1); + x_108 = x_107; + lean_ctor_set_tag(x_108, 1); } -lean_ctor_set(x_107, 0, x_72); -lean_ctor_set(x_107, 1, x_105); -return x_107; +lean_ctor_set(x_108, 0, x_73); +lean_ctor_set(x_108, 1, x_106); +return x_108; } } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_108 = lean_ctor_get(x_87, 0); -x_109 = lean_ctor_get(x_87, 1); -x_110 = lean_ctor_get(x_87, 2); -x_111 = lean_ctor_get(x_87, 3); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_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; +x_109 = lean_ctor_get(x_88, 0); +x_110 = lean_ctor_get(x_88, 1); +x_111 = lean_ctor_get(x_88, 2); +x_112 = lean_ctor_get(x_88, 3); +x_113 = lean_ctor_get(x_88, 4); +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_dec(x_87); -x_112 = lean_ctor_get_uint8(x_88, sizeof(void*)*2); -x_113 = lean_ctor_get(x_88, 0); -lean_inc(x_113); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - lean_ctor_release(x_88, 1); - x_114 = x_88; +lean_dec(x_88); +x_114 = lean_ctor_get_uint8(x_89, sizeof(void*)*2); +x_115 = lean_ctor_get(x_89, 0); +lean_inc(x_115); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_116 = x_89; } else { - lean_dec_ref(x_88); - x_114 = lean_box(0); + lean_dec_ref(x_89); + x_116 = lean_box(0); } -x_115 = l_Std_PersistentArray_append___rarg(x_19, x_82); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(0, 2, 1); -} else { - x_116 = x_114; -} -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_115); -lean_ctor_set_uint8(x_116, sizeof(void*)*2, x_112); -x_117 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_117, 0, x_108); -lean_ctor_set(x_117, 1, x_109); -lean_ctor_set(x_117, 2, x_110); -lean_ctor_set(x_117, 3, x_111); -lean_ctor_set(x_117, 4, x_116); -x_118 = lean_st_ref_set(x_3, x_117, x_89); -lean_dec(x_3); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; +x_117 = l_Std_PersistentArray_append___rarg(x_19, x_83); +if (lean_is_scalar(x_116)) { + x_118 = lean_alloc_ctor(0, 2, 1); } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + x_118 = x_116; } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_115); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_114); +x_119 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_119, 0, x_109); +lean_ctor_set(x_119, 1, x_110); +lean_ctor_set(x_119, 2, x_111); +lean_ctor_set(x_119, 3, x_112); +lean_ctor_set(x_119, 4, x_113); +lean_ctor_set(x_119, 5, x_118); +x_120 = lean_st_ref_set(x_3, x_119, x_90); +lean_dec(x_3); +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_122 = x_120; } else { - x_121 = x_120; - lean_ctor_set_tag(x_121, 1); + lean_dec_ref(x_120); + x_122 = lean_box(0); +} +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(1, 2, 0); +} else { + x_123 = x_122; + lean_ctor_set_tag(x_123, 1); } -lean_ctor_set(x_121, 0, x_72); -lean_ctor_set(x_121, 1, x_119); -return x_121; +lean_ctor_set(x_123, 0, x_73); +lean_ctor_set(x_123, 1, x_121); +return x_123; } } } @@ -7699,7 +7786,7 @@ lean_dec(x_22); x_32 = !lean_is_exclusive(x_23); if (x_32 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; x_33 = lean_ctor_get(x_23, 4); lean_dec(x_33); x_34 = lean_ctor_get(x_23, 3); @@ -7727,197 +7814,207 @@ x_41 = lean_ctor_get(x_38, 2); lean_inc(x_41); x_42 = lean_ctor_get(x_38, 3); lean_inc(x_42); +x_43 = lean_ctor_get(x_38, 4); +lean_inc(x_43); lean_dec(x_38); -x_43 = !lean_is_exclusive(x_18); -if (x_43 == 0) +x_44 = !lean_is_exclusive(x_18); +if (x_44 == 0) { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; uint8_t x_51; -x_44 = lean_ctor_get(x_18, 3); -lean_dec(x_44); -x_45 = lean_ctor_get(x_18, 2); +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; uint8_t x_53; +x_45 = lean_ctor_get(x_18, 4); lean_dec(x_45); -x_46 = lean_ctor_get(x_18, 1); +x_46 = lean_ctor_get(x_18, 3); lean_dec(x_46); -x_47 = lean_ctor_get(x_18, 0); +x_47 = lean_ctor_get(x_18, 2); lean_dec(x_47); +x_48 = lean_ctor_get(x_18, 1); +lean_dec(x_48); +x_49 = lean_ctor_get(x_18, 0); +lean_dec(x_49); +lean_ctor_set(x_18, 4, x_43); lean_ctor_set(x_18, 3, x_42); lean_ctor_set(x_18, 2, x_41); lean_ctor_set(x_18, 1, x_40); lean_ctor_set(x_18, 0, x_39); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_21); -lean_ctor_set(x_48, 1, x_18); -x_49 = 0; -x_50 = l_Lean_Elab_Term_SavedState_restore(x_48, x_49, x_2, x_3, x_4, x_5, x_6, x_7, x_24); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_21); +lean_ctor_set(x_50, 1, x_18); +x_51 = 0; +x_52 = l_Lean_Elab_Term_SavedState_restore(x_50, x_51, x_2, x_3, x_4, x_5, x_6, x_7, x_24); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_51 = !lean_is_exclusive(x_50); -if (x_51 == 0) +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) { -lean_object* x_52; -x_52 = lean_ctor_get(x_50, 0); -lean_dec(x_52); -lean_ctor_set(x_50, 0, x_13); -return x_50; +lean_object* x_54; +x_54 = lean_ctor_get(x_52, 0); +lean_dec(x_54); +lean_ctor_set(x_52, 0, x_13); +return x_52; } else { -lean_object* x_53; lean_object* x_54; -x_53 = lean_ctor_get(x_50, 1); -lean_inc(x_53); -lean_dec(x_50); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_13); -lean_ctor_set(x_54, 1, x_53); -return x_54; +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_52, 1); +lean_inc(x_55); +lean_dec(x_52); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_13); +lean_ctor_set(x_56, 1, x_55); +return x_56; } } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_55 = lean_ctor_get(x_18, 4); -lean_inc(x_55); +lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_57 = lean_ctor_get(x_18, 5); +lean_inc(x_57); lean_dec(x_18); -x_56 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_56, 0, x_39); -lean_ctor_set(x_56, 1, x_40); -lean_ctor_set(x_56, 2, x_41); -lean_ctor_set(x_56, 3, x_42); -lean_ctor_set(x_56, 4, x_55); -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_21); -lean_ctor_set(x_57, 1, x_56); -x_58 = 0; -x_59 = l_Lean_Elab_Term_SavedState_restore(x_57, x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_24); +x_58 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_58, 0, x_39); +lean_ctor_set(x_58, 1, x_40); +lean_ctor_set(x_58, 2, x_41); +lean_ctor_set(x_58, 3, x_42); +lean_ctor_set(x_58, 4, x_43); +lean_ctor_set(x_58, 5, x_57); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_21); +lean_ctor_set(x_59, 1, x_58); +x_60 = 0; +x_61 = l_Lean_Elab_Term_SavedState_restore(x_59, x_60, x_2, x_3, x_4, x_5, x_6, x_7, x_24); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_59)) { - lean_ctor_release(x_59, 0); - lean_ctor_release(x_59, 1); - x_61 = x_59; +x_62 = lean_ctor_get(x_61, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_61)) { + lean_ctor_release(x_61, 0); + lean_ctor_release(x_61, 1); + x_63 = x_61; } else { - lean_dec_ref(x_59); - x_61 = lean_box(0); + lean_dec_ref(x_61); + x_63 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(0, 2, 0); } else { - x_62 = x_61; + x_64 = x_63; } -lean_ctor_set(x_62, 0, x_13); -lean_ctor_set(x_62, 1, x_60); -return x_62; +lean_ctor_set(x_64, 0, x_13); +lean_ctor_set(x_64, 1, x_62); +return x_64; } } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_63 = lean_ctor_get(x_23, 5); -lean_inc(x_63); -lean_dec(x_23); -x_64 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_64, 0, x_27); -lean_ctor_set(x_64, 1, x_28); -lean_ctor_set(x_64, 2, x_29); -lean_ctor_set(x_64, 3, x_30); -lean_ctor_set(x_64, 4, x_31); -lean_ctor_set(x_64, 5, x_63); -lean_ctor_set(x_21, 0, x_64); -x_65 = lean_ctor_get(x_10, 1); +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; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_65 = lean_ctor_get(x_23, 5); lean_inc(x_65); -lean_dec(x_10); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); +lean_dec(x_23); +x_66 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_66, 0, x_27); +lean_ctor_set(x_66, 1, x_28); +lean_ctor_set(x_66, 2, x_29); +lean_ctor_set(x_66, 3, x_30); +lean_ctor_set(x_66, 4, x_31); +lean_ctor_set(x_66, 5, x_65); +lean_ctor_set(x_21, 0, x_66); +x_67 = lean_ctor_get(x_10, 1); lean_inc(x_67); -x_68 = lean_ctor_get(x_65, 2); +lean_dec(x_10); +x_68 = lean_ctor_get(x_67, 0); lean_inc(x_68); -x_69 = lean_ctor_get(x_65, 3); +x_69 = lean_ctor_get(x_67, 1); lean_inc(x_69); -lean_dec(x_65); -x_70 = lean_ctor_get(x_18, 4); +x_70 = lean_ctor_get(x_67, 2); lean_inc(x_70); +x_71 = lean_ctor_get(x_67, 3); +lean_inc(x_71); +x_72 = lean_ctor_get(x_67, 4); +lean_inc(x_72); +lean_dec(x_67); +x_73 = lean_ctor_get(x_18, 5); +lean_inc(x_73); if (lean_is_exclusive(x_18)) { lean_ctor_release(x_18, 0); lean_ctor_release(x_18, 1); lean_ctor_release(x_18, 2); lean_ctor_release(x_18, 3); lean_ctor_release(x_18, 4); - x_71 = x_18; + lean_ctor_release(x_18, 5); + x_74 = x_18; } else { lean_dec_ref(x_18); - x_71 = lean_box(0); + x_74 = lean_box(0); } -if (lean_is_scalar(x_71)) { - x_72 = lean_alloc_ctor(0, 5, 0); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(0, 6, 0); } else { - x_72 = x_71; + x_75 = x_74; } -lean_ctor_set(x_72, 0, x_66); -lean_ctor_set(x_72, 1, x_67); -lean_ctor_set(x_72, 2, x_68); -lean_ctor_set(x_72, 3, x_69); -lean_ctor_set(x_72, 4, x_70); -x_73 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_73, 0, x_21); -lean_ctor_set(x_73, 1, x_72); -x_74 = 0; -x_75 = l_Lean_Elab_Term_SavedState_restore(x_73, x_74, x_2, x_3, x_4, x_5, x_6, x_7, x_24); +lean_ctor_set(x_75, 0, x_68); +lean_ctor_set(x_75, 1, x_69); +lean_ctor_set(x_75, 2, x_70); +lean_ctor_set(x_75, 3, x_71); +lean_ctor_set(x_75, 4, x_72); +lean_ctor_set(x_75, 5, x_73); +x_76 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_76, 0, x_21); +lean_ctor_set(x_76, 1, x_75); +x_77 = 0; +x_78 = l_Lean_Elab_Term_SavedState_restore(x_76, x_77, x_2, x_3, x_4, x_5, x_6, x_7, x_24); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_76 = lean_ctor_get(x_75, 1); -lean_inc(x_76); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_77 = x_75; +x_79 = lean_ctor_get(x_78, 1); +lean_inc(x_79); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_80 = x_78; } else { - lean_dec_ref(x_75); - x_77 = lean_box(0); + lean_dec_ref(x_78); + x_80 = lean_box(0); } -if (lean_is_scalar(x_77)) { - x_78 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_80)) { + x_81 = lean_alloc_ctor(0, 2, 0); } else { - x_78 = x_77; + x_81 = x_80; } -lean_ctor_set(x_78, 0, x_13); -lean_ctor_set(x_78, 1, x_76); -return x_78; +lean_ctor_set(x_81, 0, x_13); +lean_ctor_set(x_81, 1, x_79); +return x_81; } } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; 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; uint8_t x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_79 = lean_ctor_get(x_21, 1); -lean_inc(x_79); -lean_dec(x_21); -x_80 = lean_ctor_get(x_22, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_22, 1); -lean_inc(x_81); -x_82 = lean_ctor_get(x_22, 2); +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_82 = lean_ctor_get(x_21, 1); lean_inc(x_82); -x_83 = lean_ctor_get(x_22, 3); +lean_dec(x_21); +x_83 = lean_ctor_get(x_22, 0); lean_inc(x_83); -x_84 = lean_ctor_get(x_22, 4); +x_84 = lean_ctor_get(x_22, 1); lean_inc(x_84); -lean_dec(x_22); -x_85 = lean_ctor_get(x_23, 5); +x_85 = lean_ctor_get(x_22, 2); lean_inc(x_85); +x_86 = lean_ctor_get(x_22, 3); +lean_inc(x_86); +x_87 = lean_ctor_get(x_22, 4); +lean_inc(x_87); +lean_dec(x_22); +x_88 = lean_ctor_get(x_23, 5); +lean_inc(x_88); if (lean_is_exclusive(x_23)) { lean_ctor_release(x_23, 0); lean_ctor_release(x_23, 1); @@ -7925,452 +8022,470 @@ if (lean_is_exclusive(x_23)) { lean_ctor_release(x_23, 3); lean_ctor_release(x_23, 4); lean_ctor_release(x_23, 5); - x_86 = x_23; + x_89 = x_23; } else { lean_dec_ref(x_23); - x_86 = lean_box(0); + x_89 = lean_box(0); } -if (lean_is_scalar(x_86)) { - x_87 = lean_alloc_ctor(0, 6, 0); +if (lean_is_scalar(x_89)) { + x_90 = lean_alloc_ctor(0, 6, 0); } else { - x_87 = x_86; + x_90 = x_89; } -lean_ctor_set(x_87, 0, x_80); -lean_ctor_set(x_87, 1, x_81); -lean_ctor_set(x_87, 2, x_82); -lean_ctor_set(x_87, 3, x_83); -lean_ctor_set(x_87, 4, x_84); -lean_ctor_set(x_87, 5, x_85); -x_88 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_88, 0, x_87); -lean_ctor_set(x_88, 1, x_79); -x_89 = lean_ctor_get(x_10, 1); -lean_inc(x_89); -lean_dec(x_10); -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_89, 1); -lean_inc(x_91); -x_92 = lean_ctor_get(x_89, 2); +lean_ctor_set(x_90, 0, x_83); +lean_ctor_set(x_90, 1, x_84); +lean_ctor_set(x_90, 2, x_85); +lean_ctor_set(x_90, 3, x_86); +lean_ctor_set(x_90, 4, x_87); +lean_ctor_set(x_90, 5, x_88); +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_82); +x_92 = lean_ctor_get(x_10, 1); lean_inc(x_92); -x_93 = lean_ctor_get(x_89, 3); +lean_dec(x_10); +x_93 = lean_ctor_get(x_92, 0); lean_inc(x_93); -lean_dec(x_89); -x_94 = lean_ctor_get(x_18, 4); +x_94 = lean_ctor_get(x_92, 1); lean_inc(x_94); +x_95 = lean_ctor_get(x_92, 2); +lean_inc(x_95); +x_96 = lean_ctor_get(x_92, 3); +lean_inc(x_96); +x_97 = lean_ctor_get(x_92, 4); +lean_inc(x_97); +lean_dec(x_92); +x_98 = lean_ctor_get(x_18, 5); +lean_inc(x_98); if (lean_is_exclusive(x_18)) { lean_ctor_release(x_18, 0); lean_ctor_release(x_18, 1); lean_ctor_release(x_18, 2); lean_ctor_release(x_18, 3); lean_ctor_release(x_18, 4); - x_95 = x_18; + lean_ctor_release(x_18, 5); + x_99 = x_18; } else { lean_dec_ref(x_18); - x_95 = lean_box(0); + x_99 = lean_box(0); } -if (lean_is_scalar(x_95)) { - x_96 = lean_alloc_ctor(0, 5, 0); +if (lean_is_scalar(x_99)) { + x_100 = lean_alloc_ctor(0, 6, 0); } else { - x_96 = x_95; + x_100 = x_99; } -lean_ctor_set(x_96, 0, x_90); -lean_ctor_set(x_96, 1, x_91); -lean_ctor_set(x_96, 2, x_92); -lean_ctor_set(x_96, 3, x_93); -lean_ctor_set(x_96, 4, x_94); -x_97 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_97, 0, x_88); -lean_ctor_set(x_97, 1, x_96); -x_98 = 0; -x_99 = l_Lean_Elab_Term_SavedState_restore(x_97, x_98, x_2, x_3, x_4, x_5, x_6, x_7, x_24); +lean_ctor_set(x_100, 0, x_93); +lean_ctor_set(x_100, 1, x_94); +lean_ctor_set(x_100, 2, x_95); +lean_ctor_set(x_100, 3, x_96); +lean_ctor_set(x_100, 4, x_97); +lean_ctor_set(x_100, 5, x_98); +x_101 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_101, 0, x_91); +lean_ctor_set(x_101, 1, x_100); +x_102 = 0; +x_103 = l_Lean_Elab_Term_SavedState_restore(x_101, x_102, x_2, x_3, x_4, x_5, x_6, x_7, x_24); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -if (lean_is_exclusive(x_99)) { - lean_ctor_release(x_99, 0); - lean_ctor_release(x_99, 1); - x_101 = x_99; +x_104 = lean_ctor_get(x_103, 1); +lean_inc(x_104); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + lean_ctor_release(x_103, 1); + x_105 = x_103; } else { - lean_dec_ref(x_99); - x_101 = lean_box(0); + lean_dec_ref(x_103); + x_105 = lean_box(0); } -if (lean_is_scalar(x_101)) { - x_102 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_105)) { + x_106 = lean_alloc_ctor(0, 2, 0); } else { - x_102 = x_101; + x_106 = x_105; } -lean_ctor_set(x_102, 0, x_13); -lean_ctor_set(x_102, 1, x_100); -return x_102; +lean_ctor_set(x_106, 0, x_13); +lean_ctor_set(x_106, 1, x_104); +return x_106; } } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; uint8_t x_115; -x_103 = lean_ctor_get(x_12, 0); -lean_inc(x_103); -x_104 = lean_ctor_get(x_12, 1); -lean_inc(x_104); -lean_dec(x_12); -x_105 = lean_st_ref_get(x_7, x_104); -x_106 = lean_ctor_get(x_105, 1); -lean_inc(x_106); -lean_dec(x_105); -x_107 = lean_st_ref_get(x_3, x_106); -x_108 = lean_ctor_get(x_107, 0); +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; +x_107 = lean_ctor_get(x_12, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_12, 1); lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = lean_st_ref_get(x_7, x_109); -x_111 = lean_ctor_get(x_10, 0); -lean_inc(x_111); +lean_dec(x_12); +x_109 = lean_st_ref_get(x_7, x_108); +x_110 = lean_ctor_get(x_109, 1); +lean_inc(x_110); +lean_dec(x_109); +x_111 = lean_st_ref_get(x_3, x_110); x_112 = lean_ctor_get(x_111, 0); lean_inc(x_112); -x_113 = lean_ctor_get(x_110, 0); +x_113 = lean_ctor_get(x_111, 1); lean_inc(x_113); -x_114 = lean_ctor_get(x_110, 1); -lean_inc(x_114); -lean_dec(x_110); -x_115 = !lean_is_exclusive(x_111); -if (x_115 == 0) -{ -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; -x_116 = lean_ctor_get(x_111, 0); -lean_dec(x_116); -x_117 = lean_ctor_get(x_112, 0); +lean_dec(x_111); +x_114 = lean_st_ref_get(x_7, x_113); +x_115 = lean_ctor_get(x_10, 0); +lean_inc(x_115); +x_116 = lean_ctor_get(x_115, 0); +lean_inc(x_116); +x_117 = lean_ctor_get(x_114, 0); lean_inc(x_117); -x_118 = lean_ctor_get(x_112, 1); +x_118 = lean_ctor_get(x_114, 1); lean_inc(x_118); -x_119 = lean_ctor_get(x_112, 2); -lean_inc(x_119); -x_120 = lean_ctor_get(x_112, 3); -lean_inc(x_120); -x_121 = lean_ctor_get(x_112, 4); +lean_dec(x_114); +x_119 = !lean_is_exclusive(x_115); +if (x_119 == 0) +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; uint8_t x_126; +x_120 = lean_ctor_get(x_115, 0); +lean_dec(x_120); +x_121 = lean_ctor_get(x_116, 0); lean_inc(x_121); -lean_dec(x_112); -x_122 = !lean_is_exclusive(x_113); -if (x_122 == 0) +x_122 = lean_ctor_get(x_116, 1); +lean_inc(x_122); +x_123 = lean_ctor_get(x_116, 2); +lean_inc(x_123); +x_124 = lean_ctor_get(x_116, 3); +lean_inc(x_124); +x_125 = lean_ctor_get(x_116, 4); +lean_inc(x_125); +lean_dec(x_116); +x_126 = !lean_is_exclusive(x_117); +if (x_126 == 0) { -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; uint8_t x_133; -x_123 = lean_ctor_get(x_113, 4); -lean_dec(x_123); -x_124 = lean_ctor_get(x_113, 3); -lean_dec(x_124); -x_125 = lean_ctor_get(x_113, 2); -lean_dec(x_125); -x_126 = lean_ctor_get(x_113, 1); -lean_dec(x_126); -x_127 = lean_ctor_get(x_113, 0); +lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; uint8_t x_138; +x_127 = lean_ctor_get(x_117, 4); lean_dec(x_127); -lean_ctor_set(x_113, 4, x_121); -lean_ctor_set(x_113, 3, x_120); -lean_ctor_set(x_113, 2, x_119); -lean_ctor_set(x_113, 1, x_118); -lean_ctor_set(x_113, 0, x_117); -lean_ctor_set(x_111, 0, x_113); -x_128 = lean_ctor_get(x_10, 1); -lean_inc(x_128); -lean_dec(x_10); -x_129 = lean_ctor_get(x_128, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_128, 1); -lean_inc(x_130); -x_131 = lean_ctor_get(x_128, 2); -lean_inc(x_131); -x_132 = lean_ctor_get(x_128, 3); -lean_inc(x_132); +x_128 = lean_ctor_get(x_117, 3); lean_dec(x_128); -x_133 = !lean_is_exclusive(x_108); -if (x_133 == 0) +x_129 = lean_ctor_get(x_117, 2); +lean_dec(x_129); +x_130 = lean_ctor_get(x_117, 1); +lean_dec(x_130); +x_131 = lean_ctor_get(x_117, 0); +lean_dec(x_131); +lean_ctor_set(x_117, 4, x_125); +lean_ctor_set(x_117, 3, x_124); +lean_ctor_set(x_117, 2, x_123); +lean_ctor_set(x_117, 1, x_122); +lean_ctor_set(x_117, 0, x_121); +lean_ctor_set(x_115, 0, x_117); +x_132 = lean_ctor_get(x_10, 1); +lean_inc(x_132); +lean_dec(x_10); +x_133 = lean_ctor_get(x_132, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_132, 1); +lean_inc(x_134); +x_135 = lean_ctor_get(x_132, 2); +lean_inc(x_135); +x_136 = lean_ctor_get(x_132, 3); +lean_inc(x_136); +x_137 = lean_ctor_get(x_132, 4); +lean_inc(x_137); +lean_dec(x_132); +x_138 = !lean_is_exclusive(x_112); +if (x_138 == 0) { -lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; lean_object* x_140; uint8_t x_141; -x_134 = lean_ctor_get(x_108, 3); -lean_dec(x_134); -x_135 = lean_ctor_get(x_108, 2); -lean_dec(x_135); -x_136 = lean_ctor_get(x_108, 1); -lean_dec(x_136); -x_137 = lean_ctor_get(x_108, 0); -lean_dec(x_137); -lean_ctor_set(x_108, 3, x_132); -lean_ctor_set(x_108, 2, x_131); -lean_ctor_set(x_108, 1, x_130); -lean_ctor_set(x_108, 0, x_129); -x_138 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_138, 0, x_111); -lean_ctor_set(x_138, 1, x_108); -x_139 = 0; -x_140 = l_Lean_Elab_Term_SavedState_restore(x_138, x_139, x_2, x_3, x_4, x_5, x_6, x_7, x_114); +lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; uint8_t x_145; lean_object* x_146; uint8_t x_147; +x_139 = lean_ctor_get(x_112, 4); +lean_dec(x_139); +x_140 = lean_ctor_get(x_112, 3); +lean_dec(x_140); +x_141 = lean_ctor_get(x_112, 2); +lean_dec(x_141); +x_142 = lean_ctor_get(x_112, 1); +lean_dec(x_142); +x_143 = lean_ctor_get(x_112, 0); +lean_dec(x_143); +lean_ctor_set(x_112, 4, x_137); +lean_ctor_set(x_112, 3, x_136); +lean_ctor_set(x_112, 2, x_135); +lean_ctor_set(x_112, 1, x_134); +lean_ctor_set(x_112, 0, x_133); +x_144 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_144, 0, x_115); +lean_ctor_set(x_144, 1, x_112); +x_145 = 0; +x_146 = l_Lean_Elab_Term_SavedState_restore(x_144, x_145, x_2, x_3, x_4, x_5, x_6, x_7, x_118); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_141 = !lean_is_exclusive(x_140); -if (x_141 == 0) +x_147 = !lean_is_exclusive(x_146); +if (x_147 == 0) { -lean_object* x_142; -x_142 = lean_ctor_get(x_140, 0); -lean_dec(x_142); -lean_ctor_set_tag(x_140, 1); -lean_ctor_set(x_140, 0, x_103); -return x_140; +lean_object* x_148; +x_148 = lean_ctor_get(x_146, 0); +lean_dec(x_148); +lean_ctor_set_tag(x_146, 1); +lean_ctor_set(x_146, 0, x_107); +return x_146; } else { -lean_object* x_143; lean_object* x_144; -x_143 = lean_ctor_get(x_140, 1); -lean_inc(x_143); -lean_dec(x_140); -x_144 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_144, 0, x_103); -lean_ctor_set(x_144, 1, x_143); -return x_144; +lean_object* x_149; lean_object* x_150; +x_149 = lean_ctor_get(x_146, 1); +lean_inc(x_149); +lean_dec(x_146); +x_150 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_150, 0, x_107); +lean_ctor_set(x_150, 1, x_149); +return x_150; } } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; uint8_t x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_145 = lean_ctor_get(x_108, 4); -lean_inc(x_145); -lean_dec(x_108); -x_146 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_146, 0, x_129); -lean_ctor_set(x_146, 1, x_130); -lean_ctor_set(x_146, 2, x_131); -lean_ctor_set(x_146, 3, x_132); -lean_ctor_set(x_146, 4, x_145); -x_147 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_147, 0, x_111); -lean_ctor_set(x_147, 1, x_146); -x_148 = 0; -x_149 = l_Lean_Elab_Term_SavedState_restore(x_147, x_148, x_2, x_3, x_4, x_5, x_6, x_7, x_114); +lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_151 = lean_ctor_get(x_112, 5); +lean_inc(x_151); +lean_dec(x_112); +x_152 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_152, 0, x_133); +lean_ctor_set(x_152, 1, x_134); +lean_ctor_set(x_152, 2, x_135); +lean_ctor_set(x_152, 3, x_136); +lean_ctor_set(x_152, 4, x_137); +lean_ctor_set(x_152, 5, x_151); +x_153 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_153, 0, x_115); +lean_ctor_set(x_153, 1, x_152); +x_154 = 0; +x_155 = l_Lean_Elab_Term_SavedState_restore(x_153, x_154, x_2, x_3, x_4, x_5, x_6, x_7, x_118); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_150 = lean_ctor_get(x_149, 1); -lean_inc(x_150); -if (lean_is_exclusive(x_149)) { - lean_ctor_release(x_149, 0); - lean_ctor_release(x_149, 1); - x_151 = x_149; +x_156 = lean_ctor_get(x_155, 1); +lean_inc(x_156); +if (lean_is_exclusive(x_155)) { + lean_ctor_release(x_155, 0); + lean_ctor_release(x_155, 1); + x_157 = x_155; } else { - lean_dec_ref(x_149); - x_151 = lean_box(0); + lean_dec_ref(x_155); + x_157 = lean_box(0); } -if (lean_is_scalar(x_151)) { - x_152 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_157)) { + x_158 = lean_alloc_ctor(1, 2, 0); } else { - x_152 = x_151; - lean_ctor_set_tag(x_152, 1); + x_158 = x_157; + lean_ctor_set_tag(x_158, 1); } -lean_ctor_set(x_152, 0, x_103); -lean_ctor_set(x_152, 1, x_150); -return x_152; +lean_ctor_set(x_158, 0, x_107); +lean_ctor_set(x_158, 1, x_156); +return x_158; } } else { -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; uint8_t x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; -x_153 = lean_ctor_get(x_113, 5); -lean_inc(x_153); -lean_dec(x_113); -x_154 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_154, 0, x_117); -lean_ctor_set(x_154, 1, x_118); -lean_ctor_set(x_154, 2, x_119); -lean_ctor_set(x_154, 3, x_120); -lean_ctor_set(x_154, 4, x_121); -lean_ctor_set(x_154, 5, x_153); -lean_ctor_set(x_111, 0, x_154); -x_155 = lean_ctor_get(x_10, 1); -lean_inc(x_155); -lean_dec(x_10); -x_156 = lean_ctor_get(x_155, 0); -lean_inc(x_156); -x_157 = lean_ctor_get(x_155, 1); -lean_inc(x_157); -x_158 = lean_ctor_get(x_155, 2); -lean_inc(x_158); -x_159 = lean_ctor_get(x_155, 3); +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; uint8_t x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_159 = lean_ctor_get(x_117, 5); lean_inc(x_159); -lean_dec(x_155); -x_160 = lean_ctor_get(x_108, 4); -lean_inc(x_160); -if (lean_is_exclusive(x_108)) { - lean_ctor_release(x_108, 0); - lean_ctor_release(x_108, 1); - lean_ctor_release(x_108, 2); - lean_ctor_release(x_108, 3); - lean_ctor_release(x_108, 4); - x_161 = x_108; +lean_dec(x_117); +x_160 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_160, 0, x_121); +lean_ctor_set(x_160, 1, x_122); +lean_ctor_set(x_160, 2, x_123); +lean_ctor_set(x_160, 3, x_124); +lean_ctor_set(x_160, 4, x_125); +lean_ctor_set(x_160, 5, x_159); +lean_ctor_set(x_115, 0, x_160); +x_161 = lean_ctor_get(x_10, 1); +lean_inc(x_161); +lean_dec(x_10); +x_162 = lean_ctor_get(x_161, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_161, 1); +lean_inc(x_163); +x_164 = lean_ctor_get(x_161, 2); +lean_inc(x_164); +x_165 = lean_ctor_get(x_161, 3); +lean_inc(x_165); +x_166 = lean_ctor_get(x_161, 4); +lean_inc(x_166); +lean_dec(x_161); +x_167 = lean_ctor_get(x_112, 5); +lean_inc(x_167); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + lean_ctor_release(x_112, 2); + lean_ctor_release(x_112, 3); + lean_ctor_release(x_112, 4); + lean_ctor_release(x_112, 5); + x_168 = x_112; } else { - lean_dec_ref(x_108); - x_161 = lean_box(0); + lean_dec_ref(x_112); + x_168 = lean_box(0); } -if (lean_is_scalar(x_161)) { - x_162 = lean_alloc_ctor(0, 5, 0); +if (lean_is_scalar(x_168)) { + x_169 = lean_alloc_ctor(0, 6, 0); } else { - x_162 = x_161; + x_169 = x_168; } -lean_ctor_set(x_162, 0, x_156); -lean_ctor_set(x_162, 1, x_157); -lean_ctor_set(x_162, 2, x_158); -lean_ctor_set(x_162, 3, x_159); -lean_ctor_set(x_162, 4, x_160); -x_163 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_163, 0, x_111); -lean_ctor_set(x_163, 1, x_162); -x_164 = 0; -x_165 = l_Lean_Elab_Term_SavedState_restore(x_163, x_164, x_2, x_3, x_4, x_5, x_6, x_7, x_114); +lean_ctor_set(x_169, 0, x_162); +lean_ctor_set(x_169, 1, x_163); +lean_ctor_set(x_169, 2, x_164); +lean_ctor_set(x_169, 3, x_165); +lean_ctor_set(x_169, 4, x_166); +lean_ctor_set(x_169, 5, x_167); +x_170 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_170, 0, x_115); +lean_ctor_set(x_170, 1, x_169); +x_171 = 0; +x_172 = l_Lean_Elab_Term_SavedState_restore(x_170, x_171, x_2, x_3, x_4, x_5, x_6, x_7, x_118); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_166 = lean_ctor_get(x_165, 1); -lean_inc(x_166); -if (lean_is_exclusive(x_165)) { - lean_ctor_release(x_165, 0); - lean_ctor_release(x_165, 1); - x_167 = x_165; +x_173 = lean_ctor_get(x_172, 1); +lean_inc(x_173); +if (lean_is_exclusive(x_172)) { + lean_ctor_release(x_172, 0); + lean_ctor_release(x_172, 1); + x_174 = x_172; } else { - lean_dec_ref(x_165); - x_167 = lean_box(0); + lean_dec_ref(x_172); + x_174 = lean_box(0); } -if (lean_is_scalar(x_167)) { - x_168 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_174)) { + x_175 = lean_alloc_ctor(1, 2, 0); } else { - x_168 = x_167; - lean_ctor_set_tag(x_168, 1); + x_175 = x_174; + lean_ctor_set_tag(x_175, 1); } -lean_ctor_set(x_168, 0, x_103); -lean_ctor_set(x_168, 1, x_166); -return x_168; +lean_ctor_set(x_175, 0, x_107); +lean_ctor_set(x_175, 1, x_173); +return x_175; } } else { -lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; 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; uint8_t x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_169 = lean_ctor_get(x_111, 1); -lean_inc(x_169); -lean_dec(x_111); -x_170 = lean_ctor_get(x_112, 0); -lean_inc(x_170); -x_171 = lean_ctor_get(x_112, 1); -lean_inc(x_171); -x_172 = lean_ctor_get(x_112, 2); -lean_inc(x_172); -x_173 = lean_ctor_get(x_112, 3); -lean_inc(x_173); -x_174 = lean_ctor_get(x_112, 4); -lean_inc(x_174); -lean_dec(x_112); -x_175 = lean_ctor_get(x_113, 5); -lean_inc(x_175); -if (lean_is_exclusive(x_113)) { - lean_ctor_release(x_113, 0); - lean_ctor_release(x_113, 1); - lean_ctor_release(x_113, 2); - lean_ctor_release(x_113, 3); - lean_ctor_release(x_113, 4); - lean_ctor_release(x_113, 5); - x_176 = x_113; -} else { - lean_dec_ref(x_113); - x_176 = lean_box(0); -} -if (lean_is_scalar(x_176)) { - x_177 = lean_alloc_ctor(0, 6, 0); -} else { - x_177 = x_176; -} -lean_ctor_set(x_177, 0, x_170); -lean_ctor_set(x_177, 1, x_171); -lean_ctor_set(x_177, 2, x_172); -lean_ctor_set(x_177, 3, x_173); -lean_ctor_set(x_177, 4, x_174); -lean_ctor_set(x_177, 5, x_175); -x_178 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_178, 0, x_177); -lean_ctor_set(x_178, 1, x_169); -x_179 = lean_ctor_get(x_10, 1); +lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; uint8_t x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_176 = lean_ctor_get(x_115, 1); +lean_inc(x_176); +lean_dec(x_115); +x_177 = lean_ctor_get(x_116, 0); +lean_inc(x_177); +x_178 = lean_ctor_get(x_116, 1); +lean_inc(x_178); +x_179 = lean_ctor_get(x_116, 2); lean_inc(x_179); -lean_dec(x_10); -x_180 = lean_ctor_get(x_179, 0); +x_180 = lean_ctor_get(x_116, 3); lean_inc(x_180); -x_181 = lean_ctor_get(x_179, 1); +x_181 = lean_ctor_get(x_116, 4); lean_inc(x_181); -x_182 = lean_ctor_get(x_179, 2); +lean_dec(x_116); +x_182 = lean_ctor_get(x_117, 5); lean_inc(x_182); -x_183 = lean_ctor_get(x_179, 3); -lean_inc(x_183); -lean_dec(x_179); -x_184 = lean_ctor_get(x_108, 4); -lean_inc(x_184); -if (lean_is_exclusive(x_108)) { - lean_ctor_release(x_108, 0); - lean_ctor_release(x_108, 1); - lean_ctor_release(x_108, 2); - lean_ctor_release(x_108, 3); - lean_ctor_release(x_108, 4); - x_185 = x_108; +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + lean_ctor_release(x_117, 2); + lean_ctor_release(x_117, 3); + lean_ctor_release(x_117, 4); + lean_ctor_release(x_117, 5); + x_183 = x_117; +} else { + lean_dec_ref(x_117); + x_183 = lean_box(0); +} +if (lean_is_scalar(x_183)) { + x_184 = lean_alloc_ctor(0, 6, 0); } else { - lean_dec_ref(x_108); - x_185 = lean_box(0); + x_184 = x_183; } -if (lean_is_scalar(x_185)) { - x_186 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_184, 0, x_177); +lean_ctor_set(x_184, 1, x_178); +lean_ctor_set(x_184, 2, x_179); +lean_ctor_set(x_184, 3, x_180); +lean_ctor_set(x_184, 4, x_181); +lean_ctor_set(x_184, 5, x_182); +x_185 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_185, 0, x_184); +lean_ctor_set(x_185, 1, x_176); +x_186 = lean_ctor_get(x_10, 1); +lean_inc(x_186); +lean_dec(x_10); +x_187 = lean_ctor_get(x_186, 0); +lean_inc(x_187); +x_188 = lean_ctor_get(x_186, 1); +lean_inc(x_188); +x_189 = lean_ctor_get(x_186, 2); +lean_inc(x_189); +x_190 = lean_ctor_get(x_186, 3); +lean_inc(x_190); +x_191 = lean_ctor_get(x_186, 4); +lean_inc(x_191); +lean_dec(x_186); +x_192 = lean_ctor_get(x_112, 5); +lean_inc(x_192); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + lean_ctor_release(x_112, 2); + lean_ctor_release(x_112, 3); + lean_ctor_release(x_112, 4); + lean_ctor_release(x_112, 5); + x_193 = x_112; } else { - x_186 = x_185; + lean_dec_ref(x_112); + x_193 = lean_box(0); +} +if (lean_is_scalar(x_193)) { + x_194 = lean_alloc_ctor(0, 6, 0); +} else { + x_194 = x_193; } -lean_ctor_set(x_186, 0, x_180); -lean_ctor_set(x_186, 1, x_181); -lean_ctor_set(x_186, 2, x_182); -lean_ctor_set(x_186, 3, x_183); -lean_ctor_set(x_186, 4, x_184); -x_187 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_187, 0, x_178); -lean_ctor_set(x_187, 1, x_186); -x_188 = 0; -x_189 = l_Lean_Elab_Term_SavedState_restore(x_187, x_188, x_2, x_3, x_4, x_5, x_6, x_7, x_114); +lean_ctor_set(x_194, 0, x_187); +lean_ctor_set(x_194, 1, x_188); +lean_ctor_set(x_194, 2, x_189); +lean_ctor_set(x_194, 3, x_190); +lean_ctor_set(x_194, 4, x_191); +lean_ctor_set(x_194, 5, x_192); +x_195 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_195, 0, x_185); +lean_ctor_set(x_195, 1, x_194); +x_196 = 0; +x_197 = l_Lean_Elab_Term_SavedState_restore(x_195, x_196, x_2, x_3, x_4, x_5, x_6, x_7, x_118); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_190 = lean_ctor_get(x_189, 1); -lean_inc(x_190); -if (lean_is_exclusive(x_189)) { - lean_ctor_release(x_189, 0); - lean_ctor_release(x_189, 1); - x_191 = x_189; +x_198 = lean_ctor_get(x_197, 1); +lean_inc(x_198); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + lean_ctor_release(x_197, 1); + x_199 = x_197; } else { - lean_dec_ref(x_189); - x_191 = lean_box(0); + lean_dec_ref(x_197); + x_199 = lean_box(0); } -if (lean_is_scalar(x_191)) { - x_192 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_199)) { + x_200 = lean_alloc_ctor(1, 2, 0); } else { - x_192 = x_191; - lean_ctor_set_tag(x_192, 1); + x_200 = x_199; + lean_ctor_set_tag(x_200, 1); } -lean_ctor_set(x_192, 0, x_103); -lean_ctor_set(x_192, 1, x_190); -return x_192; +lean_ctor_set(x_200, 0, x_107); +lean_ctor_set(x_200, 1, x_198); +return x_200; } } } @@ -8794,7 +8909,7 @@ x_8 = l_Lean_Elab_mkElabAttribute___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_2191_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_2187_(lean_object* x_1) { _start: { lean_object* x_2; @@ -8909,7 +9024,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_11, 3); +x_12 = lean_ctor_get(x_11, 4); lean_inc(x_12); lean_dec(x_11); lean_ctor_set(x_9, 0, x_12); @@ -8923,7 +9038,7 @@ x_14 = lean_ctor_get(x_9, 1); lean_inc(x_14); lean_inc(x_13); lean_dec(x_9); -x_15 = lean_ctor_get(x_13, 3); +x_15 = lean_ctor_get(x_13, 4); lean_inc(x_15); lean_dec(x_13); x_16 = lean_alloc_ctor(0, 2, 0); @@ -9136,42 +9251,45 @@ return x_22; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; x_23 = lean_ctor_get(x_12, 1); x_24 = lean_ctor_get(x_12, 2); x_25 = lean_ctor_get(x_12, 3); x_26 = lean_ctor_get(x_12, 4); +x_27 = lean_ctor_get(x_12, 5); +lean_inc(x_27); lean_inc(x_26); lean_inc(x_25); lean_inc(x_24); lean_inc(x_23); lean_dec(x_12); -x_27 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_27, 0, x_1); -lean_ctor_set(x_27, 1, x_23); -lean_ctor_set(x_27, 2, x_24); -lean_ctor_set(x_27, 3, x_25); -lean_ctor_set(x_27, 4, x_26); -x_28 = lean_st_ref_set(x_3, x_27, x_13); -x_29 = lean_ctor_get(x_28, 1); -lean_inc(x_29); -if (lean_is_exclusive(x_28)) { - lean_ctor_release(x_28, 0); - lean_ctor_release(x_28, 1); - x_30 = x_28; +x_28 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_28, 0, x_1); +lean_ctor_set(x_28, 1, x_23); +lean_ctor_set(x_28, 2, x_24); +lean_ctor_set(x_28, 3, x_25); +lean_ctor_set(x_28, 4, x_26); +lean_ctor_set(x_28, 5, x_27); +x_29 = lean_st_ref_set(x_3, x_28, x_13); +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + x_31 = x_29; } else { - lean_dec_ref(x_28); - x_30 = lean_box(0); + lean_dec_ref(x_29); + x_31 = lean_box(0); } -x_31 = lean_box(0); -if (lean_is_scalar(x_30)) { - x_32 = lean_alloc_ctor(0, 2, 0); +x_32 = lean_box(0); +if (lean_is_scalar(x_31)) { + x_33 = lean_alloc_ctor(0, 2, 0); } else { - x_32 = x_30; + x_33 = x_31; } -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_29); -return x_32; +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_30); +return x_33; } } } @@ -13746,7 +13864,7 @@ lean_dec(x_10); x_12 = lean_st_ref_get(x_4, x_11); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); -x_14 = lean_ctor_get(x_13, 4); +x_14 = lean_ctor_get(x_13, 5); lean_inc(x_14); lean_dec(x_13); x_15 = lean_ctor_get_uint8(x_14, sizeof(void*)*2); @@ -13798,7 +13916,7 @@ lean_inc(x_28); x_29 = lean_ctor_get(x_27, 1); lean_inc(x_29); lean_dec(x_27); -x_30 = lean_ctor_get(x_28, 4); +x_30 = lean_ctor_get(x_28, 5); lean_inc(x_30); lean_dec(x_28); x_31 = lean_ctor_get(x_30, 1); @@ -13823,7 +13941,7 @@ lean_dec(x_35); x_37 = lean_st_ref_take(x_4, x_36); x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -x_39 = lean_ctor_get(x_38, 4); +x_39 = lean_ctor_get(x_38, 5); lean_inc(x_39); x_40 = lean_ctor_get(x_37, 1); lean_inc(x_40); @@ -13832,7 +13950,7 @@ x_41 = !lean_is_exclusive(x_38); if (x_41 == 0) { lean_object* x_42; uint8_t x_43; -x_42 = lean_ctor_get(x_38, 4); +x_42 = lean_ctor_get(x_38, 5); lean_dec(x_42); x_43 = !lean_is_exclusive(x_39); if (x_43 == 0) @@ -13877,7 +13995,7 @@ x_54 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_54, 0, x_52); lean_ctor_set(x_54, 1, x_53); lean_ctor_set_uint8(x_54, sizeof(void*)*2, x_51); -lean_ctor_set(x_38, 4, x_54); +lean_ctor_set(x_38, 5, x_54); x_55 = lean_st_ref_set(x_4, x_38, x_40); lean_dec(x_4); x_56 = lean_ctor_get(x_55, 1); @@ -13902,298 +14020,304 @@ return x_58; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; x_59 = lean_ctor_get(x_38, 0); x_60 = lean_ctor_get(x_38, 1); x_61 = lean_ctor_get(x_38, 2); x_62 = lean_ctor_get(x_38, 3); +x_63 = lean_ctor_get(x_38, 4); +lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); lean_dec(x_38); -x_63 = lean_ctor_get_uint8(x_39, sizeof(void*)*2); -x_64 = lean_ctor_get(x_39, 0); -lean_inc(x_64); +x_64 = lean_ctor_get_uint8(x_39, sizeof(void*)*2); +x_65 = lean_ctor_get(x_39, 0); +lean_inc(x_65); if (lean_is_exclusive(x_39)) { lean_ctor_release(x_39, 0); lean_ctor_release(x_39, 1); - x_65 = x_39; + x_66 = x_39; } else { lean_dec_ref(x_39); - x_65 = lean_box(0); + x_66 = lean_box(0); } -x_66 = l_Std_PersistentArray_push___rarg(x_20, x_33); -if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 1); +x_67 = l_Std_PersistentArray_push___rarg(x_20, x_33); +if (lean_is_scalar(x_66)) { + x_68 = lean_alloc_ctor(0, 2, 1); } else { - x_67 = x_65; + x_68 = x_66; } -lean_ctor_set(x_67, 0, x_64); -lean_ctor_set(x_67, 1, x_66); -lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_63); -x_68 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_68, 0, x_59); -lean_ctor_set(x_68, 1, x_60); -lean_ctor_set(x_68, 2, x_61); -lean_ctor_set(x_68, 3, x_62); -lean_ctor_set(x_68, 4, x_67); -x_69 = lean_st_ref_set(x_4, x_68, x_40); +lean_ctor_set(x_68, 0, x_65); +lean_ctor_set(x_68, 1, x_67); +lean_ctor_set_uint8(x_68, sizeof(void*)*2, x_64); +x_69 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_69, 0, x_59); +lean_ctor_set(x_69, 1, x_60); +lean_ctor_set(x_69, 2, x_61); +lean_ctor_set(x_69, 3, x_62); +lean_ctor_set(x_69, 4, x_63); +lean_ctor_set(x_69, 5, x_68); +x_70 = lean_st_ref_set(x_4, x_69, x_40); lean_dec(x_4); -x_70 = lean_ctor_get(x_69, 1); -lean_inc(x_70); -if (lean_is_exclusive(x_69)) { - lean_ctor_release(x_69, 0); - lean_ctor_release(x_69, 1); - x_71 = x_69; +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_72 = x_70; } else { - lean_dec_ref(x_69); - x_71 = lean_box(0); + lean_dec_ref(x_70); + x_72 = lean_box(0); } -if (lean_is_scalar(x_71)) { - x_72 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_72)) { + x_73 = lean_alloc_ctor(0, 2, 0); } else { - x_72 = x_71; + x_73 = x_72; } -lean_ctor_set(x_72, 0, x_23); -lean_ctor_set(x_72, 1, x_70); -return x_72; +lean_ctor_set(x_73, 0, x_23); +lean_ctor_set(x_73, 1, x_71); +return x_73; } } else { -uint8_t x_73; +uint8_t x_74; lean_dec(x_23); lean_dec(x_20); lean_dec(x_8); lean_dec(x_4); -x_73 = !lean_is_exclusive(x_32); -if (x_73 == 0) +x_74 = !lean_is_exclusive(x_32); +if (x_74 == 0) { return x_32; } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_32, 0); -x_75 = lean_ctor_get(x_32, 1); +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_32, 0); +x_76 = lean_ctor_get(x_32, 1); +lean_inc(x_76); lean_inc(x_75); -lean_inc(x_74); lean_dec(x_32); -x_76 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_76, 0, x_74); -lean_ctor_set(x_76, 1, x_75); -return x_76; +x_77 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_77, 0, x_75); +lean_ctor_set(x_77, 1, x_76); +return x_77; } } } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_77 = lean_ctor_get(x_22, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_22, 1); +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_78 = lean_ctor_get(x_22, 0); lean_inc(x_78); +x_79 = lean_ctor_get(x_22, 1); +lean_inc(x_79); lean_dec(x_22); -x_79 = lean_st_ref_get(x_8, x_78); -x_80 = lean_ctor_get(x_79, 1); -lean_inc(x_80); -lean_dec(x_79); -x_81 = lean_st_ref_get(x_4, x_80); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_80 = lean_st_ref_get(x_8, x_79); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +lean_dec(x_80); +x_82 = lean_st_ref_get(x_4, x_81); +x_83 = lean_ctor_get(x_82, 0); lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_ctor_get(x_82, 4); +x_84 = lean_ctor_get(x_82, 1); lean_inc(x_84); lean_dec(x_82); -x_85 = lean_ctor_get(x_84, 1); +x_85 = lean_ctor_get(x_83, 5); lean_inc(x_85); -lean_dec(x_84); +lean_dec(x_83); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); lean_inc(x_8); lean_inc(x_4); -x_86 = lean_apply_8(x_2, x_85, x_3, x_4, x_5, x_6, x_7, x_8, x_83); -if (lean_obj_tag(x_86) == 0) +x_87 = lean_apply_8(x_2, x_86, x_3, x_4, x_5, x_6, x_7, x_8, x_84); +if (lean_obj_tag(x_87) == 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; uint8_t x_95; -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; +x_88 = lean_ctor_get(x_87, 0); lean_inc(x_88); -lean_dec(x_86); -x_89 = lean_st_ref_get(x_8, x_88); +x_89 = lean_ctor_get(x_87, 1); +lean_inc(x_89); +lean_dec(x_87); +x_90 = lean_st_ref_get(x_8, x_89); lean_dec(x_8); -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); -lean_dec(x_89); -x_91 = lean_st_ref_take(x_4, x_90); -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_92, 4); +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +lean_dec(x_90); +x_92 = lean_st_ref_take(x_4, x_91); +x_93 = lean_ctor_get(x_92, 0); lean_inc(x_93); -x_94 = lean_ctor_get(x_91, 1); +x_94 = lean_ctor_get(x_93, 5); lean_inc(x_94); -lean_dec(x_91); -x_95 = !lean_is_exclusive(x_92); -if (x_95 == 0) +x_95 = lean_ctor_get(x_92, 1); +lean_inc(x_95); +lean_dec(x_92); +x_96 = !lean_is_exclusive(x_93); +if (x_96 == 0) { -lean_object* x_96; uint8_t x_97; -x_96 = lean_ctor_get(x_92, 4); -lean_dec(x_96); -x_97 = !lean_is_exclusive(x_93); -if (x_97 == 0) +lean_object* x_97; uint8_t x_98; +x_97 = lean_ctor_get(x_93, 5); +lean_dec(x_97); +x_98 = !lean_is_exclusive(x_94); +if (x_98 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; uint8_t x_101; -x_98 = lean_ctor_get(x_93, 1); -lean_dec(x_98); -x_99 = l_Std_PersistentArray_push___rarg(x_20, x_87); -lean_ctor_set(x_93, 1, x_99); -x_100 = lean_st_ref_set(x_4, x_92, x_94); +lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; +x_99 = lean_ctor_get(x_94, 1); +lean_dec(x_99); +x_100 = l_Std_PersistentArray_push___rarg(x_20, x_88); +lean_ctor_set(x_94, 1, x_100); +x_101 = lean_st_ref_set(x_4, x_93, x_95); lean_dec(x_4); -x_101 = !lean_is_exclusive(x_100); -if (x_101 == 0) +x_102 = !lean_is_exclusive(x_101); +if (x_102 == 0) { -lean_object* x_102; -x_102 = lean_ctor_get(x_100, 0); -lean_dec(x_102); -lean_ctor_set_tag(x_100, 1); -lean_ctor_set(x_100, 0, x_77); -return x_100; +lean_object* x_103; +x_103 = lean_ctor_get(x_101, 0); +lean_dec(x_103); +lean_ctor_set_tag(x_101, 1); +lean_ctor_set(x_101, 0, x_78); +return x_101; } else { -lean_object* x_103; lean_object* x_104; -x_103 = lean_ctor_get(x_100, 1); -lean_inc(x_103); -lean_dec(x_100); -x_104 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_104, 0, x_77); -lean_ctor_set(x_104, 1, x_103); -return x_104; +lean_object* x_104; lean_object* x_105; +x_104 = lean_ctor_get(x_101, 1); +lean_inc(x_104); +lean_dec(x_101); +x_105 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_105, 0, x_78); +lean_ctor_set(x_105, 1, x_104); +return x_105; } } else { -uint8_t x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_105 = lean_ctor_get_uint8(x_93, sizeof(void*)*2); -x_106 = lean_ctor_get(x_93, 0); -lean_inc(x_106); -lean_dec(x_93); -x_107 = l_Std_PersistentArray_push___rarg(x_20, x_87); -x_108 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_108, 0, x_106); -lean_ctor_set(x_108, 1, x_107); -lean_ctor_set_uint8(x_108, sizeof(void*)*2, x_105); -lean_ctor_set(x_92, 4, x_108); -x_109 = lean_st_ref_set(x_4, x_92, x_94); +uint8_t x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_106 = lean_ctor_get_uint8(x_94, sizeof(void*)*2); +x_107 = lean_ctor_get(x_94, 0); +lean_inc(x_107); +lean_dec(x_94); +x_108 = l_Std_PersistentArray_push___rarg(x_20, x_88); +x_109 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 1, x_108); +lean_ctor_set_uint8(x_109, sizeof(void*)*2, x_106); +lean_ctor_set(x_93, 5, x_109); +x_110 = lean_st_ref_set(x_4, x_93, x_95); lean_dec(x_4); -x_110 = lean_ctor_get(x_109, 1); -lean_inc(x_110); -if (lean_is_exclusive(x_109)) { - lean_ctor_release(x_109, 0); - lean_ctor_release(x_109, 1); - x_111 = x_109; +x_111 = lean_ctor_get(x_110, 1); +lean_inc(x_111); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_112 = x_110; } else { - lean_dec_ref(x_109); - x_111 = lean_box(0); + lean_dec_ref(x_110); + x_112 = lean_box(0); } -if (lean_is_scalar(x_111)) { - x_112 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_112)) { + x_113 = lean_alloc_ctor(1, 2, 0); } else { - x_112 = x_111; - lean_ctor_set_tag(x_112, 1); + x_113 = x_112; + lean_ctor_set_tag(x_113, 1); } -lean_ctor_set(x_112, 0, x_77); -lean_ctor_set(x_112, 1, x_110); -return x_112; +lean_ctor_set(x_113, 0, x_78); +lean_ctor_set(x_113, 1, x_111); +return x_113; } } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; uint8_t x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_113 = lean_ctor_get(x_92, 0); -x_114 = lean_ctor_get(x_92, 1); -x_115 = lean_ctor_get(x_92, 2); -x_116 = lean_ctor_get(x_92, 3); +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_114 = lean_ctor_get(x_93, 0); +x_115 = lean_ctor_get(x_93, 1); +x_116 = lean_ctor_get(x_93, 2); +x_117 = lean_ctor_get(x_93, 3); +x_118 = lean_ctor_get(x_93, 4); +lean_inc(x_118); +lean_inc(x_117); lean_inc(x_116); lean_inc(x_115); lean_inc(x_114); -lean_inc(x_113); -lean_dec(x_92); -x_117 = lean_ctor_get_uint8(x_93, sizeof(void*)*2); -x_118 = lean_ctor_get(x_93, 0); -lean_inc(x_118); -if (lean_is_exclusive(x_93)) { - lean_ctor_release(x_93, 0); - lean_ctor_release(x_93, 1); - x_119 = x_93; +lean_dec(x_93); +x_119 = lean_ctor_get_uint8(x_94, sizeof(void*)*2); +x_120 = lean_ctor_get(x_94, 0); +lean_inc(x_120); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_121 = x_94; } else { - lean_dec_ref(x_93); - x_119 = lean_box(0); + lean_dec_ref(x_94); + x_121 = lean_box(0); } -x_120 = l_Std_PersistentArray_push___rarg(x_20, x_87); -if (lean_is_scalar(x_119)) { - x_121 = lean_alloc_ctor(0, 2, 1); +x_122 = l_Std_PersistentArray_push___rarg(x_20, x_88); +if (lean_is_scalar(x_121)) { + x_123 = lean_alloc_ctor(0, 2, 1); } else { - x_121 = x_119; + x_123 = x_121; } -lean_ctor_set(x_121, 0, x_118); -lean_ctor_set(x_121, 1, x_120); -lean_ctor_set_uint8(x_121, sizeof(void*)*2, x_117); -x_122 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_122, 0, x_113); -lean_ctor_set(x_122, 1, x_114); -lean_ctor_set(x_122, 2, x_115); -lean_ctor_set(x_122, 3, x_116); -lean_ctor_set(x_122, 4, x_121); -x_123 = lean_st_ref_set(x_4, x_122, x_94); -lean_dec(x_4); -x_124 = lean_ctor_get(x_123, 1); -lean_inc(x_124); -if (lean_is_exclusive(x_123)) { - lean_ctor_release(x_123, 0); - lean_ctor_release(x_123, 1); - x_125 = x_123; +lean_ctor_set(x_123, 0, x_120); +lean_ctor_set(x_123, 1, x_122); +lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_119); +x_124 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_124, 0, x_114); +lean_ctor_set(x_124, 1, x_115); +lean_ctor_set(x_124, 2, x_116); +lean_ctor_set(x_124, 3, x_117); +lean_ctor_set(x_124, 4, x_118); +lean_ctor_set(x_124, 5, x_123); +x_125 = lean_st_ref_set(x_4, x_124, x_95); +lean_dec(x_4); +x_126 = lean_ctor_get(x_125, 1); +lean_inc(x_126); +if (lean_is_exclusive(x_125)) { + lean_ctor_release(x_125, 0); + lean_ctor_release(x_125, 1); + x_127 = x_125; } else { - lean_dec_ref(x_123); - x_125 = lean_box(0); + lean_dec_ref(x_125); + x_127 = lean_box(0); } -if (lean_is_scalar(x_125)) { - x_126 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_127)) { + x_128 = lean_alloc_ctor(1, 2, 0); } else { - x_126 = x_125; - lean_ctor_set_tag(x_126, 1); + x_128 = x_127; + lean_ctor_set_tag(x_128, 1); } -lean_ctor_set(x_126, 0, x_77); -lean_ctor_set(x_126, 1, x_124); -return x_126; +lean_ctor_set(x_128, 0, x_78); +lean_ctor_set(x_128, 1, x_126); +return x_128; } } else { -uint8_t x_127; -lean_dec(x_77); +uint8_t x_129; +lean_dec(x_78); lean_dec(x_20); lean_dec(x_8); lean_dec(x_4); -x_127 = !lean_is_exclusive(x_86); -if (x_127 == 0) +x_129 = !lean_is_exclusive(x_87); +if (x_129 == 0) { -return x_86; +return x_87; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; -x_128 = lean_ctor_get(x_86, 0); -x_129 = lean_ctor_get(x_86, 1); -lean_inc(x_129); -lean_inc(x_128); -lean_dec(x_86); -x_130 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_130, 0, x_128); -lean_ctor_set(x_130, 1, x_129); -return x_130; +lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_130 = lean_ctor_get(x_87, 0); +x_131 = lean_ctor_get(x_87, 1); +lean_inc(x_131); +lean_inc(x_130); +lean_dec(x_87); +x_132 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_132, 0, x_130); +lean_ctor_set(x_132, 1, x_131); +return x_132; } } } @@ -14359,146 +14483,7 @@ lean_dec(x_4); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVar(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_11 = lean_st_ref_get(x_9, x_10); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_st_ref_take(x_5, x_12); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = !lean_is_exclusive(x_14); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_18, 0, x_2); -lean_ctor_set(x_18, 1, x_1); -lean_ctor_set(x_18, 2, x_3); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -lean_ctor_set(x_14, 1, x_19); -x_20 = lean_st_ref_set(x_5, x_14, x_15); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_20, 0); -lean_dec(x_22); -x_23 = lean_box(0); -lean_ctor_set(x_20, 0, x_23); -return x_20; -} -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_20, 1); -lean_inc(x_24); -lean_dec(x_20); -x_25 = lean_box(0); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -return x_26; -} -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_27 = lean_ctor_get(x_14, 0); -x_28 = lean_ctor_get(x_14, 1); -x_29 = lean_ctor_get(x_14, 2); -x_30 = lean_ctor_get(x_14, 3); -x_31 = lean_ctor_get(x_14, 4); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_14); -x_32 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_32, 0, x_2); -lean_ctor_set(x_32, 1, x_1); -lean_ctor_set(x_32, 2, x_3); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_28); -x_34 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_34, 0, x_27); -lean_ctor_set(x_34, 1, x_33); -lean_ctor_set(x_34, 2, x_29); -lean_ctor_set(x_34, 3, x_30); -lean_ctor_set(x_34, 4, x_31); -x_35 = lean_st_ref_set(x_5, x_34, x_15); -x_36 = lean_ctor_get(x_35, 1); -lean_inc(x_36); -if (lean_is_exclusive(x_35)) { - lean_ctor_release(x_35, 0); - lean_ctor_release(x_35, 1); - x_37 = x_35; -} else { - lean_dec_ref(x_35); - x_37 = lean_box(0); -} -x_38 = lean_box(0); -if (lean_is_scalar(x_37)) { - x_39 = lean_alloc_ctor(0, 2, 0); -} else { - x_39 = x_37; -} -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_36); -return x_39; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVar___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_Term_registerSyntheticMVar(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_7, 5); -lean_inc(x_10); -x_11 = l_Lean_Elab_Term_registerSyntheticMVar(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_7); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -14534,7 +14519,7 @@ switch (x_13) { case 0: { lean_object* x_14; uint8_t x_15; -x_14 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_9, x_2, x_3); +x_14 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_9, x_2, x_3); x_15 = 0; lean_ctor_set(x_1, 0, x_14); lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_15); @@ -14554,7 +14539,7 @@ return x_1; default: { lean_object* x_17; uint8_t x_18; -x_17 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_12, x_2, x_3); +x_17 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_12, x_2, x_3); x_18 = 0; lean_ctor_set(x_1, 3, x_17); lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_18); @@ -14579,7 +14564,7 @@ switch (x_23) { case 0: { lean_object* x_24; uint8_t x_25; lean_object* x_26; -x_24 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_19, x_2, x_3); +x_24 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_19, x_2, x_3); x_25 = 0; x_26 = lean_alloc_ctor(1, 4, 1); lean_ctor_set(x_26, 0, x_24); @@ -14606,7 +14591,7 @@ return x_28; default: { lean_object* x_29; uint8_t x_30; lean_object* x_31; -x_29 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_22, x_2, x_3); +x_29 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_22, x_2, x_3); x_30 = 0; x_31 = lean_alloc_ctor(1, 4, 1); lean_ctor_set(x_31, 0, x_19); @@ -14639,7 +14624,7 @@ x_38 = l_Std_RBNode_isRed___rarg(x_33); if (x_38 == 0) { lean_object* x_39; uint8_t x_40; -x_39 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_33, x_2, x_3); +x_39 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_33, x_2, x_3); x_40 = 1; lean_ctor_set(x_1, 0, x_39); lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_40); @@ -14648,7 +14633,7 @@ return x_1; else { lean_object* x_41; lean_object* x_42; -x_41 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_33, x_2, x_3); +x_41 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_33, x_2, x_3); x_42 = lean_ctor_get(x_41, 0); lean_inc(x_42); if (lean_obj_tag(x_42) == 0) @@ -15349,7 +15334,7 @@ x_201 = l_Std_RBNode_isRed___rarg(x_36); if (x_201 == 0) { lean_object* x_202; uint8_t x_203; -x_202 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_36, x_2, x_3); +x_202 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_36, x_2, x_3); x_203 = 1; lean_ctor_set(x_1, 3, x_202); lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_203); @@ -15358,7 +15343,7 @@ return x_1; else { lean_object* x_204; lean_object* x_205; -x_204 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_36, x_2, x_3); +x_204 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_36, x_2, x_3); x_205 = lean_ctor_get(x_204, 0); lean_inc(x_205); if (lean_obj_tag(x_205) == 0) @@ -16055,7 +16040,7 @@ x_367 = l_Std_RBNode_isRed___rarg(x_362); if (x_367 == 0) { lean_object* x_368; uint8_t x_369; lean_object* x_370; -x_368 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_362, x_2, x_3); +x_368 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_362, x_2, x_3); x_369 = 1; x_370 = lean_alloc_ctor(1, 4, 1); lean_ctor_set(x_370, 0, x_368); @@ -16068,7 +16053,7 @@ return x_370; else { lean_object* x_371; lean_object* x_372; -x_371 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_362, x_2, x_3); +x_371 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_362, x_2, x_3); x_372 = lean_ctor_get(x_371, 0); lean_inc(x_372); if (lean_obj_tag(x_372) == 0) @@ -16509,7 +16494,7 @@ x_455 = l_Std_RBNode_isRed___rarg(x_365); if (x_455 == 0) { lean_object* x_456; uint8_t x_457; lean_object* x_458; -x_456 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_365, x_2, x_3); +x_456 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_365, x_2, x_3); x_457 = 1; x_458 = lean_alloc_ctor(1, 4, 1); lean_ctor_set(x_458, 0, x_362); @@ -16522,7 +16507,7 @@ return x_458; else { lean_object* x_459; lean_object* x_460; -x_459 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_365, x_2, x_3); +x_459 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_365, x_2, x_3); x_460 = lean_ctor_get(x_459, 0); lean_inc(x_460); if (lean_obj_tag(x_460) == 0) @@ -16948,7 +16933,7 @@ return x_540; } } } -LEAN_EXPORT lean_object* l_Std_RBNode_insert___at_Lean_Elab_Term_registerMVarErrorInfo___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_RBNode_insert___at_Lean_Elab_Term_registerSyntheticMVar___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -16956,147 +16941,157 @@ x_4 = l_Std_RBNode_isRed___rarg(x_1); if (x_4 == 0) { lean_object* x_5; -x_5 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_1, x_2, x_3); +x_5 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_1, x_2, x_3); return x_5; } else { lean_object* x_6; lean_object* x_7; -x_6 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_1, x_2, x_3); +x_6 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerSyntheticMVar___spec__2(x_1, x_2, x_3); x_7 = l_Std_RBNode_setBlack___rarg(x_6); return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorInfo(lean_object* x_1, lean_object* x_2, lean_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_Term_registerSyntheticMVar(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_9 = lean_st_ref_get(x_7, x_8); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_st_ref_take(x_3, x_10); -x_12 = lean_ctor_get(x_11, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_11 = lean_st_ref_get(x_9, x_10); +x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); lean_dec(x_11); -x_14 = !lean_is_exclusive(x_12); -if (x_14 == 0) +x_13 = lean_st_ref_take(x_5, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = !lean_is_exclusive(x_14); +if (x_16 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_15 = lean_ctor_get(x_12, 2); -x_16 = lean_ctor_get(x_1, 0); -lean_inc(x_16); -x_17 = l_Std_RBNode_insert___at_Lean_Elab_Term_registerMVarErrorInfo___spec__1(x_15, x_16, x_1); -lean_ctor_set(x_12, 2, x_17); -x_18 = lean_st_ref_set(x_3, x_12, x_13); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_17 = lean_ctor_get(x_14, 1); +x_18 = lean_ctor_get(x_14, 2); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 1, x_3); +lean_inc(x_2); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_2); +lean_ctor_set(x_20, 1, x_18); +x_21 = l_Std_RBNode_insert___at_Lean_Elab_Term_registerSyntheticMVar___spec__1(x_17, x_2, x_19); +lean_ctor_set(x_14, 2, x_20); +lean_ctor_set(x_14, 1, x_21); +x_22 = lean_st_ref_set(x_5, x_14, x_15); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_18, 0); -lean_dec(x_20); -x_21 = lean_box(0); -lean_ctor_set(x_18, 0, x_21); -return x_18; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_22, 0); +lean_dec(x_24); +x_25 = lean_box(0); +lean_ctor_set(x_22, 0, x_25); +return x_22; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_18, 1); -lean_inc(x_22); -lean_dec(x_18); -x_23 = lean_box(0); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_22); -return x_24; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_22, 1); +lean_inc(x_26); +lean_dec(x_22); +x_27 = lean_box(0); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +return x_28; } } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_25 = lean_ctor_get(x_12, 0); -x_26 = lean_ctor_get(x_12, 1); -x_27 = lean_ctor_get(x_12, 2); -x_28 = lean_ctor_get(x_12, 3); -x_29 = lean_ctor_get(x_12, 4); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_12); -x_30 = lean_ctor_get(x_1, 0); -lean_inc(x_30); -x_31 = l_Std_RBNode_insert___at_Lean_Elab_Term_registerMVarErrorInfo___spec__1(x_27, x_30, x_1); -x_32 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_32, 0, x_25); -lean_ctor_set(x_32, 1, x_26); -lean_ctor_set(x_32, 2, x_31); -lean_ctor_set(x_32, 3, x_28); -lean_ctor_set(x_32, 4, x_29); -x_33 = lean_st_ref_set(x_3, x_32, x_13); -x_34 = lean_ctor_get(x_33, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_29 = lean_ctor_get(x_14, 0); +x_30 = lean_ctor_get(x_14, 1); +x_31 = lean_ctor_get(x_14, 2); +x_32 = lean_ctor_get(x_14, 3); +x_33 = lean_ctor_get(x_14, 4); +x_34 = lean_ctor_get(x_14, 5); lean_inc(x_34); -if (lean_is_exclusive(x_33)) { - lean_ctor_release(x_33, 0); - lean_ctor_release(x_33, 1); - x_35 = x_33; +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_14); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_1); +lean_ctor_set(x_35, 1, x_3); +lean_inc(x_2); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_2); +lean_ctor_set(x_36, 1, x_31); +x_37 = l_Std_RBNode_insert___at_Lean_Elab_Term_registerSyntheticMVar___spec__1(x_30, x_2, x_35); +x_38 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_38, 0, x_29); +lean_ctor_set(x_38, 1, x_37); +lean_ctor_set(x_38, 2, x_36); +lean_ctor_set(x_38, 3, x_32); +lean_ctor_set(x_38, 4, x_33); +lean_ctor_set(x_38, 5, x_34); +x_39 = lean_st_ref_set(x_5, x_38, x_15); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +if (lean_is_exclusive(x_39)) { + lean_ctor_release(x_39, 0); + lean_ctor_release(x_39, 1); + x_41 = x_39; } else { - lean_dec_ref(x_33); - x_35 = lean_box(0); + lean_dec_ref(x_39); + x_41 = lean_box(0); } -x_36 = lean_box(0); -if (lean_is_scalar(x_35)) { - x_37 = lean_alloc_ctor(0, 2, 0); +x_42 = lean_box(0); +if (lean_is_scalar(x_41)) { + x_43 = lean_alloc_ctor(0, 2, 0); } else { - x_37 = x_35; + x_43 = x_41; } -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_34); -return x_37; +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_40); +return x_43; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorInfo___boxed(lean_object* x_1, lean_object* x_2, lean_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_Term_registerSyntheticMVar___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_Term_registerMVarErrorInfo(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_object* x_11; +x_11 = l_Lean_Elab_Term_registerSyntheticMVar(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_9; +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorHoleInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_box(0); -x_11 = lean_box(1); -x_12 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_12, 0, x_1); -lean_ctor_set(x_12, 1, x_2); -lean_ctor_set(x_12, 2, x_11); -lean_ctor_set(x_12, 3, x_10); -x_13 = l_Lean_Elab_Term_registerMVarErrorInfo(x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_13; +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_7, 5); +lean_inc(x_10); +x_11 = l_Lean_Elab_Term_registerSyntheticMVar(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_7); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorHoleInfo___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Elab_Term_registerMVarErrorHoleInfo(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Elab_Term_registerSyntheticMVarWithCurrRef(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -17104,3773 +17099,7611 @@ lean_dec(x_3); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorImplicitArgInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_11, 0, x_3); -x_12 = lean_box(0); -x_13 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_13, 0, x_1); -lean_ctor_set(x_13, 1, x_2); -lean_ctor_set(x_13, 2, x_11); -lean_ctor_set(x_13, 3, x_12); -x_14 = l_Lean_Elab_Term_registerMVarErrorInfo(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorImplicitArgInfo___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +if (lean_obj_tag(x_1) == 0) { -lean_object* x_11; -x_11 = l_Lean_Elab_Term_registerMVarErrorImplicitArgInfo(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_11; -} +lean_object* x_4; uint8_t x_5; lean_object* x_6; +x_4 = lean_box(0); +x_5 = 0; +x_6 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_6, 0, x_4); +lean_ctor_set(x_6, 1, x_2); +lean_ctor_set(x_6, 2, x_3); +lean_ctor_set(x_6, 3, x_4); +lean_ctor_set_uint8(x_6, sizeof(void*)*4, x_5); +return x_6; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorCustomInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_11, 0, x_3); -x_12 = lean_box(0); -x_13 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_13, 0, x_1); -lean_ctor_set(x_13, 1, x_2); -lean_ctor_set(x_13, 2, x_11); -lean_ctor_set(x_13, 3, x_12); -x_14 = l_Lean_Elab_Term_registerMVarErrorInfo(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_14; +uint8_t x_7; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +if (x_7 == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_9 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 1); +x_11 = lean_ctor_get(x_1, 2); +x_12 = lean_ctor_get(x_1, 3); +x_13 = l_Lean_Name_quickCmp(x_2, x_10); +switch (x_13) { +case 0: +{ +lean_object* x_14; uint8_t x_15; +x_14 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_9, x_2, x_3); +x_15 = 0; +lean_ctor_set(x_1, 0, x_14); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_15); +return x_1; } +case 1: +{ +uint8_t x_16; +lean_dec(x_11); +lean_dec(x_10); +x_16 = 0; +lean_ctor_set(x_1, 2, x_3); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_16); +return x_1; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorCustomInfo___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +default: { -lean_object* x_11; -x_11 = l_Lean_Elab_Term_registerMVarErrorCustomInfo(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_11; +lean_object* x_17; uint8_t x_18; +x_17 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_12, x_2, x_3); +x_18 = 0; +lean_ctor_set(x_1, 3, x_17); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_18); +return x_1; } } -LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); -return x_3; } else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_4 = lean_ctor_get(x_1, 0); -x_5 = lean_ctor_get(x_1, 1); -x_6 = lean_ctor_get(x_1, 2); -x_7 = lean_ctor_get(x_1, 3); -x_8 = l_Lean_Name_quickCmp(x_2, x_5); -switch (x_8) { +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_19 = lean_ctor_get(x_1, 0); +x_20 = lean_ctor_get(x_1, 1); +x_21 = lean_ctor_get(x_1, 2); +x_22 = lean_ctor_get(x_1, 3); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_1); +x_23 = l_Lean_Name_quickCmp(x_2, x_20); +switch (x_23) { case 0: { -x_1 = x_4; -goto _start; +lean_object* x_24; uint8_t x_25; lean_object* x_26; +x_24 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_19, x_2, x_3); +x_25 = 0; +x_26 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_20); +lean_ctor_set(x_26, 2, x_21); +lean_ctor_set(x_26, 3, x_22); +lean_ctor_set_uint8(x_26, sizeof(void*)*4, x_25); +return x_26; } case 1: { -lean_object* x_10; -lean_inc(x_6); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_6); -return x_10; +uint8_t x_27; lean_object* x_28; +lean_dec(x_21); +lean_dec(x_20); +x_27 = 0; +x_28 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_28, 0, x_19); +lean_ctor_set(x_28, 1, x_2); +lean_ctor_set(x_28, 2, x_3); +lean_ctor_set(x_28, 3, x_22); +lean_ctor_set_uint8(x_28, sizeof(void*)*4, x_27); +return x_28; } default: { -x_1 = x_7; -goto _start; -} +lean_object* x_29; uint8_t x_30; lean_object* x_31; +x_29 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_22, x_2, x_3); +x_30 = 0; +x_31 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_31, 0, x_19); +lean_ctor_set(x_31, 1, x_20); +lean_ctor_set(x_31, 2, x_21); +lean_ctor_set(x_31, 3, x_29); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +return x_31; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_getMVarErrorInfo_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_9 = lean_st_ref_get(x_7, x_8); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_st_ref_get(x_3, x_10); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_32; +x_32 = !lean_is_exclusive(x_1); +if (x_32 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 2); -lean_inc(x_14); -lean_dec(x_13); -x_15 = l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1(x_14, x_1); -lean_dec(x_14); -lean_ctor_set(x_11, 0, x_15); -return x_11; -} -else +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_33 = lean_ctor_get(x_1, 0); +x_34 = lean_ctor_get(x_1, 1); +x_35 = lean_ctor_get(x_1, 2); +x_36 = lean_ctor_get(x_1, 3); +x_37 = l_Lean_Name_quickCmp(x_2, x_34); +switch (x_37) { +case 0: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_16 = lean_ctor_get(x_11, 0); -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_11); -x_18 = lean_ctor_get(x_16, 2); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1(x_18, x_1); -lean_dec(x_18); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_17); -return x_20; -} -} -} -LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: +uint8_t x_38; +x_38 = l_Std_RBNode_isRed___rarg(x_33); +if (x_38 == 0) { -lean_object* x_3; -x_3 = l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; -} +lean_object* x_39; uint8_t x_40; +x_39 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_33, x_2, x_3); +x_40 = 1; +lean_ctor_set(x_1, 0, x_39); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_40); +return x_1; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_getMVarErrorInfo_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Lean_Elab_Term_getMVarErrorInfo_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerCustomErrorIfMVar(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_41; lean_object* x_42; +x_41 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_33, x_2, x_3); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_11; -x_11 = l_Lean_Expr_getAppFn(x_1); -if (lean_obj_tag(x_11) == 2) +lean_object* x_43; +x_43 = lean_ctor_get(x_41, 3); +lean_inc(x_43); +if (lean_obj_tag(x_43) == 0) { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -lean_dec(x_11); -x_13 = l_Lean_Elab_Term_registerMVarErrorCustomInfo(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_13; +uint8_t x_44; +x_44 = !lean_is_exclusive(x_41); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; +x_45 = lean_ctor_get(x_41, 3); +lean_dec(x_45); +x_46 = lean_ctor_get(x_41, 0); +lean_dec(x_46); +x_47 = 0; +lean_ctor_set(x_41, 0, x_43); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_47); +x_48 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_48); +return x_1; } else { -lean_object* x_14; lean_object* x_15; -lean_dec(x_11); -lean_dec(x_3); -lean_dec(x_2); -x_14 = lean_box(0); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_10); -return x_15; -} +lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; uint8_t x_53; +x_49 = lean_ctor_get(x_41, 1); +x_50 = lean_ctor_get(x_41, 2); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_41); +x_51 = 0; +x_52 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_52, 0, x_43); +lean_ctor_set(x_52, 1, x_49); +lean_ctor_set(x_52, 2, x_50); +lean_ctor_set(x_52, 3, x_43); +lean_ctor_set_uint8(x_52, sizeof(void*)*4, x_51); +x_53 = 1; +lean_ctor_set(x_1, 0, x_52); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_53); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerCustomErrorIfMVar___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l_Lean_Elab_Term_registerCustomErrorIfMVar(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +uint8_t x_54; +x_54 = lean_ctor_get_uint8(x_43, sizeof(void*)*4); +if (x_54 == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_9 = lean_ctor_get(x_6, 5); -x_10 = lean_ctor_get(x_2, 2); -lean_inc(x_10); -lean_inc(x_10); -x_11 = l_Lean_Elab_getBetterRef(x_9, x_10); -x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_4, x_5, x_6, x_7, x_8); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_13, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_14); -lean_dec(x_2); -lean_dec(x_10); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_11); -lean_ctor_set(x_18, 1, x_17); -lean_ctor_set_tag(x_15, 1); -lean_ctor_set(x_15, 0, x_18); -return x_15; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_15, 0); -x_20 = lean_ctor_get(x_15, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_15); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_11); -lean_ctor_set(x_21, 1, x_19); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; -} -} -} -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1(lean_object* x_1) { -_start: +uint8_t x_55; +x_55 = !lean_is_exclusive(x_41); +if (x_55 == 0) { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg___boxed), 8, 0); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__1() { -_start: +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; +x_56 = lean_ctor_get(x_41, 1); +x_57 = lean_ctor_get(x_41, 2); +x_58 = lean_ctor_get(x_41, 3); +lean_dec(x_58); +x_59 = lean_ctor_get(x_41, 0); +lean_dec(x_59); +x_60 = !lean_is_exclusive(x_43); +if (x_60 == 0) { -lean_object* x_1; -x_1 = l_Lean_Elab_abortTermExceptionId; +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; uint8_t x_66; +x_61 = lean_ctor_get(x_43, 0); +x_62 = lean_ctor_get(x_43, 1); +x_63 = lean_ctor_get(x_43, 2); +x_64 = lean_ctor_get(x_43, 3); +x_65 = 1; +lean_ctor_set(x_43, 3, x_61); +lean_ctor_set(x_43, 2, x_57); +lean_ctor_set(x_43, 1, x_56); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set_uint8(x_43, sizeof(void*)*4, x_65); +lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 2, x_35); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 0, x_64); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_65); +x_66 = 0; +lean_ctor_set(x_1, 3, x_41); +lean_ctor_set(x_1, 2, x_63); +lean_ctor_set(x_1, 1, x_62); +lean_ctor_set(x_1, 0, x_43); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_66); return x_1; } -} -static lean_object* _init_l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__1; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; lean_object* x_72; uint8_t x_73; +x_67 = lean_ctor_get(x_43, 0); +x_68 = lean_ctor_get(x_43, 1); +x_69 = lean_ctor_get(x_43, 2); +x_70 = lean_ctor_get(x_43, 3); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_43); +x_71 = 1; +x_72 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_72, 0, x_42); +lean_ctor_set(x_72, 1, x_56); +lean_ctor_set(x_72, 2, x_57); +lean_ctor_set(x_72, 3, x_67); +lean_ctor_set_uint8(x_72, sizeof(void*)*4, x_71); +lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 2, x_35); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 0, x_70); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_71); +x_73 = 0; +lean_ctor_set(x_1, 3, x_41); +lean_ctor_set(x_1, 2, x_69); +lean_ctor_set(x_1, 1, x_68); +lean_ctor_set(x_1, 0, x_72); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_73); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg(lean_object* x_1) { -_start: +else { -lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__2; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_74 = lean_ctor_get(x_41, 1); +x_75 = lean_ctor_get(x_41, 2); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_41); +x_76 = lean_ctor_get(x_43, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_43, 1); +lean_inc(x_77); +x_78 = lean_ctor_get(x_43, 2); +lean_inc(x_78); +x_79 = lean_ctor_get(x_43, 3); +lean_inc(x_79); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + lean_ctor_release(x_43, 2); + lean_ctor_release(x_43, 3); + x_80 = x_43; +} else { + lean_dec_ref(x_43); + x_80 = lean_box(0); } +x_81 = 1; +if (lean_is_scalar(x_80)) { + x_82 = lean_alloc_ctor(1, 4, 1); +} else { + x_82 = x_80; } -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = lean_alloc_closure((void*)(l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg), 1, 0); -return x_8; +lean_ctor_set(x_82, 0, x_42); +lean_ctor_set(x_82, 1, x_74); +lean_ctor_set(x_82, 2, x_75); +lean_ctor_set(x_82, 3, x_76); +lean_ctor_set_uint8(x_82, sizeof(void*)*4, x_81); +x_83 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_83, 0, x_79); +lean_ctor_set(x_83, 1, x_34); +lean_ctor_set(x_83, 2, x_35); +lean_ctor_set(x_83, 3, x_36); +lean_ctor_set_uint8(x_83, sizeof(void*)*4, x_81); +x_84 = 0; +lean_ctor_set(x_1, 3, x_83); +lean_ctor_set(x_1, 2, x_78); +lean_ctor_set(x_1, 1, x_77); +lean_ctor_set(x_1, 0, x_82); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_84); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_9 = lean_st_ref_get(x_7, x_8); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_ctor_get(x_10, 5); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Std_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(x_12); -if (x_13 == 0) +uint8_t x_85; +x_85 = !lean_is_exclusive(x_41); +if (x_85 == 0) { -lean_object* x_14; -x_14 = l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11); -return x_14; +lean_object* x_86; lean_object* x_87; uint8_t x_88; uint8_t x_89; +x_86 = lean_ctor_get(x_41, 3); +lean_dec(x_86); +x_87 = lean_ctor_get(x_41, 0); +lean_dec(x_87); +x_88 = 0; +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_88); +x_89 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_89); +return x_1; } else { -lean_object* x_15; -lean_dec(x_2); -lean_dec(x_1); -x_15 = l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg(x_11); -return x_15; -} +lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; uint8_t x_94; +x_90 = lean_ctor_get(x_41, 1); +x_91 = lean_ctor_get(x_41, 2); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_41); +x_92 = 0; +x_93 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_93, 0, x_42); +lean_ctor_set(x_93, 1, x_90); +lean_ctor_set(x_93, 2, x_91); +lean_ctor_set(x_93, 3, x_43); +lean_ctor_set_uint8(x_93, sizeof(void*)*4, x_92); +x_94 = 1; +lean_ctor_set(x_1, 0, x_93); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_94); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_throwMVarError___rarg___boxed), 8, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +uint8_t x_95; +x_95 = lean_ctor_get_uint8(x_42, sizeof(void*)*4); +if (x_95 == 0) { -lean_object* x_8; -x_8 = l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +uint8_t x_96; +x_96 = !lean_is_exclusive(x_41); +if (x_96 == 0) { -lean_object* x_9; -x_9 = l_Lean_Elab_Term_throwMVarError___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_9; -} +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; uint8_t x_101; +x_97 = lean_ctor_get(x_41, 1); +x_98 = lean_ctor_get(x_41, 2); +x_99 = lean_ctor_get(x_41, 3); +x_100 = lean_ctor_get(x_41, 0); +lean_dec(x_100); +x_101 = !lean_is_exclusive(x_42); +if (x_101 == 0) +{ +uint8_t x_102; uint8_t x_103; +x_102 = 1; +lean_ctor_set_uint8(x_42, sizeof(void*)*4, x_102); +lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 2, x_35); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 0, x_99); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_102); +x_103 = 0; +lean_ctor_set(x_1, 3, x_41); +lean_ctor_set(x_1, 2, x_98); +lean_ctor_set(x_1, 1, x_97); +lean_ctor_set(x_1, 0, x_42); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_103); +return x_1; } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" '", 2); +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; lean_object* x_109; uint8_t x_110; +x_104 = lean_ctor_get(x_42, 0); +x_105 = lean_ctor_get(x_42, 1); +x_106 = lean_ctor_get(x_42, 2); +x_107 = lean_ctor_get(x_42, 3); +lean_inc(x_107); +lean_inc(x_106); +lean_inc(x_105); +lean_inc(x_104); +lean_dec(x_42); +x_108 = 1; +x_109 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_109, 0, x_104); +lean_ctor_set(x_109, 1, x_105); +lean_ctor_set(x_109, 2, x_106); +lean_ctor_set(x_109, 3, x_107); +lean_ctor_set_uint8(x_109, sizeof(void*)*4, x_108); +lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 2, x_35); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 0, x_99); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_108); +x_110 = 0; +lean_ctor_set(x_1, 3, x_41); +lean_ctor_set(x_1, 2, x_98); +lean_ctor_set(x_1, 1, x_97); +lean_ctor_set(x_1, 0, x_109); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_110); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; +x_111 = lean_ctor_get(x_41, 1); +x_112 = lean_ctor_get(x_41, 2); +x_113 = lean_ctor_get(x_41, 3); +lean_inc(x_113); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_41); +x_114 = lean_ctor_get(x_42, 0); +lean_inc(x_114); +x_115 = lean_ctor_get(x_42, 1); +lean_inc(x_115); +x_116 = lean_ctor_get(x_42, 2); +lean_inc(x_116); +x_117 = lean_ctor_get(x_42, 3); +lean_inc(x_117); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + lean_ctor_release(x_42, 2); + lean_ctor_release(x_42, 3); + x_118 = x_42; +} else { + lean_dec_ref(x_42); + x_118 = lean_box(0); } +x_119 = 1; +if (lean_is_scalar(x_118)) { + x_120 = lean_alloc_ctor(1, 4, 1); +} else { + x_120 = x_118; } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("'", 1); +lean_ctor_set(x_120, 0, x_114); +lean_ctor_set(x_120, 1, x_115); +lean_ctor_set(x_120, 2, x_116); +lean_ctor_set(x_120, 3, x_117); +lean_ctor_set_uint8(x_120, sizeof(void*)*4, x_119); +x_121 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_121, 0, x_113); +lean_ctor_set(x_121, 1, x_34); +lean_ctor_set(x_121, 2, x_35); +lean_ctor_set(x_121, 3, x_36); +lean_ctor_set_uint8(x_121, sizeof(void*)*4, x_119); +x_122 = 0; +lean_ctor_set(x_1, 3, x_121); +lean_ctor_set(x_1, 2, x_112); +lean_ctor_set(x_1, 1, x_111); +lean_ctor_set(x_1, 0, x_120); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_122); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +lean_object* x_123; +x_123 = lean_ctor_get(x_41, 3); +lean_inc(x_123); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_4; -x_4 = lean_ctor_get(x_1, 3); -if (lean_obj_tag(x_4) == 0) +uint8_t x_124; +x_124 = !lean_is_exclusive(x_41); +if (x_124 == 0) { -lean_dec(x_3); -return x_2; +lean_object* x_125; lean_object* x_126; uint8_t x_127; uint8_t x_128; +x_125 = lean_ctor_get(x_41, 3); +lean_dec(x_125); +x_126 = lean_ctor_get(x_41, 0); +lean_dec(x_126); +x_127 = 0; +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_127); +x_128 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_128); +return x_1; } else { -lean_object* x_5; uint8_t x_6; -x_5 = lean_ctor_get(x_4, 0); -x_6 = l_Lean_Name_hasMacroScopes(x_5); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_7 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_7, 0, x_3); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -x_9 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_9, 0, x_2); -lean_ctor_set(x_9, 1, x_8); -lean_inc(x_5); -x_10 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_10, 0, x_5); -x_11 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__2; -x_12 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -x_13 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__4; -x_14 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_14, 0, x_12); -lean_ctor_set(x_14, 1, x_13); -x_15 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_15, 0, x_9); -lean_ctor_set(x_15, 1, x_14); -return x_15; +lean_object* x_129; lean_object* x_130; uint8_t x_131; lean_object* x_132; uint8_t x_133; +x_129 = lean_ctor_get(x_41, 1); +x_130 = lean_ctor_get(x_41, 2); +lean_inc(x_130); +lean_inc(x_129); +lean_dec(x_41); +x_131 = 0; +x_132 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_132, 0, x_42); +lean_ctor_set(x_132, 1, x_129); +lean_ctor_set(x_132, 2, x_130); +lean_ctor_set(x_132, 3, x_123); +lean_ctor_set_uint8(x_132, sizeof(void*)*4, x_131); +x_133 = 1; +lean_ctor_set(x_1, 0, x_132); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_133); +return x_1; +} } else { -lean_dec(x_3); -return x_2; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +uint8_t x_134; +x_134 = lean_ctor_get_uint8(x_123, sizeof(void*)*4); +if (x_134 == 0) { -lean_object* x_4; -x_4 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(lean_object* x_1, lean_object* x_2) { -_start: +uint8_t x_135; +lean_free_object(x_1); +x_135 = !lean_is_exclusive(x_41); +if (x_135 == 0) { -if (lean_obj_tag(x_1) == 0) +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; uint8_t x_140; +x_136 = lean_ctor_get(x_41, 1); +x_137 = lean_ctor_get(x_41, 2); +x_138 = lean_ctor_get(x_41, 3); +lean_dec(x_138); +x_139 = lean_ctor_get(x_41, 0); +lean_dec(x_139); +x_140 = !lean_is_exclusive(x_123); +if (x_140 == 0) { -return x_2; -} -else +lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; uint8_t x_145; uint8_t x_146; +x_141 = lean_ctor_get(x_123, 0); +x_142 = lean_ctor_get(x_123, 1); +x_143 = lean_ctor_get(x_123, 2); +x_144 = lean_ctor_get(x_123, 3); +x_145 = 1; +lean_inc(x_42); +lean_ctor_set(x_123, 3, x_141); +lean_ctor_set(x_123, 2, x_137); +lean_ctor_set(x_123, 1, x_136); +lean_ctor_set(x_123, 0, x_42); +x_146 = !lean_is_exclusive(x_42); +if (x_146 == 0) { -lean_object* x_3; lean_object* x_4; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -x_4 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_3); -return x_4; -} -} +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; uint8_t x_151; +x_147 = lean_ctor_get(x_42, 3); +lean_dec(x_147); +x_148 = lean_ctor_get(x_42, 2); +lean_dec(x_148); +x_149 = lean_ctor_get(x_42, 1); +lean_dec(x_149); +x_150 = lean_ctor_get(x_42, 0); +lean_dec(x_150); +lean_ctor_set_uint8(x_123, sizeof(void*)*4, x_145); +lean_ctor_set(x_42, 3, x_36); +lean_ctor_set(x_42, 2, x_35); +lean_ctor_set(x_42, 1, x_34); +lean_ctor_set(x_42, 0, x_144); +lean_ctor_set_uint8(x_42, sizeof(void*)*4, x_145); +x_151 = 0; +lean_ctor_set(x_41, 3, x_42); +lean_ctor_set(x_41, 2, x_143); +lean_ctor_set(x_41, 1, x_142); +lean_ctor_set(x_41, 0, x_123); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_151); +return x_41; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; -x_3 = l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(x_1, x_2); -lean_dec(x_1); -return x_3; -} +lean_object* x_152; uint8_t x_153; +lean_dec(x_42); +lean_ctor_set_uint8(x_123, sizeof(void*)*4, x_145); +x_152 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_152, 0, x_144); +lean_ctor_set(x_152, 1, x_34); +lean_ctor_set(x_152, 2, x_35); +lean_ctor_set(x_152, 3, x_36); +lean_ctor_set_uint8(x_152, sizeof(void*)*4, x_145); +x_153 = 0; +lean_ctor_set(x_41, 3, x_152); +lean_ctor_set(x_41, 2, x_143); +lean_ctor_set(x_41, 1, x_142); +lean_ctor_set(x_41, 0, x_123); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_153); +return x_41; } -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -uint8_t x_9; -x_9 = l_Lean_Expr_hasMVar(x_1); -if (x_9 == 0) -{ -lean_object* x_10; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_1); -lean_ctor_set(x_10, 1, x_8); -return x_10; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_11 = lean_st_ref_get(x_7, x_8); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_st_ref_get(x_5, x_12); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_instantiateMVarsCore(x_16, x_1); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_st_ref_get(x_7, x_15); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -x_22 = lean_st_ref_take(x_5, x_21); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = !lean_is_exclusive(x_23); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = lean_ctor_get(x_23, 0); -lean_dec(x_26); -lean_ctor_set(x_23, 0, x_19); -x_27 = lean_st_ref_set(x_5, x_23, x_24); -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) -{ -lean_object* x_29; -x_29 = lean_ctor_get(x_27, 0); -lean_dec(x_29); -lean_ctor_set(x_27, 0, x_18); -return x_27; +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; uint8_t x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; uint8_t x_162; +x_154 = lean_ctor_get(x_123, 0); +x_155 = lean_ctor_get(x_123, 1); +x_156 = lean_ctor_get(x_123, 2); +x_157 = lean_ctor_get(x_123, 3); +lean_inc(x_157); +lean_inc(x_156); +lean_inc(x_155); +lean_inc(x_154); +lean_dec(x_123); +x_158 = 1; +lean_inc(x_42); +x_159 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_159, 0, x_42); +lean_ctor_set(x_159, 1, x_136); +lean_ctor_set(x_159, 2, x_137); +lean_ctor_set(x_159, 3, x_154); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + lean_ctor_release(x_42, 2); + lean_ctor_release(x_42, 3); + x_160 = x_42; +} else { + lean_dec_ref(x_42); + x_160 = lean_box(0); } -else -{ -lean_object* x_30; lean_object* x_31; -x_30 = lean_ctor_get(x_27, 1); -lean_inc(x_30); -lean_dec(x_27); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_18); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_ctor_set_uint8(x_159, sizeof(void*)*4, x_158); +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(1, 4, 1); +} else { + x_161 = x_160; +} +lean_ctor_set(x_161, 0, x_157); +lean_ctor_set(x_161, 1, x_34); +lean_ctor_set(x_161, 2, x_35); +lean_ctor_set(x_161, 3, x_36); +lean_ctor_set_uint8(x_161, sizeof(void*)*4, x_158); +x_162 = 0; +lean_ctor_set(x_41, 3, x_161); +lean_ctor_set(x_41, 2, x_156); +lean_ctor_set(x_41, 1, x_155); +lean_ctor_set(x_41, 0, x_159); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_162); +return x_41; } } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_23, 1); -x_33 = lean_ctor_get(x_23, 2); -x_34 = lean_ctor_get(x_23, 3); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_23); -x_35 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_35, 0, x_19); -lean_ctor_set(x_35, 1, x_32); -lean_ctor_set(x_35, 2, x_33); -lean_ctor_set(x_35, 3, x_34); -x_36 = lean_st_ref_set(x_5, x_35, x_24); -x_37 = lean_ctor_get(x_36, 1); -lean_inc(x_37); -if (lean_is_exclusive(x_36)) { - lean_ctor_release(x_36, 0); - lean_ctor_release(x_36, 1); - x_38 = x_36; +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; uint8_t x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; lean_object* x_175; +x_163 = lean_ctor_get(x_41, 1); +x_164 = lean_ctor_get(x_41, 2); +lean_inc(x_164); +lean_inc(x_163); +lean_dec(x_41); +x_165 = lean_ctor_get(x_123, 0); +lean_inc(x_165); +x_166 = lean_ctor_get(x_123, 1); +lean_inc(x_166); +x_167 = lean_ctor_get(x_123, 2); +lean_inc(x_167); +x_168 = lean_ctor_get(x_123, 3); +lean_inc(x_168); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + lean_ctor_release(x_123, 2); + lean_ctor_release(x_123, 3); + x_169 = x_123; } else { - lean_dec_ref(x_36); - x_38 = lean_box(0); + lean_dec_ref(x_123); + x_169 = lean_box(0); } -if (lean_is_scalar(x_38)) { - x_39 = lean_alloc_ctor(0, 2, 0); +x_170 = 1; +lean_inc(x_42); +if (lean_is_scalar(x_169)) { + x_171 = lean_alloc_ctor(1, 4, 1); } else { - x_39 = x_38; + x_171 = x_169; } -lean_ctor_set(x_39, 0, x_18); -lean_ctor_set(x_39, 1, x_37); -return x_39; +lean_ctor_set(x_171, 0, x_42); +lean_ctor_set(x_171, 1, x_163); +lean_ctor_set(x_171, 2, x_164); +lean_ctor_set(x_171, 3, x_165); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + lean_ctor_release(x_42, 2); + lean_ctor_release(x_42, 3); + x_172 = x_42; +} else { + lean_dec_ref(x_42); + x_172 = lean_box(0); } +lean_ctor_set_uint8(x_171, sizeof(void*)*4, x_170); +if (lean_is_scalar(x_172)) { + x_173 = lean_alloc_ctor(1, 4, 1); +} else { + x_173 = x_172; } +lean_ctor_set(x_173, 0, x_168); +lean_ctor_set(x_173, 1, x_34); +lean_ctor_set(x_173, 2, x_35); +lean_ctor_set(x_173, 3, x_36); +lean_ctor_set_uint8(x_173, sizeof(void*)*4, x_170); +x_174 = 0; +x_175 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_175, 0, x_171); +lean_ctor_set(x_175, 1, x_166); +lean_ctor_set(x_175, 2, x_167); +lean_ctor_set(x_175, 3, x_173); +lean_ctor_set_uint8(x_175, sizeof(void*)*4, x_174); +return x_175; } } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("don't know how to synthesize implicit argument", 46); +uint8_t x_176; +x_176 = !lean_is_exclusive(x_41); +if (x_176 == 0) +{ +lean_object* x_177; lean_object* x_178; uint8_t x_179; +x_177 = lean_ctor_get(x_41, 3); +lean_dec(x_177); +x_178 = lean_ctor_get(x_41, 0); +lean_dec(x_178); +x_179 = !lean_is_exclusive(x_42); +if (x_179 == 0) +{ +uint8_t x_180; uint8_t x_181; +lean_ctor_set_uint8(x_42, sizeof(void*)*4, x_134); +x_180 = 0; +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_180); +x_181 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_181); return x_1; } -} -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__1; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; uint8_t x_187; uint8_t x_188; +x_182 = lean_ctor_get(x_42, 0); +x_183 = lean_ctor_get(x_42, 1); +x_184 = lean_ctor_get(x_42, 2); +x_185 = lean_ctor_get(x_42, 3); +lean_inc(x_185); +lean_inc(x_184); +lean_inc(x_183); +lean_inc(x_182); +lean_dec(x_42); +x_186 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_186, 0, x_182); +lean_ctor_set(x_186, 1, x_183); +lean_ctor_set(x_186, 2, x_184); +lean_ctor_set(x_186, 3, x_185); +lean_ctor_set_uint8(x_186, sizeof(void*)*4, x_134); +x_187 = 0; +lean_ctor_set(x_41, 0, x_186); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_187); +x_188 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_188); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__3() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__2; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; uint8_t x_197; lean_object* x_198; uint8_t x_199; +x_189 = lean_ctor_get(x_41, 1); +x_190 = lean_ctor_get(x_41, 2); +lean_inc(x_190); +lean_inc(x_189); +lean_dec(x_41); +x_191 = lean_ctor_get(x_42, 0); +lean_inc(x_191); +x_192 = lean_ctor_get(x_42, 1); +lean_inc(x_192); +x_193 = lean_ctor_get(x_42, 2); +lean_inc(x_193); +x_194 = lean_ctor_get(x_42, 3); +lean_inc(x_194); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + lean_ctor_release(x_42, 2); + lean_ctor_release(x_42, 3); + x_195 = x_42; +} else { + lean_dec_ref(x_42); + x_195 = lean_box(0); } +if (lean_is_scalar(x_195)) { + x_196 = lean_alloc_ctor(1, 4, 1); +} else { + x_196 = x_195; } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("context:", 8); +lean_ctor_set(x_196, 0, x_191); +lean_ctor_set(x_196, 1, x_192); +lean_ctor_set(x_196, 2, x_193); +lean_ctor_set(x_196, 3, x_194); +lean_ctor_set_uint8(x_196, sizeof(void*)*4, x_134); +x_197 = 0; +x_198 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_198, 0, x_196); +lean_ctor_set(x_198, 1, x_189); +lean_ctor_set(x_198, 2, x_190); +lean_ctor_set(x_198, 3, x_123); +lean_ctor_set_uint8(x_198, sizeof(void*)*4, x_197); +x_199 = 1; +lean_ctor_set(x_1, 0, x_198); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_199); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__4; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__5; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("don't know how to synthesize placeholder", 40); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__8() { -_start: +case 1: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__7; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} +uint8_t x_200; +lean_dec(x_35); +lean_dec(x_34); +x_200 = 1; +lean_ctor_set(x_1, 2, x_3); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_200); +return x_1; } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__9() { -_start: +default: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__8; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__10() { -_start: +uint8_t x_201; +x_201 = l_Std_RBNode_isRed___rarg(x_36); +if (x_201 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" for argument", 13); +lean_object* x_202; uint8_t x_203; +x_202 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_36, x_2, x_3); +x_203 = 1; +lean_ctor_set(x_1, 3, x_202); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_203); return x_1; } -} -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__11() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__3; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +lean_object* x_204; lean_object* x_205; +x_204 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_36, x_2, x_3); +x_205 = lean_ctor_get(x_204, 0); +lean_inc(x_205); +if (lean_obj_tag(x_205) == 0) +{ +lean_object* x_206; +x_206 = lean_ctor_get(x_204, 3); +lean_inc(x_206); +if (lean_obj_tag(x_206) == 0) +{ +uint8_t x_207; +x_207 = !lean_is_exclusive(x_204); +if (x_207 == 0) +{ +lean_object* x_208; lean_object* x_209; uint8_t x_210; uint8_t x_211; +x_208 = lean_ctor_get(x_204, 3); +lean_dec(x_208); +x_209 = lean_ctor_get(x_204, 0); +lean_dec(x_209); +x_210 = 0; +lean_ctor_set(x_204, 0, x_206); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_210); +x_211 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_211); +return x_1; } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__12() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("synthPlaceholder", 16); +lean_object* x_212; lean_object* x_213; uint8_t x_214; lean_object* x_215; uint8_t x_216; +x_212 = lean_ctor_get(x_204, 1); +x_213 = lean_ctor_get(x_204, 2); +lean_inc(x_213); +lean_inc(x_212); +lean_dec(x_204); +x_214 = 0; +x_215 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_215, 0, x_206); +lean_ctor_set(x_215, 1, x_212); +lean_ctor_set(x_215, 2, x_213); +lean_ctor_set(x_215, 3, x_206); +lean_ctor_set_uint8(x_215, sizeof(void*)*4, x_214); +x_216 = 1; +lean_ctor_set(x_1, 3, x_215); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_216); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__13() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__11; -x_2 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__12; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +uint8_t x_217; +x_217 = lean_ctor_get_uint8(x_206, sizeof(void*)*4); +if (x_217 == 0) { -lean_object* x_10; -x_10 = lean_ctor_get(x_1, 2); -lean_inc(x_10); -switch (lean_obj_tag(x_10)) { -case 0: +uint8_t x_218; +x_218 = !lean_is_exclusive(x_204); +if (x_218 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_1, 1); -lean_inc(x_12); -x_13 = lean_ctor_get(x_10, 0); -lean_inc(x_13); -lean_dec(x_10); -x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__3; -x_18 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; -x_19 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(x_1, x_17, x_18); -lean_dec(x_1); -x_20 = l_Lean_Expr_setAppPPExplicitForExposingMVars(x_15); -x_21 = l_Lean_indentExpr(x_20); -x_22 = l_Lean_logTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__1___closed__5; -x_23 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -x_24 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_22); -x_25 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_25, 0, x_19); -lean_ctor_set(x_25, 1, x_24); -x_26 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1___closed__2; -x_27 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__6; -x_29 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -x_30 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_26); -x_31 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_31, 0, x_11); -x_32 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(x_2, x_32); -x_34 = 2; -x_35 = l_Lean_logAt___at_Lean_Elab_Term_traceAtCmdPos___spec__3(x_12, x_33, x_34, x_3, x_4, x_5, x_6, x_7, x_8, x_16); -lean_dec(x_12); -return x_35; -} -case 1: +lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; uint8_t x_223; +x_219 = lean_ctor_get(x_204, 1); +x_220 = lean_ctor_get(x_204, 2); +x_221 = lean_ctor_get(x_204, 3); +lean_dec(x_221); +x_222 = lean_ctor_get(x_204, 0); +lean_dec(x_222); +x_223 = !lean_is_exclusive(x_206); +if (x_223 == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; -x_36 = lean_ctor_get(x_1, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_1, 1); -lean_inc(x_37); -x_38 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__9; -x_39 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__10; -x_40 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(x_1, x_38, x_39); -lean_dec(x_1); -x_41 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1___closed__2; -x_42 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -x_43 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__6; -x_44 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -x_45 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_41); -x_46 = lean_alloc_ctor(5, 1, 0); -lean_ctor_set(x_46, 0, x_36); -x_47 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -x_48 = l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(x_2, x_47); -x_49 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__13; -x_50 = lean_alloc_ctor(11, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_48); -x_51 = 2; -x_52 = l_Lean_logAt___at_Lean_Elab_Term_traceAtCmdPos___spec__3(x_37, x_50, x_51, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_37); -return x_52; +lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; uint8_t x_228; uint8_t x_229; +x_224 = lean_ctor_get(x_206, 0); +x_225 = lean_ctor_get(x_206, 1); +x_226 = lean_ctor_get(x_206, 2); +x_227 = lean_ctor_get(x_206, 3); +x_228 = 1; +lean_ctor_set(x_206, 3, x_205); +lean_ctor_set(x_206, 2, x_35); +lean_ctor_set(x_206, 1, x_34); +lean_ctor_set(x_206, 0, x_33); +lean_ctor_set_uint8(x_206, sizeof(void*)*4, x_228); +lean_ctor_set(x_204, 3, x_227); +lean_ctor_set(x_204, 2, x_226); +lean_ctor_set(x_204, 1, x_225); +lean_ctor_set(x_204, 0, x_224); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_228); +x_229 = 0; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set(x_1, 2, x_220); +lean_ctor_set(x_1, 1, x_219); +lean_ctor_set(x_1, 0, x_206); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_229); +return x_1; } -default: +else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; -x_53 = lean_ctor_get(x_1, 1); -lean_inc(x_53); -lean_dec(x_1); -x_54 = lean_ctor_get(x_10, 0); -lean_inc(x_54); -lean_dec(x_10); -x_55 = l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(x_2, x_54); -x_56 = 2; -x_57 = l_Lean_logAt___at_Lean_Elab_Term_traceAtCmdPos___spec__3(x_53, x_55, x_56, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_53); -return x_57; -} -} +lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; uint8_t x_234; lean_object* x_235; uint8_t x_236; +x_230 = lean_ctor_get(x_206, 0); +x_231 = lean_ctor_get(x_206, 1); +x_232 = lean_ctor_get(x_206, 2); +x_233 = lean_ctor_get(x_206, 3); +lean_inc(x_233); +lean_inc(x_232); +lean_inc(x_231); +lean_inc(x_230); +lean_dec(x_206); +x_234 = 1; +x_235 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_235, 0, x_33); +lean_ctor_set(x_235, 1, x_34); +lean_ctor_set(x_235, 2, x_35); +lean_ctor_set(x_235, 3, x_205); +lean_ctor_set_uint8(x_235, sizeof(void*)*4, x_234); +lean_ctor_set(x_204, 3, x_233); +lean_ctor_set(x_204, 2, x_232); +lean_ctor_set(x_204, 1, x_231); +lean_ctor_set(x_204, 0, x_230); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_234); +x_236 = 0; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set(x_1, 2, x_220); +lean_ctor_set(x_1, 1, x_219); +lean_ctor_set(x_1, 0, x_235); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_236); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_9; +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; uint8_t x_244; lean_object* x_245; lean_object* x_246; uint8_t x_247; +x_237 = lean_ctor_get(x_204, 1); +x_238 = lean_ctor_get(x_204, 2); +lean_inc(x_238); +lean_inc(x_237); +lean_dec(x_204); +x_239 = lean_ctor_get(x_206, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_206, 1); +lean_inc(x_240); +x_241 = lean_ctor_get(x_206, 2); +lean_inc(x_241); +x_242 = lean_ctor_get(x_206, 3); +lean_inc(x_242); +if (lean_is_exclusive(x_206)) { + lean_ctor_release(x_206, 0); + lean_ctor_release(x_206, 1); + lean_ctor_release(x_206, 2); + lean_ctor_release(x_206, 3); + x_243 = x_206; +} else { + lean_dec_ref(x_206); + x_243 = lean_box(0); } +x_244 = 1; +if (lean_is_scalar(x_243)) { + x_245 = lean_alloc_ctor(1, 4, 1); +} else { + x_245 = x_243; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_Elab_Term_MVarErrorInfo_logError(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; +lean_ctor_set(x_245, 0, x_33); +lean_ctor_set(x_245, 1, x_34); +lean_ctor_set(x_245, 2, x_35); +lean_ctor_set(x_245, 3, x_205); +lean_ctor_set_uint8(x_245, sizeof(void*)*4, x_244); +x_246 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_246, 0, x_239); +lean_ctor_set(x_246, 1, x_240); +lean_ctor_set(x_246, 2, x_241); +lean_ctor_set(x_246, 3, x_242); +lean_ctor_set_uint8(x_246, sizeof(void*)*4, x_244); +x_247 = 0; +lean_ctor_set(x_1, 3, x_246); +lean_ctor_set(x_1, 2, x_238); +lean_ctor_set(x_1, 1, x_237); +lean_ctor_set(x_1, 0, x_245); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_247); +return x_1; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) +else { -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_uget(x_2, x_3); -x_7 = lean_name_eq(x_1, x_6); -lean_dec(x_6); -if (x_7 == 0) +uint8_t x_248; +x_248 = !lean_is_exclusive(x_204); +if (x_248 == 0) { -size_t x_8; size_t x_9; -x_8 = 1; -x_9 = lean_usize_add(x_3, x_8); -x_3 = x_9; -goto _start; +lean_object* x_249; lean_object* x_250; uint8_t x_251; uint8_t x_252; +x_249 = lean_ctor_get(x_204, 3); +lean_dec(x_249); +x_250 = lean_ctor_get(x_204, 0); +lean_dec(x_250); +x_251 = 0; +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_251); +x_252 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_252); +return x_1; } else { -uint8_t x_11; -x_11 = 1; -return x_11; -} +lean_object* x_253; lean_object* x_254; uint8_t x_255; lean_object* x_256; uint8_t x_257; +x_253 = lean_ctor_get(x_204, 1); +x_254 = lean_ctor_get(x_204, 2); +lean_inc(x_254); +lean_inc(x_253); +lean_dec(x_204); +x_255 = 0; +x_256 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_256, 0, x_205); +lean_ctor_set(x_256, 1, x_253); +lean_ctor_set(x_256, 2, x_254); +lean_ctor_set(x_256, 3, x_206); +lean_ctor_set_uint8(x_256, sizeof(void*)*4, x_255); +x_257 = 1; +lean_ctor_set(x_1, 3, x_256); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_257); +return x_1; } -else -{ -uint8_t x_12; -x_12 = 0; -return x_12; } } } -LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_3 = lean_array_get_size(x_1); -x_4 = lean_unsigned_to_nat(0u); -x_5 = lean_nat_dec_lt(x_4, x_3); -if (x_5 == 0) +uint8_t x_258; +x_258 = lean_ctor_get_uint8(x_205, sizeof(void*)*4); +if (x_258 == 0) { -uint8_t x_6; -lean_dec(x_3); -x_6 = 0; -return x_6; +uint8_t x_259; +x_259 = !lean_is_exclusive(x_204); +if (x_259 == 0) +{ +lean_object* x_260; uint8_t x_261; +x_260 = lean_ctor_get(x_204, 0); +lean_dec(x_260); +x_261 = !lean_is_exclusive(x_205); +if (x_261 == 0) +{ +lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; uint8_t x_266; uint8_t x_267; +x_262 = lean_ctor_get(x_205, 0); +x_263 = lean_ctor_get(x_205, 1); +x_264 = lean_ctor_get(x_205, 2); +x_265 = lean_ctor_get(x_205, 3); +x_266 = 1; +lean_ctor_set(x_205, 3, x_262); +lean_ctor_set(x_205, 2, x_35); +lean_ctor_set(x_205, 1, x_34); +lean_ctor_set(x_205, 0, x_33); +lean_ctor_set_uint8(x_205, sizeof(void*)*4, x_266); +lean_ctor_set(x_204, 0, x_265); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_266); +x_267 = 0; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set(x_1, 2, x_264); +lean_ctor_set(x_1, 1, x_263); +lean_ctor_set(x_1, 0, x_205); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_267); +return x_1; } else { -uint8_t x_7; -x_7 = lean_nat_dec_le(x_3, x_3); -if (x_7 == 0) -{ -uint8_t x_8; -lean_dec(x_3); -x_8 = 0; -return x_8; +lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; uint8_t x_272; lean_object* x_273; uint8_t x_274; +x_268 = lean_ctor_get(x_205, 0); +x_269 = lean_ctor_get(x_205, 1); +x_270 = lean_ctor_get(x_205, 2); +x_271 = lean_ctor_get(x_205, 3); +lean_inc(x_271); +lean_inc(x_270); +lean_inc(x_269); +lean_inc(x_268); +lean_dec(x_205); +x_272 = 1; +x_273 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_273, 0, x_33); +lean_ctor_set(x_273, 1, x_34); +lean_ctor_set(x_273, 2, x_35); +lean_ctor_set(x_273, 3, x_268); +lean_ctor_set_uint8(x_273, sizeof(void*)*4, x_272); +lean_ctor_set(x_204, 0, x_271); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_272); +x_274 = 0; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set(x_1, 2, x_270); +lean_ctor_set(x_1, 1, x_269); +lean_ctor_set(x_1, 0, x_273); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_274); +return x_1; +} } else { -size_t x_9; size_t x_10; uint8_t x_11; -x_9 = 0; -x_10 = lean_usize_of_nat(x_3); -lean_dec(x_3); -x_11 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(x_2, x_1, x_9, x_10); -return x_11; +lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; uint8_t x_283; lean_object* x_284; lean_object* x_285; uint8_t x_286; +x_275 = lean_ctor_get(x_204, 1); +x_276 = lean_ctor_get(x_204, 2); +x_277 = lean_ctor_get(x_204, 3); +lean_inc(x_277); +lean_inc(x_276); +lean_inc(x_275); +lean_dec(x_204); +x_278 = lean_ctor_get(x_205, 0); +lean_inc(x_278); +x_279 = lean_ctor_get(x_205, 1); +lean_inc(x_279); +x_280 = lean_ctor_get(x_205, 2); +lean_inc(x_280); +x_281 = lean_ctor_get(x_205, 3); +lean_inc(x_281); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + lean_ctor_release(x_205, 2); + lean_ctor_release(x_205, 3); + x_282 = x_205; +} else { + lean_dec_ref(x_205); + x_282 = lean_box(0); } +x_283 = 1; +if (lean_is_scalar(x_282)) { + x_284 = lean_alloc_ctor(1, 4, 1); +} else { + x_284 = x_282; } +lean_ctor_set(x_284, 0, x_33); +lean_ctor_set(x_284, 1, x_34); +lean_ctor_set(x_284, 2, x_35); +lean_ctor_set(x_284, 3, x_278); +lean_ctor_set_uint8(x_284, sizeof(void*)*4, x_283); +x_285 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_285, 0, x_281); +lean_ctor_set(x_285, 1, x_275); +lean_ctor_set(x_285, 2, x_276); +lean_ctor_set(x_285, 3, x_277); +lean_ctor_set_uint8(x_285, sizeof(void*)*4, x_283); +x_286 = 0; +lean_ctor_set(x_1, 3, x_285); +lean_ctor_set(x_1, 2, x_280); +lean_ctor_set(x_1, 1, x_279); +lean_ctor_set(x_1, 0, x_284); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_286); +return x_1; } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: +else { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) +lean_object* x_287; +x_287 = lean_ctor_get(x_204, 3); +lean_inc(x_287); +if (lean_obj_tag(x_287) == 0) { -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_uget(x_2, x_3); -x_7 = l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1(x_1, x_6); -lean_dec(x_6); -if (x_7 == 0) +uint8_t x_288; +x_288 = !lean_is_exclusive(x_204); +if (x_288 == 0) { -size_t x_8; size_t x_9; -x_8 = 1; -x_9 = lean_usize_add(x_3, x_8); -x_3 = x_9; -goto _start; +lean_object* x_289; lean_object* x_290; uint8_t x_291; uint8_t x_292; +x_289 = lean_ctor_get(x_204, 3); +lean_dec(x_289); +x_290 = lean_ctor_get(x_204, 0); +lean_dec(x_290); +x_291 = 0; +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_291); +x_292 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_292); +return x_1; } else { -uint8_t x_11; -x_11 = 1; -return x_11; +lean_object* x_293; lean_object* x_294; uint8_t x_295; lean_object* x_296; uint8_t x_297; +x_293 = lean_ctor_get(x_204, 1); +x_294 = lean_ctor_get(x_204, 2); +lean_inc(x_294); +lean_inc(x_293); +lean_dec(x_204); +x_295 = 0; +x_296 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_296, 0, x_205); +lean_ctor_set(x_296, 1, x_293); +lean_ctor_set(x_296, 2, x_294); +lean_ctor_set(x_296, 3, x_287); +lean_ctor_set_uint8(x_296, sizeof(void*)*4, x_295); +x_297 = 1; +lean_ctor_set(x_1, 3, x_296); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_297); +return x_1; } } else { -uint8_t x_12; -x_12 = 0; -return x_12; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +uint8_t x_298; +x_298 = lean_ctor_get_uint8(x_287, sizeof(void*)*4); +if (x_298 == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_apply_2(x_2, x_3, x_4); -x_11 = l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(x_1, x_10, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_11) == 0) +uint8_t x_299; +lean_free_object(x_1); +x_299 = !lean_is_exclusive(x_204); +if (x_299 == 0) { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +lean_object* x_300; lean_object* x_301; uint8_t x_302; +x_300 = lean_ctor_get(x_204, 3); +lean_dec(x_300); +x_301 = lean_ctor_get(x_204, 0); +lean_dec(x_301); +x_302 = !lean_is_exclusive(x_287); +if (x_302 == 0) { -return x_11; +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; uint8_t x_307; uint8_t x_308; +x_303 = lean_ctor_get(x_287, 0); +x_304 = lean_ctor_get(x_287, 1); +x_305 = lean_ctor_get(x_287, 2); +x_306 = lean_ctor_get(x_287, 3); +x_307 = 1; +lean_inc(x_205); +lean_ctor_set(x_287, 3, x_205); +lean_ctor_set(x_287, 2, x_35); +lean_ctor_set(x_287, 1, x_34); +lean_ctor_set(x_287, 0, x_33); +x_308 = !lean_is_exclusive(x_205); +if (x_308 == 0) +{ +lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; uint8_t x_313; +x_309 = lean_ctor_get(x_205, 3); +lean_dec(x_309); +x_310 = lean_ctor_get(x_205, 2); +lean_dec(x_310); +x_311 = lean_ctor_get(x_205, 1); +lean_dec(x_311); +x_312 = lean_ctor_get(x_205, 0); +lean_dec(x_312); +lean_ctor_set_uint8(x_287, sizeof(void*)*4, x_307); +lean_ctor_set(x_205, 3, x_306); +lean_ctor_set(x_205, 2, x_305); +lean_ctor_set(x_205, 1, x_304); +lean_ctor_set(x_205, 0, x_303); +lean_ctor_set_uint8(x_205, sizeof(void*)*4, x_307); +x_313 = 0; +lean_ctor_set(x_204, 3, x_205); +lean_ctor_set(x_204, 0, x_287); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_313); +return x_204; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -return x_15; +lean_object* x_314; uint8_t x_315; +lean_dec(x_205); +lean_ctor_set_uint8(x_287, sizeof(void*)*4, x_307); +x_314 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_314, 0, x_303); +lean_ctor_set(x_314, 1, x_304); +lean_ctor_set(x_314, 2, x_305); +lean_ctor_set(x_314, 3, x_306); +lean_ctor_set_uint8(x_314, sizeof(void*)*4, x_307); +x_315 = 0; +lean_ctor_set(x_204, 3, x_314); +lean_ctor_set(x_204, 0, x_287); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_315); +return x_204; } } else { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_11); -if (x_16 == 0) -{ -return x_11; +lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; uint8_t x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; uint8_t x_324; +x_316 = lean_ctor_get(x_287, 0); +x_317 = lean_ctor_get(x_287, 1); +x_318 = lean_ctor_get(x_287, 2); +x_319 = lean_ctor_get(x_287, 3); +lean_inc(x_319); +lean_inc(x_318); +lean_inc(x_317); +lean_inc(x_316); +lean_dec(x_287); +x_320 = 1; +lean_inc(x_205); +x_321 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_321, 0, x_33); +lean_ctor_set(x_321, 1, x_34); +lean_ctor_set(x_321, 2, x_35); +lean_ctor_set(x_321, 3, x_205); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + lean_ctor_release(x_205, 2); + lean_ctor_release(x_205, 3); + x_322 = x_205; +} else { + lean_dec_ref(x_205); + x_322 = lean_box(0); +} +lean_ctor_set_uint8(x_321, sizeof(void*)*4, x_320); +if (lean_is_scalar(x_322)) { + x_323 = lean_alloc_ctor(1, 4, 1); +} else { + x_323 = x_322; +} +lean_ctor_set(x_323, 0, x_316); +lean_ctor_set(x_323, 1, x_317); +lean_ctor_set(x_323, 2, x_318); +lean_ctor_set(x_323, 3, x_319); +lean_ctor_set_uint8(x_323, sizeof(void*)*4, x_320); +x_324 = 0; +lean_ctor_set(x_204, 3, x_323); +lean_ctor_set(x_204, 0, x_321); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_324); +return x_204; +} } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_11, 0); -x_18 = lean_ctor_get(x_11, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_11); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} +lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; uint8_t x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; uint8_t x_336; lean_object* x_337; +x_325 = lean_ctor_get(x_204, 1); +x_326 = lean_ctor_get(x_204, 2); +lean_inc(x_326); +lean_inc(x_325); +lean_dec(x_204); +x_327 = lean_ctor_get(x_287, 0); +lean_inc(x_327); +x_328 = lean_ctor_get(x_287, 1); +lean_inc(x_328); +x_329 = lean_ctor_get(x_287, 2); +lean_inc(x_329); +x_330 = lean_ctor_get(x_287, 3); +lean_inc(x_330); +if (lean_is_exclusive(x_287)) { + lean_ctor_release(x_287, 0); + lean_ctor_release(x_287, 1); + lean_ctor_release(x_287, 2); + lean_ctor_release(x_287, 3); + x_331 = x_287; +} else { + lean_dec_ref(x_287); + x_331 = lean_box(0); } +x_332 = 1; +lean_inc(x_205); +if (lean_is_scalar(x_331)) { + x_333 = lean_alloc_ctor(1, 4, 1); +} else { + x_333 = x_331; } +lean_ctor_set(x_333, 0, x_33); +lean_ctor_set(x_333, 1, x_34); +lean_ctor_set(x_333, 2, x_35); +lean_ctor_set(x_333, 3, x_205); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + lean_ctor_release(x_205, 2); + lean_ctor_release(x_205, 3); + x_334 = x_205; +} else { + lean_dec_ref(x_205); + x_334 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withMVarContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___rarg), 9, 0); -return x_2; +lean_ctor_set_uint8(x_333, sizeof(void*)*4, x_332); +if (lean_is_scalar(x_334)) { + x_335 = lean_alloc_ctor(1, 4, 1); +} else { + x_335 = x_334; } +lean_ctor_set(x_335, 0, x_327); +lean_ctor_set(x_335, 1, x_328); +lean_ctor_set(x_335, 2, x_329); +lean_ctor_set(x_335, 3, x_330); +lean_ctor_set_uint8(x_335, sizeof(void*)*4, x_332); +x_336 = 0; +x_337 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_337, 0, x_333); +lean_ctor_set(x_337, 1, x_325); +lean_ctor_set(x_337, 2, x_326); +lean_ctor_set(x_337, 3, x_335); +lean_ctor_set_uint8(x_337, sizeof(void*)*4, x_336); +return x_337; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__5(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_5); -lean_ctor_set(x_14, 1, x_12); -return x_14; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -lean_dec(x_5); -x_15 = lean_array_uget(x_2, x_4); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -lean_inc(x_1); -x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Term_MVarErrorInfo_logError___boxed), 9, 2); -lean_closure_set(x_17, 0, x_15); -lean_closure_set(x_17, 1, x_1); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_18 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___rarg(x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_18) == 0) +uint8_t x_338; +x_338 = !lean_is_exclusive(x_204); +if (x_338 == 0) { -lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -lean_dec(x_18); -x_20 = 1; -x_21 = lean_usize_add(x_4, x_20); -x_22 = lean_box(0); -x_4 = x_21; -x_5 = x_22; -x_12 = x_19; -goto _start; +lean_object* x_339; lean_object* x_340; uint8_t x_341; +x_339 = lean_ctor_get(x_204, 3); +lean_dec(x_339); +x_340 = lean_ctor_get(x_204, 0); +lean_dec(x_340); +x_341 = !lean_is_exclusive(x_205); +if (x_341 == 0) +{ +uint8_t x_342; uint8_t x_343; +lean_ctor_set_uint8(x_205, sizeof(void*)*4, x_298); +x_342 = 0; +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_342); +x_343 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_343); +return x_1; } else { -uint8_t x_24; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_24 = !lean_is_exclusive(x_18); -if (x_24 == 0) -{ -return x_18; +lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; uint8_t x_349; uint8_t x_350; +x_344 = lean_ctor_get(x_205, 0); +x_345 = lean_ctor_get(x_205, 1); +x_346 = lean_ctor_get(x_205, 2); +x_347 = lean_ctor_get(x_205, 3); +lean_inc(x_347); +lean_inc(x_346); +lean_inc(x_345); +lean_inc(x_344); +lean_dec(x_205); +x_348 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_348, 0, x_344); +lean_ctor_set(x_348, 1, x_345); +lean_ctor_set(x_348, 2, x_346); +lean_ctor_set(x_348, 3, x_347); +lean_ctor_set_uint8(x_348, sizeof(void*)*4, x_298); +x_349 = 0; +lean_ctor_set(x_204, 0, x_348); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_349); +x_350 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_350); +return x_1; +} } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_18, 0); -x_26 = lean_ctor_get(x_18, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_18); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; uint8_t x_359; lean_object* x_360; uint8_t x_361; +x_351 = lean_ctor_get(x_204, 1); +x_352 = lean_ctor_get(x_204, 2); +lean_inc(x_352); +lean_inc(x_351); +lean_dec(x_204); +x_353 = lean_ctor_get(x_205, 0); +lean_inc(x_353); +x_354 = lean_ctor_get(x_205, 1); +lean_inc(x_354); +x_355 = lean_ctor_get(x_205, 2); +lean_inc(x_355); +x_356 = lean_ctor_get(x_205, 3); +lean_inc(x_356); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + lean_ctor_release(x_205, 2); + lean_ctor_release(x_205, 3); + x_357 = x_205; +} else { + lean_dec_ref(x_205); + x_357 = lean_box(0); +} +if (lean_is_scalar(x_357)) { + x_358 = lean_alloc_ctor(1, 4, 1); +} else { + x_358 = x_357; +} +lean_ctor_set(x_358, 0, x_353); +lean_ctor_set(x_358, 1, x_354); +lean_ctor_set(x_358, 2, x_355); +lean_ctor_set(x_358, 3, x_356); +lean_ctor_set_uint8(x_358, sizeof(void*)*4, x_298); +x_359 = 0; +x_360 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_360, 0, x_358); +lean_ctor_set(x_360, 1, x_351); +lean_ctor_set(x_360, 2, x_352); +lean_ctor_set(x_360, 3, x_287); +lean_ctor_set_uint8(x_360, sizeof(void*)*4, x_359); +x_361 = 1; +lean_ctor_set(x_1, 3, x_360); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_361); +return x_1; +} } } } } } -LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___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) { -_start: -{ -uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_12 = 1; -x_13 = lean_box(x_12); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_2); -lean_ctor_set(x_14, 1, x_13); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_1); -lean_ctor_set(x_15, 1, x_14); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_15); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_11); -return x_17; } } -LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6(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) { -_start: -{ -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_5); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -return x_14; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_15 = lean_ctor_get(x_4, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_4, 2); -lean_inc(x_16); -x_17 = lean_ctor_get(x_4, 3); -lean_inc(x_17); -lean_dec(x_4); -x_18 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -x_22 = lean_ctor_get(x_18, 1); -lean_inc(x_22); -lean_dec(x_18); -x_23 = !lean_is_exclusive(x_20); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_24 = lean_ctor_get(x_20, 0); -x_25 = lean_ctor_get(x_20, 1); -lean_dec(x_25); -x_26 = !lean_is_exclusive(x_21); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_21, 0); -x_28 = lean_ctor_get(x_21, 1); -x_29 = lean_ctor_get(x_16, 0); -lean_inc(x_29); -x_30 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_24, x_29); -if (lean_obj_tag(x_30) == 0) +lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; uint8_t x_366; +x_362 = lean_ctor_get(x_1, 0); +x_363 = lean_ctor_get(x_1, 1); +x_364 = lean_ctor_get(x_1, 2); +x_365 = lean_ctor_get(x_1, 3); +lean_inc(x_365); +lean_inc(x_364); +lean_inc(x_363); +lean_inc(x_362); +lean_dec(x_1); +x_366 = l_Lean_Name_quickCmp(x_2, x_363); +switch (x_366) { +case 0: { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -lean_inc(x_29); -x_31 = l_Lean_Expr_mvar___override(x_29); -x_32 = lean_box(0); -x_33 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_24, x_29, x_32); -x_34 = l_Lean_Meta_getMVars(x_31, x_8, x_9, x_10, x_11, x_22); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_array_get_size(x_35); -x_38 = lean_unsigned_to_nat(0u); -x_39 = lean_nat_dec_lt(x_38, x_37); -if (x_39 == 0) +uint8_t x_367; +x_367 = l_Std_RBNode_isRed___rarg(x_362); +if (x_367 == 0) { -lean_dec(x_37); -lean_dec(x_35); -lean_dec(x_16); -lean_ctor_set(x_20, 0, x_33); -x_4 = x_17; -x_5 = x_20; -x_12 = x_36; -goto _start; +lean_object* x_368; uint8_t x_369; lean_object* x_370; +x_368 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_362, x_2, x_3); +x_369 = 1; +x_370 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_370, 0, x_368); +lean_ctor_set(x_370, 1, x_363); +lean_ctor_set(x_370, 2, x_364); +lean_ctor_set(x_370, 3, x_365); +lean_ctor_set_uint8(x_370, sizeof(void*)*4, x_369); +return x_370; } else { -uint8_t x_41; -x_41 = lean_nat_dec_le(x_37, x_37); -if (x_41 == 0) -{ -lean_dec(x_37); -lean_dec(x_35); -lean_dec(x_16); -lean_ctor_set(x_20, 0, x_33); -x_4 = x_17; -x_5 = x_20; -x_12 = x_36; -goto _start; -} -else +lean_object* x_371; lean_object* x_372; +x_371 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_362, x_2, x_3); +x_372 = lean_ctor_get(x_371, 0); +lean_inc(x_372); +if (lean_obj_tag(x_372) == 0) { -size_t x_43; size_t x_44; uint8_t x_45; -x_43 = 0; -x_44 = lean_usize_of_nat(x_37); -lean_dec(x_37); -x_45 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_35, x_43, x_44); -lean_dec(x_35); -if (x_45 == 0) +lean_object* x_373; +x_373 = lean_ctor_get(x_371, 3); +lean_inc(x_373); +if (lean_obj_tag(x_373) == 0) { -lean_dec(x_16); -lean_ctor_set(x_20, 0, x_33); -x_4 = x_17; -x_5 = x_20; -x_12 = x_36; -goto _start; -} -else -{ -lean_free_object(x_21); -lean_free_object(x_20); -if (x_2 == 0) -{ -lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_47 = lean_array_push(x_27, x_16); -x_48 = lean_unbox(x_28); -lean_dec(x_28); -x_49 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_33, x_47, x_48, x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_36); -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = lean_ctor_get(x_50, 0); -lean_inc(x_52); -lean_dec(x_50); -x_4 = x_17; -x_5 = x_52; -x_12 = x_51; -goto _start; -} -else -{ -uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_16); -x_54 = lean_unbox(x_28); -lean_dec(x_28); -x_55 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_33, x_27, x_54, x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_36); -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -lean_dec(x_55); -x_58 = lean_ctor_get(x_56, 0); -lean_inc(x_58); -lean_dec(x_56); -x_4 = x_17; -x_5 = x_58; -x_12 = x_57; -goto _start; -} -} -} -} +lean_object* x_374; lean_object* x_375; lean_object* x_376; uint8_t x_377; lean_object* x_378; uint8_t x_379; lean_object* x_380; +x_374 = lean_ctor_get(x_371, 1); +lean_inc(x_374); +x_375 = lean_ctor_get(x_371, 2); +lean_inc(x_375); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_376 = x_371; +} else { + lean_dec_ref(x_371); + x_376 = lean_box(0); } -else -{ -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_16); -x_4 = x_17; -x_5 = x_20; -x_12 = x_22; -goto _start; +x_377 = 0; +if (lean_is_scalar(x_376)) { + x_378 = lean_alloc_ctor(1, 4, 1); +} else { + x_378 = x_376; } +lean_ctor_set(x_378, 0, x_373); +lean_ctor_set(x_378, 1, x_374); +lean_ctor_set(x_378, 2, x_375); +lean_ctor_set(x_378, 3, x_373); +lean_ctor_set_uint8(x_378, sizeof(void*)*4, x_377); +x_379 = 1; +x_380 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_380, 0, x_378); +lean_ctor_set(x_380, 1, x_363); +lean_ctor_set(x_380, 2, x_364); +lean_ctor_set(x_380, 3, x_365); +lean_ctor_set_uint8(x_380, sizeof(void*)*4, x_379); +return x_380; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_61 = lean_ctor_get(x_21, 0); -x_62 = lean_ctor_get(x_21, 1); -lean_inc(x_62); -lean_inc(x_61); -lean_dec(x_21); -x_63 = lean_ctor_get(x_16, 0); -lean_inc(x_63); -x_64 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_24, x_63); -if (lean_obj_tag(x_64) == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; -lean_inc(x_63); -x_65 = l_Lean_Expr_mvar___override(x_63); -x_66 = lean_box(0); -x_67 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_24, x_63, x_66); -x_68 = l_Lean_Meta_getMVars(x_65, x_8, x_9, x_10, x_11, x_22); -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_68, 1); -lean_inc(x_70); -lean_dec(x_68); -x_71 = lean_array_get_size(x_69); -x_72 = lean_unsigned_to_nat(0u); -x_73 = lean_nat_dec_lt(x_72, x_71); -if (x_73 == 0) +uint8_t x_381; +x_381 = lean_ctor_get_uint8(x_373, sizeof(void*)*4); +if (x_381 == 0) { -lean_object* x_74; -lean_dec(x_71); -lean_dec(x_69); -lean_dec(x_16); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_61); -lean_ctor_set(x_74, 1, x_62); -lean_ctor_set(x_20, 1, x_74); -lean_ctor_set(x_20, 0, x_67); -x_4 = x_17; -x_5 = x_20; -x_12 = x_70; -goto _start; +lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; uint8_t x_390; lean_object* x_391; lean_object* x_392; uint8_t x_393; lean_object* x_394; +x_382 = lean_ctor_get(x_371, 1); +lean_inc(x_382); +x_383 = lean_ctor_get(x_371, 2); +lean_inc(x_383); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_384 = x_371; +} else { + lean_dec_ref(x_371); + x_384 = lean_box(0); } -else -{ -uint8_t x_76; -x_76 = lean_nat_dec_le(x_71, x_71); -if (x_76 == 0) -{ -lean_object* x_77; -lean_dec(x_71); -lean_dec(x_69); -lean_dec(x_16); -x_77 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_77, 0, x_61); -lean_ctor_set(x_77, 1, x_62); -lean_ctor_set(x_20, 1, x_77); -lean_ctor_set(x_20, 0, x_67); -x_4 = x_17; -x_5 = x_20; -x_12 = x_70; -goto _start; +x_385 = lean_ctor_get(x_373, 0); +lean_inc(x_385); +x_386 = lean_ctor_get(x_373, 1); +lean_inc(x_386); +x_387 = lean_ctor_get(x_373, 2); +lean_inc(x_387); +x_388 = lean_ctor_get(x_373, 3); +lean_inc(x_388); +if (lean_is_exclusive(x_373)) { + lean_ctor_release(x_373, 0); + lean_ctor_release(x_373, 1); + lean_ctor_release(x_373, 2); + lean_ctor_release(x_373, 3); + x_389 = x_373; +} else { + lean_dec_ref(x_373); + x_389 = lean_box(0); } -else -{ -size_t x_79; size_t x_80; uint8_t x_81; -x_79 = 0; -x_80 = lean_usize_of_nat(x_71); -lean_dec(x_71); -x_81 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_69, x_79, x_80); -lean_dec(x_69); -if (x_81 == 0) -{ -lean_object* x_82; -lean_dec(x_16); -x_82 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_82, 0, x_61); -lean_ctor_set(x_82, 1, x_62); -lean_ctor_set(x_20, 1, x_82); -lean_ctor_set(x_20, 0, x_67); -x_4 = x_17; -x_5 = x_20; -x_12 = x_70; -goto _start; +x_390 = 1; +if (lean_is_scalar(x_389)) { + x_391 = lean_alloc_ctor(1, 4, 1); +} else { + x_391 = x_389; } -else -{ -lean_free_object(x_20); -if (x_2 == 0) -{ -lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_84 = lean_array_push(x_61, x_16); -x_85 = lean_unbox(x_62); -lean_dec(x_62); -x_86 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_67, x_84, x_85, x_66, x_6, x_7, x_8, x_9, x_10, x_11, x_70); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); -lean_inc(x_88); -lean_dec(x_86); -x_89 = lean_ctor_get(x_87, 0); -lean_inc(x_89); -lean_dec(x_87); -x_4 = x_17; -x_5 = x_89; -x_12 = x_88; -goto _start; +lean_ctor_set(x_391, 0, x_372); +lean_ctor_set(x_391, 1, x_382); +lean_ctor_set(x_391, 2, x_383); +lean_ctor_set(x_391, 3, x_385); +lean_ctor_set_uint8(x_391, sizeof(void*)*4, x_390); +if (lean_is_scalar(x_384)) { + x_392 = lean_alloc_ctor(1, 4, 1); +} else { + x_392 = x_384; +} +lean_ctor_set(x_392, 0, x_388); +lean_ctor_set(x_392, 1, x_363); +lean_ctor_set(x_392, 2, x_364); +lean_ctor_set(x_392, 3, x_365); +lean_ctor_set_uint8(x_392, sizeof(void*)*4, x_390); +x_393 = 0; +x_394 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_394, 0, x_391); +lean_ctor_set(x_394, 1, x_386); +lean_ctor_set(x_394, 2, x_387); +lean_ctor_set(x_394, 3, x_392); +lean_ctor_set_uint8(x_394, sizeof(void*)*4, x_393); +return x_394; } else { -uint8_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -lean_dec(x_16); -x_91 = lean_unbox(x_62); -lean_dec(x_62); -x_92 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_67, x_61, x_91, x_66, x_6, x_7, x_8, x_9, x_10, x_11, x_70); -x_93 = lean_ctor_get(x_92, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_92, 1); -lean_inc(x_94); -lean_dec(x_92); -x_95 = lean_ctor_get(x_93, 0); -lean_inc(x_95); -lean_dec(x_93); -x_4 = x_17; -x_5 = x_95; -x_12 = x_94; -goto _start; +lean_object* x_395; lean_object* x_396; lean_object* x_397; uint8_t x_398; lean_object* x_399; uint8_t x_400; lean_object* x_401; +x_395 = lean_ctor_get(x_371, 1); +lean_inc(x_395); +x_396 = lean_ctor_get(x_371, 2); +lean_inc(x_396); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_397 = x_371; +} else { + lean_dec_ref(x_371); + x_397 = lean_box(0); } +x_398 = 0; +if (lean_is_scalar(x_397)) { + x_399 = lean_alloc_ctor(1, 4, 1); +} else { + x_399 = x_397; } +lean_ctor_set(x_399, 0, x_372); +lean_ctor_set(x_399, 1, x_395); +lean_ctor_set(x_399, 2, x_396); +lean_ctor_set(x_399, 3, x_373); +lean_ctor_set_uint8(x_399, sizeof(void*)*4, x_398); +x_400 = 1; +x_401 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_401, 0, x_399); +lean_ctor_set(x_401, 1, x_363); +lean_ctor_set(x_401, 2, x_364); +lean_ctor_set(x_401, 3, x_365); +lean_ctor_set_uint8(x_401, sizeof(void*)*4, x_400); +return x_401; } } } else { -lean_object* x_97; -lean_dec(x_64); -lean_dec(x_63); -lean_dec(x_16); -x_97 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_97, 0, x_61); -lean_ctor_set(x_97, 1, x_62); -lean_ctor_set(x_20, 1, x_97); -x_4 = x_17; -x_5 = x_20; -x_12 = x_22; -goto _start; -} -} -} -else +uint8_t x_402; +x_402 = lean_ctor_get_uint8(x_372, sizeof(void*)*4); +if (x_402 == 0) { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_99 = lean_ctor_get(x_20, 0); -lean_inc(x_99); -lean_dec(x_20); -x_100 = lean_ctor_get(x_21, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_21, 1); -lean_inc(x_101); -if (lean_is_exclusive(x_21)) { - lean_ctor_release(x_21, 0); - lean_ctor_release(x_21, 1); - x_102 = x_21; +lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; uint8_t x_412; lean_object* x_413; lean_object* x_414; uint8_t x_415; lean_object* x_416; +x_403 = lean_ctor_get(x_371, 1); +lean_inc(x_403); +x_404 = lean_ctor_get(x_371, 2); +lean_inc(x_404); +x_405 = lean_ctor_get(x_371, 3); +lean_inc(x_405); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_406 = x_371; } else { - lean_dec_ref(x_21); - x_102 = lean_box(0); + lean_dec_ref(x_371); + x_406 = lean_box(0); } -x_103 = lean_ctor_get(x_16, 0); -lean_inc(x_103); -x_104 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_99, x_103); -if (lean_obj_tag(x_104) == 0) -{ -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; -lean_inc(x_103); -x_105 = l_Lean_Expr_mvar___override(x_103); -x_106 = lean_box(0); -x_107 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_99, x_103, x_106); -x_108 = l_Lean_Meta_getMVars(x_105, x_8, x_9, x_10, x_11, x_22); -x_109 = lean_ctor_get(x_108, 0); -lean_inc(x_109); -x_110 = lean_ctor_get(x_108, 1); -lean_inc(x_110); -lean_dec(x_108); -x_111 = lean_array_get_size(x_109); -x_112 = lean_unsigned_to_nat(0u); -x_113 = lean_nat_dec_lt(x_112, x_111); -if (x_113 == 0) -{ -lean_object* x_114; lean_object* x_115; -lean_dec(x_111); -lean_dec(x_109); -lean_dec(x_16); -if (lean_is_scalar(x_102)) { - x_114 = lean_alloc_ctor(0, 2, 0); +x_407 = lean_ctor_get(x_372, 0); +lean_inc(x_407); +x_408 = lean_ctor_get(x_372, 1); +lean_inc(x_408); +x_409 = lean_ctor_get(x_372, 2); +lean_inc(x_409); +x_410 = lean_ctor_get(x_372, 3); +lean_inc(x_410); +if (lean_is_exclusive(x_372)) { + lean_ctor_release(x_372, 0); + lean_ctor_release(x_372, 1); + lean_ctor_release(x_372, 2); + lean_ctor_release(x_372, 3); + x_411 = x_372; } else { - x_114 = x_102; + lean_dec_ref(x_372); + x_411 = lean_box(0); } -lean_ctor_set(x_114, 0, x_100); -lean_ctor_set(x_114, 1, x_101); -x_115 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_115, 0, x_107); -lean_ctor_set(x_115, 1, x_114); -x_4 = x_17; -x_5 = x_115; -x_12 = x_110; -goto _start; +x_412 = 1; +if (lean_is_scalar(x_411)) { + x_413 = lean_alloc_ctor(1, 4, 1); +} else { + x_413 = x_411; } -else -{ -uint8_t x_117; -x_117 = lean_nat_dec_le(x_111, x_111); -if (x_117 == 0) -{ -lean_object* x_118; lean_object* x_119; -lean_dec(x_111); -lean_dec(x_109); -lean_dec(x_16); -if (lean_is_scalar(x_102)) { - x_118 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_413, 0, x_407); +lean_ctor_set(x_413, 1, x_408); +lean_ctor_set(x_413, 2, x_409); +lean_ctor_set(x_413, 3, x_410); +lean_ctor_set_uint8(x_413, sizeof(void*)*4, x_412); +if (lean_is_scalar(x_406)) { + x_414 = lean_alloc_ctor(1, 4, 1); } else { - x_118 = x_102; + x_414 = x_406; } -lean_ctor_set(x_118, 0, x_100); -lean_ctor_set(x_118, 1, x_101); -x_119 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_119, 0, x_107); -lean_ctor_set(x_119, 1, x_118); -x_4 = x_17; -x_5 = x_119; -x_12 = x_110; -goto _start; +lean_ctor_set(x_414, 0, x_405); +lean_ctor_set(x_414, 1, x_363); +lean_ctor_set(x_414, 2, x_364); +lean_ctor_set(x_414, 3, x_365); +lean_ctor_set_uint8(x_414, sizeof(void*)*4, x_412); +x_415 = 0; +x_416 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_416, 0, x_413); +lean_ctor_set(x_416, 1, x_403); +lean_ctor_set(x_416, 2, x_404); +lean_ctor_set(x_416, 3, x_414); +lean_ctor_set_uint8(x_416, sizeof(void*)*4, x_415); +return x_416; } else { -size_t x_121; size_t x_122; uint8_t x_123; -x_121 = 0; -x_122 = lean_usize_of_nat(x_111); -lean_dec(x_111); -x_123 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_109, x_121, x_122); -lean_dec(x_109); -if (x_123 == 0) +lean_object* x_417; +x_417 = lean_ctor_get(x_371, 3); +lean_inc(x_417); +if (lean_obj_tag(x_417) == 0) { -lean_object* x_124; lean_object* x_125; -lean_dec(x_16); -if (lean_is_scalar(x_102)) { - x_124 = lean_alloc_ctor(0, 2, 0); +lean_object* x_418; lean_object* x_419; lean_object* x_420; uint8_t x_421; lean_object* x_422; uint8_t x_423; lean_object* x_424; +x_418 = lean_ctor_get(x_371, 1); +lean_inc(x_418); +x_419 = lean_ctor_get(x_371, 2); +lean_inc(x_419); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_420 = x_371; } else { - x_124 = x_102; + lean_dec_ref(x_371); + x_420 = lean_box(0); } -lean_ctor_set(x_124, 0, x_100); -lean_ctor_set(x_124, 1, x_101); -x_125 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_125, 0, x_107); -lean_ctor_set(x_125, 1, x_124); -x_4 = x_17; -x_5 = x_125; -x_12 = x_110; -goto _start; +x_421 = 0; +if (lean_is_scalar(x_420)) { + x_422 = lean_alloc_ctor(1, 4, 1); +} else { + x_422 = x_420; +} +lean_ctor_set(x_422, 0, x_372); +lean_ctor_set(x_422, 1, x_418); +lean_ctor_set(x_422, 2, x_419); +lean_ctor_set(x_422, 3, x_417); +lean_ctor_set_uint8(x_422, sizeof(void*)*4, x_421); +x_423 = 1; +x_424 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_424, 0, x_422); +lean_ctor_set(x_424, 1, x_363); +lean_ctor_set(x_424, 2, x_364); +lean_ctor_set(x_424, 3, x_365); +lean_ctor_set_uint8(x_424, sizeof(void*)*4, x_423); +return x_424; } else { -lean_dec(x_102); -if (x_2 == 0) +uint8_t x_425; +x_425 = lean_ctor_get_uint8(x_417, sizeof(void*)*4); +if (x_425 == 0) { -lean_object* x_127; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_127 = lean_array_push(x_100, x_16); -x_128 = lean_unbox(x_101); -lean_dec(x_101); -x_129 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_107, x_127, x_128, x_106, x_6, x_7, x_8, x_9, x_10, x_11, x_110); -x_130 = lean_ctor_get(x_129, 0); -lean_inc(x_130); -x_131 = lean_ctor_get(x_129, 1); -lean_inc(x_131); -lean_dec(x_129); -x_132 = lean_ctor_get(x_130, 0); -lean_inc(x_132); -lean_dec(x_130); -x_4 = x_17; -x_5 = x_132; -x_12 = x_131; -goto _start; +lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; uint8_t x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; uint8_t x_438; lean_object* x_439; +x_426 = lean_ctor_get(x_371, 1); +lean_inc(x_426); +x_427 = lean_ctor_get(x_371, 2); +lean_inc(x_427); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_428 = x_371; +} else { + lean_dec_ref(x_371); + x_428 = lean_box(0); } -else -{ -uint8_t x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; -lean_dec(x_16); -x_134 = lean_unbox(x_101); -lean_dec(x_101); -x_135 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_107, x_100, x_134, x_106, x_6, x_7, x_8, x_9, x_10, x_11, x_110); -x_136 = lean_ctor_get(x_135, 0); -lean_inc(x_136); -x_137 = lean_ctor_get(x_135, 1); -lean_inc(x_137); -lean_dec(x_135); -x_138 = lean_ctor_get(x_136, 0); -lean_inc(x_138); -lean_dec(x_136); -x_4 = x_17; -x_5 = x_138; -x_12 = x_137; -goto _start; +x_429 = lean_ctor_get(x_417, 0); +lean_inc(x_429); +x_430 = lean_ctor_get(x_417, 1); +lean_inc(x_430); +x_431 = lean_ctor_get(x_417, 2); +lean_inc(x_431); +x_432 = lean_ctor_get(x_417, 3); +lean_inc(x_432); +if (lean_is_exclusive(x_417)) { + lean_ctor_release(x_417, 0); + lean_ctor_release(x_417, 1); + lean_ctor_release(x_417, 2); + lean_ctor_release(x_417, 3); + x_433 = x_417; +} else { + lean_dec_ref(x_417); + x_433 = lean_box(0); +} +x_434 = 1; +lean_inc(x_372); +if (lean_is_scalar(x_433)) { + x_435 = lean_alloc_ctor(1, 4, 1); +} else { + x_435 = x_433; } +lean_ctor_set(x_435, 0, x_372); +lean_ctor_set(x_435, 1, x_426); +lean_ctor_set(x_435, 2, x_427); +lean_ctor_set(x_435, 3, x_429); +if (lean_is_exclusive(x_372)) { + lean_ctor_release(x_372, 0); + lean_ctor_release(x_372, 1); + lean_ctor_release(x_372, 2); + lean_ctor_release(x_372, 3); + x_436 = x_372; +} else { + lean_dec_ref(x_372); + x_436 = lean_box(0); } +lean_ctor_set_uint8(x_435, sizeof(void*)*4, x_434); +if (lean_is_scalar(x_436)) { + x_437 = lean_alloc_ctor(1, 4, 1); +} else { + x_437 = x_436; } +lean_ctor_set(x_437, 0, x_432); +lean_ctor_set(x_437, 1, x_363); +lean_ctor_set(x_437, 2, x_364); +lean_ctor_set(x_437, 3, x_365); +lean_ctor_set_uint8(x_437, sizeof(void*)*4, x_434); +x_438 = 0; +if (lean_is_scalar(x_428)) { + x_439 = lean_alloc_ctor(1, 4, 1); +} else { + x_439 = x_428; } +lean_ctor_set(x_439, 0, x_435); +lean_ctor_set(x_439, 1, x_430); +lean_ctor_set(x_439, 2, x_431); +lean_ctor_set(x_439, 3, x_437); +lean_ctor_set_uint8(x_439, sizeof(void*)*4, x_438); +return x_439; } else { -lean_object* x_140; lean_object* x_141; -lean_dec(x_104); -lean_dec(x_103); -lean_dec(x_16); -if (lean_is_scalar(x_102)) { - x_140 = lean_alloc_ctor(0, 2, 0); +lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; uint8_t x_449; lean_object* x_450; uint8_t x_451; lean_object* x_452; +x_440 = lean_ctor_get(x_371, 1); +lean_inc(x_440); +x_441 = lean_ctor_get(x_371, 2); +lean_inc(x_441); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_442 = x_371; } else { - x_140 = x_102; + lean_dec_ref(x_371); + x_442 = lean_box(0); } -lean_ctor_set(x_140, 0, x_100); -lean_ctor_set(x_140, 1, x_101); -x_141 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_141, 0, x_99); -lean_ctor_set(x_141, 1, x_140); -x_4 = x_17; -x_5 = x_141; -x_12 = x_22; -goto _start; +x_443 = lean_ctor_get(x_372, 0); +lean_inc(x_443); +x_444 = lean_ctor_get(x_372, 1); +lean_inc(x_444); +x_445 = lean_ctor_get(x_372, 2); +lean_inc(x_445); +x_446 = lean_ctor_get(x_372, 3); +lean_inc(x_446); +if (lean_is_exclusive(x_372)) { + lean_ctor_release(x_372, 0); + lean_ctor_release(x_372, 1); + lean_ctor_release(x_372, 2); + lean_ctor_release(x_372, 3); + x_447 = x_372; +} else { + lean_dec_ref(x_372); + x_447 = lean_box(0); } +if (lean_is_scalar(x_447)) { + x_448 = lean_alloc_ctor(1, 4, 1); +} else { + x_448 = x_447; } +lean_ctor_set(x_448, 0, x_443); +lean_ctor_set(x_448, 1, x_444); +lean_ctor_set(x_448, 2, x_445); +lean_ctor_set(x_448, 3, x_446); +lean_ctor_set_uint8(x_448, sizeof(void*)*4, x_425); +x_449 = 0; +if (lean_is_scalar(x_442)) { + x_450 = lean_alloc_ctor(1, 4, 1); +} else { + x_450 = x_442; } +lean_ctor_set(x_450, 0, x_448); +lean_ctor_set(x_450, 1, x_440); +lean_ctor_set(x_450, 2, x_441); +lean_ctor_set(x_450, 3, x_417); +lean_ctor_set_uint8(x_450, sizeof(void*)*4, x_449); +x_451 = 1; +x_452 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_452, 0, x_450); +lean_ctor_set(x_452, 1, x_363); +lean_ctor_set(x_452, 2, x_364); +lean_ctor_set(x_452, 3, x_365); +lean_ctor_set_uint8(x_452, sizeof(void*)*4, x_451); +return x_452; } } -LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(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) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -lean_object* x_12; lean_object* x_13; -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_4); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; } -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_14 = lean_ctor_get(x_3, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_3, 2); -lean_inc(x_15); -x_16 = lean_ctor_get(x_3, 3); -lean_inc(x_16); -lean_dec(x_3); -x_17 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(x_1, x_2, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_17, 1); -lean_inc(x_21); -lean_dec(x_17); -x_22 = !lean_is_exclusive(x_19); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_23 = lean_ctor_get(x_19, 0); -x_24 = lean_ctor_get(x_19, 1); -lean_dec(x_24); -x_25 = !lean_is_exclusive(x_20); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_26 = lean_ctor_get(x_20, 0); -x_27 = lean_ctor_get(x_20, 1); -x_28 = lean_ctor_get(x_15, 0); -lean_inc(x_28); -x_29 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_23, x_28); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -lean_inc(x_28); -x_30 = l_Lean_Expr_mvar___override(x_28); -x_31 = lean_box(0); -x_32 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_23, x_28, x_31); -x_33 = l_Lean_Meta_getMVars(x_30, x_7, x_8, x_9, x_10, x_21); -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_array_get_size(x_34); -x_37 = lean_unsigned_to_nat(0u); -x_38 = lean_nat_dec_lt(x_37, x_36); -if (x_38 == 0) -{ -lean_dec(x_36); -lean_dec(x_34); -lean_dec(x_15); -lean_ctor_set(x_19, 0, x_32); -x_3 = x_16; -x_4 = x_19; -x_11 = x_35; -goto _start; } -else -{ -uint8_t x_40; -x_40 = lean_nat_dec_le(x_36, x_36); -if (x_40 == 0) +} +} +case 1: { -lean_dec(x_36); -lean_dec(x_34); -lean_dec(x_15); -lean_ctor_set(x_19, 0, x_32); -x_3 = x_16; -x_4 = x_19; -x_11 = x_35; -goto _start; +uint8_t x_453; lean_object* x_454; +lean_dec(x_364); +lean_dec(x_363); +x_453 = 1; +x_454 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_454, 0, x_362); +lean_ctor_set(x_454, 1, x_2); +lean_ctor_set(x_454, 2, x_3); +lean_ctor_set(x_454, 3, x_365); +lean_ctor_set_uint8(x_454, sizeof(void*)*4, x_453); +return x_454; } -else +default: { -size_t x_42; size_t x_43; uint8_t x_44; -x_42 = 0; -x_43 = lean_usize_of_nat(x_36); -lean_dec(x_36); -x_44 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_34, x_42, x_43); -lean_dec(x_34); -if (x_44 == 0) +uint8_t x_455; +x_455 = l_Std_RBNode_isRed___rarg(x_365); +if (x_455 == 0) { -lean_dec(x_15); -lean_ctor_set(x_19, 0, x_32); -x_3 = x_16; -x_4 = x_19; -x_11 = x_35; -goto _start; +lean_object* x_456; uint8_t x_457; lean_object* x_458; +x_456 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_365, x_2, x_3); +x_457 = 1; +x_458 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_458, 0, x_362); +lean_ctor_set(x_458, 1, x_363); +lean_ctor_set(x_458, 2, x_364); +lean_ctor_set(x_458, 3, x_456); +lean_ctor_set_uint8(x_458, sizeof(void*)*4, x_457); +return x_458; } else { -lean_free_object(x_20); -lean_free_object(x_19); -if (x_2 == 0) +lean_object* x_459; lean_object* x_460; +x_459 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_365, x_2, x_3); +x_460 = lean_ctor_get(x_459, 0); +lean_inc(x_460); +if (lean_obj_tag(x_460) == 0) { -lean_object* x_46; uint8_t x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_46 = lean_array_push(x_26, x_15); -x_47 = lean_unbox(x_27); -lean_dec(x_27); -x_48 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_32, x_46, x_47, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_35); -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_48, 1); -lean_inc(x_50); -lean_dec(x_48); -x_51 = lean_ctor_get(x_49, 0); -lean_inc(x_51); -lean_dec(x_49); -x_3 = x_16; -x_4 = x_51; -x_11 = x_50; -goto _start; +lean_object* x_461; +x_461 = lean_ctor_get(x_459, 3); +lean_inc(x_461); +if (lean_obj_tag(x_461) == 0) +{ +lean_object* x_462; lean_object* x_463; lean_object* x_464; uint8_t x_465; lean_object* x_466; uint8_t x_467; lean_object* x_468; +x_462 = lean_ctor_get(x_459, 1); +lean_inc(x_462); +x_463 = lean_ctor_get(x_459, 2); +lean_inc(x_463); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_464 = x_459; +} else { + lean_dec_ref(x_459); + x_464 = lean_box(0); +} +x_465 = 0; +if (lean_is_scalar(x_464)) { + x_466 = lean_alloc_ctor(1, 4, 1); +} else { + x_466 = x_464; +} +lean_ctor_set(x_466, 0, x_461); +lean_ctor_set(x_466, 1, x_462); +lean_ctor_set(x_466, 2, x_463); +lean_ctor_set(x_466, 3, x_461); +lean_ctor_set_uint8(x_466, sizeof(void*)*4, x_465); +x_467 = 1; +x_468 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_468, 0, x_362); +lean_ctor_set(x_468, 1, x_363); +lean_ctor_set(x_468, 2, x_364); +lean_ctor_set(x_468, 3, x_466); +lean_ctor_set_uint8(x_468, sizeof(void*)*4, x_467); +return x_468; } else { -uint8_t x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -lean_dec(x_15); -x_53 = lean_unbox(x_27); -lean_dec(x_27); -x_54 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_32, x_26, x_53, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_35); -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_54, 1); -lean_inc(x_56); -lean_dec(x_54); -x_57 = lean_ctor_get(x_55, 0); -lean_inc(x_57); -lean_dec(x_55); -x_3 = x_16; -x_4 = x_57; -x_11 = x_56; -goto _start; +uint8_t x_469; +x_469 = lean_ctor_get_uint8(x_461, sizeof(void*)*4); +if (x_469 == 0) +{ +lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; uint8_t x_478; lean_object* x_479; lean_object* x_480; uint8_t x_481; lean_object* x_482; +x_470 = lean_ctor_get(x_459, 1); +lean_inc(x_470); +x_471 = lean_ctor_get(x_459, 2); +lean_inc(x_471); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_472 = x_459; +} else { + lean_dec_ref(x_459); + x_472 = lean_box(0); } +x_473 = lean_ctor_get(x_461, 0); +lean_inc(x_473); +x_474 = lean_ctor_get(x_461, 1); +lean_inc(x_474); +x_475 = lean_ctor_get(x_461, 2); +lean_inc(x_475); +x_476 = lean_ctor_get(x_461, 3); +lean_inc(x_476); +if (lean_is_exclusive(x_461)) { + lean_ctor_release(x_461, 0); + lean_ctor_release(x_461, 1); + lean_ctor_release(x_461, 2); + lean_ctor_release(x_461, 3); + x_477 = x_461; +} else { + lean_dec_ref(x_461); + x_477 = lean_box(0); } +x_478 = 1; +if (lean_is_scalar(x_477)) { + x_479 = lean_alloc_ctor(1, 4, 1); +} else { + x_479 = x_477; } +lean_ctor_set(x_479, 0, x_362); +lean_ctor_set(x_479, 1, x_363); +lean_ctor_set(x_479, 2, x_364); +lean_ctor_set(x_479, 3, x_460); +lean_ctor_set_uint8(x_479, sizeof(void*)*4, x_478); +if (lean_is_scalar(x_472)) { + x_480 = lean_alloc_ctor(1, 4, 1); +} else { + x_480 = x_472; } +lean_ctor_set(x_480, 0, x_473); +lean_ctor_set(x_480, 1, x_474); +lean_ctor_set(x_480, 2, x_475); +lean_ctor_set(x_480, 3, x_476); +lean_ctor_set_uint8(x_480, sizeof(void*)*4, x_478); +x_481 = 0; +x_482 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_482, 0, x_479); +lean_ctor_set(x_482, 1, x_470); +lean_ctor_set(x_482, 2, x_471); +lean_ctor_set(x_482, 3, x_480); +lean_ctor_set_uint8(x_482, sizeof(void*)*4, x_481); +return x_482; } else { -lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_15); -x_3 = x_16; -x_4 = x_19; -x_11 = x_21; -goto _start; +lean_object* x_483; lean_object* x_484; lean_object* x_485; uint8_t x_486; lean_object* x_487; uint8_t x_488; lean_object* x_489; +x_483 = lean_ctor_get(x_459, 1); +lean_inc(x_483); +x_484 = lean_ctor_get(x_459, 2); +lean_inc(x_484); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_485 = x_459; +} else { + lean_dec_ref(x_459); + x_485 = lean_box(0); +} +x_486 = 0; +if (lean_is_scalar(x_485)) { + x_487 = lean_alloc_ctor(1, 4, 1); +} else { + x_487 = x_485; +} +lean_ctor_set(x_487, 0, x_460); +lean_ctor_set(x_487, 1, x_483); +lean_ctor_set(x_487, 2, x_484); +lean_ctor_set(x_487, 3, x_461); +lean_ctor_set_uint8(x_487, sizeof(void*)*4, x_486); +x_488 = 1; +x_489 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_489, 0, x_362); +lean_ctor_set(x_489, 1, x_363); +lean_ctor_set(x_489, 2, x_364); +lean_ctor_set(x_489, 3, x_487); +lean_ctor_set_uint8(x_489, sizeof(void*)*4, x_488); +return x_489; +} } } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_60 = lean_ctor_get(x_20, 0); -x_61 = lean_ctor_get(x_20, 1); -lean_inc(x_61); -lean_inc(x_60); -lean_dec(x_20); -x_62 = lean_ctor_get(x_15, 0); -lean_inc(x_62); -x_63 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_23, x_62); -if (lean_obj_tag(x_63) == 0) +uint8_t x_490; +x_490 = lean_ctor_get_uint8(x_460, sizeof(void*)*4); +if (x_490 == 0) { -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -lean_inc(x_62); -x_64 = l_Lean_Expr_mvar___override(x_62); -x_65 = lean_box(0); -x_66 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_23, x_62, x_65); -x_67 = l_Lean_Meta_getMVars(x_64, x_7, x_8, x_9, x_10, x_21); -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_array_get_size(x_68); -x_71 = lean_unsigned_to_nat(0u); -x_72 = lean_nat_dec_lt(x_71, x_70); -if (x_72 == 0) -{ -lean_object* x_73; -lean_dec(x_70); -lean_dec(x_68); -lean_dec(x_15); -x_73 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_73, 0, x_60); -lean_ctor_set(x_73, 1, x_61); -lean_ctor_set(x_19, 1, x_73); -lean_ctor_set(x_19, 0, x_66); -x_3 = x_16; -x_4 = x_19; -x_11 = x_69; -goto _start; +lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; uint8_t x_500; lean_object* x_501; lean_object* x_502; uint8_t x_503; lean_object* x_504; +x_491 = lean_ctor_get(x_459, 1); +lean_inc(x_491); +x_492 = lean_ctor_get(x_459, 2); +lean_inc(x_492); +x_493 = lean_ctor_get(x_459, 3); +lean_inc(x_493); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_494 = x_459; +} else { + lean_dec_ref(x_459); + x_494 = lean_box(0); } -else -{ -uint8_t x_75; -x_75 = lean_nat_dec_le(x_70, x_70); -if (x_75 == 0) -{ -lean_object* x_76; -lean_dec(x_70); -lean_dec(x_68); -lean_dec(x_15); -x_76 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_76, 0, x_60); -lean_ctor_set(x_76, 1, x_61); -lean_ctor_set(x_19, 1, x_76); -lean_ctor_set(x_19, 0, x_66); -x_3 = x_16; -x_4 = x_19; -x_11 = x_69; -goto _start; +x_495 = lean_ctor_get(x_460, 0); +lean_inc(x_495); +x_496 = lean_ctor_get(x_460, 1); +lean_inc(x_496); +x_497 = lean_ctor_get(x_460, 2); +lean_inc(x_497); +x_498 = lean_ctor_get(x_460, 3); +lean_inc(x_498); +if (lean_is_exclusive(x_460)) { + lean_ctor_release(x_460, 0); + lean_ctor_release(x_460, 1); + lean_ctor_release(x_460, 2); + lean_ctor_release(x_460, 3); + x_499 = x_460; +} else { + lean_dec_ref(x_460); + x_499 = lean_box(0); } -else -{ -size_t x_78; size_t x_79; uint8_t x_80; -x_78 = 0; -x_79 = lean_usize_of_nat(x_70); -lean_dec(x_70); -x_80 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_68, x_78, x_79); -lean_dec(x_68); -if (x_80 == 0) -{ -lean_object* x_81; -lean_dec(x_15); -x_81 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_81, 0, x_60); -lean_ctor_set(x_81, 1, x_61); -lean_ctor_set(x_19, 1, x_81); -lean_ctor_set(x_19, 0, x_66); -x_3 = x_16; -x_4 = x_19; -x_11 = x_69; -goto _start; +x_500 = 1; +if (lean_is_scalar(x_499)) { + x_501 = lean_alloc_ctor(1, 4, 1); +} else { + x_501 = x_499; } -else -{ -lean_free_object(x_19); -if (x_2 == 0) -{ -lean_object* x_83; uint8_t x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_83 = lean_array_push(x_60, x_15); -x_84 = lean_unbox(x_61); -lean_dec(x_61); -x_85 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_66, x_83, x_84, x_65, x_5, x_6, x_7, x_8, x_9, x_10, x_69); -x_86 = lean_ctor_get(x_85, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_85, 1); -lean_inc(x_87); -lean_dec(x_85); -x_88 = lean_ctor_get(x_86, 0); -lean_inc(x_88); -lean_dec(x_86); -x_3 = x_16; -x_4 = x_88; -x_11 = x_87; -goto _start; +lean_ctor_set(x_501, 0, x_362); +lean_ctor_set(x_501, 1, x_363); +lean_ctor_set(x_501, 2, x_364); +lean_ctor_set(x_501, 3, x_495); +lean_ctor_set_uint8(x_501, sizeof(void*)*4, x_500); +if (lean_is_scalar(x_494)) { + x_502 = lean_alloc_ctor(1, 4, 1); +} else { + x_502 = x_494; +} +lean_ctor_set(x_502, 0, x_498); +lean_ctor_set(x_502, 1, x_491); +lean_ctor_set(x_502, 2, x_492); +lean_ctor_set(x_502, 3, x_493); +lean_ctor_set_uint8(x_502, sizeof(void*)*4, x_500); +x_503 = 0; +x_504 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_504, 0, x_501); +lean_ctor_set(x_504, 1, x_496); +lean_ctor_set(x_504, 2, x_497); +lean_ctor_set(x_504, 3, x_502); +lean_ctor_set_uint8(x_504, sizeof(void*)*4, x_503); +return x_504; } else { -uint8_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -lean_dec(x_15); -x_90 = lean_unbox(x_61); -lean_dec(x_61); -x_91 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_66, x_60, x_90, x_65, x_5, x_6, x_7, x_8, x_9, x_10, x_69); -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); -lean_dec(x_91); -x_94 = lean_ctor_get(x_92, 0); -lean_inc(x_94); -lean_dec(x_92); -x_3 = x_16; -x_4 = x_94; -x_11 = x_93; -goto _start; -} -} +lean_object* x_505; +x_505 = lean_ctor_get(x_459, 3); +lean_inc(x_505); +if (lean_obj_tag(x_505) == 0) +{ +lean_object* x_506; lean_object* x_507; lean_object* x_508; uint8_t x_509; lean_object* x_510; uint8_t x_511; lean_object* x_512; +x_506 = lean_ctor_get(x_459, 1); +lean_inc(x_506); +x_507 = lean_ctor_get(x_459, 2); +lean_inc(x_507); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_508 = x_459; +} else { + lean_dec_ref(x_459); + x_508 = lean_box(0); } +x_509 = 0; +if (lean_is_scalar(x_508)) { + x_510 = lean_alloc_ctor(1, 4, 1); +} else { + x_510 = x_508; } +lean_ctor_set(x_510, 0, x_460); +lean_ctor_set(x_510, 1, x_506); +lean_ctor_set(x_510, 2, x_507); +lean_ctor_set(x_510, 3, x_505); +lean_ctor_set_uint8(x_510, sizeof(void*)*4, x_509); +x_511 = 1; +x_512 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_512, 0, x_362); +lean_ctor_set(x_512, 1, x_363); +lean_ctor_set(x_512, 2, x_364); +lean_ctor_set(x_512, 3, x_510); +lean_ctor_set_uint8(x_512, sizeof(void*)*4, x_511); +return x_512; } else { -lean_object* x_96; -lean_dec(x_63); -lean_dec(x_62); -lean_dec(x_15); -x_96 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_96, 0, x_60); -lean_ctor_set(x_96, 1, x_61); -lean_ctor_set(x_19, 1, x_96); -x_3 = x_16; -x_4 = x_19; -x_11 = x_21; -goto _start; +uint8_t x_513; +x_513 = lean_ctor_get_uint8(x_505, sizeof(void*)*4); +if (x_513 == 0) +{ +lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; uint8_t x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; uint8_t x_526; lean_object* x_527; +x_514 = lean_ctor_get(x_459, 1); +lean_inc(x_514); +x_515 = lean_ctor_get(x_459, 2); +lean_inc(x_515); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_516 = x_459; +} else { + lean_dec_ref(x_459); + x_516 = lean_box(0); +} +x_517 = lean_ctor_get(x_505, 0); +lean_inc(x_517); +x_518 = lean_ctor_get(x_505, 1); +lean_inc(x_518); +x_519 = lean_ctor_get(x_505, 2); +lean_inc(x_519); +x_520 = lean_ctor_get(x_505, 3); +lean_inc(x_520); +if (lean_is_exclusive(x_505)) { + lean_ctor_release(x_505, 0); + lean_ctor_release(x_505, 1); + lean_ctor_release(x_505, 2); + lean_ctor_release(x_505, 3); + x_521 = x_505; +} else { + lean_dec_ref(x_505); + x_521 = lean_box(0); } +x_522 = 1; +lean_inc(x_460); +if (lean_is_scalar(x_521)) { + x_523 = lean_alloc_ctor(1, 4, 1); +} else { + x_523 = x_521; } +lean_ctor_set(x_523, 0, x_362); +lean_ctor_set(x_523, 1, x_363); +lean_ctor_set(x_523, 2, x_364); +lean_ctor_set(x_523, 3, x_460); +if (lean_is_exclusive(x_460)) { + lean_ctor_release(x_460, 0); + lean_ctor_release(x_460, 1); + lean_ctor_release(x_460, 2); + lean_ctor_release(x_460, 3); + x_524 = x_460; +} else { + lean_dec_ref(x_460); + x_524 = lean_box(0); } -else -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_98 = lean_ctor_get(x_19, 0); -lean_inc(x_98); -lean_dec(x_19); -x_99 = lean_ctor_get(x_20, 0); -lean_inc(x_99); -x_100 = lean_ctor_get(x_20, 1); -lean_inc(x_100); -if (lean_is_exclusive(x_20)) { - lean_ctor_release(x_20, 0); - lean_ctor_release(x_20, 1); - x_101 = x_20; +lean_ctor_set_uint8(x_523, sizeof(void*)*4, x_522); +if (lean_is_scalar(x_524)) { + x_525 = lean_alloc_ctor(1, 4, 1); } else { - lean_dec_ref(x_20); - x_101 = lean_box(0); + x_525 = x_524; } -x_102 = lean_ctor_get(x_15, 0); -lean_inc(x_102); -x_103 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_98, x_102); -if (lean_obj_tag(x_103) == 0) -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; -lean_inc(x_102); -x_104 = l_Lean_Expr_mvar___override(x_102); -x_105 = lean_box(0); -x_106 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_98, x_102, x_105); -x_107 = l_Lean_Meta_getMVars(x_104, x_7, x_8, x_9, x_10, x_21); -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = lean_array_get_size(x_108); -x_111 = lean_unsigned_to_nat(0u); -x_112 = lean_nat_dec_lt(x_111, x_110); -if (x_112 == 0) -{ -lean_object* x_113; lean_object* x_114; -lean_dec(x_110); -lean_dec(x_108); -lean_dec(x_15); -if (lean_is_scalar(x_101)) { - x_113 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_525, 0, x_517); +lean_ctor_set(x_525, 1, x_518); +lean_ctor_set(x_525, 2, x_519); +lean_ctor_set(x_525, 3, x_520); +lean_ctor_set_uint8(x_525, sizeof(void*)*4, x_522); +x_526 = 0; +if (lean_is_scalar(x_516)) { + x_527 = lean_alloc_ctor(1, 4, 1); } else { - x_113 = x_101; + x_527 = x_516; } -lean_ctor_set(x_113, 0, x_99); -lean_ctor_set(x_113, 1, x_100); -x_114 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_114, 0, x_106); -lean_ctor_set(x_114, 1, x_113); -x_3 = x_16; -x_4 = x_114; -x_11 = x_109; -goto _start; +lean_ctor_set(x_527, 0, x_523); +lean_ctor_set(x_527, 1, x_514); +lean_ctor_set(x_527, 2, x_515); +lean_ctor_set(x_527, 3, x_525); +lean_ctor_set_uint8(x_527, sizeof(void*)*4, x_526); +return x_527; } else { -uint8_t x_116; -x_116 = lean_nat_dec_le(x_110, x_110); -if (x_116 == 0) -{ -lean_object* x_117; lean_object* x_118; -lean_dec(x_110); -lean_dec(x_108); -lean_dec(x_15); -if (lean_is_scalar(x_101)) { - x_117 = lean_alloc_ctor(0, 2, 0); +lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; uint8_t x_537; lean_object* x_538; uint8_t x_539; lean_object* x_540; +x_528 = lean_ctor_get(x_459, 1); +lean_inc(x_528); +x_529 = lean_ctor_get(x_459, 2); +lean_inc(x_529); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_530 = x_459; } else { - x_117 = x_101; + lean_dec_ref(x_459); + x_530 = lean_box(0); } -lean_ctor_set(x_117, 0, x_99); -lean_ctor_set(x_117, 1, x_100); -x_118 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_118, 0, x_106); -lean_ctor_set(x_118, 1, x_117); -x_3 = x_16; -x_4 = x_118; -x_11 = x_109; -goto _start; +x_531 = lean_ctor_get(x_460, 0); +lean_inc(x_531); +x_532 = lean_ctor_get(x_460, 1); +lean_inc(x_532); +x_533 = lean_ctor_get(x_460, 2); +lean_inc(x_533); +x_534 = lean_ctor_get(x_460, 3); +lean_inc(x_534); +if (lean_is_exclusive(x_460)) { + lean_ctor_release(x_460, 0); + lean_ctor_release(x_460, 1); + lean_ctor_release(x_460, 2); + lean_ctor_release(x_460, 3); + x_535 = x_460; +} else { + lean_dec_ref(x_460); + x_535 = lean_box(0); } -else -{ -size_t x_120; size_t x_121; uint8_t x_122; -x_120 = 0; -x_121 = lean_usize_of_nat(x_110); -lean_dec(x_110); -x_122 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_108, x_120, x_121); -lean_dec(x_108); -if (x_122 == 0) -{ -lean_object* x_123; lean_object* x_124; -lean_dec(x_15); -if (lean_is_scalar(x_101)) { - x_123 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_535)) { + x_536 = lean_alloc_ctor(1, 4, 1); } else { - x_123 = x_101; + x_536 = x_535; } -lean_ctor_set(x_123, 0, x_99); -lean_ctor_set(x_123, 1, x_100); -x_124 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_124, 0, x_106); -lean_ctor_set(x_124, 1, x_123); -x_3 = x_16; -x_4 = x_124; -x_11 = x_109; -goto _start; +lean_ctor_set(x_536, 0, x_531); +lean_ctor_set(x_536, 1, x_532); +lean_ctor_set(x_536, 2, x_533); +lean_ctor_set(x_536, 3, x_534); +lean_ctor_set_uint8(x_536, sizeof(void*)*4, x_513); +x_537 = 0; +if (lean_is_scalar(x_530)) { + x_538 = lean_alloc_ctor(1, 4, 1); +} else { + x_538 = x_530; } -else -{ -lean_dec(x_101); -if (x_2 == 0) -{ -lean_object* x_126; uint8_t x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; -x_126 = lean_array_push(x_99, x_15); -x_127 = lean_unbox(x_100); -lean_dec(x_100); -x_128 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_106, x_126, x_127, x_105, x_5, x_6, x_7, x_8, x_9, x_10, x_109); -x_129 = lean_ctor_get(x_128, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_128, 1); -lean_inc(x_130); -lean_dec(x_128); -x_131 = lean_ctor_get(x_129, 0); -lean_inc(x_131); -lean_dec(x_129); -x_3 = x_16; -x_4 = x_131; -x_11 = x_130; -goto _start; +lean_ctor_set(x_538, 0, x_536); +lean_ctor_set(x_538, 1, x_528); +lean_ctor_set(x_538, 2, x_529); +lean_ctor_set(x_538, 3, x_505); +lean_ctor_set_uint8(x_538, sizeof(void*)*4, x_537); +x_539 = 1; +x_540 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_540, 0, x_362); +lean_ctor_set(x_540, 1, x_363); +lean_ctor_set(x_540, 2, x_364); +lean_ctor_set(x_540, 3, x_538); +lean_ctor_set_uint8(x_540, sizeof(void*)*4, x_539); +return x_540; } -else -{ -uint8_t x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; -lean_dec(x_15); -x_133 = lean_unbox(x_100); -lean_dec(x_100); -x_134 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_106, x_99, x_133, x_105, x_5, x_6, x_7, x_8, x_9, x_10, x_109); -x_135 = lean_ctor_get(x_134, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_134, 1); -lean_inc(x_136); -lean_dec(x_134); -x_137 = lean_ctor_get(x_135, 0); -lean_inc(x_137); -lean_dec(x_135); -x_3 = x_16; -x_4 = x_137; -x_11 = x_136; -goto _start; } } } } } -else -{ -lean_object* x_139; lean_object* x_140; -lean_dec(x_103); -lean_dec(x_102); -lean_dec(x_15); -if (lean_is_scalar(x_101)) { - x_139 = lean_alloc_ctor(0, 2, 0); -} else { - x_139 = x_101; } -lean_ctor_set(x_139, 0, x_99); -lean_ctor_set(x_139, 1, x_100); -x_140 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_140, 0, x_98); -lean_ctor_set(x_140, 1, x_139); -x_3 = x_16; -x_4 = x_140; -x_11 = x_21; -goto _start; } } } } } -static lean_object* _init_l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__1() { +LEAN_EXPORT lean_object* l_Std_RBNode_insert___at_Lean_Elab_Term_registerMVarErrorInfo___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Term_instInhabitedLetRecToLift___closed__1; -x_2 = 0; -x_3 = lean_box(x_2); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_3); -return x_4; -} +uint8_t x_4; +x_4 = l_Std_RBNode_isRed___rarg(x_1); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_1, x_2, x_3); +return x_5; } -static lean_object* _init_l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__1; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_6; lean_object* x_7; +x_6 = l_Std_RBNode_ins___at_Lean_Elab_Term_registerMVarErrorInfo___spec__2(x_1, x_2, x_3); +x_7 = l_Std_RBNode_setBlack___rarg(x_6); +return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_logUnassignedUsingErrorInfos(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -uint8_t x_10; -x_10 = l_Array_isEmpty___rarg(x_1); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; 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_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_11 = lean_st_ref_get(x_8, x_9); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_9 = lean_st_ref_get(x_7, x_8); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = lean_st_ref_take(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = lean_ctor_get(x_12, 5); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l_Std_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(x_14); -x_16 = lean_st_ref_get(x_8, x_13); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = lean_st_ref_get(x_4, x_17); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_19, 2); -lean_inc(x_21); -lean_dec(x_19); -x_41 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__2; -x_42 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(x_1, x_15, x_21, x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_20); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_ctor_get(x_43, 0); -lean_inc(x_45); -lean_dec(x_43); -x_22 = x_45; -x_23 = x_44; -goto block_40; -block_40: -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; size_t x_28; size_t x_29; lean_object* x_30; lean_object* x_31; -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_array_get_size(x_25); -x_28 = lean_usize_of_nat(x_27); -lean_dec(x_27); -x_29 = 0; -x_30 = lean_box(0); -x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__5(x_2, x_25, x_28, x_29, x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_23); -lean_dec(x_25); -if (lean_obj_tag(x_31) == 0) +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_15 = lean_ctor_get(x_12, 3); +x_16 = lean_ctor_get(x_1, 0); +lean_inc(x_16); +x_17 = l_Std_RBNode_insert___at_Lean_Elab_Term_registerMVarErrorInfo___spec__1(x_15, x_16, x_1); +lean_ctor_set(x_12, 3, x_17); +x_18 = lean_st_ref_set(x_3, x_12, x_13); +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -lean_object* x_33; -x_33 = lean_ctor_get(x_31, 0); -lean_dec(x_33); -lean_ctor_set(x_31, 0, x_26); -return x_31; +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_18, 0); +lean_dec(x_20); +x_21 = lean_box(0); +lean_ctor_set(x_18, 0, x_21); +return x_18; } else { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_31, 1); -lean_inc(x_34); -lean_dec(x_31); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_26); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_18, 1); +lean_inc(x_22); +lean_dec(x_18); +x_23 = lean_box(0); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; } } else { -uint8_t x_36; -lean_dec(x_26); -x_36 = !lean_is_exclusive(x_31); -if (x_36 == 0) -{ -return x_31; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_25 = lean_ctor_get(x_12, 0); +x_26 = lean_ctor_get(x_12, 1); +x_27 = lean_ctor_get(x_12, 2); +x_28 = lean_ctor_get(x_12, 3); +x_29 = lean_ctor_get(x_12, 4); +x_30 = lean_ctor_get(x_12, 5); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_12); +x_31 = lean_ctor_get(x_1, 0); +lean_inc(x_31); +x_32 = l_Std_RBNode_insert___at_Lean_Elab_Term_registerMVarErrorInfo___spec__1(x_28, x_31, x_1); +x_33 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_33, 0, x_25); +lean_ctor_set(x_33, 1, x_26); +lean_ctor_set(x_33, 2, x_27); +lean_ctor_set(x_33, 3, x_32); +lean_ctor_set(x_33, 4, x_29); +lean_ctor_set(x_33, 5, x_30); +x_34 = lean_st_ref_set(x_3, x_33, x_13); +x_35 = lean_ctor_get(x_34, 1); +lean_inc(x_35); +if (lean_is_exclusive(x_34)) { + lean_ctor_release(x_34, 0); + lean_ctor_release(x_34, 1); + x_36 = x_34; +} else { + lean_dec_ref(x_34); + x_36 = lean_box(0); } -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_31, 0); -x_38 = lean_ctor_get(x_31, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_31); -x_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; +x_37 = lean_box(0); +if (lean_is_scalar(x_36)) { + x_38 = lean_alloc_ctor(0, 2, 0); +} else { + x_38 = x_36; } +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_35); +return x_38; } } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorInfo___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -uint8_t x_46; lean_object* x_47; lean_object* x_48; -lean_dec(x_8); +lean_object* x_9; +x_9 = l_Lean_Elab_Term_registerMVarErrorInfo(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_46 = 0; -x_47 = lean_box(x_46); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_47); -lean_ctor_set(x_48, 1, x_9); -return x_48; +return x_9; +} } +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorHoleInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_box(0); +x_11 = lean_box(1); +x_12 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_2); +lean_ctor_set(x_12, 2, x_11); +lean_ctor_set(x_12, 3, x_10); +x_13 = l_Lean_Elab_Term_registerMVarErrorInfo(x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_13; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorHoleInfo___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); +lean_object* x_10; +x_10 = l_Lean_Elab_Term_registerMVarErrorHoleInfo(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(x_1, x_2, x_5, x_6); -lean_dec(x_2); -lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; +lean_dec(x_3); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorImplicitArgInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_3); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_13, 0, x_1); +lean_ctor_set(x_13, 1, x_2); +lean_ctor_set(x_13, 2, x_11); +lean_ctor_set(x_13, 3, x_12); +x_14 = l_Lean_Elab_Term_registerMVarErrorInfo(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_14; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorImplicitArgInfo___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); +lean_object* x_11; +x_11 = l_Lean_Elab_Term_registerMVarErrorImplicitArgInfo(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_2, x_5, x_6); -lean_dec(x_2); -lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; +return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorCustomInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__5(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_2); -return x_15; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_11, 0, x_3); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_13, 0, x_1); +lean_ctor_set(x_13, 1, x_2); +lean_ctor_set(x_13, 2, x_11); +lean_ctor_set(x_13, 3, x_12); +x_14 = l_Lean_Elab_Term_registerMVarErrorInfo(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_14; } } -LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerMVarErrorCustomInfo___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_12; lean_object* x_13; -x_12 = lean_unbox(x_3); -lean_dec(x_3); -x_13 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); +lean_object* x_11; +x_11 = l_Lean_Elab_Term_registerMVarErrorCustomInfo(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_13; +return x_11; } } -LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1(lean_object* x_1, lean_object* x_2) { _start: { -uint8_t x_13; lean_object* x_14; -x_13 = lean_unbox(x_2); -lean_dec(x_2); -x_14 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6(x_1, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_10); +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_4 = lean_ctor_get(x_1, 0); +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_1, 2); +x_7 = lean_ctor_get(x_1, 3); +x_8 = l_Lean_Name_quickCmp(x_2, x_5); +switch (x_8) { +case 0: +{ +x_1 = x_4; +goto _start; +} +case 1: +{ +lean_object* x_10; +lean_inc(x_6); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_6); +return x_10; +} +default: +{ +x_1 = x_7; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_getMVarErrorInfo_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_9 = lean_st_ref_get(x_7, x_8); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); lean_dec(x_9); -lean_dec(x_8); +x_11 = lean_st_ref_get(x_3, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_13, 3); +lean_inc(x_14); +lean_dec(x_13); +x_15 = l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1(x_14, x_1); +lean_dec(x_14); +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_11, 0); +x_17 = lean_ctor_get(x_11, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_11); +x_18 = lean_ctor_get(x_16, 3); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1(x_18, x_1); +lean_dec(x_18); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_17); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_RBNode_find___at_Lean_Elab_Term_getMVarErrorInfo_x3f___spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_getMVarErrorInfo_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Term_getMVarErrorInfo_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -return x_14; +return x_9; } } -LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerCustomErrorIfMVar(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_12; lean_object* x_13; -x_12 = lean_unbox(x_2); +lean_object* x_11; +x_11 = l_Lean_Expr_getAppFn(x_1); +if (lean_obj_tag(x_11) == 2) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Elab_Term_registerMVarErrorCustomInfo(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_11); +lean_dec(x_3); lean_dec(x_2); -x_13 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(x_1, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_10); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_registerCustomErrorIfMVar___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_Term_registerCustomErrorIfMVar(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_1); -return x_13; +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_logUnassignedUsingErrorInfos___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_10; -x_10 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_1); -return x_10; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_9 = lean_ctor_get(x_6, 5); +x_10 = lean_ctor_get(x_2, 2); +lean_inc(x_10); +lean_inc(x_10); +x_11 = l_Lean_Elab_getBetterRef(x_9, x_10); +x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_4, x_5, x_6, x_7, x_8); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_13, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_14); +lean_dec(x_2); +lean_dec(x_10); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_11); +lean_ctor_set(x_18, 1, x_17); +lean_ctor_set_tag(x_15, 1); +lean_ctor_set(x_15, 0, x_18); +return x_15; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_15, 0); +x_20 = lean_ctor_get(x_15, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_15); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_11); +lean_ctor_set(x_21, 1, x_19); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; } } -static lean_object* _init_l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg___closed__1() { +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg___boxed), 8, 0); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__1() { _start: { lean_object* x_1; -x_1 = l_Lean_Elab_abortCommandExceptionId; +x_1 = l_Lean_Elab_abortTermExceptionId; return x_1; } } -static lean_object* _init_l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg___closed__2() { +static lean_object* _init_l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg___closed__1; +x_2 = l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__1; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg___closed__2; +x_2 = l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_7; -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg), 1, 0); -return x_7; +lean_object* x_8; +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg), 1, 0); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_ensureNoUnassignedMVars(lean_object* x_1, lean_object* x_2, lean_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_Term_throwMVarError___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_9 = l_Lean_Meta_getMVarsAtDecl(x_1, x_4, x_5, x_6, x_7, x_8); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_9 = lean_st_ref_get(x_7, x_8); x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); -x_12 = lean_box(0); -x_13 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos(x_10, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_11); +x_12 = lean_ctor_get(x_10, 5); +lean_inc(x_12); lean_dec(x_10); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; uint8_t x_15; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_unbox(x_14); -lean_dec(x_14); -if (x_15 == 0) -{ -uint8_t x_16; -x_16 = !lean_is_exclusive(x_13); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_13, 0); -lean_dec(x_17); -x_18 = lean_box(0); -lean_ctor_set(x_13, 0, x_18); -return x_13; -} -else +x_13 = l_Std_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(x_12); +if (x_13 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_13, 1); -lean_inc(x_19); -lean_dec(x_13); -x_20 = lean_box(0); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -return x_21; -} +lean_object* x_14; +x_14 = l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11); +return x_14; } else { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_13, 1); -lean_inc(x_22); -lean_dec(x_13); -x_23 = l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg(x_22); -return x_23; +lean_object* x_15; +lean_dec(x_2); +lean_dec(x_1); +x_15 = l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___rarg(x_11); +return x_15; } } -else -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_13); -if (x_24 == 0) -{ -return x_13; } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError(lean_object* x_1) { +_start: { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_13, 0); -x_26 = lean_ctor_get(x_13, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_13); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} -} +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_throwMVarError___rarg___boxed), 8, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_7; -x_7 = l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_object* x_9; +x_9 = l_Lean_throwError___at_Lean_Elab_Term_throwMVarError___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_7; +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutPostponing___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_2); -if (x_9 == 0) -{ -uint8_t x_10; lean_object* x_11; -x_10 = 0; -lean_ctor_set_uint8(x_2, sizeof(void*)*8, x_10); -x_11 = lean_apply_7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; uint8_t x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; uint8_t x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; -x_12 = lean_ctor_get(x_2, 0); -x_13 = lean_ctor_get(x_2, 1); -x_14 = lean_ctor_get(x_2, 2); -x_15 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 1); -x_16 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 2); -x_17 = lean_ctor_get(x_2, 3); -x_18 = lean_ctor_get(x_2, 4); -x_19 = lean_ctor_get(x_2, 5); -x_20 = lean_ctor_get(x_2, 6); -x_21 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 3); -x_22 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 4); -x_23 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 5); -x_24 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 6); -x_25 = lean_ctor_get(x_2, 7); -x_26 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 7); -lean_inc(x_25); -lean_inc(x_20); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); +lean_object* x_8; +x_8 = l_Lean_Elab_throwAbortTerm___at_Lean_Elab_Term_throwMVarError___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -x_27 = 0; -x_28 = lean_alloc_ctor(0, 8, 8); -lean_ctor_set(x_28, 0, x_12); -lean_ctor_set(x_28, 1, x_13); -lean_ctor_set(x_28, 2, x_14); -lean_ctor_set(x_28, 3, x_17); -lean_ctor_set(x_28, 4, x_18); -lean_ctor_set(x_28, 5, x_19); -lean_ctor_set(x_28, 6, x_20); -lean_ctor_set(x_28, 7, x_25); -lean_ctor_set_uint8(x_28, sizeof(void*)*8, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 1, x_15); -lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 2, x_16); -lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 3, x_21); -lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 4, x_22); -lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 5, x_23); -lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 6, x_24); -lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 7, x_26); -x_29 = lean_apply_7(x_1, x_28, x_3, x_4, x_5, x_6, x_7, x_8); -return x_29; -} +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutPostponing(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwMVarError___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutPostponing___rarg), 8, 0); -return x_2; +lean_object* x_9; +x_9 = l_Lean_Elab_Term_throwMVarError___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__1() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("explicitBinder", 14); +x_1 = lean_mk_string_from_bytes(" '", 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__2() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__15; -x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__3() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("(", 1); +x_1 = lean_mk_string_from_bytes("'", 1); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__4() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(2); -x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__3; -x_3 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__5() { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1u); -x_2 = lean_mk_empty_array_with_capacity(x_1); +lean_object* x_4; +x_4 = lean_ctor_get(x_1, 3); +if (lean_obj_tag(x_4) == 0) +{ +lean_dec(x_3); return x_2; } +else +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_ctor_get(x_4, 0); +x_6 = l_Lean_Name_hasMacroScopes(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_7 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_9, 0, x_2); +lean_ctor_set(x_9, 1, x_8); +lean_inc(x_5); +x_10 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_10, 0, x_5); +x_11 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__2; +x_12 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +x_13 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__4; +x_14 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_15, 0, x_9); +lean_ctor_set(x_15, 1, x_14); +return x_15; } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__6() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("null", 4); -return x_1; +lean_dec(x_3); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__7() { +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__6; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_4; +x_4 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__8() { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(":", 1); -return x_1; +if (lean_obj_tag(x_1) == 0) +{ +return x_2; +} +else +{ +lean_object* x_3; lean_object* x_4; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__9() { +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(2); -x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__8; -x_3 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); +lean_object* x_3; +x_3 = l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(x_1, x_2); +lean_dec(x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__10() { +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(2u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; +uint8_t x_9; +x_9 = l_Lean_Expr_hasMVar(x_1); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_8); +return x_10; } +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_11 = lean_st_ref_get(x_7, x_8); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_st_ref_get(x_5, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_instantiateMVarsCore(x_16, x_1); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_st_ref_get(x_7, x_15); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_st_ref_take(x_5, x_21); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = !lean_is_exclusive(x_23); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = lean_ctor_get(x_23, 0); +lean_dec(x_26); +lean_ctor_set(x_23, 0, x_19); +x_27 = lean_st_ref_set(x_5, x_23, x_24); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +lean_object* x_29; +x_29 = lean_ctor_get(x_27, 0); +lean_dec(x_29); +lean_ctor_set(x_27, 0, x_18); +return x_27; } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__11() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_mkExplicitBinder___closed__10; -x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__9; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_dec(x_27); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_18); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__12() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__7; -x_3 = l_Lean_Elab_Term_instInhabitedLetRecToLift___closed__1; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_32 = lean_ctor_get(x_23, 1); +x_33 = lean_ctor_get(x_23, 2); +x_34 = lean_ctor_get(x_23, 3); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_23); +x_35 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_35, 0, x_19); +lean_ctor_set(x_35, 1, x_32); +lean_ctor_set(x_35, 2, x_33); +lean_ctor_set(x_35, 3, x_34); +x_36 = lean_st_ref_set(x_5, x_35, x_24); +x_37 = lean_ctor_get(x_36, 1); +lean_inc(x_37); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + lean_ctor_release(x_36, 1); + x_38 = x_36; +} else { + lean_dec_ref(x_36); + x_38 = lean_box(0); +} +if (lean_is_scalar(x_38)) { + x_39 = lean_alloc_ctor(0, 2, 0); +} else { + x_39 = x_38; +} +lean_ctor_set(x_39, 0, x_18); +lean_ctor_set(x_39, 1, x_37); +return x_39; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__13() { +} +} +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes(")", 1); +x_1 = lean_mk_string_from_bytes("don't know how to synthesize implicit argument", 46); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__14() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(2); -x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__13; -x_3 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__1; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__15() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(5u); -x_2 = lean_mk_empty_array_with_capacity(x_1); +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__2; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__16() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_mkExplicitBinder___closed__15; -x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__4; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("context:", 8); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkExplicitBinder(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__5() { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_3 = l_Lean_Elab_Term_mkExplicitBinder___closed__5; -x_4 = lean_array_push(x_3, x_1); -x_5 = lean_box(2); -x_6 = l_Lean_Elab_Term_mkExplicitBinder___closed__7; -x_7 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_7, 0, x_5); -lean_ctor_set(x_7, 1, x_6); -lean_ctor_set(x_7, 2, x_4); -x_8 = l_Lean_Elab_Term_mkExplicitBinder___closed__11; -x_9 = lean_array_push(x_8, x_2); -x_10 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_10, 0, x_5); -lean_ctor_set(x_10, 1, x_6); -lean_ctor_set(x_10, 2, x_9); -x_11 = l_Lean_Elab_Term_mkExplicitBinder___closed__16; -x_12 = lean_array_push(x_11, x_7); -x_13 = lean_array_push(x_12, x_10); -x_14 = l_Lean_Elab_Term_mkExplicitBinder___closed__12; -x_15 = lean_array_push(x_13, x_14); -x_16 = l_Lean_Elab_Term_mkExplicitBinder___closed__14; -x_17 = lean_array_push(x_15, x_16); -x_18 = l_Lean_Elab_Term_mkExplicitBinder___closed__2; -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_5); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set(x_19, 2, x_17); -return x_19; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__4; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT uint8_t l_Lean_Elab_Term_levelMVarToParam___lambda__1(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__6() { _start: { -uint8_t x_3; -x_3 = l_List_elem___at_Lean_NameHashSet_insert___spec__2(x_2, x_1); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__5; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l_Lean_Elab_Term_levelMVarToParam___closed__1() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__7() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("u", 1); +x_1 = lean_mk_string_from_bytes("don't know how to synthesize placeholder", 40); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_levelMVarToParam___closed__2() { +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__8() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Term_levelMVarToParam___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__7; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__9() { +_start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_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_11 = l_Lean_Elab_Term_getLevelNames___rarg(x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__8; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(" for argument", 13); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("synthPlaceholder", 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_MVarErrorInfo_logError___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__11; +x_2 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__12; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = lean_ctor_get(x_1, 2); +lean_inc(x_10); +switch (lean_obj_tag(x_10)) { +case 0: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 1); lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); +x_13 = lean_ctor_get(x_10, 0); lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_st_ref_get(x_9, x_13); -x_15 = lean_ctor_get(x_14, 1); +lean_dec(x_10); +x_14 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); lean_dec(x_14); -x_16 = lean_st_ref_get(x_7, x_15); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 0); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_alloc_closure((void*)(l_Lean_Elab_Term_levelMVarToParam___lambda__1___boxed), 2, 1); -lean_closure_set(x_20, 0, x_12); -x_21 = l_Lean_Elab_Term_levelMVarToParam___closed__2; -x_22 = l_Lean_MetavarContext_levelMVarToParam(x_19, x_20, x_3, x_1, x_21, x_2); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_st_ref_get(x_9, x_18); -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = lean_st_ref_take(x_7, x_25); -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get_uint8(x_23, sizeof(void*)*8); -if (x_28 == 0) +x_17 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__3; +x_18 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; +x_19 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(x_1, x_17, x_18); +lean_dec(x_1); +x_20 = l_Lean_Expr_setAppPPExplicitForExposingMVars(x_15); +x_21 = l_Lean_indentExpr(x_20); +x_22 = l_Lean_logTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__1___closed__5; +x_23 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +x_24 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +x_25 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_25, 0, x_19); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1___closed__2; +x_27 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_28 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__6; +x_29 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +x_30 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_26); +x_31 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_31, 0, x_11); +x_32 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(x_2, x_32); +x_34 = 2; +x_35 = l_Lean_logAt___at_Lean_Elab_Term_traceAtCmdPos___spec__3(x_12, x_33, x_34, x_3, x_4, x_5, x_6, x_7, x_8, x_16); +lean_dec(x_12); +return x_35; +} +case 1: { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_29 = lean_ctor_get(x_27, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_26, 1); -lean_inc(x_30); -lean_dec(x_26); -x_31 = lean_ctor_get(x_23, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_23, 1); -lean_inc(x_32); -x_33 = lean_ctor_get(x_23, 2); -lean_inc(x_33); -x_34 = lean_ctor_get(x_23, 3); -lean_inc(x_34); -x_35 = lean_ctor_get(x_23, 4); -lean_inc(x_35); -x_36 = lean_ctor_get(x_23, 5); +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; uint8_t x_51; lean_object* x_52; +x_36 = lean_ctor_get(x_1, 0); lean_inc(x_36); -x_37 = lean_ctor_get(x_23, 6); +x_37 = lean_ctor_get(x_1, 1); lean_inc(x_37); -x_38 = lean_ctor_get(x_23, 7); -lean_inc(x_38); -lean_dec(x_23); -x_39 = !lean_is_exclusive(x_27); -if (x_39 == 0) +x_38 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__9; +x_39 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__10; +x_40 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName(x_1, x_38, x_39); +lean_dec(x_1); +x_41 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1___closed__2; +x_42 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__6; +x_44 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_41); +x_46 = lean_alloc_ctor(5, 1, 0); +lean_ctor_set(x_46, 0, x_36); +x_47 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(x_2, x_47); +x_49 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__13; +x_50 = lean_alloc_ctor(11, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_48); +x_51 = 2; +x_52 = l_Lean_logAt___at_Lean_Elab_Term_traceAtCmdPos___spec__3(x_37, x_50, x_51, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_37); +return x_52; +} +default: { -lean_object* x_40; uint8_t x_41; -x_40 = lean_ctor_get(x_27, 0); -lean_dec(x_40); -x_41 = !lean_is_exclusive(x_29); -if (x_41 == 0) +lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; +x_53 = lean_ctor_get(x_1, 1); +lean_inc(x_53); +lean_dec(x_1); +x_54 = lean_ctor_get(x_10, 0); +lean_inc(x_54); +lean_dec(x_10); +x_55 = l_Lean_Elab_Term_MVarErrorInfo_logError_appendExtra(x_2, x_54); +x_56 = 2; +x_57 = l_Lean_logAt___at_Lean_Elab_Term_traceAtCmdPos___spec__3(x_53, x_55, x_56, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_53); +return x_57; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; -x_42 = lean_ctor_get(x_29, 7); -lean_dec(x_42); -x_43 = lean_ctor_get(x_29, 6); -lean_dec(x_43); -x_44 = lean_ctor_get(x_29, 5); -lean_dec(x_44); -x_45 = lean_ctor_get(x_29, 4); -lean_dec(x_45); -x_46 = lean_ctor_get(x_29, 3); -lean_dec(x_46); -x_47 = lean_ctor_get(x_29, 2); -lean_dec(x_47); -x_48 = lean_ctor_get(x_29, 1); -lean_dec(x_48); -x_49 = lean_ctor_get(x_29, 0); -lean_dec(x_49); -lean_ctor_set(x_29, 7, x_38); -lean_ctor_set(x_29, 6, x_37); -lean_ctor_set(x_29, 5, x_36); -lean_ctor_set(x_29, 4, x_35); -lean_ctor_set(x_29, 3, x_34); -lean_ctor_set(x_29, 2, x_33); -lean_ctor_set(x_29, 1, x_32); -lean_ctor_set(x_29, 0, x_31); -x_50 = lean_st_ref_set(x_7, x_27, x_30); -x_51 = !lean_is_exclusive(x_50); -if (x_51 == 0) +lean_object* x_9; +x_9 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_MVarErrorInfo_logError___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Term_MVarErrorInfo_logError(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_uget(x_2, x_3); +x_7 = lean_name_eq(x_1, x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +size_t x_8; size_t x_9; +x_8 = 1; +x_9 = lean_usize_add(x_3, x_8); +x_3 = x_9; +goto _start; +} +else +{ +uint8_t x_11; +x_11 = 1; +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = 0; +return x_12; +} +} +} +LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_array_get_size(x_1); +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_lt(x_4, x_3); +if (x_5 == 0) +{ +uint8_t x_6; +lean_dec(x_3); +x_6 = 0; +return x_6; +} +else +{ +uint8_t x_7; +x_7 = lean_nat_dec_le(x_3, x_3); +if (x_7 == 0) +{ +uint8_t x_8; +lean_dec(x_3); +x_8 = 0; +return x_8; +} +else +{ +size_t x_9; size_t x_10; uint8_t x_11; +x_9 = 0; +x_10 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_11 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(x_2, x_1, x_9, x_10); +return x_11; +} +} +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_uget(x_2, x_3); +x_7 = l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1(x_1, x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +size_t x_8; size_t x_9; +x_8 = 1; +x_9 = lean_usize_add(x_3, x_8); +x_3 = x_9; +goto _start; +} +else +{ +uint8_t x_11; +x_11 = 1; +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = 0; +return x_12; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_apply_2(x_2, x_3, x_4); +x_11 = l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(x_1, x_10, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +return x_11; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +else +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_11); +if (x_16 == 0) +{ +return x_11; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_11, 0); +x_18 = lean_ctor_get(x_11, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_11); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withMVarContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___rarg), 9, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__5(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_4, x_3); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_5); +lean_ctor_set(x_14, 1, x_12); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_5); +x_15 = lean_array_uget(x_2, x_4); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Lean_Elab_Term_MVarErrorInfo_logError___boxed), 9, 2); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_1); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_18 = l_Lean_Meta_withMVarContext___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__4___rarg(x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = 1; +x_21 = lean_usize_add(x_4, x_20); +x_22 = lean_box(0); +x_4 = x_21; +x_5 = x_22; +x_12 = x_19; +goto _start; +} +else +{ +uint8_t x_24; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) +{ +return x_18; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_18, 0); +x_26 = lean_ctor_get(x_18, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_18); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___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) { +_start: +{ +uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_12 = 1; +x_13 = lean_box(x_12); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_2); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_1); +lean_ctor_set(x_15, 1, x_14); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_11); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6(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) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_5); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_15 = lean_ctor_get(x_4, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_4, 2); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 3); +lean_inc(x_17); +lean_dec(x_4); +x_18 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +x_22 = lean_ctor_get(x_18, 1); +lean_inc(x_22); +lean_dec(x_18); +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = lean_ctor_get(x_20, 0); +x_25 = lean_ctor_get(x_20, 1); +lean_dec(x_25); +x_26 = !lean_is_exclusive(x_21); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_21, 0); +x_28 = lean_ctor_get(x_21, 1); +x_29 = lean_ctor_get(x_16, 0); +lean_inc(x_29); +x_30 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_24, x_29); +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; lean_object* x_37; lean_object* x_38; uint8_t x_39; +lean_inc(x_29); +x_31 = l_Lean_Expr_mvar___override(x_29); +x_32 = lean_box(0); +x_33 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_24, x_29, x_32); +x_34 = l_Lean_Meta_getMVars(x_31, x_8, x_9, x_10, x_11, x_22); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = lean_array_get_size(x_35); +x_38 = lean_unsigned_to_nat(0u); +x_39 = lean_nat_dec_lt(x_38, x_37); +if (x_39 == 0) +{ +lean_dec(x_37); +lean_dec(x_35); +lean_dec(x_16); +lean_ctor_set(x_20, 0, x_33); +x_4 = x_17; +x_5 = x_20; +x_12 = x_36; +goto _start; +} +else +{ +uint8_t x_41; +x_41 = lean_nat_dec_le(x_37, x_37); +if (x_41 == 0) +{ +lean_dec(x_37); +lean_dec(x_35); +lean_dec(x_16); +lean_ctor_set(x_20, 0, x_33); +x_4 = x_17; +x_5 = x_20; +x_12 = x_36; +goto _start; +} +else +{ +size_t x_43; size_t x_44; uint8_t x_45; +x_43 = 0; +x_44 = lean_usize_of_nat(x_37); +lean_dec(x_37); +x_45 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_35, x_43, x_44); +lean_dec(x_35); +if (x_45 == 0) +{ +lean_dec(x_16); +lean_ctor_set(x_20, 0, x_33); +x_4 = x_17; +x_5 = x_20; +x_12 = x_36; +goto _start; +} +else +{ +lean_free_object(x_21); +lean_free_object(x_20); +if (x_2 == 0) +{ +lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_47 = lean_array_push(x_27, x_16); +x_48 = lean_unbox(x_28); +lean_dec(x_28); +x_49 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_33, x_47, x_48, x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_36); +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = lean_ctor_get(x_50, 0); +lean_inc(x_52); +lean_dec(x_50); +x_4 = x_17; +x_5 = x_52; +x_12 = x_51; +goto _start; +} +else +{ +uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_dec(x_16); +x_54 = lean_unbox(x_28); +lean_dec(x_28); +x_55 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_33, x_27, x_54, x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_36); +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +lean_dec(x_55); +x_58 = lean_ctor_get(x_56, 0); +lean_inc(x_58); +lean_dec(x_56); +x_4 = x_17; +x_5 = x_58; +x_12 = x_57; +goto _start; +} +} +} +} +} +else +{ +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_16); +x_4 = x_17; +x_5 = x_20; +x_12 = x_22; +goto _start; +} +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_61 = lean_ctor_get(x_21, 0); +x_62 = lean_ctor_get(x_21, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_21); +x_63 = lean_ctor_get(x_16, 0); +lean_inc(x_63); +x_64 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_24, x_63); +if (lean_obj_tag(x_64) == 0) +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; +lean_inc(x_63); +x_65 = l_Lean_Expr_mvar___override(x_63); +x_66 = lean_box(0); +x_67 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_24, x_63, x_66); +x_68 = l_Lean_Meta_getMVars(x_65, x_8, x_9, x_10, x_11, x_22); +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = lean_array_get_size(x_69); +x_72 = lean_unsigned_to_nat(0u); +x_73 = lean_nat_dec_lt(x_72, x_71); +if (x_73 == 0) +{ +lean_object* x_74; +lean_dec(x_71); +lean_dec(x_69); +lean_dec(x_16); +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_61); +lean_ctor_set(x_74, 1, x_62); +lean_ctor_set(x_20, 1, x_74); +lean_ctor_set(x_20, 0, x_67); +x_4 = x_17; +x_5 = x_20; +x_12 = x_70; +goto _start; +} +else +{ +uint8_t x_76; +x_76 = lean_nat_dec_le(x_71, x_71); +if (x_76 == 0) +{ +lean_object* x_77; +lean_dec(x_71); +lean_dec(x_69); +lean_dec(x_16); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_61); +lean_ctor_set(x_77, 1, x_62); +lean_ctor_set(x_20, 1, x_77); +lean_ctor_set(x_20, 0, x_67); +x_4 = x_17; +x_5 = x_20; +x_12 = x_70; +goto _start; +} +else +{ +size_t x_79; size_t x_80; uint8_t x_81; +x_79 = 0; +x_80 = lean_usize_of_nat(x_71); +lean_dec(x_71); +x_81 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_69, x_79, x_80); +lean_dec(x_69); +if (x_81 == 0) +{ +lean_object* x_82; +lean_dec(x_16); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_61); +lean_ctor_set(x_82, 1, x_62); +lean_ctor_set(x_20, 1, x_82); +lean_ctor_set(x_20, 0, x_67); +x_4 = x_17; +x_5 = x_20; +x_12 = x_70; +goto _start; +} +else +{ +lean_free_object(x_20); +if (x_2 == 0) +{ +lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_84 = lean_array_push(x_61, x_16); +x_85 = lean_unbox(x_62); +lean_dec(x_62); +x_86 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_67, x_84, x_85, x_66, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +x_89 = lean_ctor_get(x_87, 0); +lean_inc(x_89); +lean_dec(x_87); +x_4 = x_17; +x_5 = x_89; +x_12 = x_88; +goto _start; +} +else +{ +uint8_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +lean_dec(x_16); +x_91 = lean_unbox(x_62); +lean_dec(x_62); +x_92 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_67, x_61, x_91, x_66, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +lean_dec(x_92); +x_95 = lean_ctor_get(x_93, 0); +lean_inc(x_95); +lean_dec(x_93); +x_4 = x_17; +x_5 = x_95; +x_12 = x_94; +goto _start; +} +} +} +} +} +else +{ +lean_object* x_97; +lean_dec(x_64); +lean_dec(x_63); +lean_dec(x_16); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_61); +lean_ctor_set(x_97, 1, x_62); +lean_ctor_set(x_20, 1, x_97); +x_4 = x_17; +x_5 = x_20; +x_12 = x_22; +goto _start; +} +} +} +else +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; +x_99 = lean_ctor_get(x_20, 0); +lean_inc(x_99); +lean_dec(x_20); +x_100 = lean_ctor_get(x_21, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_21, 1); +lean_inc(x_101); +if (lean_is_exclusive(x_21)) { + lean_ctor_release(x_21, 0); + lean_ctor_release(x_21, 1); + x_102 = x_21; +} else { + lean_dec_ref(x_21); + x_102 = lean_box(0); +} +x_103 = lean_ctor_get(x_16, 0); +lean_inc(x_103); +x_104 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_99, x_103); +if (lean_obj_tag(x_104) == 0) +{ +lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; +lean_inc(x_103); +x_105 = l_Lean_Expr_mvar___override(x_103); +x_106 = lean_box(0); +x_107 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_99, x_103, x_106); +x_108 = l_Lean_Meta_getMVars(x_105, x_8, x_9, x_10, x_11, x_22); +x_109 = lean_ctor_get(x_108, 0); +lean_inc(x_109); +x_110 = lean_ctor_get(x_108, 1); +lean_inc(x_110); +lean_dec(x_108); +x_111 = lean_array_get_size(x_109); +x_112 = lean_unsigned_to_nat(0u); +x_113 = lean_nat_dec_lt(x_112, x_111); +if (x_113 == 0) +{ +lean_object* x_114; lean_object* x_115; +lean_dec(x_111); +lean_dec(x_109); +lean_dec(x_16); +if (lean_is_scalar(x_102)) { + x_114 = lean_alloc_ctor(0, 2, 0); +} else { + x_114 = x_102; +} +lean_ctor_set(x_114, 0, x_100); +lean_ctor_set(x_114, 1, x_101); +x_115 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_115, 0, x_107); +lean_ctor_set(x_115, 1, x_114); +x_4 = x_17; +x_5 = x_115; +x_12 = x_110; +goto _start; +} +else +{ +uint8_t x_117; +x_117 = lean_nat_dec_le(x_111, x_111); +if (x_117 == 0) +{ +lean_object* x_118; lean_object* x_119; +lean_dec(x_111); +lean_dec(x_109); +lean_dec(x_16); +if (lean_is_scalar(x_102)) { + x_118 = lean_alloc_ctor(0, 2, 0); +} else { + x_118 = x_102; +} +lean_ctor_set(x_118, 0, x_100); +lean_ctor_set(x_118, 1, x_101); +x_119 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_119, 0, x_107); +lean_ctor_set(x_119, 1, x_118); +x_4 = x_17; +x_5 = x_119; +x_12 = x_110; +goto _start; +} +else +{ +size_t x_121; size_t x_122; uint8_t x_123; +x_121 = 0; +x_122 = lean_usize_of_nat(x_111); +lean_dec(x_111); +x_123 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_109, x_121, x_122); +lean_dec(x_109); +if (x_123 == 0) +{ +lean_object* x_124; lean_object* x_125; +lean_dec(x_16); +if (lean_is_scalar(x_102)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_102; +} +lean_ctor_set(x_124, 0, x_100); +lean_ctor_set(x_124, 1, x_101); +x_125 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_125, 0, x_107); +lean_ctor_set(x_125, 1, x_124); +x_4 = x_17; +x_5 = x_125; +x_12 = x_110; +goto _start; +} +else +{ +lean_dec(x_102); +if (x_2 == 0) +{ +lean_object* x_127; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_127 = lean_array_push(x_100, x_16); +x_128 = lean_unbox(x_101); +lean_dec(x_101); +x_129 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_107, x_127, x_128, x_106, x_6, x_7, x_8, x_9, x_10, x_11, x_110); +x_130 = lean_ctor_get(x_129, 0); +lean_inc(x_130); +x_131 = lean_ctor_get(x_129, 1); +lean_inc(x_131); +lean_dec(x_129); +x_132 = lean_ctor_get(x_130, 0); +lean_inc(x_132); +lean_dec(x_130); +x_4 = x_17; +x_5 = x_132; +x_12 = x_131; +goto _start; +} +else +{ +uint8_t x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; +lean_dec(x_16); +x_134 = lean_unbox(x_101); +lean_dec(x_101); +x_135 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_107, x_100, x_134, x_106, x_6, x_7, x_8, x_9, x_10, x_11, x_110); +x_136 = lean_ctor_get(x_135, 0); +lean_inc(x_136); +x_137 = lean_ctor_get(x_135, 1); +lean_inc(x_137); +lean_dec(x_135); +x_138 = lean_ctor_get(x_136, 0); +lean_inc(x_138); +lean_dec(x_136); +x_4 = x_17; +x_5 = x_138; +x_12 = x_137; +goto _start; +} +} +} +} +} +else +{ +lean_object* x_140; lean_object* x_141; +lean_dec(x_104); +lean_dec(x_103); +lean_dec(x_16); +if (lean_is_scalar(x_102)) { + x_140 = lean_alloc_ctor(0, 2, 0); +} else { + x_140 = x_102; +} +lean_ctor_set(x_140, 0, x_100); +lean_ctor_set(x_140, 1, x_101); +x_141 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_141, 0, x_99); +lean_ctor_set(x_141, 1, x_140); +x_4 = x_17; +x_5 = x_141; +x_12 = x_22; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(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) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_12, 0, x_4); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_14 = lean_ctor_get(x_3, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_3, 2); +lean_inc(x_15); +x_16 = lean_ctor_get(x_3, 3); +lean_inc(x_16); +lean_dec(x_3); +x_17 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(x_1, x_2, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = !lean_is_exclusive(x_19); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_23 = lean_ctor_get(x_19, 0); +x_24 = lean_ctor_get(x_19, 1); +lean_dec(x_24); +x_25 = !lean_is_exclusive(x_20); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_26 = lean_ctor_get(x_20, 0); +x_27 = lean_ctor_get(x_20, 1); +x_28 = lean_ctor_get(x_15, 0); +lean_inc(x_28); +x_29 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_23, x_28); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +lean_inc(x_28); +x_30 = l_Lean_Expr_mvar___override(x_28); +x_31 = lean_box(0); +x_32 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_23, x_28, x_31); +x_33 = l_Lean_Meta_getMVars(x_30, x_7, x_8, x_9, x_10, x_21); +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_array_get_size(x_34); +x_37 = lean_unsigned_to_nat(0u); +x_38 = lean_nat_dec_lt(x_37, x_36); +if (x_38 == 0) +{ +lean_dec(x_36); +lean_dec(x_34); +lean_dec(x_15); +lean_ctor_set(x_19, 0, x_32); +x_3 = x_16; +x_4 = x_19; +x_11 = x_35; +goto _start; +} +else +{ +uint8_t x_40; +x_40 = lean_nat_dec_le(x_36, x_36); +if (x_40 == 0) +{ +lean_dec(x_36); +lean_dec(x_34); +lean_dec(x_15); +lean_ctor_set(x_19, 0, x_32); +x_3 = x_16; +x_4 = x_19; +x_11 = x_35; +goto _start; +} +else +{ +size_t x_42; size_t x_43; uint8_t x_44; +x_42 = 0; +x_43 = lean_usize_of_nat(x_36); +lean_dec(x_36); +x_44 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_34, x_42, x_43); +lean_dec(x_34); +if (x_44 == 0) +{ +lean_dec(x_15); +lean_ctor_set(x_19, 0, x_32); +x_3 = x_16; +x_4 = x_19; +x_11 = x_35; +goto _start; +} +else +{ +lean_free_object(x_20); +lean_free_object(x_19); +if (x_2 == 0) +{ +lean_object* x_46; uint8_t x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_46 = lean_array_push(x_26, x_15); +x_47 = lean_unbox(x_27); +lean_dec(x_27); +x_48 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_32, x_46, x_47, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_35); +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_ctor_get(x_49, 0); +lean_inc(x_51); +lean_dec(x_49); +x_3 = x_16; +x_4 = x_51; +x_11 = x_50; +goto _start; +} +else +{ +uint8_t x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +lean_dec(x_15); +x_53 = lean_unbox(x_27); +lean_dec(x_27); +x_54 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_32, x_26, x_53, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_35); +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +lean_dec(x_54); +x_57 = lean_ctor_get(x_55, 0); +lean_inc(x_57); +lean_dec(x_55); +x_3 = x_16; +x_4 = x_57; +x_11 = x_56; +goto _start; +} +} +} +} +} +else +{ +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_15); +x_3 = x_16; +x_4 = x_19; +x_11 = x_21; +goto _start; +} +} +else +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_60 = lean_ctor_get(x_20, 0); +x_61 = lean_ctor_get(x_20, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_20); +x_62 = lean_ctor_get(x_15, 0); +lean_inc(x_62); +x_63 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_23, x_62); +if (lean_obj_tag(x_63) == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +lean_inc(x_62); +x_64 = l_Lean_Expr_mvar___override(x_62); +x_65 = lean_box(0); +x_66 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_23, x_62, x_65); +x_67 = l_Lean_Meta_getMVars(x_64, x_7, x_8, x_9, x_10, x_21); +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); +x_70 = lean_array_get_size(x_68); +x_71 = lean_unsigned_to_nat(0u); +x_72 = lean_nat_dec_lt(x_71, x_70); +if (x_72 == 0) +{ +lean_object* x_73; +lean_dec(x_70); +lean_dec(x_68); +lean_dec(x_15); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_60); +lean_ctor_set(x_73, 1, x_61); +lean_ctor_set(x_19, 1, x_73); +lean_ctor_set(x_19, 0, x_66); +x_3 = x_16; +x_4 = x_19; +x_11 = x_69; +goto _start; +} +else +{ +uint8_t x_75; +x_75 = lean_nat_dec_le(x_70, x_70); +if (x_75 == 0) +{ +lean_object* x_76; +lean_dec(x_70); +lean_dec(x_68); +lean_dec(x_15); +x_76 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_76, 0, x_60); +lean_ctor_set(x_76, 1, x_61); +lean_ctor_set(x_19, 1, x_76); +lean_ctor_set(x_19, 0, x_66); +x_3 = x_16; +x_4 = x_19; +x_11 = x_69; +goto _start; +} +else +{ +size_t x_78; size_t x_79; uint8_t x_80; +x_78 = 0; +x_79 = lean_usize_of_nat(x_70); +lean_dec(x_70); +x_80 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_68, x_78, x_79); +lean_dec(x_68); +if (x_80 == 0) +{ +lean_object* x_81; +lean_dec(x_15); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_60); +lean_ctor_set(x_81, 1, x_61); +lean_ctor_set(x_19, 1, x_81); +lean_ctor_set(x_19, 0, x_66); +x_3 = x_16; +x_4 = x_19; +x_11 = x_69; +goto _start; +} +else +{ +lean_free_object(x_19); +if (x_2 == 0) +{ +lean_object* x_83; uint8_t x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_83 = lean_array_push(x_60, x_15); +x_84 = lean_unbox(x_61); +lean_dec(x_61); +x_85 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_66, x_83, x_84, x_65, x_5, x_6, x_7, x_8, x_9, x_10, x_69); +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_85, 1); +lean_inc(x_87); +lean_dec(x_85); +x_88 = lean_ctor_get(x_86, 0); +lean_inc(x_88); +lean_dec(x_86); +x_3 = x_16; +x_4 = x_88; +x_11 = x_87; +goto _start; +} +else +{ +uint8_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +lean_dec(x_15); +x_90 = lean_unbox(x_61); +lean_dec(x_61); +x_91 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_66, x_60, x_90, x_65, x_5, x_6, x_7, x_8, x_9, x_10, x_69); +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_91, 1); +lean_inc(x_93); +lean_dec(x_91); +x_94 = lean_ctor_get(x_92, 0); +lean_inc(x_94); +lean_dec(x_92); +x_3 = x_16; +x_4 = x_94; +x_11 = x_93; +goto _start; +} +} +} +} +} +else +{ +lean_object* x_96; +lean_dec(x_63); +lean_dec(x_62); +lean_dec(x_15); +x_96 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_60); +lean_ctor_set(x_96, 1, x_61); +lean_ctor_set(x_19, 1, x_96); +x_3 = x_16; +x_4 = x_19; +x_11 = x_21; +goto _start; +} +} +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_98 = lean_ctor_get(x_19, 0); +lean_inc(x_98); +lean_dec(x_19); +x_99 = lean_ctor_get(x_20, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_20, 1); +lean_inc(x_100); +if (lean_is_exclusive(x_20)) { + lean_ctor_release(x_20, 0); + lean_ctor_release(x_20, 1); + x_101 = x_20; +} else { + lean_dec_ref(x_20); + x_101 = lean_box(0); +} +x_102 = lean_ctor_get(x_15, 0); +lean_inc(x_102); +x_103 = l_Std_RBNode_findCore___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__5(x_98, x_102); +if (lean_obj_tag(x_103) == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; +lean_inc(x_102); +x_104 = l_Lean_Expr_mvar___override(x_102); +x_105 = lean_box(0); +x_106 = l_Std_RBNode_insert___at_Lean_Level_collectMVars___spec__1(x_98, x_102, x_105); +x_107 = l_Lean_Meta_getMVars(x_104, x_7, x_8, x_9, x_10, x_21); +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +x_110 = lean_array_get_size(x_108); +x_111 = lean_unsigned_to_nat(0u); +x_112 = lean_nat_dec_lt(x_111, x_110); +if (x_112 == 0) +{ +lean_object* x_113; lean_object* x_114; +lean_dec(x_110); +lean_dec(x_108); +lean_dec(x_15); +if (lean_is_scalar(x_101)) { + x_113 = lean_alloc_ctor(0, 2, 0); +} else { + x_113 = x_101; +} +lean_ctor_set(x_113, 0, x_99); +lean_ctor_set(x_113, 1, x_100); +x_114 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_114, 0, x_106); +lean_ctor_set(x_114, 1, x_113); +x_3 = x_16; +x_4 = x_114; +x_11 = x_109; +goto _start; +} +else +{ +uint8_t x_116; +x_116 = lean_nat_dec_le(x_110, x_110); +if (x_116 == 0) +{ +lean_object* x_117; lean_object* x_118; +lean_dec(x_110); +lean_dec(x_108); +lean_dec(x_15); +if (lean_is_scalar(x_101)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_101; +} +lean_ctor_set(x_117, 0, x_99); +lean_ctor_set(x_117, 1, x_100); +x_118 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_118, 0, x_106); +lean_ctor_set(x_118, 1, x_117); +x_3 = x_16; +x_4 = x_118; +x_11 = x_109; +goto _start; +} +else +{ +size_t x_120; size_t x_121; uint8_t x_122; +x_120 = 0; +x_121 = lean_usize_of_nat(x_110); +lean_dec(x_110); +x_122 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_108, x_120, x_121); +lean_dec(x_108); +if (x_122 == 0) +{ +lean_object* x_123; lean_object* x_124; +lean_dec(x_15); +if (lean_is_scalar(x_101)) { + x_123 = lean_alloc_ctor(0, 2, 0); +} else { + x_123 = x_101; +} +lean_ctor_set(x_123, 0, x_99); +lean_ctor_set(x_123, 1, x_100); +x_124 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_124, 0, x_106); +lean_ctor_set(x_124, 1, x_123); +x_3 = x_16; +x_4 = x_124; +x_11 = x_109; +goto _start; +} +else +{ +lean_dec(x_101); +if (x_2 == 0) +{ +lean_object* x_126; uint8_t x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_126 = lean_array_push(x_99, x_15); +x_127 = lean_unbox(x_100); +lean_dec(x_100); +x_128 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_106, x_126, x_127, x_105, x_5, x_6, x_7, x_8, x_9, x_10, x_109); +x_129 = lean_ctor_get(x_128, 0); +lean_inc(x_129); +x_130 = lean_ctor_get(x_128, 1); +lean_inc(x_130); +lean_dec(x_128); +x_131 = lean_ctor_get(x_129, 0); +lean_inc(x_131); +lean_dec(x_129); +x_3 = x_16; +x_4 = x_131; +x_11 = x_130; +goto _start; +} +else +{ +uint8_t x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; +lean_dec(x_15); +x_133 = lean_unbox(x_100); +lean_dec(x_100); +x_134 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_106, x_99, x_133, x_105, x_5, x_6, x_7, x_8, x_9, x_10, x_109); +x_135 = lean_ctor_get(x_134, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_134, 1); +lean_inc(x_136); +lean_dec(x_134); +x_137 = lean_ctor_get(x_135, 0); +lean_inc(x_137); +lean_dec(x_135); +x_3 = x_16; +x_4 = x_137; +x_11 = x_136; +goto _start; +} +} +} +} +} +else +{ +lean_object* x_139; lean_object* x_140; +lean_dec(x_103); +lean_dec(x_102); +lean_dec(x_15); +if (lean_is_scalar(x_101)) { + x_139 = lean_alloc_ctor(0, 2, 0); +} else { + x_139 = x_101; +} +lean_ctor_set(x_139, 0, x_99); +lean_ctor_set(x_139, 1, x_100); +x_140 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_140, 0, x_98); +lean_ctor_set(x_140, 1, x_139); +x_3 = x_16; +x_4 = x_140; +x_11 = x_21; +goto _start; +} +} +} +} +} +static lean_object* _init_l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Term_instInhabitedLetRecToLift___closed__1; +x_2 = 0; +x_3 = lean_box(x_2); +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__1; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_logUnassignedUsingErrorInfos(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; +x_10 = l_Array_isEmpty___rarg(x_1); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; 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_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_11 = lean_st_ref_get(x_8, x_9); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_ctor_get(x_12, 5); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Std_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(x_14); +x_16 = lean_st_ref_get(x_8, x_13); +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = lean_st_ref_get(x_4, x_17); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_ctor_get(x_19, 3); +lean_inc(x_21); +lean_dec(x_19); +x_41 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos___closed__2; +x_42 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(x_1, x_15, x_21, x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_20); +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = lean_ctor_get(x_43, 0); +lean_inc(x_45); +lean_dec(x_43); +x_22 = x_45; +x_23 = x_44; +goto block_40; +block_40: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; size_t x_28; size_t x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_array_get_size(x_25); +x_28 = lean_usize_of_nat(x_27); +lean_dec(x_27); +x_29 = 0; +x_30 = lean_box(0); +x_31 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__5(x_2, x_25, x_28, x_29, x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_23); +lean_dec(x_25); +if (lean_obj_tag(x_31) == 0) +{ +uint8_t x_32; +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) +{ +lean_object* x_33; +x_33 = lean_ctor_get(x_31, 0); +lean_dec(x_33); +lean_ctor_set(x_31, 0, x_26); +return x_31; +} +else +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_31, 1); +lean_inc(x_34); +lean_dec(x_31); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_26); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +} +else +{ +uint8_t x_36; +lean_dec(x_26); +x_36 = !lean_is_exclusive(x_31); +if (x_36 == 0) +{ +return x_31; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_31, 0); +x_38 = lean_ctor_get(x_31, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_31); +x_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_46; lean_object* x_47; lean_object* x_48; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_46 = 0; +x_47 = lean_box(x_46); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_9); +return x_48; +} +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_7 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__2(x_1, x_2, x_5, x_6); +lean_dec(x_2); +lean_dec(x_1); +x_8 = lean_box(x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Array_contains___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_7 = l_Array_anyMUnsafe_any___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__3(x_1, x_2, x_5, x_6); +lean_dec(x_2); +lean_dec(x_1); +x_8 = lean_box(x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__5(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_2); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_3); +lean_dec(x_3); +x_13 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___lambda__1(x_1, x_2, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +uint8_t x_13; lean_object* x_14; +x_13 = lean_unbox(x_2); +lean_dec(x_2); +x_14 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6(x_1, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_2); +lean_dec(x_2); +x_13 = l_Std_RBNode_forIn_visit___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__6___at_Lean_Elab_Term_logUnassignedUsingErrorInfos___spec__7(x_1, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_logUnassignedUsingErrorInfos___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_1); +return x_10; +} +} +static lean_object* _init_l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_abortCommandExceptionId; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg___closed__1; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg___closed__2; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = lean_alloc_closure((void*)(l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg), 1, 0); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_ensureNoUnassignedMVars(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = l_Lean_Meta_getMVarsAtDecl(x_1, x_4, x_5, x_6, x_7, x_8); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_box(0); +x_13 = l_Lean_Elab_Term_logUnassignedUsingErrorInfos(x_10, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_11); +lean_dec(x_10); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_unbox(x_14); +lean_dec(x_14); +if (x_15 == 0) +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_13); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_13, 0); +lean_dec(x_17); +x_18 = lean_box(0); +lean_ctor_set(x_13, 0, x_18); +return x_13; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_13, 1); +lean_inc(x_19); +lean_dec(x_13); +x_20 = lean_box(0); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +return x_21; +} +} +else +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_13, 1); +lean_inc(x_22); +lean_dec(x_13); +x_23 = l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___rarg(x_22); +return x_23; +} +} +else +{ +uint8_t x_24; +x_24 = !lean_is_exclusive(x_13); +if (x_24 == 0) +{ +return x_13; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_13, 0); +x_26 = lean_ctor_get(x_13, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_13); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Elab_throwAbortCommand___at_Lean_Elab_Term_ensureNoUnassignedMVars___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutPostponing___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; +x_9 = !lean_is_exclusive(x_2); +if (x_9 == 0) +{ +uint8_t x_10; lean_object* x_11; +x_10 = 0; +lean_ctor_set_uint8(x_2, sizeof(void*)*8, x_10); +x_11 = lean_apply_7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; uint8_t x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; uint8_t x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; +x_12 = lean_ctor_get(x_2, 0); +x_13 = lean_ctor_get(x_2, 1); +x_14 = lean_ctor_get(x_2, 2); +x_15 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 1); +x_16 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 2); +x_17 = lean_ctor_get(x_2, 3); +x_18 = lean_ctor_get(x_2, 4); +x_19 = lean_ctor_get(x_2, 5); +x_20 = lean_ctor_get(x_2, 6); +x_21 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 3); +x_22 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 4); +x_23 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 5); +x_24 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 6); +x_25 = lean_ctor_get(x_2, 7); +x_26 = lean_ctor_get_uint8(x_2, sizeof(void*)*8 + 7); +lean_inc(x_25); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_2); +x_27 = 0; +x_28 = lean_alloc_ctor(0, 8, 8); +lean_ctor_set(x_28, 0, x_12); +lean_ctor_set(x_28, 1, x_13); +lean_ctor_set(x_28, 2, x_14); +lean_ctor_set(x_28, 3, x_17); +lean_ctor_set(x_28, 4, x_18); +lean_ctor_set(x_28, 5, x_19); +lean_ctor_set(x_28, 6, x_20); +lean_ctor_set(x_28, 7, x_25); +lean_ctor_set_uint8(x_28, sizeof(void*)*8, x_27); +lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 1, x_15); +lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 2, x_16); +lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 3, x_21); +lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 4, x_22); +lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 5, x_23); +lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 6, x_24); +lean_ctor_set_uint8(x_28, sizeof(void*)*8 + 7, x_26); +x_29 = lean_apply_7(x_1, x_28, x_3, x_4, x_5, x_6, x_7, x_8); +return x_29; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutPostponing(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutPostponing___rarg), 8, 0); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("explicitBinder", 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__15; +x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("(", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(2); +x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__3; +x_3 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("null", 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__6; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(":", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(2); +x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__8; +x_3 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(2u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Term_mkExplicitBinder___closed__10; +x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__9; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__7; +x_3 = l_Lean_Elab_Term_instInhabitedLetRecToLift___closed__1; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(")", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(2); +x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__13; +x_3 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(5u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkExplicitBinder___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Term_mkExplicitBinder___closed__15; +x_2 = l_Lean_Elab_Term_mkExplicitBinder___closed__4; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkExplicitBinder(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; 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; +x_3 = l_Lean_Elab_Term_mkExplicitBinder___closed__5; +x_4 = lean_array_push(x_3, x_1); +x_5 = lean_box(2); +x_6 = l_Lean_Elab_Term_mkExplicitBinder___closed__7; +x_7 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_6); +lean_ctor_set(x_7, 2, x_4); +x_8 = l_Lean_Elab_Term_mkExplicitBinder___closed__11; +x_9 = lean_array_push(x_8, x_2); +x_10 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_10, 0, x_5); +lean_ctor_set(x_10, 1, x_6); +lean_ctor_set(x_10, 2, x_9); +x_11 = l_Lean_Elab_Term_mkExplicitBinder___closed__16; +x_12 = lean_array_push(x_11, x_7); +x_13 = lean_array_push(x_12, x_10); +x_14 = l_Lean_Elab_Term_mkExplicitBinder___closed__12; +x_15 = lean_array_push(x_13, x_14); +x_16 = l_Lean_Elab_Term_mkExplicitBinder___closed__14; +x_17 = lean_array_push(x_15, x_16); +x_18 = l_Lean_Elab_Term_mkExplicitBinder___closed__2; +x_19 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_19, 0, x_5); +lean_ctor_set(x_19, 1, x_18); +lean_ctor_set(x_19, 2, x_17); +return x_19; +} +} +LEAN_EXPORT uint8_t l_Lean_Elab_Term_levelMVarToParam___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; +x_3 = l_List_elem___at_Lean_NameHashSet_insert___spec__2(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Term_levelMVarToParam___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("u", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_levelMVarToParam___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Term_levelMVarToParam___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; 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_11 = l_Lean_Elab_Term_getLevelNames___rarg(x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_st_ref_get(x_9, x_13); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = lean_st_ref_get(x_7, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_alloc_closure((void*)(l_Lean_Elab_Term_levelMVarToParam___lambda__1___boxed), 2, 1); +lean_closure_set(x_20, 0, x_12); +x_21 = l_Lean_Elab_Term_levelMVarToParam___closed__2; +x_22 = l_Lean_MetavarContext_levelMVarToParam(x_19, x_20, x_3, x_1, x_21, x_2); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_st_ref_get(x_9, x_18); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_st_ref_take(x_7, x_25); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get_uint8(x_23, sizeof(void*)*8); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_29 = lean_ctor_get(x_27, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_26, 1); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_ctor_get(x_23, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_23, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_23, 2); +lean_inc(x_33); +x_34 = lean_ctor_get(x_23, 3); +lean_inc(x_34); +x_35 = lean_ctor_get(x_23, 4); +lean_inc(x_35); +x_36 = lean_ctor_get(x_23, 5); +lean_inc(x_36); +x_37 = lean_ctor_get(x_23, 6); +lean_inc(x_37); +x_38 = lean_ctor_get(x_23, 7); +lean_inc(x_38); +lean_dec(x_23); +x_39 = !lean_is_exclusive(x_27); +if (x_39 == 0) +{ +lean_object* x_40; uint8_t x_41; +x_40 = lean_ctor_get(x_27, 0); +lean_dec(x_40); +x_41 = !lean_is_exclusive(x_29); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; +x_42 = lean_ctor_get(x_29, 7); +lean_dec(x_42); +x_43 = lean_ctor_get(x_29, 6); +lean_dec(x_43); +x_44 = lean_ctor_get(x_29, 5); +lean_dec(x_44); +x_45 = lean_ctor_get(x_29, 4); +lean_dec(x_45); +x_46 = lean_ctor_get(x_29, 3); +lean_dec(x_46); +x_47 = lean_ctor_get(x_29, 2); +lean_dec(x_47); +x_48 = lean_ctor_get(x_29, 1); +lean_dec(x_48); +x_49 = lean_ctor_get(x_29, 0); +lean_dec(x_49); +lean_ctor_set(x_29, 7, x_38); +lean_ctor_set(x_29, 6, x_37); +lean_ctor_set(x_29, 5, x_36); +lean_ctor_set(x_29, 4, x_35); +lean_ctor_set(x_29, 3, x_34); +lean_ctor_set(x_29, 2, x_33); +lean_ctor_set(x_29, 1, x_32); +lean_ctor_set(x_29, 0, x_31); +x_50 = lean_st_ref_set(x_7, x_27, x_30); +x_51 = !lean_is_exclusive(x_50); +if (x_51 == 0) +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_52 = lean_ctor_get(x_50, 0); +lean_dec(x_52); +x_53 = lean_ctor_get(x_22, 3); +lean_inc(x_53); +x_54 = lean_ctor_get(x_22, 2); +lean_inc(x_54); +lean_dec(x_22); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +lean_ctor_set(x_50, 0, x_55); +return x_50; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_56 = lean_ctor_get(x_50, 1); +lean_inc(x_56); +lean_dec(x_50); +x_57 = lean_ctor_get(x_22, 3); +lean_inc(x_57); +x_58 = lean_ctor_get(x_22, 2); +lean_inc(x_58); +lean_dec(x_22); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_56); +return x_60; +} +} +else +{ +uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_61 = lean_ctor_get_uint8(x_29, sizeof(void*)*8); +lean_dec(x_29); +x_62 = lean_alloc_ctor(0, 8, 1); +lean_ctor_set(x_62, 0, x_31); +lean_ctor_set(x_62, 1, x_32); +lean_ctor_set(x_62, 2, x_33); +lean_ctor_set(x_62, 3, x_34); +lean_ctor_set(x_62, 4, x_35); +lean_ctor_set(x_62, 5, x_36); +lean_ctor_set(x_62, 6, x_37); +lean_ctor_set(x_62, 7, x_38); +lean_ctor_set_uint8(x_62, sizeof(void*)*8, x_61); +lean_ctor_set(x_27, 0, x_62); +x_63 = lean_st_ref_set(x_7, x_27, x_30); +x_64 = lean_ctor_get(x_63, 1); +lean_inc(x_64); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + x_65 = x_63; +} else { + lean_dec_ref(x_63); + x_65 = lean_box(0); +} +x_66 = lean_ctor_get(x_22, 3); +lean_inc(x_66); +x_67 = lean_ctor_get(x_22, 2); +lean_inc(x_67); +lean_dec(x_22); +x_68 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +if (lean_is_scalar(x_65)) { + x_69 = lean_alloc_ctor(0, 2, 0); +} else { + x_69 = x_65; +} +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_64); +return x_69; +} +} +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_70 = lean_ctor_get(x_27, 1); +x_71 = lean_ctor_get(x_27, 2); +x_72 = lean_ctor_get(x_27, 3); +lean_inc(x_72); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_27); +x_73 = lean_ctor_get_uint8(x_29, sizeof(void*)*8); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + lean_ctor_release(x_29, 2); + lean_ctor_release(x_29, 3); + lean_ctor_release(x_29, 4); + lean_ctor_release(x_29, 5); + lean_ctor_release(x_29, 6); + lean_ctor_release(x_29, 7); + x_74 = x_29; +} else { + lean_dec_ref(x_29); + x_74 = lean_box(0); +} +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(0, 8, 1); +} else { + x_75 = x_74; +} +lean_ctor_set(x_75, 0, x_31); +lean_ctor_set(x_75, 1, x_32); +lean_ctor_set(x_75, 2, x_33); +lean_ctor_set(x_75, 3, x_34); +lean_ctor_set(x_75, 4, x_35); +lean_ctor_set(x_75, 5, x_36); +lean_ctor_set(x_75, 6, x_37); +lean_ctor_set(x_75, 7, x_38); +lean_ctor_set_uint8(x_75, sizeof(void*)*8, x_73); +x_76 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_70); +lean_ctor_set(x_76, 2, x_71); +lean_ctor_set(x_76, 3, x_72); +x_77 = lean_st_ref_set(x_7, x_76, x_30); +x_78 = lean_ctor_get(x_77, 1); +lean_inc(x_78); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_79 = x_77; +} else { + lean_dec_ref(x_77); + x_79 = lean_box(0); +} +x_80 = lean_ctor_get(x_22, 3); +lean_inc(x_80); +x_81 = lean_ctor_get(x_22, 2); +lean_inc(x_81); +lean_dec(x_22); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +if (lean_is_scalar(x_79)) { + x_83 = lean_alloc_ctor(0, 2, 0); +} else { + x_83 = x_79; +} +lean_ctor_set(x_83, 0, x_82); +lean_ctor_set(x_83, 1, x_78); +return x_83; +} +} +else +{ +lean_object* x_84; uint8_t x_85; +x_84 = lean_ctor_get(x_26, 1); +lean_inc(x_84); +lean_dec(x_26); +x_85 = !lean_is_exclusive(x_23); +if (x_85 == 0) +{ +uint8_t x_86; +x_86 = !lean_is_exclusive(x_27); +if (x_86 == 0) +{ +lean_object* x_87; uint8_t x_88; lean_object* x_89; uint8_t x_90; +x_87 = lean_ctor_get(x_27, 0); +lean_dec(x_87); +x_88 = 1; +lean_ctor_set_uint8(x_23, sizeof(void*)*8, x_88); +lean_ctor_set(x_27, 0, x_23); +x_89 = lean_st_ref_set(x_7, x_27, x_84); +x_90 = !lean_is_exclusive(x_89); +if (x_90 == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_91 = lean_ctor_get(x_89, 0); +lean_dec(x_91); +x_92 = lean_ctor_get(x_22, 3); +lean_inc(x_92); +x_93 = lean_ctor_get(x_22, 2); +lean_inc(x_93); +lean_dec(x_22); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_93); +lean_ctor_set(x_89, 0, x_94); +return x_89; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_95 = lean_ctor_get(x_89, 1); +lean_inc(x_95); +lean_dec(x_89); +x_96 = lean_ctor_get(x_22, 3); +lean_inc(x_96); +x_97 = lean_ctor_get(x_22, 2); +lean_inc(x_97); +lean_dec(x_22); +x_98 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_97); +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set(x_99, 1, x_95); +return x_99; +} +} +else +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_100 = lean_ctor_get(x_27, 1); +x_101 = lean_ctor_get(x_27, 2); +x_102 = lean_ctor_get(x_27, 3); +lean_inc(x_102); +lean_inc(x_101); +lean_inc(x_100); +lean_dec(x_27); +x_103 = 1; +lean_ctor_set_uint8(x_23, sizeof(void*)*8, x_103); +x_104 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_104, 0, x_23); +lean_ctor_set(x_104, 1, x_100); +lean_ctor_set(x_104, 2, x_101); +lean_ctor_set(x_104, 3, x_102); +x_105 = lean_st_ref_set(x_7, x_104, x_84); +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; +} else { + lean_dec_ref(x_105); + x_107 = lean_box(0); +} +x_108 = lean_ctor_get(x_22, 3); +lean_inc(x_108); +x_109 = lean_ctor_get(x_22, 2); +lean_inc(x_109); +lean_dec(x_22); +x_110 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_110, 0, x_108); +lean_ctor_set(x_110, 1, x_109); +if (lean_is_scalar(x_107)) { + x_111 = lean_alloc_ctor(0, 2, 0); +} else { + x_111 = x_107; +} +lean_ctor_set(x_111, 0, x_110); +lean_ctor_set(x_111, 1, x_106); +return x_111; +} +} +else +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; uint8_t x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_112 = lean_ctor_get(x_23, 0); +x_113 = lean_ctor_get(x_23, 1); +x_114 = lean_ctor_get(x_23, 2); +x_115 = lean_ctor_get(x_23, 3); +x_116 = lean_ctor_get(x_23, 4); +x_117 = lean_ctor_get(x_23, 5); +x_118 = lean_ctor_get(x_23, 6); +x_119 = lean_ctor_get(x_23, 7); +lean_inc(x_119); +lean_inc(x_118); +lean_inc(x_117); +lean_inc(x_116); +lean_inc(x_115); +lean_inc(x_114); +lean_inc(x_113); +lean_inc(x_112); +lean_dec(x_23); +x_120 = lean_ctor_get(x_27, 1); +lean_inc(x_120); +x_121 = lean_ctor_get(x_27, 2); +lean_inc(x_121); +x_122 = lean_ctor_get(x_27, 3); +lean_inc(x_122); +if (lean_is_exclusive(x_27)) { + lean_ctor_release(x_27, 0); + lean_ctor_release(x_27, 1); + lean_ctor_release(x_27, 2); + lean_ctor_release(x_27, 3); + x_123 = x_27; +} else { + lean_dec_ref(x_27); + x_123 = lean_box(0); +} +x_124 = 1; +x_125 = lean_alloc_ctor(0, 8, 1); +lean_ctor_set(x_125, 0, x_112); +lean_ctor_set(x_125, 1, x_113); +lean_ctor_set(x_125, 2, x_114); +lean_ctor_set(x_125, 3, x_115); +lean_ctor_set(x_125, 4, x_116); +lean_ctor_set(x_125, 5, x_117); +lean_ctor_set(x_125, 6, x_118); +lean_ctor_set(x_125, 7, x_119); +lean_ctor_set_uint8(x_125, sizeof(void*)*8, x_124); +if (lean_is_scalar(x_123)) { + x_126 = lean_alloc_ctor(0, 4, 0); +} else { + x_126 = x_123; +} +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_120); +lean_ctor_set(x_126, 2, x_121); +lean_ctor_set(x_126, 3, x_122); +x_127 = lean_st_ref_set(x_7, x_126, x_84); +x_128 = lean_ctor_get(x_127, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_129 = x_127; +} else { + lean_dec_ref(x_127); + x_129 = lean_box(0); +} +x_130 = lean_ctor_get(x_22, 3); +lean_inc(x_130); +x_131 = lean_ctor_get(x_22, 2); +lean_inc(x_131); +lean_dec(x_22); +x_132 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_132, 0, x_130); +lean_ctor_set(x_132, 1, x_131); +if (lean_is_scalar(x_129)) { + x_133 = lean_alloc_ctor(0, 2, 0); +} else { + x_133 = x_129; +} +lean_ctor_set(x_133, 0, x_132); +lean_ctor_set(x_133, 1, x_128); +return x_133; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Lean_Elab_Term_levelMVarToParam___lambda__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_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_Term_levelMVarToParam(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam_x27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_11 = lean_st_ref_get(x_9, x_10); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_st_ref_get(x_3, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l_Lean_Elab_Term_levelMVarToParam(x_1, x_14, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +x_21 = lean_st_ref_get(x_9, x_18); +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_23 = lean_st_ref_set(x_3, x_20, x_22); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; +x_25 = lean_ctor_get(x_23, 0); +lean_dec(x_25); +lean_ctor_set(x_23, 0, x_19); +return x_23; +} +else +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_19); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam_x27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Term_levelMVarToParam_x27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = l_Lean_addMacroScope(x_2, x_3, x_4); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__1), 4, 3); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_5); +lean_closure_set(x_7, 2, x_3); +x_8 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_6, x_7); +return x_8; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("x", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_3 = lean_ctor_get(x_2, 3); +lean_inc(x_3); +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +x_5 = lean_ctor_get(x_2, 2); +lean_inc(x_5); +x_6 = l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__2; +lean_inc(x_4); +x_7 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__2), 5, 4); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_1); +lean_closure_set(x_7, 2, x_6); +lean_closure_set(x_7, 3, x_4); +x_8 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_5, x_7); +x_9 = lean_apply_2(x_3, lean_box(0), x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshBinderName___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = l_Lean_mkIdentFrom(x_2, x_3); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +lean_inc(x_1); +x_5 = l_Lean_Elab_Term_mkFreshBinderName___rarg(x_1, x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshIdent___rarg___lambda__1), 3, 2); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_3); +x_7 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_5, x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshIdent___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_9 = lean_ctor_get(x_6, 5); +x_10 = lean_ctor_get(x_2, 2); +lean_inc(x_10); +lean_inc(x_10); +x_11 = l_Lean_Elab_getBetterRef(x_9, x_10); +x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_4, x_5, x_6, x_7, x_8); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_13, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_14); +lean_dec(x_2); +lean_dec(x_10); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_11); +lean_ctor_set(x_18, 1, x_17); +lean_ctor_set_tag(x_15, 1); +lean_ctor_set(x_15, 0, x_18); +return x_15; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_15, 0); +x_20 = lean_ctor_get(x_15, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_15); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_11); +lean_ctor_set(x_21, 1, x_19); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_254; uint8_t x_255; +x_254 = 2; +x_255 = l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_101_(x_3, x_254); +if (x_255 == 0) +{ +lean_object* x_256; +x_256 = lean_box(0); +x_11 = x_256; +goto block_253; +} +else +{ +uint8_t x_257; +lean_inc(x_2); +x_257 = l_Lean_MessageData_hasSyntheticSorry(x_2); +if (x_257 == 0) +{ +lean_object* x_258; +x_258 = lean_box(0); +x_11 = x_258; +goto block_253; +} +else +{ +lean_object* x_259; lean_object* x_260; +lean_dec(x_2); +x_259 = lean_box(0); +x_260 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_260, 0, x_259); +lean_ctor_set(x_260, 1, x_10); +return x_260; +} +} +block_253: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; +lean_dec(x_11); +x_12 = lean_ctor_get(x_8, 0); +x_13 = lean_ctor_get(x_8, 1); +x_14 = lean_ctor_get(x_8, 5); +x_15 = lean_ctor_get(x_8, 6); +x_16 = lean_ctor_get(x_8, 7); +x_17 = l_Lean_replaceRef(x_1, x_14); +x_18 = 0; +x_19 = l_Lean_Syntax_getPos_x3f(x_17, x_18); +x_20 = l_Lean_Syntax_getTailPos_x3f(x_17, x_18); +if (lean_obj_tag(x_19) == 0) +{ +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_21 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_unsigned_to_nat(0u); +x_25 = l_Lean_FileMap_toPosition(x_13, x_24); +lean_inc(x_25); +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_25); +lean_inc(x_16); +lean_inc(x_15); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_15); +lean_ctor_set(x_27, 1, x_16); +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_22); +x_29 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; +lean_inc(x_12); +x_30 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_30, 0, x_12); +lean_ctor_set(x_30, 1, x_25); +lean_ctor_set(x_30, 2, x_26); +lean_ctor_set(x_30, 3, x_29); +lean_ctor_set(x_30, 4, x_28); +lean_ctor_set_uint8(x_30, sizeof(void*)*5, x_3); +x_31 = lean_st_ref_take(x_9, x_23); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = !lean_is_exclusive(x_32); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_35 = lean_ctor_get(x_32, 5); +x_36 = l_Std_PersistentArray_push___rarg(x_35, x_30); +lean_ctor_set(x_32, 5, x_36); +x_37 = lean_st_ref_set(x_9, x_32, x_33); +x_38 = !lean_is_exclusive(x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_37, 0); +lean_dec(x_39); +x_40 = lean_box(0); +lean_ctor_set(x_37, 0, x_40); +return x_37; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_37, 1); +lean_inc(x_41); +lean_dec(x_37); +x_42 = lean_box(0); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_41); +return x_43; +} +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_44 = lean_ctor_get(x_32, 0); +x_45 = lean_ctor_get(x_32, 1); +x_46 = lean_ctor_get(x_32, 2); +x_47 = lean_ctor_get(x_32, 3); +x_48 = lean_ctor_get(x_32, 4); +x_49 = lean_ctor_get(x_32, 5); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_32); +x_50 = l_Std_PersistentArray_push___rarg(x_49, x_30); +x_51 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_51, 0, x_44); +lean_ctor_set(x_51, 1, x_45); +lean_ctor_set(x_51, 2, x_46); +lean_ctor_set(x_51, 3, x_47); +lean_ctor_set(x_51, 4, x_48); +lean_ctor_set(x_51, 5, x_50); +x_52 = lean_st_ref_set(x_9, x_51, x_33); +x_53 = lean_ctor_get(x_52, 1); +lean_inc(x_53); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + x_54 = x_52; +} else { + lean_dec_ref(x_52); + x_54 = lean_box(0); +} +x_55 = lean_box(0); +if (lean_is_scalar(x_54)) { + x_56 = lean_alloc_ctor(0, 2, 0); +} else { + x_56 = x_54; +} +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_53); +return x_56; +} +} +else +{ +uint8_t x_57; +x_57 = !lean_is_exclusive(x_20); +if (x_57 == 0) +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +x_58 = lean_ctor_get(x_20, 0); +x_59 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = lean_unsigned_to_nat(0u); +x_63 = l_Lean_FileMap_toPosition(x_13, x_62); +x_64 = l_Lean_FileMap_toPosition(x_13, x_58); +lean_dec(x_58); +lean_ctor_set(x_20, 0, x_64); +lean_inc(x_16); +lean_inc(x_15); +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_15); +lean_ctor_set(x_65, 1, x_16); +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_60); +x_67 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; +lean_inc(x_12); +x_68 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_68, 0, x_12); +lean_ctor_set(x_68, 1, x_63); +lean_ctor_set(x_68, 2, x_20); +lean_ctor_set(x_68, 3, x_67); +lean_ctor_set(x_68, 4, x_66); +lean_ctor_set_uint8(x_68, sizeof(void*)*5, x_3); +x_69 = lean_st_ref_take(x_9, x_61); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); +lean_dec(x_69); +x_72 = !lean_is_exclusive(x_70); +if (x_72 == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_73 = lean_ctor_get(x_70, 5); +x_74 = l_Std_PersistentArray_push___rarg(x_73, x_68); +lean_ctor_set(x_70, 5, x_74); +x_75 = lean_st_ref_set(x_9, x_70, x_71); +x_76 = !lean_is_exclusive(x_75); +if (x_76 == 0) +{ +lean_object* x_77; lean_object* x_78; +x_77 = lean_ctor_get(x_75, 0); +lean_dec(x_77); +x_78 = lean_box(0); +lean_ctor_set(x_75, 0, x_78); +return x_75; +} +else +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_75, 1); +lean_inc(x_79); +lean_dec(x_75); +x_80 = lean_box(0); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_79); +return x_81; +} +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_82 = lean_ctor_get(x_70, 0); +x_83 = lean_ctor_get(x_70, 1); +x_84 = lean_ctor_get(x_70, 2); +x_85 = lean_ctor_get(x_70, 3); +x_86 = lean_ctor_get(x_70, 4); +x_87 = lean_ctor_get(x_70, 5); +lean_inc(x_87); +lean_inc(x_86); +lean_inc(x_85); +lean_inc(x_84); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_70); +x_88 = l_Std_PersistentArray_push___rarg(x_87, x_68); +x_89 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_89, 0, x_82); +lean_ctor_set(x_89, 1, x_83); +lean_ctor_set(x_89, 2, x_84); +lean_ctor_set(x_89, 3, x_85); +lean_ctor_set(x_89, 4, x_86); +lean_ctor_set(x_89, 5, x_88); +x_90 = lean_st_ref_set(x_9, x_89, x_71); +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_90)) { + lean_ctor_release(x_90, 0); + lean_ctor_release(x_90, 1); + x_92 = x_90; +} else { + lean_dec_ref(x_90); + x_92 = lean_box(0); +} +x_93 = lean_box(0); +if (lean_is_scalar(x_92)) { + x_94 = lean_alloc_ctor(0, 2, 0); +} else { + x_94 = x_92; +} +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_91); +return x_94; +} +} +else +{ +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; +x_95 = lean_ctor_get(x_20, 0); +lean_inc(x_95); +lean_dec(x_20); +x_96 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +lean_dec(x_96); +x_99 = lean_unsigned_to_nat(0u); +x_100 = l_Lean_FileMap_toPosition(x_13, x_99); +x_101 = l_Lean_FileMap_toPosition(x_13, x_95); +lean_dec(x_95); +x_102 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_102, 0, x_101); +lean_inc(x_16); +lean_inc(x_15); +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_15); +lean_ctor_set(x_103, 1, x_16); +x_104 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_97); +x_105 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; +lean_inc(x_12); +x_106 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_106, 0, x_12); +lean_ctor_set(x_106, 1, x_100); +lean_ctor_set(x_106, 2, x_102); +lean_ctor_set(x_106, 3, x_105); +lean_ctor_set(x_106, 4, x_104); +lean_ctor_set_uint8(x_106, sizeof(void*)*5, x_3); +x_107 = lean_st_ref_take(x_9, x_98); +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +x_110 = lean_ctor_get(x_108, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_108, 1); +lean_inc(x_111); +x_112 = lean_ctor_get(x_108, 2); +lean_inc(x_112); +x_113 = lean_ctor_get(x_108, 3); +lean_inc(x_113); +x_114 = lean_ctor_get(x_108, 4); +lean_inc(x_114); +x_115 = lean_ctor_get(x_108, 5); +lean_inc(x_115); +if (lean_is_exclusive(x_108)) { + lean_ctor_release(x_108, 0); + lean_ctor_release(x_108, 1); + lean_ctor_release(x_108, 2); + lean_ctor_release(x_108, 3); + lean_ctor_release(x_108, 4); + lean_ctor_release(x_108, 5); + x_116 = x_108; +} else { + lean_dec_ref(x_108); + x_116 = lean_box(0); +} +x_117 = l_Std_PersistentArray_push___rarg(x_115, x_106); +if (lean_is_scalar(x_116)) { + x_118 = lean_alloc_ctor(0, 6, 0); +} else { + x_118 = x_116; +} +lean_ctor_set(x_118, 0, x_110); +lean_ctor_set(x_118, 1, x_111); +lean_ctor_set(x_118, 2, x_112); +lean_ctor_set(x_118, 3, x_113); +lean_ctor_set(x_118, 4, x_114); +lean_ctor_set(x_118, 5, x_117); +x_119 = lean_st_ref_set(x_9, x_118, x_109); +x_120 = lean_ctor_get(x_119, 1); +lean_inc(x_120); +if (lean_is_exclusive(x_119)) { + lean_ctor_release(x_119, 0); + lean_ctor_release(x_119, 1); + x_121 = x_119; +} else { + lean_dec_ref(x_119); + x_121 = lean_box(0); +} +x_122 = lean_box(0); +if (lean_is_scalar(x_121)) { + x_123 = lean_alloc_ctor(0, 2, 0); +} else { + x_123 = x_121; +} +lean_ctor_set(x_123, 0, x_122); +lean_ctor_set(x_123, 1, x_120); +return x_123; +} +} +} +else +{ +if (lean_obj_tag(x_20) == 0) +{ +uint8_t x_124; +x_124 = !lean_is_exclusive(x_19); +if (x_124 == 0) +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; uint8_t x_137; +x_125 = lean_ctor_get(x_19, 0); +x_126 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); +x_127 = lean_ctor_get(x_126, 0); +lean_inc(x_127); +x_128 = lean_ctor_get(x_126, 1); +lean_inc(x_128); +lean_dec(x_126); +x_129 = l_Lean_FileMap_toPosition(x_13, x_125); +lean_dec(x_125); +lean_inc(x_129); +lean_ctor_set(x_19, 0, x_129); +lean_inc(x_16); +lean_inc(x_15); +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_15); +lean_ctor_set(x_130, 1, x_16); +x_131 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_127); +x_132 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; +lean_inc(x_12); +x_133 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_133, 0, x_12); +lean_ctor_set(x_133, 1, x_129); +lean_ctor_set(x_133, 2, x_19); +lean_ctor_set(x_133, 3, x_132); +lean_ctor_set(x_133, 4, x_131); +lean_ctor_set_uint8(x_133, sizeof(void*)*5, x_3); +x_134 = lean_st_ref_take(x_9, x_128); +x_135 = lean_ctor_get(x_134, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_134, 1); +lean_inc(x_136); +lean_dec(x_134); +x_137 = !lean_is_exclusive(x_135); +if (x_137 == 0) { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_50, 0); -lean_dec(x_52); -x_53 = lean_ctor_get(x_22, 3); -lean_inc(x_53); -x_54 = lean_ctor_get(x_22, 2); -lean_inc(x_54); -lean_dec(x_22); -x_55 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -lean_ctor_set(x_50, 0, x_55); -return x_50; +lean_object* x_138; lean_object* x_139; lean_object* x_140; uint8_t x_141; +x_138 = lean_ctor_get(x_135, 5); +x_139 = l_Std_PersistentArray_push___rarg(x_138, x_133); +lean_ctor_set(x_135, 5, x_139); +x_140 = lean_st_ref_set(x_9, x_135, x_136); +x_141 = !lean_is_exclusive(x_140); +if (x_141 == 0) +{ +lean_object* x_142; lean_object* x_143; +x_142 = lean_ctor_get(x_140, 0); +lean_dec(x_142); +x_143 = lean_box(0); +lean_ctor_set(x_140, 0, x_143); +return x_140; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_56 = lean_ctor_get(x_50, 1); -lean_inc(x_56); -lean_dec(x_50); -x_57 = lean_ctor_get(x_22, 3); -lean_inc(x_57); -x_58 = lean_ctor_get(x_22, 2); -lean_inc(x_58); -lean_dec(x_22); -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -x_60 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_56); -return x_60; +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_140, 1); +lean_inc(x_144); +lean_dec(x_140); +x_145 = lean_box(0); +x_146 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_146, 0, x_145); +lean_ctor_set(x_146, 1, x_144); +return x_146; } } else { -uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_61 = lean_ctor_get_uint8(x_29, sizeof(void*)*8); -lean_dec(x_29); -x_62 = lean_alloc_ctor(0, 8, 1); -lean_ctor_set(x_62, 0, x_31); -lean_ctor_set(x_62, 1, x_32); -lean_ctor_set(x_62, 2, x_33); -lean_ctor_set(x_62, 3, x_34); -lean_ctor_set(x_62, 4, x_35); -lean_ctor_set(x_62, 5, x_36); -lean_ctor_set(x_62, 6, x_37); -lean_ctor_set(x_62, 7, x_38); -lean_ctor_set_uint8(x_62, sizeof(void*)*8, x_61); -lean_ctor_set(x_27, 0, x_62); -x_63 = lean_st_ref_set(x_7, x_27, x_30); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; +x_147 = lean_ctor_get(x_135, 0); +x_148 = lean_ctor_get(x_135, 1); +x_149 = lean_ctor_get(x_135, 2); +x_150 = lean_ctor_get(x_135, 3); +x_151 = lean_ctor_get(x_135, 4); +x_152 = lean_ctor_get(x_135, 5); +lean_inc(x_152); +lean_inc(x_151); +lean_inc(x_150); +lean_inc(x_149); +lean_inc(x_148); +lean_inc(x_147); +lean_dec(x_135); +x_153 = l_Std_PersistentArray_push___rarg(x_152, x_133); +x_154 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_154, 0, x_147); +lean_ctor_set(x_154, 1, x_148); +lean_ctor_set(x_154, 2, x_149); +lean_ctor_set(x_154, 3, x_150); +lean_ctor_set(x_154, 4, x_151); +lean_ctor_set(x_154, 5, x_153); +x_155 = lean_st_ref_set(x_9, x_154, x_136); +x_156 = lean_ctor_get(x_155, 1); +lean_inc(x_156); +if (lean_is_exclusive(x_155)) { + lean_ctor_release(x_155, 0); + lean_ctor_release(x_155, 1); + x_157 = x_155; } else { - lean_dec_ref(x_63); - x_65 = lean_box(0); + lean_dec_ref(x_155); + x_157 = lean_box(0); } -x_66 = lean_ctor_get(x_22, 3); -lean_inc(x_66); -x_67 = lean_ctor_get(x_22, 2); -lean_inc(x_67); -lean_dec(x_22); -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -if (lean_is_scalar(x_65)) { - x_69 = lean_alloc_ctor(0, 2, 0); +x_158 = lean_box(0); +if (lean_is_scalar(x_157)) { + x_159 = lean_alloc_ctor(0, 2, 0); } else { - x_69 = x_65; + x_159 = x_157; } -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_64); -return x_69; +lean_ctor_set(x_159, 0, x_158); +lean_ctor_set(x_159, 1, x_156); +return x_159; } } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_70 = lean_ctor_get(x_27, 1); -x_71 = lean_ctor_get(x_27, 2); -x_72 = lean_ctor_get(x_27, 3); -lean_inc(x_72); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_27); -x_73 = lean_ctor_get_uint8(x_29, sizeof(void*)*8); -if (lean_is_exclusive(x_29)) { - lean_ctor_release(x_29, 0); - lean_ctor_release(x_29, 1); - lean_ctor_release(x_29, 2); - lean_ctor_release(x_29, 3); - lean_ctor_release(x_29, 4); - lean_ctor_release(x_29, 5); - lean_ctor_release(x_29, 6); - lean_ctor_release(x_29, 7); - x_74 = x_29; +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; +x_160 = lean_ctor_get(x_19, 0); +lean_inc(x_160); +lean_dec(x_19); +x_161 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); +x_162 = lean_ctor_get(x_161, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_161, 1); +lean_inc(x_163); +lean_dec(x_161); +x_164 = l_Lean_FileMap_toPosition(x_13, x_160); +lean_dec(x_160); +lean_inc(x_164); +x_165 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_165, 0, x_164); +lean_inc(x_16); +lean_inc(x_15); +x_166 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_166, 0, x_15); +lean_ctor_set(x_166, 1, x_16); +x_167 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_167, 0, x_166); +lean_ctor_set(x_167, 1, x_162); +x_168 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; +lean_inc(x_12); +x_169 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_169, 0, x_12); +lean_ctor_set(x_169, 1, x_164); +lean_ctor_set(x_169, 2, x_165); +lean_ctor_set(x_169, 3, x_168); +lean_ctor_set(x_169, 4, x_167); +lean_ctor_set_uint8(x_169, sizeof(void*)*5, x_3); +x_170 = lean_st_ref_take(x_9, x_163); +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 = lean_ctor_get(x_171, 0); +lean_inc(x_173); +x_174 = lean_ctor_get(x_171, 1); +lean_inc(x_174); +x_175 = lean_ctor_get(x_171, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_171, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_171, 4); +lean_inc(x_177); +x_178 = lean_ctor_get(x_171, 5); +lean_inc(x_178); +if (lean_is_exclusive(x_171)) { + lean_ctor_release(x_171, 0); + lean_ctor_release(x_171, 1); + lean_ctor_release(x_171, 2); + lean_ctor_release(x_171, 3); + lean_ctor_release(x_171, 4); + lean_ctor_release(x_171, 5); + x_179 = x_171; } else { - lean_dec_ref(x_29); - x_74 = lean_box(0); + lean_dec_ref(x_171); + x_179 = lean_box(0); } -if (lean_is_scalar(x_74)) { - x_75 = lean_alloc_ctor(0, 8, 1); +x_180 = l_Std_PersistentArray_push___rarg(x_178, x_169); +if (lean_is_scalar(x_179)) { + x_181 = lean_alloc_ctor(0, 6, 0); } else { - x_75 = x_74; + x_181 = x_179; } -lean_ctor_set(x_75, 0, x_31); -lean_ctor_set(x_75, 1, x_32); -lean_ctor_set(x_75, 2, x_33); -lean_ctor_set(x_75, 3, x_34); -lean_ctor_set(x_75, 4, x_35); -lean_ctor_set(x_75, 5, x_36); -lean_ctor_set(x_75, 6, x_37); -lean_ctor_set(x_75, 7, x_38); -lean_ctor_set_uint8(x_75, sizeof(void*)*8, x_73); -x_76 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_70); -lean_ctor_set(x_76, 2, x_71); -lean_ctor_set(x_76, 3, x_72); -x_77 = lean_st_ref_set(x_7, x_76, x_30); -x_78 = lean_ctor_get(x_77, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_79 = x_77; +lean_ctor_set(x_181, 0, x_173); +lean_ctor_set(x_181, 1, x_174); +lean_ctor_set(x_181, 2, x_175); +lean_ctor_set(x_181, 3, x_176); +lean_ctor_set(x_181, 4, x_177); +lean_ctor_set(x_181, 5, x_180); +x_182 = lean_st_ref_set(x_9, x_181, x_172); +x_183 = lean_ctor_get(x_182, 1); +lean_inc(x_183); +if (lean_is_exclusive(x_182)) { + lean_ctor_release(x_182, 0); + lean_ctor_release(x_182, 1); + x_184 = x_182; } else { - lean_dec_ref(x_77); - x_79 = lean_box(0); + lean_dec_ref(x_182); + x_184 = lean_box(0); } -x_80 = lean_ctor_get(x_22, 3); -lean_inc(x_80); -x_81 = lean_ctor_get(x_22, 2); -lean_inc(x_81); -lean_dec(x_22); -x_82 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -if (lean_is_scalar(x_79)) { - x_83 = lean_alloc_ctor(0, 2, 0); +x_185 = lean_box(0); +if (lean_is_scalar(x_184)) { + x_186 = lean_alloc_ctor(0, 2, 0); } else { - x_83 = x_79; + x_186 = x_184; } -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_78); -return x_83; +lean_ctor_set(x_186, 0, x_185); +lean_ctor_set(x_186, 1, x_183); +return x_186; } } else { -lean_object* x_84; uint8_t x_85; -x_84 = lean_ctor_get(x_26, 1); -lean_inc(x_84); -lean_dec(x_26); -x_85 = !lean_is_exclusive(x_23); -if (x_85 == 0) +lean_object* x_187; uint8_t x_188; +x_187 = lean_ctor_get(x_19, 0); +lean_inc(x_187); +lean_dec(x_19); +x_188 = !lean_is_exclusive(x_20); +if (x_188 == 0) { -uint8_t x_86; -x_86 = !lean_is_exclusive(x_27); -if (x_86 == 0) +lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; uint8_t x_202; +x_189 = lean_ctor_get(x_20, 0); +x_190 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); +x_191 = lean_ctor_get(x_190, 0); +lean_inc(x_191); +x_192 = lean_ctor_get(x_190, 1); +lean_inc(x_192); +lean_dec(x_190); +x_193 = l_Lean_FileMap_toPosition(x_13, x_187); +lean_dec(x_187); +x_194 = l_Lean_FileMap_toPosition(x_13, x_189); +lean_dec(x_189); +lean_ctor_set(x_20, 0, x_194); +lean_inc(x_16); +lean_inc(x_15); +x_195 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_195, 0, x_15); +lean_ctor_set(x_195, 1, x_16); +x_196 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_196, 0, x_195); +lean_ctor_set(x_196, 1, x_191); +x_197 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; +lean_inc(x_12); +x_198 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_198, 0, x_12); +lean_ctor_set(x_198, 1, x_193); +lean_ctor_set(x_198, 2, x_20); +lean_ctor_set(x_198, 3, x_197); +lean_ctor_set(x_198, 4, x_196); +lean_ctor_set_uint8(x_198, sizeof(void*)*5, x_3); +x_199 = lean_st_ref_take(x_9, x_192); +x_200 = lean_ctor_get(x_199, 0); +lean_inc(x_200); +x_201 = lean_ctor_get(x_199, 1); +lean_inc(x_201); +lean_dec(x_199); +x_202 = !lean_is_exclusive(x_200); +if (x_202 == 0) { -lean_object* x_87; uint8_t x_88; lean_object* x_89; uint8_t x_90; -x_87 = lean_ctor_get(x_27, 0); -lean_dec(x_87); -x_88 = 1; -lean_ctor_set_uint8(x_23, sizeof(void*)*8, x_88); -lean_ctor_set(x_27, 0, x_23); -x_89 = lean_st_ref_set(x_7, x_27, x_84); -x_90 = !lean_is_exclusive(x_89); -if (x_90 == 0) +lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_206; +x_203 = lean_ctor_get(x_200, 5); +x_204 = l_Std_PersistentArray_push___rarg(x_203, x_198); +lean_ctor_set(x_200, 5, x_204); +x_205 = lean_st_ref_set(x_9, x_200, x_201); +x_206 = !lean_is_exclusive(x_205); +if (x_206 == 0) { -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_91 = lean_ctor_get(x_89, 0); -lean_dec(x_91); -x_92 = lean_ctor_get(x_22, 3); -lean_inc(x_92); -x_93 = lean_ctor_get(x_22, 2); -lean_inc(x_93); -lean_dec(x_22); -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_92); -lean_ctor_set(x_94, 1, x_93); -lean_ctor_set(x_89, 0, x_94); -return x_89; +lean_object* x_207; lean_object* x_208; +x_207 = lean_ctor_get(x_205, 0); +lean_dec(x_207); +x_208 = lean_box(0); +lean_ctor_set(x_205, 0, x_208); +return x_205; } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_95 = lean_ctor_get(x_89, 1); -lean_inc(x_95); -lean_dec(x_89); -x_96 = lean_ctor_get(x_22, 3); -lean_inc(x_96); -x_97 = lean_ctor_get(x_22, 2); -lean_inc(x_97); -lean_dec(x_22); -x_98 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_98, 0, x_96); -lean_ctor_set(x_98, 1, x_97); -x_99 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_99, 0, x_98); -lean_ctor_set(x_99, 1, x_95); -return x_99; +lean_object* x_209; lean_object* x_210; lean_object* x_211; +x_209 = lean_ctor_get(x_205, 1); +lean_inc(x_209); +lean_dec(x_205); +x_210 = lean_box(0); +x_211 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_211, 0, x_210); +lean_ctor_set(x_211, 1, x_209); +return x_211; } } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_100 = lean_ctor_get(x_27, 1); -x_101 = lean_ctor_get(x_27, 2); -x_102 = lean_ctor_get(x_27, 3); -lean_inc(x_102); -lean_inc(x_101); -lean_inc(x_100); -lean_dec(x_27); -x_103 = 1; -lean_ctor_set_uint8(x_23, sizeof(void*)*8, x_103); -x_104 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_104, 0, x_23); -lean_ctor_set(x_104, 1, x_100); -lean_ctor_set(x_104, 2, x_101); -lean_ctor_set(x_104, 3, x_102); -x_105 = lean_st_ref_set(x_7, x_104, x_84); -x_106 = lean_ctor_get(x_105, 1); -lean_inc(x_106); -if (lean_is_exclusive(x_105)) { - lean_ctor_release(x_105, 0); - lean_ctor_release(x_105, 1); - x_107 = x_105; +lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; +x_212 = lean_ctor_get(x_200, 0); +x_213 = lean_ctor_get(x_200, 1); +x_214 = lean_ctor_get(x_200, 2); +x_215 = lean_ctor_get(x_200, 3); +x_216 = lean_ctor_get(x_200, 4); +x_217 = lean_ctor_get(x_200, 5); +lean_inc(x_217); +lean_inc(x_216); +lean_inc(x_215); +lean_inc(x_214); +lean_inc(x_213); +lean_inc(x_212); +lean_dec(x_200); +x_218 = l_Std_PersistentArray_push___rarg(x_217, x_198); +x_219 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_219, 0, x_212); +lean_ctor_set(x_219, 1, x_213); +lean_ctor_set(x_219, 2, x_214); +lean_ctor_set(x_219, 3, x_215); +lean_ctor_set(x_219, 4, x_216); +lean_ctor_set(x_219, 5, x_218); +x_220 = lean_st_ref_set(x_9, x_219, x_201); +x_221 = lean_ctor_get(x_220, 1); +lean_inc(x_221); +if (lean_is_exclusive(x_220)) { + lean_ctor_release(x_220, 0); + lean_ctor_release(x_220, 1); + x_222 = x_220; } else { - lean_dec_ref(x_105); - x_107 = lean_box(0); + lean_dec_ref(x_220); + x_222 = lean_box(0); } -x_108 = lean_ctor_get(x_22, 3); -lean_inc(x_108); -x_109 = lean_ctor_get(x_22, 2); -lean_inc(x_109); -lean_dec(x_22); -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -if (lean_is_scalar(x_107)) { - x_111 = lean_alloc_ctor(0, 2, 0); +x_223 = lean_box(0); +if (lean_is_scalar(x_222)) { + x_224 = lean_alloc_ctor(0, 2, 0); } else { - x_111 = x_107; -} -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_106); -return x_111; -} + x_224 = x_222; } -else -{ -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; uint8_t x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_112 = lean_ctor_get(x_23, 0); -x_113 = lean_ctor_get(x_23, 1); -x_114 = lean_ctor_get(x_23, 2); -x_115 = lean_ctor_get(x_23, 3); -x_116 = lean_ctor_get(x_23, 4); -x_117 = lean_ctor_get(x_23, 5); -x_118 = lean_ctor_get(x_23, 6); -x_119 = lean_ctor_get(x_23, 7); -lean_inc(x_119); -lean_inc(x_118); -lean_inc(x_117); -lean_inc(x_116); -lean_inc(x_115); -lean_inc(x_114); -lean_inc(x_113); -lean_inc(x_112); -lean_dec(x_23); -x_120 = lean_ctor_get(x_27, 1); -lean_inc(x_120); -x_121 = lean_ctor_get(x_27, 2); -lean_inc(x_121); -x_122 = lean_ctor_get(x_27, 3); -lean_inc(x_122); -if (lean_is_exclusive(x_27)) { - lean_ctor_release(x_27, 0); - lean_ctor_release(x_27, 1); - lean_ctor_release(x_27, 2); - lean_ctor_release(x_27, 3); - x_123 = x_27; +lean_ctor_set(x_224, 0, x_223); +lean_ctor_set(x_224, 1, x_221); +return x_224; +} +} +else +{ +lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; +x_225 = lean_ctor_get(x_20, 0); +lean_inc(x_225); +lean_dec(x_20); +x_226 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); +x_227 = lean_ctor_get(x_226, 0); +lean_inc(x_227); +x_228 = lean_ctor_get(x_226, 1); +lean_inc(x_228); +lean_dec(x_226); +x_229 = l_Lean_FileMap_toPosition(x_13, x_187); +lean_dec(x_187); +x_230 = l_Lean_FileMap_toPosition(x_13, x_225); +lean_dec(x_225); +x_231 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_231, 0, x_230); +lean_inc(x_16); +lean_inc(x_15); +x_232 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_232, 0, x_15); +lean_ctor_set(x_232, 1, x_16); +x_233 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_233, 0, x_232); +lean_ctor_set(x_233, 1, x_227); +x_234 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; +lean_inc(x_12); +x_235 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_235, 0, x_12); +lean_ctor_set(x_235, 1, x_229); +lean_ctor_set(x_235, 2, x_231); +lean_ctor_set(x_235, 3, x_234); +lean_ctor_set(x_235, 4, x_233); +lean_ctor_set_uint8(x_235, sizeof(void*)*5, x_3); +x_236 = lean_st_ref_take(x_9, x_228); +x_237 = lean_ctor_get(x_236, 0); +lean_inc(x_237); +x_238 = lean_ctor_get(x_236, 1); +lean_inc(x_238); +lean_dec(x_236); +x_239 = lean_ctor_get(x_237, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_237, 1); +lean_inc(x_240); +x_241 = lean_ctor_get(x_237, 2); +lean_inc(x_241); +x_242 = lean_ctor_get(x_237, 3); +lean_inc(x_242); +x_243 = lean_ctor_get(x_237, 4); +lean_inc(x_243); +x_244 = lean_ctor_get(x_237, 5); +lean_inc(x_244); +if (lean_is_exclusive(x_237)) { + lean_ctor_release(x_237, 0); + lean_ctor_release(x_237, 1); + lean_ctor_release(x_237, 2); + lean_ctor_release(x_237, 3); + lean_ctor_release(x_237, 4); + lean_ctor_release(x_237, 5); + x_245 = x_237; } else { - lean_dec_ref(x_27); - x_123 = lean_box(0); + lean_dec_ref(x_237); + x_245 = lean_box(0); } -x_124 = 1; -x_125 = lean_alloc_ctor(0, 8, 1); -lean_ctor_set(x_125, 0, x_112); -lean_ctor_set(x_125, 1, x_113); -lean_ctor_set(x_125, 2, x_114); -lean_ctor_set(x_125, 3, x_115); -lean_ctor_set(x_125, 4, x_116); -lean_ctor_set(x_125, 5, x_117); -lean_ctor_set(x_125, 6, x_118); -lean_ctor_set(x_125, 7, x_119); -lean_ctor_set_uint8(x_125, sizeof(void*)*8, x_124); -if (lean_is_scalar(x_123)) { - x_126 = lean_alloc_ctor(0, 4, 0); +x_246 = l_Std_PersistentArray_push___rarg(x_244, x_235); +if (lean_is_scalar(x_245)) { + x_247 = lean_alloc_ctor(0, 6, 0); } else { - x_126 = x_123; + x_247 = x_245; } -lean_ctor_set(x_126, 0, x_125); -lean_ctor_set(x_126, 1, x_120); -lean_ctor_set(x_126, 2, x_121); -lean_ctor_set(x_126, 3, x_122); -x_127 = lean_st_ref_set(x_7, x_126, x_84); -x_128 = lean_ctor_get(x_127, 1); -lean_inc(x_128); -if (lean_is_exclusive(x_127)) { - lean_ctor_release(x_127, 0); - lean_ctor_release(x_127, 1); - x_129 = x_127; +lean_ctor_set(x_247, 0, x_239); +lean_ctor_set(x_247, 1, x_240); +lean_ctor_set(x_247, 2, x_241); +lean_ctor_set(x_247, 3, x_242); +lean_ctor_set(x_247, 4, x_243); +lean_ctor_set(x_247, 5, x_246); +x_248 = lean_st_ref_set(x_9, x_247, x_238); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; } else { - lean_dec_ref(x_127); - x_129 = lean_box(0); + lean_dec_ref(x_248); + x_250 = lean_box(0); } -x_130 = lean_ctor_get(x_22, 3); -lean_inc(x_130); -x_131 = lean_ctor_get(x_22, 2); -lean_inc(x_131); -lean_dec(x_22); -x_132 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); -if (lean_is_scalar(x_129)) { - x_133 = lean_alloc_ctor(0, 2, 0); +x_251 = lean_box(0); +if (lean_is_scalar(x_250)) { + x_252 = lean_alloc_ctor(0, 2, 0); } else { - x_133 = x_129; + x_252 = x_250; } -lean_ctor_set(x_133, 0, x_132); -lean_ctor_set(x_133, 1, x_128); -return x_133; +lean_ctor_set(x_252, 0, x_251); +lean_ctor_set(x_252, 1, x_249); +return x_252; } } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Elab_Term_levelMVarToParam___lambda__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5(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) { _start: { -lean_object* x_11; -x_11 = l_Lean_Elab_Term_levelMVarToParam(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_7, 5); +lean_inc(x_10); +x_11 = l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_10); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam_x27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__1() { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_11 = lean_st_ref_get(x_9, x_10); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_st_ref_get(x_3, x_12); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l_Lean_Elab_Term_levelMVarToParam(x_1, x_14, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_15); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); -lean_dec(x_17); -x_21 = lean_st_ref_get(x_9, x_18); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_st_ref_set(x_3, x_20, x_22); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) -{ -lean_object* x_25; -x_25 = lean_ctor_get(x_23, 0); -lean_dec(x_25); -lean_ctor_set(x_23, 0, x_19); -return x_23; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("internal exception: ", 20); +return x_1; } -else -{ -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_dec(x_23); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_19); -lean_ctor_set(x_27, 1, x_26); -return x_27; } +static lean_object* _init_l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_levelMVarToParam_x27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_11; -x_11 = l_Lean_Elab_Term_levelMVarToParam_x27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_1, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_1, 1); +lean_inc(x_10); +lean_dec(x_1); +x_11 = 2; +x_12 = l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4(x_9, x_10, x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -return x_11; +lean_dec(x_2); +lean_dec(x_9); +return x_12; } +else +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_1); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_1, 0); +x_15 = lean_ctor_get(x_1, 1); +lean_dec(x_15); +x_16 = l_Lean_Elab_isAbortExceptionId(x_14); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_st_ref_get(x_7, x_8); +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_ctor_get(x_6, 5); +lean_inc(x_19); +x_20 = l_Lean_InternalExceptionId_getName(x_14, x_18); +lean_dec(x_14); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; +lean_dec(x_19); +lean_free_object(x_1); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_23, 0, x_21); +x_24 = l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2; +x_25 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +x_26 = l_Lean_logTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__1___closed__5; +x_27 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_28 = 2; +x_29 = l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5(x_27, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_22); +return x_29; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); +uint8_t x_30; +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -x_7 = l_Lean_addMacroScope(x_2, x_3, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; -} +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_30 = !lean_is_exclusive(x_20); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_20, 0); +x_32 = lean_io_error_to_string(x_31); +x_33 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_33, 0, x_32); +x_34 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set_tag(x_1, 0); +lean_ctor_set(x_1, 1, x_34); +lean_ctor_set(x_1, 0, x_19); +lean_ctor_set(x_20, 0, x_1); +return x_20; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -lean_dec(x_1); -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__1), 4, 3); -lean_closure_set(x_7, 0, x_2); -lean_closure_set(x_7, 1, x_5); -lean_closure_set(x_7, 2, x_3); -x_8 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_6, x_7); -return x_8; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_35 = lean_ctor_get(x_20, 0); +x_36 = lean_ctor_get(x_20, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_20); +x_37 = lean_io_error_to_string(x_35); +x_38 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set_tag(x_1, 0); +lean_ctor_set(x_1, 1, x_39); +lean_ctor_set(x_1, 0, x_19); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_1); +lean_ctor_set(x_40, 1, x_36); +return x_40; } } -static lean_object* _init_l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__1() { -_start: +} +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("x", 1); -return x_1; +lean_object* x_41; lean_object* x_42; +lean_free_object(x_1); +lean_dec(x_14); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_41 = lean_box(0); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_8); +return x_42; } } -static lean_object* _init_l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +lean_object* x_43; uint8_t x_44; +x_43 = lean_ctor_get(x_1, 0); +lean_inc(x_43); +lean_dec(x_1); +x_44 = l_Lean_Elab_isAbortExceptionId(x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_45 = lean_st_ref_get(x_7, x_8); +x_46 = lean_ctor_get(x_45, 1); +lean_inc(x_46); +lean_dec(x_45); +x_47 = lean_ctor_get(x_6, 5); +lean_inc(x_47); +x_48 = l_Lean_InternalExceptionId_getName(x_43, x_46); +lean_dec(x_43); +if (lean_obj_tag(x_48) == 0) +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; +lean_dec(x_47); +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_51, 0, x_49); +x_52 = l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2; +x_53 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +x_54 = l_Lean_logTrace___at_Lean_Elab_Term_traceAtCmdPos___spec__1___closed__5; +x_55 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +x_56 = 2; +x_57 = l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5(x_55, x_56, x_2, x_3, x_4, x_5, x_6, x_7, x_50); +return x_57; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___rarg(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_3 = lean_ctor_get(x_2, 3); -lean_inc(x_3); -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -x_5 = lean_ctor_get(x_2, 2); -lean_inc(x_5); -x_6 = l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__2; -lean_inc(x_4); -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshBinderName___rarg___lambda__2), 5, 4); -lean_closure_set(x_7, 0, x_2); -lean_closure_set(x_7, 1, x_1); -lean_closure_set(x_7, 2, x_6); -lean_closure_set(x_7, 3, x_4); -x_8 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_5, x_7); -x_9 = lean_apply_2(x_3, lean_box(0), x_8); -return x_9; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_58 = lean_ctor_get(x_48, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_48, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_60 = x_48; +} else { + lean_dec_ref(x_48); + x_60 = lean_box(0); } +x_61 = lean_io_error_to_string(x_58); +x_62 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_62, 0, x_61); +x_63 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_63, 0, x_62); +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_47); +lean_ctor_set(x_64, 1, x_63); +if (lean_is_scalar(x_60)) { + x_65 = lean_alloc_ctor(1, 2, 0); +} else { + x_65 = x_60; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshBinderName___rarg), 2, 0); -return x_2; +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_59); +return x_65; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); +lean_object* x_66; lean_object* x_67; +lean_dec(x_43); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -x_6 = l_Lean_mkIdentFrom(x_2, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; -} +lean_dec(x_3); +lean_dec(x_2); +x_66 = lean_box(0); +x_67 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_8); +return x_67; } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -lean_inc(x_1); -x_5 = l_Lean_Elab_Term_mkFreshBinderName___rarg(x_1, x_2); -x_6 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshIdent___rarg___lambda__1), 3, 2); -lean_closure_set(x_6, 0, x_1); -lean_closure_set(x_6, 1, x_3); -x_7 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_5, x_6); -return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshIdent(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_mkFreshIdent___rarg), 3, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Elab_withLogging___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_9 = lean_ctor_get(x_6, 5); -x_10 = lean_ctor_get(x_2, 2); -lean_inc(x_10); -lean_inc(x_10); -x_11 = l_Lean_Elab_getBetterRef(x_9, x_10); -x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_4, x_5, x_6, x_7, x_8); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_13, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_14); +lean_object* x_9; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_9 = lean_apply_7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) +{ +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_10); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_11); -lean_ctor_set(x_18, 1, x_17); -lean_ctor_set_tag(x_15, 1); -lean_ctor_set(x_15, 0, x_18); -return x_15; +return x_9; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_15, 0); -x_20 = lean_ctor_get(x_15, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_15); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_11); -lean_ctor_set(x_21, 1, x_19); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3(x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_11); +return x_12; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___closed__1() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +lean_object* x_12; uint8_t x_13; +x_12 = lean_st_ref_get(x_10, x_11); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) { -uint8_t x_14; -x_14 = lean_usize_dec_lt(x_5, x_4); -if (x_14 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); +x_18 = l_Lean_getAttributeImpl(x_16, x_17); +lean_dec(x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_15; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_7); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +lean_free_object(x_12); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_6); -lean_ctor_set(x_15, 1, x_13); -return x_15; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_20, 0, x_19); +x_21 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_21, 0, x_20); +x_22 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +return x_22; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; 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_dec(x_8); +lean_dec(x_7); lean_dec(x_6); -x_16 = lean_array_uget(x_3, x_5); -x_24 = lean_st_ref_get(x_12, x_13); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_ctor_get(x_25, 0); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_ctor_get(x_16, 0); -lean_inc(x_28); -x_29 = l_Lean_getAttributeImpl(x_27, x_28); -lean_dec(x_27); -if (lean_obj_tag(x_29) == 0) +lean_dec(x_5); +if (lean_obj_tag(x_2) == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -lean_dec(x_16); -lean_dec(x_2); +lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; +lean_free_object(x_12); +x_23 = lean_ctor_get(x_18, 0); +lean_inc(x_23); +lean_dec(x_18); +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +x_25 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); lean_dec(x_1); -x_30 = lean_ctor_get(x_29, 0); +x_26 = lean_box(x_25); +x_27 = lean_apply_6(x_24, x_3, x_4, x_26, x_9, x_10, x_15); +return x_27; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; uint8_t x_32; uint8_t x_33; +x_28 = lean_ctor_get(x_18, 0); +lean_inc(x_28); +lean_dec(x_18); +x_29 = lean_ctor_get(x_2, 0); +lean_inc(x_29); +lean_dec(x_2); +x_30 = lean_ctor_get(x_28, 0); lean_inc(x_30); +x_31 = lean_ctor_get_uint8(x_30, sizeof(void*)*2); +lean_dec(x_30); +x_32 = lean_unbox(x_29); lean_dec(x_29); -x_31 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_31, 0, x_30); -x_32 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_26); -lean_dec(x_12); -lean_dec(x_11); -x_34 = !lean_is_exclusive(x_33); -if (x_34 == 0) +x_33 = l___private_Lean_Attributes_0__Lean_beqAttributeApplicationTime____x40_Lean_Attributes___hyg_15_(x_32, x_31); +if (x_33 == 0) { -return x_33; +lean_object* x_34; +lean_dec(x_28); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_34 = lean_box(0); +lean_ctor_set(x_12, 0, x_34); +return x_12; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_33, 0); -x_36 = lean_ctor_get(x_33, 1); -lean_inc(x_36); +lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; +lean_free_object(x_12); +x_35 = lean_ctor_get(x_28, 1); lean_inc(x_35); -lean_dec(x_33); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_dec(x_28); +x_36 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +lean_dec(x_1); +x_37 = lean_box(x_36); +x_38 = lean_apply_6(x_35, x_3, x_4, x_37, x_9, x_10, x_15); +return x_38; +} +} } } else { -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; -x_38 = lean_ctor_get(x_29, 0); -lean_inc(x_38); -lean_dec(x_29); -x_39 = lean_ctor_get(x_38, 1); -lean_inc(x_39); -lean_dec(x_38); -x_40 = lean_ctor_get(x_16, 1); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_39 = lean_ctor_get(x_12, 0); +x_40 = lean_ctor_get(x_12, 1); lean_inc(x_40); -x_41 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); -lean_dec(x_16); -x_42 = lean_box(x_41); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_1); -x_43 = lean_apply_6(x_39, x_1, x_40, x_42, x_11, x_12, x_26); +lean_inc(x_39); +lean_dec(x_12); +x_41 = lean_ctor_get(x_39, 0); +lean_inc(x_41); +lean_dec(x_39); +x_42 = lean_ctor_get(x_1, 0); +lean_inc(x_42); +x_43 = l_Lean_getAttributeImpl(x_41, x_42); +lean_dec(x_41); if (lean_obj_tag(x_43) == 0) { -lean_object* x_44; lean_object* x_45; -x_44 = lean_ctor_get(x_43, 1); +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_44 = lean_ctor_get(x_43, 0); lean_inc(x_44); lean_dec(x_43); -x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___closed__1; -x_17 = x_45; -x_18 = x_44; -goto block_23; +x_45 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_46 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_46, x_5, x_6, x_7, x_8, x_9, x_10, x_40); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +return x_47; } else { -uint8_t x_46; -lean_dec(x_12); -lean_dec(x_11); +lean_dec(x_8); lean_dec(x_7); -lean_dec(x_1); -x_46 = !lean_is_exclusive(x_43); -if (x_46 == 0) +lean_dec(x_6); +lean_dec(x_5); +if (lean_obj_tag(x_2) == 0) { -return x_43; +lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; +x_48 = lean_ctor_get(x_43, 0); +lean_inc(x_48); +lean_dec(x_43); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +lean_dec(x_1); +x_51 = lean_box(x_50); +x_52 = lean_apply_6(x_49, x_3, x_4, x_51, x_9, x_10, x_40); +return x_52; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_43, 0); -x_48 = lean_ctor_get(x_43, 1); -lean_inc(x_48); -lean_inc(x_47); +lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; uint8_t x_57; uint8_t x_58; +x_53 = lean_ctor_get(x_43, 0); +lean_inc(x_53); lean_dec(x_43); -x_49 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); -return x_49; +x_54 = lean_ctor_get(x_2, 0); +lean_inc(x_54); +lean_dec(x_2); +x_55 = lean_ctor_get(x_53, 0); +lean_inc(x_55); +x_56 = lean_ctor_get_uint8(x_55, sizeof(void*)*2); +lean_dec(x_55); +x_57 = lean_unbox(x_54); +lean_dec(x_54); +x_58 = l___private_Lean_Attributes_0__Lean_beqAttributeApplicationTime____x40_Lean_Attributes___hyg_15_(x_57, x_56); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; +lean_dec(x_53); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_59 = lean_box(0); +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_40); +return x_60; +} +else +{ +lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; +x_61 = lean_ctor_get(x_53, 1); +lean_inc(x_61); +lean_dec(x_53); +x_62 = lean_ctor_get_uint8(x_1, sizeof(void*)*2); +lean_dec(x_1); +x_63 = lean_box(x_62); +x_64 = lean_apply_6(x_61, x_3, x_4, x_63, x_9, x_10, x_40); +return x_64; } } } -else +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; uint8_t x_54; uint8_t x_55; -x_50 = lean_ctor_get(x_29, 0); -lean_inc(x_50); -lean_dec(x_29); -x_51 = lean_ctor_get(x_2, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 0); -lean_inc(x_52); -x_53 = lean_ctor_get_uint8(x_52, sizeof(void*)*2); -lean_dec(x_52); -x_54 = lean_unbox(x_51); -lean_dec(x_51); -x_55 = l___private_Lean_Attributes_0__Lean_beqAttributeApplicationTime____x40_Lean_Attributes___hyg_15_(x_54, x_53); -if (x_55 == 0) +uint8_t x_14; +x_14 = lean_usize_dec_lt(x_5, x_4); +if (x_14 == 0) { -lean_object* x_56; -lean_dec(x_50); -lean_dec(x_16); -x_56 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___closed__1; -x_17 = x_56; -x_18 = x_26; -goto block_23; +lean_object* x_15; +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_6); +lean_ctor_set(x_15, 1, x_13); +return x_15; } else { -lean_object* x_57; lean_object* x_58; uint8_t x_59; lean_object* x_60; lean_object* x_61; -x_57 = lean_ctor_get(x_50, 1); -lean_inc(x_57); -lean_dec(x_50); -x_58 = lean_ctor_get(x_16, 1); -lean_inc(x_58); -x_59 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); -lean_dec(x_16); -x_60 = lean_box(x_59); -lean_inc(x_12); -lean_inc(x_11); +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_dec(x_6); +x_16 = lean_array_uget(x_3, x_5); +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_inc(x_17); lean_inc(x_1); -x_61 = lean_apply_6(x_57, x_1, x_58, x_60, x_11, x_12, x_26); -if (lean_obj_tag(x_61) == 0) +lean_inc(x_2); +x_18 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6___lambda__1), 11, 4); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_2); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_17); +x_19 = lean_ctor_get(x_11, 0); +x_20 = lean_ctor_get(x_11, 1); +x_21 = lean_ctor_get(x_11, 2); +x_22 = lean_ctor_get(x_11, 3); +x_23 = lean_ctor_get(x_11, 4); +x_24 = lean_ctor_get(x_11, 5); +x_25 = lean_ctor_get(x_11, 6); +x_26 = lean_ctor_get(x_11, 7); +x_27 = lean_ctor_get(x_11, 8); +x_28 = lean_ctor_get(x_11, 9); +x_29 = lean_ctor_get(x_11, 10); +x_30 = l_Lean_replaceRef(x_17, x_24); +lean_dec(x_17); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_23); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +x_31 = lean_alloc_ctor(0, 11, 0); +lean_ctor_set(x_31, 0, x_19); +lean_ctor_set(x_31, 1, x_20); +lean_ctor_set(x_31, 2, x_21); +lean_ctor_set(x_31, 3, x_22); +lean_ctor_set(x_31, 4, x_23); +lean_ctor_set(x_31, 5, x_30); +lean_ctor_set(x_31, 6, x_25); +lean_ctor_set(x_31, 7, x_26); +lean_ctor_set(x_31, 8, x_27); +lean_ctor_set(x_31, 9, x_28); +lean_ctor_set(x_31, 10, x_29); +lean_inc(x_12); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_32 = l_Lean_Elab_withLogging___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(x_18, x_7, x_8, x_9, x_10, x_31, x_12, x_13); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_62; lean_object* x_63; -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___closed__1; -x_17 = x_63; -x_18 = x_62; -goto block_23; +lean_object* x_33; size_t x_34; size_t x_35; lean_object* x_36; +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = 1; +x_35 = lean_usize_add(x_5, x_34); +x_36 = lean_box(0); +x_5 = x_35; +x_6 = x_36; +x_13 = x_33; +goto _start; } else { -uint8_t x_64; +uint8_t x_38; lean_dec(x_12); -lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -x_64 = !lean_is_exclusive(x_61); -if (x_64 == 0) +x_38 = !lean_is_exclusive(x_32); +if (x_38 == 0) { -return x_61; +return x_32; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_61, 0); -x_66 = lean_ctor_get(x_61, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_61); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -return x_67; -} -} -} -} +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_32, 0); +x_40 = lean_ctor_get(x_32, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_32); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; } -block_23: -{ -lean_object* x_19; size_t x_20; size_t x_21; -x_19 = lean_ctor_get(x_17, 0); -lean_inc(x_19); -lean_dec(x_17); -x_20 = 1; -x_21 = lean_usize_add(x_5, x_20); -x_5 = x_21; -x_6 = x_19; -x_13 = x_18; -goto _start; } } } @@ -20884,7 +24717,7 @@ x_12 = lean_usize_of_nat(x_11); lean_dec(x_11); x_13 = 0; x_14 = lean_box(0); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(x_1, x_3, x_2, x_12, x_13, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6(x_1, x_3, x_2, x_12, x_13, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); if (lean_obj_tag(x_15) == 0) { uint8_t x_16; @@ -20946,7 +24779,34 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_3); +lean_dec(x_3); +x_12 = l_Lean_logAt___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__4(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; lean_object* x_11; +x_10 = lean_unbox(x_2); +lean_dec(x_2); +x_11 = l_Lean_log___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__5(x_1, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { size_t x_14; size_t x_15; lean_object* x_16; @@ -20954,10 +24814,8 @@ x_14 = lean_unbox_usize(x_4); lean_dec(x_4); x_15 = lean_unbox_usize(x_5); lean_dec(x_5); -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__6(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_11); lean_dec(x_3); return x_16; } @@ -20967,9 +24825,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttri { lean_object* x_11; x_11 = l___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_8); lean_dec(x_2); return x_11; } @@ -20992,9 +24848,7 @@ uint8_t x_11; lean_object* x_12; x_11 = lean_unbox(x_3); lean_dec(x_3); x_12 = l_Lean_Elab_Term_applyAttributesAt(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_dec(x_8); lean_dec(x_2); return x_12; } @@ -21013,9 +24867,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_applyAttributes___boxed(lean_object* x { lean_object* x_10; x_10 = l_Lean_Elab_Term_applyAttributes(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_7); lean_dec(x_2); return x_10; } @@ -25294,7 +29146,7 @@ lean_dec(x_3); return x_12; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__1() { _start: { lean_object* x_1; @@ -25302,17 +29154,17 @@ x_1 = lean_mk_string_from_bytes("autoLift", 8); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__3() { _start: { lean_object* x_1; @@ -25320,13 +29172,13 @@ x_1 = lean_mk_string_from_bytes("insert monadic lifts (i.e., `liftM` and coercio return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__4() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 1; x_2 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__3; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__3; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -25335,17 +29187,17 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__2; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__4; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__2; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__4; x_4 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_1); return x_4; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__1() { _start: { lean_object* x_1; @@ -25353,17 +29205,17 @@ x_1 = lean_mk_string_from_bytes("maxCoeSize", 10); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__3() { _start: { lean_object* x_1; @@ -25371,13 +29223,13 @@ x_1 = lean_mk_string_from_bytes("maximum number of instances used to construct a return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_unsigned_to_nat(16u); x_2 = l_Lean_Elab_ContextInfo_saveNoFileMap___at_Lean_Elab_Term_withoutModifyingElabMetaStateWithInfo___spec__4___rarg___closed__1; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__3; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__3; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -25385,12 +29237,12 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__2; -x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__4; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__2; +x_3 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__4; x_4 = l_Lean_Option_register___at_Lean_initFn____x40_Lean_Util_RecDepth___hyg_6____spec__1(x_2, x_3, x_1); return x_4; } @@ -30822,23 +34674,6 @@ lean_dec(x_2); return x_9; } } -static lean_object* _init_l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("internal exception: ", 20); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { @@ -30895,7 +34730,7 @@ lean_inc(x_22); lean_dec(x_20); x_23 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_23, 0, x_21); -x_24 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__2; +x_24 = l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2; x_25 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_23); @@ -31002,7 +34837,7 @@ lean_inc(x_50); lean_dec(x_48); x_51 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_51, 0, x_49); -x_52 = l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__2; +x_52 = l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2; x_53 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_53, 0, x_52); lean_ctor_set(x_53, 1, x_51); @@ -32355,13 +36190,44 @@ lean_dec(x_3); return x_11; } } -LEAN_EXPORT uint8_t l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Elab_Term_getSyntheticMVarDecl_x3f___spec__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; uint8_t x_4; -x_3 = lean_ctor_get(x_2, 0); -x_4 = lean_name_eq(x_3, x_1); -return x_4; +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_4 = lean_ctor_get(x_1, 0); +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_1, 2); +x_7 = lean_ctor_get(x_1, 3); +x_8 = l_Lean_Name_quickCmp(x_2, x_5); +switch (x_8) { +case 0: +{ +x_1 = x_4; +goto _start; +} +case 1: +{ +lean_object* x_10; +lean_inc(x_6); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_6); +return x_10; +} +default: +{ +x_1 = x_7; +goto _start; +} +} +} } } LEAN_EXPORT lean_object* l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { @@ -32376,47 +36242,44 @@ x_11 = lean_st_ref_get(x_3, x_10); x_12 = !lean_is_exclusive(x_11); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_13; lean_object* x_14; lean_object* x_15; x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_alloc_closure((void*)(l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___lambda__1___boxed), 2, 1); -lean_closure_set(x_14, 0, x_1); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); lean_dec(x_13); -x_16 = l_List_find_x3f___rarg(x_14, x_15); -lean_ctor_set(x_11, 0, x_16); +x_15 = l_Std_RBNode_find___at_Lean_Elab_Term_getSyntheticMVarDecl_x3f___spec__1(x_14, x_1); +lean_dec(x_14); +lean_ctor_set(x_11, 0, x_15); return x_11; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_11, 0); -x_18 = lean_ctor_get(x_11, 1); -lean_inc(x_18); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_11, 0); +x_17 = lean_ctor_get(x_11, 1); lean_inc(x_17); +lean_inc(x_16); lean_dec(x_11); -x_19 = lean_alloc_closure((void*)(l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___lambda__1___boxed), 2, 1); -lean_closure_set(x_19, 0, x_1); -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); -lean_dec(x_17); -x_21 = l_List_find_x3f___rarg(x_19, x_20); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_18); -return x_22; +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Std_RBNode_find___at_Lean_Elab_Term_getSyntheticMVarDecl_x3f___spec__1(x_18, x_1); +lean_dec(x_18); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_17); +return x_20; } } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Elab_Term_getSyntheticMVarDecl_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___lambda__1(x_1, x_2); +lean_object* x_3; +x_3 = l_Std_RBNode_find___at_Lean_Elab_Term_getSyntheticMVarDecl_x3f___spec__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +return x_3; } } LEAN_EXPORT lean_object* l_Lean_Elab_Term_getSyntheticMVarDecl_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { @@ -32430,6 +36293,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); return x_9; } } @@ -32515,16 +36379,12 @@ if (lean_obj_tag(x_1) == 2) { lean_object* x_9; lean_object* x_10; lean_object* x_11; x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -lean_dec(x_1); -lean_inc(x_9); x_10 = l_Lean_Elab_Term_getSyntheticMVarDecl_x3f(x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); if (lean_obj_tag(x_11) == 0) { uint8_t x_12; -lean_dec(x_9); x_12 = !lean_is_exclusive(x_10); if (x_12 == 0) { @@ -32556,7 +36416,7 @@ if (x_18 == 0) { lean_object* x_19; lean_object* x_20; x_19 = lean_ctor_get(x_11, 0); -x_20 = lean_ctor_get(x_19, 2); +x_20 = lean_ctor_get(x_19, 1); lean_inc(x_20); lean_dec(x_19); switch (lean_obj_tag(x_20)) { @@ -32570,6 +36430,7 @@ if (x_21 == 0) lean_object* x_22; x_22 = lean_ctor_get(x_10, 0); lean_dec(x_22); +lean_inc(x_9); lean_ctor_set(x_11, 0, x_9); return x_10; } @@ -32579,6 +36440,7 @@ lean_object* x_23; lean_object* x_24; x_23 = lean_ctor_get(x_10, 1); lean_inc(x_23); lean_dec(x_10); +lean_inc(x_9); lean_ctor_set(x_11, 0, x_9); x_24 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_24, 0, x_11); @@ -32596,6 +36458,7 @@ if (x_25 == 0) lean_object* x_26; x_26 = lean_ctor_get(x_10, 0); lean_dec(x_26); +lean_inc(x_9); lean_ctor_set(x_11, 0, x_9); return x_10; } @@ -32605,6 +36468,7 @@ lean_object* x_27; lean_object* x_28; x_27 = lean_ctor_get(x_10, 1); lean_inc(x_27); lean_dec(x_10); +lean_inc(x_9); lean_ctor_set(x_11, 0, x_9); x_28 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_28, 0, x_11); @@ -32617,7 +36481,6 @@ return x_28; uint8_t x_29; lean_dec(x_20); lean_free_object(x_11); -lean_dec(x_9); x_29 = !lean_is_exclusive(x_10); if (x_29 == 0) { @@ -32649,7 +36512,7 @@ lean_object* x_35; lean_object* x_36; x_35 = lean_ctor_get(x_11, 0); lean_inc(x_35); lean_dec(x_11); -x_36 = lean_ctor_get(x_35, 2); +x_36 = lean_ctor_get(x_35, 1); lean_inc(x_36); lean_dec(x_35); switch (lean_obj_tag(x_36)) { @@ -32667,6 +36530,7 @@ if (lean_is_exclusive(x_10)) { lean_dec_ref(x_10); x_38 = lean_box(0); } +lean_inc(x_9); x_39 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_39, 0, x_9); if (lean_is_scalar(x_38)) { @@ -32692,6 +36556,7 @@ if (lean_is_exclusive(x_10)) { lean_dec_ref(x_10); x_42 = lean_box(0); } +lean_inc(x_9); x_43 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_43, 0, x_9); if (lean_is_scalar(x_42)) { @@ -32707,7 +36572,6 @@ return x_44; { lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_dec(x_36); -lean_dec(x_9); x_45 = lean_ctor_get(x_10, 1); lean_inc(x_45); if (lean_is_exclusive(x_10)) { @@ -32735,7 +36599,6 @@ return x_48; else { lean_object* x_49; lean_object* x_50; -lean_dec(x_1); x_49 = lean_box(0); x_50 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_50, 0, x_49); @@ -32755,6 +36618,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); return x_9; } } @@ -32762,7 +36626,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkTermInfo(lean_object* x_1, lean_obje _start: { lean_object* x_14; lean_object* x_15; -lean_inc(x_3); x_14 = l_Lean_Elab_Term_isTacticOrPostponedHole_x3f(x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); @@ -32954,7 +36817,7 @@ lean_dec(x_23); x_25 = lean_st_ref_get(x_4, x_24); x_26 = lean_ctor_get(x_25, 0); lean_inc(x_26); -x_27 = lean_ctor_get(x_26, 4); +x_27 = lean_ctor_get(x_26, 5); lean_inc(x_27); lean_dec(x_26); x_28 = lean_ctor_get_uint8(x_27, sizeof(void*)*2); @@ -33016,7 +36879,7 @@ lean_dec(x_41); x_43 = lean_st_ref_take(x_4, x_42); x_44 = lean_ctor_get(x_43, 0); lean_inc(x_44); -x_45 = lean_ctor_get(x_44, 4); +x_45 = lean_ctor_get(x_44, 5); lean_inc(x_45); if (lean_obj_tag(x_39) == 0) { @@ -33028,7 +36891,7 @@ x_47 = !lean_is_exclusive(x_44); if (x_47 == 0) { lean_object* x_48; uint8_t x_49; -x_48 = lean_ctor_get(x_44, 4); +x_48 = lean_ctor_get(x_44, 5); lean_dec(x_48); x_49 = !lean_is_exclusive(x_45); if (x_49 == 0) @@ -33096,7 +36959,7 @@ x_69 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_69, 0, x_64); lean_ctor_set(x_69, 1, x_68); lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_63); -lean_ctor_set(x_44, 4, x_69); +lean_ctor_set(x_44, 5, x_69); x_70 = lean_st_ref_set(x_4, x_44, x_46); lean_dec(x_4); x_71 = lean_ctor_get(x_70, 1); @@ -33126,439 +36989,448 @@ goto block_22; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_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_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; x_76 = lean_ctor_get(x_44, 0); x_77 = lean_ctor_get(x_44, 1); x_78 = lean_ctor_get(x_44, 2); x_79 = lean_ctor_get(x_44, 3); +x_80 = lean_ctor_get(x_44, 4); +lean_inc(x_80); lean_inc(x_79); lean_inc(x_78); lean_inc(x_77); lean_inc(x_76); lean_dec(x_44); -x_80 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); -x_81 = lean_ctor_get(x_45, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_45, 1); +x_81 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); +x_82 = lean_ctor_get(x_45, 0); lean_inc(x_82); +x_83 = lean_ctor_get(x_45, 1); +lean_inc(x_83); if (lean_is_exclusive(x_45)) { lean_ctor_release(x_45, 0); lean_ctor_release(x_45, 1); - x_83 = x_45; + x_84 = x_45; } else { lean_dec_ref(x_45); - x_83 = lean_box(0); + x_84 = lean_box(0); } -x_84 = lean_ctor_get(x_39, 0); -lean_inc(x_84); +x_85 = lean_ctor_get(x_39, 0); +lean_inc(x_85); lean_dec(x_39); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_84); -lean_ctor_set(x_85, 1, x_82); -x_86 = l_Std_PersistentArray_push___rarg(x_33, x_85); -if (lean_is_scalar(x_83)) { - x_87 = lean_alloc_ctor(0, 2, 1); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_83); +x_87 = l_Std_PersistentArray_push___rarg(x_33, x_86); +if (lean_is_scalar(x_84)) { + x_88 = lean_alloc_ctor(0, 2, 1); } else { - x_87 = x_83; + x_88 = x_84; } -lean_ctor_set(x_87, 0, x_81); -lean_ctor_set(x_87, 1, x_86); -lean_ctor_set_uint8(x_87, sizeof(void*)*2, x_80); -x_88 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_88, 0, x_76); -lean_ctor_set(x_88, 1, x_77); -lean_ctor_set(x_88, 2, x_78); -lean_ctor_set(x_88, 3, x_79); -lean_ctor_set(x_88, 4, x_87); -x_89 = lean_st_ref_set(x_4, x_88, x_46); +lean_ctor_set(x_88, 0, x_82); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set_uint8(x_88, sizeof(void*)*2, x_81); +x_89 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_89, 0, x_76); +lean_ctor_set(x_89, 1, x_77); +lean_ctor_set(x_89, 2, x_78); +lean_ctor_set(x_89, 3, x_79); +lean_ctor_set(x_89, 4, x_80); +lean_ctor_set(x_89, 5, x_88); +x_90 = lean_st_ref_set(x_4, x_89, x_46); lean_dec(x_4); -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_91 = x_89; +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_90)) { + lean_ctor_release(x_90, 0); + lean_ctor_release(x_90, 1); + x_92 = x_90; } else { - lean_dec_ref(x_89); - x_91 = lean_box(0); + lean_dec_ref(x_90); + x_92 = lean_box(0); } -x_92 = lean_box(0); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_36); -lean_ctor_set(x_93, 1, x_92); -if (lean_is_scalar(x_91)) { - x_94 = lean_alloc_ctor(0, 2, 0); +x_93 = lean_box(0); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_36); +lean_ctor_set(x_94, 1, x_93); +if (lean_is_scalar(x_92)) { + x_95 = lean_alloc_ctor(0, 2, 0); } else { - x_94 = x_91; + x_95 = x_92; } -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_90); -x_10 = x_94; +lean_ctor_set(x_95, 0, x_94); +lean_ctor_set(x_95, 1, x_91); +x_10 = x_95; goto block_22; } } else { -lean_object* x_95; uint8_t x_96; -x_95 = lean_ctor_get(x_43, 1); -lean_inc(x_95); +lean_object* x_96; uint8_t x_97; +x_96 = lean_ctor_get(x_43, 1); +lean_inc(x_96); lean_dec(x_43); -x_96 = !lean_is_exclusive(x_44); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_44); +if (x_97 == 0) { -lean_object* x_97; uint8_t x_98; -x_97 = lean_ctor_get(x_44, 4); -lean_dec(x_97); -x_98 = !lean_is_exclusive(x_45); -if (x_98 == 0) +lean_object* x_98; uint8_t x_99; +x_98 = lean_ctor_get(x_44, 5); +lean_dec(x_98); +x_99 = !lean_is_exclusive(x_45); +if (x_99 == 0) { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; -x_99 = lean_ctor_get(x_45, 1); -lean_dec(x_99); -x_100 = lean_ctor_get(x_39, 0); -lean_inc(x_100); +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; +x_100 = lean_ctor_get(x_45, 1); +lean_dec(x_100); +x_101 = lean_ctor_get(x_39, 0); +lean_inc(x_101); lean_dec(x_39); -x_101 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_101, 0, x_100); -x_102 = l_Std_PersistentArray_push___rarg(x_33, x_101); -lean_ctor_set(x_45, 1, x_102); -x_103 = lean_st_ref_set(x_4, x_44, x_95); +x_102 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_102, 0, x_101); +x_103 = l_Std_PersistentArray_push___rarg(x_33, x_102); +lean_ctor_set(x_45, 1, x_103); +x_104 = lean_st_ref_set(x_4, x_44, x_96); lean_dec(x_4); -x_104 = !lean_is_exclusive(x_103); -if (x_104 == 0) +x_105 = !lean_is_exclusive(x_104); +if (x_105 == 0) { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_103, 0); -lean_dec(x_105); -x_106 = lean_box(0); -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_36); -lean_ctor_set(x_107, 1, x_106); -lean_ctor_set(x_103, 0, x_107); -x_10 = x_103; +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_104, 0); +lean_dec(x_106); +x_107 = lean_box(0); +x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_108, 0, x_36); +lean_ctor_set(x_108, 1, x_107); +lean_ctor_set(x_104, 0, x_108); +x_10 = x_104; goto block_22; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_108 = lean_ctor_get(x_103, 1); -lean_inc(x_108); -lean_dec(x_103); -x_109 = lean_box(0); -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_36); -lean_ctor_set(x_110, 1, x_109); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_109 = lean_ctor_get(x_104, 1); +lean_inc(x_109); +lean_dec(x_104); +x_110 = lean_box(0); x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_108); -x_10 = x_111; +lean_ctor_set(x_111, 0, x_36); +lean_ctor_set(x_111, 1, x_110); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_109); +x_10 = x_112; goto block_22; } } else { -uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_112 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); -x_113 = lean_ctor_get(x_45, 0); -lean_inc(x_113); -lean_dec(x_45); -x_114 = lean_ctor_get(x_39, 0); +uint8_t x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_113 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); +x_114 = lean_ctor_get(x_45, 0); lean_inc(x_114); +lean_dec(x_45); +x_115 = lean_ctor_get(x_39, 0); +lean_inc(x_115); lean_dec(x_39); -x_115 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_115, 0, x_114); -x_116 = l_Std_PersistentArray_push___rarg(x_33, x_115); -x_117 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_117, 0, x_113); -lean_ctor_set(x_117, 1, x_116); -lean_ctor_set_uint8(x_117, sizeof(void*)*2, x_112); -lean_ctor_set(x_44, 4, x_117); -x_118 = lean_st_ref_set(x_4, x_44, x_95); +x_116 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_116, 0, x_115); +x_117 = l_Std_PersistentArray_push___rarg(x_33, x_116); +x_118 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_118, 0, x_114); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_113); +lean_ctor_set(x_44, 5, x_118); +x_119 = lean_st_ref_set(x_4, x_44, x_96); lean_dec(x_4); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; +x_120 = lean_ctor_get(x_119, 1); +lean_inc(x_120); +if (lean_is_exclusive(x_119)) { + lean_ctor_release(x_119, 0); + lean_ctor_release(x_119, 1); + x_121 = x_119; } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + lean_dec_ref(x_119); + x_121 = lean_box(0); } -x_121 = lean_box(0); -x_122 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_122, 0, x_36); -lean_ctor_set(x_122, 1, x_121); -if (lean_is_scalar(x_120)) { - x_123 = lean_alloc_ctor(0, 2, 0); +x_122 = lean_box(0); +x_123 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_123, 0, x_36); +lean_ctor_set(x_123, 1, x_122); +if (lean_is_scalar(x_121)) { + x_124 = lean_alloc_ctor(0, 2, 0); } else { - x_123 = x_120; + x_124 = x_121; } -lean_ctor_set(x_123, 0, x_122); -lean_ctor_set(x_123, 1, x_119); -x_10 = x_123; +lean_ctor_set(x_124, 0, x_123); +lean_ctor_set(x_124, 1, x_120); +x_10 = x_124; goto block_22; } } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; -x_124 = lean_ctor_get(x_44, 0); -x_125 = lean_ctor_get(x_44, 1); -x_126 = lean_ctor_get(x_44, 2); -x_127 = lean_ctor_get(x_44, 3); +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; uint8_t x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; +x_125 = lean_ctor_get(x_44, 0); +x_126 = lean_ctor_get(x_44, 1); +x_127 = lean_ctor_get(x_44, 2); +x_128 = lean_ctor_get(x_44, 3); +x_129 = lean_ctor_get(x_44, 4); +lean_inc(x_129); +lean_inc(x_128); lean_inc(x_127); lean_inc(x_126); lean_inc(x_125); -lean_inc(x_124); lean_dec(x_44); -x_128 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); -x_129 = lean_ctor_get(x_45, 0); -lean_inc(x_129); +x_130 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); +x_131 = lean_ctor_get(x_45, 0); +lean_inc(x_131); if (lean_is_exclusive(x_45)) { lean_ctor_release(x_45, 0); lean_ctor_release(x_45, 1); - x_130 = x_45; + x_132 = x_45; } else { lean_dec_ref(x_45); - x_130 = lean_box(0); + x_132 = lean_box(0); } -x_131 = lean_ctor_get(x_39, 0); -lean_inc(x_131); +x_133 = lean_ctor_get(x_39, 0); +lean_inc(x_133); lean_dec(x_39); -x_132 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_132, 0, x_131); -x_133 = l_Std_PersistentArray_push___rarg(x_33, x_132); -if (lean_is_scalar(x_130)) { - x_134 = lean_alloc_ctor(0, 2, 1); -} else { - x_134 = x_130; -} -lean_ctor_set(x_134, 0, x_129); -lean_ctor_set(x_134, 1, x_133); -lean_ctor_set_uint8(x_134, sizeof(void*)*2, x_128); -x_135 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_135, 0, x_124); -lean_ctor_set(x_135, 1, x_125); -lean_ctor_set(x_135, 2, x_126); -lean_ctor_set(x_135, 3, x_127); -lean_ctor_set(x_135, 4, x_134); -x_136 = lean_st_ref_set(x_4, x_135, x_95); -lean_dec(x_4); -x_137 = lean_ctor_get(x_136, 1); -lean_inc(x_137); -if (lean_is_exclusive(x_136)) { - lean_ctor_release(x_136, 0); - lean_ctor_release(x_136, 1); - x_138 = x_136; +x_134 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_134, 0, x_133); +x_135 = l_Std_PersistentArray_push___rarg(x_33, x_134); +if (lean_is_scalar(x_132)) { + x_136 = lean_alloc_ctor(0, 2, 1); +} else { + x_136 = x_132; +} +lean_ctor_set(x_136, 0, x_131); +lean_ctor_set(x_136, 1, x_135); +lean_ctor_set_uint8(x_136, sizeof(void*)*2, x_130); +x_137 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_137, 0, x_125); +lean_ctor_set(x_137, 1, x_126); +lean_ctor_set(x_137, 2, x_127); +lean_ctor_set(x_137, 3, x_128); +lean_ctor_set(x_137, 4, x_129); +lean_ctor_set(x_137, 5, x_136); +x_138 = lean_st_ref_set(x_4, x_137, x_96); +lean_dec(x_4); +x_139 = lean_ctor_get(x_138, 1); +lean_inc(x_139); +if (lean_is_exclusive(x_138)) { + lean_ctor_release(x_138, 0); + lean_ctor_release(x_138, 1); + x_140 = x_138; } else { - lean_dec_ref(x_136); - x_138 = lean_box(0); + lean_dec_ref(x_138); + x_140 = lean_box(0); } -x_139 = lean_box(0); -x_140 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_140, 0, x_36); -lean_ctor_set(x_140, 1, x_139); -if (lean_is_scalar(x_138)) { - x_141 = lean_alloc_ctor(0, 2, 0); +x_141 = lean_box(0); +x_142 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_142, 0, x_36); +lean_ctor_set(x_142, 1, x_141); +if (lean_is_scalar(x_140)) { + x_143 = lean_alloc_ctor(0, 2, 0); } else { - x_141 = x_138; + x_143 = x_140; } -lean_ctor_set(x_141, 0, x_140); -lean_ctor_set(x_141, 1, x_137); -x_10 = x_141; +lean_ctor_set(x_143, 0, x_142); +lean_ctor_set(x_143, 1, x_139); +x_10 = x_143; goto block_22; } } } else { -uint8_t x_142; +uint8_t x_144; lean_dec(x_36); lean_dec(x_33); lean_dec(x_8); lean_dec(x_4); -x_142 = !lean_is_exclusive(x_38); -if (x_142 == 0) +x_144 = !lean_is_exclusive(x_38); +if (x_144 == 0) { x_10 = x_38; goto block_22; } else { -lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_143 = lean_ctor_get(x_38, 0); -x_144 = lean_ctor_get(x_38, 1); -lean_inc(x_144); -lean_inc(x_143); +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_38, 0); +x_146 = lean_ctor_get(x_38, 1); +lean_inc(x_146); +lean_inc(x_145); lean_dec(x_38); -x_145 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_145, 0, x_143); -lean_ctor_set(x_145, 1, x_144); -x_10 = x_145; +x_147 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_147, 0, x_145); +lean_ctor_set(x_147, 1, x_146); +x_10 = x_147; goto block_22; } } } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; uint8_t x_156; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); -x_146 = lean_ctor_get(x_35, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_35, 1); -lean_inc(x_147); +x_148 = lean_ctor_get(x_35, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_35, 1); +lean_inc(x_149); lean_dec(x_35); -x_148 = lean_st_ref_get(x_8, x_147); +x_150 = lean_st_ref_get(x_8, x_149); lean_dec(x_8); -x_149 = lean_ctor_get(x_148, 1); -lean_inc(x_149); -lean_dec(x_148); -x_150 = lean_st_ref_take(x_4, x_149); -x_151 = lean_ctor_get(x_150, 0); +x_151 = lean_ctor_get(x_150, 1); lean_inc(x_151); -x_152 = lean_ctor_get(x_151, 4); -lean_inc(x_152); -x_153 = lean_ctor_get(x_150, 1); -lean_inc(x_153); lean_dec(x_150); -x_154 = !lean_is_exclusive(x_151); -if (x_154 == 0) -{ -lean_object* x_155; uint8_t x_156; -x_155 = lean_ctor_get(x_151, 4); -lean_dec(x_155); -x_156 = !lean_is_exclusive(x_152); +x_152 = lean_st_ref_take(x_4, x_151); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +x_154 = lean_ctor_get(x_153, 5); +lean_inc(x_154); +x_155 = lean_ctor_get(x_152, 1); +lean_inc(x_155); +lean_dec(x_152); +x_156 = !lean_is_exclusive(x_153); if (x_156 == 0) { -lean_object* x_157; lean_object* x_158; uint8_t x_159; -x_157 = lean_ctor_get(x_152, 1); +lean_object* x_157; uint8_t x_158; +x_157 = lean_ctor_get(x_153, 5); lean_dec(x_157); -lean_ctor_set(x_152, 1, x_33); -x_158 = lean_st_ref_set(x_4, x_151, x_153); +x_158 = !lean_is_exclusive(x_154); +if (x_158 == 0) +{ +lean_object* x_159; lean_object* x_160; uint8_t x_161; +x_159 = lean_ctor_get(x_154, 1); +lean_dec(x_159); +lean_ctor_set(x_154, 1, x_33); +x_160 = lean_st_ref_set(x_4, x_153, x_155); lean_dec(x_4); -x_159 = !lean_is_exclusive(x_158); -if (x_159 == 0) +x_161 = !lean_is_exclusive(x_160); +if (x_161 == 0) { -lean_object* x_160; -x_160 = lean_ctor_get(x_158, 0); -lean_dec(x_160); -lean_ctor_set_tag(x_158, 1); -lean_ctor_set(x_158, 0, x_146); -x_10 = x_158; +lean_object* x_162; +x_162 = lean_ctor_get(x_160, 0); +lean_dec(x_162); +lean_ctor_set_tag(x_160, 1); +lean_ctor_set(x_160, 0, x_148); +x_10 = x_160; goto block_22; } else { -lean_object* x_161; lean_object* x_162; -x_161 = lean_ctor_get(x_158, 1); -lean_inc(x_161); -lean_dec(x_158); -x_162 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_162, 0, x_146); -lean_ctor_set(x_162, 1, x_161); -x_10 = x_162; +lean_object* x_163; lean_object* x_164; +x_163 = lean_ctor_get(x_160, 1); +lean_inc(x_163); +lean_dec(x_160); +x_164 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_164, 0, x_148); +lean_ctor_set(x_164, 1, x_163); +x_10 = x_164; goto block_22; } } else { -uint8_t x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -x_163 = lean_ctor_get_uint8(x_152, sizeof(void*)*2); -x_164 = lean_ctor_get(x_152, 0); -lean_inc(x_164); -lean_dec(x_152); -x_165 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_165, 0, x_164); -lean_ctor_set(x_165, 1, x_33); -lean_ctor_set_uint8(x_165, sizeof(void*)*2, x_163); -lean_ctor_set(x_151, 4, x_165); -x_166 = lean_st_ref_set(x_4, x_151, x_153); +uint8_t x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +x_165 = lean_ctor_get_uint8(x_154, sizeof(void*)*2); +x_166 = lean_ctor_get(x_154, 0); +lean_inc(x_166); +lean_dec(x_154); +x_167 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_167, 0, x_166); +lean_ctor_set(x_167, 1, x_33); +lean_ctor_set_uint8(x_167, sizeof(void*)*2, x_165); +lean_ctor_set(x_153, 5, x_167); +x_168 = lean_st_ref_set(x_4, x_153, x_155); lean_dec(x_4); -x_167 = lean_ctor_get(x_166, 1); -lean_inc(x_167); -if (lean_is_exclusive(x_166)) { - lean_ctor_release(x_166, 0); - lean_ctor_release(x_166, 1); - x_168 = x_166; +x_169 = lean_ctor_get(x_168, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_168)) { + lean_ctor_release(x_168, 0); + lean_ctor_release(x_168, 1); + x_170 = x_168; } else { - lean_dec_ref(x_166); - x_168 = lean_box(0); + lean_dec_ref(x_168); + x_170 = lean_box(0); } -if (lean_is_scalar(x_168)) { - x_169 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_169 = x_168; - lean_ctor_set_tag(x_169, 1); + x_171 = x_170; + lean_ctor_set_tag(x_171, 1); } -lean_ctor_set(x_169, 0, x_146); -lean_ctor_set(x_169, 1, x_167); -x_10 = x_169; +lean_ctor_set(x_171, 0, x_148); +lean_ctor_set(x_171, 1, x_169); +x_10 = x_171; goto block_22; } } else { -lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_170 = lean_ctor_get(x_151, 0); -x_171 = lean_ctor_get(x_151, 1); -x_172 = lean_ctor_get(x_151, 2); -x_173 = lean_ctor_get(x_151, 3); +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; uint8_t x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; +x_172 = lean_ctor_get(x_153, 0); +x_173 = lean_ctor_get(x_153, 1); +x_174 = lean_ctor_get(x_153, 2); +x_175 = lean_ctor_get(x_153, 3); +x_176 = lean_ctor_get(x_153, 4); +lean_inc(x_176); +lean_inc(x_175); +lean_inc(x_174); lean_inc(x_173); lean_inc(x_172); -lean_inc(x_171); -lean_inc(x_170); -lean_dec(x_151); -x_174 = lean_ctor_get_uint8(x_152, sizeof(void*)*2); -x_175 = lean_ctor_get(x_152, 0); -lean_inc(x_175); -if (lean_is_exclusive(x_152)) { - lean_ctor_release(x_152, 0); - lean_ctor_release(x_152, 1); - x_176 = x_152; -} else { - lean_dec_ref(x_152); - x_176 = lean_box(0); -} -if (lean_is_scalar(x_176)) { - x_177 = lean_alloc_ctor(0, 2, 1); +lean_dec(x_153); +x_177 = lean_ctor_get_uint8(x_154, sizeof(void*)*2); +x_178 = lean_ctor_get(x_154, 0); +lean_inc(x_178); +if (lean_is_exclusive(x_154)) { + lean_ctor_release(x_154, 0); + lean_ctor_release(x_154, 1); + x_179 = x_154; } else { - x_177 = x_176; + lean_dec_ref(x_154); + x_179 = lean_box(0); } -lean_ctor_set(x_177, 0, x_175); -lean_ctor_set(x_177, 1, x_33); -lean_ctor_set_uint8(x_177, sizeof(void*)*2, x_174); -x_178 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_178, 0, x_170); -lean_ctor_set(x_178, 1, x_171); -lean_ctor_set(x_178, 2, x_172); -lean_ctor_set(x_178, 3, x_173); -lean_ctor_set(x_178, 4, x_177); -x_179 = lean_st_ref_set(x_4, x_178, x_153); +if (lean_is_scalar(x_179)) { + x_180 = lean_alloc_ctor(0, 2, 1); +} else { + x_180 = x_179; +} +lean_ctor_set(x_180, 0, x_178); +lean_ctor_set(x_180, 1, x_33); +lean_ctor_set_uint8(x_180, sizeof(void*)*2, x_177); +x_181 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_181, 0, x_172); +lean_ctor_set(x_181, 1, x_173); +lean_ctor_set(x_181, 2, x_174); +lean_ctor_set(x_181, 3, x_175); +lean_ctor_set(x_181, 4, x_176); +lean_ctor_set(x_181, 5, x_180); +x_182 = lean_st_ref_set(x_4, x_181, x_155); lean_dec(x_4); -x_180 = lean_ctor_get(x_179, 1); -lean_inc(x_180); -if (lean_is_exclusive(x_179)) { - lean_ctor_release(x_179, 0); - lean_ctor_release(x_179, 1); - x_181 = x_179; +x_183 = lean_ctor_get(x_182, 1); +lean_inc(x_183); +if (lean_is_exclusive(x_182)) { + lean_ctor_release(x_182, 0); + lean_ctor_release(x_182, 1); + x_184 = x_182; } else { - lean_dec_ref(x_179); - x_181 = lean_box(0); + lean_dec_ref(x_182); + x_184 = lean_box(0); } -if (lean_is_scalar(x_181)) { - x_182 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_184)) { + x_185 = lean_alloc_ctor(1, 2, 0); } else { - x_182 = x_181; - lean_ctor_set_tag(x_182, 1); + x_185 = x_184; + lean_ctor_set_tag(x_185, 1); } -lean_ctor_set(x_182, 0, x_146); -lean_ctor_set(x_182, 1, x_180); -x_10 = x_182; +lean_ctor_set(x_185, 0, x_148); +lean_ctor_set(x_185, 1, x_183); +x_10 = x_185; goto block_22; } } @@ -33836,7 +37708,7 @@ lean_dec(x_23); x_25 = lean_st_ref_get(x_4, x_24); x_26 = lean_ctor_get(x_25, 0); lean_inc(x_26); -x_27 = lean_ctor_get(x_26, 4); +x_27 = lean_ctor_get(x_26, 5); lean_inc(x_27); lean_dec(x_26); x_28 = lean_ctor_get_uint8(x_27, sizeof(void*)*2); @@ -33898,7 +37770,7 @@ lean_dec(x_41); x_43 = lean_st_ref_take(x_4, x_42); x_44 = lean_ctor_get(x_43, 0); lean_inc(x_44); -x_45 = lean_ctor_get(x_44, 4); +x_45 = lean_ctor_get(x_44, 5); lean_inc(x_45); if (lean_obj_tag(x_39) == 0) { @@ -33910,7 +37782,7 @@ x_47 = !lean_is_exclusive(x_44); if (x_47 == 0) { lean_object* x_48; uint8_t x_49; -x_48 = lean_ctor_get(x_44, 4); +x_48 = lean_ctor_get(x_44, 5); lean_dec(x_48); x_49 = !lean_is_exclusive(x_45); if (x_49 == 0) @@ -33978,7 +37850,7 @@ x_69 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_69, 0, x_64); lean_ctor_set(x_69, 1, x_68); lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_63); -lean_ctor_set(x_44, 4, x_69); +lean_ctor_set(x_44, 5, x_69); x_70 = lean_st_ref_set(x_4, x_44, x_46); lean_dec(x_4); x_71 = lean_ctor_get(x_70, 1); @@ -34008,439 +37880,448 @@ goto block_22; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_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_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; x_76 = lean_ctor_get(x_44, 0); x_77 = lean_ctor_get(x_44, 1); x_78 = lean_ctor_get(x_44, 2); x_79 = lean_ctor_get(x_44, 3); +x_80 = lean_ctor_get(x_44, 4); +lean_inc(x_80); lean_inc(x_79); lean_inc(x_78); lean_inc(x_77); lean_inc(x_76); lean_dec(x_44); -x_80 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); -x_81 = lean_ctor_get(x_45, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_45, 1); +x_81 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); +x_82 = lean_ctor_get(x_45, 0); lean_inc(x_82); +x_83 = lean_ctor_get(x_45, 1); +lean_inc(x_83); if (lean_is_exclusive(x_45)) { lean_ctor_release(x_45, 0); lean_ctor_release(x_45, 1); - x_83 = x_45; + x_84 = x_45; } else { lean_dec_ref(x_45); - x_83 = lean_box(0); + x_84 = lean_box(0); } -x_84 = lean_ctor_get(x_39, 0); -lean_inc(x_84); +x_85 = lean_ctor_get(x_39, 0); +lean_inc(x_85); lean_dec(x_39); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_84); -lean_ctor_set(x_85, 1, x_82); -x_86 = l_Std_PersistentArray_push___rarg(x_33, x_85); -if (lean_is_scalar(x_83)) { - x_87 = lean_alloc_ctor(0, 2, 1); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_83); +x_87 = l_Std_PersistentArray_push___rarg(x_33, x_86); +if (lean_is_scalar(x_84)) { + x_88 = lean_alloc_ctor(0, 2, 1); } else { - x_87 = x_83; + x_88 = x_84; } -lean_ctor_set(x_87, 0, x_81); -lean_ctor_set(x_87, 1, x_86); -lean_ctor_set_uint8(x_87, sizeof(void*)*2, x_80); -x_88 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_88, 0, x_76); -lean_ctor_set(x_88, 1, x_77); -lean_ctor_set(x_88, 2, x_78); -lean_ctor_set(x_88, 3, x_79); -lean_ctor_set(x_88, 4, x_87); -x_89 = lean_st_ref_set(x_4, x_88, x_46); +lean_ctor_set(x_88, 0, x_82); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set_uint8(x_88, sizeof(void*)*2, x_81); +x_89 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_89, 0, x_76); +lean_ctor_set(x_89, 1, x_77); +lean_ctor_set(x_89, 2, x_78); +lean_ctor_set(x_89, 3, x_79); +lean_ctor_set(x_89, 4, x_80); +lean_ctor_set(x_89, 5, x_88); +x_90 = lean_st_ref_set(x_4, x_89, x_46); lean_dec(x_4); -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_91 = x_89; +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_90)) { + lean_ctor_release(x_90, 0); + lean_ctor_release(x_90, 1); + x_92 = x_90; } else { - lean_dec_ref(x_89); - x_91 = lean_box(0); + lean_dec_ref(x_90); + x_92 = lean_box(0); } -x_92 = lean_box(0); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_36); -lean_ctor_set(x_93, 1, x_92); -if (lean_is_scalar(x_91)) { - x_94 = lean_alloc_ctor(0, 2, 0); +x_93 = lean_box(0); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_36); +lean_ctor_set(x_94, 1, x_93); +if (lean_is_scalar(x_92)) { + x_95 = lean_alloc_ctor(0, 2, 0); } else { - x_94 = x_91; + x_95 = x_92; } -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_90); -x_10 = x_94; +lean_ctor_set(x_95, 0, x_94); +lean_ctor_set(x_95, 1, x_91); +x_10 = x_95; goto block_22; } } else { -lean_object* x_95; uint8_t x_96; -x_95 = lean_ctor_get(x_43, 1); -lean_inc(x_95); +lean_object* x_96; uint8_t x_97; +x_96 = lean_ctor_get(x_43, 1); +lean_inc(x_96); lean_dec(x_43); -x_96 = !lean_is_exclusive(x_44); -if (x_96 == 0) +x_97 = !lean_is_exclusive(x_44); +if (x_97 == 0) { -lean_object* x_97; uint8_t x_98; -x_97 = lean_ctor_get(x_44, 4); -lean_dec(x_97); -x_98 = !lean_is_exclusive(x_45); -if (x_98 == 0) +lean_object* x_98; uint8_t x_99; +x_98 = lean_ctor_get(x_44, 5); +lean_dec(x_98); +x_99 = !lean_is_exclusive(x_45); +if (x_99 == 0) { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; -x_99 = lean_ctor_get(x_45, 1); -lean_dec(x_99); -x_100 = lean_ctor_get(x_39, 0); -lean_inc(x_100); +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; +x_100 = lean_ctor_get(x_45, 1); +lean_dec(x_100); +x_101 = lean_ctor_get(x_39, 0); +lean_inc(x_101); lean_dec(x_39); -x_101 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_101, 0, x_100); -x_102 = l_Std_PersistentArray_push___rarg(x_33, x_101); -lean_ctor_set(x_45, 1, x_102); -x_103 = lean_st_ref_set(x_4, x_44, x_95); +x_102 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_102, 0, x_101); +x_103 = l_Std_PersistentArray_push___rarg(x_33, x_102); +lean_ctor_set(x_45, 1, x_103); +x_104 = lean_st_ref_set(x_4, x_44, x_96); lean_dec(x_4); -x_104 = !lean_is_exclusive(x_103); -if (x_104 == 0) +x_105 = !lean_is_exclusive(x_104); +if (x_105 == 0) { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_103, 0); -lean_dec(x_105); -x_106 = lean_box(0); -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_36); -lean_ctor_set(x_107, 1, x_106); -lean_ctor_set(x_103, 0, x_107); -x_10 = x_103; +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_104, 0); +lean_dec(x_106); +x_107 = lean_box(0); +x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_108, 0, x_36); +lean_ctor_set(x_108, 1, x_107); +lean_ctor_set(x_104, 0, x_108); +x_10 = x_104; goto block_22; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_108 = lean_ctor_get(x_103, 1); -lean_inc(x_108); -lean_dec(x_103); -x_109 = lean_box(0); -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_36); -lean_ctor_set(x_110, 1, x_109); +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_109 = lean_ctor_get(x_104, 1); +lean_inc(x_109); +lean_dec(x_104); +x_110 = lean_box(0); x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_108); -x_10 = x_111; +lean_ctor_set(x_111, 0, x_36); +lean_ctor_set(x_111, 1, x_110); +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_109); +x_10 = x_112; goto block_22; } } else { -uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_112 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); -x_113 = lean_ctor_get(x_45, 0); -lean_inc(x_113); -lean_dec(x_45); -x_114 = lean_ctor_get(x_39, 0); +uint8_t x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_113 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); +x_114 = lean_ctor_get(x_45, 0); lean_inc(x_114); +lean_dec(x_45); +x_115 = lean_ctor_get(x_39, 0); +lean_inc(x_115); lean_dec(x_39); -x_115 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_115, 0, x_114); -x_116 = l_Std_PersistentArray_push___rarg(x_33, x_115); -x_117 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_117, 0, x_113); -lean_ctor_set(x_117, 1, x_116); -lean_ctor_set_uint8(x_117, sizeof(void*)*2, x_112); -lean_ctor_set(x_44, 4, x_117); -x_118 = lean_st_ref_set(x_4, x_44, x_95); +x_116 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_116, 0, x_115); +x_117 = l_Std_PersistentArray_push___rarg(x_33, x_116); +x_118 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_118, 0, x_114); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set_uint8(x_118, sizeof(void*)*2, x_113); +lean_ctor_set(x_44, 5, x_118); +x_119 = lean_st_ref_set(x_4, x_44, x_96); lean_dec(x_4); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_120 = x_118; +x_120 = lean_ctor_get(x_119, 1); +lean_inc(x_120); +if (lean_is_exclusive(x_119)) { + lean_ctor_release(x_119, 0); + lean_ctor_release(x_119, 1); + x_121 = x_119; } else { - lean_dec_ref(x_118); - x_120 = lean_box(0); + lean_dec_ref(x_119); + x_121 = lean_box(0); } -x_121 = lean_box(0); -x_122 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_122, 0, x_36); -lean_ctor_set(x_122, 1, x_121); -if (lean_is_scalar(x_120)) { - x_123 = lean_alloc_ctor(0, 2, 0); +x_122 = lean_box(0); +x_123 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_123, 0, x_36); +lean_ctor_set(x_123, 1, x_122); +if (lean_is_scalar(x_121)) { + x_124 = lean_alloc_ctor(0, 2, 0); } else { - x_123 = x_120; + x_124 = x_121; } -lean_ctor_set(x_123, 0, x_122); -lean_ctor_set(x_123, 1, x_119); -x_10 = x_123; +lean_ctor_set(x_124, 0, x_123); +lean_ctor_set(x_124, 1, x_120); +x_10 = x_124; goto block_22; } } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; -x_124 = lean_ctor_get(x_44, 0); -x_125 = lean_ctor_get(x_44, 1); -x_126 = lean_ctor_get(x_44, 2); -x_127 = lean_ctor_get(x_44, 3); +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; uint8_t x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; +x_125 = lean_ctor_get(x_44, 0); +x_126 = lean_ctor_get(x_44, 1); +x_127 = lean_ctor_get(x_44, 2); +x_128 = lean_ctor_get(x_44, 3); +x_129 = lean_ctor_get(x_44, 4); +lean_inc(x_129); +lean_inc(x_128); lean_inc(x_127); lean_inc(x_126); lean_inc(x_125); -lean_inc(x_124); lean_dec(x_44); -x_128 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); -x_129 = lean_ctor_get(x_45, 0); -lean_inc(x_129); +x_130 = lean_ctor_get_uint8(x_45, sizeof(void*)*2); +x_131 = lean_ctor_get(x_45, 0); +lean_inc(x_131); if (lean_is_exclusive(x_45)) { lean_ctor_release(x_45, 0); lean_ctor_release(x_45, 1); - x_130 = x_45; + x_132 = x_45; } else { lean_dec_ref(x_45); - x_130 = lean_box(0); + x_132 = lean_box(0); } -x_131 = lean_ctor_get(x_39, 0); -lean_inc(x_131); +x_133 = lean_ctor_get(x_39, 0); +lean_inc(x_133); lean_dec(x_39); -x_132 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_132, 0, x_131); -x_133 = l_Std_PersistentArray_push___rarg(x_33, x_132); -if (lean_is_scalar(x_130)) { - x_134 = lean_alloc_ctor(0, 2, 1); -} else { - x_134 = x_130; -} -lean_ctor_set(x_134, 0, x_129); -lean_ctor_set(x_134, 1, x_133); -lean_ctor_set_uint8(x_134, sizeof(void*)*2, x_128); -x_135 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_135, 0, x_124); -lean_ctor_set(x_135, 1, x_125); -lean_ctor_set(x_135, 2, x_126); -lean_ctor_set(x_135, 3, x_127); -lean_ctor_set(x_135, 4, x_134); -x_136 = lean_st_ref_set(x_4, x_135, x_95); -lean_dec(x_4); -x_137 = lean_ctor_get(x_136, 1); -lean_inc(x_137); -if (lean_is_exclusive(x_136)) { - lean_ctor_release(x_136, 0); - lean_ctor_release(x_136, 1); - x_138 = x_136; +x_134 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_134, 0, x_133); +x_135 = l_Std_PersistentArray_push___rarg(x_33, x_134); +if (lean_is_scalar(x_132)) { + x_136 = lean_alloc_ctor(0, 2, 1); +} else { + x_136 = x_132; +} +lean_ctor_set(x_136, 0, x_131); +lean_ctor_set(x_136, 1, x_135); +lean_ctor_set_uint8(x_136, sizeof(void*)*2, x_130); +x_137 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_137, 0, x_125); +lean_ctor_set(x_137, 1, x_126); +lean_ctor_set(x_137, 2, x_127); +lean_ctor_set(x_137, 3, x_128); +lean_ctor_set(x_137, 4, x_129); +lean_ctor_set(x_137, 5, x_136); +x_138 = lean_st_ref_set(x_4, x_137, x_96); +lean_dec(x_4); +x_139 = lean_ctor_get(x_138, 1); +lean_inc(x_139); +if (lean_is_exclusive(x_138)) { + lean_ctor_release(x_138, 0); + lean_ctor_release(x_138, 1); + x_140 = x_138; } else { - lean_dec_ref(x_136); - x_138 = lean_box(0); + lean_dec_ref(x_138); + x_140 = lean_box(0); } -x_139 = lean_box(0); -x_140 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_140, 0, x_36); -lean_ctor_set(x_140, 1, x_139); -if (lean_is_scalar(x_138)) { - x_141 = lean_alloc_ctor(0, 2, 0); +x_141 = lean_box(0); +x_142 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_142, 0, x_36); +lean_ctor_set(x_142, 1, x_141); +if (lean_is_scalar(x_140)) { + x_143 = lean_alloc_ctor(0, 2, 0); } else { - x_141 = x_138; + x_143 = x_140; } -lean_ctor_set(x_141, 0, x_140); -lean_ctor_set(x_141, 1, x_137); -x_10 = x_141; +lean_ctor_set(x_143, 0, x_142); +lean_ctor_set(x_143, 1, x_139); +x_10 = x_143; goto block_22; } } } else { -uint8_t x_142; +uint8_t x_144; lean_dec(x_36); lean_dec(x_33); lean_dec(x_8); lean_dec(x_4); -x_142 = !lean_is_exclusive(x_38); -if (x_142 == 0) +x_144 = !lean_is_exclusive(x_38); +if (x_144 == 0) { x_10 = x_38; goto block_22; } else { -lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_143 = lean_ctor_get(x_38, 0); -x_144 = lean_ctor_get(x_38, 1); -lean_inc(x_144); -lean_inc(x_143); +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_38, 0); +x_146 = lean_ctor_get(x_38, 1); +lean_inc(x_146); +lean_inc(x_145); lean_dec(x_38); -x_145 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_145, 0, x_143); -lean_ctor_set(x_145, 1, x_144); -x_10 = x_145; +x_147 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_147, 0, x_145); +lean_ctor_set(x_147, 1, x_146); +x_10 = x_147; goto block_22; } } } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; uint8_t x_156; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); -x_146 = lean_ctor_get(x_35, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_35, 1); -lean_inc(x_147); +x_148 = lean_ctor_get(x_35, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_35, 1); +lean_inc(x_149); lean_dec(x_35); -x_148 = lean_st_ref_get(x_8, x_147); +x_150 = lean_st_ref_get(x_8, x_149); lean_dec(x_8); -x_149 = lean_ctor_get(x_148, 1); -lean_inc(x_149); -lean_dec(x_148); -x_150 = lean_st_ref_take(x_4, x_149); -x_151 = lean_ctor_get(x_150, 0); +x_151 = lean_ctor_get(x_150, 1); lean_inc(x_151); -x_152 = lean_ctor_get(x_151, 4); -lean_inc(x_152); -x_153 = lean_ctor_get(x_150, 1); -lean_inc(x_153); lean_dec(x_150); -x_154 = !lean_is_exclusive(x_151); -if (x_154 == 0) -{ -lean_object* x_155; uint8_t x_156; -x_155 = lean_ctor_get(x_151, 4); -lean_dec(x_155); -x_156 = !lean_is_exclusive(x_152); +x_152 = lean_st_ref_take(x_4, x_151); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +x_154 = lean_ctor_get(x_153, 5); +lean_inc(x_154); +x_155 = lean_ctor_get(x_152, 1); +lean_inc(x_155); +lean_dec(x_152); +x_156 = !lean_is_exclusive(x_153); if (x_156 == 0) { -lean_object* x_157; lean_object* x_158; uint8_t x_159; -x_157 = lean_ctor_get(x_152, 1); +lean_object* x_157; uint8_t x_158; +x_157 = lean_ctor_get(x_153, 5); lean_dec(x_157); -lean_ctor_set(x_152, 1, x_33); -x_158 = lean_st_ref_set(x_4, x_151, x_153); +x_158 = !lean_is_exclusive(x_154); +if (x_158 == 0) +{ +lean_object* x_159; lean_object* x_160; uint8_t x_161; +x_159 = lean_ctor_get(x_154, 1); +lean_dec(x_159); +lean_ctor_set(x_154, 1, x_33); +x_160 = lean_st_ref_set(x_4, x_153, x_155); lean_dec(x_4); -x_159 = !lean_is_exclusive(x_158); -if (x_159 == 0) +x_161 = !lean_is_exclusive(x_160); +if (x_161 == 0) { -lean_object* x_160; -x_160 = lean_ctor_get(x_158, 0); -lean_dec(x_160); -lean_ctor_set_tag(x_158, 1); -lean_ctor_set(x_158, 0, x_146); -x_10 = x_158; +lean_object* x_162; +x_162 = lean_ctor_get(x_160, 0); +lean_dec(x_162); +lean_ctor_set_tag(x_160, 1); +lean_ctor_set(x_160, 0, x_148); +x_10 = x_160; goto block_22; } else { -lean_object* x_161; lean_object* x_162; -x_161 = lean_ctor_get(x_158, 1); -lean_inc(x_161); -lean_dec(x_158); -x_162 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_162, 0, x_146); -lean_ctor_set(x_162, 1, x_161); -x_10 = x_162; +lean_object* x_163; lean_object* x_164; +x_163 = lean_ctor_get(x_160, 1); +lean_inc(x_163); +lean_dec(x_160); +x_164 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_164, 0, x_148); +lean_ctor_set(x_164, 1, x_163); +x_10 = x_164; goto block_22; } } else { -uint8_t x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -x_163 = lean_ctor_get_uint8(x_152, sizeof(void*)*2); -x_164 = lean_ctor_get(x_152, 0); -lean_inc(x_164); -lean_dec(x_152); -x_165 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_165, 0, x_164); -lean_ctor_set(x_165, 1, x_33); -lean_ctor_set_uint8(x_165, sizeof(void*)*2, x_163); -lean_ctor_set(x_151, 4, x_165); -x_166 = lean_st_ref_set(x_4, x_151, x_153); +uint8_t x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +x_165 = lean_ctor_get_uint8(x_154, sizeof(void*)*2); +x_166 = lean_ctor_get(x_154, 0); +lean_inc(x_166); +lean_dec(x_154); +x_167 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_167, 0, x_166); +lean_ctor_set(x_167, 1, x_33); +lean_ctor_set_uint8(x_167, sizeof(void*)*2, x_165); +lean_ctor_set(x_153, 5, x_167); +x_168 = lean_st_ref_set(x_4, x_153, x_155); lean_dec(x_4); -x_167 = lean_ctor_get(x_166, 1); -lean_inc(x_167); -if (lean_is_exclusive(x_166)) { - lean_ctor_release(x_166, 0); - lean_ctor_release(x_166, 1); - x_168 = x_166; +x_169 = lean_ctor_get(x_168, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_168)) { + lean_ctor_release(x_168, 0); + lean_ctor_release(x_168, 1); + x_170 = x_168; } else { - lean_dec_ref(x_166); - x_168 = lean_box(0); + lean_dec_ref(x_168); + x_170 = lean_box(0); } -if (lean_is_scalar(x_168)) { - x_169 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_169 = x_168; - lean_ctor_set_tag(x_169, 1); + x_171 = x_170; + lean_ctor_set_tag(x_171, 1); } -lean_ctor_set(x_169, 0, x_146); -lean_ctor_set(x_169, 1, x_167); -x_10 = x_169; +lean_ctor_set(x_171, 0, x_148); +lean_ctor_set(x_171, 1, x_169); +x_10 = x_171; goto block_22; } } else { -lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_170 = lean_ctor_get(x_151, 0); -x_171 = lean_ctor_get(x_151, 1); -x_172 = lean_ctor_get(x_151, 2); -x_173 = lean_ctor_get(x_151, 3); +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; uint8_t x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; +x_172 = lean_ctor_get(x_153, 0); +x_173 = lean_ctor_get(x_153, 1); +x_174 = lean_ctor_get(x_153, 2); +x_175 = lean_ctor_get(x_153, 3); +x_176 = lean_ctor_get(x_153, 4); +lean_inc(x_176); +lean_inc(x_175); +lean_inc(x_174); lean_inc(x_173); lean_inc(x_172); -lean_inc(x_171); -lean_inc(x_170); -lean_dec(x_151); -x_174 = lean_ctor_get_uint8(x_152, sizeof(void*)*2); -x_175 = lean_ctor_get(x_152, 0); -lean_inc(x_175); -if (lean_is_exclusive(x_152)) { - lean_ctor_release(x_152, 0); - lean_ctor_release(x_152, 1); - x_176 = x_152; -} else { - lean_dec_ref(x_152); - x_176 = lean_box(0); -} -if (lean_is_scalar(x_176)) { - x_177 = lean_alloc_ctor(0, 2, 1); +lean_dec(x_153); +x_177 = lean_ctor_get_uint8(x_154, sizeof(void*)*2); +x_178 = lean_ctor_get(x_154, 0); +lean_inc(x_178); +if (lean_is_exclusive(x_154)) { + lean_ctor_release(x_154, 0); + lean_ctor_release(x_154, 1); + x_179 = x_154; } else { - x_177 = x_176; + lean_dec_ref(x_154); + x_179 = lean_box(0); } -lean_ctor_set(x_177, 0, x_175); -lean_ctor_set(x_177, 1, x_33); -lean_ctor_set_uint8(x_177, sizeof(void*)*2, x_174); -x_178 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_178, 0, x_170); -lean_ctor_set(x_178, 1, x_171); -lean_ctor_set(x_178, 2, x_172); -lean_ctor_set(x_178, 3, x_173); -lean_ctor_set(x_178, 4, x_177); -x_179 = lean_st_ref_set(x_4, x_178, x_153); +if (lean_is_scalar(x_179)) { + x_180 = lean_alloc_ctor(0, 2, 1); +} else { + x_180 = x_179; +} +lean_ctor_set(x_180, 0, x_178); +lean_ctor_set(x_180, 1, x_33); +lean_ctor_set_uint8(x_180, sizeof(void*)*2, x_177); +x_181 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_181, 0, x_172); +lean_ctor_set(x_181, 1, x_173); +lean_ctor_set(x_181, 2, x_174); +lean_ctor_set(x_181, 3, x_175); +lean_ctor_set(x_181, 4, x_176); +lean_ctor_set(x_181, 5, x_180); +x_182 = lean_st_ref_set(x_4, x_181, x_155); lean_dec(x_4); -x_180 = lean_ctor_get(x_179, 1); -lean_inc(x_180); -if (lean_is_exclusive(x_179)) { - lean_ctor_release(x_179, 0); - lean_ctor_release(x_179, 1); - x_181 = x_179; +x_183 = lean_ctor_get(x_182, 1); +lean_inc(x_183); +if (lean_is_exclusive(x_182)) { + lean_ctor_release(x_182, 0); + lean_ctor_release(x_182, 1); + x_184 = x_182; } else { - lean_dec_ref(x_179); - x_181 = lean_box(0); + lean_dec_ref(x_182); + x_184 = lean_box(0); } -if (lean_is_scalar(x_181)) { - x_182 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_184)) { + x_185 = lean_alloc_ctor(1, 2, 0); } else { - x_182 = x_181; - lean_ctor_set_tag(x_182, 1); + x_185 = x_184; + lean_ctor_set_tag(x_185, 1); } -lean_ctor_set(x_182, 0, x_146); -lean_ctor_set(x_182, 1, x_180); -x_10 = x_182; +lean_ctor_set(x_185, 0, x_148); +lean_ctor_set(x_185, 1, x_183); +x_10 = x_185; goto block_22; } } @@ -37798,7 +41679,7 @@ static lean_object* _init_l___private_Lean_Util_Trace_0__Lean_withNestedTracesFi 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_Util_Trace_0__Lean_withNestedTracesFinalizer___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__1___closed__1; x_2 = l___private_Lean_Util_Trace_0__Lean_withNestedTracesFinalizer___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Util_Trace_0__Lean_withNestedTracesFinalizer___at___private_Lean_Elab_Term_0__Lean_Elab_Term_elabTermAux___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -41243,7 +45124,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -41288,7 +45169,7 @@ lean_dec(x_22); x_24 = lean_st_ref_take(x_3, x_23); x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -x_26 = lean_ctor_get(x_25, 4); +x_26 = lean_ctor_get(x_25, 5); lean_inc(x_26); x_27 = lean_ctor_get(x_24, 1); lean_inc(x_27); @@ -41297,7 +45178,7 @@ x_28 = !lean_is_exclusive(x_25); if (x_28 == 0) { lean_object* x_29; uint8_t x_30; -x_29 = lean_ctor_get(x_25, 4); +x_29 = lean_ctor_get(x_25, 5); lean_dec(x_29); x_30 = !lean_is_exclusive(x_26); if (x_30 == 0) @@ -41344,7 +45225,7 @@ x_44 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_44, 0, x_41); lean_ctor_set(x_44, 1, x_43); lean_ctor_set_uint8(x_44, sizeof(void*)*2, x_40); -lean_ctor_set(x_25, 4, x_44); +lean_ctor_set(x_25, 5, x_44); x_45 = lean_st_ref_set(x_3, x_25, x_27); x_46 = lean_ctor_get(x_45, 1); lean_inc(x_46); @@ -41369,64 +45250,67 @@ return x_49; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; x_50 = lean_ctor_get(x_25, 0); x_51 = lean_ctor_get(x_25, 1); x_52 = lean_ctor_get(x_25, 2); x_53 = lean_ctor_get(x_25, 3); +x_54 = lean_ctor_get(x_25, 4); +lean_inc(x_54); lean_inc(x_53); lean_inc(x_52); lean_inc(x_51); lean_inc(x_50); lean_dec(x_25); -x_54 = lean_ctor_get_uint8(x_26, sizeof(void*)*2); -x_55 = lean_ctor_get(x_26, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_26, 1); +x_55 = lean_ctor_get_uint8(x_26, sizeof(void*)*2); +x_56 = lean_ctor_get(x_26, 0); lean_inc(x_56); +x_57 = lean_ctor_get(x_26, 1); +lean_inc(x_57); if (lean_is_exclusive(x_26)) { lean_ctor_release(x_26, 0); lean_ctor_release(x_26, 1); - x_57 = x_26; + x_58 = x_26; } else { lean_dec_ref(x_26); - x_57 = lean_box(0); + x_58 = lean_box(0); } -x_58 = l_Std_PersistentArray_push___rarg(x_56, x_1); -if (lean_is_scalar(x_57)) { - x_59 = lean_alloc_ctor(0, 2, 1); +x_59 = l_Std_PersistentArray_push___rarg(x_57, x_1); +if (lean_is_scalar(x_58)) { + x_60 = lean_alloc_ctor(0, 2, 1); } else { - x_59 = x_57; + x_60 = x_58; } -lean_ctor_set(x_59, 0, x_55); -lean_ctor_set(x_59, 1, x_58); -lean_ctor_set_uint8(x_59, sizeof(void*)*2, x_54); -x_60 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_60, 0, x_50); -lean_ctor_set(x_60, 1, x_51); -lean_ctor_set(x_60, 2, x_52); -lean_ctor_set(x_60, 3, x_53); -lean_ctor_set(x_60, 4, x_59); -x_61 = lean_st_ref_set(x_3, x_60, x_27); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_63 = x_61; +lean_ctor_set(x_60, 0, x_56); +lean_ctor_set(x_60, 1, x_59); +lean_ctor_set_uint8(x_60, sizeof(void*)*2, x_55); +x_61 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_61, 0, x_50); +lean_ctor_set(x_61, 1, x_51); +lean_ctor_set(x_61, 2, x_52); +lean_ctor_set(x_61, 3, x_53); +lean_ctor_set(x_61, 4, x_54); +lean_ctor_set(x_61, 5, x_60); +x_62 = lean_st_ref_set(x_3, x_61, x_27); +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + x_64 = x_62; } else { - lean_dec_ref(x_61); - x_63 = lean_box(0); + lean_dec_ref(x_62); + x_64 = lean_box(0); } -x_64 = lean_box(0); -if (lean_is_scalar(x_63)) { - x_65 = lean_alloc_ctor(0, 2, 0); +x_65 = lean_box(0); +if (lean_is_scalar(x_64)) { + x_66 = lean_alloc_ctor(0, 2, 0); } else { - x_65 = x_63; + x_66 = x_64; } -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_62); -return x_65; +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_63); +return x_66; } } } @@ -41442,7 +45326,7 @@ lean_dec(x_9); x_11 = lean_st_ref_get(x_3, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 4); +x_13 = lean_ctor_get(x_12, 5); lean_inc(x_13); lean_dec(x_12); x_14 = lean_ctor_get_uint8(x_13, sizeof(void*)*2); @@ -41776,237 +45660,6 @@ x_15 = l_Lean_Elab_Term_elabTermEnsuringType(x_1, x_2, x_13, x_14, x_5, x_6, x_7 return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutPending___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_st_ref_get(x_7, x_8); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_st_ref_get(x_3, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -lean_inc(x_7); -lean_inc(x_3); -x_14 = lean_apply_7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_13); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_st_ref_get(x_7, x_16); -lean_dec(x_7); -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -x_19 = lean_st_ref_take(x_3, x_18); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_ctor_get(x_12, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_12, 1); -lean_inc(x_23); -x_24 = lean_ctor_get(x_12, 2); -lean_inc(x_24); -x_25 = lean_ctor_get(x_12, 3); -lean_inc(x_25); -lean_dec(x_12); -x_26 = !lean_is_exclusive(x_20); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_27 = lean_ctor_get(x_20, 3); -lean_dec(x_27); -x_28 = lean_ctor_get(x_20, 2); -lean_dec(x_28); -x_29 = lean_ctor_get(x_20, 1); -lean_dec(x_29); -x_30 = lean_ctor_get(x_20, 0); -lean_dec(x_30); -lean_ctor_set(x_20, 3, x_25); -lean_ctor_set(x_20, 2, x_24); -lean_ctor_set(x_20, 1, x_23); -lean_ctor_set(x_20, 0, x_22); -x_31 = lean_st_ref_set(x_3, x_20, x_21); -lean_dec(x_3); -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) -{ -lean_object* x_33; -x_33 = lean_ctor_get(x_31, 0); -lean_dec(x_33); -lean_ctor_set(x_31, 0, x_15); -return x_31; -} -else -{ -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_31, 1); -lean_inc(x_34); -lean_dec(x_31); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_15); -lean_ctor_set(x_35, 1, x_34); -return x_35; -} -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_36 = lean_ctor_get(x_20, 4); -lean_inc(x_36); -lean_dec(x_20); -x_37 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_37, 0, x_22); -lean_ctor_set(x_37, 1, x_23); -lean_ctor_set(x_37, 2, x_24); -lean_ctor_set(x_37, 3, x_25); -lean_ctor_set(x_37, 4, x_36); -x_38 = lean_st_ref_set(x_3, x_37, x_21); -lean_dec(x_3); -x_39 = lean_ctor_get(x_38, 1); -lean_inc(x_39); -if (lean_is_exclusive(x_38)) { - lean_ctor_release(x_38, 0); - lean_ctor_release(x_38, 1); - x_40 = x_38; -} else { - lean_dec_ref(x_38); - x_40 = lean_box(0); -} -if (lean_is_scalar(x_40)) { - x_41 = lean_alloc_ctor(0, 2, 0); -} else { - x_41 = x_40; -} -lean_ctor_set(x_41, 0, x_15); -lean_ctor_set(x_41, 1, x_39); -return x_41; -} -} -else -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; -x_42 = lean_ctor_get(x_14, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_14, 1); -lean_inc(x_43); -lean_dec(x_14); -x_44 = lean_st_ref_get(x_7, x_43); -lean_dec(x_7); -x_45 = lean_ctor_get(x_44, 1); -lean_inc(x_45); -lean_dec(x_44); -x_46 = lean_st_ref_take(x_3, x_45); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = lean_ctor_get(x_12, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_12, 1); -lean_inc(x_50); -x_51 = lean_ctor_get(x_12, 2); -lean_inc(x_51); -x_52 = lean_ctor_get(x_12, 3); -lean_inc(x_52); -lean_dec(x_12); -x_53 = !lean_is_exclusive(x_47); -if (x_53 == 0) -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; -x_54 = lean_ctor_get(x_47, 3); -lean_dec(x_54); -x_55 = lean_ctor_get(x_47, 2); -lean_dec(x_55); -x_56 = lean_ctor_get(x_47, 1); -lean_dec(x_56); -x_57 = lean_ctor_get(x_47, 0); -lean_dec(x_57); -lean_ctor_set(x_47, 3, x_52); -lean_ctor_set(x_47, 2, x_51); -lean_ctor_set(x_47, 1, x_50); -lean_ctor_set(x_47, 0, x_49); -x_58 = lean_st_ref_set(x_3, x_47, x_48); -lean_dec(x_3); -x_59 = !lean_is_exclusive(x_58); -if (x_59 == 0) -{ -lean_object* x_60; -x_60 = lean_ctor_get(x_58, 0); -lean_dec(x_60); -lean_ctor_set_tag(x_58, 1); -lean_ctor_set(x_58, 0, x_42); -return x_58; -} -else -{ -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_58, 1); -lean_inc(x_61); -lean_dec(x_58); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_42); -lean_ctor_set(x_62, 1, x_61); -return x_62; -} -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_63 = lean_ctor_get(x_47, 4); -lean_inc(x_63); -lean_dec(x_47); -x_64 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_64, 0, x_49); -lean_ctor_set(x_64, 1, x_50); -lean_ctor_set(x_64, 2, x_51); -lean_ctor_set(x_64, 3, x_52); -lean_ctor_set(x_64, 4, x_63); -x_65 = lean_st_ref_set(x_3, x_64, x_48); -lean_dec(x_3); -x_66 = lean_ctor_get(x_65, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_65)) { - lean_ctor_release(x_65, 0); - lean_ctor_release(x_65, 1); - x_67 = x_65; -} else { - lean_dec_ref(x_65); - x_67 = lean_box(0); -} -if (lean_is_scalar(x_67)) { - x_68 = lean_alloc_ctor(1, 2, 0); -} else { - x_68 = x_67; - lean_ctor_set_tag(x_68, 1); -} -lean_ctor_set(x_68, 0, x_42); -lean_ctor_set(x_68, 1, x_66); -return x_68; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Term_withoutPending(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Term_withoutPending___rarg), 8, 0); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_Elab_Term_commitIfNoErrors_x3f___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { @@ -49806,7 +53459,55 @@ goto block_233; } } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__1() { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_9 = lean_ctor_get(x_6, 5); +x_10 = lean_ctor_get(x_2, 2); +lean_inc(x_10); +lean_inc(x_10); +x_11 = l_Lean_Elab_getBetterRef(x_9, x_10); +x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_4, x_5, x_6, x_7, x_8); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(x_13, x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_14); +lean_dec(x_2); +lean_dec(x_10); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_11); +lean_ctor_set(x_18, 1, x_17); +lean_ctor_set_tag(x_15, 1); +lean_ctor_set(x_15, 0, x_18); +return x_15; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_15, 0); +x_20 = lean_ctor_get(x_15, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_15); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_11); +lean_ctor_set(x_21, 1, x_19); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__1() { _start: { lean_object* x_1; @@ -49814,16 +53515,16 @@ x_1 = lean_mk_string_from_bytes("invalid auto implicit argument '", 32); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__1; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__3() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__3() { _start: { lean_object* x_1; @@ -49831,16 +53532,16 @@ x_1 = lean_mk_string_from_bytes("', it depends on explicitly provided argument ' return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__4() { +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__3; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { uint8_t x_14; @@ -49894,11 +53595,11 @@ lean_inc(x_26); lean_dec(x_18); x_27 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_27, 0, x_1); -x_28 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__2; +x_28 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__2; x_29 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_29, 0, x_28); lean_ctor_set(x_29, 1, x_27); -x_30 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__4; +x_30 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__4; x_31 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_31, 0, x_29); lean_ctor_set(x_31, 1, x_30); @@ -49911,7 +53612,7 @@ x_34 = l_Lean_Elab_Term_MVarErrorInfo_logError_addArgName___closed__4; x_35 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_35, 0, x_33); lean_ctor_set(x_35, 1, x_34); -x_36 = l_Lean_throwError___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__1(x_35, x_7, x_8, x_9, x_10, x_11, x_12, x_26); +x_36 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_35, x_7, x_8, x_9, x_10, x_11, x_12, x_26); x_37 = !lean_is_exclusive(x_36); if (x_37 == 0) { @@ -49934,7 +53635,7 @@ return x_40; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__52(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; @@ -49987,7 +53688,7 @@ lean_dec(x_25); x_27 = 0; x_28 = lean_box(0); lean_inc(x_6); -x_29 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_15, x_23, x_1, x_26, x_27, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_24); +x_29 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51(x_15, x_23, x_1, x_26, x_27, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_24); if (lean_obj_tag(x_29) == 0) { lean_object* x_30; size_t x_31; size_t x_32; @@ -50082,7 +53783,7 @@ x_12 = lean_usize_of_nat(x_11); lean_dec(x_11); x_13 = 0; x_14 = lean_box(0); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51(x_1, x_3, x_12, x_13, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__52(x_1, x_3, x_12, x_13, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -50773,7 +54474,20 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_throwError___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { size_t x_14; size_t x_15; lean_object* x_16; @@ -50781,7 +54495,7 @@ x_14 = lean_unbox_usize(x_4); lean_dec(x_4); x_15 = lean_unbox_usize(x_5); lean_dec(x_5); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -50791,7 +54505,7 @@ lean_dec(x_3); return x_16; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__52___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { size_t x_13; size_t x_14; lean_object* x_15; @@ -50799,7 +54513,7 @@ x_13 = lean_unbox_usize(x_3); lean_dec(x_3); x_14 = lean_unbox_usize(x_4); lean_dec(x_4); -x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__52(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -51281,7 +54995,7 @@ lean_dec(x_3); return x_10; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__1() { _start: { lean_object* x_1; @@ -51289,21 +55003,21 @@ x_1 = lean_mk_string_from_bytes("letrec", 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__11; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__2; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__2; x_3 = l_Lean_registerTraceClass(x_2, x_1); return x_3; } @@ -51558,7 +55272,7 @@ if (x_13 == 0) { lean_object* x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_14, 3); +x_15 = lean_ctor_get(x_14, 4); lean_inc(x_15); lean_dec(x_14); x_16 = 0; @@ -51576,7 +55290,7 @@ x_20 = lean_ctor_get(x_12, 1); lean_inc(x_20); lean_inc(x_19); lean_dec(x_12); -x_21 = lean_ctor_get(x_19, 3); +x_21 = lean_ctor_get(x_19, 4); lean_inc(x_21); lean_dec(x_19); x_22 = 0; @@ -51746,7 +55460,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_isLetRecAuxMVar(lean_object* x_1, lean _start: { lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_9 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__2; +x_9 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__2; x_38 = lean_st_ref_get(x_7, x_8); x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); @@ -51818,7 +55532,7 @@ x_23 = l_Lean_Elab_Term_isLetRecAuxMVar___closed__4; x_24 = lean_alloc_ctor(10, 2, 0); lean_ctor_set(x_24, 0, x_22); lean_ctor_set(x_24, 1, x_23); -x_25 = lean_ctor_get(x_17, 3); +x_25 = lean_ctor_get(x_17, 4); lean_inc(x_25); lean_dec(x_17); x_26 = lean_box(0); @@ -59159,12 +62873,13 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(0); x_2 = lean_box(0); x_3 = l_Lean_Elab_Term_instMetaEvalTermElabM___rarg___closed__3; -x_4 = lean_alloc_ctor(0, 5, 0); +x_4 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_1); -lean_ctor_set(x_4, 3, x_2); -lean_ctor_set(x_4, 4, x_3); +lean_ctor_set(x_4, 1, x_1); +lean_ctor_set(x_4, 2, x_2); +lean_ctor_set(x_4, 3, x_1); +lean_ctor_set(x_4, 4, x_2); +lean_ctor_set(x_4, 5, x_3); return x_4; } } @@ -61420,183 +65135,185 @@ lean_dec(x_10); x_13 = !lean_is_exclusive(x_11); if (x_13 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; x_14 = lean_ctor_get(x_11, 0); x_15 = lean_ctor_get(x_11, 4); lean_dec(x_15); -x_16 = l_Lean_addDocString___at_Lean_Elab_Term_expandDeclId___spec__10___closed__1; -x_17 = l_Lean_MapDeclarationExtension_insert___rarg(x_16, x_14, x_1, x_2); -x_18 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__9; -lean_ctor_set(x_11, 4, x_18); -lean_ctor_set(x_11, 0, x_17); -x_19 = lean_st_ref_set(x_8, x_11, x_12); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_st_ref_get(x_8, x_20); -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_st_ref_take(x_6, x_22); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); +x_16 = l___private_Lean_DocString_0__Lean_removeLeadingSpaces(x_2); +x_17 = l_Lean_addDocString___at_Lean_Elab_Term_expandDeclId___spec__10___closed__1; +x_18 = l_Lean_MapDeclarationExtension_insert___rarg(x_17, x_14, x_1, x_16); +x_19 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__9; +lean_ctor_set(x_11, 4, x_19); +lean_ctor_set(x_11, 0, x_18); +x_20 = lean_st_ref_set(x_8, x_11, x_12); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_st_ref_get(x_8, x_21); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_st_ref_take(x_6, x_23); +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_dec(x_23); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = !lean_is_exclusive(x_25); +if (x_27 == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_27 = lean_ctor_get(x_24, 1); -lean_dec(x_27); -x_28 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__19; -lean_ctor_set(x_24, 1, x_28); -x_29 = lean_st_ref_set(x_6, x_24, x_25); -x_30 = !lean_is_exclusive(x_29); -if (x_30 == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_28 = lean_ctor_get(x_25, 1); +lean_dec(x_28); +x_29 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__19; +lean_ctor_set(x_25, 1, x_29); +x_30 = lean_st_ref_set(x_6, x_25, x_26); +x_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) { -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_29, 0); -lean_dec(x_31); -x_32 = lean_box(0); -lean_ctor_set(x_29, 0, x_32); -return x_29; +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_30, 0); +lean_dec(x_32); +x_33 = lean_box(0); +lean_ctor_set(x_30, 0, x_33); +return x_30; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_29, 1); -lean_inc(x_33); -lean_dec(x_29); -x_34 = lean_box(0); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_33); -return x_35; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_30, 1); +lean_inc(x_34); +lean_dec(x_30); +x_35 = lean_box(0); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_34); +return x_36; } } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_36 = lean_ctor_get(x_24, 0); -x_37 = lean_ctor_get(x_24, 2); -x_38 = lean_ctor_get(x_24, 3); +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_37 = lean_ctor_get(x_25, 0); +x_38 = lean_ctor_get(x_25, 2); +x_39 = lean_ctor_get(x_25, 3); +lean_inc(x_39); lean_inc(x_38); lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_24); -x_39 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__19; -x_40 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_40, 0, x_36); -lean_ctor_set(x_40, 1, x_39); -lean_ctor_set(x_40, 2, x_37); -lean_ctor_set(x_40, 3, x_38); -x_41 = lean_st_ref_set(x_6, x_40, x_25); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -if (lean_is_exclusive(x_41)) { - lean_ctor_release(x_41, 0); - lean_ctor_release(x_41, 1); - x_43 = x_41; +lean_dec(x_25); +x_40 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__19; +x_41 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_41, 0, x_37); +lean_ctor_set(x_41, 1, x_40); +lean_ctor_set(x_41, 2, x_38); +lean_ctor_set(x_41, 3, x_39); +x_42 = lean_st_ref_set(x_6, x_41, x_26); +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + x_44 = x_42; } else { - lean_dec_ref(x_41); - x_43 = lean_box(0); + lean_dec_ref(x_42); + x_44 = lean_box(0); } -x_44 = lean_box(0); -if (lean_is_scalar(x_43)) { - x_45 = lean_alloc_ctor(0, 2, 0); +x_45 = lean_box(0); +if (lean_is_scalar(x_44)) { + x_46 = lean_alloc_ctor(0, 2, 0); } else { - x_45 = x_43; + x_46 = x_44; } -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_42); -return x_45; +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_43); +return x_46; } } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_46 = lean_ctor_get(x_11, 0); -x_47 = lean_ctor_get(x_11, 1); -x_48 = lean_ctor_get(x_11, 2); -x_49 = lean_ctor_get(x_11, 3); -x_50 = lean_ctor_get(x_11, 5); +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; +x_47 = lean_ctor_get(x_11, 0); +x_48 = lean_ctor_get(x_11, 1); +x_49 = lean_ctor_get(x_11, 2); +x_50 = lean_ctor_get(x_11, 3); +x_51 = lean_ctor_get(x_11, 5); +lean_inc(x_51); lean_inc(x_50); lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); -lean_inc(x_46); lean_dec(x_11); -x_51 = l_Lean_addDocString___at_Lean_Elab_Term_expandDeclId___spec__10___closed__1; -x_52 = l_Lean_MapDeclarationExtension_insert___rarg(x_51, x_46, x_1, x_2); -x_53 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__9; -x_54 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_47); -lean_ctor_set(x_54, 2, x_48); -lean_ctor_set(x_54, 3, x_49); -lean_ctor_set(x_54, 4, x_53); -lean_ctor_set(x_54, 5, x_50); -x_55 = lean_st_ref_set(x_8, x_54, x_12); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -x_57 = lean_st_ref_get(x_8, x_56); +x_52 = l___private_Lean_DocString_0__Lean_removeLeadingSpaces(x_2); +x_53 = l_Lean_addDocString___at_Lean_Elab_Term_expandDeclId___spec__10___closed__1; +x_54 = l_Lean_MapDeclarationExtension_insert___rarg(x_53, x_47, x_1, x_52); +x_55 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__9; +x_56 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_48); +lean_ctor_set(x_56, 2, x_49); +lean_ctor_set(x_56, 3, x_50); +lean_ctor_set(x_56, 4, x_55); +lean_ctor_set(x_56, 5, x_51); +x_57 = lean_st_ref_set(x_8, x_56, x_12); x_58 = lean_ctor_get(x_57, 1); lean_inc(x_58); lean_dec(x_57); -x_59 = lean_st_ref_take(x_6, x_58); -x_60 = lean_ctor_get(x_59, 0); +x_59 = lean_st_ref_get(x_8, x_58); +x_60 = lean_ctor_get(x_59, 1); lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); lean_dec(x_59); -x_62 = lean_ctor_get(x_60, 0); +x_61 = lean_st_ref_take(x_6, x_60); +x_62 = lean_ctor_get(x_61, 0); lean_inc(x_62); -x_63 = lean_ctor_get(x_60, 2); +x_63 = lean_ctor_get(x_61, 1); lean_inc(x_63); -x_64 = lean_ctor_get(x_60, 3); +lean_dec(x_61); +x_64 = lean_ctor_get(x_62, 0); lean_inc(x_64); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - lean_ctor_release(x_60, 2); - lean_ctor_release(x_60, 3); - x_65 = x_60; +x_65 = lean_ctor_get(x_62, 2); +lean_inc(x_65); +x_66 = lean_ctor_get(x_62, 3); +lean_inc(x_66); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + lean_ctor_release(x_62, 2); + lean_ctor_release(x_62, 3); + x_67 = x_62; } else { - lean_dec_ref(x_60); - x_65 = lean_box(0); + lean_dec_ref(x_62); + x_67 = lean_box(0); } -x_66 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__19; -if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 4, 0); +x_68 = l_Lean_Elab_Tactic_instInhabitedSnapshot___closed__19; +if (lean_is_scalar(x_67)) { + x_69 = lean_alloc_ctor(0, 4, 0); } else { - x_67 = x_65; + x_69 = x_67; } -lean_ctor_set(x_67, 0, x_62); -lean_ctor_set(x_67, 1, x_66); -lean_ctor_set(x_67, 2, x_63); -lean_ctor_set(x_67, 3, x_64); -x_68 = lean_st_ref_set(x_6, x_67, x_61); -x_69 = lean_ctor_get(x_68, 1); -lean_inc(x_69); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_70 = x_68; +lean_ctor_set(x_69, 0, x_64); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_69, 2, x_65); +lean_ctor_set(x_69, 3, x_66); +x_70 = lean_st_ref_set(x_6, x_69, x_63); +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_72 = x_70; } else { - lean_dec_ref(x_68); - x_70 = lean_box(0); + lean_dec_ref(x_70); + x_72 = lean_box(0); } -x_71 = lean_box(0); -if (lean_is_scalar(x_70)) { - x_72 = lean_alloc_ctor(0, 2, 0); +x_73 = lean_box(0); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(0, 2, 0); } else { - x_72 = x_70; + x_74 = x_72; } -lean_ctor_set(x_72, 0, x_71); -lean_ctor_set(x_72, 1, x_69); -return x_72; +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_71); +return x_74; } } } @@ -63059,7 +66776,7 @@ x_3 = lean_alloc_closure((void*)(l_Lean_Elab_withoutModifyingStateWithInfoAndMes return x_3; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__1() { _start: { lean_object* x_1; @@ -63067,17 +66784,17 @@ x_1 = lean_mk_string_from_bytes("debug", 5); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Term_MVarErrorInfo_logError___closed__11; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__1; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -63097,7 +66814,7 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); -x_8 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__2; +x_8 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__2; x_9 = l_Lean_registerTraceClass(x_8, x_7); return x_9; } @@ -63229,6 +66946,8 @@ lean_dec_ref(res); res = initialize_Lean_Elab_DeclModifiers(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l_Lean_Elab_Term_instInhabitedSyntheticMVarKind = _init_l_Lean_Elab_Term_instInhabitedSyntheticMVarKind(); +lean_mark_persistent(l_Lean_Elab_Term_instInhabitedSyntheticMVarKind); l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__1 = _init_l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__1); l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__2 = _init_l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__2(); @@ -63237,6 +66956,10 @@ l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__3 = _init_l_Lean_Elab_T lean_mark_persistent(l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__3); l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__4 = _init_l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__4(); lean_mark_persistent(l_Lean_Elab_Term_instToStringSyntheticMVarKind___closed__4); +l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl___closed__1 = _init_l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl___closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl___closed__1); +l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl = _init_l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl(); +lean_mark_persistent(l_Lean_Elab_Term_instInhabitedSyntheticMVarDecl); l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__1 = _init_l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__1); l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__2 = _init_l_Lean_Elab_Term_instInhabitedMVarErrorKind___closed__2(); @@ -63278,6 +67001,8 @@ l_Lean_Elab_Term_State_levelNames___default = _init_l_Lean_Elab_Term_State_level lean_mark_persistent(l_Lean_Elab_Term_State_levelNames___default); l_Lean_Elab_Term_State_syntheticMVars___default = _init_l_Lean_Elab_Term_State_syntheticMVars___default(); lean_mark_persistent(l_Lean_Elab_Term_State_syntheticMVars___default); +l_Lean_Elab_Term_State_pendingMVars___default = _init_l_Lean_Elab_Term_State_pendingMVars___default(); +lean_mark_persistent(l_Lean_Elab_Term_State_pendingMVars___default); l_Lean_Elab_Term_State_mvarErrorInfos___default = _init_l_Lean_Elab_Term_State_mvarErrorInfos___default(); lean_mark_persistent(l_Lean_Elab_Term_State_mvarErrorInfos___default); l_Lean_Elab_Term_State_letRecsToLift___default = _init_l_Lean_Elab_Term_State_letRecsToLift___default(); @@ -63501,7 +67226,7 @@ l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__17 = _init_l_Lean_Elab_Term lean_mark_persistent(l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__17); l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__18 = _init_l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__18(); lean_mark_persistent(l_Lean_Elab_Term_mkTermElabAttributeUnsafe___closed__18); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_2191_(lean_io_mk_world()); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_2187_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Term_termElabAttribute = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Term_termElabAttribute); @@ -63606,8 +67331,10 @@ l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__1 = _init_l_Lean_Elab_Term_m lean_mark_persistent(l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__1); l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__2 = _init_l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__2(); lean_mark_persistent(l_Lean_Elab_Term_mkFreshBinderName___rarg___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__2___closed__1); +l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__1 = _init_l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__1); +l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2 = _init_l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_logException___at___private_Lean_Elab_Term_0__Lean_Elab_Term_applyAttributesCore___spec__3___closed__2); l_Lean_Elab_Term_mkTypeMismatchError___closed__1 = _init_l_Lean_Elab_Term_mkTypeMismatchError___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_mkTypeMismatchError___closed__1); l_Lean_Elab_Term_mkTypeMismatchError___closed__2 = _init_l_Lean_Elab_Term_mkTypeMismatchError___closed__2(); @@ -63652,28 +67379,28 @@ l_Lean_Elab_Term_synthesizeInstMVarCore___closed__4 = _init_l_Lean_Elab_Term_syn lean_mark_persistent(l_Lean_Elab_Term_synthesizeInstMVarCore___closed__4); l_Lean_Elab_Term_synthesizeInstMVarCore___closed__5 = _init_l_Lean_Elab_Term_synthesizeInstMVarCore___closed__5(); lean_mark_persistent(l_Lean_Elab_Term_synthesizeInstMVarCore___closed__5); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818____closed__4); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5818_(lean_io_mk_world()); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741____closed__4); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5741_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Term_autoLift = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Term_autoLift); lean_dec_ref(res); -}l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844____closed__4); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5844_(lean_io_mk_world()); +}l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767____closed__4); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_5767_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Term_maxCoeSize = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Term_maxCoeSize); @@ -63748,10 +67475,6 @@ l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__15 = _init_ lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_tryLiftAndCoe___closed__15); l___private_Lean_Elab_Term_0__Lean_Elab_Term_mkSyntheticSorryFor___closed__1 = _init_l___private_Lean_Elab_Term_0__Lean_Elab_Term_mkSyntheticSorryFor___closed__1(); lean_mark_persistent(l___private_Lean_Elab_Term_0__Lean_Elab_Term_mkSyntheticSorryFor___closed__1); -l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__1 = _init_l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__1); -l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__2 = _init_l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_logException___at_Lean_Elab_Term_exceptionToSorry___spec__1___closed__2); l_Lean_Elab_throwPostpone___at_Lean_Elab_Term_tryPostpone___spec__1___rarg___closed__1 = _init_l_Lean_Elab_throwPostpone___at_Lean_Elab_Term_tryPostpone___spec__1___rarg___closed__1(); lean_mark_persistent(l_Lean_Elab_throwPostpone___at_Lean_Elab_Term_tryPostpone___spec__1___rarg___closed__1); l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__1 = _init_l_Lean_Elab_Term_tryPostponeIfHasMVars___closed__1(); @@ -63941,25 +67664,25 @@ l_Lean_Elab_Term_collectUnassignedMVars_go___closed__2 = _init_l_Lean_Elab_Term_ lean_mark_persistent(l_Lean_Elab_Term_collectUnassignedMVars_go___closed__2); l_Lean_localDeclDependsOn___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__1___closed__1 = _init_l_Lean_localDeclDependsOn___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__1___closed__1(); lean_mark_persistent(l_Lean_localDeclDependsOn___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__1___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__1); -l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__2); -l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__3); -l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__50___closed__4); +l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__1); +l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__2); +l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__3 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__3); +l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__4 = _init_l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Elab_Term_addAutoBoundImplicits_go___spec__51___closed__4); l_Lean_Elab_Term_addAutoBoundImplicits_go___closed__1 = _init_l_Lean_Elab_Term_addAutoBoundImplicits_go___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_addAutoBoundImplicits_go___closed__1); l_Lean_Elab_Term_mkAuxName___closed__1 = _init_l_Lean_Elab_Term_mkAuxName___closed__1(); lean_mark_persistent(l_Lean_Elab_Term_mkAuxName___closed__1); l_Lean_Elab_Term_mkAuxName___closed__2 = _init_l_Lean_Elab_Term_mkAuxName___closed__2(); lean_mark_persistent(l_Lean_Elab_Term_mkAuxName___closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425____closed__2); -res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13425_(lean_io_mk_world()); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268____closed__2); +res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_Term___hyg_13268_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Elab_Term_isLetRecAuxMVar___lambda__2___closed__1 = _init_l_Lean_Elab_Term_isLetRecAuxMVar___lambda__2___closed__1(); @@ -64120,11 +67843,11 @@ l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4 = _init_l_Lean_Elab_Term_e lean_mark_persistent(l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__4); l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__5 = _init_l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__5(); lean_mark_persistent(l_Lean_Elab_Term_exprToSyntax___lambda__1___closed__5); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077____closed__2); -res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_16077_(lean_io_mk_world()); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920____closed__2); +res = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_15920_(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/Util.c b/stage0/stdlib/Lean/Elab/Util.c index e194b5580c04..589d53de14a9 100644 --- a/stage0/stdlib/Lean/Elab/Util.c +++ b/stage0/stdlib/Lean/Elab/Util.c @@ -125,6 +125,7 @@ lean_object* l_Lean_Name_toString(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Elab_mkElabAttribute___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldl___at_Lean_Elab_addMacroStack___spec__1___closed__3; lean_object* l_Lean_ResolveName_resolveNamespace(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_withLogging___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_name_append_index_after(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkSyntaxNodeKind___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_mkMacroAttributeUnsafe___closed__10; @@ -136,7 +137,7 @@ lean_object* l_Lean_Name_toExprAux(lean_object*); static lean_object* l_Lean_Elab_mkElabAttribute___rarg___lambda__2___closed__17; lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_expandMacroImpl_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_291_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_930_(lean_object*); static lean_object* l_Lean_Elab_mkElabAttribute___rarg___lambda__2___closed__8; @@ -244,7 +245,6 @@ uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); lean_object* l_Lean_InternalExceptionId_getName___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_expandOptNamedPrio___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_expandOptNamedPrio___closed__8; -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_checkSyntaxNodeKind___at_Lean_Elab_checkSyntaxNodeKindAtCurrentNamespaces___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_logException___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_expandOptNamedPrio___closed__1; @@ -257,10 +257,11 @@ LEAN_EXPORT lean_object* l_Lean_Elab_nestedExceptionToMessageData___rarg___lambd lean_object* l_Lean_mkNatLit(lean_object*); lean_object* l_Lean_mkStrLit(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkSyntaxNodeKindAtCurrentNamespaces(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__2; +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__2; static lean_object* l_Lean_Elab_mkMacroAttributeUnsafe___closed__2; lean_object* l_Lean_log___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Elab_liftMacroM___spec__3___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__1; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Elab_expandMacroImpl_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_expandOptNamedPrio___closed__4; uint8_t l_List_isEmpty___rarg(lean_object*); @@ -268,6 +269,7 @@ static lean_object* l_Lean_Elab_mkElabAttribute___rarg___lambda__2___closed__20; lean_object* l_Lean_KeyedDeclsAttribute_init___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_checkSyntaxNodeKindAtNamespaces___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_mkElabAttribute___rarg___lambda__2___closed__10; +LEAN_EXPORT lean_object* l_Lean_Elab_withLogging(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_liftMacroM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_addMacroStack___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_addMacroStack___rarg___lambda__1___closed__1; @@ -3862,6 +3864,30 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Elab_logException___rarg), 5, 0); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Elab_withLogging___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 1); +lean_inc(x_7); +lean_dec(x_3); +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_logException___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +lean_closure_set(x_8, 3, x_5); +x_9 = lean_apply_3(x_7, lean_box(0), x_6, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_withLogging(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_withLogging___rarg), 6, 0); +return x_2; +} +} LEAN_EXPORT lean_object* l_Lean_Elab_trace___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) { _start: { @@ -4368,7 +4394,7 @@ x_8 = l_Array_mapMUnsafe_map___at_Lean_Elab_throwErrorWithNestedErrors___spec__1 return x_8; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__1() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__1() { _start: { lean_object* x_1; @@ -4376,17 +4402,17 @@ x_1 = lean_mk_string_from_bytes("step", 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__2() { +static lean_object* _init_l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_logDbgTrace___rarg___closed__1; -x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__1; +x_2 = l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -4398,7 +4424,7 @@ lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_ctor_get(x_3, 1); lean_inc(x_4); lean_dec(x_3); -x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__2; +x_5 = l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__2; x_6 = l_Lean_registerTraceClass(x_5, x_4); return x_6; } @@ -4647,11 +4673,11 @@ l_Lean_Elab_throwErrorWithNestedErrors___rarg___lambda__1___closed__1 = _init_l_ lean_mark_persistent(l_Lean_Elab_throwErrorWithNestedErrors___rarg___lambda__1___closed__1); l_Lean_Elab_throwErrorWithNestedErrors___rarg___lambda__1___closed__2 = _init_l_Lean_Elab_throwErrorWithNestedErrors___rarg___lambda__1___closed__2(); lean_mark_persistent(l_Lean_Elab_throwErrorWithNestedErrors___rarg___lambda__1___closed__2); -l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__1(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__1); -l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__2(); -lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344____closed__2); -res = l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2344_(lean_io_mk_world()); +l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__1 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__1(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__1); +l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__2 = _init_l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__2(); +lean_mark_persistent(l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386____closed__2); +res = l_Lean_Elab_initFn____x40_Lean_Elab_Util___hyg_2386_(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/Expr.c b/stage0/stdlib/Lean/Expr.c index 43fa2d30a0af..909e1a78e56a 100644 --- a/stage0/stdlib/Lean/Expr.c +++ b/stage0/stdlib/Lean/Expr.c @@ -13,6 +13,7 @@ #ifdef __cplusplus extern "C" { #endif +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__45; lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_BinderInfo_isImplicit___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isBinding___boxed(lean_object*); @@ -22,8 +23,7 @@ static lean_object* l_Lean_mkNatLit___closed__8; LEAN_EXPORT lean_object* l_Lean_instLTLiteral; static lean_object* l_Lean_mkLHSGoal___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_bindingInfo_x21(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateSort___boxed(lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__40; lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_mkDecIsFalse___closed__2; @@ -31,6 +31,7 @@ static lean_object* l_Lean_Expr_bvarIdx_x21___closed__3; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__16; size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Expr_Data_hash___boxed(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__2; LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instReprData__1___lambda__3___closed__1; static lean_object* l_Lean_mkNatLit___closed__4; @@ -43,11 +44,11 @@ LEAN_EXPORT lean_object* l_Lean_Expr_letName_x21(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isNatLit(lean_object*); static lean_object* l_Lean_Expr_replaceFVar___closed__1; LEAN_EXPORT lean_object* l_Lean_mkFreshMVarId___rarg(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_replaceFVar___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Expr_projIdx_x21___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateLambda___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getAppNumArgs___boxed(lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lean_Expr_projExpr_x21___closed__3; @@ -60,6 +61,7 @@ LEAN_EXPORT uint8_t l_Lean_Expr_isHeadBetaTargetFn(uint8_t, lean_object*); uint8_t lean_uint64_dec_eq(uint64_t, uint64_t); static lean_object* l_Lean_Expr_bindingDomain_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_letBody_x21(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__27; LEAN_EXPORT lean_object* l_Lean_Expr_abstract___boxed(lean_object*, lean_object*); static lean_object* l_Lean_instReprExpr___closed__1; static lean_object* l_Lean_Expr_getRevArg_x21___closed__1; @@ -68,15 +70,14 @@ static lean_object* l_Lean_mkNatLit___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Expr_traverseApp___spec__1(lean_object*); static lean_object* l_Lean_Expr_letBody_x21___closed__1; -LEAN_EXPORT lean_object* l_Lean_Expr_updateConst___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_mkDecIsTrue___closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_withApp(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_eqv___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isMData(lean_object*); -LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_patternAnnotation_x3f___boxed(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__9; LEAN_EXPORT lean_object* l_Lean_Expr_letBody_x21___boxed(lean_object*); uint8_t lean_uint8_dec_eq(uint8_t, uint8_t); static lean_object* l_Lean_mkDecIsFalse___closed__1; @@ -94,12 +95,14 @@ static lean_object* l_Lean_Expr_instHashableExpr___closed__1; static lean_object* l_Lean_mkInaccessible___closed__1; LEAN_EXPORT uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1848_(lean_object*); static lean_object* l_Lean_Expr_litValue_x21___closed__1; -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); uint32_t lean_uint8_to_uint32(uint8_t); LEAN_EXPORT lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); static lean_object* l_Lean_Expr_letBody_x21___closed__2; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__17; LEAN_EXPORT lean_object* l_Lean_Expr_getAppArgs(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__8; static lean_object* l_Lean_Expr_projIdx_x21___closed__2; +lean_object* l_Lean_Level_succ___override(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_etaExpandedBody(lean_object*, lean_object*, lean_object*); extern lean_object* l_Std_Format_defWidth; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_mkAppN___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -107,18 +110,17 @@ static lean_object* l_Lean_mkEM___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_isLit___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_replaceFVars___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_approxDepth___boxed(lean_object*); -static lean_object* l_Lean_Expr_updateLambda_x21___closed__3; uint64_t lean_uint64_add(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_bindingInfo_x21___closed__1; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__24; +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ExprStructEq_instHashableExprStructEq; LEAN_EXPORT lean_object* l_Lean_Expr_letE___override___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_bool_to_uint64(uint8_t); -static lean_object* l_Lean_Expr_updateMData_x21___closed__2; static lean_object* l_Lean_mkNatLit___closed__9; LEAN_EXPORT uint8_t l_Lean_Expr_isArrow(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__3; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkOr(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Expr_instantiateLevelParams___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); @@ -128,10 +130,8 @@ static lean_object* l_Lean_Expr_letValue_x21___closed__2; static lean_object* l_Lean_Expr_mkAppData___closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_isOptParam___boxed(lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__11; -static lean_object* l_Lean_Expr_updateMData_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_mkForallEx___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkLambda___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__49; LEAN_EXPORT lean_object* l_Lean_Expr_getAutoParamTactic_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkLit(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getAppRevArgs(lean_object*); @@ -142,6 +142,7 @@ LEAN_EXPORT lean_object* l_Lean_mkLHSGoal(lean_object*); uint8_t lean_uint32_to_uint8(uint32_t); static lean_object* l_Lean_mkDecIsTrue___closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_mkAppData(uint64_t, uint64_t); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__28; LEAN_EXPORT lean_object* l_Lean_instFVarIdSetEmptyCollection; LEAN_EXPORT lean_object* l_Lean_mkMVar(lean_object*); size_t lean_usize_sub(size_t, size_t); @@ -149,15 +150,17 @@ LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_etaExpandedAux(lean_ LEAN_EXPORT lean_object* l_Lean_Expr_hash___boxed(lean_object*); static lean_object* l_Lean_Expr_appFn_x21_x27___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_betaRev___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__18; +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl(lean_object*, lean_object*); static lean_object* l_Lean_Literal_type___closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_mvarId_x21___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_appFn_x21_x27___boxed(lean_object*); static lean_object* l_Lean_instReprData__1___lambda__3___closed__2; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__16; static lean_object* l_Lean_Expr_ctorName___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParamsArray(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_litValue_x21___closed__3; static lean_object* l_Lean_Expr_constName_x21___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); static lean_object* l_Lean_Expr_mvarId_x21___closed__1; uint8_t l_Lean_Level_hasMVar(lean_object*); @@ -167,6 +170,8 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppRev___rarg(lean_object*, lean_object lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); static lean_object* l_Lean_Expr_mkData___closed__3; LEAN_EXPORT lean_object* l_Lean_annotation_x3f___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__14; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__30; LEAN_EXPORT lean_object* l_Lean_Expr_mkDataForBinder(uint64_t, lean_object*, uint32_t, uint8_t, uint8_t, uint8_t, uint8_t, uint8_t); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_patternWithRef_x3f___boxed(lean_object*); @@ -180,19 +185,18 @@ LEAN_EXPORT lean_object* l_Lean_Expr_binderInfoEx___boxed(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isApp(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_Data_binderInfo___boxed(lean_object*); static lean_object* l_Lean_Expr_ctorName___closed__2; -static lean_object* l_Lean_Expr_updateApp_x21___closed__2; LEAN_EXPORT uint8_t l_Lean_Expr_hasLooseBVarInExplicitDomain(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Expr_hasFVarEx___boxed(lean_object*); uint64_t l_Lean_Level_hash(lean_object*); static lean_object* l_Lean_Expr_ctorName___closed__8; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__26; LEAN_EXPORT lean_object* l_Lean_Expr_lt___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateLet___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_appFn_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_hasLevelMVar___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isAutoParam___boxed(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); static lean_object* l_Lean_Expr_mkData___closed__5; +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl(lean_object*, lean_object*); static lean_object* l_Lean_Expr_mvarId_x21___closed__2; static lean_object* l_Lean_mkSimpleThunkType___closed__1; LEAN_EXPORT lean_object* l_Lean_BinderInfo_toUInt64___boxed(lean_object*); @@ -201,26 +205,28 @@ LEAN_EXPORT lean_object* l_Lean_BinderInfo_toCtorIdx(uint8_t); static lean_object* l_Lean_Expr_ctorName___closed__4; LEAN_EXPORT uint8_t l_Lean_Expr_isBVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__3; lean_object* lean_expr_instantiate1(lean_object*, lean_object*); static lean_object* l_Lean_Literal_type___closed__3; lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__15; lean_object* lean_expr_lift_loose_bvars(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Expr_traverseApp___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Expr_traverseApp___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkLetFunAnnotation(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l_Lean_Expr_appFn_x21_x27___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__1; LEAN_EXPORT uint8_t lean_expr_has_level_mvar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_ExprStructEq_instBEqExprStructEq___closed__1; -static lean_object* l_Lean_Expr_updateForall_x21___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__44; static lean_object* l_Lean_ExprStructEq_instHashableExprStructEq___closed__1; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__32; static lean_object* l_Lean_Expr_appFn_x21___closed__3; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__20; +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getOptParamDefault_x3f(lean_object*); -LEAN_EXPORT uint8_t l_Lean_Expr_ptrEq(lean_object*, lean_object*); +uint8_t l_ptrEqList___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getRevArgD(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Expr_instantiateLevelParams___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_getAppArgs___closed__1; @@ -228,41 +234,34 @@ static lean_object* l_Lean_mkNatLit___closed__2; uint8_t l_Lean_Level_hasParam(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Expr_0__Lean_beqFVarId____x40_Lean_Expr___hyg_1793_(lean_object*, lean_object*); lean_object* l_Std_mkHashSetImp___rarg(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__43; LEAN_EXPORT uint8_t l_Lean_instDecidableLtLiteralInstLTLiteral(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateApp_x21(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_mkAppRevRange(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Expr_const___override___spec__2___boxed(lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__14; -LEAN_EXPORT lean_object* l_Lean_Expr_updateForall_x21___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__10; LEAN_EXPORT lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l_Lean_Expr_fvarId_x21___closed__2; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__2; uint8_t lean_expr_lt(lean_object*, lean_object*); static lean_object* l_Lean_Expr_sortLevel_x21___closed__3; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__47; +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); static lean_object* l_Lean_Expr_letName_x21___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__2; static lean_object* l_Lean_Expr_projExpr_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_replaceFVars(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_mdataExpr_x21(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__18; uint32_t lean_uint32_of_nat(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_letName_x21___boxed(lean_object*); static lean_object* l_Lean_Expr_projExpr_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_instCoeExprExprStructEq___boxed(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__30; LEAN_EXPORT lean_object* l_Lean_Expr_projExpr_x21___boxed(lean_object*); -static lean_object* l_Lean_Expr_updateForall_x21___closed__3; -LEAN_EXPORT lean_object* l_Lean_Expr_updateForall_x21(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_looseBVarRange___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_mkDataForBinder___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_BinderInfo_hash___boxed(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__15; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_mkAppRev___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_lit___override(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__28; LEAN_EXPORT lean_object* l_Lean_Expr_containsFVar___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ctorName___boxed(lean_object*); LEAN_EXPORT lean_object* lean_expr_mk_forall(lean_object*, lean_object*, lean_object*, uint8_t); @@ -271,11 +270,12 @@ static lean_object* l_Lean_Expr_bindingName_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_setOption(lean_object*); extern lean_object* l_Lean_levelZero; LEAN_EXPORT lean_object* l_Lean_ExprStructEq_instBEqExprStructEq; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__3; lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__6; LEAN_EXPORT lean_object* l_Lean_Expr_hasExprMVarEx___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_instReprLiteral; LEAN_EXPORT lean_object* l_Lean_Expr_hasExprMVar___boxed(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__46; static lean_object* l_Lean_Expr_setPPExplicit___closed__4; uint16_t lean_uint16_add(uint16_t, uint16_t); LEAN_EXPORT lean_object* l_Lean_Expr_getAppNumArgs(lean_object*); @@ -284,9 +284,9 @@ LEAN_EXPORT lean_object* l_Lean_instReprFVarId(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_bindingName_x21___boxed(lean_object*); static lean_object* l_Lean_Expr_updateLambdaE_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_getAppFn___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_mkOr___closed__1; static lean_object* l_Lean_instReprData__1___lambda__5___closed__1; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__42; uint32_t lean_uint32_add(uint32_t, uint32_t); static lean_object* l_Lean_Expr_sortLevel_x21___closed__2; LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Expr_const___override___spec__2(uint8_t, lean_object*); @@ -294,17 +294,19 @@ static lean_object* l_Lean_instReprData__1___lambda__4___closed__1; uint8_t lean_expr_has_loose_bvar(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkAppN(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_natLit_x3f___boxed(lean_object*); +lean_object* l_Lean_simpLevelIMax_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkMData(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__25; static lean_object* l_Lean_mkOr___closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_Data_approxDepth___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParamsCore(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__29; LEAN_EXPORT lean_object* l_Lean_Expr_updateFn___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_sortLevel_x21___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkDecIsTrue(lean_object*, lean_object*); extern uint64_t l_instInhabitedUInt64; LEAN_EXPORT lean_object* l_Lean_mkLet___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__19; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__37; LEAN_EXPORT lean_object* l_Lean_BinderInfo_noConfusion___rarg(uint8_t, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_forallE___override___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_lower_loose_bvars(lean_object*, lean_object*, lean_object*); @@ -324,16 +326,15 @@ LEAN_EXPORT lean_object* l_Lean_Expr_isConstOf___boxed(lean_object*, lean_object LEAN_EXPORT lean_object* lean_expr_mk_mdata(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instBEqBinderInfo; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__1; -static lean_object* l_Lean_Expr_updateSort_x21___closed__3; LEAN_EXPORT uint64_t l_Lean_BinderInfo_toUInt64(uint8_t); LEAN_EXPORT lean_object* l_Lean_Expr_lam___override___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_letName_x21___closed__3; static lean_object* l_Lean_mkEM___closed__3; -LEAN_EXPORT lean_object* l_Lean_Expr_updateLambda_x21(lean_object*, uint8_t, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__35; LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprLiteral____x40_Lean_Expr___hyg_109_(lean_object*, lean_object*); static lean_object* l_Lean_instHashableFVarId___closed__1; -static lean_object* l_Lean_Expr_updateForall_x21___closed__2; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__39; static lean_object* l_Lean_Expr_updateLambdaE_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_mkProj(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instReprFVarId___boxed(lean_object*, lean_object*); @@ -343,42 +344,42 @@ lean_object* lean_expr_instantiate_rev_range(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_Lean_Expr_updateFn(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_ExprStructEq_beq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateApp___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__48; static lean_object* l_Lean_instReprData__1___lambda__6___closed__1; LEAN_EXPORT lean_object* l_Lean_ExprStructEq_beq___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateSort_x21(lean_object*, lean_object*); LEAN_EXPORT uint8_t lean_expr_has_expr_mvar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_setPPUniverses(lean_object*, uint8_t); LEAN_EXPORT lean_object* lean_expr_consume_type_annotations(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_mvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_traverseApp___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__7; LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____boxed(lean_object*, lean_object*); static lean_object* l_Lean_Expr_constName_x21___closed__3; static lean_object* l_Lean_Literal_type___closed__6; LEAN_EXPORT uint8_t l_Lean_Expr_hasLevelParam(lean_object*); LEAN_EXPORT lean_object* l_Lean_instCoeExprExprStructEq(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateConst_x21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instEmptyCollectionFVarIdMap(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__11; LEAN_EXPORT lean_object* l_Lean_Expr_projExpr_x21(lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__2; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__3; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__36; LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__46; LEAN_EXPORT lean_object* l_Lean_Expr_constLevels_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_hasLevelParam___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_beqLiteral____x40_Lean_Expr___hyg_31____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_patternAnnotation_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_instFVarIdSetInhabited; static lean_object* l_Lean_Expr_sortLevel_x21___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__2; LEAN_EXPORT uint8_t lean_expr_has_mvar(lean_object*); static lean_object* l_Lean_Expr_mkData___closed__7; LEAN_EXPORT lean_object* l_Lean_mkRawNatLit(lean_object*); static lean_object* l_Lean_mkNatLit___closed__6; +LEAN_EXPORT lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); uint8_t l_Lean_KVMap_getBool(lean_object*, lean_object*, uint8_t); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__9; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__25; static lean_object* l_Lean_Expr_ctorName___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_mkAppRevRangeAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_BinderInfo_noConfusion___rarg___closed__1; @@ -389,11 +390,13 @@ lean_object* l_panic___at_Lean_Level_normalize___spec__1(lean_object*); static lean_object* l_Lean_isLHSGoal_x3f___closed__1; LEAN_EXPORT uint8_t lean_expr_binder_info(lean_object*); static lean_object* l_Lean_Expr_mkData___closed__2; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__29; -lean_object* lean_level_update_max(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkAnnotation(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_letFunAnnotation_x3f___boxed(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__1; +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_BinderInfo_isStrictImplicit(uint8_t); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__43; LEAN_EXPORT lean_object* l_Lean_Expr_looseBVarRangeEx___boxed(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_hasExprMVar(lean_object*); LEAN_EXPORT uint8_t lean_is_out_param(lean_object*); @@ -401,6 +404,7 @@ lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_abstractRange___boxed(lean_object*, lean_object*, lean_object*); uint32_t lean_uint64_to_uint32(uint64_t); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__27; +lean_object* l_Lean_simpLevelMax_x27(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkFreshId___rarg(lean_object*, lean_object*); uint8_t lean_uint32_dec_lt(uint32_t, uint32_t); LEAN_EXPORT lean_object* l_Lean_instInhabitedLiteral; @@ -417,7 +421,7 @@ LEAN_EXPORT uint8_t l_Lean_Expr_isHeadBetaTarget(lean_object*, uint8_t); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__17; LEAN_EXPORT uint8_t l_Lean_Expr_isBinding(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_bindingBody_x21___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateProj_x21(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); static uint32_t l_Lean_Expr_mkAppData___closed__1; static lean_object* l_Lean_Expr_appArg_x21_x27___closed__2; @@ -427,23 +431,22 @@ static lean_object* l_Lean_mkDecIsTrue___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParams(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getAutoParamTactic_x3f___boxed(lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__8; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__33; LEAN_EXPORT lean_object* l_Lean_Expr_Data_hasLevelParam___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isFVar___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Expr_setAppPPExplicitForExposingMVars___spec__1(size_t, size_t, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__22; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__6; lean_object* l_Nat_repr(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_Data_hasFVar(uint64_t); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__22; static lean_object* l_Lean_Expr_instBEqExpr___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_hasMVarEx___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkAppRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint32_t l_Lean_Expr_approxDepth(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_ptrEq___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_setAppPPExplicitForExposingMVars(lean_object*); static lean_object* l_Lean_Expr_fvarId_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_isType___boxed(lean_object*); -static lean_object* l_Lean_Expr_updateConst_x21___closed__2; LEAN_EXPORT lean_object* lean_expr_mk_bvar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_instHashableExpr; static lean_object* l_Lean_mkDecIsTrue___closed__2; @@ -469,60 +472,59 @@ static lean_object* l_Lean_isLHSGoal_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_natLit_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_BinderInfo_noConfusion___rarg___lambda__1(lean_object*); LEAN_EXPORT lean_object* lean_expr_mk_const(lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__38; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__21; LEAN_EXPORT lean_object* l_Lean_mkAppRange(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_isCharLit___closed__3; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__33; static lean_object* l_Lean_mkEM___closed__5; static lean_object* l_Lean_mkOr___closed__2; static lean_object* l_Lean_Expr_mkAppData___closed__2; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__24; static lean_object* l_Lean_Expr_mdataExpr_x21___closed__3; static lean_object* l_Lean_Literal_type___closed__4; static lean_object* l_Lean_mkDecIsTrue___closed__4; LEAN_EXPORT lean_object* lean_expr_mk_lit(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateMData_x21(lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__23; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__7; LEAN_EXPORT uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_Data_hasLevelMVar(uint64_t); lean_object* lean_expr_dbg_to_string(lean_object*); static lean_object* l_Lean_Expr_withAppAux___at_Lean_Expr_traverseApp___spec__1___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Expr_updateConst_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_instInhabitedExpr; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__41; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__13; LEAN_EXPORT lean_object* l_Lean_Expr_mkDataForLet(uint64_t, lean_object*, uint32_t, uint8_t, uint8_t, uint8_t, uint8_t, uint8_t); static lean_object* l_Lean_mkSimpleThunk___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_mkAppRangeAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instReprData__1___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_appFn_x21_x27(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Expr_const___override___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Expr_updateProj_x21___closed__3; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__4; static lean_object* l_Lean_Literal_type___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_mkDataForLet___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__23; uint64_t l___private_Lean_Level_0__Lean_hashMVarId____x40_Lean_Level___hyg_478_(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_instantiate___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Expr_0__Lean_beqLiteral____x40_Lean_Expr___hyg_31_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isLetFun___boxed(lean_object*); static lean_object* l_Lean_mkSimpleThunk___closed__1; lean_object* l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isAppOfArity_x27(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_appFn_x21___closed__1; -static lean_object* l_Lean_Expr_updateApp_x21___closed__1; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_reverse___rarg(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__34; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__49; LEAN_EXPORT uint8_t l_Lean_Expr_isConst(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__20; LEAN_EXPORT uint8_t l_Lean_Expr_hasLevelMVar(lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__13; static lean_object* l_Lean_Expr_mkAppData___closed__5; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__16; LEAN_EXPORT lean_object* lean_expr_mk_let(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); static lean_object* l_Lean_Expr_fvarId_x21___closed__3; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__48; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__3; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_instantiateRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_hasFVar___boxed(lean_object*); LEAN_EXPORT uint8_t l_Lean_isLetFun(lean_object*); @@ -545,7 +547,6 @@ static lean_object* l_Lean_Expr_mkAppData___closed__3; LEAN_EXPORT lean_object* lean_expr_mk_app(lean_object*, lean_object*); static lean_object* l_Lean_Expr_constName_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__4(lean_object*, uint64_t, lean_object*, lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isForall(lean_object*); LEAN_EXPORT uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); LEAN_EXPORT lean_object* l_Lean_mkDecIsFalse(lean_object*, lean_object*); @@ -554,6 +555,7 @@ uint8_t lean_expr_quick_lt(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isLit(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFVar(lean_object*); static lean_object* l_Lean_Expr_getAutoParamTactic_x3f___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__34; LEAN_EXPORT uint8_t l_Lean_Expr_Data_binderInfo(uint64_t); LEAN_EXPORT lean_object* l_Lean_Expr_letValue_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_MData_empty; @@ -567,66 +569,50 @@ static lean_object* l_Lean_Expr_getAutoParamTactic_x3f___closed__2; LEAN_EXPORT uint8_t l_Lean_Expr_isLambda(lean_object*); static uint64_t l_Lean_Expr_mkAppData___closed__6; static lean_object* l_Lean_instInhabitedLiteral___closed__1; -static lean_object* l_Lean_Expr_updateSort_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_ctorName(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_replaceFVarId(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkApp9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_data___boxed(lean_object*); static lean_object* l_Lean_Expr_setPPExplicit___closed__1; -lean_object* lean_expr_update_proj(lean_object*, lean_object*); static lean_object* l_Lean_Expr_setPPExplicit___closed__2; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__6; LEAN_EXPORT uint8_t l_Lean_BinderInfo_isImplicit(uint8_t); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__50; LEAN_EXPORT lean_object* l_Lean_Expr_traverseApp(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getForallBody___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_setPPExplicit___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_looseBVarRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_bvarIdx_x21(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__45; -static lean_object* l_Lean_Expr_updateProj_x21___closed__2; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl(lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__40; LEAN_EXPORT lean_object* l_panic___at_Lean_Expr_mkData___spec__1___boxed__const__1; LEAN_EXPORT lean_object* l_Lean_Expr_setAppPPExplicit(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__27; static lean_object* l_Lean_Expr_ctorName___closed__9; LEAN_EXPORT lean_object* l_Lean_Expr_instantiateRevRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__50; static lean_object* l_Lean_mkNatLit___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378_(uint8_t, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Expr_bindingInfo_x21___spec__1(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__4; static lean_object* l_Lean_Expr_mkData___closed__6; LEAN_EXPORT uint8_t l_Lean_instInhabitedBinderInfo; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__29; -static lean_object* l_Lean_Expr_updateLambda_x21___closed__1; -LEAN_EXPORT lean_object* l_repr___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____spec__1(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__3; LEAN_EXPORT lean_object* l_Lean_instBEqFVarId; LEAN_EXPORT lean_object* l_Lean_Expr_fvar___override(lean_object*); uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); LEAN_EXPORT lean_object* l_Lean_instInhabitedFVarId; -static lean_object* l_Lean_Expr_updateProj_x21___closed__1; size_t lean_ptr_addr(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isType(lean_object*); -lean_object* lean_level_update_imax(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__17; static lean_object* l_Lean_mkNatLit___closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_isProj___boxed(lean_object*); -static lean_object* l_Lean_Expr_updateLambda_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__8; LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__7(lean_object*, uint64_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Expr_mkData___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getOptParamDefault_x3f___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateMData___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_repr___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Expr_traverseApp___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_appFn_x21___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_hasLevelMVarEx___boxed(lean_object*); static lean_object* l_Lean_instHashableBinderInfo___closed__1; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__44; LEAN_EXPORT lean_object* l_Lean_Expr_eta(lean_object*); LEAN_EXPORT lean_object* lean_expr_mk_mvar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_bindingName_x21(lean_object*); @@ -635,14 +621,13 @@ static lean_object* l_Lean_Expr_constLevels_x21___closed__1; uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l_Lean_mkAnd___closed__3; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_mkAppRev___spec__1(lean_object*, size_t, size_t, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__1; static lean_object* l_Lean_Expr_getOptParamDefault_x3f___closed__1; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__25; LEAN_EXPORT uint8_t l_Lean_Expr_isMVar(lean_object*); uint8_t lean_expr_equal(lean_object*, lean_object*); LEAN_EXPORT uint8_t lean_expr_has_fvar(lean_object*); -lean_object* lean_expr_update_sort(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____boxed(lean_object*, lean_object*); uint8_t lean_uint64_to_uint8(uint64_t); LEAN_EXPORT lean_object* l_Lean_Expr_hasAnyFVar(lean_object*, lean_object*); static lean_object* l_Lean_Expr_setPPExplicit___closed__3; @@ -651,11 +636,9 @@ LEAN_EXPORT lean_object* l_Lean_mkForall___boxed(lean_object*, lean_object*, lea uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkNot(lean_object*); static lean_object* l_Lean_Expr_constLevels_x21___closed__2; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_beta(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkApp(lean_object*, lean_object*); lean_object* l_String_quote(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_getAppNumArgsAux___boxed(lean_object*, lean_object*); LEAN_EXPORT uint64_t l_Lean_Literal_hash(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkLambdaEx___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_hasMVar(lean_object*); @@ -669,35 +652,33 @@ LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__5(lean_object*, uint64 LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Expr_instantiateLevelParamsArray___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_BinderInfo_isExplicit(uint8_t); LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Expr_const___override___spec__3(uint8_t, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__2; -static lean_object* l_Lean_Expr_updateMData_x21___closed__3; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__24; LEAN_EXPORT lean_object* l_Lean_mkApp5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_Data_looseBVarRange___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkAppRev(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_BinderInfo_noConfusion(lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__7; -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__47; static lean_object* l_Lean_Expr_bvarIdx_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_BinderInfo_isStrictImplicit___boxed(lean_object*); static lean_object* l_Lean_mkNatLit___closed__10; static lean_object* l_Lean_mkAnd___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__19; lean_object* l___private_Lean_Data_KVMap_0__Lean_reprKVMap____x40_Lean_Data_KVMap___hyg_855_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withApp___rarg(lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__11; LEAN_EXPORT lean_object* l_Lean_Expr_isAppOfArity___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_appArg_x21___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_getParamSubst(lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_shift_left(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Expr_binderInfo___boxed(lean_object*); static lean_object* l_Lean_instInhabitedExpr___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__1; LEAN_EXPORT lean_object* l_Lean_Literal_lt___boxed(lean_object*, lean_object*); lean_object* l_Lean_KVMap_insertCore(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__32; static lean_object* l_Lean_Expr_appArg_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_patternWithRef_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkApp7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___rarg___lambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateLambda_x21___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* lean_expr_mk_proj(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_projIdx_x21___closed__1; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__22; @@ -705,10 +686,12 @@ static lean_object* l_Lean_Expr_appFn_x21___closed__2; uint64_t lean_uint64_lor(uint64_t, uint64_t); static lean_object* l_Lean_mkNatLit___closed__5; LEAN_EXPORT lean_object* l_Lean_Expr_Data_hasExprMVar___boxed(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__2; LEAN_EXPORT lean_object* l_Lean_instReprBinderInfo; LEAN_EXPORT lean_object* l_Lean_Expr_etaExpanded_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_liftLooseBVars___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_bvarIdx_x21___closed__2; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__10; LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParamsCore_visit(lean_object*, lean_object*); static lean_object* l_Lean_Expr_appArg_x21___closed__1; uint8_t lean_uint16_dec_lt(uint16_t, uint16_t); @@ -735,7 +718,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Expr_setAppPPExplicit_ LEAN_EXPORT lean_object* l_Lean_BinderInfo_isAuxDecl___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_mkAppRevRangeAux(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Expr_instantiateLevelParamsArray___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__19; LEAN_EXPORT uint8_t l_Lean_Expr_isFVar(lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprLiteral____x40_Lean_Expr___hyg_109____closed__4; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -743,26 +725,23 @@ static lean_object* l_Lean_Expr_setPPUniverses___closed__1; LEAN_EXPORT lean_object* l_Lean_mkForall(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_instantiate1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getRevArgD___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instReprData__1___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_instantiateRev___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_isSort___boxed(lean_object*); static lean_object* l_Lean_Expr_isOutParam___closed__1; uint8_t lean_uint16_to_uint8(uint16_t); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__39; -static lean_object* l_Lean_Expr_updateLet_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_constName_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Expr_mkData___closed__4; lean_object* l_panic___at_Lean_TSyntax_getNat___spec__1(lean_object*); LEAN_EXPORT lean_object* lean_expr_mk_sort(lean_object*); LEAN_EXPORT lean_object* l_Lean_Literal_hash___boxed(lean_object*); -lean_object* lean_level_update_succ(lean_object*, lean_object*); lean_object* l_Lean_KVMap_findCore(lean_object*, lean_object*); static lean_object* l_Lean_instReprData__1___lambda__2___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_isBVar___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_consumeMDataAndTypeAnnotations(lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__15; static lean_object* l_Lean_instHashableLiteral___closed__1; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__18; @@ -773,28 +752,33 @@ LEAN_EXPORT lean_object* lean_expr_mk_fvar(lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l_Lean_Expr_letType_x21___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Expr_setAppPPExplicitForExposingMVars___spec__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__35; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__2; LEAN_EXPORT lean_object* l_Lean_instFVarIdHashSetInhabited; static lean_object* l___private_Lean_Expr_0__Lean_patternRefAnnotationKey___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkLet(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__3; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__12; lean_object* l_Lean_Name_quickCmp___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__26; static lean_object* l_Lean_instForInFVarIdSetFVarId___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_letType_x21___boxed(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__36; -LEAN_EXPORT lean_object* l_Lean_Expr_updateProj___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_letType_x21___closed__2; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isStringLit(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshMVarId(lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__5; lean_object* lean_uint64_to_nat(uint64_t); LEAN_EXPORT uint64_t lean_expr_hash(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_Data_hasFVar___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_mkAppRangeAux(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__30; +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__2; LEAN_EXPORT uint8_t l_Lean_Expr_isProj(lean_object*); LEAN_EXPORT lean_object* l_Lean_instFVarIdHashSetEmptyCollection; static lean_object* l_Lean_instReprLiteral___closed__1; @@ -809,10 +793,12 @@ LEAN_EXPORT uint8_t l_Lean_Expr_isAtomic(lean_object*); lean_object* lean_expr_abstract(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getArg_x21(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_ctorName___closed__12; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__37; LEAN_EXPORT lean_object* l_Lean_mkApp2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instForInFVarIdSetFVarId___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_instBEqExpr; LEAN_EXPORT lean_object* l_Lean_instInhabitedExprStructEq; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__42; LEAN_EXPORT uint64_t l_List_foldl___at_Lean_Expr_const___override___spec__1(uint64_t, lean_object*); static lean_object* l_Lean_Expr_ctorName___closed__6; LEAN_EXPORT lean_object* l_Lean_mkAnd(lean_object*, lean_object*); @@ -825,6 +811,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_updateForallE_x21(lean_object*, lean_object LEAN_EXPORT lean_object* l_Lean_mkPatternWithRef(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_instBEqData__1(uint64_t, uint64_t); lean_object* lean_string_length(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_mkAppN___spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_projIdx_x21(lean_object*); @@ -845,11 +832,9 @@ static lean_object* l___private_Lean_Expr_0__Lean_reprLiteral____x40_Lean_Expr__ static lean_object* l_Lean_mkDecIsFalse___closed__3; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__20; LEAN_EXPORT lean_object* l_Lean_Expr_isHeadBetaTarget___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Expr_updateLet_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_setOption___at_Lean_Expr_setPPExplicit___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isAtomic___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_Data_nonDepLet___boxed(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__12; LEAN_EXPORT lean_object* l_Lean_instInhabitedFVarIdMap(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkNatLit(lean_object*); lean_object* l_Lean_Level_instantiateParams(lean_object*, lean_object*); @@ -858,12 +843,14 @@ LEAN_EXPORT lean_object* l_Lean_Expr_sortLevel_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getArgD(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_getAppFn(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isAppOfArity_x27___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__26; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__38; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__21; LEAN_EXPORT lean_object* l_Lean_Expr_etaExpandedStrict_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_updateLambdaE_x21(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_hasLooseBVar___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Expr_ctorName___closed__11; static lean_object* l_Lean_mkNot___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__23; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Expr_setAppPPExplicit___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_letValue_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_instReprData__1(uint64_t, lean_object*); @@ -878,11 +865,12 @@ LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Ex static lean_object* l___private_Lean_Expr_0__Lean_reprLiteral____x40_Lean_Expr___hyg_109____closed__5; static lean_object* l_Lean_mkLetFunAnnotation___closed__2; static lean_object* l_Lean_instBEqBinderInfo___closed__1; -lean_object* lean_expr_update_app(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_isCharLit___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_setOption___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint64_t l_Lean_BinderInfo_hash(uint8_t); +LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____spec__2(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__1; static lean_object* l_Lean_Expr_setPPUniverses___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1___boxed(lean_object*, lean_object*, lean_object*); uint8_t lean_uint32_dec_le(uint32_t, uint32_t); @@ -901,14 +889,12 @@ LEAN_EXPORT lean_object* lean_expr_mk_lambda(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l_Lean_Expr_consumeMData___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_bindingBody_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_equal___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_updateLet_x21(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Literal_lt(lean_object*, lean_object*); static lean_object* l_Lean_mkLetFunAnnotation___closed__1; -LEAN_EXPORT lean_object* l_Lean_Expr_updateForall___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_casesOn___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkConst(lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__1; LEAN_EXPORT lean_object* l_Lean_mkSimpleThunk(lean_object*); -static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__31; static lean_object* l_Lean_mkNot___closed__2; LEAN_EXPORT lean_object* l_Lean_BinderInfo_toCtorIdx___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isLambda___boxed(lean_object*); @@ -930,13 +916,13 @@ static lean_object* l_Lean_instFVarIdHashSetInhabited___closed__1; static lean_object* l___private_Lean_Expr_0__Lean_reprBinderInfo____x40_Lean_Expr___hyg_378____closed__10; static lean_object* l_Lean_Expr_isOutParam___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_hasAnyFVar_visit(lean_object*, lean_object*); -lean_object* lean_expr_update_const(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Level_mvarId_x21___spec__1(lean_object*); static lean_object* l___private_Lean_Expr_0__Lean_patternRefAnnotationKey___closed__2; -static lean_object* l_Lean_Expr_updateSort_x21___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_isConst___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkInaccessible(lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__13; static lean_object* l_Lean_Expr_mdataExpr_x21___closed__1; +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__41; uint64_t lean_string_hash(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_isNatLit___boxed(lean_object*); lean_object* l_List_mapTRAux___rarg(lean_object*, lean_object*, lean_object*); @@ -952,6 +938,7 @@ static lean_object* l___private_Lean_Expr_0__Lean_reprLiteral____x40_Lean_Expr__ static lean_object* l_Lean_Expr_isCharLit___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_isCharLit___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_instReprData__1___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__31; uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT uint32_t l_Lean_Expr_Data_looseBVarRange(uint64_t); LEAN_EXPORT lean_object* l_Lean_Expr_setPPUniverses___boxed(lean_object*, lean_object*); @@ -2520,7 +2507,7 @@ static lean_object* _init_l_Lean_Expr_mkData___closed__7() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_mkData___closed__6; -x_3 = lean_unsigned_to_nat(163u); +x_3 = lean_unsigned_to_nat(200u); x_4 = lean_unsigned_to_nat(2u); x_5 = l_Lean_Expr_mkData___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2677,7 +2664,7 @@ static lean_object* _init_l_Lean_Expr_mkAppData___closed__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; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_mkAppData___closed__4; -x_3 = lean_unsigned_to_nat(184u); +x_3 = lean_unsigned_to_nat(221u); x_4 = lean_unsigned_to_nat(2u); x_5 = l_Lean_Expr_mkAppData___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -5531,7 +5518,7 @@ x_1 = l_Lean_instInhabitedExpr___closed__1; return x_1; } } -LEAN_EXPORT lean_object* l_repr___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_repr___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____spec__1(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -5540,7 +5527,7 @@ x_3 = l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935_(x_1, return x_3; } } -LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -5578,7 +5565,7 @@ lean_inc(x_2); x_11 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_2); -x_12 = l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____spec__2(x_4, x_2); +x_12 = l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____spec__2(x_4, x_2); x_13 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_13, 0, x_11); lean_ctor_set(x_13, 1, x_12); @@ -5587,7 +5574,7 @@ return x_13; } } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__1() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__1() { _start: { lean_object* x_1; @@ -5595,21 +5582,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.bvar", 14); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__1; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__1; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__3() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__2; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__2; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5617,7 +5604,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__4() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__4() { _start: { lean_object* x_1; @@ -5625,21 +5612,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.fvar", 14); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__5() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__4; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__4; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__6() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__5; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__5; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5647,7 +5634,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__7() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__7() { _start: { lean_object* x_1; @@ -5655,21 +5642,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.mvar", 14); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__8() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__7; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__7; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__9() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__8; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__8; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5677,7 +5664,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__10() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__10() { _start: { lean_object* x_1; @@ -5685,21 +5672,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.sort", 14); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__11() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__10; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__10; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__12() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__11; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__11; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5707,7 +5694,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__13() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__13() { _start: { lean_object* x_1; @@ -5715,21 +5702,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.const", 15); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__14() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__13; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__13; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__15() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__14; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__14; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5737,7 +5724,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__16() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__16() { _start: { lean_object* x_1; @@ -5745,17 +5732,17 @@ x_1 = lean_mk_string_from_bytes("[]", 2); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__17() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__17() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__16; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__16; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__18() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__18() { _start: { lean_object* x_1; @@ -5763,21 +5750,21 @@ x_1 = lean_mk_string_from_bytes(",", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__19() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__19() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__18; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__18; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__20() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__19; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__19; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5785,7 +5772,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__21() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__21() { _start: { lean_object* x_1; @@ -5793,35 +5780,35 @@ x_1 = lean_mk_string_from_bytes("[", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__22() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__21; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__21; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__23() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__23() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__22; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__22; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__24() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__24() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__21; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__21; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__25() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__25() { _start: { lean_object* x_1; @@ -5829,17 +5816,17 @@ x_1 = lean_mk_string_from_bytes("]", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__26() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__26() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__25; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__25; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__27() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__27() { _start: { lean_object* x_1; @@ -5847,21 +5834,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.app", 13); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__28() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__28() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__27; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__27; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__29() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__29() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__28; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__28; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5869,7 +5856,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__30() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__30() { _start: { lean_object* x_1; @@ -5877,21 +5864,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.lam", 13); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__31() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__31() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__30; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__30; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__32() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__32() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__31; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__31; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5899,7 +5886,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__33() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__33() { _start: { lean_object* x_1; @@ -5907,21 +5894,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.forallE", 17); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__34() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__34() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__33; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__33; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__35() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__35() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__34; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__34; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5929,7 +5916,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__36() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__36() { _start: { lean_object* x_1; @@ -5937,21 +5924,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.letE", 14); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__37() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__37() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__36; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__36; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__38() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__38() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__37; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__37; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -5959,7 +5946,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__39() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__39() { _start: { lean_object* x_1; @@ -5967,17 +5954,17 @@ x_1 = lean_mk_string_from_bytes("false", 5); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__40() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__40() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__39; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__39; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__41() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__41() { _start: { lean_object* x_1; lean_object* x_2; @@ -5987,7 +5974,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__42() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__42() { _start: { lean_object* x_1; @@ -5995,21 +5982,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.lit", 13); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__43() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__43() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__42; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__42; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__44() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__44() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__43; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__43; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -6017,7 +6004,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__45() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__45() { _start: { lean_object* x_1; @@ -6025,21 +6012,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.mdata", 15); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__46() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__46() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__45; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__45; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__47() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__47() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__46; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__46; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -6047,7 +6034,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__48() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__48() { _start: { lean_object* x_1; @@ -6055,21 +6042,21 @@ x_1 = lean_mk_string_from_bytes("Lean.Expr.proj", 14); return x_1; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__49() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__49() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__48; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__48; x_2 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__50() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__50() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__49; +x_1 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__49; x_2 = lean_box(1); x_3 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -6077,7 +6064,7 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(lean_object* x_1, lean_object* x_2) { _start: { switch (lean_obj_tag(x_1)) { @@ -6092,7 +6079,7 @@ x_5 = lean_nat_dec_le(x_4, x_2); x_6 = l_Nat_repr(x_3); x_7 = lean_alloc_ctor(2, 1, 0); lean_ctor_set(x_7, 0, x_6); -x_8 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__3; +x_8 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__3; x_9 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_9, 0, x_8); lean_ctor_set(x_9, 1, x_7); @@ -6134,7 +6121,7 @@ lean_dec(x_1); x_21 = lean_unsigned_to_nat(1024u); x_22 = lean_nat_dec_le(x_21, x_2); x_23 = l_Lean_Name_reprPrec(x_20, x_21); -x_24 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__6; +x_24 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__6; x_25 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_25, 0, x_24); lean_ctor_set(x_25, 1, x_23); @@ -6176,7 +6163,7 @@ lean_dec(x_1); x_37 = lean_unsigned_to_nat(1024u); x_38 = lean_nat_dec_le(x_37, x_2); x_39 = l_Lean_Name_reprPrec(x_36, x_37); -x_40 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__9; +x_40 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__9; x_41 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_41, 0, x_40); lean_ctor_set(x_41, 1, x_39); @@ -6218,7 +6205,7 @@ lean_dec(x_1); x_53 = lean_unsigned_to_nat(1024u); x_54 = lean_nat_dec_le(x_53, x_2); x_55 = l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935_(x_52, x_53); -x_56 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__12; +x_56 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__12; x_57 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_57, 0, x_56); lean_ctor_set(x_57, 1, x_55); @@ -6262,7 +6249,7 @@ lean_dec(x_1); x_70 = lean_unsigned_to_nat(1024u); x_71 = lean_nat_dec_le(x_70, x_2); x_72 = l_Lean_Name_reprPrec(x_68, x_70); -x_73 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__15; +x_73 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__15; x_74 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_74, 0, x_73); lean_ctor_set(x_74, 1, x_72); @@ -6275,7 +6262,7 @@ if (x_71 == 0) if (lean_obj_tag(x_69) == 0) { lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; -x_77 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__17; +x_77 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__17; x_78 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_78, 0, x_76); lean_ctor_set(x_78, 1, x_77); @@ -6293,17 +6280,17 @@ return x_83; else { lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_84 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__20; -x_85 = l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____spec__2(x_69, x_84); -x_86 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__24; +x_84 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__20; +x_85 = l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____spec__2(x_69, x_84); +x_86 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__24; x_87 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_87, 0, x_86); lean_ctor_set(x_87, 1, x_85); -x_88 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__26; +x_88 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__26; x_89 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_89, 0, x_87); lean_ctor_set(x_89, 1, x_88); -x_90 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__23; +x_90 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__23; x_91 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_91, 0, x_90); lean_ctor_set(x_91, 1, x_89); @@ -6330,7 +6317,7 @@ else if (lean_obj_tag(x_69) == 0) { lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; -x_99 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__17; +x_99 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__17; x_100 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_100, 0, x_76); lean_ctor_set(x_100, 1, x_99); @@ -6348,17 +6335,17 @@ return x_105; else { 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; uint8_t x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_106 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__20; -x_107 = l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____spec__2(x_69, x_106); -x_108 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__24; +x_106 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__20; +x_107 = l_Std_Format_joinSep___at___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____spec__2(x_69, x_106); +x_108 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__24; x_109 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_109, 0, x_108); lean_ctor_set(x_109, 1, x_107); -x_110 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__26; +x_110 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__26; x_111 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_111, 0, x_109); lean_ctor_set(x_111, 1, x_110); -x_112 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__23; +x_112 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__23; x_113 = lean_alloc_ctor(3, 2, 0); lean_ctor_set(x_113, 0, x_112); lean_ctor_set(x_113, 1, x_111); @@ -6391,8 +6378,8 @@ lean_inc(x_122); lean_dec(x_1); x_123 = lean_unsigned_to_nat(1024u); x_124 = lean_nat_dec_le(x_123, x_2); -x_125 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_121, x_123); -x_126 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__29; +x_125 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_121, x_123); +x_126 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__29; x_127 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_127, 0, x_126); lean_ctor_set(x_127, 1, x_125); @@ -6400,7 +6387,7 @@ x_128 = lean_box(1); x_129 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_129, 0, x_127); lean_ctor_set(x_129, 1, x_128); -x_130 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_122, x_123); +x_130 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_122, x_123); x_131 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_131, 0, x_129); lean_ctor_set(x_131, 1, x_130); @@ -6447,7 +6434,7 @@ lean_dec(x_1); x_146 = lean_unsigned_to_nat(1024u); x_147 = lean_nat_dec_le(x_146, x_2); x_148 = l_Lean_Name_reprPrec(x_142, x_146); -x_149 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__32; +x_149 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__32; x_150 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_150, 0, x_149); lean_ctor_set(x_150, 1, x_148); @@ -6455,14 +6442,14 @@ x_151 = lean_box(1); x_152 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_152, 0, x_150); lean_ctor_set(x_152, 1, x_151); -x_153 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_143, x_146); +x_153 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_143, x_146); x_154 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_154, 0, x_152); lean_ctor_set(x_154, 1, x_153); x_155 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_155, 0, x_154); lean_ctor_set(x_155, 1, x_151); -x_156 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_144, x_146); +x_156 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_144, x_146); x_157 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_157, 0, x_155); lean_ctor_set(x_157, 1, x_156); @@ -6516,7 +6503,7 @@ lean_dec(x_1); x_175 = lean_unsigned_to_nat(1024u); x_176 = lean_nat_dec_le(x_175, x_2); x_177 = l_Lean_Name_reprPrec(x_171, x_175); -x_178 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__35; +x_178 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__35; x_179 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_179, 0, x_178); lean_ctor_set(x_179, 1, x_177); @@ -6524,14 +6511,14 @@ x_180 = lean_box(1); x_181 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_181, 0, x_179); lean_ctor_set(x_181, 1, x_180); -x_182 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_172, x_175); +x_182 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_172, x_175); x_183 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_183, 0, x_181); lean_ctor_set(x_183, 1, x_182); x_184 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_184, 0, x_183); lean_ctor_set(x_184, 1, x_180); -x_185 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_173, x_175); +x_185 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_173, x_175); x_186 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_186, 0, x_184); lean_ctor_set(x_186, 1, x_185); @@ -6587,7 +6574,7 @@ lean_dec(x_1); x_205 = lean_unsigned_to_nat(1024u); x_206 = lean_nat_dec_le(x_205, x_2); x_207 = l_Lean_Name_reprPrec(x_200, x_205); -x_208 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__38; +x_208 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__38; x_209 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_209, 0, x_208); lean_ctor_set(x_209, 1, x_207); @@ -6595,21 +6582,21 @@ x_210 = lean_box(1); x_211 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_211, 0, x_209); lean_ctor_set(x_211, 1, x_210); -x_212 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_201, x_205); +x_212 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_201, x_205); x_213 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_213, 0, x_211); lean_ctor_set(x_213, 1, x_212); x_214 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_214, 0, x_213); lean_ctor_set(x_214, 1, x_210); -x_215 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_202, x_205); +x_215 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_202, x_205); x_216 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_216, 0, x_214); lean_ctor_set(x_216, 1, x_215); x_217 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_217, 0, x_216); lean_ctor_set(x_217, 1, x_210); -x_218 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_203, x_205); +x_218 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_203, x_205); x_219 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_219, 0, x_217); lean_ctor_set(x_219, 1, x_218); @@ -6621,7 +6608,7 @@ if (x_206 == 0) if (x_204 == 0) { lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; uint8_t x_225; lean_object* x_226; lean_object* x_227; -x_221 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__40; +x_221 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__40; x_222 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_222, 0, x_220); lean_ctor_set(x_222, 1, x_221); @@ -6639,7 +6626,7 @@ return x_227; else { lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; uint8_t x_232; lean_object* x_233; lean_object* x_234; -x_228 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__41; +x_228 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__41; x_229 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_229, 0, x_220); lean_ctor_set(x_229, 1, x_228); @@ -6660,7 +6647,7 @@ else if (x_204 == 0) { lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; uint8_t x_239; lean_object* x_240; lean_object* x_241; -x_235 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__40; +x_235 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__40; x_236 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_236, 0, x_220); lean_ctor_set(x_236, 1, x_235); @@ -6678,7 +6665,7 @@ return x_241; else { lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; uint8_t x_246; lean_object* x_247; lean_object* x_248; -x_242 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__41; +x_242 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__41; x_243 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_243, 0, x_220); lean_ctor_set(x_243, 1, x_242); @@ -6704,7 +6691,7 @@ lean_dec(x_1); x_250 = lean_unsigned_to_nat(1024u); x_251 = lean_nat_dec_le(x_250, x_2); x_252 = l___private_Lean_Expr_0__Lean_reprLiteral____x40_Lean_Expr___hyg_109_(x_249, x_250); -x_253 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__44; +x_253 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__44; x_254 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_254, 0, x_253); lean_ctor_set(x_254, 1, x_252); @@ -6748,7 +6735,7 @@ lean_dec(x_1); x_267 = lean_unsigned_to_nat(1024u); x_268 = lean_nat_dec_le(x_267, x_2); x_269 = l___private_Lean_Data_KVMap_0__Lean_reprKVMap____x40_Lean_Data_KVMap___hyg_855_(x_265, x_267); -x_270 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__47; +x_270 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__47; x_271 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_271, 0, x_270); lean_ctor_set(x_271, 1, x_269); @@ -6756,7 +6743,7 @@ x_272 = lean_box(1); x_273 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_273, 0, x_271); lean_ctor_set(x_273, 1, x_272); -x_274 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_266, x_267); +x_274 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_266, x_267); x_275 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_275, 0, x_273); lean_ctor_set(x_275, 1, x_274); @@ -6802,7 +6789,7 @@ lean_dec(x_1); x_289 = lean_unsigned_to_nat(1024u); x_290 = lean_nat_dec_le(x_289, x_2); x_291 = l_Lean_Name_reprPrec(x_286, x_289); -x_292 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__50; +x_292 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__50; x_293 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_293, 0, x_292); lean_ctor_set(x_293, 1, x_291); @@ -6819,7 +6806,7 @@ lean_ctor_set(x_298, 1, x_297); x_299 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_299, 0, x_298); lean_ctor_set(x_299, 1, x_294); -x_300 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_288, x_289); +x_300 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_288, x_289); x_301 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_301, 0, x_299); lean_ctor_set(x_301, 1, x_300); @@ -6855,11 +6842,11 @@ return x_311; } } } -LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_1, x_2); +x_3 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -6868,7 +6855,7 @@ static lean_object* _init_l_Lean_instReprExpr___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____boxed), 2, 0); return x_1; } } @@ -8271,27 +8258,6 @@ x_1 = l_Lean_Expr_instBEqExpr___closed__1; return x_1; } } -LEAN_EXPORT uint8_t l_Lean_Expr_ptrEq(lean_object* x_1, lean_object* x_2) { -_start: -{ -size_t x_3; size_t x_4; uint8_t x_5; -x_3 = lean_ptr_addr(x_1); -x_4 = lean_ptr_addr(x_2); -x_5 = lean_usize_dec_eq(x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Expr_ptrEq___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Expr_ptrEq(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} -} LEAN_EXPORT lean_object* l_Lean_Expr_equal___boxed(lean_object* x_1, lean_object* x_2) { _start: { @@ -8819,7 +8785,7 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 5) @@ -8839,11 +8805,11 @@ return x_2; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_getAppNumArgsAux___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Expr_getAppNumArgsAux(x_1, x_2); +x_3 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_2); lean_dec(x_1); return x_3; } @@ -8853,7 +8819,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_getAppNumArgs(lean_object* x_1) { { lean_object* x_2; lean_object* x_3; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Expr_getAppNumArgsAux(x_1, x_2); +x_3 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_2); return x_3; } } @@ -8908,7 +8874,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_getAppArgs(lean_object* x_1) { { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Expr_getAppNumArgsAux(x_1, x_2); +x_3 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_2); x_4 = l_Lean_Expr_getAppArgs___closed__1; lean_inc(x_3); x_5 = lean_mk_array(x_3, x_4); @@ -8947,7 +8913,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_getAppRevArgs(lean_object* x_1) { { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Expr_getAppNumArgsAux(x_1, x_2); +x_3 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_2); x_4 = lean_mk_empty_array_with_capacity(x_3); lean_dec(x_3); x_5 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_4); @@ -8996,7 +8962,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withApp___rarg(lean_object* x_1, lean_objec { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_3 = lean_unsigned_to_nat(0u); -x_4 = l_Lean_Expr_getAppNumArgsAux(x_1, x_3); +x_4 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_3); x_5 = l_Lean_Expr_getAppArgs___closed__1; lean_inc(x_4); x_6 = lean_mk_array(x_4, x_5); @@ -9095,7 +9061,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_traverseApp___rarg(lean_object* x_1, lean_o { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; x_4 = lean_unsigned_to_nat(0u); -x_5 = l_Lean_Expr_getAppNumArgsAux(x_3, x_4); +x_5 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_4); x_6 = l_Lean_Expr_getAppArgs___closed__1; lean_inc(x_5); x_7 = lean_mk_array(x_5, x_6); @@ -9160,7 +9126,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppRev___rarg(lean_object* x_1, lean_ob { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_3 = lean_unsigned_to_nat(0u); -x_4 = l_Lean_Expr_getAppNumArgsAux(x_1, x_3); +x_4 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_3); x_5 = lean_mk_empty_array_with_capacity(x_4); lean_dec(x_4); x_6 = l___private_Lean_Expr_0__Lean_Expr_withAppRevAux___rarg(x_2, x_1, x_5); @@ -9251,7 +9217,7 @@ static lean_object* _init_l_Lean_Expr_getRevArg_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_getRevArg_x21___closed__1; -x_3 = lean_unsigned_to_nat(624u); +x_3 = lean_unsigned_to_nat(904u); x_4 = lean_unsigned_to_nat(20u); x_5 = l_Lean_Expr_getRevArg_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9548,7 +9514,7 @@ static lean_object* _init_l_Lean_Expr_appFn_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_appFn_x21___closed__1; -x_3 = lean_unsigned_to_nat(656u); +x_3 = lean_unsigned_to_nat(938u); x_4 = lean_unsigned_to_nat(15u); x_5 = l_Lean_Expr_appFn_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9597,7 +9563,7 @@ static lean_object* _init_l_Lean_Expr_appArg_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_appArg_x21___closed__1; -x_3 = lean_unsigned_to_nat(660u); +x_3 = lean_unsigned_to_nat(942u); x_4 = lean_unsigned_to_nat(15u); x_5 = l_Lean_Expr_appFn_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9646,7 +9612,7 @@ static lean_object* _init_l_Lean_Expr_appFn_x21_x27___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_appFn_x21_x27___closed__1; -x_3 = lean_unsigned_to_nat(665u); +x_3 = lean_unsigned_to_nat(947u); x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_Expr_appFn_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9704,7 +9670,7 @@ static lean_object* _init_l_Lean_Expr_appArg_x21_x27___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_appArg_x21_x27___closed__1; -x_3 = lean_unsigned_to_nat(670u); +x_3 = lean_unsigned_to_nat(952u); x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_Expr_appFn_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9770,7 +9736,7 @@ static lean_object* _init_l_Lean_Expr_sortLevel_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_sortLevel_x21___closed__1; -x_3 = lean_unsigned_to_nat(674u); +x_3 = lean_unsigned_to_nat(956u); x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_Expr_sortLevel_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9836,7 +9802,7 @@ static lean_object* _init_l_Lean_Expr_litValue_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_litValue_x21___closed__1; -x_3 = lean_unsigned_to_nat(678u); +x_3 = lean_unsigned_to_nat(960u); x_4 = lean_unsigned_to_nat(13u); x_5 = l_Lean_Expr_litValue_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10063,7 +10029,7 @@ static lean_object* _init_l_Lean_Expr_constName_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_constName_x21___closed__1; -x_3 = lean_unsigned_to_nat(697u); +x_3 = lean_unsigned_to_nat(979u); x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_Expr_constName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10150,7 +10116,7 @@ static lean_object* _init_l_Lean_Expr_constLevels_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_constLevels_x21___closed__1; -x_3 = lean_unsigned_to_nat(705u); +x_3 = lean_unsigned_to_nat(987u); x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Expr_constName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10200,7 +10166,7 @@ static lean_object* _init_l_Lean_Expr_bvarIdx_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_bvarIdx_x21___closed__1; -x_3 = lean_unsigned_to_nat(709u); +x_3 = lean_unsigned_to_nat(991u); x_4 = lean_unsigned_to_nat(16u); x_5 = l_Lean_Expr_bvarIdx_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10266,7 +10232,7 @@ static lean_object* _init_l_Lean_Expr_fvarId_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_fvarId_x21___closed__1; -x_3 = lean_unsigned_to_nat(713u); +x_3 = lean_unsigned_to_nat(995u); x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_Expr_fvarId_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10316,7 +10282,7 @@ static lean_object* _init_l_Lean_Expr_mvarId_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_mvarId_x21___closed__1; -x_3 = lean_unsigned_to_nat(717u); +x_3 = lean_unsigned_to_nat(999u); x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_Expr_mvarId_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10373,7 +10339,7 @@ static lean_object* _init_l_Lean_Expr_bindingName_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_bindingName_x21___closed__1; -x_3 = lean_unsigned_to_nat(722u); +x_3 = lean_unsigned_to_nat(1004u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Lean_Expr_bindingName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10431,7 +10397,7 @@ static lean_object* _init_l_Lean_Expr_bindingDomain_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_bindingDomain_x21___closed__1; -x_3 = lean_unsigned_to_nat(727u); +x_3 = lean_unsigned_to_nat(1009u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Lean_Expr_bindingName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10489,7 +10455,7 @@ static lean_object* _init_l_Lean_Expr_bindingBody_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_bindingBody_x21___closed__1; -x_3 = lean_unsigned_to_nat(732u); +x_3 = lean_unsigned_to_nat(1014u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Lean_Expr_bindingName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10557,7 +10523,7 @@ static lean_object* _init_l_Lean_Expr_bindingInfo_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_bindingInfo_x21___closed__1; -x_3 = lean_unsigned_to_nat(737u); +x_3 = lean_unsigned_to_nat(1019u); x_4 = lean_unsigned_to_nat(24u); x_5 = l_Lean_Expr_bindingName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10617,7 +10583,7 @@ static lean_object* _init_l_Lean_Expr_letName_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_letName_x21___closed__1; -x_3 = lean_unsigned_to_nat(741u); +x_3 = lean_unsigned_to_nat(1023u); x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_Expr_letName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10666,7 +10632,7 @@ static lean_object* _init_l_Lean_Expr_letType_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_letType_x21___closed__1; -x_3 = lean_unsigned_to_nat(745u); +x_3 = lean_unsigned_to_nat(1027u); x_4 = lean_unsigned_to_nat(19u); x_5 = l_Lean_Expr_letName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10715,7 +10681,7 @@ static lean_object* _init_l_Lean_Expr_letValue_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_letValue_x21___closed__1; -x_3 = lean_unsigned_to_nat(749u); +x_3 = lean_unsigned_to_nat(1031u); x_4 = lean_unsigned_to_nat(21u); x_5 = l_Lean_Expr_letName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10764,7 +10730,7 @@ static lean_object* _init_l_Lean_Expr_letBody_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_letBody_x21___closed__1; -x_3 = lean_unsigned_to_nat(753u); +x_3 = lean_unsigned_to_nat(1035u); x_4 = lean_unsigned_to_nat(23u); x_5 = l_Lean_Expr_letName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10847,7 +10813,7 @@ static lean_object* _init_l_Lean_Expr_mdataExpr_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_mdataExpr_x21___closed__1; -x_3 = lean_unsigned_to_nat(761u); +x_3 = lean_unsigned_to_nat(1043u); x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_Expr_mdataExpr_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10904,7 +10870,7 @@ static lean_object* _init_l_Lean_Expr_projExpr_x21___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_projExpr_x21___closed__1; -x_3 = lean_unsigned_to_nat(765u); +x_3 = lean_unsigned_to_nat(1047u); x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Expr_projExpr_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10953,7 +10919,7 @@ static lean_object* _init_l_Lean_Expr_projIdx_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_projIdx_x21___closed__1; -x_3 = lean_unsigned_to_nat(769u); +x_3 = lean_unsigned_to_nat(1051u); x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Expr_projExpr_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -11956,7 +11922,7 @@ else { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Lean_Expr_getAppNumArgsAux(x_1, x_5); +x_6 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_5); x_7 = lean_mk_empty_array_with_capacity(x_6); lean_dec(x_6); x_8 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_7); @@ -12415,7 +12381,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_consumeMDataAndTypeAnnotations(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Expr_cleanupAnnotations(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; @@ -12787,122 +12753,152 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateApp___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = lean_expr_update_app(x_1, x_2, x_3); -return x_5; -} -} -static lean_object* _init_l_Lean_Expr_updateApp_x21___closed__1() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateApp!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateApp!Impl", 45); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateApp_x21___closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; -x_2 = l_Lean_Expr_updateApp_x21___closed__1; -x_3 = lean_unsigned_to_nat(1081u); -x_4 = lean_unsigned_to_nat(14u); +x_2 = l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(1401u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Expr_appFn_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateApp_x21(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 5) { -lean_object* x_4; -x_4 = lean_expr_update_app(x_1, x_2, x_3); -return x_4; +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; uint8_t x_8; +x_4 = lean_ctor_get(x_1, 0); +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ptr_addr(x_4); +x_7 = lean_ptr_addr(x_2); +x_8 = lean_usize_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Lean_Expr_app___override(x_2, x_3); +return x_9; +} +else +{ +size_t x_10; size_t x_11; uint8_t x_12; +x_10 = lean_ptr_addr(x_5); +x_11 = lean_ptr_addr(x_3); +x_12 = lean_usize_dec_eq(x_10, x_11); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = l_Lean_Expr_app___override(x_2, x_3); +return x_13; } else { -lean_object* x_5; lean_object* x_6; lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_5 = l_Lean_Expr_updateApp_x21___closed__2; -x_6 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_5); -return x_6; +lean_inc(x_1); +return x_1; +} +} +} +else +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_3); +lean_dec(x_2); +x_14 = l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__2; +x_15 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_14); +return x_15; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateConst___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = lean_expr_update_const(x_1, x_2); +x_4 = l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl(x_1, x_2, x_3); +lean_dec(x_1); return x_4; } } -static lean_object* _init_l_Lean_Expr_updateConst_x21___closed__1() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateConst!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateConst!Impl", 47); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateConst_x21___closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; -x_2 = l_Lean_Expr_updateConst_x21___closed__1; -x_3 = lean_unsigned_to_nat(1090u); -x_4 = lean_unsigned_to_nat(20u); +x_2 = l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(1412u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Expr_constName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateConst_x21(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 4) { -lean_object* x_3; -x_3 = lean_expr_update_const(x_1, x_2); -return x_3; +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +x_5 = l_ptrEqList___rarg(x_4, x_2); +lean_dec(x_4); +if (x_5 == 0) +{ +lean_object* x_6; +lean_dec(x_1); +x_6 = l_Lean_Expr_const___override(x_3, x_2); +return x_6; } else { -lean_object* x_4; lean_object* x_5; +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_4 = l_Lean_Expr_updateConst_x21___closed__2; -x_5 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_4); -return x_5; -} +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateSort___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = lean_expr_update_sort(x_1, x_2); -return x_4; +lean_object* x_7; lean_object* x_8; +lean_dec(x_2); +lean_dec(x_1); +x_7 = l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__2; +x_8 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_7); +return x_8; +} } } -static lean_object* _init_l_Lean_Expr_updateSort_x21___closed__1() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateSort!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateSort!Impl", 46); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateSort_x21___closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__2() { _start: { lean_object* x_1; @@ -12910,64 +12906,70 @@ x_1 = lean_mk_string_from_bytes("level expected", 14); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateSort_x21___closed__3() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; -x_2 = l_Lean_Expr_updateSort_x21___closed__1; -x_3 = lean_unsigned_to_nat(1099u); -x_4 = lean_unsigned_to_nat(16u); -x_5 = l_Lean_Expr_updateSort_x21___closed__2; +x_2 = l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(1423u); +x_4 = lean_unsigned_to_nat(14u); +x_5 = l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateSort_x21(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 3) { -lean_object* x_3; -x_3 = lean_expr_update_sort(x_1, x_2); -return x_3; +lean_object* x_3; size_t x_4; size_t x_5; uint8_t x_6; +x_3 = lean_ctor_get(x_1, 0); +x_4 = lean_ptr_addr(x_3); +x_5 = lean_ptr_addr(x_2); +x_6 = lean_usize_dec_eq(x_4, x_5); +if (x_6 == 0) +{ +lean_object* x_7; +x_7 = l_Lean_Expr_sort___override(x_2); +return x_7; } else { -lean_object* x_4; lean_object* x_5; lean_dec(x_2); -lean_dec(x_1); -x_4 = l_Lean_Expr_updateSort_x21___closed__3; -x_5 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_4); -return x_5; -} +lean_inc(x_1); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateProj___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = lean_expr_update_proj(x_1, x_2); -return x_4; +lean_object* x_8; lean_object* x_9; +lean_dec(x_2); +x_8 = l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__3; +x_9 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_8); +return x_9; +} } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateMData___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_4; -x_4 = lean_expr_update_mdata(x_1, x_2); -return x_4; +lean_object* x_3; +x_3 = l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl(x_1, x_2); +lean_dec(x_1); +return x_3; } } -static lean_object* _init_l_Lean_Expr_updateMData_x21___closed__1() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateMData!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateMData!Impl", 47); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateMData_x21___closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__2() { _start: { lean_object* x_1; @@ -12975,48 +12977,67 @@ x_1 = lean_mk_string_from_bytes("mdata expected", 14); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateMData_x21___closed__3() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; -x_2 = l_Lean_Expr_updateMData_x21___closed__1; -x_3 = lean_unsigned_to_nat(1116u); -x_4 = lean_unsigned_to_nat(16u); -x_5 = l_Lean_Expr_updateMData_x21___closed__2; +x_2 = l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(1434u); +x_4 = lean_unsigned_to_nat(17u); +x_5 = l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateMData_x21(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 10) { -lean_object* x_3; -x_3 = lean_expr_update_mdata(x_1, x_2); -return x_3; +lean_object* x_3; lean_object* x_4; size_t x_5; size_t x_6; uint8_t x_7; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +x_5 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_6 = lean_ptr_addr(x_2); +x_7 = lean_usize_dec_eq(x_5, x_6); +if (x_7 == 0) +{ +lean_object* x_8; +lean_dec(x_1); +x_8 = l_Lean_Expr_mdata___override(x_3, x_2); +return x_8; } else { -lean_object* x_4; lean_object* x_5; +lean_dec(x_3); +lean_dec(x_2); +return x_1; +} +} +else +{ +lean_object* x_9; lean_object* x_10; lean_dec(x_2); lean_dec(x_1); -x_4 = l_Lean_Expr_updateMData_x21___closed__3; -x_5 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_4); -return x_5; +x_9 = l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__3; +x_10 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_9); +return x_10; } } } -static lean_object* _init_l_Lean_Expr_updateProj_x21___closed__1() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateProj!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateProj!Impl", 46); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateProj_x21___closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__2() { _start: { lean_object* x_1; @@ -13024,58 +13045,70 @@ x_1 = lean_mk_string_from_bytes("proj expected", 13); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateProj_x21___closed__3() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; -x_2 = l_Lean_Expr_updateProj_x21___closed__1; -x_3 = lean_unsigned_to_nat(1121u); -x_4 = lean_unsigned_to_nat(15u); -x_5 = l_Lean_Expr_updateProj_x21___closed__2; +x_2 = l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(1445u); +x_4 = lean_unsigned_to_nat(18u); +x_5 = l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateProj_x21(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 11) { -lean_object* x_3; -x_3 = lean_expr_update_proj(x_1, x_2); -return x_3; +lean_object* x_3; lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; uint8_t x_8; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +x_6 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_7 = lean_ptr_addr(x_2); +x_8 = lean_usize_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +lean_dec(x_1); +x_9 = l_Lean_Expr_proj___override(x_3, x_4, x_2); +return x_9; } else { -lean_object* x_4; lean_object* x_5; +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_4 = l_Lean_Expr_updateProj_x21___closed__3; -x_5 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_4); -return x_5; -} +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateForall___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -uint8_t x_6; lean_object* x_7; -x_6 = lean_unbox(x_2); +lean_object* x_10; lean_object* x_11; lean_dec(x_2); -x_7 = lean_expr_update_forall(x_1, x_6, x_3, x_4); -return x_7; +lean_dec(x_1); +x_10 = l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__3; +x_11 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_10); +return x_11; +} } } -static lean_object* _init_l_Lean_Expr_updateForall_x21___closed__1() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateForall!", 23); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateForall!Impl", 48); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateForall_x21___closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__2() { _start: { lean_object* x_1; @@ -13083,47 +13116,98 @@ x_1 = lean_mk_string_from_bytes("forall expected", 15); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateForall_x21___closed__3() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; -x_2 = l_Lean_Expr_updateForall_x21___closed__1; -x_3 = lean_unsigned_to_nat(1130u); -x_4 = lean_unsigned_to_nat(18u); -x_5 = l_Lean_Expr_updateForall_x21___closed__2; +x_2 = l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(1460u); +x_4 = lean_unsigned_to_nat(23u); +x_5 = l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateForall_x21(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 7) { -lean_object* x_5; -x_5 = lean_expr_update_forall(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; size_t x_9; size_t x_10; uint8_t x_11; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_1, 2); +lean_inc(x_7); +x_8 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +x_9 = lean_ptr_addr(x_6); +lean_dec(x_6); +x_10 = lean_ptr_addr(x_3); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_7); +lean_dec(x_1); +x_12 = l_Lean_Expr_forallE___override(x_5, x_3, x_4, x_2); +return x_12; } else { -lean_object* x_6; lean_object* x_7; +size_t x_13; size_t x_14; uint8_t x_15; +x_13 = lean_ptr_addr(x_7); +lean_dec(x_7); +x_14 = lean_ptr_addr(x_4); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_1); +x_16 = l_Lean_Expr_forallE___override(x_5, x_3, x_4, x_2); +return x_16; +} +else +{ +uint8_t x_17; +x_17 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_8, x_2); +if (x_17 == 0) +{ +lean_object* x_18; +lean_dec(x_1); +x_18 = l_Lean_Expr_forallE___override(x_5, x_3, x_4, x_2); +return x_18; +} +else +{ +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_1; +} +} +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_6 = l_Lean_Expr_updateForall_x21___closed__3; -x_7 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_6); -return x_7; +x_19 = l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__3; +x_20 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_19); +return x_20; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateForall_x21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; x_5 = lean_unbox(x_2); lean_dec(x_2); -x_6 = l_Lean_Expr_updateForall_x21(x_1, x_5, x_3, x_4); +x_6 = l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl(x_1, x_5, x_3, x_4); return x_6; } } @@ -13141,9 +13225,9 @@ static lean_object* _init_l_Lean_Expr_updateForallE_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_updateForallE_x21___closed__1; -x_3 = lean_unsigned_to_nat(1135u); -x_4 = lean_unsigned_to_nat(23u); -x_5 = l_Lean_Expr_updateForall_x21___closed__2; +x_3 = lean_unsigned_to_nat(1471u); +x_4 = lean_unsigned_to_nat(24u); +x_5 = l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } @@ -13153,42 +13237,87 @@ LEAN_EXPORT lean_object* l_Lean_Expr_updateForallE_x21(lean_object* x_1, lean_ob { if (lean_obj_tag(x_1) == 7) { -uint8_t x_4; lean_object* x_5; -x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_5 = lean_expr_update_forall(x_1, x_4, x_2, x_3); -return x_5; +lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_8 = l_Lean_Expr_forallE___override(x_4, x_5, x_6, x_7); +x_9 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_10 = lean_ptr_addr(x_2); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_8); +lean_dec(x_6); +x_12 = l_Lean_Expr_forallE___override(x_4, x_2, x_3, x_7); +return x_12; } else { -lean_object* x_6; lean_object* x_7; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_6 = l_Lean_Expr_updateForallE_x21___closed__2; -x_7 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_6); -return x_7; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Expr_updateLambda___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +size_t x_13; size_t x_14; uint8_t x_15; +x_13 = lean_ptr_addr(x_6); +lean_dec(x_6); +x_14 = lean_ptr_addr(x_3); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) { -uint8_t x_6; lean_object* x_7; -x_6 = lean_unbox(x_2); -lean_dec(x_2); -x_7 = lean_expr_update_lambda(x_1, x_6, x_3, x_4); -return x_7; +lean_object* x_16; +lean_dec(x_8); +x_16 = l_Lean_Expr_forallE___override(x_4, x_2, x_3, x_7); +return x_16; +} +else +{ +uint8_t x_17; +x_17 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_7, x_7); +if (x_17 == 0) +{ +lean_object* x_18; +lean_dec(x_8); +x_18 = l_Lean_Expr_forallE___override(x_4, x_2, x_3, x_7); +return x_18; +} +else +{ +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_8; +} +} +} +} +else +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_19 = l_Lean_Expr_updateForallE_x21___closed__2; +x_20 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_19); +return x_20; } } -static lean_object* _init_l_Lean_Expr_updateLambda_x21___closed__1() { +} +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateLambda!", 23); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateLambda!Impl", 48); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateLambda_x21___closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__2() { _start: { lean_object* x_1; @@ -13196,47 +13325,98 @@ x_1 = lean_mk_string_from_bytes("lambda expected", 15); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateLambda_x21___closed__3() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; -x_2 = l_Lean_Expr_updateLambda_x21___closed__1; -x_3 = lean_unsigned_to_nat(1144u); -x_4 = lean_unsigned_to_nat(14u); -x_5 = l_Lean_Expr_updateLambda_x21___closed__2; +x_2 = l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(1480u); +x_4 = lean_unsigned_to_nat(19u); +x_5 = l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateLambda_x21(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 6) { -lean_object* x_5; -x_5 = lean_expr_update_lambda(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; size_t x_9; size_t x_10; uint8_t x_11; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_1, 2); +lean_inc(x_7); +x_8 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +x_9 = lean_ptr_addr(x_6); +lean_dec(x_6); +x_10 = lean_ptr_addr(x_3); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_7); +lean_dec(x_1); +x_12 = l_Lean_Expr_lam___override(x_5, x_3, x_4, x_2); +return x_12; } else { -lean_object* x_6; lean_object* x_7; +size_t x_13; size_t x_14; uint8_t x_15; +x_13 = lean_ptr_addr(x_7); +lean_dec(x_7); +x_14 = lean_ptr_addr(x_4); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_1); +x_16 = l_Lean_Expr_lam___override(x_5, x_3, x_4, x_2); +return x_16; +} +else +{ +uint8_t x_17; +x_17 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_8, x_2); +if (x_17 == 0) +{ +lean_object* x_18; +lean_dec(x_1); +x_18 = l_Lean_Expr_lam___override(x_5, x_3, x_4, x_2); +return x_18; +} +else +{ +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_1; +} +} +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_6 = l_Lean_Expr_updateLambda_x21___closed__3; -x_7 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_6); -return x_7; +x_19 = l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__3; +x_20 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_19); +return x_20; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateLambda_x21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { uint8_t x_5; lean_object* x_6; x_5 = lean_unbox(x_2); lean_dec(x_2); -x_6 = l_Lean_Expr_updateLambda_x21(x_1, x_5, x_3, x_4); +x_6 = l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl(x_1, x_5, x_3, x_4); return x_6; } } @@ -13254,9 +13434,9 @@ static lean_object* _init_l_Lean_Expr_updateLambdaE_x21___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; x_2 = l_Lean_Expr_updateLambdaE_x21___closed__1; -x_3 = lean_unsigned_to_nat(1149u); -x_4 = lean_unsigned_to_nat(19u); -x_5 = l_Lean_Expr_updateLambda_x21___closed__2; +x_3 = lean_unsigned_to_nat(1491u); +x_4 = lean_unsigned_to_nat(20u); +x_5 = l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } @@ -13266,71 +13446,177 @@ LEAN_EXPORT lean_object* l_Lean_Expr_updateLambdaE_x21(lean_object* x_1, lean_ob { if (lean_obj_tag(x_1) == 6) { -uint8_t x_4; lean_object* x_5; -x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_5 = lean_expr_update_lambda(x_1, x_4, x_2, x_3); -return x_5; +lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_8 = l_Lean_Expr_lam___override(x_4, x_5, x_6, x_7); +x_9 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_10 = lean_ptr_addr(x_2); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_8); +lean_dec(x_6); +x_12 = l_Lean_Expr_lam___override(x_4, x_2, x_3, x_7); +return x_12; } else { -lean_object* x_6; lean_object* x_7; +size_t x_13; size_t x_14; uint8_t x_15; +x_13 = lean_ptr_addr(x_6); +lean_dec(x_6); +x_14 = lean_ptr_addr(x_3); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_8); +x_16 = l_Lean_Expr_lam___override(x_4, x_2, x_3, x_7); +return x_16; +} +else +{ +uint8_t x_17; +x_17 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_7, x_7); +if (x_17 == 0) +{ +lean_object* x_18; +lean_dec(x_8); +x_18 = l_Lean_Expr_lam___override(x_4, x_2, x_3, x_7); +return x_18; +} +else +{ +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_6 = l_Lean_Expr_updateLambdaE_x21___closed__2; -x_7 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_6); -return x_7; +return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateLet___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +} +else { -lean_object* x_6; -x_6 = lean_expr_update_let(x_1, x_2, x_3, x_4); -return x_6; +lean_object* x_19; lean_object* x_20; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_19 = l_Lean_Expr_updateLambdaE_x21___closed__2; +x_20 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_19); +return x_20; } } -static lean_object* _init_l_Lean_Expr_updateLet_x21___closed__1() { +} +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateLet!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateLet!Impl", 45); return x_1; } } -static lean_object* _init_l_Lean_Expr_updateLet_x21___closed__2() { +static lean_object* _init_l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_mkData___closed__5; -x_2 = l_Lean_Expr_updateLet_x21___closed__1; -x_3 = lean_unsigned_to_nat(1158u); -x_4 = lean_unsigned_to_nat(15u); +x_2 = l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(1500u); +x_4 = lean_unsigned_to_nat(22u); x_5 = l_Lean_Expr_letName_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Expr_updateLet_x21(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_1) == 8) { -lean_object* x_5; -x_5 = lean_expr_update_let(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; size_t x_10; size_t x_11; uint8_t x_12; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_1, 2); +lean_inc(x_7); +x_8 = lean_ctor_get(x_1, 3); +lean_inc(x_8); +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); +x_10 = lean_ptr_addr(x_6); +lean_dec(x_6); +x_11 = lean_ptr_addr(x_2); +x_12 = lean_usize_dec_eq(x_10, x_11); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_1); +x_13 = l_Lean_Expr_letE___override(x_5, x_2, x_3, x_4, x_9); +return x_13; } else { -lean_object* x_6; lean_object* x_7; +size_t x_14; size_t x_15; uint8_t x_16; +x_14 = lean_ptr_addr(x_7); +lean_dec(x_7); +x_15 = lean_ptr_addr(x_3); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; +lean_dec(x_8); +lean_dec(x_1); +x_17 = l_Lean_Expr_letE___override(x_5, x_2, x_3, x_4, x_9); +return x_17; +} +else +{ +size_t x_18; size_t x_19; uint8_t x_20; +x_18 = lean_ptr_addr(x_8); +lean_dec(x_8); +x_19 = lean_ptr_addr(x_4); +x_20 = lean_usize_dec_eq(x_18, x_19); +if (x_20 == 0) +{ +lean_object* x_21; +lean_dec(x_1); +x_21 = l_Lean_Expr_letE___override(x_5, x_2, x_3, x_4, x_9); +return x_21; +} +else +{ +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_1; +} +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_6 = l_Lean_Expr_updateLet_x21___closed__2; -x_7 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_6); -return x_7; +x_22 = l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__2; +x_23 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_22); +return x_23; } } } @@ -13339,14 +13625,43 @@ LEAN_EXPORT lean_object* l_Lean_Expr_updateFn(lean_object* x_1, lean_object* x_2 { if (lean_obj_tag(x_1) == 5) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_3; lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; uint8_t x_8; x_3 = lean_ctor_get(x_1, 0); lean_inc(x_3); x_4 = lean_ctor_get(x_1, 1); lean_inc(x_4); +lean_inc(x_3); x_5 = l_Lean_Expr_updateFn(x_3, x_2); -x_6 = lean_expr_update_app(x_1, x_5, x_4); -return x_6; +x_6 = lean_ptr_addr(x_3); +lean_dec(x_3); +x_7 = lean_ptr_addr(x_5); +x_8 = lean_usize_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +lean_dec(x_1); +x_9 = l_Lean_Expr_app___override(x_5, x_4); +return x_9; +} +else +{ +size_t x_10; uint8_t x_11; +x_10 = lean_ptr_addr(x_4); +x_11 = lean_usize_dec_eq(x_10, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_1); +x_12 = l_Lean_Expr_app___override(x_5, x_4); +return x_12; +} +else +{ +lean_dec(x_5); +lean_dec(x_4); +return x_1; +} +} } else { @@ -13370,190 +13685,644 @@ LEAN_EXPORT lean_object* l_Lean_Expr_eta(lean_object* x_1) { { if (lean_obj_tag(x_1) == 6) { -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_2 = lean_ctor_get(x_1, 1); +lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; +x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); -x_3 = lean_ctor_get(x_1, 2); +x_3 = lean_ctor_get(x_1, 1); lean_inc(x_3); -x_4 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_5 = l_Lean_Expr_eta(x_3); -if (lean_obj_tag(x_5) == 5) -{ -lean_object* x_6; -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -if (lean_obj_tag(x_6) == 0) +x_4 = lean_ctor_get(x_1, 2); +lean_inc(x_4); +x_5 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_4); +x_6 = l_Lean_Expr_eta(x_4); +if (lean_obj_tag(x_6) == 5) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_7 = lean_ctor_get(x_5, 0); +lean_object* x_7; +x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; x_8 = lean_ctor_get(x_6, 0); lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_unsigned_to_nat(0u); -x_10 = lean_nat_dec_eq(x_8, x_9); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_eq(x_9, x_10); +lean_dec(x_9); +if (x_11 == 0) +{ +lean_object* x_12; size_t x_13; uint8_t x_14; lean_dec(x_8); -if (x_10 == 0) +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_12 = l_Lean_Expr_lam___override(x_2, x_3, x_4, x_5); +x_13 = lean_ptr_addr(x_3); +x_14 = lean_usize_dec_eq(x_13, x_13); +if (x_14 == 0) { -lean_object* x_11; -lean_dec(x_7); -x_11 = lean_expr_update_lambda(x_1, x_4, x_2, x_5); -return x_11; +lean_object* x_15; +lean_dec(x_12); +lean_dec(x_4); +x_15 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_15; } else { -uint8_t x_12; -x_12 = lean_expr_has_loose_bvar(x_7, x_9); -if (x_12 == 0) +size_t x_16; size_t x_17; uint8_t x_18; +x_16 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_17 = lean_ptr_addr(x_6); +x_18 = lean_usize_dec_eq(x_16, x_17); +if (x_18 == 0) { -lean_object* x_13; lean_object* x_14; -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_13 = lean_unsigned_to_nat(1u); -x_14 = lean_expr_lower_loose_bvars(x_7, x_13, x_13); -lean_dec(x_7); -return x_14; +lean_object* x_19; +lean_dec(x_12); +x_19 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_19; } else { -lean_object* x_15; +uint8_t x_20; +x_20 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_5, x_5); +if (x_20 == 0) +{ +lean_object* x_21; +lean_dec(x_12); +x_21 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_21; +} +else +{ +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_12; +} +} +} +} +else +{ +uint8_t x_22; +x_22 = lean_expr_has_loose_bvar(x_8, x_10); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_23 = lean_unsigned_to_nat(1u); +x_24 = lean_expr_lower_loose_bvars(x_8, x_23, x_23); +lean_dec(x_8); +return x_24; +} +else +{ +lean_object* x_25; size_t x_26; uint8_t x_27; +lean_dec(x_8); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_25 = l_Lean_Expr_lam___override(x_2, x_3, x_4, x_5); +x_26 = lean_ptr_addr(x_3); +x_27 = lean_usize_dec_eq(x_26, x_26); +if (x_27 == 0) +{ +lean_object* x_28; +lean_dec(x_25); +lean_dec(x_4); +x_28 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_28; +} +else +{ +size_t x_29; size_t x_30; uint8_t x_31; +x_29 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_30 = lean_ptr_addr(x_6); +x_31 = lean_usize_dec_eq(x_29, x_30); +if (x_31 == 0) +{ +lean_object* x_32; +lean_dec(x_25); +x_32 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_32; +} +else +{ +uint8_t x_33; +x_33 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_5, x_5); +if (x_33 == 0) +{ +lean_object* x_34; +lean_dec(x_25); +x_34 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_34; +} +else +{ +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_25; +} +} +} +} +} +} +else +{ +lean_object* x_35; size_t x_36; uint8_t x_37; lean_dec(x_7); -x_15 = lean_expr_update_lambda(x_1, x_4, x_2, x_5); -return x_15; +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_35 = l_Lean_Expr_lam___override(x_2, x_3, x_4, x_5); +x_36 = lean_ptr_addr(x_3); +x_37 = lean_usize_dec_eq(x_36, x_36); +if (x_37 == 0) +{ +lean_object* x_38; +lean_dec(x_35); +lean_dec(x_4); +x_38 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_38; +} +else +{ +size_t x_39; size_t x_40; uint8_t x_41; +x_39 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_40 = lean_ptr_addr(x_6); +x_41 = lean_usize_dec_eq(x_39, x_40); +if (x_41 == 0) +{ +lean_object* x_42; +lean_dec(x_35); +x_42 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_42; +} +else +{ +uint8_t x_43; +x_43 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_5, x_5); +if (x_43 == 0) +{ +lean_object* x_44; +lean_dec(x_35); +x_44 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_44; +} +else +{ +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_35; +} +} } } } else { -lean_object* x_16; +lean_object* x_45; size_t x_46; uint8_t x_47; +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_45 = l_Lean_Expr_lam___override(x_2, x_3, x_4, x_5); +x_46 = lean_ptr_addr(x_3); +x_47 = lean_usize_dec_eq(x_46, x_46); +if (x_47 == 0) +{ +lean_object* x_48; +lean_dec(x_45); +lean_dec(x_4); +x_48 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_48; +} +else +{ +size_t x_49; size_t x_50; uint8_t x_51; +x_49 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_50 = lean_ptr_addr(x_6); +x_51 = lean_usize_dec_eq(x_49, x_50); +if (x_51 == 0) +{ +lean_object* x_52; +lean_dec(x_45); +x_52 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_52; +} +else +{ +uint8_t x_53; +x_53 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_5, x_5); +if (x_53 == 0) +{ +lean_object* x_54; +lean_dec(x_45); +x_54 = l_Lean_Expr_lam___override(x_2, x_3, x_6, x_5); +return x_54; +} +else +{ lean_dec(x_6); -x_16 = lean_expr_update_lambda(x_1, x_4, x_2, x_5); +lean_dec(x_3); +lean_dec(x_2); +return x_45; +} +} +} +} +} +else +{ +return x_1; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParamsCore_visit(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; +x_3 = l_Lean_Expr_hasLevelParam(x_2); +if (x_3 == 0) +{ +lean_dec(x_1); +return x_2; +} +else +{ +switch (lean_obj_tag(x_2)) { +case 3: +{ +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; uint8_t x_8; +x_4 = lean_ctor_get(x_2, 0); +lean_inc(x_4); +lean_inc(x_4); +x_5 = l_Lean_Level_instantiateParams(x_1, x_4); +x_6 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_7 = lean_ptr_addr(x_5); +x_8 = lean_usize_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +lean_dec(x_2); +x_9 = l_Lean_Expr_sort___override(x_5); +return x_9; +} +else +{ +lean_dec(x_5); +return x_2; +} +} +case 4: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_10 = lean_ctor_get(x_2, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_Lean_Level_instantiateParams), 2, 1); +lean_closure_set(x_12, 0, x_1); +x_13 = lean_box(0); +lean_inc(x_11); +x_14 = l_List_mapTRAux___rarg(x_12, x_11, x_13); +x_15 = l_ptrEqList___rarg(x_11, x_14); +lean_dec(x_11); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_2); +x_16 = l_Lean_Expr_const___override(x_10, x_14); return x_16; } +else +{ +lean_dec(x_14); +lean_dec(x_10); +return x_2; +} +} +case 5: +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; uint8_t x_23; +x_17 = lean_ctor_get(x_2, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_2, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_1); +x_19 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_17); +lean_inc(x_18); +x_20 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_18); +x_21 = lean_ptr_addr(x_17); +lean_dec(x_17); +x_22 = lean_ptr_addr(x_19); +x_23 = lean_usize_dec_eq(x_21, x_22); +if (x_23 == 0) +{ +lean_object* x_24; +lean_dec(x_18); +lean_dec(x_2); +x_24 = l_Lean_Expr_app___override(x_19, x_20); +return x_24; +} +else +{ +size_t x_25; size_t x_26; uint8_t x_27; +x_25 = lean_ptr_addr(x_18); +lean_dec(x_18); +x_26 = lean_ptr_addr(x_20); +x_27 = lean_usize_dec_eq(x_25, x_26); +if (x_27 == 0) +{ +lean_object* x_28; +lean_dec(x_2); +x_28 = l_Lean_Expr_app___override(x_19, x_20); +return x_28; +} +else +{ +lean_dec(x_20); +lean_dec(x_19); +return x_2; +} +} +} +case 6: +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; size_t x_36; size_t x_37; uint8_t x_38; +x_29 = lean_ctor_get(x_2, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_2, 1); +lean_inc(x_30); +x_31 = lean_ctor_get(x_2, 2); +lean_inc(x_31); +x_32 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_30); +lean_inc(x_1); +x_33 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_30); +lean_inc(x_31); +x_34 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_31); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +x_35 = l_Lean_Expr_lam___override(x_29, x_30, x_31, x_32); +x_36 = lean_ptr_addr(x_30); +lean_dec(x_30); +x_37 = lean_ptr_addr(x_33); +x_38 = lean_usize_dec_eq(x_36, x_37); +if (x_38 == 0) +{ +lean_object* x_39; +lean_dec(x_35); +lean_dec(x_31); +x_39 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_39; +} +else +{ +size_t x_40; size_t x_41; uint8_t x_42; +x_40 = lean_ptr_addr(x_31); +lean_dec(x_31); +x_41 = lean_ptr_addr(x_34); +x_42 = lean_usize_dec_eq(x_40, x_41); +if (x_42 == 0) +{ +lean_object* x_43; +lean_dec(x_35); +x_43 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_43; +} +else +{ +uint8_t x_44; +x_44 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_32, x_32); +if (x_44 == 0) +{ +lean_object* x_45; +lean_dec(x_35); +x_45 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_45; +} +else +{ +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_29); +return x_35; +} +} +} +} +case 7: +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; size_t x_53; size_t x_54; uint8_t x_55; +x_46 = lean_ctor_get(x_2, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_2, 1); +lean_inc(x_47); +x_48 = lean_ctor_get(x_2, 2); +lean_inc(x_48); +x_49 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_47); +lean_inc(x_1); +x_50 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_47); +lean_inc(x_48); +x_51 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_48); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +x_52 = l_Lean_Expr_forallE___override(x_46, x_47, x_48, x_49); +x_53 = lean_ptr_addr(x_47); +lean_dec(x_47); +x_54 = lean_ptr_addr(x_50); +x_55 = lean_usize_dec_eq(x_53, x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_52); +lean_dec(x_48); +x_56 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_56; +} +else +{ +size_t x_57; size_t x_58; uint8_t x_59; +x_57 = lean_ptr_addr(x_48); +lean_dec(x_48); +x_58 = lean_ptr_addr(x_51); +x_59 = lean_usize_dec_eq(x_57, x_58); +if (x_59 == 0) +{ +lean_object* x_60; +lean_dec(x_52); +x_60 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_60; } else { -lean_object* x_17; -x_17 = lean_expr_update_lambda(x_1, x_4, x_2, x_5); -return x_17; -} +uint8_t x_61; +x_61 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_49, x_49); +if (x_61 == 0) +{ +lean_object* x_62; +lean_dec(x_52); +x_62 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_62; } else { -return x_1; +lean_dec(x_51); +lean_dec(x_50); +lean_dec(x_46); +return x_52; } } } -LEAN_EXPORT lean_object* l_Lean_Expr_instantiateLevelParamsCore_visit(lean_object* x_1, lean_object* x_2) { -_start: +} +case 8: { -uint8_t x_3; -x_3 = l_Lean_Expr_hasLevelParam(x_2); -if (x_3 == 0) +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; uint8_t x_73; +x_63 = lean_ctor_get(x_2, 0); +lean_inc(x_63); +x_64 = lean_ctor_get(x_2, 1); +lean_inc(x_64); +x_65 = lean_ctor_get(x_2, 2); +lean_inc(x_65); +x_66 = lean_ctor_get(x_2, 3); +lean_inc(x_66); +x_67 = lean_ctor_get_uint8(x_2, sizeof(void*)*4 + 8); +lean_inc(x_64); +lean_inc(x_1); +x_68 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_64); +lean_inc(x_65); +lean_inc(x_1); +x_69 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_65); +lean_inc(x_66); +x_70 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_66); +x_71 = lean_ptr_addr(x_64); +lean_dec(x_64); +x_72 = lean_ptr_addr(x_68); +x_73 = lean_usize_dec_eq(x_71, x_72); +if (x_73 == 0) { -lean_dec(x_1); -return x_2; +lean_object* x_74; +lean_dec(x_66); +lean_dec(x_65); +lean_dec(x_2); +x_74 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_74; } else { -switch (lean_obj_tag(x_2)) { -case 3: +size_t x_75; size_t x_76; uint8_t x_77; +x_75 = lean_ptr_addr(x_65); +lean_dec(x_65); +x_76 = lean_ptr_addr(x_69); +x_77 = lean_usize_dec_eq(x_75, x_76); +if (x_77 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = l_Lean_Level_instantiateParams(x_1, x_4); -x_6 = lean_expr_update_sort(x_2, x_5); -return x_6; +lean_object* x_78; +lean_dec(x_66); +lean_dec(x_2); +x_78 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_78; } -case 4: +else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_ctor_get(x_2, 1); -lean_inc(x_7); -x_8 = lean_alloc_closure((void*)(l_Lean_Level_instantiateParams), 2, 1); -lean_closure_set(x_8, 0, x_1); -x_9 = lean_box(0); -x_10 = l_List_mapTRAux___rarg(x_8, x_7, x_9); -x_11 = lean_expr_update_const(x_2, x_10); -return x_11; -} -case 5: +size_t x_79; size_t x_80; uint8_t x_81; +x_79 = lean_ptr_addr(x_66); +lean_dec(x_66); +x_80 = lean_ptr_addr(x_70); +x_81 = lean_usize_dec_eq(x_79, x_80); +if (x_81 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_12 = lean_ctor_get(x_2, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_2, 1); -lean_inc(x_13); -lean_inc(x_1); -x_14 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_12); -x_15 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_13); -x_16 = lean_expr_update_app(x_2, x_14, x_15); -return x_16; +lean_object* x_82; +lean_dec(x_2); +x_82 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_82; } -case 6: +else { -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_2, 1); -lean_inc(x_17); -x_18 = lean_ctor_get(x_2, 2); -lean_inc(x_18); -x_19 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -lean_inc(x_1); -x_20 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_17); -x_21 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_18); -x_22 = lean_expr_update_lambda(x_2, x_19, x_20, x_21); -return x_22; +lean_dec(x_70); +lean_dec(x_69); +lean_dec(x_68); +lean_dec(x_63); +return x_2; +} } -case 7: -{ -lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_23 = lean_ctor_get(x_2, 1); -lean_inc(x_23); -x_24 = lean_ctor_get(x_2, 2); -lean_inc(x_24); -x_25 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -lean_inc(x_1); -x_26 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_23); -x_27 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_24); -x_28 = lean_expr_update_forall(x_2, x_25, x_26, x_27); -return x_28; } -case 8: -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_29 = lean_ctor_get(x_2, 1); -lean_inc(x_29); -x_30 = lean_ctor_get(x_2, 2); -lean_inc(x_30); -x_31 = lean_ctor_get(x_2, 3); -lean_inc(x_31); -lean_inc(x_1); -x_32 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_29); -lean_inc(x_1); -x_33 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_30); -x_34 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_31); -x_35 = lean_expr_update_let(x_2, x_32, x_33, x_34); -return x_35; } case 10: { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_2, 1); -lean_inc(x_36); -x_37 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_36); -x_38 = lean_expr_update_mdata(x_2, x_37); -return x_38; +lean_object* x_83; lean_object* x_84; lean_object* x_85; size_t x_86; size_t x_87; uint8_t x_88; +x_83 = lean_ctor_get(x_2, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_2, 1); +lean_inc(x_84); +lean_inc(x_84); +x_85 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_84); +x_86 = lean_ptr_addr(x_84); +lean_dec(x_84); +x_87 = lean_ptr_addr(x_85); +x_88 = lean_usize_dec_eq(x_86, x_87); +if (x_88 == 0) +{ +lean_object* x_89; +lean_dec(x_2); +x_89 = l_Lean_Expr_mdata___override(x_83, x_85); +return x_89; +} +else +{ +lean_dec(x_85); +lean_dec(x_83); +return x_2; +} } case 11: { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_2, 2); -lean_inc(x_39); -x_40 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_39); -x_41 = lean_expr_update_proj(x_2, x_40); -return x_41; +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; size_t x_94; size_t x_95; uint8_t x_96; +x_90 = lean_ctor_get(x_2, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_2, 1); +lean_inc(x_91); +x_92 = lean_ctor_get(x_2, 2); +lean_inc(x_92); +lean_inc(x_92); +x_93 = l_Lean_Expr_instantiateLevelParamsCore_visit(x_1, x_92); +x_94 = lean_ptr_addr(x_92); +lean_dec(x_92); +x_95 = lean_ptr_addr(x_93); +x_96 = lean_usize_dec_eq(x_94, x_95); +if (x_96 == 0) +{ +lean_object* x_97; +lean_dec(x_2); +x_97 = l_Lean_Expr_proj___override(x_90, x_91, x_93); +return x_97; +} +else +{ +lean_dec(x_93); +lean_dec(x_91); +lean_dec(x_90); +return x_2; +} } default: { @@ -13634,90 +14403,149 @@ case 1: { lean_object* x_4; uint8_t x_5; x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); x_5 = l_Lean_Level_hasParam(x_3); if (x_5 == 0) { -lean_dec(x_4); +lean_inc(x_3); return x_3; } else { -lean_object* x_6; lean_object* x_7; +lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_6 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_4); -x_7 = lean_level_update_succ(x_3, x_6); -return x_7; +x_7 = lean_ptr_addr(x_4); +x_8 = lean_ptr_addr(x_6); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_Lean_Level_succ___override(x_6); +return x_10; +} +else +{ +lean_dec(x_6); +lean_inc(x_3); +return x_3; +} } } case 2: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_ctor_get(x_3, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_3, 1); -lean_inc(x_9); -x_10 = l_Lean_Level_hasParam(x_3); -if (x_10 == 0) +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = l_Lean_Level_hasParam(x_3); +if (x_13 == 0) { -lean_dec(x_9); -lean_dec(x_8); +lean_inc(x_3); return x_3; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_8); -x_12 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_9); -x_13 = lean_level_update_max(x_3, x_11, x_12); -return x_13; -} +lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; uint8_t x_18; +x_14 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_11); +x_15 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_12); +x_16 = lean_ptr_addr(x_11); +x_17 = lean_ptr_addr(x_14); +x_18 = lean_usize_dec_eq(x_16, x_17); +if (x_18 == 0) +{ +lean_object* x_19; +x_19 = l_Lean_mkLevelMax_x27(x_14, x_15); +return x_19; } -case 3: +else { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_ctor_get(x_3, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_3, 1); -lean_inc(x_15); -x_16 = l_Lean_Level_hasParam(x_3); -if (x_16 == 0) +size_t x_20; size_t x_21; uint8_t x_22; +x_20 = lean_ptr_addr(x_12); +x_21 = lean_ptr_addr(x_15); +x_22 = lean_usize_dec_eq(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = l_Lean_mkLevelMax_x27(x_14, x_15); +return x_23; +} +else { +lean_object* x_24; +x_24 = l_Lean_simpLevelMax_x27(x_14, x_15, x_3); lean_dec(x_15); lean_dec(x_14); +return x_24; +} +} +} +} +case 3: +{ +lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_25 = lean_ctor_get(x_3, 0); +x_26 = lean_ctor_get(x_3, 1); +x_27 = l_Lean_Level_hasParam(x_3); +if (x_27 == 0) +{ +lean_inc(x_3); return x_3; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_14); -x_18 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_15); -x_19 = lean_level_update_imax(x_3, x_17, x_18); -return x_19; +lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; uint8_t x_32; +x_28 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_25); +x_29 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_26); +x_30 = lean_ptr_addr(x_25); +x_31 = lean_ptr_addr(x_28); +x_32 = lean_usize_dec_eq(x_30, x_31); +if (x_32 == 0) +{ +lean_object* x_33; +x_33 = l_Lean_mkLevelIMax_x27(x_28, x_29); +return x_33; +} +else +{ +size_t x_34; size_t x_35; uint8_t x_36; +x_34 = lean_ptr_addr(x_26); +x_35 = lean_ptr_addr(x_29); +x_36 = lean_usize_dec_eq(x_34, x_35); +if (x_36 == 0) +{ +lean_object* x_37; +x_37 = l_Lean_mkLevelIMax_x27(x_28, x_29); +return x_37; +} +else +{ +lean_object* x_38; +x_38 = l_Lean_simpLevelIMax_x27(x_28, x_29, x_3); +return x_38; +} +} } } case 4: { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_3, 0); -lean_inc(x_20); -x_21 = l___private_Lean_Expr_0__Lean_Expr_getParamSubst(x_1, x_2, x_20); -lean_dec(x_20); -if (lean_obj_tag(x_21) == 0) +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_3, 0); +x_40 = l___private_Lean_Expr_0__Lean_Expr_getParamSubst(x_1, x_2, x_39); +if (lean_obj_tag(x_40) == 0) { +lean_inc(x_3); return x_3; } else { -lean_object* x_22; -lean_dec(x_3); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -return x_22; +lean_object* x_41; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +lean_dec(x_40); +return x_41; } } default: { +lean_inc(x_3); return x_3; } } @@ -13731,90 +14559,149 @@ case 1: { lean_object* x_4; uint8_t x_5; x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); x_5 = l_Lean_Level_hasParam(x_3); if (x_5 == 0) { -lean_dec(x_4); +lean_inc(x_3); return x_3; } else { -lean_object* x_6; lean_object* x_7; +lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_6 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_4); -x_7 = lean_level_update_succ(x_3, x_6); -return x_7; +x_7 = lean_ptr_addr(x_4); +x_8 = lean_ptr_addr(x_6); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_Lean_Level_succ___override(x_6); +return x_10; +} +else +{ +lean_dec(x_6); +lean_inc(x_3); +return x_3; +} } } case 2: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_ctor_get(x_3, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_3, 1); -lean_inc(x_9); -x_10 = l_Lean_Level_hasParam(x_3); -if (x_10 == 0) +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = l_Lean_Level_hasParam(x_3); +if (x_13 == 0) { -lean_dec(x_9); -lean_dec(x_8); +lean_inc(x_3); return x_3; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_8); -x_12 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_9); -x_13 = lean_level_update_max(x_3, x_11, x_12); -return x_13; -} +lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; uint8_t x_18; +x_14 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_11); +x_15 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_12); +x_16 = lean_ptr_addr(x_11); +x_17 = lean_ptr_addr(x_14); +x_18 = lean_usize_dec_eq(x_16, x_17); +if (x_18 == 0) +{ +lean_object* x_19; +x_19 = l_Lean_mkLevelMax_x27(x_14, x_15); +return x_19; } -case 3: +else { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_ctor_get(x_3, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_3, 1); -lean_inc(x_15); -x_16 = l_Lean_Level_hasParam(x_3); -if (x_16 == 0) +size_t x_20; size_t x_21; uint8_t x_22; +x_20 = lean_ptr_addr(x_12); +x_21 = lean_ptr_addr(x_15); +x_22 = lean_usize_dec_eq(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = l_Lean_mkLevelMax_x27(x_14, x_15); +return x_23; +} +else { +lean_object* x_24; +x_24 = l_Lean_simpLevelMax_x27(x_14, x_15, x_3); lean_dec(x_15); lean_dec(x_14); +return x_24; +} +} +} +} +case 3: +{ +lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_25 = lean_ctor_get(x_3, 0); +x_26 = lean_ctor_get(x_3, 1); +x_27 = l_Lean_Level_hasParam(x_3); +if (x_27 == 0) +{ +lean_inc(x_3); return x_3; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_14); -x_18 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_15); -x_19 = lean_level_update_imax(x_3, x_17, x_18); -return x_19; +lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; uint8_t x_32; +x_28 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_25); +x_29 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_26); +x_30 = lean_ptr_addr(x_25); +x_31 = lean_ptr_addr(x_28); +x_32 = lean_usize_dec_eq(x_30, x_31); +if (x_32 == 0) +{ +lean_object* x_33; +x_33 = l_Lean_mkLevelIMax_x27(x_28, x_29); +return x_33; +} +else +{ +size_t x_34; size_t x_35; uint8_t x_36; +x_34 = lean_ptr_addr(x_26); +x_35 = lean_ptr_addr(x_29); +x_36 = lean_usize_dec_eq(x_34, x_35); +if (x_36 == 0) +{ +lean_object* x_37; +x_37 = l_Lean_mkLevelIMax_x27(x_28, x_29); +return x_37; +} +else +{ +lean_object* x_38; +x_38 = l_Lean_simpLevelIMax_x27(x_28, x_29, x_3); +return x_38; +} +} } } case 4: { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_3, 0); -lean_inc(x_20); -x_21 = l___private_Lean_Expr_0__Lean_Expr_getParamSubst(x_1, x_2, x_20); -lean_dec(x_20); -if (lean_obj_tag(x_21) == 0) +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_3, 0); +x_40 = l___private_Lean_Expr_0__Lean_Expr_getParamSubst(x_1, x_2, x_39); +if (lean_obj_tag(x_40) == 0) { +lean_inc(x_3); return x_3; } else { -lean_object* x_22; -lean_dec(x_3); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -return x_22; +lean_object* x_41; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +lean_dec(x_40); +return x_41; } } default: { +lean_inc(x_3); return x_3; } } @@ -13839,6 +14726,7 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_3, 0); x_8 = lean_ctor_get(x_3, 1); x_9 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_7); +lean_dec(x_7); lean_ctor_set(x_3, 1, x_4); lean_ctor_set(x_3, 0, x_9); { @@ -13858,6 +14746,7 @@ lean_inc(x_12); lean_inc(x_11); lean_dec(x_3); x_13 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_11); +lean_dec(x_11); x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_13); lean_ctor_set(x_14, 1, x_4); @@ -13882,93 +14771,357 @@ else switch (lean_obj_tag(x_3)) { case 3: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_5 = lean_ctor_get(x_3, 0); lean_inc(x_5); x_6 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_5); -x_7 = lean_expr_update_sort(x_3, x_6); -return x_7; +x_7 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_8 = lean_ptr_addr(x_6); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_3); +x_10 = l_Lean_Expr_sort___override(x_6); +return x_10; } -case 4: +else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_3, 1); -lean_inc(x_8); -x_9 = lean_box(0); -x_10 = l_List_mapTRAux___at_Lean_Expr_instantiateLevelParams___spec__4(x_1, x_2, x_8, x_9); -x_11 = lean_expr_update_const(x_3, x_10); -return x_11; +lean_dec(x_6); +return x_3; } -case 5: +} +case 4: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_12 = lean_ctor_get(x_3, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_11 = lean_ctor_get(x_3, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_3, 1); lean_inc(x_12); -x_13 = lean_ctor_get(x_3, 1); -lean_inc(x_13); -x_14 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_12); -x_15 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_13); -x_16 = lean_expr_update_app(x_3, x_14, x_15); +x_13 = lean_box(0); +lean_inc(x_12); +x_14 = l_List_mapTRAux___at_Lean_Expr_instantiateLevelParams___spec__4(x_1, x_2, x_12, x_13); +x_15 = l_ptrEqList___rarg(x_12, x_14); +lean_dec(x_12); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_3); +x_16 = l_Lean_Expr_const___override(x_11, x_14); return x_16; } -case 6: +else +{ +lean_dec(x_14); +lean_dec(x_11); +return x_3; +} +} +case 5: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_3, 1); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; uint8_t x_23; +x_17 = lean_ctor_get(x_3, 0); lean_inc(x_17); -x_18 = lean_ctor_get(x_3, 2); +x_18 = lean_ctor_get(x_3, 1); lean_inc(x_18); -x_19 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); -x_20 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_17); -x_21 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_18); -x_22 = lean_expr_update_lambda(x_3, x_19, x_20, x_21); -return x_22; +lean_inc(x_17); +x_19 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_17); +lean_inc(x_18); +x_20 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_18); +x_21 = lean_ptr_addr(x_17); +lean_dec(x_17); +x_22 = lean_ptr_addr(x_19); +x_23 = lean_usize_dec_eq(x_21, x_22); +if (x_23 == 0) +{ +lean_object* x_24; +lean_dec(x_18); +lean_dec(x_3); +x_24 = l_Lean_Expr_app___override(x_19, x_20); +return x_24; } -case 7: +else { -lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_23 = lean_ctor_get(x_3, 1); -lean_inc(x_23); -x_24 = lean_ctor_get(x_3, 2); -lean_inc(x_24); -x_25 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); -x_26 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_23); -x_27 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_24); -x_28 = lean_expr_update_forall(x_3, x_25, x_26, x_27); +size_t x_25; size_t x_26; uint8_t x_27; +x_25 = lean_ptr_addr(x_18); +lean_dec(x_18); +x_26 = lean_ptr_addr(x_20); +x_27 = lean_usize_dec_eq(x_25, x_26); +if (x_27 == 0) +{ +lean_object* x_28; +lean_dec(x_3); +x_28 = l_Lean_Expr_app___override(x_19, x_20); return x_28; } -case 8: +else +{ +lean_dec(x_20); +lean_dec(x_19); +return x_3; +} +} +} +case 6: { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_29 = lean_ctor_get(x_3, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; size_t x_36; size_t x_37; uint8_t x_38; +x_29 = lean_ctor_get(x_3, 0); lean_inc(x_29); -x_30 = lean_ctor_get(x_3, 2); +x_30 = lean_ctor_get(x_3, 1); lean_inc(x_30); -x_31 = lean_ctor_get(x_3, 3); +x_31 = lean_ctor_get(x_3, 2); lean_inc(x_31); -x_32 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_29); +x_32 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +lean_dec(x_3); +lean_inc(x_30); x_33 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_30); +lean_inc(x_31); x_34 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_31); -x_35 = lean_expr_update_let(x_3, x_32, x_33, x_34); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +x_35 = l_Lean_Expr_lam___override(x_29, x_30, x_31, x_32); +x_36 = lean_ptr_addr(x_30); +lean_dec(x_30); +x_37 = lean_ptr_addr(x_33); +x_38 = lean_usize_dec_eq(x_36, x_37); +if (x_38 == 0) +{ +lean_object* x_39; +lean_dec(x_35); +lean_dec(x_31); +x_39 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_39; +} +else +{ +size_t x_40; size_t x_41; uint8_t x_42; +x_40 = lean_ptr_addr(x_31); +lean_dec(x_31); +x_41 = lean_ptr_addr(x_34); +x_42 = lean_usize_dec_eq(x_40, x_41); +if (x_42 == 0) +{ +lean_object* x_43; +lean_dec(x_35); +x_43 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_43; +} +else +{ +uint8_t x_44; +x_44 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_32, x_32); +if (x_44 == 0) +{ +lean_object* x_45; +lean_dec(x_35); +x_45 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_45; +} +else +{ +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_29); return x_35; } +} +} +} +case 7: +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; size_t x_53; size_t x_54; uint8_t x_55; +x_46 = lean_ctor_get(x_3, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_3, 1); +lean_inc(x_47); +x_48 = lean_ctor_get(x_3, 2); +lean_inc(x_48); +x_49 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +lean_dec(x_3); +lean_inc(x_47); +x_50 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_47); +lean_inc(x_48); +x_51 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_48); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +x_52 = l_Lean_Expr_forallE___override(x_46, x_47, x_48, x_49); +x_53 = lean_ptr_addr(x_47); +lean_dec(x_47); +x_54 = lean_ptr_addr(x_50); +x_55 = lean_usize_dec_eq(x_53, x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_52); +lean_dec(x_48); +x_56 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_56; +} +else +{ +size_t x_57; size_t x_58; uint8_t x_59; +x_57 = lean_ptr_addr(x_48); +lean_dec(x_48); +x_58 = lean_ptr_addr(x_51); +x_59 = lean_usize_dec_eq(x_57, x_58); +if (x_59 == 0) +{ +lean_object* x_60; +lean_dec(x_52); +x_60 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_60; +} +else +{ +uint8_t x_61; +x_61 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_49, x_49); +if (x_61 == 0) +{ +lean_object* x_62; +lean_dec(x_52); +x_62 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_62; +} +else +{ +lean_dec(x_51); +lean_dec(x_50); +lean_dec(x_46); +return x_52; +} +} +} +} +case 8: +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; uint8_t x_73; +x_63 = lean_ctor_get(x_3, 0); +lean_inc(x_63); +x_64 = lean_ctor_get(x_3, 1); +lean_inc(x_64); +x_65 = lean_ctor_get(x_3, 2); +lean_inc(x_65); +x_66 = lean_ctor_get(x_3, 3); +lean_inc(x_66); +x_67 = lean_ctor_get_uint8(x_3, sizeof(void*)*4 + 8); +lean_inc(x_64); +x_68 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_64); +lean_inc(x_65); +x_69 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_65); +lean_inc(x_66); +x_70 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_66); +x_71 = lean_ptr_addr(x_64); +lean_dec(x_64); +x_72 = lean_ptr_addr(x_68); +x_73 = lean_usize_dec_eq(x_71, x_72); +if (x_73 == 0) +{ +lean_object* x_74; +lean_dec(x_66); +lean_dec(x_65); +lean_dec(x_3); +x_74 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_74; +} +else +{ +size_t x_75; size_t x_76; uint8_t x_77; +x_75 = lean_ptr_addr(x_65); +lean_dec(x_65); +x_76 = lean_ptr_addr(x_69); +x_77 = lean_usize_dec_eq(x_75, x_76); +if (x_77 == 0) +{ +lean_object* x_78; +lean_dec(x_66); +lean_dec(x_3); +x_78 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_78; +} +else +{ +size_t x_79; size_t x_80; uint8_t x_81; +x_79 = lean_ptr_addr(x_66); +lean_dec(x_66); +x_80 = lean_ptr_addr(x_70); +x_81 = lean_usize_dec_eq(x_79, x_80); +if (x_81 == 0) +{ +lean_object* x_82; +lean_dec(x_3); +x_82 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_82; +} +else +{ +lean_dec(x_70); +lean_dec(x_69); +lean_dec(x_68); +lean_dec(x_63); +return x_3; +} +} +} +} case 10: { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_3, 1); -lean_inc(x_36); -x_37 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_36); -x_38 = lean_expr_update_mdata(x_3, x_37); -return x_38; +lean_object* x_83; lean_object* x_84; lean_object* x_85; size_t x_86; size_t x_87; uint8_t x_88; +x_83 = lean_ctor_get(x_3, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_3, 1); +lean_inc(x_84); +lean_inc(x_84); +x_85 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_84); +x_86 = lean_ptr_addr(x_84); +lean_dec(x_84); +x_87 = lean_ptr_addr(x_85); +x_88 = lean_usize_dec_eq(x_86, x_87); +if (x_88 == 0) +{ +lean_object* x_89; +lean_dec(x_3); +x_89 = l_Lean_Expr_mdata___override(x_83, x_85); +return x_89; +} +else +{ +lean_dec(x_85); +lean_dec(x_83); +return x_3; +} } case 11: { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_3, 2); -lean_inc(x_39); -x_40 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_39); -x_41 = lean_expr_update_proj(x_3, x_40); -return x_41; +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; size_t x_94; size_t x_95; uint8_t x_96; +x_90 = lean_ctor_get(x_3, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_3, 1); +lean_inc(x_91); +x_92 = lean_ctor_get(x_3, 2); +lean_inc(x_92); +lean_inc(x_92); +x_93 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParams___spec__1(x_1, x_2, x_92); +x_94 = lean_ptr_addr(x_92); +lean_dec(x_92); +x_95 = lean_ptr_addr(x_93); +x_96 = lean_usize_dec_eq(x_94, x_95); +if (x_96 == 0) +{ +lean_object* x_97; +lean_dec(x_3); +x_97 = l_Lean_Expr_proj___override(x_90, x_91, x_93); +return x_97; +} +else +{ +lean_dec(x_93); +lean_dec(x_91); +lean_dec(x_90); +return x_3; +} } default: { @@ -13993,6 +15146,7 @@ LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantia { lean_object* x_4; x_4 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__2(x_1, x_2, x_3); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_4; @@ -14003,6 +15157,7 @@ LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantia { lean_object* x_4; x_4 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParams___spec__3(x_1, x_2, x_3); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_4; @@ -14104,91 +15259,150 @@ case 1: { lean_object* x_4; uint8_t x_5; x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); x_5 = l_Lean_Level_hasParam(x_3); if (x_5 == 0) { -lean_dec(x_4); +lean_inc(x_3); return x_3; } else { -lean_object* x_6; lean_object* x_7; +lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_6 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_4); -x_7 = lean_level_update_succ(x_3, x_6); -return x_7; +x_7 = lean_ptr_addr(x_4); +x_8 = lean_ptr_addr(x_6); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_Lean_Level_succ___override(x_6); +return x_10; +} +else +{ +lean_dec(x_6); +lean_inc(x_3); +return x_3; +} } } case 2: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_ctor_get(x_3, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_3, 1); -lean_inc(x_9); -x_10 = l_Lean_Level_hasParam(x_3); -if (x_10 == 0) +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = l_Lean_Level_hasParam(x_3); +if (x_13 == 0) { -lean_dec(x_9); -lean_dec(x_8); +lean_inc(x_3); return x_3; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_8); -x_12 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_9); -x_13 = lean_level_update_max(x_3, x_11, x_12); -return x_13; -} +lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; uint8_t x_18; +x_14 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_11); +x_15 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_12); +x_16 = lean_ptr_addr(x_11); +x_17 = lean_ptr_addr(x_14); +x_18 = lean_usize_dec_eq(x_16, x_17); +if (x_18 == 0) +{ +lean_object* x_19; +x_19 = l_Lean_mkLevelMax_x27(x_14, x_15); +return x_19; } -case 3: +else { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_ctor_get(x_3, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_3, 1); -lean_inc(x_15); -x_16 = l_Lean_Level_hasParam(x_3); -if (x_16 == 0) +size_t x_20; size_t x_21; uint8_t x_22; +x_20 = lean_ptr_addr(x_12); +x_21 = lean_ptr_addr(x_15); +x_22 = lean_usize_dec_eq(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = l_Lean_mkLevelMax_x27(x_14, x_15); +return x_23; +} +else { +lean_object* x_24; +x_24 = l_Lean_simpLevelMax_x27(x_14, x_15, x_3); lean_dec(x_15); lean_dec(x_14); +return x_24; +} +} +} +} +case 3: +{ +lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_25 = lean_ctor_get(x_3, 0); +x_26 = lean_ctor_get(x_3, 1); +x_27 = l_Lean_Level_hasParam(x_3); +if (x_27 == 0) +{ +lean_inc(x_3); return x_3; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_14); -x_18 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_15); -x_19 = lean_level_update_imax(x_3, x_17, x_18); -return x_19; +lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; uint8_t x_32; +x_28 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_25); +x_29 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_26); +x_30 = lean_ptr_addr(x_25); +x_31 = lean_ptr_addr(x_28); +x_32 = lean_usize_dec_eq(x_30, x_31); +if (x_32 == 0) +{ +lean_object* x_33; +x_33 = l_Lean_mkLevelIMax_x27(x_28, x_29); +return x_33; +} +else +{ +size_t x_34; size_t x_35; uint8_t x_36; +x_34 = lean_ptr_addr(x_26); +x_35 = lean_ptr_addr(x_29); +x_36 = lean_usize_dec_eq(x_34, x_35); +if (x_36 == 0) +{ +lean_object* x_37; +x_37 = l_Lean_mkLevelIMax_x27(x_28, x_29); +return x_37; +} +else +{ +lean_object* x_38; +x_38 = l_Lean_simpLevelIMax_x27(x_28, x_29, x_3); +return x_38; +} +} } } case 4: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_3, 0); -lean_inc(x_20); -x_21 = lean_unsigned_to_nat(0u); -x_22 = l___private_Lean_Expr_0__Lean_Expr_getParamSubstArray(x_1, x_2, x_20, x_21); -lean_dec(x_20); -if (lean_obj_tag(x_22) == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_3, 0); +x_40 = lean_unsigned_to_nat(0u); +x_41 = l___private_Lean_Expr_0__Lean_Expr_getParamSubstArray(x_1, x_2, x_39, x_40); +if (lean_obj_tag(x_41) == 0) { +lean_inc(x_3); return x_3; } else { -lean_object* x_23; -lean_dec(x_3); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -return x_23; +lean_object* x_42; +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +lean_dec(x_41); +return x_42; } } default: { +lean_inc(x_3); return x_3; } } @@ -14202,91 +15416,150 @@ case 1: { lean_object* x_4; uint8_t x_5; x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); x_5 = l_Lean_Level_hasParam(x_3); if (x_5 == 0) { -lean_dec(x_4); +lean_inc(x_3); return x_3; } else { -lean_object* x_6; lean_object* x_7; +lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_6 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_4); -x_7 = lean_level_update_succ(x_3, x_6); -return x_7; +x_7 = lean_ptr_addr(x_4); +x_8 = lean_ptr_addr(x_6); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_Lean_Level_succ___override(x_6); +return x_10; +} +else +{ +lean_dec(x_6); +lean_inc(x_3); +return x_3; +} } } case 2: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_ctor_get(x_3, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_3, 1); -lean_inc(x_9); -x_10 = l_Lean_Level_hasParam(x_3); -if (x_10 == 0) +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = l_Lean_Level_hasParam(x_3); +if (x_13 == 0) { -lean_dec(x_9); -lean_dec(x_8); +lean_inc(x_3); return x_3; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_8); -x_12 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_9); -x_13 = lean_level_update_max(x_3, x_11, x_12); -return x_13; -} +lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; uint8_t x_18; +x_14 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_11); +x_15 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_12); +x_16 = lean_ptr_addr(x_11); +x_17 = lean_ptr_addr(x_14); +x_18 = lean_usize_dec_eq(x_16, x_17); +if (x_18 == 0) +{ +lean_object* x_19; +x_19 = l_Lean_mkLevelMax_x27(x_14, x_15); +return x_19; } -case 3: +else { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_ctor_get(x_3, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_3, 1); -lean_inc(x_15); -x_16 = l_Lean_Level_hasParam(x_3); -if (x_16 == 0) +size_t x_20; size_t x_21; uint8_t x_22; +x_20 = lean_ptr_addr(x_12); +x_21 = lean_ptr_addr(x_15); +x_22 = lean_usize_dec_eq(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = l_Lean_mkLevelMax_x27(x_14, x_15); +return x_23; +} +else { +lean_object* x_24; +x_24 = l_Lean_simpLevelMax_x27(x_14, x_15, x_3); lean_dec(x_15); lean_dec(x_14); +return x_24; +} +} +} +} +case 3: +{ +lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_25 = lean_ctor_get(x_3, 0); +x_26 = lean_ctor_get(x_3, 1); +x_27 = l_Lean_Level_hasParam(x_3); +if (x_27 == 0) +{ +lean_inc(x_3); return x_3; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_14); -x_18 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_15); -x_19 = lean_level_update_imax(x_3, x_17, x_18); -return x_19; +lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; uint8_t x_32; +x_28 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_25); +x_29 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_26); +x_30 = lean_ptr_addr(x_25); +x_31 = lean_ptr_addr(x_28); +x_32 = lean_usize_dec_eq(x_30, x_31); +if (x_32 == 0) +{ +lean_object* x_33; +x_33 = l_Lean_mkLevelIMax_x27(x_28, x_29); +return x_33; +} +else +{ +size_t x_34; size_t x_35; uint8_t x_36; +x_34 = lean_ptr_addr(x_26); +x_35 = lean_ptr_addr(x_29); +x_36 = lean_usize_dec_eq(x_34, x_35); +if (x_36 == 0) +{ +lean_object* x_37; +x_37 = l_Lean_mkLevelIMax_x27(x_28, x_29); +return x_37; +} +else +{ +lean_object* x_38; +x_38 = l_Lean_simpLevelIMax_x27(x_28, x_29, x_3); +return x_38; +} +} } } case 4: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_3, 0); -lean_inc(x_20); -x_21 = lean_unsigned_to_nat(0u); -x_22 = l___private_Lean_Expr_0__Lean_Expr_getParamSubstArray(x_1, x_2, x_20, x_21); -lean_dec(x_20); -if (lean_obj_tag(x_22) == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_3, 0); +x_40 = lean_unsigned_to_nat(0u); +x_41 = l___private_Lean_Expr_0__Lean_Expr_getParamSubstArray(x_1, x_2, x_39, x_40); +if (lean_obj_tag(x_41) == 0) { +lean_inc(x_3); return x_3; } else { -lean_object* x_23; -lean_dec(x_3); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -return x_23; +lean_object* x_42; +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +lean_dec(x_41); +return x_42; } } default: { +lean_inc(x_3); return x_3; } } @@ -14311,6 +15584,7 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_3, 0); x_8 = lean_ctor_get(x_3, 1); x_9 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_7); +lean_dec(x_7); lean_ctor_set(x_3, 1, x_4); lean_ctor_set(x_3, 0, x_9); { @@ -14330,6 +15604,7 @@ lean_inc(x_12); lean_inc(x_11); lean_dec(x_3); x_13 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_11); +lean_dec(x_11); x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_13); lean_ctor_set(x_14, 1, x_4); @@ -14354,93 +15629,357 @@ else switch (lean_obj_tag(x_3)) { case 3: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_5 = lean_ctor_get(x_3, 0); lean_inc(x_5); x_6 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_5); -x_7 = lean_expr_update_sort(x_3, x_6); -return x_7; +x_7 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_8 = lean_ptr_addr(x_6); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_3); +x_10 = l_Lean_Expr_sort___override(x_6); +return x_10; } -case 4: +else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_3, 1); -lean_inc(x_8); -x_9 = lean_box(0); -x_10 = l_List_mapTRAux___at_Lean_Expr_instantiateLevelParamsArray___spec__4(x_1, x_2, x_8, x_9); -x_11 = lean_expr_update_const(x_3, x_10); -return x_11; +lean_dec(x_6); +return x_3; } -case 5: +} +case 4: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_12 = lean_ctor_get(x_3, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_11 = lean_ctor_get(x_3, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_3, 1); lean_inc(x_12); -x_13 = lean_ctor_get(x_3, 1); -lean_inc(x_13); -x_14 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_12); -x_15 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_13); -x_16 = lean_expr_update_app(x_3, x_14, x_15); +x_13 = lean_box(0); +lean_inc(x_12); +x_14 = l_List_mapTRAux___at_Lean_Expr_instantiateLevelParamsArray___spec__4(x_1, x_2, x_12, x_13); +x_15 = l_ptrEqList___rarg(x_12, x_14); +lean_dec(x_12); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_3); +x_16 = l_Lean_Expr_const___override(x_11, x_14); return x_16; } -case 6: +else { -lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_3, 1); +lean_dec(x_14); +lean_dec(x_11); +return x_3; +} +} +case 5: +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; uint8_t x_23; +x_17 = lean_ctor_get(x_3, 0); lean_inc(x_17); -x_18 = lean_ctor_get(x_3, 2); +x_18 = lean_ctor_get(x_3, 1); lean_inc(x_18); -x_19 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); -x_20 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_17); -x_21 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_18); -x_22 = lean_expr_update_lambda(x_3, x_19, x_20, x_21); -return x_22; +lean_inc(x_17); +x_19 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_17); +lean_inc(x_18); +x_20 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_18); +x_21 = lean_ptr_addr(x_17); +lean_dec(x_17); +x_22 = lean_ptr_addr(x_19); +x_23 = lean_usize_dec_eq(x_21, x_22); +if (x_23 == 0) +{ +lean_object* x_24; +lean_dec(x_18); +lean_dec(x_3); +x_24 = l_Lean_Expr_app___override(x_19, x_20); +return x_24; } -case 7: +else { -lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_23 = lean_ctor_get(x_3, 1); -lean_inc(x_23); -x_24 = lean_ctor_get(x_3, 2); -lean_inc(x_24); -x_25 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); -x_26 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_23); -x_27 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_24); -x_28 = lean_expr_update_forall(x_3, x_25, x_26, x_27); +size_t x_25; size_t x_26; uint8_t x_27; +x_25 = lean_ptr_addr(x_18); +lean_dec(x_18); +x_26 = lean_ptr_addr(x_20); +x_27 = lean_usize_dec_eq(x_25, x_26); +if (x_27 == 0) +{ +lean_object* x_28; +lean_dec(x_3); +x_28 = l_Lean_Expr_app___override(x_19, x_20); return x_28; } -case 8: +else +{ +lean_dec(x_20); +lean_dec(x_19); +return x_3; +} +} +} +case 6: { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_29 = lean_ctor_get(x_3, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; size_t x_36; size_t x_37; uint8_t x_38; +x_29 = lean_ctor_get(x_3, 0); lean_inc(x_29); -x_30 = lean_ctor_get(x_3, 2); +x_30 = lean_ctor_get(x_3, 1); lean_inc(x_30); -x_31 = lean_ctor_get(x_3, 3); +x_31 = lean_ctor_get(x_3, 2); lean_inc(x_31); -x_32 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_29); +x_32 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +lean_dec(x_3); +lean_inc(x_30); x_33 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_30); +lean_inc(x_31); x_34 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_31); -x_35 = lean_expr_update_let(x_3, x_32, x_33, x_34); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +x_35 = l_Lean_Expr_lam___override(x_29, x_30, x_31, x_32); +x_36 = lean_ptr_addr(x_30); +lean_dec(x_30); +x_37 = lean_ptr_addr(x_33); +x_38 = lean_usize_dec_eq(x_36, x_37); +if (x_38 == 0) +{ +lean_object* x_39; +lean_dec(x_35); +lean_dec(x_31); +x_39 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_39; +} +else +{ +size_t x_40; size_t x_41; uint8_t x_42; +x_40 = lean_ptr_addr(x_31); +lean_dec(x_31); +x_41 = lean_ptr_addr(x_34); +x_42 = lean_usize_dec_eq(x_40, x_41); +if (x_42 == 0) +{ +lean_object* x_43; +lean_dec(x_35); +x_43 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_43; +} +else +{ +uint8_t x_44; +x_44 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_32, x_32); +if (x_44 == 0) +{ +lean_object* x_45; +lean_dec(x_35); +x_45 = l_Lean_Expr_lam___override(x_29, x_33, x_34, x_32); +return x_45; +} +else +{ +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_29); return x_35; } +} +} +} +case 7: +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; size_t x_53; size_t x_54; uint8_t x_55; +x_46 = lean_ctor_get(x_3, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_3, 1); +lean_inc(x_47); +x_48 = lean_ctor_get(x_3, 2); +lean_inc(x_48); +x_49 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +lean_dec(x_3); +lean_inc(x_47); +x_50 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_47); +lean_inc(x_48); +x_51 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_48); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +x_52 = l_Lean_Expr_forallE___override(x_46, x_47, x_48, x_49); +x_53 = lean_ptr_addr(x_47); +lean_dec(x_47); +x_54 = lean_ptr_addr(x_50); +x_55 = lean_usize_dec_eq(x_53, x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_52); +lean_dec(x_48); +x_56 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_56; +} +else +{ +size_t x_57; size_t x_58; uint8_t x_59; +x_57 = lean_ptr_addr(x_48); +lean_dec(x_48); +x_58 = lean_ptr_addr(x_51); +x_59 = lean_usize_dec_eq(x_57, x_58); +if (x_59 == 0) +{ +lean_object* x_60; +lean_dec(x_52); +x_60 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_60; +} +else +{ +uint8_t x_61; +x_61 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_49, x_49); +if (x_61 == 0) +{ +lean_object* x_62; +lean_dec(x_52); +x_62 = l_Lean_Expr_forallE___override(x_46, x_50, x_51, x_49); +return x_62; +} +else +{ +lean_dec(x_51); +lean_dec(x_50); +lean_dec(x_46); +return x_52; +} +} +} +} +case 8: +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; uint8_t x_73; +x_63 = lean_ctor_get(x_3, 0); +lean_inc(x_63); +x_64 = lean_ctor_get(x_3, 1); +lean_inc(x_64); +x_65 = lean_ctor_get(x_3, 2); +lean_inc(x_65); +x_66 = lean_ctor_get(x_3, 3); +lean_inc(x_66); +x_67 = lean_ctor_get_uint8(x_3, sizeof(void*)*4 + 8); +lean_inc(x_64); +x_68 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_64); +lean_inc(x_65); +x_69 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_65); +lean_inc(x_66); +x_70 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_66); +x_71 = lean_ptr_addr(x_64); +lean_dec(x_64); +x_72 = lean_ptr_addr(x_68); +x_73 = lean_usize_dec_eq(x_71, x_72); +if (x_73 == 0) +{ +lean_object* x_74; +lean_dec(x_66); +lean_dec(x_65); +lean_dec(x_3); +x_74 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_74; +} +else +{ +size_t x_75; size_t x_76; uint8_t x_77; +x_75 = lean_ptr_addr(x_65); +lean_dec(x_65); +x_76 = lean_ptr_addr(x_69); +x_77 = lean_usize_dec_eq(x_75, x_76); +if (x_77 == 0) +{ +lean_object* x_78; +lean_dec(x_66); +lean_dec(x_3); +x_78 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_78; +} +else +{ +size_t x_79; size_t x_80; uint8_t x_81; +x_79 = lean_ptr_addr(x_66); +lean_dec(x_66); +x_80 = lean_ptr_addr(x_70); +x_81 = lean_usize_dec_eq(x_79, x_80); +if (x_81 == 0) +{ +lean_object* x_82; +lean_dec(x_3); +x_82 = l_Lean_Expr_letE___override(x_63, x_68, x_69, x_70, x_67); +return x_82; +} +else +{ +lean_dec(x_70); +lean_dec(x_69); +lean_dec(x_68); +lean_dec(x_63); +return x_3; +} +} +} +} case 10: { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_3, 1); -lean_inc(x_36); -x_37 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_36); -x_38 = lean_expr_update_mdata(x_3, x_37); -return x_38; +lean_object* x_83; lean_object* x_84; lean_object* x_85; size_t x_86; size_t x_87; uint8_t x_88; +x_83 = lean_ctor_get(x_3, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_3, 1); +lean_inc(x_84); +lean_inc(x_84); +x_85 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_84); +x_86 = lean_ptr_addr(x_84); +lean_dec(x_84); +x_87 = lean_ptr_addr(x_85); +x_88 = lean_usize_dec_eq(x_86, x_87); +if (x_88 == 0) +{ +lean_object* x_89; +lean_dec(x_3); +x_89 = l_Lean_Expr_mdata___override(x_83, x_85); +return x_89; +} +else +{ +lean_dec(x_85); +lean_dec(x_83); +return x_3; +} } case 11: { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_3, 2); -lean_inc(x_39); -x_40 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_39); -x_41 = lean_expr_update_proj(x_3, x_40); -return x_41; +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; size_t x_94; size_t x_95; uint8_t x_96; +x_90 = lean_ctor_get(x_3, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_3, 1); +lean_inc(x_91); +x_92 = lean_ctor_get(x_3, 2); +lean_inc(x_92); +lean_inc(x_92); +x_93 = l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(x_1, x_2, x_92); +x_94 = lean_ptr_addr(x_92); +lean_dec(x_92); +x_95 = lean_ptr_addr(x_93); +x_96 = lean_usize_dec_eq(x_94, x_95); +if (x_96 == 0) +{ +lean_object* x_97; +lean_dec(x_3); +x_97 = l_Lean_Expr_proj___override(x_90, x_91, x_93); +return x_97; +} +else +{ +lean_dec(x_93); +lean_dec(x_91); +lean_dec(x_90); +return x_3; +} } default: { @@ -14465,6 +16004,7 @@ LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantia { lean_object* x_4; x_4 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__2(x_1, x_2, x_3); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_4; @@ -14475,6 +16015,7 @@ LEAN_EXPORT lean_object* l_Lean_Level_instantiateParams___at_Lean_Expr_instantia { lean_object* x_4; x_4 = l_Lean_Level_instantiateParams___at_Lean_Expr_instantiateLevelParamsArray___spec__3(x_1, x_2, x_3); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_4; @@ -14672,7 +16213,7 @@ x_2 = l_Lean_Expr_getAppFn(x_1); x_3 = 0; x_4 = l_Lean_Expr_setPPExplicit(x_2, x_3); x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Lean_Expr_getAppNumArgsAux(x_1, x_5); +x_6 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_5); x_7 = l_Lean_Expr_getAppArgs___closed__1; lean_inc(x_6); x_8 = lean_mk_array(x_6, x_7); @@ -14757,7 +16298,7 @@ x_2 = l_Lean_Expr_getAppFn(x_1); x_3 = 0; x_4 = l_Lean_Expr_setPPExplicit(x_2, x_3); x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Lean_Expr_getAppNumArgsAux(x_1, x_5); +x_6 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_5); x_7 = l_Lean_Expr_getAppArgs___closed__1; lean_inc(x_6); x_8 = lean_mk_array(x_6, x_7); @@ -15779,106 +17320,106 @@ l_Lean_instInhabitedExpr___closed__1 = _init_l_Lean_instInhabitedExpr___closed__ lean_mark_persistent(l_Lean_instInhabitedExpr___closed__1); l_Lean_instInhabitedExpr = _init_l_Lean_instInhabitedExpr(); lean_mark_persistent(l_Lean_instInhabitedExpr); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__1 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__1(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__1); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__2 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__2(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__2); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__3 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__3(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__3); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__4 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__4(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__4); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__5 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__5(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__5); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__6 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__6(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__6); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__7 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__7(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__7); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__8 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__8(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__8); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__9 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__9(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__9); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__10 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__10(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__10); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__11 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__11(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__11); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__12 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__12(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__12); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__13 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__13(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__13); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__14 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__14(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__14); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__15 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__15(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__15); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__16 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__16(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__16); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__17 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__17(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__17); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__18 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__18(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__18); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__19 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__19(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__19); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__20 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__20(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__20); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__21 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__21(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__21); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__22 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__22(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__22); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__23 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__23(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__23); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__24 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__24(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__24); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__25 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__25(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__25); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__26 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__26(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__26); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__27 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__27(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__27); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__28 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__28(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__28); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__29 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__29(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__29); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__30 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__30(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__30); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__31 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__31(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__31); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__32 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__32(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__32); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__33 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__33(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__33); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__34 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__34(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__34); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__35 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__35(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__35); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__36 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__36(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__36); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__37 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__37(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__37); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__38 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__38(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__38); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__39 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__39(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__39); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__40 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__40(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__40); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__41 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__41(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__41); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__42 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__42(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__42); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__43 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__43(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__43); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__44 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__44(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__44); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__45 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__45(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__45); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__46 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__46(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__46); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__47 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__47(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__47); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__48 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__48(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__48); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__49 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__49(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__49); -l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__50 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__50(); -lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803____closed__50); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__1 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__1); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__2 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__2); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__3 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__3(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__3); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__4 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__4(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__4); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__5 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__5(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__5); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__6 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__6(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__6); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__7 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__7(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__7); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__8 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__8(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__8); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__9 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__9(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__9); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__10 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__10(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__10); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__11 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__11(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__11); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__12 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__12(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__12); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__13 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__13(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__13); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__14 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__14(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__14); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__15 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__15(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__15); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__16 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__16(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__16); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__17 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__17(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__17); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__18 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__18(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__18); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__19 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__19(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__19); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__20 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__20(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__20); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__21 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__21(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__21); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__22 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__22(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__22); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__23 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__23(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__23); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__24 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__24(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__24); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__25 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__25(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__25); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__26 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__26(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__26); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__27 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__27(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__27); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__28 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__28(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__28); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__29 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__29(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__29); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__30 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__30(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__30); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__31 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__31(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__31); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__32 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__32(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__32); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__33 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__33(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__33); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__34 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__34(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__34); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__35 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__35(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__35); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__36 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__36(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__36); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__37 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__37(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__37); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__38 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__38(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__38); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__39 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__39(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__39); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__40 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__40(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__40); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__41 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__41(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__41); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__42 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__42(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__42); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__43 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__43(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__43); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__44 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__44(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__44); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__45 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__45(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__45); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__46 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__46(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__46); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__47 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__47(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__47); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__48 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__48(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__48); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__49 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__49(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__49); +l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__50 = _init_l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__50(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766____closed__50); l_Lean_instReprExpr___closed__1 = _init_l_Lean_instReprExpr___closed__1(); lean_mark_persistent(l_Lean_instReprExpr___closed__1); l_Lean_instReprExpr = _init_l_Lean_instReprExpr(); @@ -16127,56 +17668,56 @@ l_Lean_Expr_isOutParam___closed__1 = _init_l_Lean_Expr_isOutParam___closed__1(); lean_mark_persistent(l_Lean_Expr_isOutParam___closed__1); l_Lean_Expr_isOutParam___closed__2 = _init_l_Lean_Expr_isOutParam___closed__2(); lean_mark_persistent(l_Lean_Expr_isOutParam___closed__2); -l_Lean_Expr_updateApp_x21___closed__1 = _init_l_Lean_Expr_updateApp_x21___closed__1(); -lean_mark_persistent(l_Lean_Expr_updateApp_x21___closed__1); -l_Lean_Expr_updateApp_x21___closed__2 = _init_l_Lean_Expr_updateApp_x21___closed__2(); -lean_mark_persistent(l_Lean_Expr_updateApp_x21___closed__2); -l_Lean_Expr_updateConst_x21___closed__1 = _init_l_Lean_Expr_updateConst_x21___closed__1(); -lean_mark_persistent(l_Lean_Expr_updateConst_x21___closed__1); -l_Lean_Expr_updateConst_x21___closed__2 = _init_l_Lean_Expr_updateConst_x21___closed__2(); -lean_mark_persistent(l_Lean_Expr_updateConst_x21___closed__2); -l_Lean_Expr_updateSort_x21___closed__1 = _init_l_Lean_Expr_updateSort_x21___closed__1(); -lean_mark_persistent(l_Lean_Expr_updateSort_x21___closed__1); -l_Lean_Expr_updateSort_x21___closed__2 = _init_l_Lean_Expr_updateSort_x21___closed__2(); -lean_mark_persistent(l_Lean_Expr_updateSort_x21___closed__2); -l_Lean_Expr_updateSort_x21___closed__3 = _init_l_Lean_Expr_updateSort_x21___closed__3(); -lean_mark_persistent(l_Lean_Expr_updateSort_x21___closed__3); -l_Lean_Expr_updateMData_x21___closed__1 = _init_l_Lean_Expr_updateMData_x21___closed__1(); -lean_mark_persistent(l_Lean_Expr_updateMData_x21___closed__1); -l_Lean_Expr_updateMData_x21___closed__2 = _init_l_Lean_Expr_updateMData_x21___closed__2(); -lean_mark_persistent(l_Lean_Expr_updateMData_x21___closed__2); -l_Lean_Expr_updateMData_x21___closed__3 = _init_l_Lean_Expr_updateMData_x21___closed__3(); -lean_mark_persistent(l_Lean_Expr_updateMData_x21___closed__3); -l_Lean_Expr_updateProj_x21___closed__1 = _init_l_Lean_Expr_updateProj_x21___closed__1(); -lean_mark_persistent(l_Lean_Expr_updateProj_x21___closed__1); -l_Lean_Expr_updateProj_x21___closed__2 = _init_l_Lean_Expr_updateProj_x21___closed__2(); -lean_mark_persistent(l_Lean_Expr_updateProj_x21___closed__2); -l_Lean_Expr_updateProj_x21___closed__3 = _init_l_Lean_Expr_updateProj_x21___closed__3(); -lean_mark_persistent(l_Lean_Expr_updateProj_x21___closed__3); -l_Lean_Expr_updateForall_x21___closed__1 = _init_l_Lean_Expr_updateForall_x21___closed__1(); -lean_mark_persistent(l_Lean_Expr_updateForall_x21___closed__1); -l_Lean_Expr_updateForall_x21___closed__2 = _init_l_Lean_Expr_updateForall_x21___closed__2(); -lean_mark_persistent(l_Lean_Expr_updateForall_x21___closed__2); -l_Lean_Expr_updateForall_x21___closed__3 = _init_l_Lean_Expr_updateForall_x21___closed__3(); -lean_mark_persistent(l_Lean_Expr_updateForall_x21___closed__3); +l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__1 = _init_l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__1); +l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__2 = _init_l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___closed__2); +l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__1 = _init_l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__1); +l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__2 = _init_l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateConst_x21Impl___closed__2); +l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__1 = _init_l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__1); +l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__2 = _init_l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__2); +l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__3 = _init_l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__3(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateSort_x21Impl___closed__3); +l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__1 = _init_l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__1); +l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__2 = _init_l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__2); +l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__3 = _init_l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__3(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl___closed__3); +l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__1 = _init_l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__1); +l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__2 = _init_l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__2); +l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__3 = _init_l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__3(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl___closed__3); +l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__1 = _init_l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__1); +l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__2 = _init_l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__2); +l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__3 = _init_l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__3(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateForall_x21Impl___closed__3); l_Lean_Expr_updateForallE_x21___closed__1 = _init_l_Lean_Expr_updateForallE_x21___closed__1(); lean_mark_persistent(l_Lean_Expr_updateForallE_x21___closed__1); l_Lean_Expr_updateForallE_x21___closed__2 = _init_l_Lean_Expr_updateForallE_x21___closed__2(); lean_mark_persistent(l_Lean_Expr_updateForallE_x21___closed__2); -l_Lean_Expr_updateLambda_x21___closed__1 = _init_l_Lean_Expr_updateLambda_x21___closed__1(); -lean_mark_persistent(l_Lean_Expr_updateLambda_x21___closed__1); -l_Lean_Expr_updateLambda_x21___closed__2 = _init_l_Lean_Expr_updateLambda_x21___closed__2(); -lean_mark_persistent(l_Lean_Expr_updateLambda_x21___closed__2); -l_Lean_Expr_updateLambda_x21___closed__3 = _init_l_Lean_Expr_updateLambda_x21___closed__3(); -lean_mark_persistent(l_Lean_Expr_updateLambda_x21___closed__3); +l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__1 = _init_l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__1); +l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__2 = _init_l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__2); +l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__3 = _init_l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__3(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateLambda_x21Impl___closed__3); l_Lean_Expr_updateLambdaE_x21___closed__1 = _init_l_Lean_Expr_updateLambdaE_x21___closed__1(); lean_mark_persistent(l_Lean_Expr_updateLambdaE_x21___closed__1); l_Lean_Expr_updateLambdaE_x21___closed__2 = _init_l_Lean_Expr_updateLambdaE_x21___closed__2(); lean_mark_persistent(l_Lean_Expr_updateLambdaE_x21___closed__2); -l_Lean_Expr_updateLet_x21___closed__1 = _init_l_Lean_Expr_updateLet_x21___closed__1(); -lean_mark_persistent(l_Lean_Expr_updateLet_x21___closed__1); -l_Lean_Expr_updateLet_x21___closed__2 = _init_l_Lean_Expr_updateLet_x21___closed__2(); -lean_mark_persistent(l_Lean_Expr_updateLet_x21___closed__2); +l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__1 = _init_l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__1); +l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__2 = _init_l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Expr_0__Lean_Expr_updateLet_x21Impl___closed__2); l_Lean_Expr_setPPExplicit___closed__1 = _init_l_Lean_Expr_setPPExplicit___closed__1(); lean_mark_persistent(l_Lean_Expr_setPPExplicit___closed__1); l_Lean_Expr_setPPExplicit___closed__2 = _init_l_Lean_Expr_setPPExplicit___closed__2(); diff --git a/stage0/stdlib/Lean/Level.c b/stage0/stdlib/Lean/Level.c index 1e6cc552b811..225fc712c32b 100644 --- a/stage0/stdlib/Lean/Level.c +++ b/stage0/stdlib/Lean/Level.c @@ -15,6 +15,7 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lean_Level_dec(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_getMaxArgsAux(lean_object*, lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_simpLevelIMax_x27___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Level_PP_Result_quote___lambda__3___closed__9; size_t lean_usize_add(size_t, size_t); LEAN_EXPORT uint8_t l_Lean_Level_isNeverZero(lean_object*); @@ -36,6 +37,8 @@ static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level__ static lean_object* l_Lean_Level_PP_Result_quote___lambda__3___closed__8; static lean_object* l_Lean_Level_PP_Result_format___closed__1; LEAN_EXPORT lean_object* l_Lean_Level_quote___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__3; +uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l_Lean_Level_normalize___closed__6; lean_object* l_Array_append___rarg(lean_object*, lean_object*); @@ -43,7 +46,6 @@ LEAN_EXPORT lean_object* l_Lean_instForInMVarIdMapProdMVarId(lean_object*, lean_ static lean_object* l___private_Lean_Level_0__Lean_reprMVarId____x40_Lean_Level___hyg_506____closed__11; LEAN_EXPORT lean_object* l_Lean_Level_isMVar___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_getMaxArgsAux___at_Lean_Level_normalize___spec__2(lean_object*, uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Level_updateIMax___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_succ___override(lean_object*); static lean_object* l_Lean_Level_mkData___closed__3; extern lean_object* l_Std_Format_defWidth; @@ -59,7 +61,6 @@ lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Level_PP_Result_quote___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_instReprData___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_getOffsetAux___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Level_updateMax_x21(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* lean_level_mk_max(lean_object*, lean_object*); static lean_object* l_Lean_Level_PP_toResult___closed__4; static lean_object* l_Lean_Level_instHashableLevel___closed__1; @@ -75,10 +76,12 @@ static lean_object* l_Lean_Level_mkData___closed__2; lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Level_geq_go(lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); +static lean_object* l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__1; LEAN_EXPORT uint8_t l_Lean_Level_isEquiv(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_instBEqLevel; LEAN_EXPORT lean_object* l_Lean_instReprData___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Level_PP_Result_quote___spec__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__2; LEAN_EXPORT uint8_t lean_level_has_param(lean_object*); LEAN_EXPORT uint64_t l_Lean_Level_hash(lean_object*); static lean_object* l_Lean_instReprData___lambda__3___closed__1; @@ -86,8 +89,10 @@ LEAN_EXPORT lean_object* l_Lean_instReprData___lambda__3___boxed(lean_object*, l static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__4; static lean_object* l___private_Lean_Level_0__Lean_Level_PP_parenIfFalse___closed__4; static lean_object* l_Lean_instForInMVarIdMapProdMVarId___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_isExplicit___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_instForInMVarIdSetMVarId(lean_object*); +static lean_object* l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__3; LEAN_EXPORT uint32_t lean_level_hash(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_hasParamEx___boxed(lean_object*); @@ -106,7 +111,6 @@ lean_object* l_Array_qpartition_loop___rarg(lean_object*, lean_object*, lean_obj LEAN_EXPORT lean_object* l_Lean_Level_depth(lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__22; LEAN_EXPORT lean_object* l_Lean_Level_isSucc___boxed(lean_object*); -static lean_object* l_Lean_Level_updateIMax_x21___closed__1; LEAN_EXPORT uint8_t l___private_Lean_Level_0__Lean_Level_isAlreadyNormalizedCheap(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_getMaxArgsAux___at_Lean_Level_normalize___spec__2___boxed(lean_object*, lean_object*, lean_object*); @@ -119,11 +123,11 @@ static lean_object* l_Lean_Level_data___override___closed__1; lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__12; LEAN_EXPORT lean_object* l_Lean_Level_geq___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Level_updateMax_x21___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_isAlreadyNormalizedCheap___boxed(lean_object*); static lean_object* l_Lean_Level_PP_Result_format___closed__6; +static lean_object* l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__2; static lean_object* l_Lean_instForInMVarIdSetMVarId___closed__2; -LEAN_EXPORT lean_object* lean_level_simp_imax(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_simpLevelIMax_x27(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__8; static lean_object* l_Lean_Level_mvarId_x21___closed__3; extern uint64_t l_instInhabitedUInt64; @@ -135,7 +139,6 @@ static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level__ LEAN_EXPORT lean_object* l_Lean_Level_Data_hasMVar___boxed(lean_object*); lean_object* l_Std_RBTree_forIn___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Name_hash___override(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Level_updateIMax_x21(lean_object*, lean_object*, lean_object*); lean_object* l_Std_RBNode_setBlack___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkLevelIMax(lean_object*, lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__1; @@ -150,13 +153,12 @@ LEAN_EXPORT lean_object* l_Lean_Level_imax___override(lean_object*, lean_object* static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__2; LEAN_EXPORT uint8_t l_Lean_Level_isParam(lean_object*); static lean_object* l_Lean_Level_PP_Result_format___closed__2; -LEAN_EXPORT lean_object* l_Lean_Level_updateSucc_x21(lean_object*, lean_object*); -static lean_object* l_Lean_Level_updateMax_x21___closed__1; lean_object* l_ReaderT_bind___at_Lean_Unhygienic_instMonadQuotationUnhygienic___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_isParam___boxed(lean_object*); static lean_object* l_Lean_Level_PP_toResult___closed__2; static lean_object* l___private_Lean_Level_0__Lean_reprMVarId____x40_Lean_Level___hyg_506____closed__10; lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__1; LEAN_EXPORT uint8_t l_Lean_Level_geq(lean_object*, lean_object*); LEAN_EXPORT uint32_t lean_level_depth(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_isIMax___boxed(lean_object*); @@ -167,18 +169,18 @@ LEAN_EXPORT lean_object* l_Lean_Level_instHashableLevel; LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Level_normalize___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_any___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Level_PP_Result_quote___lambda__3___closed__7; +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_mkData(uint64_t, lean_object*, uint8_t, uint8_t); LEAN_EXPORT lean_object* l_panic___at_Lean_Level_normalize___spec__1(lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__11; -lean_object* lean_level_update_max(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Level_any(lean_object*, lean_object*); -LEAN_EXPORT lean_object* lean_level_mk_max_simp(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t); static lean_object* l_Lean_Level_normalize___closed__1; lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); uint32_t lean_uint64_to_uint32(uint64_t); static lean_object* l_Lean_instHashableMVarId___closed__1; -LEAN_EXPORT lean_object* lean_level_simp_max(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_simpLevelMax_x27(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Unhygienic_run___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkLevelMax(lean_object*, lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprMVarId____x40_Lean_Level___hyg_506____closed__5; @@ -187,16 +189,16 @@ LEAN_EXPORT lean_object* l_Lean_instMVarIdSetEmptyCollection; LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_depth___boxed(lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprMVarId____x40_Lean_Level___hyg_506____closed__3; -LEAN_EXPORT lean_object* lean_level_mk_imax_simp(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_toNat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_geq_go___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_normLtAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instInhabitedMVarIdMap(lean_object*); +static lean_object* l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__2; LEAN_EXPORT uint8_t l___private_Lean_Level_0__Lean_beqMVarId____x40_Lean_Level___hyg_423_(lean_object*, lean_object*); static lean_object* l_Lean_instReprMVarId___closed__1; lean_object* l_Nat_repr(lean_object*); -static lean_object* l_Lean_Level_updateSucc_x21___closed__3; LEAN_EXPORT lean_object* l_Lean_Level_casesOn___override___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Level_PP_Result_quote___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -210,16 +212,13 @@ LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Le static lean_object* l___private_Lean_Level_0__Lean_reprMVarId____x40_Lean_Level___hyg_506____closed__7; static lean_object* l_Lean_Level_PP_Result_quote___lambda__4___closed__2; lean_object* lean_format_pretty(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Level_updateMax___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_isExplicitSubsumedAux___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_occurs___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_isZero___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_ctorToNat(lean_object*); -static lean_object* l_Lean_Level_updateMax_x21___closed__3; static lean_object* l_Lean_instReprData___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Level_ofNat___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_instBEqData___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Level_updateSucc___boxed(lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); static lean_object* l_Lean_Level_PP_toResult___closed__5; LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Level_normalize___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -240,6 +239,7 @@ LEAN_EXPORT uint8_t l___private_Lean_Level_0__Lean_Level_isExplicitSubsumedAux(l static lean_object* l_Lean_Level_normalize___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_skipExplicit___boxed(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_simpLevelMax_x27___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Level_isIMax(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -252,6 +252,7 @@ LEAN_EXPORT lean_object* l_Nat_toLevel(lean_object*); LEAN_EXPORT uint8_t l_Lean_Level_normLt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_casesOn___override___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Level_PP_Result_format___closed__3; +static lean_object* l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__3; static lean_object* l_Lean_Level_PP_Result_quote___lambda__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_imax(lean_object*, lean_object*); lean_object* l_Lean_Syntax_mkNumLit(lean_object*, lean_object*); @@ -263,11 +264,10 @@ static lean_object* l_Lean_Level_normalize___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_mkLevelMaxCore(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__20; uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); -lean_object* lean_level_update_imax(lean_object*, lean_object*, lean_object*); +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l_Nat_imax___boxed(lean_object*, lean_object*); lean_object* l_List_redLength___rarg(lean_object*); LEAN_EXPORT uint8_t l_Lean_instBEqData(uint64_t, uint64_t); -static lean_object* l_Lean_Level_updateIMax_x21___closed__3; LEAN_EXPORT lean_object* l_Lean_instInhabitedMVarId; LEAN_EXPORT lean_object* l_Lean_Level_zero___override; static lean_object* l_Lean_levelOne___closed__1; @@ -282,6 +282,7 @@ static lean_object* l_Lean_Level_PP_toResult___closed__3; static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__16; LEAN_EXPORT lean_object* l_Lean_Level_find_x3f(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl(lean_object*, lean_object*); uint8_t l_Std_RBNode_isRed___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Level_Data_hasMVar(uint64_t); @@ -296,7 +297,6 @@ static lean_object* l_Lean_Level_PP_Result_quote___lambda__6___closed__1; LEAN_EXPORT lean_object* l_Lean_instReprMVarId__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Level_updateSucc_x21___closed__2; static lean_object* l_Lean_Level_PP_Result_quote___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_instReprMVarId__1___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Level_isMVar(lean_object*); @@ -314,7 +314,6 @@ LEAN_EXPORT lean_object* l_Lean_Level_depthEx___boxed(lean_object*); static lean_object* l_Lean_instReprData___lambda__2___closed__2; static lean_object* l___private_Lean_Level_0__Lean_Level_PP_parenIfFalse___closed__3; lean_object* l_List_toArrayAux___rarg(lean_object*, lean_object*); -lean_object* lean_level_update_succ(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_getLevelOffset(lean_object*); static lean_object* l_Lean_Level_PP_Result_quote___lambda__5___closed__3; static lean_object* l___private_Lean_Level_0__Lean_reprMVarId____x40_Lean_Level___hyg_506____closed__9; @@ -337,6 +336,7 @@ LEAN_EXPORT lean_object* l_Lean_Level_isEquiv___boxed(lean_object*, lean_object* LEAN_EXPORT lean_object* l_Lean_Level_instQuoteLevelStrAnonymous(lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); LEAN_EXPORT lean_object* lean_level_mk_zero(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Level_normalize___closed__7; LEAN_EXPORT uint8_t l_Lean_Level_isZero(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_casesOn___override(lean_object*); @@ -355,6 +355,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_PP_parenIfFalse___ lean_object* lean_mk_syntax_ident(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_hashMVarId____x40_Lean_Level___hyg_478____boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_ofNat(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Level_isMaxIMax(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_hash___boxed(lean_object*); @@ -364,8 +365,9 @@ LEAN_EXPORT lean_object* l_Lean_instReprData___boxed(lean_object*, lean_object*) LEAN_EXPORT uint8_t l_Lean_Level_isSucc(lean_object*); static lean_object* l_Lean_Level_PP_Result_quote___lambda__5___closed__1; static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__18; +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Level_isExplicit(lean_object*); -static lean_object* l_Lean_Level_updateSucc_x21___closed__1; +static lean_object* l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__1; LEAN_EXPORT lean_object* l_Lean_Level_mvar___override(lean_object*); static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level___hyg_935____closed__14; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); @@ -389,7 +391,6 @@ static lean_object* l___private_Lean_Level_0__Lean_reprLevel____x40_Lean_Level__ lean_object* lean_nat_to_int(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_Data_hasParam___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Level_updateIMax_x21___closed__2; LEAN_EXPORT lean_object* l_Lean_Level_PP_toResult(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Level_mvarId_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_PP_Result_quote___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -4197,7 +4198,7 @@ static lean_object* _init_l_Lean_Level_normalize___closed__8() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Level_normalize___closed__5; x_2 = l_Lean_Level_normalize___closed__6; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Level_normalize___closed__7; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -6046,7 +6047,7 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* lean_level_mk_max_simp(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_mkLevelMax_x27(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_13; uint8_t x_32; @@ -6331,7 +6332,7 @@ return x_2; } } } -LEAN_EXPORT lean_object* lean_level_simp_max(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_simpLevelMax_x27(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_13; uint8_t x_32; @@ -6354,16 +6355,12 @@ if (lean_obj_tag(x_1) == 2) { lean_object* x_36; lean_object* x_37; uint8_t x_38; x_36 = lean_ctor_get(x_1, 0); -lean_inc(x_36); x_37 = lean_ctor_get(x_1, 1); -lean_inc(x_37); x_38 = lean_level_eq(x_2, x_36); -lean_dec(x_36); if (x_38 == 0) { uint8_t x_39; x_39 = lean_level_eq(x_2, x_37); -lean_dec(x_37); if (x_39 == 0) { lean_object* x_40; @@ -6373,16 +6370,13 @@ goto block_31; } else { -lean_dec(x_3); -lean_dec(x_2); +lean_inc(x_1); return x_1; } } else { -lean_dec(x_37); -lean_dec(x_3); -lean_dec(x_2); +lean_inc(x_1); return x_1; } } @@ -6409,16 +6403,12 @@ if (lean_obj_tag(x_1) == 2) { lean_object* x_46; lean_object* x_47; uint8_t x_48; x_46 = lean_ctor_get(x_1, 0); -lean_inc(x_46); x_47 = lean_ctor_get(x_1, 1); -lean_inc(x_47); x_48 = lean_level_eq(x_2, x_46); -lean_dec(x_46); if (x_48 == 0) { uint8_t x_49; x_49 = lean_level_eq(x_2, x_47); -lean_dec(x_47); if (x_49 == 0) { lean_object* x_50; @@ -6428,16 +6418,13 @@ goto block_31; } else { -lean_dec(x_3); -lean_dec(x_2); +lean_inc(x_1); return x_1; } } else { -lean_dec(x_47); -lean_dec(x_3); -lean_dec(x_2); +lean_inc(x_1); return x_1; } } @@ -6451,30 +6438,26 @@ goto block_31; } else { -lean_dec(x_3); -lean_dec(x_2); +lean_inc(x_1); return x_1; } } } else { -lean_dec(x_3); -lean_dec(x_2); +lean_inc(x_1); return x_1; } } else { -lean_dec(x_3); -lean_dec(x_1); +lean_inc(x_2); return x_2; } } else { -lean_dec(x_3); -lean_dec(x_2); +lean_inc(x_1); return x_1; } block_12: @@ -6488,14 +6471,12 @@ lean_dec(x_6); lean_dec(x_5); if (x_7 == 0) { -lean_dec(x_2); -lean_dec(x_1); +lean_inc(x_3); return x_3; } else { lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -lean_dec(x_3); x_8 = lean_unsigned_to_nat(0u); x_9 = l_Lean_Level_getOffsetAux(x_2, x_8); x_10 = l_Lean_Level_getOffsetAux(x_1, x_8); @@ -6504,12 +6485,12 @@ lean_dec(x_10); lean_dec(x_9); if (x_11 == 0) { -lean_dec(x_1); +lean_inc(x_2); return x_2; } else { -lean_dec(x_2); +lean_inc(x_1); return x_1; } } @@ -6525,16 +6506,12 @@ if (lean_obj_tag(x_2) == 2) { lean_object* x_15; lean_object* x_16; uint8_t x_17; x_15 = lean_ctor_get(x_2, 0); -lean_inc(x_15); x_16 = lean_ctor_get(x_2, 1); -lean_inc(x_16); x_17 = lean_level_eq(x_1, x_15); -lean_dec(x_15); if (x_17 == 0) { uint8_t x_18; x_18 = lean_level_eq(x_1, x_16); -lean_dec(x_16); if (x_18 == 0) { lean_object* x_19; @@ -6544,16 +6521,13 @@ goto block_12; } else { -lean_dec(x_3); -lean_dec(x_1); +lean_inc(x_2); return x_2; } } else { -lean_dec(x_16); -lean_dec(x_3); -lean_dec(x_1); +lean_inc(x_2); return x_2; } } @@ -6580,16 +6554,12 @@ if (lean_obj_tag(x_2) == 2) { lean_object* x_25; lean_object* x_26; uint8_t x_27; x_25 = lean_ctor_get(x_2, 0); -lean_inc(x_25); x_26 = lean_ctor_get(x_2, 1); -lean_inc(x_26); x_27 = lean_level_eq(x_1, x_25); -lean_dec(x_25); if (x_27 == 0) { uint8_t x_28; x_28 = lean_level_eq(x_1, x_26); -lean_dec(x_26); if (x_28 == 0) { lean_object* x_29; @@ -6599,16 +6569,13 @@ goto block_12; } else { -lean_dec(x_3); -lean_dec(x_1); +lean_inc(x_2); return x_2; } } else { -lean_dec(x_26); -lean_dec(x_3); -lean_dec(x_1); +lean_inc(x_2); return x_2; } } @@ -6622,14 +6589,24 @@ goto block_12; } else { -lean_dec(x_3); -lean_dec(x_1); +lean_inc(x_2); return x_2; } } } } } +LEAN_EXPORT lean_object* l_Lean_simpLevelMax_x27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_simpLevelMax_x27(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_mkLevelIMaxCore(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -6680,12 +6657,12 @@ else { lean_object* x_10; lean_dec(x_3); -x_10 = lean_level_mk_max_simp(x_1, x_2); +x_10 = l_Lean_mkLevelMax_x27(x_1, x_2); return x_10; } } } -LEAN_EXPORT lean_object* lean_level_mk_imax_simp(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_mkLevelIMax_x27(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; @@ -6729,12 +6706,12 @@ return x_2; else { lean_object* x_8; -x_8 = lean_level_mk_max_simp(x_1, x_2); +x_8 = l_Lean_mkLevelMax_x27(x_1, x_2); return x_8; } } } -LEAN_EXPORT lean_object* lean_level_simp_imax(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_simpLevelIMax_x27(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -6755,24 +6732,22 @@ lean_dec(x_2); if (x_7 == 0) { lean_dec(x_1); +lean_inc(x_3); return x_3; } else { -lean_dec(x_3); return x_1; } } else { -lean_dec(x_3); lean_dec(x_1); return x_2; } } else { -lean_dec(x_3); lean_dec(x_1); return x_2; } @@ -6780,29 +6755,29 @@ return x_2; else { lean_object* x_8; -lean_dec(x_3); -x_8 = lean_level_mk_max_simp(x_1, x_2); +x_8 = l_Lean_mkLevelMax_x27(x_1, x_2); return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_Level_updateSucc___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_simpLevelIMax_x27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = lean_level_update_succ(x_1, x_2); +x_4 = l_Lean_simpLevelIMax_x27(x_1, x_2, x_3); +lean_dec(x_3); return x_4; } } -static lean_object* _init_l_Lean_Level_updateSucc_x21___closed__1() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateSucc!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateSucc!Impl", 48); return x_1; } } -static lean_object* _init_l_Lean_Level_updateSucc_x21___closed__2() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__2() { _start: { lean_object* x_1; @@ -6810,56 +6785,70 @@ x_1 = lean_mk_string_from_bytes("succ level expected", 19); return x_1; } } -static lean_object* _init_l_Lean_Level_updateSucc_x21___closed__3() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Level_mkData___closed__2; -x_2 = l_Lean_Level_updateSucc_x21___closed__1; -x_3 = lean_unsigned_to_nat(538u); -x_4 = lean_unsigned_to_nat(15u); -x_5 = l_Lean_Level_updateSucc_x21___closed__2; +x_2 = l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(527u); +x_4 = lean_unsigned_to_nat(14u); +x_5 = l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Level_updateSucc_x21(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 1) { -lean_object* x_3; -x_3 = lean_level_update_succ(x_1, x_2); -return x_3; +lean_object* x_3; size_t x_4; size_t x_5; uint8_t x_6; +x_3 = lean_ctor_get(x_1, 0); +x_4 = lean_ptr_addr(x_3); +x_5 = lean_ptr_addr(x_2); +x_6 = lean_usize_dec_eq(x_4, x_5); +if (x_6 == 0) +{ +lean_object* x_7; +x_7 = l_Lean_Level_succ___override(x_2); +return x_7; } else { -lean_object* x_4; lean_object* x_5; lean_dec(x_2); -lean_dec(x_1); -x_4 = l_Lean_Level_updateSucc_x21___closed__3; -x_5 = l_panic___at_Lean_Level_normalize___spec__1(x_4); -return x_5; +lean_inc(x_1); +return x_1; +} +} +else +{ +lean_object* x_8; lean_object* x_9; +lean_dec(x_2); +x_8 = l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__3; +x_9 = l_panic___at_Lean_Level_normalize___spec__1(x_8); +return x_9; } } } -LEAN_EXPORT lean_object* l_Lean_Level_updateMax___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_5; -x_5 = lean_level_update_max(x_1, x_2, x_3); -return x_5; +lean_object* x_3; +x_3 = l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl(x_1, x_2); +lean_dec(x_1); +return x_3; } } -static lean_object* _init_l_Lean_Level_updateMax_x21___closed__1() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateMax!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateMax!Impl", 47); return x_1; } } -static lean_object* _init_l_Lean_Level_updateMax_x21___closed__2() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__2() { _start: { lean_object* x_1; @@ -6867,57 +6856,87 @@ x_1 = lean_mk_string_from_bytes("max level expected", 18); return x_1; } } -static lean_object* _init_l_Lean_Level_updateMax_x21___closed__3() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Level_mkData___closed__2; -x_2 = l_Lean_Level_updateMax_x21___closed__1; -x_3 = lean_unsigned_to_nat(547u); -x_4 = lean_unsigned_to_nat(14u); -x_5 = l_Lean_Level_updateMax_x21___closed__2; +x_2 = l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(538u); +x_4 = lean_unsigned_to_nat(19u); +x_5 = l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Level_updateMax_x21(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 2) { -lean_object* x_4; -x_4 = lean_level_update_max(x_1, x_2, x_3); -return x_4; +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; uint8_t x_8; +x_4 = lean_ctor_get(x_1, 0); +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ptr_addr(x_4); +x_7 = lean_ptr_addr(x_2); +x_8 = lean_usize_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Lean_mkLevelMax_x27(x_2, x_3); +return x_9; } else { -lean_object* x_5; lean_object* x_6; +size_t x_10; size_t x_11; uint8_t x_12; +x_10 = lean_ptr_addr(x_5); +x_11 = lean_ptr_addr(x_3); +x_12 = lean_usize_dec_eq(x_10, x_11); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = l_Lean_mkLevelMax_x27(x_2, x_3); +return x_13; +} +else +{ +lean_object* x_14; +x_14 = l_Lean_simpLevelMax_x27(x_2, x_3, x_1); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_5 = l_Lean_Level_updateMax_x21___closed__3; -x_6 = l_panic___at_Lean_Level_normalize___spec__1(x_5); -return x_6; +return x_14; +} +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_3); +lean_dec(x_2); +x_15 = l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__3; +x_16 = l_panic___at_Lean_Level_normalize___spec__1(x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l_Lean_Level_updateIMax___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; -x_5 = lean_level_update_imax(x_1, x_2, x_3); -return x_5; +lean_object* x_4; +x_4 = l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; } } -static lean_object* _init_l_Lean_Level_updateIMax_x21___closed__1() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateIMax!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateIMax!Impl", 48); return x_1; } } -static lean_object* _init_l_Lean_Level_updateIMax_x21___closed__2() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__2() { _start: { lean_object* x_1; @@ -6925,40 +6944,76 @@ x_1 = lean_mk_string_from_bytes("imax level expected", 19); return x_1; } } -static lean_object* _init_l_Lean_Level_updateIMax_x21___closed__3() { +static lean_object* _init_l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Level_mkData___closed__2; -x_2 = l_Lean_Level_updateIMax_x21___closed__1; -x_3 = lean_unsigned_to_nat(556u); -x_4 = lean_unsigned_to_nat(15u); -x_5 = l_Lean_Level_updateIMax_x21___closed__2; +x_2 = l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__1; +x_3 = lean_unsigned_to_nat(549u); +x_4 = lean_unsigned_to_nat(20u); +x_5 = l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Level_updateIMax_x21(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 3) { -lean_object* x_4; -x_4 = lean_level_update_imax(x_1, x_2, x_3); -return x_4; +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; uint8_t x_8; +x_4 = lean_ctor_get(x_1, 0); +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ptr_addr(x_4); +x_7 = lean_ptr_addr(x_2); +x_8 = lean_usize_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = l_Lean_mkLevelIMax_x27(x_2, x_3); +return x_9; } else { -lean_object* x_5; lean_object* x_6; +size_t x_10; size_t x_11; uint8_t x_12; +x_10 = lean_ptr_addr(x_5); +x_11 = lean_ptr_addr(x_3); +x_12 = lean_usize_dec_eq(x_10, x_11); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = l_Lean_mkLevelIMax_x27(x_2, x_3); +return x_13; +} +else +{ +lean_object* x_14; +x_14 = l_Lean_simpLevelIMax_x27(x_2, x_3, x_1); +return x_14; +} +} +} +else +{ +lean_object* x_15; lean_object* x_16; lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_5 = l_Lean_Level_updateIMax_x21___closed__3; -x_6 = l_panic___at_Lean_Level_normalize___spec__1(x_5); -return x_6; +x_15 = l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__3; +x_16 = l_panic___at_Lean_Level_normalize___spec__1(x_15); +return x_16; } } } +LEAN_EXPORT lean_object* l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Level_mkNaryMax(lean_object* x_1) { _start: { @@ -6988,7 +7043,7 @@ x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = l_Lean_Level_mkNaryMax(x_3); -x_7 = lean_level_mk_max_simp(x_5, x_6); +x_7 = l_Lean_mkLevelMax_x27(x_5, x_6); return x_7; } } @@ -7012,80 +7067,165 @@ return x_2; } else { -lean_object* x_5; lean_object* x_6; +lean_object* x_5; size_t x_6; size_t x_7; uint8_t x_8; +lean_inc(x_3); x_5 = l_Lean_Level_instantiateParams(x_1, x_3); -x_6 = lean_level_update_succ(x_2, x_5); -return x_6; +x_6 = lean_ptr_addr(x_3); +lean_dec(x_3); +x_7 = lean_ptr_addr(x_5); +x_8 = lean_usize_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; +lean_dec(x_2); +x_9 = l_Lean_Level_succ___override(x_5); +return x_9; +} +else +{ +lean_dec(x_5); +return x_2; +} } } case 2: { -lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_2, 1); -lean_inc(x_8); -x_9 = l_Lean_Level_hasParam(x_2); -if (x_9 == 0) +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_2, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = l_Lean_Level_hasParam(x_2); +if (x_12 == 0) { -lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_1); return x_2; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; uint8_t x_17; +lean_inc(x_10); lean_inc(x_1); -x_10 = l_Lean_Level_instantiateParams(x_1, x_7); -x_11 = l_Lean_Level_instantiateParams(x_1, x_8); -x_12 = lean_level_update_max(x_2, x_10, x_11); -return x_12; -} +x_13 = l_Lean_Level_instantiateParams(x_1, x_10); +lean_inc(x_11); +x_14 = l_Lean_Level_instantiateParams(x_1, x_11); +x_15 = lean_ptr_addr(x_10); +lean_dec(x_10); +x_16 = lean_ptr_addr(x_13); +x_17 = lean_usize_dec_eq(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; +lean_dec(x_11); +lean_dec(x_2); +x_18 = l_Lean_mkLevelMax_x27(x_13, x_14); +return x_18; } -case 3: +else { -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = lean_ctor_get(x_2, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_2, 1); -lean_inc(x_14); -x_15 = l_Lean_Level_hasParam(x_2); -if (x_15 == 0) +size_t x_19; size_t x_20; uint8_t x_21; +x_19 = lean_ptr_addr(x_11); +lean_dec(x_11); +x_20 = lean_ptr_addr(x_14); +x_21 = lean_usize_dec_eq(x_19, x_20); +if (x_21 == 0) +{ +lean_object* x_22; +lean_dec(x_2); +x_22 = l_Lean_mkLevelMax_x27(x_13, x_14); +return x_22; +} +else { +lean_object* x_23; +x_23 = l_Lean_simpLevelMax_x27(x_13, x_14, x_2); +lean_dec(x_2); lean_dec(x_14); lean_dec(x_13); +return x_23; +} +} +} +} +case 3: +{ +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = lean_ctor_get(x_2, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_2, 1); +lean_inc(x_25); +x_26 = l_Lean_Level_hasParam(x_2); +if (x_26 == 0) +{ +lean_dec(x_25); +lean_dec(x_24); lean_dec(x_1); return x_2; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_object* x_27; lean_object* x_28; size_t x_29; size_t x_30; uint8_t x_31; +lean_inc(x_24); lean_inc(x_1); -x_16 = l_Lean_Level_instantiateParams(x_1, x_13); -x_17 = l_Lean_Level_instantiateParams(x_1, x_14); -x_18 = lean_level_update_imax(x_2, x_16, x_17); -return x_18; +x_27 = l_Lean_Level_instantiateParams(x_1, x_24); +lean_inc(x_25); +x_28 = l_Lean_Level_instantiateParams(x_1, x_25); +x_29 = lean_ptr_addr(x_24); +lean_dec(x_24); +x_30 = lean_ptr_addr(x_27); +x_31 = lean_usize_dec_eq(x_29, x_30); +if (x_31 == 0) +{ +lean_object* x_32; +lean_dec(x_25); +lean_dec(x_2); +x_32 = l_Lean_mkLevelIMax_x27(x_27, x_28); +return x_32; +} +else +{ +size_t x_33; size_t x_34; uint8_t x_35; +x_33 = lean_ptr_addr(x_25); +lean_dec(x_25); +x_34 = lean_ptr_addr(x_28); +x_35 = lean_usize_dec_eq(x_33, x_34); +if (x_35 == 0) +{ +lean_object* x_36; +lean_dec(x_2); +x_36 = l_Lean_mkLevelIMax_x27(x_27, x_28); +return x_36; +} +else +{ +lean_object* x_37; +x_37 = l_Lean_simpLevelIMax_x27(x_27, x_28, x_2); +lean_dec(x_2); +return x_37; +} +} } } case 4: { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_2, 0); -lean_inc(x_19); -x_20 = lean_apply_1(x_1, x_19); -if (lean_obj_tag(x_20) == 0) +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_2, 0); +lean_inc(x_38); +x_39 = lean_apply_1(x_1, x_38); +if (lean_obj_tag(x_39) == 0) { return x_2; } else { -lean_object* x_21; +lean_object* x_40; lean_dec(x_2); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -lean_dec(x_20); -return x_21; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +lean_dec(x_39); +return x_40; } } default: @@ -10427,24 +10567,24 @@ l_Lean_Level_PP_Result_quote___lambda__6___closed__1 = _init_l_Lean_Level_PP_Res lean_mark_persistent(l_Lean_Level_PP_Result_quote___lambda__6___closed__1); l_Lean_Level_PP_Result_quote___closed__1 = _init_l_Lean_Level_PP_Result_quote___closed__1(); lean_mark_persistent(l_Lean_Level_PP_Result_quote___closed__1); -l_Lean_Level_updateSucc_x21___closed__1 = _init_l_Lean_Level_updateSucc_x21___closed__1(); -lean_mark_persistent(l_Lean_Level_updateSucc_x21___closed__1); -l_Lean_Level_updateSucc_x21___closed__2 = _init_l_Lean_Level_updateSucc_x21___closed__2(); -lean_mark_persistent(l_Lean_Level_updateSucc_x21___closed__2); -l_Lean_Level_updateSucc_x21___closed__3 = _init_l_Lean_Level_updateSucc_x21___closed__3(); -lean_mark_persistent(l_Lean_Level_updateSucc_x21___closed__3); -l_Lean_Level_updateMax_x21___closed__1 = _init_l_Lean_Level_updateMax_x21___closed__1(); -lean_mark_persistent(l_Lean_Level_updateMax_x21___closed__1); -l_Lean_Level_updateMax_x21___closed__2 = _init_l_Lean_Level_updateMax_x21___closed__2(); -lean_mark_persistent(l_Lean_Level_updateMax_x21___closed__2); -l_Lean_Level_updateMax_x21___closed__3 = _init_l_Lean_Level_updateMax_x21___closed__3(); -lean_mark_persistent(l_Lean_Level_updateMax_x21___closed__3); -l_Lean_Level_updateIMax_x21___closed__1 = _init_l_Lean_Level_updateIMax_x21___closed__1(); -lean_mark_persistent(l_Lean_Level_updateIMax_x21___closed__1); -l_Lean_Level_updateIMax_x21___closed__2 = _init_l_Lean_Level_updateIMax_x21___closed__2(); -lean_mark_persistent(l_Lean_Level_updateIMax_x21___closed__2); -l_Lean_Level_updateIMax_x21___closed__3 = _init_l_Lean_Level_updateIMax_x21___closed__3(); -lean_mark_persistent(l_Lean_Level_updateIMax_x21___closed__3); +l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__1 = _init_l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__1); +l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__2 = _init_l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__2); +l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__3 = _init_l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__3(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateSucc_x21Impl___closed__3); +l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__1 = _init_l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__1); +l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__2 = _init_l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__2); +l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__3 = _init_l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__3(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateMax_x21Impl___closed__3); +l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__1 = _init_l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__1(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__1); +l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__2 = _init_l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__2(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__2); +l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__3 = _init_l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__3(); +lean_mark_persistent(l___private_Lean_Level_0__Lean_Level_updateIMax_x21Impl___closed__3); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Linter/Basic.c b/stage0/stdlib/Lean/Linter/Basic.c index b4671c7ff9ac..1c57d270dc96 100644 --- a/stage0/stdlib/Lean/Linter/Basic.c +++ b/stage0/stdlib/Lean/Linter/Basic.c @@ -13,28 +13,35 @@ #ifdef __cplusplus extern "C" { #endif +lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInFun___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7____closed__6; static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__2; static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__6; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__7; +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__9; size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__8; static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__7; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__23(lean_object*, lean_object*, size_t, size_t); +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__4; LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInFun___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___boxed(lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__16; +LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Linter_unusedVariables___spec__28(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__5; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__1; lean_object* l_Std_HashMapImp_find_x3f___at_Lean_ForEachExpr_visit___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__3; static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__3; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__10; lean_object* l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(lean_object*); +LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables___spec__30(lean_object*, lean_object*, uint8_t, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); -static lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__1; +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__1; lean_object* l_Lean_Elab_InfoTree_hasSorry(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__1; -LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__3; uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); @@ -43,24 +50,30 @@ uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1848_(l LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___boxed(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInStructure___rarg(lean_object*); -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__2; -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInStructure___rarg___closed__6; +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_contains___at_Lean_Linter_unusedVariables___spec__15___boxed(lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__13; +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__3(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Server_InfoUtils_0__String_beqRange____x40_Lean_Server_InfoUtils___hyg_75_(lean_object*, lean_object*); +static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___closed__1; static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__10; -LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___spec__1(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__9; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__8; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__33(lean_object*, lean_object*, size_t, size_t); +static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___closed__1; static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_matchesUnusedPattern___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25___boxed(lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashSetImp_expand___at_Lean_Linter_unusedVariables___spec__4(lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__2; +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__5; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__1; +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__3; LEAN_EXPORT lean_object* l_Std_mkHashSet___at_Lean_Linter_unusedVariables___spec__2(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__6; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___boxed(lean_object*); @@ -72,34 +85,33 @@ LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isPatternVar___rarg___box static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__9; LEAN_EXPORT lean_object* l_Std_HashMapImp_moveEntries___at_Lean_Linter_unusedVariables___spec__11(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isVariable(lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariablesPatternVars___boxed(lean_object*); lean_object* l_Lean_Elab_Command_addLinter(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___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_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInLetDeclaration___rarg(lean_object*); +lean_object* l_Lean_Elab_Info_updateContext_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariablesFunArgs___boxed(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__2___closed__1; -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__6; -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__8; -LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isInConstantOrAxiom___spec__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__1; +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__32(lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* l_Std_mkHashSetImp___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___boxed(lean_object*); LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1(uint8_t, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__4; static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__4; lean_object* l_List_get_x3f___rarg(lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__4; static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__1; static lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__6; static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__5; LEAN_EXPORT uint8_t l_Std_AssocList_contains___at_Lean_Linter_unusedVariables___spec__9(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__14; static lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1___closed__3; -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__11; -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__9; +extern lean_object* l_Lean_Elab_Command_instMonadCommandElabM; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__32___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_matchesUnusedPattern___closed__1; static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__11; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isTopLevelDecl___boxed(lean_object*, lean_object*, lean_object*); @@ -113,6 +125,7 @@ static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7____clo static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__4; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isInCtorOrStructBinder___spec__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__6; static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__10; uint8_t l_Lean_Linter_stackMatches(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_elem___at_Lean_Linter_unusedVariables_isTopLevelDecl___spec__2___boxed(lean_object*, lean_object*); @@ -122,6 +135,7 @@ LEAN_EXPORT lean_object* l_Std_PersistentHashMap_foldlM___at_Lean_Linter_unusedV static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__7; LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInLetDeclaration___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInStructure(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Linter_unusedVariables___spec__6(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isTopLevelDecl___closed__4; @@ -131,117 +145,134 @@ static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__7; static lean_object* l_Lean_Linter_unusedVariables_isInLetDeclaration___rarg___closed__3; uint8_t l_Lean_Name_hasMacroScopes(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___boxed(lean_object*); +static lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___closed__1; LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariablesFunArgs(lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Linter_unusedVariables___spec__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__33___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_unusedVariables___spec__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__8; LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isInDeclarationSignature___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isVariable___boxed(lean_object*); lean_object* l_Lean_Option_register___at_Lean_initFn____x40_Lean_PrettyPrinter_Delaborator_Options___hyg_6____spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInInductive___rarg(lean_object*); uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Linter_unusedVariables_isInStructure___rarg___closed__7; lean_object* lean_st_ref_take(lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__11; -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__6; static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__13; static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__8; LEAN_EXPORT lean_object* l_List_replace___at_Lean_Linter_unusedVariables___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_List_elem___at_Lean_Linter_unusedVariables_isTopLevelDecl___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___boxed(lean_object*); -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__4; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__36___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__11; -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__9; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___boxed(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__9; -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__9; -LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariables(lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterUnusedVariablesPatternVars(lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Elab_Info_contains(lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__14; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__4; LEAN_EXPORT lean_object* l_Lean_ForEachExpr_visit___at_Lean_Linter_unusedVariables___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__3___closed__1; lean_object* l_Lean_Name_toString(lean_object*, uint8_t); -static lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__2; +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_37____closed__2; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__5; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___boxed(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_67____closed__3; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___boxed(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__8; +lean_object* l_instInhabited___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__1; lean_object* l_Std_PersistentHashMap_foldlMAux_traverse___at_Lean_mkModuleData___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashSetImp_insert___at_Lean_Linter_unusedVariables___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDeclarationSignature___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_67_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_37_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577_(lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__3; static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__4; static lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__4; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7____closed__1; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDepArrow(lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__2; static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__1; lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInDeclarationSignature___rarg(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInLetDeclaration___rarg___closed__5; +LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__36(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__4; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7____closed__2; static lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__2; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__21(lean_object*, lean_object*); lean_object* l_Lean_Linter_publishMessage(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Std_HashSetImp_insert___at_Lean_Meta_getNondepPropHyps___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_foldlMAux___at_Lean_Linter_unusedVariables___spec__17(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_67____closed__2; -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__12; static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__9; LEAN_EXPORT lean_object* l_Lean_ForEachExpr_visit___at_Lean_Linter_unusedVariables___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Linter_findSyntaxStack_x3f(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isVariable___rarg(lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__1; +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__2; +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_37____closed__1; LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at_Lean_Linter_unusedVariables___spec__10(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_replace___at_Lean_Linter_unusedVariables___spec__7___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__3; +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__1; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__8; LEAN_EXPORT lean_object* l_Lean_Linter_getLinterUnusedVariables___boxed(lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__3; +LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg(lean_object*); size_t lean_usize_modn(size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables; uint64_t l___private_Lean_Level_0__Lean_hashMVarId____x40_Lean_Level___hyg_478_(lean_object*); LEAN_EXPORT uint8_t l_Std_HashMapImp_contains___at_Lean_Linter_unusedVariables___spec__15(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashSetImp_moveEntries___at_Lean_Linter_unusedVariables___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Linter_unusedVariables___spec__8(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__3; +lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDeclarationSignature(lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isInInductive___spec__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__9; static lean_object* l_Lean_Linter_unusedVariables_isTopLevelDecl___closed__5; static lean_object* l_Lean_Linter_unusedVariables_isInDeclarationSignature___rarg___closed__3; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__27(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__9; +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDepArrow___rarg___closed__6; +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__10; static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__6; +lean_object* l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isPatternVar___rarg(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInLetDeclaration___rarg___closed__2; -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___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*); uint8_t l_Lean_Linter_getLinterAll(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__2; LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables_isInDeclarationSignature___spec__1(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDeclarationSignature___rarg___closed__1; size_t lean_usize_of_nat(lean_object*); lean_object* l_Std_HashMap_insert___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__4(lean_object*, lean_object*, lean_object*); @@ -249,143 +280,154 @@ static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__8; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_foldlMAux___at_Lean_Linter_unusedVariables___spec__17___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__2; static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__3; -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__10; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInDeclarationSignature___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables___spec__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__7; +LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom(lean_object*); lean_object* l_Lean_Elab_InfoTree_foldInfo___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_HashSetImp_contains___at_Lean_Linter_unusedVariables_isTopLevelDecl___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__6; +lean_object* l_Std_PersistentArray_toList___rarg(lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__15; static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__8; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7____closed__5; static lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1___closed__4; -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__7; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__13; static lean_object* l_Lean_Linter_unusedVariables_isInLetDeclaration___rarg___closed__6; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInFun(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_toList___at_Lean_Linter_unusedVariables___spec__20(lean_object*); -static lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___closed__1; +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__8; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isPatternVar(lean_object*); static lean_object* l_Lean_Linter_unusedVariables___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_matchesUnusedPattern(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInLetDeclaration___rarg___closed__1; static lean_object* l_Lean_Linter_unusedVariables_isTopLevelDecl___closed__6; static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__10; LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables_funArgs; -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__10; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7____closed__3; -lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t); +lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInStructure___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Std_PersistentHashMap_foldlMAux___at_Lean_Linter_unusedVariables___spec__17___closed__1; +static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577____closed__1; lean_object* l_Std_PersistentArray_toArray___rarg(lean_object*); +lean_object* l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInStructure___rarg___closed__1; lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__18(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables_isInConstantOrAxiom___spec__1(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___boxed(lean_object*); LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables_isInCtorOrStructBinder___spec__1(lean_object*, uint8_t, lean_object*); static lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1___closed__2; +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isTopLevelDecl(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInStructure___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__2; LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables_isInInductive___spec__1(lean_object*, uint8_t, lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__2; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_37____closed__3; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInLetDeclaration___rarg___boxed(lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__12; static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__1; static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__3; static lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1___closed__1; static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__11; static lean_object* l_Lean_Linter_unusedVariables_isInStructure___rarg___closed__2; -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__22(lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__5; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__1; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___boxed(lean_object*); +static lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__11; uint64_t l___private_Lean_Server_InfoUtils_0__String_hashRange____x40_Lean_Server_InfoUtils___hyg_146_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables___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_nat_mul(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg(lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__7___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Linter_linter_unusedVariables_patternVars; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__12(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29(lean_object*, lean_object*, lean_object*, size_t, size_t); static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__2; uint8_t l_String_startsWith(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__24(lean_object*, lean_object*, lean_object*, size_t, size_t); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; static lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1___closed__6; lean_object* l_Lean_KVMap_findCore(lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__2; static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__6; +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__12; +lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__7; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__31(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7____closed__4; -LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__3; lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInStructure___rarg___closed__4; uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isVariable___rarg___closed__3; +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__11; static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__1; static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__3; -static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429____closed__1; static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_unusedVariables___spec__27(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInInductive(lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__1; -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__16; -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__14; uint8_t l_Std_AssocList_contains___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__5(lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__15; -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__5; +static lean_object* l_panic___at_Lean_Linter_unusedVariables___spec__27___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_37____closed__4; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashSetImp_contains___at_Lean_Linter_unusedVariables_isTopLevelDecl___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__5; static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__7; static lean_object* l_Lean_Linter_unusedVariables_isInFun___rarg___closed__5; LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__21___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__6; static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__12; uint8_t l_Std_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Linter_unusedVariables___spec__1(lean_object*); lean_object* lean_local_ctx_find(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_67____closed__4; static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__10; uint8_t l_Std_HashSetImp_contains___at_Lean_Meta_getNondepPropHyps___spec__12(lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_lctx(lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isTopLevelDecl___closed__3; +static lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__2; LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_Linter_unusedVariables___spec__13(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInLetDeclaration___rarg___closed__4; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInInductive___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isPatternVar___boxed(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__5; lean_object* l_Std_HashMap_insert___at_Lean_ForEachExpr_visit___spec__3(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__7; +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__38(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__2; static lean_object* l_Lean_Linter_unusedVariables_isInStructure___rarg___closed__3; +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_unusedVariables_isInStructure___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder(lean_object*); static lean_object* l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__7; -static lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__3; static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__10; static lean_object* l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__7; static lean_object* l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___closed__5; static lean_object* l_Lean_Linter_unusedVariables_isInInductive___rarg___closed__8; LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInDepArrow___rarg(lean_object*); -LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__2(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_7____closed__1() { _start: { @@ -1773,7 +1815,7 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables_isInConstantOrAxiom___spec__1(lean_object* x_1, uint8_t x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___spec__1(lean_object* x_1, uint8_t x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -1787,7 +1829,7 @@ lean_object* x_4; lean_object* x_5; uint8_t x_6; uint8_t x_7; x_4 = lean_ctor_get(x_3, 0); x_5 = lean_ctor_get(x_3, 1); lean_inc(x_1); -x_6 = l_List_foldr___at_Lean_Linter_unusedVariables_isInConstantOrAxiom___spec__1(x_1, x_2, x_5); +x_6 = l_List_foldr___at_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___spec__1(x_1, x_2, x_5); x_7 = l_Lean_Syntax_isOfKind(x_1, x_4); if (x_7 == 0) { @@ -1802,7 +1844,7 @@ return x_8; } } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__1() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -1812,11 +1854,11 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__2() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__1; +x_1 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__1; x_2 = l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -1824,43 +1866,43 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__3() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Linter_unusedVariables_isVariable___rarg___closed__3; -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__2; +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__2; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__4() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__3; +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__3; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__5() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Linter_unusedVariables_isVariable___rarg___closed__3; -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__4; +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__6() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__6() { _start: { lean_object* x_1; @@ -1868,17 +1910,17 @@ x_1 = lean_mk_string_from_bytes("opaque", 6); return x_1; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__7() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__6; -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__6; +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__8() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__8() { _start: { lean_object* x_1; @@ -1886,45 +1928,45 @@ x_1 = lean_mk_string_from_bytes("axiom", 5); return x_1; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__9() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Linter_unusedVariables_skipDeclIdIfPresent___closed__6; -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__8; +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__10() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__9; +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__9; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__11() { +static lean_object* _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__7; -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__10; +x_1 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__7; +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__10; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg(lean_object* x_1) { +LEAN_EXPORT uint8_t l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__5; +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__5; lean_inc(x_1); x_3 = l_Lean_Linter_stackMatches(x_1, x_2); if (x_3 == 0) @@ -1956,47 +1998,47 @@ x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); lean_dec(x_8); x_10 = 0; -x_11 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__11; -x_12 = l_List_foldr___at_Lean_Linter_unusedVariables_isInConstantOrAxiom___spec__1(x_9, x_10, x_11); +x_11 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__11; +x_12 = l_List_foldr___at_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___spec__1(x_9, x_10, x_11); return x_12; } } } } -LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___boxed), 1, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___boxed), 1, 0); return x_2; } } -LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isInConstantOrAxiom___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; uint8_t x_5; lean_object* x_6; x_4 = lean_unbox(x_2); lean_dec(x_2); -x_5 = l_List_foldr___at_Lean_Linter_unusedVariables_isInConstantOrAxiom___spec__1(x_1, x_4, x_3); +x_5 = l_List_foldr___at_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___spec__1(x_1, x_4, x_3); lean_dec(x_3); x_6 = lean_box(x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___boxed(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg(x_1); +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg(x_1); x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInConstantOrAxiom___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Linter_unusedVariables_isInConstantOrAxiom(x_1); +x_2 = l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom(x_1); lean_dec(x_1); return x_2; } @@ -5771,55 +5813,1320 @@ return x_10; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__23(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +static lean_object* _init_l_panic___at_Lean_Linter_unusedVariables___spec__27___closed__1() { _start: { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Command_instMonadCommandElabM; +x_3 = l_instInhabited___rarg(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Linter_unusedVariables___spec__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = l_panic___at_Lean_Linter_unusedVariables___spec__27___closed__1; +x_6 = lean_panic_fn(x_5, x_1); +x_7 = lean_apply_3(x_6, x_2, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Linter_unusedVariables___spec__28(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_8; lean_object* x_9; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; +} +else +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_4); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_4, 0); +x_12 = lean_ctor_get(x_4, 1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_13 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26(x_1, x_2, x_3, x_11, x_5, x_6, x_7); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l_List_mapM___at_Lean_Linter_unusedVariables___spec__28(x_1, x_2, x_3, x_12, x_5, x_6, x_15); +if (lean_obj_tag(x_16) == 0) +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_16, 0); +lean_ctor_set(x_4, 1, x_18); +lean_ctor_set(x_4, 0, x_14); +lean_ctor_set(x_16, 0, x_4); +return x_16; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_16, 0); +x_20 = lean_ctor_get(x_16, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_16); +lean_ctor_set(x_4, 1, x_19); +lean_ctor_set(x_4, 0, x_14); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_4); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} +} +else +{ +uint8_t x_22; +lean_dec(x_14); +lean_free_object(x_4); +x_22 = !lean_is_exclusive(x_16); +if (x_22 == 0) +{ +return x_16; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_16, 0); +x_24 = lean_ctor_get(x_16, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_16); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; +} +} +} +else +{ +uint8_t x_26; +lean_free_object(x_4); +lean_dec(x_12); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_13); +if (x_26 == 0) +{ +return x_13; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_13, 0); +x_28 = lean_ctor_get(x_13, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_13); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_4, 0); +x_31 = lean_ctor_get(x_4, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_4); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_32 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26(x_1, x_2, x_3, x_30, x_5, x_6, x_7); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = l_List_mapM___at_Lean_Linter_unusedVariables___spec__28(x_1, x_2, x_3, x_31, x_5, x_6, x_34); +if (lean_obj_tag(x_35) == 0) +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +if (lean_is_exclusive(x_35)) { + lean_ctor_release(x_35, 0); + lean_ctor_release(x_35, 1); + x_38 = x_35; +} else { + lean_dec_ref(x_35); + x_38 = lean_box(0); +} +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_33); +lean_ctor_set(x_39, 1, x_36); +if (lean_is_scalar(x_38)) { + x_40 = lean_alloc_ctor(0, 2, 0); +} else { + x_40 = x_38; +} +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_37); +return x_40; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_dec(x_33); +x_41 = lean_ctor_get(x_35, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_35, 1); +lean_inc(x_42); +if (lean_is_exclusive(x_35)) { + lean_ctor_release(x_35, 0); + lean_ctor_release(x_35, 1); + x_43 = x_35; +} else { + lean_dec_ref(x_35); + x_43 = lean_box(0); +} +if (lean_is_scalar(x_43)) { + x_44 = lean_alloc_ctor(1, 2, 0); +} else { + x_44 = x_43; +} +lean_ctor_set(x_44, 0, x_41); +lean_ctor_set(x_44, 1, x_42); +return x_44; +} +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +lean_dec(x_31); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_45 = lean_ctor_get(x_32, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_32, 1); +lean_inc(x_46); +if (lean_is_exclusive(x_32)) { + lean_ctor_release(x_32, 0); + lean_ctor_release(x_32, 1); + x_47 = x_32; +} else { + lean_dec_ref(x_32); + x_47 = lean_box(0); +} +if (lean_is_scalar(x_47)) { + x_48 = lean_alloc_ctor(1, 2, 0); +} else { + x_48 = x_47; +} +lean_ctor_set(x_48, 0, x_45); +lean_ctor_set(x_48, 1, x_46); +return x_48; +} +} +} +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Lean.Server.InfoUtils", 21); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Lean.Elab.InfoTree.visitM.go", 28); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("unexpected context-free info tree node", 38); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__1; +x_2 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__2; +x_3 = lean_unsigned_to_nat(39u); +x_4 = lean_unsigned_to_nat(21u); +x_5 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +switch (lean_obj_tag(x_4)) { +case 0: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_4, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_4, 1); +lean_inc(x_9); +lean_dec(x_4); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_8); +x_3 = x_10; +x_4 = x_9; +goto _start; +} +case 1: +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_12 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__4; +x_13 = l_panic___at_Lean_Linter_unusedVariables___spec__27(x_12, x_5, x_6, x_7); +return x_13; +} +default: +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_7); +return x_15; +} +} +} +else +{ +switch (lean_obj_tag(x_4)) { +case 0: +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_3); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_3, 0); +lean_dec(x_17); +x_18 = lean_ctor_get(x_4, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_4, 1); +lean_inc(x_19); +lean_dec(x_4); +lean_ctor_set(x_3, 0, x_18); +x_4 = x_19; +goto _start; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_3); +x_21 = lean_ctor_get(x_4, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_4, 1); +lean_inc(x_22); +lean_dec(x_4); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_21); +x_3 = x_23; +x_4 = x_22; +goto _start; +} +} +case 1: +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_3); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_26 = lean_ctor_get(x_3, 0); +x_27 = lean_ctor_get(x_4, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_4, 1); +lean_inc(x_28); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +x_29 = lean_apply_6(x_1, x_26, x_27, x_28, x_5, x_6, x_7); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +lean_inc(x_26); +x_31 = l_Lean_Elab_Info_updateContext_x3f(x_3, x_27); +lean_inc(x_28); +x_32 = l_Std_PersistentArray_toList___rarg(x_28); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_33 = l_List_mapM___at_Lean_Linter_unusedVariables___spec__28(x_1, x_2, x_31, x_32, x_5, x_6, x_30); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_apply_7(x_2, x_26, x_27, x_28, x_34, x_5, x_6, x_35); +if (lean_obj_tag(x_36) == 0) +{ +uint8_t x_37; +x_37 = !lean_is_exclusive(x_36); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_36, 0); +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_36, 0, x_39); +return x_36; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_40 = lean_ctor_get(x_36, 0); +x_41 = lean_ctor_get(x_36, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_36); +x_42 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_42, 0, x_40); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_41); +return x_43; +} +} +else +{ +uint8_t x_44; +x_44 = !lean_is_exclusive(x_36); +if (x_44 == 0) +{ +return x_36; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_36, 0); +x_46 = lean_ctor_get(x_36, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_36); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; +} +} +} +else +{ +uint8_t x_48; +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_48 = !lean_is_exclusive(x_33); +if (x_48 == 0) +{ +return x_33; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_33, 0); +x_50 = lean_ctor_get(x_33, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_33); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} +} +} +else +{ +uint8_t x_52; +lean_dec(x_28); +lean_dec(x_27); +lean_free_object(x_3); +lean_dec(x_26); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_52 = !lean_is_exclusive(x_29); +if (x_52 == 0) +{ +return x_29; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_29, 0); +x_54 = lean_ctor_get(x_29, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_29); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; +} +} +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_56 = lean_ctor_get(x_3, 0); +lean_inc(x_56); +lean_dec(x_3); +x_57 = lean_ctor_get(x_4, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_4, 1); +lean_inc(x_58); +lean_dec(x_4); +lean_inc(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +x_59 = lean_apply_6(x_1, x_56, x_57, x_58, x_5, x_6, x_7); +if (lean_obj_tag(x_59) == 0) +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_60 = lean_ctor_get(x_59, 1); +lean_inc(x_60); +lean_dec(x_59); +lean_inc(x_56); +x_61 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_61, 0, x_56); +x_62 = l_Lean_Elab_Info_updateContext_x3f(x_61, x_57); +lean_inc(x_58); +x_63 = l_Std_PersistentArray_toList___rarg(x_58); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_64 = l_List_mapM___at_Lean_Linter_unusedVariables___spec__28(x_1, x_2, x_62, x_63, x_5, x_6, x_60); +if (lean_obj_tag(x_64) == 0) +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_64, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_64, 1); +lean_inc(x_66); +lean_dec(x_64); +x_67 = lean_apply_7(x_2, x_56, x_57, x_58, x_65, x_5, x_6, x_66); +if (lean_obj_tag(x_67) == 0) +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +if (lean_is_exclusive(x_67)) { + lean_ctor_release(x_67, 0); + lean_ctor_release(x_67, 1); + x_70 = x_67; +} else { + lean_dec_ref(x_67); + x_70 = lean_box(0); +} +x_71 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_71, 0, x_68); +if (lean_is_scalar(x_70)) { + x_72 = lean_alloc_ctor(0, 2, 0); +} else { + x_72 = x_70; +} +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_69); +return x_72; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_73 = lean_ctor_get(x_67, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_67, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_67)) { + lean_ctor_release(x_67, 0); + lean_ctor_release(x_67, 1); + x_75 = x_67; +} else { + lean_dec_ref(x_67); + x_75 = lean_box(0); +} +if (lean_is_scalar(x_75)) { + x_76 = lean_alloc_ctor(1, 2, 0); +} else { + x_76 = x_75; +} +lean_ctor_set(x_76, 0, x_73); +lean_ctor_set(x_76, 1, x_74); +return x_76; +} +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_56); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_77 = lean_ctor_get(x_64, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_64, 1); +lean_inc(x_78); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_79 = x_64; +} else { + lean_dec_ref(x_64); + x_79 = lean_box(0); +} +if (lean_is_scalar(x_79)) { + x_80 = lean_alloc_ctor(1, 2, 0); +} else { + x_80 = x_79; +} +lean_ctor_set(x_80, 0, x_77); +lean_ctor_set(x_80, 1, x_78); +return x_80; +} +} +else +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +lean_dec(x_58); +lean_dec(x_57); +lean_dec(x_56); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_81 = lean_ctor_get(x_59, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_59, 1); +lean_inc(x_82); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_83 = x_59; +} else { + lean_dec_ref(x_59); + x_83 = lean_box(0); +} +if (lean_is_scalar(x_83)) { + x_84 = lean_alloc_ctor(1, 2, 0); +} else { + x_84 = x_83; +} +lean_ctor_set(x_84, 0, x_81); +lean_ctor_set(x_84, 1, x_82); +return x_84; +} +} +} +default: +{ +lean_object* x_85; lean_object* x_86; +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_85 = lean_box(0); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_7); +return x_86; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_box(0); +x_8 = l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26(x_1, x_2, x_7, x_3, x_4, x_5, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25___rarg), 6, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_6); +return x_8; +} +} +static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(x_6); +x_11 = l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; uint8_t x_13; uint8_t x_14; +x_12 = lean_ctor_get(x_1, 0); +x_13 = 0; +x_14 = l_Lean_Elab_Info_contains(x_4, x_12, x_13); +if (x_14 == 0) +{ +lean_object* x_15; +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_9); +return x_15; +} +else +{ +lean_object* x_16; uint8_t x_17; uint8_t x_18; +x_16 = lean_ctor_get(x_1, 1); +x_17 = 1; +x_18 = l_Lean_Elab_Info_contains(x_4, x_16, x_17); +if (x_18 == 0) +{ +lean_object* x_19; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_2); +lean_ctor_set(x_19, 1, x_9); +return x_19; +} +else +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 3) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_20 = lean_ctor_get(x_4, 0); +x_21 = lean_box(0); +lean_inc(x_20); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_22); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_9); +return x_24; +} +else +{ +lean_object* x_25; lean_object* x_26; +x_25 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___closed__1; +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_9); +return x_26; +} +} +} +} +else +{ +lean_dec(x_2); +if (lean_obj_tag(x_4) == 3) +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_11); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_28 = lean_ctor_get(x_11, 0); +x_29 = lean_ctor_get(x_11, 1); +lean_dec(x_29); +x_30 = lean_ctor_get(x_4, 0); +lean_inc(x_30); +lean_ctor_set(x_11, 1, x_28); +lean_ctor_set(x_11, 0, x_30); +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_11); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_9); +return x_32; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_33 = lean_ctor_get(x_11, 0); +lean_inc(x_33); +lean_dec(x_11); +x_34 = lean_ctor_get(x_4, 0); +lean_inc(x_34); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_33); +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_35); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_9); +return x_37; +} +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_11, 0); +lean_inc(x_38); +lean_dec(x_11); +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_38); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_9); +return x_40; +} +} +} +} +static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__1___boxed), 6, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_box(0); +x_7 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___boxed), 9, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_6); +x_8 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___closed__1; +x_9 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25___rarg(x_8, x_7, x_2, x_3, x_4, x_5); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_unusedVariables___spec__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24(x_1, x_2, x_3, x_4, x_5); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +if (lean_obj_tag(x_7) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_6, 0); +lean_dec(x_9); +x_10 = lean_box(0); +lean_ctor_set(x_6, 0, x_10); +return x_6; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_6, 1); +lean_inc(x_11); +lean_dec(x_6); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +} +else +{ +lean_object* x_14; +x_14 = lean_ctor_get(x_7, 0); +lean_inc(x_14); +lean_dec(x_7); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_6); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_6, 0); +lean_dec(x_16); +x_17 = lean_box(0); +lean_ctor_set(x_6, 0, x_17); +return x_6; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_6, 1); +lean_inc(x_18); +lean_dec(x_6); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; +} +} +else +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_6); +if (x_21 == 0) +{ +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_6, 0); +lean_dec(x_22); +x_23 = !lean_is_exclusive(x_14); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_14, 0); +x_25 = l_List_reverse___rarg(x_24); +lean_ctor_set(x_14, 0, x_25); +lean_ctor_set(x_6, 0, x_14); +return x_6; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_14, 0); +lean_inc(x_26); +lean_dec(x_14); +x_27 = l_List_reverse___rarg(x_26); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_6, 0, x_28); +return x_6; +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_29 = lean_ctor_get(x_6, 1); +lean_inc(x_29); +lean_dec(x_6); +x_30 = lean_ctor_get(x_14, 0); +lean_inc(x_30); +if (lean_is_exclusive(x_14)) { + lean_ctor_release(x_14, 0); + x_31 = x_14; +} else { + lean_dec_ref(x_14); + x_31 = lean_box(0); +} +x_32 = l_List_reverse___rarg(x_30); +if (lean_is_scalar(x_31)) { + x_33 = lean_alloc_ctor(1, 1, 0); +} else { + x_33 = x_31; +} +lean_ctor_set(x_33, 0, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_29); +return x_34; +} +} +} +} +else +{ +uint8_t x_35; +x_35 = !lean_is_exclusive(x_6); +if (x_35 == 0) +{ +return x_6; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_6, 0); +x_37 = lean_ctor_get(x_6, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_6); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} +} +} +} +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_eq(x_4, x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_7 = lean_array_uget(x_3, x_4); +lean_inc(x_2); +lean_inc(x_1); +x_8 = lean_apply_2(x_7, x_1, x_2); +x_9 = lean_unbox(x_8); +lean_dec(x_8); +if (x_9 == 0) +{ +size_t x_10; size_t x_11; +x_10 = 1; +x_11 = lean_usize_add(x_4, x_10); +x_4 = x_11; +goto _start; +} +else +{ +uint8_t x_13; +lean_dec(x_2); +lean_dec(x_1); +x_13 = 1; +return x_13; +} +} +else +{ +uint8_t x_14; +lean_dec(x_2); +lean_dec(x_1); +x_14 = 0; +return x_14; +} +} +} +LEAN_EXPORT uint8_t l_List_foldr___at_Lean_Linter_unusedVariables___spec__30(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_dec(x_1); +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_4, 1); +lean_inc(x_6); +lean_dec(x_4); +lean_inc(x_1); +x_7 = l_List_foldr___at_Lean_Linter_unusedVariables___spec__30(x_1, x_2, x_3, x_6); +x_8 = lean_ctor_get(x_5, 2); +lean_inc(x_8); +lean_dec(x_5); +lean_inc(x_1); +x_9 = l_Lean_Linter_findSyntaxStack_x3f(x_8, x_1); +if (lean_obj_tag(x_9) == 0) +{ +lean_dec(x_1); +return x_7; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +lean_dec(x_9); +x_11 = lean_array_get_size(x_2); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_nat_dec_lt(x_12, x_11); +if (x_13 == 0) +{ +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_1); +return x_7; +} +else +{ +uint8_t x_14; +x_14 = lean_nat_dec_le(x_11, x_11); +if (x_14 == 0) +{ +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_1); +return x_7; +} +else +{ +size_t x_15; size_t x_16; uint8_t x_17; +x_15 = 0; +x_16 = lean_usize_of_nat(x_11); +lean_dec(x_11); +x_17 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29(x_1, x_10, x_2, x_15, x_16); +if (x_17 == 0) +{ +return x_7; +} +else +{ +uint8_t x_18; +x_18 = 1; +return x_18; +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__31(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_6; -x_6 = lean_array_uget(x_2, x_3); -if (lean_obj_tag(x_6) == 0) +uint8_t x_10; +x_10 = lean_usize_dec_eq(x_5, x_6); +if (x_10 == 0) { -uint8_t x_7; -lean_dec(x_6); -x_7 = 1; -return x_7; +lean_object* x_11; lean_object* x_12; +x_11 = lean_array_uget(x_4, x_5); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_12 = l_Lean_Linter_collectMacroExpansions_x3f___at_Lean_Linter_unusedVariables___spec__23(x_2, x_11, x_7, x_8, x_9); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; size_t x_15; size_t x_16; +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = 1; +x_16 = lean_usize_add(x_5, x_15); +x_5 = x_16; +x_9 = x_14; +goto _start; } else { -lean_object* x_8; uint8_t x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -x_9 = l_Std_HashSetImp_contains___at_Lean_Meta_getNondepPropHyps___spec__12(x_1, x_8); +uint8_t x_18; +x_18 = !lean_is_exclusive(x_12); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; uint8_t x_23; +x_19 = lean_ctor_get(x_12, 1); +x_20 = lean_ctor_get(x_12, 0); +lean_dec(x_20); +x_21 = lean_ctor_get(x_13, 0); +lean_inc(x_21); +lean_dec(x_13); +x_22 = 0; +lean_inc(x_1); +x_23 = l_List_foldr___at_Lean_Linter_unusedVariables___spec__30(x_1, x_3, x_22, x_21); +if (x_23 == 0) +{ +size_t x_24; size_t x_25; +lean_free_object(x_12); +x_24 = 1; +x_25 = lean_usize_add(x_5, x_24); +x_5 = x_25; +x_9 = x_19; +goto _start; +} +else +{ +uint8_t x_27; lean_object* x_28; lean_dec(x_8); -if (x_9 == 0) +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_27 = 1; +x_28 = lean_box(x_27); +lean_ctor_set(x_12, 0, x_28); +return x_12; +} +} +else { -size_t x_10; size_t x_11; -x_10 = 1; -x_11 = lean_usize_add(x_3, x_10); -x_3 = x_11; +lean_object* x_29; lean_object* x_30; uint8_t x_31; uint8_t x_32; +x_29 = lean_ctor_get(x_12, 1); +lean_inc(x_29); +lean_dec(x_12); +x_30 = lean_ctor_get(x_13, 0); +lean_inc(x_30); +lean_dec(x_13); +x_31 = 0; +lean_inc(x_1); +x_32 = l_List_foldr___at_Lean_Linter_unusedVariables___spec__30(x_1, x_3, x_31, x_30); +if (x_32 == 0) +{ +size_t x_33; size_t x_34; +x_33 = 1; +x_34 = lean_usize_add(x_5, x_33); +x_5 = x_34; +x_9 = x_29; goto _start; } else { -uint8_t x_13; -x_13 = 1; -return x_13; +uint8_t x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_36 = 1; +x_37 = lean_box(x_36); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_29); +return x_38; +} } } } else { -uint8_t x_14; -x_14 = 0; -return x_14; +uint8_t x_39; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_39 = !lean_is_exclusive(x_12); +if (x_39 == 0) +{ +return x_12; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_12, 0); +x_41 = lean_ctor_get(x_12, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_12); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; +} +} +} +else +{ +uint8_t x_43; lean_object* x_44; lean_object* x_45; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +x_43 = 0; +x_44 = lean_box(x_43); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_9); +return x_45; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__32(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5) { _start: { uint8_t x_6; @@ -5860,7 +7167,57 @@ return x_14; } } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__1() { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__33(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; +x_6 = lean_array_uget(x_2, x_3); +if (lean_obj_tag(x_6) == 0) +{ +size_t x_7; size_t x_8; +lean_dec(x_6); +x_7 = 1; +x_8 = lean_usize_add(x_3, x_7); +x_3 = x_8; +goto _start; +} +else +{ +lean_object* x_10; uint8_t x_11; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = l_Std_HashSetImp_contains___at_Lean_Meta_getNondepPropHyps___spec__12(x_1, x_10); +lean_dec(x_10); +if (x_11 == 0) +{ +size_t x_12; size_t x_13; +x_12 = 1; +x_13 = lean_usize_add(x_3, x_12); +x_3 = x_13; +goto _start; +} +else +{ +uint8_t x_15; +x_15 = 1; +return x_15; +} +} +} +else +{ +uint8_t x_16; +x_16 = 0; +return x_16; +} +} +} +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -5868,7 +7225,7 @@ x_1 = lean_mk_string_from_bytes("unused variable `", 17); return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__2() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__2() { _start: { lean_object* x_1; @@ -5876,7 +7233,7 @@ x_1 = lean_mk_string_from_bytes("`", 1); return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -5886,148 +7243,165 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_11; uint8_t x_28; -x_28 = l_Array_isEmpty___rarg(x_3); -if (x_28 == 0) +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; uint8_t x_14; lean_object* x_15; uint8_t x_16; +x_7 = l_Lean_LocalDecl_userName(x_1); +x_8 = 1; +x_9 = l_Lean_Name_toString(x_7, x_8); +x_10 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__1; +x_11 = lean_string_append(x_10, x_9); +lean_dec(x_9); +x_12 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__2; +x_13 = lean_string_append(x_11, x_12); +x_14 = 1; +x_15 = l_Lean_Linter_publishMessage(x_13, x_2, x_14, x_4, x_5, x_6); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) { -lean_object* x_29; lean_object* x_30; -lean_dec(x_8); -x_29 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_10); -return x_30; +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +lean_dec(x_17); +x_18 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; +lean_ctor_set(x_15, 0, x_18); +return x_15; } else { -uint8_t x_31; -x_31 = l_Std_HashSetImp_contains___at_Lean_Meta_getNondepPropHyps___spec__12(x_4, x_5); -if (x_31 == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_15, 1); +lean_inc(x_19); +lean_dec(x_15); +x_20 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = lean_ctor_get(x_6, 1); -x_33 = lean_array_get_size(x_32); -x_34 = lean_unsigned_to_nat(0u); -x_35 = lean_nat_dec_lt(x_34, x_33); -if (x_35 == 0) +uint8_t x_13; lean_object* x_14; +if (x_3 == 0) { -lean_object* x_36; -lean_dec(x_33); -x_36 = lean_box(0); -x_11 = x_36; -goto block_27; +uint8_t x_20; +lean_dec(x_6); +lean_dec(x_5); +x_20 = 0; +x_13 = x_20; +x_14 = x_12; +goto block_19; } else { -uint8_t x_37; -x_37 = lean_nat_dec_le(x_33, x_33); -if (x_37 == 0) +if (x_4 == 0) { -lean_object* x_38; -lean_dec(x_33); -x_38 = lean_box(0); -x_11 = x_38; -goto block_27; +uint8_t x_21; +lean_dec(x_6); +lean_dec(x_5); +x_21 = 0; +x_13 = x_21; +x_14 = x_12; +goto block_19; } else { -size_t x_39; size_t x_40; uint8_t x_41; -x_39 = 0; -x_40 = lean_usize_of_nat(x_33); -lean_dec(x_33); -x_41 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__23(x_4, x_32, x_39, x_40); -if (x_41 == 0) +size_t x_22; size_t x_23; lean_object* x_24; +x_22 = 0; +x_23 = lean_usize_of_nat(x_5); +lean_dec(x_5); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_2); +x_24 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__31(x_6, x_2, x_7, x_8, x_22, x_23, x_10, x_11, x_12); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_42; -x_42 = lean_box(0); -x_11 = x_42; -goto block_27; +lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_unbox(x_25); +lean_dec(x_25); +x_13 = x_27; +x_14 = x_26; +goto block_19; } else { -lean_object* x_43; lean_object* x_44; -lean_dec(x_8); -x_43 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_10); -return x_44; -} -} -} +uint8_t x_28; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_2); +x_28 = !lean_is_exclusive(x_24); +if (x_28 == 0) +{ +return x_24; } else { -lean_object* x_45; lean_object* x_46; -lean_dec(x_8); -x_45 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_10); -return x_46; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_24, 0); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_24); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } -block_27: +} +} +block_19: { -lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; uint8_t x_21; -lean_dec(x_11); -x_12 = l_Lean_LocalDecl_userName(x_1); -x_13 = 1; -x_14 = l_Lean_Name_toString(x_12, x_13); -x_15 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__1; -x_16 = lean_string_append(x_15, x_14); -lean_dec(x_14); -x_17 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__2; -x_18 = lean_string_append(x_16, x_17); -x_19 = 1; -x_20 = l_Lean_Linter_publishMessage(x_18, x_2, x_19, x_8, x_9, x_10); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +if (x_13 == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_20, 0); -lean_dec(x_22); -x_23 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; -lean_ctor_set(x_20, 0, x_23); -return x_20; +lean_object* x_15; lean_object* x_16; +x_15 = lean_box(0); +x_16 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1(x_1, x_2, x_15, x_10, x_11, x_14); +lean_dec(x_11); +lean_dec(x_2); +return x_16; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_20, 1); -lean_inc(x_24); -lean_dec(x_20); -x_25 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -return x_26; +lean_object* x_17; lean_object* x_18; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_2); +x_17 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_14); +return x_18; } } } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__3(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { lean_object* x_14; lean_dec(x_10); -lean_inc(x_2); -x_14 = l_Lean_Linter_findSyntaxStack_x3f(x_1, x_2); +lean_inc(x_6); +x_14 = l_Lean_Linter_findSyntaxStack_x3f(x_8, x_6); if (lean_obj_tag(x_14) == 0) { lean_object* x_15; lean_object* x_16; +lean_dec(x_12); lean_dec(x_11); -lean_dec(x_8); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); -x_15 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; +x_15 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_15); lean_ctor_set(x_16, 1, x_13); @@ -6047,15 +7421,10 @@ if (x_20 == 0) lean_object* x_21; lean_object* x_22; lean_dec(x_18); lean_dec(x_17); -lean_dec(x_2); x_21 = lean_box(0); -x_22 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1(x_3, x_4, x_5, x_6, x_7, x_8, x_21, x_11, x_12, x_13); -lean_dec(x_8); +x_22 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_9, x_7, x_21, x_11, x_12, x_13); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +lean_dec(x_9); return x_22; } else @@ -6067,15 +7436,10 @@ if (x_23 == 0) lean_object* x_24; lean_object* x_25; lean_dec(x_18); lean_dec(x_17); -lean_dec(x_2); x_24 = lean_box(0); -x_25 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1(x_3, x_4, x_5, x_6, x_7, x_8, x_24, x_11, x_12, x_13); -lean_dec(x_8); +x_25 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_9, x_7, x_24, x_11, x_12, x_13); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +lean_dec(x_9); return x_25; } else @@ -6084,31 +7448,28 @@ size_t x_26; size_t x_27; uint8_t x_28; x_26 = 0; x_27 = lean_usize_of_nat(x_18); lean_dec(x_18); -x_28 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__24(x_2, x_17, x_9, x_26, x_27); +lean_inc(x_6); +x_28 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__32(x_6, x_17, x_9, x_26, x_27); if (x_28 == 0) { lean_object* x_29; lean_object* x_30; x_29 = lean_box(0); -x_30 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1(x_3, x_4, x_5, x_6, x_7, x_8, x_29, x_11, x_12, x_13); -lean_dec(x_8); +x_30 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_9, x_7, x_29, x_11, x_12, x_13); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +lean_dec(x_9); return x_30; } else { lean_object* x_31; lean_object* x_32; +lean_dec(x_12); lean_dec(x_11); -lean_dec(x_8); +lean_dec(x_9); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_31 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; +lean_dec(x_2); +x_31 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; x_32 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_32, 0, x_31); lean_ctor_set(x_32, 1, x_13); @@ -6119,7 +7480,7 @@ return x_32; } } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__1() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -6128,7 +7489,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__2() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__2() { _start: { lean_object* x_1; @@ -6136,17 +7497,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isPatternVar___bo return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__3() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__1; -x_2 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__2; +x_1 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__1; +x_2 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__2; x_3 = lean_array_push(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { uint8_t x_15; @@ -6156,26 +7517,22 @@ lean_dec(x_9); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__3; +x_16 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__3; x_17 = l_Array_append___rarg(x_10, x_16); x_18 = lean_box(0); -x_19 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_17, x_18, x_12, x_13, x_14); -lean_dec(x_13); -lean_dec(x_17); +x_19 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_17, x_18, x_12, x_13, x_14); return x_19; } else { lean_object* x_20; lean_object* x_21; x_20 = lean_box(0); -x_21 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_10, x_20, x_12, x_13, x_14); -lean_dec(x_13); -lean_dec(x_10); +x_21 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_10, x_20, x_12, x_13, x_14); return x_21; } } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__1() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -6184,7 +7541,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__2() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__2() { _start: { lean_object* x_1; @@ -6192,7 +7549,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_matchesUnusedPatt return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__3() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__3() { _start: { lean_object* x_1; @@ -6200,7 +7557,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isVariable___boxe return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__4() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__4() { _start: { lean_object* x_1; @@ -6208,7 +7565,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInStructure___b return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__5() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__5() { _start: { lean_object* x_1; @@ -6216,7 +7573,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInInductive___b return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__6() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__6() { _start: { lean_object* x_1; @@ -6224,15 +7581,15 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInCtorOrStructB return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__7() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__7() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__8() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__8() { _start: { lean_object* x_1; @@ -6240,7 +7597,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInDefWithForeig return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__9() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__9() { _start: { lean_object* x_1; @@ -6248,7 +7605,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInDepArrow___bo return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__10() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__10() { _start: { lean_object* x_1; lean_object* x_2; @@ -6257,7 +7614,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__11() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__11() { _start: { lean_object* x_1; @@ -6265,17 +7622,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInLetDeclaratio return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__12() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__10; -x_2 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__11; +x_1 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__10; +x_2 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__11; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__13() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__13() { _start: { lean_object* x_1; @@ -6283,17 +7640,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInDeclarationSi return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__14() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__12; -x_2 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__13; +x_1 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__12; +x_2 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__13; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__15() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__15() { _start: { lean_object* x_1; @@ -6301,263 +7658,470 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isInFun___boxed), return x_1; } } -static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__16() { +static lean_object* _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__14; -x_2 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__15; +x_1 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__14; +x_2 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__15; x_3 = lean_array_push(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_dec(x_11); x_15 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables_isTopLevelDecl___boxed), 3, 1); lean_closure_set(x_15, 0, x_1); -x_16 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__1; +x_16 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__1; x_17 = lean_array_push(x_16, x_15); -x_18 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__2; +x_18 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__2; x_19 = lean_array_push(x_17, x_18); -x_20 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__3; +x_20 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__3; x_21 = lean_array_push(x_19, x_20); -x_22 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__4; +x_22 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__4; x_23 = lean_array_push(x_21, x_22); -x_24 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__5; +x_24 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__5; x_25 = lean_array_push(x_23, x_24); -x_26 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__6; +x_26 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__6; x_27 = lean_array_push(x_25, x_26); -x_28 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__7; +x_28 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__7; x_29 = lean_array_push(x_27, x_28); -x_30 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__8; +x_30 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__8; x_31 = lean_array_push(x_29, x_30); -x_32 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__9; +x_32 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__9; x_33 = lean_array_push(x_31, x_32); x_34 = l_Lean_Linter_getLinterUnusedVariablesFunArgs(x_10); if (x_34 == 0) { lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_35 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__16; +x_35 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__16; x_36 = l_Array_append___rarg(x_33, x_35); x_37 = lean_box(0); -x_38 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_36, x_37, x_12, x_13, x_14); +x_38 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_36, x_37, x_12, x_13, x_14); +lean_dec(x_2); return x_38; } else { lean_object* x_39; lean_object* x_40; x_39 = lean_box(0); -x_40 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_33, x_39, x_12, x_13, x_14); +x_40 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_33, x_39, x_12, x_13, x_14); +lean_dec(x_2); return x_40; } } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -lean_dec(x_10); -x_14 = lean_ctor_get(x_1, 4); -lean_inc(x_14); -x_15 = lean_ctor_get(x_14, 3); +lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_dec(x_11); +x_15 = lean_ctor_get(x_1, 4); lean_inc(x_15); -lean_dec(x_14); -x_16 = l_Lean_Linter_getLinterUnusedVariables(x_15); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; +lean_dec(x_1); +x_16 = lean_ctor_get(x_15, 3); +lean_inc(x_16); lean_dec(x_15); +x_17 = l_Lean_Linter_getLinterUnusedVariables(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_16); +lean_dec(x_13); lean_dec(x_12); -lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_17 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_13); -return x_18; +x_18 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_14); +return x_19; } else { +lean_object* x_20; lean_object* x_21; +x_20 = lean_box(0); +x_21 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_16, x_20, x_12, x_13, x_14); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +_start: +{ +uint8_t x_18; +lean_dec(x_14); +x_18 = l_Array_isEmpty___rarg(x_11); +lean_dec(x_11); +if (x_18 == 0) +{ lean_object* x_19; lean_object* x_20; -x_19 = lean_box(0); -x_20 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_1, x_15, x_19, x_11, x_12, x_13); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_19 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_17); return x_20; } +else +{ +uint8_t x_21; +x_21 = l_Std_HashSetImp_contains___at_Lean_Meta_getNondepPropHyps___spec__12(x_12, x_13); +lean_dec(x_13); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_22 = lean_ctor_get(x_1, 1); +lean_inc(x_22); +x_23 = lean_array_get_size(x_22); +x_24 = lean_unsigned_to_nat(0u); +x_25 = lean_nat_dec_lt(x_24, x_23); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_12); +x_26 = lean_box(0); +x_27 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_26, x_15, x_16, x_17); +return x_27; } +else +{ +uint8_t x_28; +x_28 = lean_nat_dec_le(x_23, x_23); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_12); +x_29 = lean_box(0); +x_30 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_29, x_15, x_16, x_17); +return x_30; } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -if (lean_obj_tag(x_5) == 0) +size_t x_31; size_t x_32; uint8_t x_33; +x_31 = 0; +x_32 = lean_usize_of_nat(x_23); +lean_dec(x_23); +x_33 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__33(x_12, x_22, x_31, x_32); +lean_dec(x_22); +lean_dec(x_12); +if (x_33 == 0) { -lean_object* x_10; +lean_object* x_34; lean_object* x_35; +x_34 = lean_box(0); +x_35 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_34, x_15, x_16, x_17); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_6); -lean_ctor_set(x_10, 1, x_9); -return x_10; +x_36 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_17); +return x_37; +} +} +} } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -lean_dec(x_6); -x_11 = lean_ctor_get(x_5, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -if (lean_obj_tag(x_13) == 0) +lean_object* x_38; lean_object* x_39; +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_38 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3; +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_17); +return x_39; +} +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_14; lean_object* x_15; +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_14; lean_dec(x_12); lean_dec(x_11); -x_14 = lean_ctor_get(x_5, 1); -lean_inc(x_14); -lean_dec(x_5); -x_15 = lean_box(0); -x_5 = x_14; -x_6 = x_15; -goto _start; +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_10); +lean_ctor_set(x_14, 1, x_13); +return x_14; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; -x_17 = lean_ctor_get(x_5, 1); +lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_dec(x_10); +x_15 = lean_ctor_get(x_9, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); -lean_dec(x_5); -x_18 = lean_ctor_get(x_11, 0); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_16); +lean_dec(x_15); +x_18 = lean_ctor_get(x_9, 1); lean_inc(x_18); -lean_dec(x_11); -x_19 = lean_ctor_get(x_12, 1); -lean_inc(x_19); -lean_dec(x_12); -x_20 = lean_ctor_get(x_13, 0); -lean_inc(x_20); -lean_dec(x_13); -x_21 = lean_ctor_get(x_20, 3); +lean_dec(x_9); +x_19 = lean_box(0); +x_9 = x_18; +x_10 = x_19; +goto _start; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; +x_21 = lean_ctor_get(x_9, 1); lean_inc(x_21); -x_22 = l_Lean_Linter_unusedVariables_skipDeclIdIfPresent(x_21); -x_23 = 0; +lean_dec(x_9); +x_22 = lean_ctor_get(x_15, 0); lean_inc(x_22); -x_24 = l_Lean_Syntax_getRange_x3f(x_22, x_23); -if (lean_obj_tag(x_24) == 0) +lean_dec(x_15); +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); +lean_dec(x_16); +x_24 = lean_ctor_get(x_17, 0); +lean_inc(x_24); +lean_dec(x_17); +x_25 = lean_ctor_get(x_24, 3); +lean_inc(x_25); +x_26 = l_Lean_Linter_unusedVariables_skipDeclIdIfPresent(x_25); +x_27 = 0; +lean_inc(x_26); +x_28 = l_Lean_Syntax_getRange_x3f(x_26, x_27); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_25; +lean_object* x_29; +lean_dec(x_26); +lean_dec(x_24); +lean_dec(x_23); lean_dec(x_22); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -x_25 = lean_box(0); -x_5 = x_17; -x_6 = x_25; +x_29 = lean_box(0); +x_9 = x_21; +x_10 = x_29; goto _start; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_24, 0); -lean_inc(x_27); -lean_dec(x_24); -x_28 = lean_ctor_get(x_20, 5); -lean_inc(x_28); -x_29 = l_Lean_Elab_Info_lctx(x_28); +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_28, 0); +lean_inc(x_31); lean_dec(x_28); -lean_inc(x_18); -x_30 = lean_local_ctx_find(x_29, x_18); -if (lean_obj_tag(x_30) == 0) +x_32 = lean_ctor_get(x_24, 5); +lean_inc(x_32); +x_33 = l_Lean_Elab_Info_lctx(x_32); +lean_dec(x_32); +lean_inc(x_22); +x_34 = lean_local_ctx_find(x_33, x_22); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_31; -lean_dec(x_27); +lean_object* x_35; +lean_dec(x_31); +lean_dec(x_26); +lean_dec(x_24); +lean_dec(x_23); lean_dec(x_22); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -x_31 = lean_box(0); -x_5 = x_17; -x_6 = x_31; +x_35 = lean_box(0); +x_9 = x_21; +x_10 = x_35; +goto _start; +} +else +{ +lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_37 = lean_ctor_get(x_34, 0); +lean_inc(x_37); +lean_dec(x_34); +x_38 = lean_ctor_get(x_31, 0); +lean_inc(x_38); +x_39 = l_String_Range_contains(x_2, x_38, x_27); +lean_dec(x_38); +if (x_39 == 0) +{ +lean_object* x_40; +lean_dec(x_37); +lean_dec(x_31); +lean_dec(x_26); +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_22); +x_40 = lean_box(0); +x_9 = x_21; +x_10 = x_40; goto _start; } else { -lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_33 = lean_ctor_get(x_30, 0); -lean_inc(x_33); -lean_dec(x_30); -x_34 = lean_ctor_get(x_27, 0); -lean_inc(x_34); -x_35 = l_String_Range_contains(x_2, x_34, x_23); -lean_dec(x_34); -if (x_35 == 0) +lean_object* x_42; uint8_t x_43; +x_42 = l_Lean_LocalDecl_userName(x_37); +x_43 = l_Lean_Name_hasMacroScopes(x_42); +lean_dec(x_42); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +x_44 = lean_box(0); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_8); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_4); +lean_inc(x_6); +x_45 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__7(x_24, x_6, x_37, x_31, x_5, x_7, x_4, x_26, x_3, x_1, x_23, x_8, x_22, x_44, x_11, x_12, x_13); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +if (lean_obj_tag(x_46) == 0) +{ +uint8_t x_47; +lean_dec(x_21); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_47 = !lean_is_exclusive(x_45); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_45, 0); +lean_dec(x_48); +x_49 = lean_ctor_get(x_46, 0); +lean_inc(x_49); +lean_dec(x_46); +lean_ctor_set(x_45, 0, x_49); +return x_45; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_45, 1); +lean_inc(x_50); +lean_dec(x_45); +x_51 = lean_ctor_get(x_46, 0); +lean_inc(x_51); +lean_dec(x_46); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_50); +return x_52; +} +} +else { -lean_object* x_36; -lean_dec(x_33); -lean_dec(x_27); -lean_dec(x_22); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -x_36 = lean_box(0); -x_5 = x_17; -x_6 = x_36; +lean_object* x_53; lean_object* x_54; +x_53 = lean_ctor_get(x_45, 1); +lean_inc(x_53); +lean_dec(x_45); +x_54 = lean_ctor_get(x_46, 0); +lean_inc(x_54); +lean_dec(x_46); +x_9 = x_21; +x_10 = x_54; +x_13 = x_53; goto _start; } +} else { -lean_object* x_38; uint8_t x_39; -x_38 = l_Lean_LocalDecl_userName(x_33); -x_39 = l_Lean_Name_hasMacroScopes(x_38); -lean_dec(x_38); -if (x_39 == 0) +uint8_t x_56; +lean_dec(x_21); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_56 = !lean_is_exclusive(x_45); +if (x_56 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_40 = lean_box(0); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_4); -lean_inc(x_1); -lean_inc(x_3); -x_41 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__5(x_20, x_3, x_1, x_22, x_33, x_27, x_19, x_4, x_18, x_40, x_7, x_8, x_9); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = lean_ctor_get(x_42, 0); -lean_inc(x_44); -lean_dec(x_42); -x_5 = x_17; -x_6 = x_44; -x_9 = x_43; -goto _start; +return x_45; } else { -lean_object* x_46; -lean_dec(x_33); -lean_dec(x_27); +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_45, 0); +x_58 = lean_ctor_get(x_45, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_45); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; +} +} +} +else +{ +lean_object* x_60; +lean_dec(x_37); +lean_dec(x_31); +lean_dec(x_26); +lean_dec(x_24); +lean_dec(x_23); lean_dec(x_22); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -x_46 = lean_box(0); -x_5 = x_17; -x_6 = x_46; +x_60 = lean_box(0); +x_9 = x_21; +x_10 = x_60; goto _start; } } @@ -6567,7 +8131,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; @@ -6634,7 +8198,7 @@ return x_17; } } } -static lean_object* _init_l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__1() { +static lean_object* _init_l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -6643,15 +8207,15 @@ x_2 = l_Std_mkHashMapImp___rarg(x_1); return x_2; } } -static lean_object* _init_l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__2() { +static lean_object* _init_l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___lambda__1___boxed), 5, 0); +x_1 = lean_alloc_closure((void*)(l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___lambda__1___boxed), 5, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_2) == 0) @@ -6672,14 +8236,14 @@ lean_inc(x_7); x_8 = lean_ctor_get(x_2, 2); lean_inc(x_8); lean_dec(x_2); -x_9 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__1; +x_9 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__1; x_10 = lean_st_mk_ref(x_9, x_5); x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); -x_13 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__2; +x_13 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__2; lean_inc(x_4); lean_inc(x_3); x_14 = l_Lean_ForEachExpr_visit___at_Lean_Linter_unusedVariables___spec__19(x_13, x_7, x_11, x_1, x_3, x_4, x_12); @@ -6733,7 +8297,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__27(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__36(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { uint8_t x_8; @@ -6744,7 +8308,7 @@ lean_object* x_9; lean_object* x_10; x_9 = lean_array_uget(x_1, x_2); lean_inc(x_6); lean_inc(x_5); -x_10 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26(x_4, x_9, x_5, x_6, x_7); +x_10 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35(x_4, x_9, x_5, x_6, x_7); if (lean_obj_tag(x_10) == 0) { lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; @@ -6797,7 +8361,7 @@ return x_20; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_dec(x_1); @@ -6823,15 +8387,15 @@ return x_3; } } } -static lean_object* _init_l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___closed__1() { +static lean_object* _init_l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___lambda__1), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___lambda__1), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -6842,7 +8406,7 @@ size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; x_6 = 1; x_7 = lean_usize_sub(x_2, x_6); x_8 = lean_array_uget(x_1, x_7); -x_9 = l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___closed__1; +x_9 = l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___closed__1; x_10 = l_Lean_Elab_InfoTree_foldInfo___rarg(x_9, x_4, x_8); x_2 = x_7; x_4 = x_10; @@ -6854,7 +8418,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__38(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -6979,12 +8543,12 @@ x_2 = l_Std_mkHashSetImp___rarg(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -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; +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; uint8_t x_24; lean_object* x_25; x_11 = 1; -x_12 = l_Lean_Server_findModuleRefs(x_1, x_2, x_11); +x_12 = l_Lean_Server_findModuleRefs(x_1, x_2, x_11, x_11); x_13 = lean_unsigned_to_nat(0u); x_14 = l_Std_mkHashMapImp___rarg(x_13); x_15 = lean_unsigned_to_nat(8u); @@ -7004,132 +8568,161 @@ lean_inc(x_22); x_23 = lean_ctor_get(x_20, 1); lean_inc(x_23); lean_dec(x_20); -if (x_5 == 0) +x_24 = lean_nat_dec_le(x_3, x_3); +if (x_6 == 0) { -lean_object* x_52; -x_52 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__1; -x_24 = x_52; -goto block_51; +lean_object* x_57; +x_57 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__1; +x_25 = x_57; +goto block_56; } else { -size_t x_53; size_t x_54; lean_object* x_55; lean_object* x_56; -x_53 = lean_usize_of_nat(x_6); -x_54 = 0; -x_55 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__1; -x_56 = l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28(x_2, x_53, x_54, x_55); -x_24 = x_56; -goto block_51; +size_t x_58; size_t x_59; lean_object* x_60; lean_object* x_61; +x_58 = lean_usize_of_nat(x_3); +x_59 = 0; +x_60 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__1; +x_61 = l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37(x_2, x_58, x_59, x_60); +x_25 = x_61; +goto block_56; } -block_51: +block_56: { -lean_object* x_25; lean_object* x_26; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_35 = lean_ctor_get(x_24, 1); -lean_inc(x_35); -lean_dec(x_24); -x_36 = lean_array_get_size(x_35); -x_37 = lean_nat_dec_lt(x_13, x_36); -if (x_37 == 0) +lean_object* x_26; lean_object* x_27; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_40 = lean_ctor_get(x_25, 1); +lean_inc(x_40); +lean_dec(x_25); +x_41 = lean_array_get_size(x_40); +x_42 = lean_nat_dec_lt(x_13, x_41); +if (x_42 == 0) { -lean_object* x_38; -lean_dec(x_36); -lean_dec(x_35); -x_38 = l_Lean_Linter_unusedVariables___lambda__1___closed__1; -x_25 = x_38; -x_26 = x_21; -goto block_34; +lean_object* x_43; +lean_dec(x_41); +lean_dec(x_40); +x_43 = l_Lean_Linter_unusedVariables___lambda__1___closed__1; +x_26 = x_43; +x_27 = x_21; +goto block_39; } else { -uint8_t x_39; -x_39 = lean_nat_dec_le(x_36, x_36); -if (x_39 == 0) +uint8_t x_44; +x_44 = lean_nat_dec_le(x_41, x_41); +if (x_44 == 0) { -lean_object* x_40; -lean_dec(x_36); -lean_dec(x_35); -x_40 = l_Lean_Linter_unusedVariables___lambda__1___closed__1; -x_25 = x_40; -x_26 = x_21; -goto block_34; +lean_object* x_45; +lean_dec(x_41); +lean_dec(x_40); +x_45 = l_Lean_Linter_unusedVariables___lambda__1___closed__1; +x_26 = x_45; +x_27 = x_21; +goto block_39; } else { -size_t x_41; size_t x_42; lean_object* x_43; lean_object* x_44; -x_41 = 0; -x_42 = lean_usize_of_nat(x_36); -lean_dec(x_36); -x_43 = l_Lean_Linter_unusedVariables___lambda__1___closed__1; +size_t x_46; size_t x_47; lean_object* x_48; lean_object* x_49; +x_46 = 0; +x_47 = lean_usize_of_nat(x_41); +lean_dec(x_41); +x_48 = l_Lean_Linter_unusedVariables___lambda__1___closed__1; lean_inc(x_9); lean_inc(x_8); -x_44 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__27(x_35, x_41, x_42, x_43, x_8, x_9, x_21); -lean_dec(x_35); -if (lean_obj_tag(x_44) == 0) +x_49 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__36(x_40, x_46, x_47, x_48, x_8, x_9, x_21); +lean_dec(x_40); +if (lean_obj_tag(x_49) == 0) { -lean_object* x_45; lean_object* x_46; -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_25 = x_45; -x_26 = x_46; -goto block_34; +lean_object* x_50; lean_object* x_51; +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_26 = x_50; +x_27 = x_51; +goto block_39; } else { -uint8_t x_47; +uint8_t x_52; lean_dec(x_23); lean_dec(x_22); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_4); lean_dec(x_3); -x_47 = !lean_is_exclusive(x_44); -if (x_47 == 0) +lean_dec(x_2); +x_52 = !lean_is_exclusive(x_49); +if (x_52 == 0) { -return x_44; +return x_49; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_44, 0); -x_49 = lean_ctor_get(x_44, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_44); -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_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_49, 0); +x_54 = lean_ctor_get(x_49, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_49); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; +} +} } } +block_39: +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = l_Std_HashMap_toList___at_Lean_Linter_unusedVariables___spec__20(x_23); +x_29 = lean_box(0); +x_30 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34(x_4, x_5, x_2, x_3, x_6, x_22, x_24, x_26, x_28, x_29, x_8, x_9, x_27); +if (lean_obj_tag(x_30) == 0) +{ +uint8_t x_31; +x_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) +{ +lean_object* x_32; +x_32 = lean_ctor_get(x_30, 0); +lean_dec(x_32); +lean_ctor_set(x_30, 0, x_29); +return x_30; +} +else +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +lean_dec(x_30); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_29); +lean_ctor_set(x_34, 1, x_33); +return x_34; } } -block_34: +else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_27 = l_Std_HashMap_toList___at_Lean_Linter_unusedVariables___spec__20(x_23); -x_28 = lean_box(0); -x_29 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25(x_3, x_4, x_22, x_25, x_27, x_28, x_8, x_9, x_26); -x_30 = !lean_is_exclusive(x_29); -if (x_30 == 0) +uint8_t x_35; +x_35 = !lean_is_exclusive(x_30); +if (x_35 == 0) { -lean_object* x_31; -x_31 = lean_ctor_get(x_29, 0); -lean_dec(x_31); -lean_ctor_set(x_29, 0, x_28); -return x_29; +return x_30; } else { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_29, 1); -lean_inc(x_32); -lean_dec(x_29); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_28); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_30, 0); +x_37 = lean_ctor_get(x_30, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_30); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} } } } @@ -7207,7 +8800,7 @@ else size_t x_30; size_t x_31; lean_object* x_32; x_30 = 0; x_31 = lean_usize_of_nat(x_19); -x_32 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29(x_17, x_30, x_31, x_3, x_4, x_13); +x_32 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__38(x_17, x_30, x_31, x_3, x_4, x_13); if (lean_obj_tag(x_32) == 0) { lean_object* x_33; lean_object* x_34; uint8_t x_35; @@ -7261,10 +8854,8 @@ if (x_22 == 0) lean_object* x_24; lean_object* x_25; lean_dec(x_14); x_24 = lean_box(0); -x_25 = l_Lean_Linter_unusedVariables___lambda__1(x_18, x_17, x_1, x_10, x_21, x_19, x_24, x_3, x_4, x_23); -lean_dec(x_19); +x_25 = l_Lean_Linter_unusedVariables___lambda__1(x_18, x_17, x_19, x_1, x_10, x_21, x_24, x_3, x_4, x_23); lean_dec(x_10); -lean_dec(x_17); return x_25; } else @@ -7453,22 +9044,43 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25___boxed(lean_object* x_1) { _start: { -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); +lean_object* x_2; +x_2 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_unusedVariables___spec__25(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__23(x_1, x_2, x_5, x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { size_t x_6; size_t x_7; uint8_t x_8; lean_object* x_9; @@ -7476,58 +9088,198 @@ x_6 = lean_unbox_usize(x_4); lean_dec(x_4); x_7 = lean_unbox_usize(x_5); lean_dec(x_5); -x_8 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__24(x_1, x_2, x_3, x_6, x_7); +x_8 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29(x_1, x_2, x_3, x_6, x_7); lean_dec(x_3); x_9 = lean_box(x_8); return x_9; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_List_foldr___at_Lean_Linter_unusedVariables___spec__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_11; -x_11 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_7); +uint8_t x_5; uint8_t x_6; lean_object* x_7; +x_5 = lean_unbox(x_3); +lean_dec(x_3); +x_6 = l_List_foldr___at_Lean_Linter_unusedVariables___spec__30(x_1, x_2, x_5, x_4); +lean_dec(x_2); +x_7 = lean_box(x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__31___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +size_t x_10; size_t x_11; lean_object* x_12; +x_10 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_11 = lean_unbox_usize(x_6); lean_dec(x_6); +x_12 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__31(x_1, x_2, x_3, x_4, x_10, x_11, x_7, x_8, x_9); +lean_dec(x_4); +lean_dec(x_3); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__32___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; uint8_t x_8; lean_object* x_9; +x_6 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_7 = lean_unbox_usize(x_5); lean_dec(x_5); +x_8 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__32(x_1, x_2, x_3, x_6, x_7); +lean_dec(x_3); +x_9 = lean_box(x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__33___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = lean_unbox_usize(x_4); lean_dec(x_4); +x_7 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__33(x_1, x_2, x_5, x_6); +lean_dec(x_2); +lean_dec(x_1); +x_8 = lean_box(x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_11; +return x_7; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_14; -x_14 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_12); +uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_13 = lean_unbox(x_3); +lean_dec(x_3); +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__2(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_9); -return x_14; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_1); +return x_15; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_10; -x_10 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +uint8_t x_14; uint8_t x_15; lean_object* x_16; +x_14 = lean_unbox(x_3); +lean_dec(x_3); +x_15 = lean_unbox(x_4); +lean_dec(x_4); +x_16 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__3(x_1, x_2, x_14, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_15 = lean_unbox(x_3); +lean_dec(x_3); +x_16 = lean_unbox(x_4); +lean_dec(x_4); +x_17 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4(x_1, x_2, x_15, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_1); +return x_17; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_15 = lean_unbox(x_4); +lean_dec(x_4); +x_16 = lean_unbox(x_5); +lean_dec(x_5); +x_17 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5(x_1, x_2, x_3, x_15, x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_17; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_15 = lean_unbox(x_5); +lean_dec(x_5); +x_16 = lean_unbox(x_6); +lean_dec(x_6); +x_17 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__6(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_17; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__7___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +uint8_t x_18; uint8_t x_19; lean_object* x_20; +x_18 = lean_unbox(x_5); +lean_dec(x_5); +x_19 = lean_unbox(x_6); +lean_dec(x_6); +x_20 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__7(x_1, x_2, x_3, x_4, x_18, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +return x_20; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; uint8_t x_15; lean_object* x_16; +x_14 = lean_unbox(x_5); +lean_dec(x_5); +x_15 = lean_unbox(x_7); +lean_dec(x_7); +x_16 = l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34(x_1, x_2, x_3, x_4, x_14, x_6, x_15, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_2); -return x_10; +return x_16; } } -LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___lambda__1(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___lambda__1(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__36___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -7535,12 +9287,12 @@ x_8 = lean_unbox_usize(x_2); lean_dec(x_2); x_9 = lean_unbox_usize(x_3); lean_dec(x_3); -x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__27(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__36(x_1, x_8, x_9, x_4, x_5, x_6, x_7); lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -7548,12 +9300,12 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__38___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; size_t x_8; lean_object* x_9; @@ -7561,7 +9313,7 @@ x_7 = lean_unbox_usize(x_2); lean_dec(x_2); x_8 = lean_unbox_usize(x_3); lean_dec(x_3); -x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__29(x_1, x_7, x_8, x_4, x_5, x_6); +x_9 = l_Array_anyMUnsafe_any___at_Lean_Linter_unusedVariables___spec__38(x_1, x_7, x_8, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); @@ -7572,17 +9324,15 @@ LEAN_EXPORT lean_object* l_Lean_Linter_unusedVariables___lambda__1___boxed(lean_ _start: { uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_5); -lean_dec(x_5); -x_12 = l_Lean_Linter_unusedVariables___lambda__1(x_1, x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_7); +x_11 = lean_unbox(x_6); lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_2); +x_12 = l_Lean_Linter_unusedVariables___lambda__1(x_1, x_2, x_3, x_4, x_5, x_11, x_7, x_8, x_9, x_10); +lean_dec(x_7); +lean_dec(x_5); return x_12; } } -static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429____closed__1() { +static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577____closed__1() { _start: { lean_object* x_1; @@ -7590,11 +9340,11 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Linter_unusedVariables), 4, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429____closed__1; +x_2 = l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577____closed__1; x_3 = l_Lean_Elab_Command_addLinter(x_2, x_1); return x_3; } @@ -7793,28 +9543,28 @@ l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__11 = _init lean_mark_persistent(l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__11); l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__12 = _init_l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__12(); lean_mark_persistent(l_Lean_Linter_unusedVariables_isInCtorOrStructBinder___rarg___closed__12); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__1 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__1(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__1); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__2 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__2(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__2); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__3 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__3(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__3); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__4 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__4(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__4); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__5 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__5(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__5); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__6 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__6(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__6); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__7 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__7(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__7); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__8 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__8(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__8); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__9 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__9(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__9); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__10 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__10(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__10); -l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__11 = _init_l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__11(); -lean_mark_persistent(l_Lean_Linter_unusedVariables_isInConstantOrAxiom___rarg___closed__11); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__1 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__1(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__1); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__2 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__2(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__2); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__3 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__3(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__3); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__4 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__4(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__4); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__5 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__5(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__5); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__6 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__6(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__6); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__7 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__7(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__7); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__8 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__8(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__8); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__9 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__9(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__9); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__10 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__10(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__10); +l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__11 = _init_l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__11(); +lean_mark_persistent(l_Lean_Linter_unusedVariables_isInOpaqueOrAxiom___rarg___closed__11); l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__1 = _init_l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__1); l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__2 = _init_l_Lean_Linter_unusedVariables_isInDefWithForeignDefinition___rarg___lambda__1___closed__2(); @@ -7921,61 +9671,75 @@ l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1___closed__6 lean_mark_persistent(l_List_foldr___at_Lean_Linter_unusedVariables_isPatternVar___spec__1___closed__6); l_Std_PersistentHashMap_foldlMAux___at_Lean_Linter_unusedVariables___spec__17___closed__1 = _init_l_Std_PersistentHashMap_foldlMAux___at_Lean_Linter_unusedVariables___spec__17___closed__1(); lean_mark_persistent(l_Std_PersistentHashMap_foldlMAux___at_Lean_Linter_unusedVariables___spec__17___closed__1); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__1 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__1(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__1); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__2 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__2(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__2); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__1___closed__3); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__1 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__1(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__1); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__2 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__2(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__2); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__3 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__3(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__3___closed__3); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__1 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__1(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__1); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__2 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__2(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__2); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__3 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__3(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__3); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__4 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__4(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__4); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__5 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__5(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__5); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__6 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__6(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__6); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__7 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__7(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__7); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__8 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__8(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__8); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__9 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__9(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__9); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__10 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__10(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__10); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__11 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__11(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__11); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__12 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__12(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__12); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__13 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__13(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__13); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__14 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__14(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__14); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__15 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__15(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__15); -l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__16 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__16(); -lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__25___lambda__4___closed__16); -l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__1 = _init_l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__1(); -lean_mark_persistent(l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__1); -l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__2 = _init_l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__2(); -lean_mark_persistent(l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__26___closed__2); -l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___closed__1 = _init_l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___closed__1(); -lean_mark_persistent(l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__28___closed__1); +l_panic___at_Lean_Linter_unusedVariables___spec__27___closed__1 = _init_l_panic___at_Lean_Linter_unusedVariables___spec__27___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Linter_unusedVariables___spec__27___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__1 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__1(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__1); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__2 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__2(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__2); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__3 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__3(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__3); +l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__4 = _init_l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__4(); +lean_mark_persistent(l_Lean_Elab_InfoTree_visitM_go___at_Lean_Linter_unusedVariables___spec__26___closed__4); +l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___lambda__2___closed__1); +l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___closed__1(); +lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___at_Lean_Linter_unusedVariables___spec__24___closed__1); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__1 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__1(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__1); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__2 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__2(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__2); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__1___closed__3); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__1 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__1(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__1); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__2 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__2(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__2); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__3 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__3(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__4___closed__3); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__1 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__1(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__1); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__2 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__2(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__2); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__3 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__3(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__3); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__4 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__4(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__4); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__5 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__5(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__5); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__6 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__6(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__6); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__7 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__7(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__7); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__8 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__8(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__8); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__9 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__9(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__9); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__10 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__10(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__10); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__11 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__11(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__11); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__12 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__12(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__12); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__13 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__13(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__13); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__14 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__14(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__14); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__15 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__15(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__15); +l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__16 = _init_l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__16(); +lean_mark_persistent(l_List_forIn_loop___at_Lean_Linter_unusedVariables___spec__34___lambda__5___closed__16); +l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__1 = _init_l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__1(); +lean_mark_persistent(l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__1); +l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__2 = _init_l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__2(); +lean_mark_persistent(l_Std_AssocList_foldlM___at_Lean_Linter_unusedVariables___spec__35___closed__2); +l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___closed__1 = _init_l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___closed__1(); +lean_mark_persistent(l_Array_foldrMUnsafe_fold___at_Lean_Linter_unusedVariables___spec__37___closed__1); l_Lean_Linter_unusedVariables___lambda__1___closed__1 = _init_l_Lean_Linter_unusedVariables___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Linter_unusedVariables___lambda__1___closed__1); -l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429____closed__1(); -lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429____closed__1); -res = l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2429_(lean_io_mk_world()); +l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577____closed__1 = _init_l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577____closed__1(); +lean_mark_persistent(l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577____closed__1); +res = l_Lean_Linter_initFn____x40_Lean_Linter_Basic___hyg_2577_(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/Linter/Util.c b/stage0/stdlib/Lean/Linter/Util.c index 1c876d892a6c..54ecbc37f3b1 100644 --- a/stage0/stdlib/Lean/Linter/Util.c +++ b/stage0/stdlib/Lean/Linter/Util.c @@ -13,6 +13,7 @@ #ifdef __cplusplus extern "C" { #endif +lean_object* l_List_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Util___hyg_6_(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__3; @@ -20,6 +21,7 @@ static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Util___hyg_6____clos uint8_t l___private_Lean_Server_InfoUtils_0__String_beqRange____x40_Lean_Server_InfoUtils___hyg_75_(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); +lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_range(lean_object*); lean_object* l_List_zipWith___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_stackMatches___boxed(lean_object*, lean_object*); @@ -30,7 +32,9 @@ LEAN_EXPORT uint8_t l_Lean_Linter_stackMatches___lambda__1(lean_object*, lean_ob LEAN_EXPORT lean_object* l_Lean_Linter_publishMessage___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_stackMatches(lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Util___hyg_6____closed__3; +static lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1; static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Util___hyg_6____closed__5; +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__2; lean_object* l_Lean_Option_register___at_Lean_initFn____x40_Lean_PrettyPrinter_Delaborator_Options___hyg_6____spec__1(lean_object*, lean_object*, lean_object*); uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); @@ -38,25 +42,36 @@ lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_linter_all; static lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__1; lean_object* l_Lean_Elab_mkMessageCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +uint8_t l_Lean_Elab_Info_contains(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Util___hyg_6____closed__7; LEAN_EXPORT lean_object* l_Lean_Linter_publishMessage(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_findSyntaxStack_x3f(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object*); LEAN_EXPORT uint8_t l_Lean_Linter_getLinterAll(lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Util___hyg_6____closed__1; uint8_t l_List_foldr___at_List_and___spec__1(uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___rarg___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__1___boxed(lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getNumArgs(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_stackMatches___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); lean_object* l_Lean_Syntax_getKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_findSyntaxStack_x3f_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Linter_getLinterAll___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KVMap_findCore(lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); @@ -64,7 +79,10 @@ LEAN_EXPORT lean_object* l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2(lean_o lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_findSyntaxStack_x3f_go___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_Util___hyg_6____closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object*); static lean_object* _init_l_Lean_Linter_initFn____x40_Lean_Linter_Util___hyg_6____closed__1() { _start: { @@ -324,6 +342,475 @@ lean_dec(x_2); return x_8; } } +LEAN_EXPORT lean_object* l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_2; +x_2 = lean_box(0); +return x_2; +} +else +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +lean_dec(x_1); +x_1 = x_4; +goto _start; +} +else +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_1); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 1); +x_8 = lean_ctor_get(x_1, 0); +lean_dec(x_8); +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(x_7); +lean_ctor_set(x_1, 1, x_10); +lean_ctor_set(x_1, 0, x_9); +return x_1; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(x_11); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +} +} +} +} +LEAN_EXPORT lean_object* l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_2; +x_2 = lean_box(0); +return x_2; +} +else +{ +lean_object* x_3; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +lean_dec(x_1); +x_1 = x_4; +goto _start; +} +else +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_1); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 1); +x_8 = lean_ctor_get(x_1, 0); +lean_dec(x_8); +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(x_7); +lean_ctor_set(x_1, 1, x_10); +lean_ctor_set(x_1, 0, x_9); +return x_1; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); +lean_dec(x_3); +x_13 = l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(x_11); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_box(0); +x_7 = l_Lean_Elab_InfoTree_visitM_go___rarg(x_1, x_3, x_4, x_6, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_box(0); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +} +static lean_object* _init_l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; +x_8 = l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__1(x_7); +x_9 = l_List_filterMap___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__2(x_8); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; uint8_t x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_1, 0); +x_11 = 0; +x_12 = l_Lean_Elab_Info_contains(x_5, x_10, x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_2, 0); +lean_inc(x_13); +lean_dec(x_2); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_apply_2(x_14, lean_box(0), x_3); +return x_15; +} +else +{ +lean_object* x_16; uint8_t x_17; uint8_t x_18; +x_16 = lean_ctor_get(x_1, 1); +x_17 = 1; +x_18 = l_Lean_Elab_Info_contains(x_5, x_16, x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_2, 0); +lean_inc(x_19); +lean_dec(x_2); +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_apply_2(x_20, lean_box(0), x_3); +return x_21; +} +else +{ +lean_dec(x_3); +if (lean_obj_tag(x_5) == 3) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_22 = lean_ctor_get(x_5, 0); +x_23 = lean_ctor_get(x_2, 0); +lean_inc(x_23); +lean_dec(x_2); +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +x_25 = lean_box(0); +lean_inc(x_22); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_22); +lean_ctor_set(x_26, 1, x_25); +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_26); +x_28 = lean_apply_2(x_24, lean_box(0), x_27); +return x_28; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_2, 0); +lean_inc(x_29); +lean_dec(x_2); +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +x_31 = l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1; +x_32 = lean_apply_2(x_30, lean_box(0), x_31); +return x_32; +} +} +} +} +else +{ +lean_dec(x_3); +if (lean_obj_tag(x_5) == 3) +{ +uint8_t x_33; +x_33 = !lean_is_exclusive(x_9); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_34 = lean_ctor_get(x_9, 0); +x_35 = lean_ctor_get(x_9, 1); +lean_dec(x_35); +x_36 = lean_ctor_get(x_5, 0); +x_37 = lean_ctor_get(x_2, 0); +lean_inc(x_37); +lean_dec(x_2); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +lean_inc(x_36); +lean_ctor_set(x_9, 1, x_34); +lean_ctor_set(x_9, 0, x_36); +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_9); +x_40 = lean_apply_2(x_38, lean_box(0), x_39); +return x_40; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_41 = lean_ctor_get(x_9, 0); +lean_inc(x_41); +lean_dec(x_9); +x_42 = lean_ctor_get(x_5, 0); +x_43 = lean_ctor_get(x_2, 0); +lean_inc(x_43); +lean_dec(x_2); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +lean_inc(x_42); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_42); +lean_ctor_set(x_45, 1, x_41); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = lean_apply_2(x_44, lean_box(0), x_46); +return x_47; +} +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_48 = lean_ctor_get(x_9, 0); +lean_inc(x_48); +lean_dec(x_9); +x_49 = lean_ctor_get(x_2, 0); +lean_inc(x_49); +lean_dec(x_2); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +lean_dec(x_49); +x_51 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_51, 0, x_48); +x_52 = lean_apply_2(x_50, lean_box(0), x_51); +return x_52; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_box(0); +lean_inc(x_1); +x_5 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed), 4, 1); +lean_closure_set(x_5, 0, x_1); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___boxed), 7, 3); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_1); +lean_closure_set(x_6, 2, x_4); +x_7 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(x_1, x_4, x_5, x_6, x_3); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Elab_InfoTree_visitM___at_Lean_Linter_collectMacroExpansions_x3f_go___spec__3___rarg(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_2); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_dec(x_1); +x_4 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_box(0); +x_6 = lean_apply_2(x_4, lean_box(0), x_5); +return x_6; +} +else +{ +lean_object* x_7; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(0); +x_11 = lean_apply_2(x_9, lean_box(0), x_10); +return x_11; +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_7); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_7, 0); +x_14 = lean_ctor_get(x_1, 0); +lean_inc(x_14); +lean_dec(x_1); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = l_List_reverse___rarg(x_13); +lean_ctor_set(x_7, 0, x_16); +x_17 = lean_apply_2(x_15, lean_box(0), x_7); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_7, 0); +lean_inc(x_18); +lean_dec(x_7); +x_19 = lean_ctor_get(x_1, 0); +lean_inc(x_19); +lean_dec(x_1); +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = l_List_reverse___rarg(x_18); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = lean_apply_2(x_20, lean_box(0), x_22); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +lean_inc(x_1); +x_5 = l_Lean_Linter_collectMacroExpansions_x3f_go___rarg(x_1, x_2, x_3); +x_6 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f___rarg___lambda__1), 2, 1); +lean_closure_set(x_6, 0, x_1); +x_7 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_5, x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Linter_collectMacroExpansions_x3f(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Linter_collectMacroExpansions_x3f___rarg), 3, 0); +return x_2; +} +} LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Linter_findSyntaxStack_x3f_go___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { @@ -812,7 +1299,9 @@ if (lean_io_result_is_error(res)) return res; l_Lean_Linter_linter_all = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Linter_linter_all); lean_dec_ref(res); -}l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__1 = _init_l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__1(); +}l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1 = _init_l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Linter_collectMacroExpansions_x3f_go___rarg___lambda__2___closed__1); +l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__1 = _init_l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__1); l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__2 = _init_l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__2(); lean_mark_persistent(l_Lean_Linter_findSyntaxStack_x3f_go___lambda__2___closed__2); diff --git a/stage0/stdlib/Lean/LocalContext.c b/stage0/stdlib/Lean/LocalContext.c index 2ca25a6e00bc..d56069b5c1c6 100644 --- a/stage0/stdlib/Lean/LocalContext.c +++ b/stage0/stdlib/Lean/LocalContext.c @@ -88,6 +88,7 @@ static lean_object* l_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___spec__ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_LocalContext_foldr___spec__21___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_LocalContext_foldr___spec__12___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_findSomeRevM_x3f___at_Lean_LocalContext_findFromUserName_x3f___spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_LocalContext_foldlM___at_Lean_LocalContext_size___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_LocalContext_instForInLocalContextLocalDecl___spec__1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* lean_local_ctx_erase(lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); @@ -133,6 +134,7 @@ LEAN_EXPORT lean_object* l_Lean_LocalContext_findDeclM_x3f___rarg(lean_object*, lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_LocalContext_foldr___spec__22(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_LocalContext_instForInLocalContextLocalDecl___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_LocalContext_allM___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___spec__1___closed__6; LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_LocalContext_instForInLocalContextLocalDecl___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -164,7 +166,9 @@ lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_foldrM___at_Lean_LocalContext_foldr___spec__1(lean_object*); static lean_object* l_Lean_LocalContext_mkEmpty___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_LocalContext_instForInLocalContextLocalDecl___spec__5___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_LocalContext_size___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentHashMap_containsAtAux___at_Lean_LocalContext_contains___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_LocalContext_size(lean_object*); static lean_object* l_Lean_LocalDecl_value___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_getFVarIds___spec__5(lean_object*, size_t, size_t, lean_object*); uint8_t lean_expr_has_loose_bvar(lean_object*, lean_object*); @@ -237,6 +241,7 @@ static size_t l_Std_PersistentHashMap_insertAux___at_Lean_LocalContext_mkLocalDe LEAN_EXPORT lean_object* l_Lean_LocalContext_findDeclM_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_foldl___spec__14___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at_Lean_LocalContext_allM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_LocalContext_size___spec__3(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_LocalContext_any___spec__4(lean_object*, lean_object*, size_t, size_t); lean_object* lean_name_append_index_after(lean_object*, lean_object*); static size_t l_Std_PersistentHashMap_insertAux___at_Lean_LocalContext_mkLocalDecl___spec__2___closed__1; @@ -349,6 +354,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_LocalContext_foldr_ lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); static lean_object* l_Lean_instInhabitedLocalDecl___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_LocalContext_anyM___spec__4___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_PersistentArray_foldlM___at_Lean_LocalContext_size___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_findDeclRev_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalDecl_index(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_LocalContext_instForInLocalContextLocalDecl___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); @@ -391,6 +397,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_LocalContext_instFor LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_LocalContext_anyM___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at_Lean_LocalContext_any___spec__2(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_LocalDecl_hasExprMVar(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_LocalContext_foldr___spec__24___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_LocalContext_get_x21___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at_Lean_LocalContext_anyM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t); @@ -432,6 +439,7 @@ static lean_object* l_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___spec__ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_LocalContext_foldr___spec__13___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l_Std_PersistentArray_findSomeMAux___at_Lean_LocalContext_findDecl_x3f___spec__3___rarg___closed__2; +LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlMAux___at_Lean_LocalContext_size___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_findSomeMAux___at_Lean_LocalContext_findDecl_x3f___spec__3___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instMonadLCtx___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at_Lean_LocalContext_mkLocalDecl___spec__1(lean_object*, lean_object*, lean_object*); @@ -479,6 +487,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_LocalContext_foldr_ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_LocalContext_anyM___spec__4(lean_object*); LEAN_EXPORT lean_object* lean_local_ctx_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_allM(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__5(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_anyM(lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalContext_mkForall(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_LocalDecl_binderInfoEx___boxed(lean_object*); @@ -494,6 +503,7 @@ LEAN_EXPORT lean_object* l_Lean_LocalContext_contains___boxed(lean_object*, lean LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_LocalContext_foldr___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_LocalContext_allM___spec__3___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_LocalContext_instForInLocalContextLocalDecl___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_LocalContext_allM___spec__5___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_pp_sanitizeNames; LEAN_EXPORT lean_object* l_Lean_LocalDecl_hasValue___boxed(lean_object*); @@ -8495,6 +8505,430 @@ lean_dec(x_2); return x_8; } } +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__5(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; +x_6 = lean_array_uget(x_1, x_2); +x_7 = l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlMAux___at_Lean_LocalContext_size___spec__4(x_6, x_4); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_2 = x_9; +x_4 = x_7; +goto _start; +} +else +{ +return x_4; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) +{ +lean_object* x_6; size_t x_7; size_t x_8; +x_6 = lean_array_uget(x_1, x_2); +x_7 = 1; +x_8 = lean_usize_add(x_2, x_7); +if (lean_obj_tag(x_6) == 0) +{ +x_2 = x_8; +goto _start; +} +else +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_6); +x_10 = lean_unsigned_to_nat(1u); +x_11 = lean_nat_add(x_4, x_10); +lean_dec(x_4); +x_2 = x_8; +x_4 = x_11; +goto _start; +} +} +else +{ +return x_4; +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlMAux___at_Lean_LocalContext_size___spec__4(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_dec(x_1); +x_4 = lean_array_get_size(x_3); +x_5 = lean_unsigned_to_nat(0u); +x_6 = lean_nat_dec_lt(x_5, x_4); +if (x_6 == 0) +{ +lean_dec(x_4); +lean_dec(x_3); +return x_2; +} +else +{ +uint8_t x_7; +x_7 = lean_nat_dec_le(x_4, x_4); +if (x_7 == 0) +{ +lean_dec(x_4); +lean_dec(x_3); +return x_2; +} +else +{ +size_t x_8; size_t x_9; lean_object* x_10; +x_8 = 0; +x_9 = lean_usize_of_nat(x_4); +lean_dec(x_4); +x_10 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__5(x_3, x_8, x_9, x_2); +lean_dec(x_3); +return x_10; +} +} +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_array_get_size(x_11); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_nat_dec_lt(x_13, x_12); +if (x_14 == 0) +{ +lean_dec(x_12); +lean_dec(x_11); +return x_2; +} +else +{ +uint8_t x_15; +x_15 = lean_nat_dec_le(x_12, x_12); +if (x_15 == 0) +{ +lean_dec(x_12); +lean_dec(x_11); +return x_2; +} +else +{ +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = 0; +x_17 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_18 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6(x_11, x_16, x_17, x_2); +lean_dec(x_11); +return x_18; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_LocalContext_size___spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_5; size_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_usize_shift_right(x_2, x_3); +x_7 = lean_usize_to_nat(x_6); +x_8 = l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_LocalContext_getFVarIds___spec__2___closed__1; +x_9 = lean_array_get(x_8, x_5, x_7); +x_10 = 1; +x_11 = lean_usize_shift_left(x_10, x_3); +x_12 = lean_usize_sub(x_11, x_10); +x_13 = lean_usize_land(x_2, x_12); +x_14 = 5; +x_15 = lean_usize_sub(x_3, x_14); +x_16 = l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_LocalContext_size___spec__3(x_9, x_13, x_15, x_4); +lean_dec(x_9); +x_17 = lean_unsigned_to_nat(1u); +x_18 = lean_nat_add(x_7, x_17); +lean_dec(x_7); +x_19 = lean_array_get_size(x_5); +x_20 = lean_nat_dec_lt(x_18, x_19); +if (x_20 == 0) +{ +lean_dec(x_19); +lean_dec(x_18); +return x_16; +} +else +{ +uint8_t x_21; +x_21 = lean_nat_dec_le(x_19, x_19); +if (x_21 == 0) +{ +lean_dec(x_19); +lean_dec(x_18); +return x_16; +} +else +{ +size_t x_22; size_t x_23; lean_object* x_24; +x_22 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_23 = lean_usize_of_nat(x_19); +lean_dec(x_19); +x_24 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__5(x_5, x_22, x_23, x_16); +return x_24; +} +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = lean_ctor_get(x_1, 0); +x_26 = lean_usize_to_nat(x_2); +x_27 = lean_array_get_size(x_25); +x_28 = lean_nat_dec_lt(x_26, x_27); +if (x_28 == 0) +{ +lean_dec(x_27); +lean_dec(x_26); +return x_4; +} +else +{ +uint8_t x_29; +x_29 = lean_nat_dec_le(x_27, x_27); +if (x_29 == 0) +{ +lean_dec(x_27); +lean_dec(x_26); +return x_4; +} +else +{ +size_t x_30; size_t x_31; lean_object* x_32; +x_30 = lean_usize_of_nat(x_26); +lean_dec(x_26); +x_31 = lean_usize_of_nat(x_27); +lean_dec(x_27); +x_32 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6(x_25, x_30, x_31, x_4); +return x_32; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_PersistentArray_foldlM___at_Lean_LocalContext_size___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_nat_dec_eq(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_ctor_get(x_1, 3); +lean_inc(x_6); +x_7 = lean_nat_dec_le(x_6, x_3); +if (x_7 == 0) +{ +lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +lean_dec(x_6); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +x_9 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_10 = lean_ctor_get_usize(x_1, 4); +x_11 = l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_LocalContext_size___spec__3(x_8, x_9, x_10, x_2); +lean_dec(x_8); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_array_get_size(x_12); +x_14 = lean_nat_dec_lt(x_4, x_13); +if (x_14 == 0) +{ +lean_dec(x_13); +lean_dec(x_12); +return x_11; +} +else +{ +uint8_t x_15; +x_15 = lean_nat_dec_le(x_13, x_13); +if (x_15 == 0) +{ +lean_dec(x_13); +lean_dec(x_12); +return x_11; +} +else +{ +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = 0; +x_17 = lean_usize_of_nat(x_13); +lean_dec(x_13); +x_18 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6(x_12, x_16, x_17, x_11); +lean_dec(x_12); +return x_18; +} +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +lean_dec(x_1); +x_20 = lean_nat_sub(x_3, x_6); +lean_dec(x_6); +lean_dec(x_3); +x_21 = lean_array_get_size(x_19); +x_22 = lean_nat_dec_lt(x_20, x_21); +if (x_22 == 0) +{ +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +return x_2; +} +else +{ +uint8_t x_23; +x_23 = lean_nat_dec_le(x_21, x_21); +if (x_23 == 0) +{ +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +return x_2; +} +else +{ +size_t x_24; size_t x_25; lean_object* x_26; +x_24 = lean_usize_of_nat(x_20); +lean_dec(x_20); +x_25 = lean_usize_of_nat(x_21); +lean_dec(x_21); +x_26 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6(x_19, x_24, x_25, x_2); +lean_dec(x_19); +return x_26; +} +} +} +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_dec(x_3); +x_27 = lean_ctor_get(x_1, 0); +lean_inc(x_27); +x_28 = l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlMAux___at_Lean_LocalContext_size___spec__4(x_27, x_2); +x_29 = lean_ctor_get(x_1, 1); +lean_inc(x_29); +lean_dec(x_1); +x_30 = lean_array_get_size(x_29); +x_31 = lean_nat_dec_lt(x_4, x_30); +if (x_31 == 0) +{ +lean_dec(x_30); +lean_dec(x_29); +return x_28; +} +else +{ +uint8_t x_32; +x_32 = lean_nat_dec_le(x_30, x_30); +if (x_32 == 0) +{ +lean_dec(x_30); +lean_dec(x_29); +return x_28; +} +else +{ +size_t x_33; size_t x_34; lean_object* x_35; +x_33 = 0; +x_34 = lean_usize_of_nat(x_30); +lean_dec(x_30); +x_35 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6(x_29, x_33, x_34, x_28); +lean_dec(x_29); +return x_35; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_LocalContext_foldlM___at_Lean_LocalContext_size___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +lean_dec(x_1); +x_5 = l_Std_PersistentArray_foldlM___at_Lean_LocalContext_size___spec__2(x_4, x_2, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_LocalContext_size(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Lean_LocalContext_foldlM___at_Lean_LocalContext_size___spec__1(x_1, x_2, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__5(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_LocalContext_size___spec__6(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_LocalContext_size___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_LocalContext_size___spec__3(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_LocalContext_findDecl_x3f___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { @@ -9738,7 +10172,7 @@ static lean_object* _init_l_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___ 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_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___spec__1___closed__1; x_2 = l_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9759,7 +10193,7 @@ static lean_object* _init_l_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_LocalDecl_value___closed__1; x_2 = l_Nat_foldRev_loop___at_Lean_LocalContext_mkBinding___spec__1___closed__5; -x_3 = lean_unsigned_to_nat(365u); +x_3 = lean_unsigned_to_nat(368u); x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_LocalContext_get_x21___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/ACLt.c b/stage0/stdlib/Lean/Meta/ACLt.c index 23e2bfcd3057..0cd76e921ed8 100644 --- a/stage0/stdlib/Lean/Meta/ACLt.c +++ b/stage0/stdlib/Lean/Meta/ACLt.c @@ -55,6 +55,7 @@ lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_ACLt_lt_lpo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); static lean_object* l_panic___at_Lean_Meta_ACLt_lt_lexSameCtor___spec__1___closed__1; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_ACLt_lt_ltApp___spec__2___closed__5; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_ACLt_lt_allChildrenLt___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Meta_ParamInfo_isInstImplicit(lean_object*); @@ -75,7 +76,6 @@ static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_ACLt_lt_ltApp___spec__ static lean_object* l_Lean_Meta_ACLt_lt_ltApp___lambda__2___closed__1; static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_ACLt_lt_ltApp___spec__2___closed__6; size_t lean_ptr_addr(lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); uint8_t l_Lean_Name_lt(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_ACLt_lt_ltApp___spec__1(lean_object*); @@ -1206,7 +1206,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Meta_ACLt_lt_ltApp___ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Meta_ACLt_lt_ltApp___spec__2___closed__7; x_2 = l_Std_Range_forIn_loop___at_Lean_Meta_ACLt_lt_ltApp___spec__2___closed__8; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Meta_ACLt_lt_ltApp___spec__2___closed__9; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2500,7 +2500,7 @@ x_18 = lean_ctor_get(x_14, 1); x_19 = lean_ctor_get(x_14, 0); lean_dec(x_19); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_1, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_20); x_22 = l_Lean_Meta_ACLt_lt_ltApp___closed__1; lean_inc(x_21); x_23 = lean_mk_array(x_21, x_22); @@ -2508,7 +2508,7 @@ x_24 = lean_unsigned_to_nat(1u); x_25 = lean_nat_sub(x_21, x_24); lean_dec(x_21); x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_23, x_25); -x_27 = l_Lean_Expr_getAppNumArgsAux(x_2, x_20); +x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_20); lean_inc(x_27); x_28 = lean_mk_array(x_27, x_22); x_29 = lean_nat_sub(x_27, x_24); @@ -2718,7 +2718,7 @@ x_65 = lean_ctor_get(x_14, 1); lean_inc(x_65); lean_dec(x_14); x_66 = lean_unsigned_to_nat(0u); -x_67 = l_Lean_Expr_getAppNumArgsAux(x_1, x_66); +x_67 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_66); x_68 = l_Lean_Meta_ACLt_lt_ltApp___closed__1; lean_inc(x_67); x_69 = lean_mk_array(x_67, x_68); @@ -2726,7 +2726,7 @@ x_70 = lean_unsigned_to_nat(1u); x_71 = lean_nat_sub(x_67, x_70); lean_dec(x_67); x_72 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_69, x_71); -x_73 = l_Lean_Expr_getAppNumArgsAux(x_2, x_66); +x_73 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_66); lean_inc(x_73); x_74 = lean_mk_array(x_73, x_68); x_75 = lean_nat_sub(x_73, x_70); @@ -3920,7 +3920,7 @@ case 5: { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Lean_Expr_getAppNumArgsAux(x_1, x_8); +x_9 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_8); x_10 = l_Lean_Meta_ACLt_lt_ltApp___closed__1; lean_inc(x_9); x_11 = lean_mk_array(x_9, x_10); diff --git a/stage0/stdlib/Lean/Meta/AbstractMVars.c b/stage0/stdlib/Lean/Meta/AbstractMVars.c index f801878116bf..b571d82eca00 100644 --- a/stage0/stdlib/Lean/Meta/AbstractMVars.c +++ b/stage0/stdlib/Lean/Meta/AbstractMVars.c @@ -14,21 +14,24 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Std_AssocList_contains___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__4___boxed(lean_object*, lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_openAbstractMVarsResult___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); lean_object* l_Lean_Meta_mkFreshLevelMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Level_param___override(lean_object*); +lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(lean_object*); +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); +uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__8(lean_object*, lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); +lean_object* l_Lean_Level_succ___override(lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Meta_AbstractMVars_State_lmap___default___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_instMonadMCtxM; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); uint8_t l_Lean_Level_hasMVar(lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); @@ -38,7 +41,9 @@ lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_StateT_get___at_Lean_Meta_AbstractMVars_instMonadMCtxM___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__7(lean_object*, lean_object*); +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_instInhabitedAbstractMVarsResult; +uint8_t l_ptrEqList___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insert___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AbstractMVars_instMonadMCtxM___closed__3; LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__2(lean_object*, lean_object*); @@ -51,6 +56,7 @@ static lean_object* l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVa LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__9(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_openAbstractMVarsResult___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_AbstractMVars_instMonadMCtxM___closed__1; +lean_object* l_Lean_simpLevelIMax_x27(lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); lean_object* lean_array_fget(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); @@ -59,12 +65,14 @@ LEAN_EXPORT lean_object* l_Lean_Meta_abstractMVars(lean_object*, lean_object*, l lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_abstractExprMVars(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___closed__2; -lean_object* lean_level_update_max(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Meta_instBEqAbstractMVarsResult___closed__1; +lean_object* l_Lean_simpLevelMax_x27(lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); lean_object* lean_name_append_index_after(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_mkFreshFVarId(lean_object*); LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__10(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__1(lean_object*, lean_object*); @@ -74,15 +82,14 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_instMonadMCtxM___lambda__1(le static lean_object* l_Lean_Meta_AbstractMVars_instMonadMCtxM___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_mkFreshId(lean_object*); LEAN_EXPORT uint8_t l_Std_AssocList_contains___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__4(lean_object*, lean_object*); +lean_object* l_Lean_Expr_sort___override(lean_object*); lean_object* l_Lean_Meta_lambdaMetaTelescope(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_isEqvAux___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_beqAbstractMVarsResult____x40_Lean_Meta_AbstractMVars___hyg_42____spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_modn(size_t, lean_object*); uint64_t l___private_Lean_Level_0__Lean_hashMVarId____x40_Lean_Level___hyg_478_(lean_object*); lean_object* l_Lean_Expr_bvar___override(lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__4(lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); static lean_object* l_Lean_Meta_AbstractMVars_abstractExprMVars___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_State_emap___default; LEAN_EXPORT lean_object* l_Std_HashMapImp_moveEntries___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__6(lean_object*, lean_object*, lean_object*); @@ -90,13 +97,13 @@ lean_object* lean_local_ctx_mk_local_decl(lean_object*, lean_object*, lean_objec LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_instMonadMCtxM___lambda__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Meta_AbstractMVars_State_emap___default___spec__1___boxed(lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); -lean_object* lean_level_update_imax(lean_object*, lean_object*, lean_object*); +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__5(lean_object*, lean_object*); +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_State_nextParamIdx___default; uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l_Lean_Meta_instInhabitedAbstractMVarsResult___closed__3; -lean_object* lean_expr_update_sort(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t l_Lean_Expr_hasMVar(lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Meta_AbstractMVars_State_lmap___default___spec__1___boxed(lean_object*); @@ -113,15 +120,16 @@ lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_instInhabitedAbstractMVarsResult___closed__1; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_State_lmap___default; -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); -lean_object* lean_level_update_succ(lean_object*, lean_object*); +lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_openAbstractMVarsResult(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_beqAbstractMVarsResult____x40_Lean_Meta_AbstractMVars___hyg_42____boxed(lean_object*, lean_object*); lean_object* l_Lean_MetavarContext_getLevelDepth(lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_instBEqAbstractMVarsResult; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_openAbstractMVarsResult___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_instantiateLevelParamsCore_visit___at_Lean_Expr_instantiateLevelParamsArray___spec__1(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_abstractMVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_AssocList_contains___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_Meta_AbstractMVars_instMonadMCtxM___spec__2(lean_object*, lean_object*); @@ -129,10 +137,8 @@ LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at___private_Lean_Meta_Abstr lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_State_paramNames___default; lean_object* l_Lean_MetavarContext_getDecl(lean_object*, lean_object*); -lean_object* lean_expr_update_app(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AbstractMVars_State_fvars___default; LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_Meta_AbstractMVars_instMonadMCtxM___spec__2___rarg(lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_const(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__6(lean_object*, lean_object*); static lean_object* _init_l_Lean_Meta_instInhabitedAbstractMVarsResult___closed__1() { @@ -1082,205 +1088,391 @@ case 1: lean_object* x_5; lean_object* x_6; uint8_t x_7; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); +lean_inc(x_5); x_6 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_5, x_2); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) { -lean_object* x_8; lean_object* x_9; +lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_level_update_succ(x_1, x_8); -lean_ctor_set(x_6, 0, x_9); +x_9 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_10 = lean_ptr_addr(x_8); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_1); +x_12 = l_Lean_Level_succ___override(x_8); +lean_ctor_set(x_6, 0, x_12); return x_6; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_6, 0); -x_11 = lean_ctor_get(x_6, 1); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_6); -x_12 = lean_level_update_succ(x_1, x_10); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +lean_dec(x_8); +lean_ctor_set(x_6, 0, x_1); +return x_6; } } -case 2: +else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_14 = lean_ctor_get(x_1, 0); +lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_6, 0); +x_14 = lean_ctor_get(x_6, 1); lean_inc(x_14); -x_15 = lean_ctor_get(x_1, 1); -lean_inc(x_15); -x_16 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_14, x_2); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_15, x_18); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_level_update_max(x_1, x_17, x_21); -lean_ctor_set(x_19, 0, x_22); +lean_inc(x_13); +lean_dec(x_6); +x_15 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_16 = lean_ptr_addr(x_13); +x_17 = lean_usize_dec_eq(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_1); +x_18 = l_Lean_Level_succ___override(x_13); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_14); return x_19; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_19, 0); -x_24 = lean_ctor_get(x_19, 1); +lean_object* x_20; +lean_dec(x_13); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_1); +lean_ctor_set(x_20, 1, x_14); +return x_20; +} +} +} +case 2: +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_21 = lean_ctor_get(x_1, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_1, 1); +lean_inc(x_22); +lean_inc(x_21); +x_23 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_21, x_2); +x_24 = lean_ctor_get(x_23, 0); lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_19); -x_25 = lean_level_update_max(x_1, x_17, x_23); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +lean_inc(x_22); +x_26 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_22, x_25); +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) +{ +lean_object* x_28; size_t x_29; size_t x_30; uint8_t x_31; +x_28 = lean_ctor_get(x_26, 0); +x_29 = lean_ptr_addr(x_21); +lean_dec(x_21); +x_30 = lean_ptr_addr(x_24); +x_31 = lean_usize_dec_eq(x_29, x_30); +if (x_31 == 0) +{ +lean_object* x_32; +lean_dec(x_22); +lean_dec(x_1); +x_32 = l_Lean_mkLevelMax_x27(x_24, x_28); +lean_ctor_set(x_26, 0, x_32); return x_26; } -} -case 3: +else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_27 = lean_ctor_get(x_1, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_1, 1); -lean_inc(x_28); -x_29 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_27, x_2); -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_28, x_31); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) +size_t x_33; size_t x_34; uint8_t x_35; +x_33 = lean_ptr_addr(x_22); +lean_dec(x_22); +x_34 = lean_ptr_addr(x_28); +x_35 = lean_usize_dec_eq(x_33, x_34); +if (x_35 == 0) { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_level_update_imax(x_1, x_30, x_34); -lean_ctor_set(x_32, 0, x_35); -return x_32; +lean_object* x_36; +lean_dec(x_1); +x_36 = l_Lean_mkLevelMax_x27(x_24, x_28); +lean_ctor_set(x_26, 0, x_36); +return x_26; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_32, 0); -x_37 = lean_ctor_get(x_32, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_32); -x_38 = lean_level_update_imax(x_1, x_30, x_36); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_37); -return x_39; +lean_object* x_37; +x_37 = l_Lean_simpLevelMax_x27(x_24, x_28, x_1); +lean_dec(x_1); +lean_dec(x_28); +lean_dec(x_24); +lean_ctor_set(x_26, 0, x_37); +return x_26; } } -case 5: +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_40 = lean_ctor_get(x_1, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_2, 2); -lean_inc(x_41); -lean_inc(x_40); -lean_inc(x_41); -x_42 = l_Lean_MetavarContext_getLevelDepth(x_41, x_40); -x_43 = lean_ctor_get(x_41, 0); -lean_inc(x_43); -x_44 = lean_nat_dec_eq(x_42, x_43); -lean_dec(x_43); -lean_dec(x_42); -if (x_44 == 0) +lean_object* x_38; lean_object* x_39; size_t x_40; size_t x_41; uint8_t x_42; +x_38 = lean_ctor_get(x_26, 0); +x_39 = lean_ctor_get(x_26, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_26); +x_40 = lean_ptr_addr(x_21); +lean_dec(x_21); +x_41 = lean_ptr_addr(x_24); +x_42 = lean_usize_dec_eq(x_40, x_41); +if (x_42 == 0) { -lean_object* x_45; -lean_dec(x_41); -lean_dec(x_40); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_1); -lean_ctor_set(x_45, 1, x_2); -return x_45; +lean_object* x_43; lean_object* x_44; +lean_dec(x_22); +lean_dec(x_1); +x_43 = l_Lean_mkLevelMax_x27(x_24, x_38); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_39); +return x_44; } else { -lean_object* x_46; lean_object* x_47; +size_t x_45; size_t x_46; uint8_t x_47; +x_45 = lean_ptr_addr(x_22); +lean_dec(x_22); +x_46 = lean_ptr_addr(x_38); +x_47 = lean_usize_dec_eq(x_45, x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_dec(x_1); -x_46 = lean_ctor_get(x_2, 6); -lean_inc(x_46); -lean_inc(x_40); -lean_inc(x_46); -x_47 = l_Std_HashMapImp_find_x3f___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__1(x_46, x_40); -if (lean_obj_tag(x_47) == 0) +x_48 = l_Lean_mkLevelMax_x27(x_24, x_38); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_39); +return x_49; +} +else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_48 = lean_ctor_get(x_2, 3); -lean_inc(x_48); -x_49 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___closed__2; -lean_inc(x_48); -x_50 = l_Lean_Name_num___override(x_49, x_48); -lean_inc(x_50); -x_51 = l_Lean_Level_param___override(x_50); -x_52 = lean_ctor_get(x_2, 0); +lean_object* x_50; lean_object* x_51; +x_50 = l_Lean_simpLevelMax_x27(x_24, x_38, x_1); +lean_dec(x_1); +lean_dec(x_38); +lean_dec(x_24); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_39); +return x_51; +} +} +} +} +case 3: +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; +x_52 = lean_ctor_get(x_1, 0); lean_inc(x_52); -x_53 = lean_ctor_get(x_2, 1); +x_53 = lean_ctor_get(x_1, 1); lean_inc(x_53); -x_54 = lean_unsigned_to_nat(1u); -x_55 = lean_nat_add(x_48, x_54); -lean_dec(x_48); -x_56 = lean_ctor_get(x_2, 4); +lean_inc(x_52); +x_54 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_52, x_2); +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_array_push(x_56, x_50); -x_58 = lean_ctor_get(x_2, 5); -lean_inc(x_58); -lean_inc(x_51); -x_59 = l_Std_HashMap_insert___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__3(x_46, x_40, x_51); -x_60 = lean_ctor_get(x_2, 7); -lean_inc(x_60); +lean_dec(x_54); +lean_inc(x_53); +x_57 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_53, x_56); +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) +{ +lean_object* x_59; size_t x_60; size_t x_61; uint8_t x_62; +x_59 = lean_ctor_get(x_57, 0); +x_60 = lean_ptr_addr(x_52); +lean_dec(x_52); +x_61 = lean_ptr_addr(x_55); +x_62 = lean_usize_dec_eq(x_60, x_61); +if (x_62 == 0) +{ +lean_object* x_63; +lean_dec(x_53); +lean_dec(x_1); +x_63 = l_Lean_mkLevelIMax_x27(x_55, x_59); +lean_ctor_set(x_57, 0, x_63); +return x_57; +} +else +{ +size_t x_64; size_t x_65; uint8_t x_66; +x_64 = lean_ptr_addr(x_53); +lean_dec(x_53); +x_65 = lean_ptr_addr(x_59); +x_66 = lean_usize_dec_eq(x_64, x_65); +if (x_66 == 0) +{ +lean_object* x_67; +lean_dec(x_1); +x_67 = l_Lean_mkLevelIMax_x27(x_55, x_59); +lean_ctor_set(x_57, 0, x_67); +return x_57; +} +else +{ +lean_object* x_68; +x_68 = l_Lean_simpLevelIMax_x27(x_55, x_59, x_1); +lean_dec(x_1); +lean_ctor_set(x_57, 0, x_68); +return x_57; +} +} +} +else +{ +lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; uint8_t x_73; +x_69 = lean_ctor_get(x_57, 0); +x_70 = lean_ctor_get(x_57, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_57); +x_71 = lean_ptr_addr(x_52); +lean_dec(x_52); +x_72 = lean_ptr_addr(x_55); +x_73 = lean_usize_dec_eq(x_71, x_72); +if (x_73 == 0) +{ +lean_object* x_74; lean_object* x_75; +lean_dec(x_53); +lean_dec(x_1); +x_74 = l_Lean_mkLevelIMax_x27(x_55, x_69); +x_75 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_70); +return x_75; +} +else +{ +size_t x_76; size_t x_77; uint8_t x_78; +x_76 = lean_ptr_addr(x_53); +lean_dec(x_53); +x_77 = lean_ptr_addr(x_69); +x_78 = lean_usize_dec_eq(x_76, x_77); +if (x_78 == 0) +{ +lean_object* x_79; lean_object* x_80; +lean_dec(x_1); +x_79 = l_Lean_mkLevelIMax_x27(x_55, x_69); +x_80 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_80, 0, x_79); +lean_ctor_set(x_80, 1, x_70); +return x_80; +} +else +{ +lean_object* x_81; lean_object* x_82; +x_81 = l_Lean_simpLevelIMax_x27(x_55, x_69, x_1); +lean_dec(x_1); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_70); +return x_82; +} +} +} +} +case 5: +{ +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; +x_83 = lean_ctor_get(x_1, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_2, 2); +lean_inc(x_84); +lean_inc(x_83); +lean_inc(x_84); +x_85 = l_Lean_MetavarContext_getLevelDepth(x_84, x_83); +x_86 = lean_ctor_get(x_84, 0); +lean_inc(x_86); +x_87 = lean_nat_dec_eq(x_85, x_86); +lean_dec(x_86); +lean_dec(x_85); +if (x_87 == 0) +{ +lean_object* x_88; +lean_dec(x_84); +lean_dec(x_83); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_1); +lean_ctor_set(x_88, 1, x_2); +return x_88; +} +else +{ +lean_object* x_89; lean_object* x_90; +lean_dec(x_1); +x_89 = lean_ctor_get(x_2, 6); +lean_inc(x_89); +lean_inc(x_83); +lean_inc(x_89); +x_90 = l_Std_HashMapImp_find_x3f___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__1(x_89, x_83); +if (lean_obj_tag(x_90) == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_91 = lean_ctor_get(x_2, 3); +lean_inc(x_91); +x_92 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___closed__2; +lean_inc(x_91); +x_93 = l_Lean_Name_num___override(x_92, x_91); +lean_inc(x_93); +x_94 = l_Lean_Level_param___override(x_93); +x_95 = lean_ctor_get(x_2, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_2, 1); +lean_inc(x_96); +x_97 = lean_unsigned_to_nat(1u); +x_98 = lean_nat_add(x_91, x_97); +lean_dec(x_91); +x_99 = lean_ctor_get(x_2, 4); +lean_inc(x_99); +x_100 = lean_array_push(x_99, x_93); +x_101 = lean_ctor_get(x_2, 5); +lean_inc(x_101); +lean_inc(x_94); +x_102 = l_Std_HashMap_insert___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__3(x_89, x_83, x_94); +x_103 = lean_ctor_get(x_2, 7); +lean_inc(x_103); lean_dec(x_2); -x_61 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_61, 0, x_52); -lean_ctor_set(x_61, 1, x_53); -lean_ctor_set(x_61, 2, x_41); -lean_ctor_set(x_61, 3, x_55); -lean_ctor_set(x_61, 4, x_57); -lean_ctor_set(x_61, 5, x_58); -lean_ctor_set(x_61, 6, x_59); -lean_ctor_set(x_61, 7, x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_51); -lean_ctor_set(x_62, 1, x_61); -return x_62; -} -else -{ -lean_object* x_63; lean_object* x_64; -lean_dec(x_46); -lean_dec(x_41); -lean_dec(x_40); -x_63 = lean_ctor_get(x_47, 0); -lean_inc(x_63); -lean_dec(x_47); -x_64 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_2); -return x_64; +x_104 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_104, 0, x_95); +lean_ctor_set(x_104, 1, x_96); +lean_ctor_set(x_104, 2, x_84); +lean_ctor_set(x_104, 3, x_98); +lean_ctor_set(x_104, 4, x_100); +lean_ctor_set(x_104, 5, x_101); +lean_ctor_set(x_104, 6, x_102); +lean_ctor_set(x_104, 7, x_103); +x_105 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_94); +lean_ctor_set(x_105, 1, x_104); +return x_105; +} +else +{ +lean_object* x_106; lean_object* x_107; +lean_dec(x_89); +lean_dec(x_84); +lean_dec(x_83); +x_106 = lean_ctor_get(x_90, 0); +lean_inc(x_106); +lean_dec(x_90); +x_107 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set(x_107, 1, x_2); +return x_107; } } } default: { -lean_object* x_65; -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_1); -lean_ctor_set(x_65, 1, x_2); -return x_65; +lean_object* x_108; +x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_108, 0, x_1); +lean_ctor_set(x_108, 1, x_2); +return x_108; } } } @@ -2305,290 +2497,858 @@ case 3: lean_object* x_117; lean_object* x_118; uint8_t x_119; x_117 = lean_ctor_get(x_1, 0); lean_inc(x_117); +lean_inc(x_117); x_118 = l___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars(x_117, x_2); x_119 = !lean_is_exclusive(x_118); if (x_119 == 0) { -lean_object* x_120; lean_object* x_121; +lean_object* x_120; size_t x_121; size_t x_122; uint8_t x_123; x_120 = lean_ctor_get(x_118, 0); -x_121 = lean_expr_update_sort(x_1, x_120); -lean_ctor_set(x_118, 0, x_121); +x_121 = lean_ptr_addr(x_117); +lean_dec(x_117); +x_122 = lean_ptr_addr(x_120); +x_123 = lean_usize_dec_eq(x_121, x_122); +if (x_123 == 0) +{ +lean_object* x_124; +lean_dec(x_1); +x_124 = l_Lean_Expr_sort___override(x_120); +lean_ctor_set(x_118, 0, x_124); return x_118; } else { -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_122 = lean_ctor_get(x_118, 0); -x_123 = lean_ctor_get(x_118, 1); -lean_inc(x_123); -lean_inc(x_122); -lean_dec(x_118); -x_124 = lean_expr_update_sort(x_1, x_122); -x_125 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_125, 0, x_124); -lean_ctor_set(x_125, 1, x_123); -return x_125; +lean_dec(x_120); +lean_ctor_set(x_118, 0, x_1); +return x_118; } } -case 4: +else { -lean_object* x_126; lean_object* x_127; uint8_t x_128; -x_126 = lean_ctor_get(x_1, 1); +lean_object* x_125; lean_object* x_126; size_t x_127; size_t x_128; uint8_t x_129; +x_125 = lean_ctor_get(x_118, 0); +x_126 = lean_ctor_get(x_118, 1); lean_inc(x_126); -x_127 = l_List_mapM___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__10(x_126, x_2); -x_128 = !lean_is_exclusive(x_127); -if (x_128 == 0) +lean_inc(x_125); +lean_dec(x_118); +x_127 = lean_ptr_addr(x_117); +lean_dec(x_117); +x_128 = lean_ptr_addr(x_125); +x_129 = lean_usize_dec_eq(x_127, x_128); +if (x_129 == 0) { -lean_object* x_129; lean_object* x_130; -x_129 = lean_ctor_get(x_127, 0); -x_130 = lean_expr_update_const(x_1, x_129); -lean_ctor_set(x_127, 0, x_130); -return x_127; +lean_object* x_130; lean_object* x_131; +lean_dec(x_1); +x_130 = l_Lean_Expr_sort___override(x_125); +x_131 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_126); +return x_131; } else { -lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; -x_131 = lean_ctor_get(x_127, 0); -x_132 = lean_ctor_get(x_127, 1); -lean_inc(x_132); -lean_inc(x_131); -lean_dec(x_127); -x_133 = lean_expr_update_const(x_1, x_131); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_133); -lean_ctor_set(x_134, 1, x_132); -return x_134; +lean_object* x_132; +lean_dec(x_125); +x_132 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_132, 0, x_1); +lean_ctor_set(x_132, 1, x_126); +return x_132; } } -case 5: +} +case 4: +{ +lean_object* x_133; lean_object* x_134; lean_object* x_135; uint8_t x_136; +x_133 = lean_ctor_get(x_1, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_1, 1); +lean_inc(x_134); +lean_inc(x_134); +x_135 = l_List_mapM___at_Lean_Meta_AbstractMVars_abstractExprMVars___spec__10(x_134, x_2); +x_136 = !lean_is_exclusive(x_135); +if (x_136 == 0) +{ +lean_object* x_137; uint8_t x_138; +x_137 = lean_ctor_get(x_135, 0); +x_138 = l_ptrEqList___rarg(x_134, x_137); +lean_dec(x_134); +if (x_138 == 0) +{ +lean_object* x_139; +lean_dec(x_1); +x_139 = l_Lean_Expr_const___override(x_133, x_137); +lean_ctor_set(x_135, 0, x_139); +return x_135; +} +else { -lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; uint8_t x_141; -x_135 = lean_ctor_get(x_1, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_1, 1); -lean_inc(x_136); -x_137 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_135, x_2); -x_138 = lean_ctor_get(x_137, 0); -lean_inc(x_138); -x_139 = lean_ctor_get(x_137, 1); -lean_inc(x_139); lean_dec(x_137); -x_140 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_136, x_139); -x_141 = !lean_is_exclusive(x_140); -if (x_141 == 0) +lean_dec(x_133); +lean_ctor_set(x_135, 0, x_1); +return x_135; +} +} +else +{ +lean_object* x_140; lean_object* x_141; uint8_t x_142; +x_140 = lean_ctor_get(x_135, 0); +x_141 = lean_ctor_get(x_135, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_135); +x_142 = l_ptrEqList___rarg(x_134, x_140); +lean_dec(x_134); +if (x_142 == 0) { -lean_object* x_142; lean_object* x_143; -x_142 = lean_ctor_get(x_140, 0); -x_143 = lean_expr_update_app(x_1, x_138, x_142); -lean_ctor_set(x_140, 0, x_143); -return x_140; +lean_object* x_143; lean_object* x_144; +lean_dec(x_1); +x_143 = l_Lean_Expr_const___override(x_133, x_140); +x_144 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_141); +return x_144; } else { -lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_144 = lean_ctor_get(x_140, 0); -x_145 = lean_ctor_get(x_140, 1); -lean_inc(x_145); -lean_inc(x_144); +lean_object* x_145; lean_dec(x_140); -x_146 = lean_expr_update_app(x_1, x_138, x_144); -x_147 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_147, 0, x_146); -lean_ctor_set(x_147, 1, x_145); -return x_147; +lean_dec(x_133); +x_145 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_145, 0, x_1); +lean_ctor_set(x_145, 1, x_141); +return x_145; } } -case 6: +} +case 5: { -lean_object* x_148; lean_object* x_149; uint8_t x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; uint8_t x_155; -x_148 = lean_ctor_get(x_1, 1); -lean_inc(x_148); -x_149 = lean_ctor_get(x_1, 2); +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; uint8_t x_152; +x_146 = lean_ctor_get(x_1, 0); +lean_inc(x_146); +x_147 = lean_ctor_get(x_1, 1); +lean_inc(x_147); +lean_inc(x_146); +x_148 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_146, x_2); +x_149 = lean_ctor_get(x_148, 0); lean_inc(x_149); -x_150 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_151 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_148, x_2); -x_152 = lean_ctor_get(x_151, 0); -lean_inc(x_152); -x_153 = lean_ctor_get(x_151, 1); -lean_inc(x_153); -lean_dec(x_151); -x_154 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_149, x_153); -x_155 = !lean_is_exclusive(x_154); -if (x_155 == 0) +x_150 = lean_ctor_get(x_148, 1); +lean_inc(x_150); +lean_dec(x_148); +lean_inc(x_147); +x_151 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_147, x_150); +x_152 = !lean_is_exclusive(x_151); +if (x_152 == 0) +{ +lean_object* x_153; size_t x_154; size_t x_155; uint8_t x_156; +x_153 = lean_ctor_get(x_151, 0); +x_154 = lean_ptr_addr(x_146); +lean_dec(x_146); +x_155 = lean_ptr_addr(x_149); +x_156 = lean_usize_dec_eq(x_154, x_155); +if (x_156 == 0) +{ +lean_object* x_157; +lean_dec(x_147); +lean_dec(x_1); +x_157 = l_Lean_Expr_app___override(x_149, x_153); +lean_ctor_set(x_151, 0, x_157); +return x_151; +} +else +{ +size_t x_158; size_t x_159; uint8_t x_160; +x_158 = lean_ptr_addr(x_147); +lean_dec(x_147); +x_159 = lean_ptr_addr(x_153); +x_160 = lean_usize_dec_eq(x_158, x_159); +if (x_160 == 0) { -lean_object* x_156; lean_object* x_157; -x_156 = lean_ctor_get(x_154, 0); -x_157 = lean_expr_update_lambda(x_1, x_150, x_152, x_156); -lean_ctor_set(x_154, 0, x_157); -return x_154; +lean_object* x_161; +lean_dec(x_1); +x_161 = l_Lean_Expr_app___override(x_149, x_153); +lean_ctor_set(x_151, 0, x_161); +return x_151; } else { -lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; -x_158 = lean_ctor_get(x_154, 0); -x_159 = lean_ctor_get(x_154, 1); -lean_inc(x_159); -lean_inc(x_158); -lean_dec(x_154); -x_160 = lean_expr_update_lambda(x_1, x_150, x_152, x_158); -x_161 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_161, 0, x_160); -lean_ctor_set(x_161, 1, x_159); -return x_161; +lean_dec(x_153); +lean_dec(x_149); +lean_ctor_set(x_151, 0, x_1); +return x_151; } } -case 7: +} +else { -lean_object* x_162; lean_object* x_163; uint8_t x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_169; -x_162 = lean_ctor_get(x_1, 1); -lean_inc(x_162); -x_163 = lean_ctor_get(x_1, 2); +lean_object* x_162; lean_object* x_163; size_t x_164; size_t x_165; uint8_t x_166; +x_162 = lean_ctor_get(x_151, 0); +x_163 = lean_ctor_get(x_151, 1); lean_inc(x_163); -x_164 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_165 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_162, x_2); -x_166 = lean_ctor_get(x_165, 0); -lean_inc(x_166); -x_167 = lean_ctor_get(x_165, 1); -lean_inc(x_167); -lean_dec(x_165); -x_168 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_163, x_167); -x_169 = !lean_is_exclusive(x_168); -if (x_169 == 0) -{ -lean_object* x_170; lean_object* x_171; -x_170 = lean_ctor_get(x_168, 0); -x_171 = lean_expr_update_forall(x_1, x_164, x_166, x_170); -lean_ctor_set(x_168, 0, x_171); +lean_inc(x_162); +lean_dec(x_151); +x_164 = lean_ptr_addr(x_146); +lean_dec(x_146); +x_165 = lean_ptr_addr(x_149); +x_166 = lean_usize_dec_eq(x_164, x_165); +if (x_166 == 0) +{ +lean_object* x_167; lean_object* x_168; +lean_dec(x_147); +lean_dec(x_1); +x_167 = l_Lean_Expr_app___override(x_149, x_162); +x_168 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_168, 0, x_167); +lean_ctor_set(x_168, 1, x_163); return x_168; } else { -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; -x_172 = lean_ctor_get(x_168, 0); -x_173 = lean_ctor_get(x_168, 1); -lean_inc(x_173); -lean_inc(x_172); -lean_dec(x_168); -x_174 = lean_expr_update_forall(x_1, x_164, x_166, x_172); -x_175 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_175, 0, x_174); -lean_ctor_set(x_175, 1, x_173); -return x_175; +size_t x_169; size_t x_170; uint8_t x_171; +x_169 = lean_ptr_addr(x_147); +lean_dec(x_147); +x_170 = lean_ptr_addr(x_162); +x_171 = lean_usize_dec_eq(x_169, x_170); +if (x_171 == 0) +{ +lean_object* x_172; lean_object* x_173; +lean_dec(x_1); +x_172 = l_Lean_Expr_app___override(x_149, x_162); +x_173 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_173, 0, x_172); +lean_ctor_set(x_173, 1, x_163); +return x_173; } +else +{ +lean_object* x_174; +lean_dec(x_162); +lean_dec(x_149); +x_174 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_174, 0, x_1); +lean_ctor_set(x_174, 1, x_163); +return x_174; } -case 8: +} +} +} +case 6: { -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; uint8_t x_186; +lean_object* x_175; lean_object* x_176; lean_object* x_177; uint8_t x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_175 = lean_ctor_get(x_1, 0); +lean_inc(x_175); x_176 = lean_ctor_get(x_1, 1); lean_inc(x_176); x_177 = lean_ctor_get(x_1, 2); lean_inc(x_177); -x_178 = lean_ctor_get(x_1, 3); -lean_inc(x_178); +x_178 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_176); x_179 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_176, x_2); x_180 = lean_ctor_get(x_179, 0); lean_inc(x_180); x_181 = lean_ctor_get(x_179, 1); lean_inc(x_181); lean_dec(x_179); +lean_inc(x_177); x_182 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_177, x_181); -x_183 = lean_ctor_get(x_182, 0); -lean_inc(x_183); -x_184 = lean_ctor_get(x_182, 1); -lean_inc(x_184); -lean_dec(x_182); -x_185 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_178, x_184); -x_186 = !lean_is_exclusive(x_185); -if (x_186 == 0) +x_183 = !lean_is_exclusive(x_182); +if (x_183 == 0) +{ +lean_object* x_184; lean_object* x_185; size_t x_186; size_t x_187; uint8_t x_188; +x_184 = lean_ctor_get(x_182, 0); +lean_inc(x_177); +lean_inc(x_176); +lean_inc(x_175); +x_185 = l_Lean_Expr_lam___override(x_175, x_176, x_177, x_178); +x_186 = lean_ptr_addr(x_176); +lean_dec(x_176); +x_187 = lean_ptr_addr(x_180); +x_188 = lean_usize_dec_eq(x_186, x_187); +if (x_188 == 0) +{ +lean_object* x_189; +lean_dec(x_185); +lean_dec(x_177); +x_189 = l_Lean_Expr_lam___override(x_175, x_180, x_184, x_178); +lean_ctor_set(x_182, 0, x_189); +return x_182; +} +else +{ +size_t x_190; size_t x_191; uint8_t x_192; +x_190 = lean_ptr_addr(x_177); +lean_dec(x_177); +x_191 = lean_ptr_addr(x_184); +x_192 = lean_usize_dec_eq(x_190, x_191); +if (x_192 == 0) { -lean_object* x_187; lean_object* x_188; -x_187 = lean_ctor_get(x_185, 0); -x_188 = lean_expr_update_let(x_1, x_180, x_183, x_187); -lean_ctor_set(x_185, 0, x_188); -return x_185; +lean_object* x_193; +lean_dec(x_185); +x_193 = l_Lean_Expr_lam___override(x_175, x_180, x_184, x_178); +lean_ctor_set(x_182, 0, x_193); +return x_182; } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_189 = lean_ctor_get(x_185, 0); -x_190 = lean_ctor_get(x_185, 1); -lean_inc(x_190); -lean_inc(x_189); +uint8_t x_194; +x_194 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_178, x_178); +if (x_194 == 0) +{ +lean_object* x_195; lean_dec(x_185); -x_191 = lean_expr_update_let(x_1, x_180, x_183, x_189); -x_192 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_192, 0, x_191); -lean_ctor_set(x_192, 1, x_190); -return x_192; +x_195 = l_Lean_Expr_lam___override(x_175, x_180, x_184, x_178); +lean_ctor_set(x_182, 0, x_195); +return x_182; +} +else +{ +lean_dec(x_184); +lean_dec(x_180); +lean_dec(x_175); +lean_ctor_set(x_182, 0, x_185); +return x_182; +} +} +} +} +else +{ +lean_object* x_196; lean_object* x_197; lean_object* x_198; size_t x_199; size_t x_200; uint8_t x_201; +x_196 = lean_ctor_get(x_182, 0); +x_197 = lean_ctor_get(x_182, 1); +lean_inc(x_197); +lean_inc(x_196); +lean_dec(x_182); +lean_inc(x_177); +lean_inc(x_176); +lean_inc(x_175); +x_198 = l_Lean_Expr_lam___override(x_175, x_176, x_177, x_178); +x_199 = lean_ptr_addr(x_176); +lean_dec(x_176); +x_200 = lean_ptr_addr(x_180); +x_201 = lean_usize_dec_eq(x_199, x_200); +if (x_201 == 0) +{ +lean_object* x_202; lean_object* x_203; +lean_dec(x_198); +lean_dec(x_177); +x_202 = l_Lean_Expr_lam___override(x_175, x_180, x_196, x_178); +x_203 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_203, 0, x_202); +lean_ctor_set(x_203, 1, x_197); +return x_203; +} +else +{ +size_t x_204; size_t x_205; uint8_t x_206; +x_204 = lean_ptr_addr(x_177); +lean_dec(x_177); +x_205 = lean_ptr_addr(x_196); +x_206 = lean_usize_dec_eq(x_204, x_205); +if (x_206 == 0) +{ +lean_object* x_207; lean_object* x_208; +lean_dec(x_198); +x_207 = l_Lean_Expr_lam___override(x_175, x_180, x_196, x_178); +x_208 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_208, 0, x_207); +lean_ctor_set(x_208, 1, x_197); +return x_208; +} +else +{ +uint8_t x_209; +x_209 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_178, x_178); +if (x_209 == 0) +{ +lean_object* x_210; lean_object* x_211; +lean_dec(x_198); +x_210 = l_Lean_Expr_lam___override(x_175, x_180, x_196, x_178); +x_211 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_211, 0, x_210); +lean_ctor_set(x_211, 1, x_197); +return x_211; +} +else +{ +lean_object* x_212; +lean_dec(x_196); +lean_dec(x_180); +lean_dec(x_175); +x_212 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_212, 0, x_198); +lean_ctor_set(x_212, 1, x_197); +return x_212; +} +} +} +} +} +case 7: +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; uint8_t x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; uint8_t x_221; +x_213 = lean_ctor_get(x_1, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_1, 1); +lean_inc(x_214); +x_215 = lean_ctor_get(x_1, 2); +lean_inc(x_215); +x_216 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_214); +x_217 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_214, x_2); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +x_219 = lean_ctor_get(x_217, 1); +lean_inc(x_219); +lean_dec(x_217); +lean_inc(x_215); +x_220 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_215, x_219); +x_221 = !lean_is_exclusive(x_220); +if (x_221 == 0) +{ +lean_object* x_222; lean_object* x_223; size_t x_224; size_t x_225; uint8_t x_226; +x_222 = lean_ctor_get(x_220, 0); +lean_inc(x_215); +lean_inc(x_214); +lean_inc(x_213); +x_223 = l_Lean_Expr_forallE___override(x_213, x_214, x_215, x_216); +x_224 = lean_ptr_addr(x_214); +lean_dec(x_214); +x_225 = lean_ptr_addr(x_218); +x_226 = lean_usize_dec_eq(x_224, x_225); +if (x_226 == 0) +{ +lean_object* x_227; +lean_dec(x_223); +lean_dec(x_215); +x_227 = l_Lean_Expr_forallE___override(x_213, x_218, x_222, x_216); +lean_ctor_set(x_220, 0, x_227); +return x_220; +} +else +{ +size_t x_228; size_t x_229; uint8_t x_230; +x_228 = lean_ptr_addr(x_215); +lean_dec(x_215); +x_229 = lean_ptr_addr(x_222); +x_230 = lean_usize_dec_eq(x_228, x_229); +if (x_230 == 0) +{ +lean_object* x_231; +lean_dec(x_223); +x_231 = l_Lean_Expr_forallE___override(x_213, x_218, x_222, x_216); +lean_ctor_set(x_220, 0, x_231); +return x_220; +} +else +{ +uint8_t x_232; +x_232 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_216, x_216); +if (x_232 == 0) +{ +lean_object* x_233; +lean_dec(x_223); +x_233 = l_Lean_Expr_forallE___override(x_213, x_218, x_222, x_216); +lean_ctor_set(x_220, 0, x_233); +return x_220; +} +else +{ +lean_dec(x_222); +lean_dec(x_218); +lean_dec(x_213); +lean_ctor_set(x_220, 0, x_223); +return x_220; +} +} +} +} +else +{ +lean_object* x_234; lean_object* x_235; lean_object* x_236; size_t x_237; size_t x_238; uint8_t x_239; +x_234 = lean_ctor_get(x_220, 0); +x_235 = lean_ctor_get(x_220, 1); +lean_inc(x_235); +lean_inc(x_234); +lean_dec(x_220); +lean_inc(x_215); +lean_inc(x_214); +lean_inc(x_213); +x_236 = l_Lean_Expr_forallE___override(x_213, x_214, x_215, x_216); +x_237 = lean_ptr_addr(x_214); +lean_dec(x_214); +x_238 = lean_ptr_addr(x_218); +x_239 = lean_usize_dec_eq(x_237, x_238); +if (x_239 == 0) +{ +lean_object* x_240; lean_object* x_241; +lean_dec(x_236); +lean_dec(x_215); +x_240 = l_Lean_Expr_forallE___override(x_213, x_218, x_234, x_216); +x_241 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_241, 0, x_240); +lean_ctor_set(x_241, 1, x_235); +return x_241; +} +else +{ +size_t x_242; size_t x_243; uint8_t x_244; +x_242 = lean_ptr_addr(x_215); +lean_dec(x_215); +x_243 = lean_ptr_addr(x_234); +x_244 = lean_usize_dec_eq(x_242, x_243); +if (x_244 == 0) +{ +lean_object* x_245; lean_object* x_246; +lean_dec(x_236); +x_245 = l_Lean_Expr_forallE___override(x_213, x_218, x_234, x_216); +x_246 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_246, 0, x_245); +lean_ctor_set(x_246, 1, x_235); +return x_246; +} +else +{ +uint8_t x_247; +x_247 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_216, x_216); +if (x_247 == 0) +{ +lean_object* x_248; lean_object* x_249; +lean_dec(x_236); +x_248 = l_Lean_Expr_forallE___override(x_213, x_218, x_234, x_216); +x_249 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_249, 0, x_248); +lean_ctor_set(x_249, 1, x_235); +return x_249; +} +else +{ +lean_object* x_250; +lean_dec(x_234); +lean_dec(x_218); +lean_dec(x_213); +x_250 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_250, 0, x_236); +lean_ctor_set(x_250, 1, x_235); +return x_250; +} +} +} +} +} +case 8: +{ +lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; uint8_t x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; uint8_t x_263; +x_251 = lean_ctor_get(x_1, 0); +lean_inc(x_251); +x_252 = lean_ctor_get(x_1, 1); +lean_inc(x_252); +x_253 = lean_ctor_get(x_1, 2); +lean_inc(x_253); +x_254 = lean_ctor_get(x_1, 3); +lean_inc(x_254); +x_255 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); +lean_inc(x_252); +x_256 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_252, x_2); +x_257 = lean_ctor_get(x_256, 0); +lean_inc(x_257); +x_258 = lean_ctor_get(x_256, 1); +lean_inc(x_258); +lean_dec(x_256); +lean_inc(x_253); +x_259 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_253, x_258); +x_260 = lean_ctor_get(x_259, 0); +lean_inc(x_260); +x_261 = lean_ctor_get(x_259, 1); +lean_inc(x_261); +lean_dec(x_259); +lean_inc(x_254); +x_262 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_254, x_261); +x_263 = !lean_is_exclusive(x_262); +if (x_263 == 0) +{ +lean_object* x_264; size_t x_265; size_t x_266; uint8_t x_267; +x_264 = lean_ctor_get(x_262, 0); +x_265 = lean_ptr_addr(x_252); +lean_dec(x_252); +x_266 = lean_ptr_addr(x_257); +x_267 = lean_usize_dec_eq(x_265, x_266); +if (x_267 == 0) +{ +lean_object* x_268; +lean_dec(x_254); +lean_dec(x_253); +lean_dec(x_1); +x_268 = l_Lean_Expr_letE___override(x_251, x_257, x_260, x_264, x_255); +lean_ctor_set(x_262, 0, x_268); +return x_262; +} +else +{ +size_t x_269; size_t x_270; uint8_t x_271; +x_269 = lean_ptr_addr(x_253); +lean_dec(x_253); +x_270 = lean_ptr_addr(x_260); +x_271 = lean_usize_dec_eq(x_269, x_270); +if (x_271 == 0) +{ +lean_object* x_272; +lean_dec(x_254); +lean_dec(x_1); +x_272 = l_Lean_Expr_letE___override(x_251, x_257, x_260, x_264, x_255); +lean_ctor_set(x_262, 0, x_272); +return x_262; +} +else +{ +size_t x_273; size_t x_274; uint8_t x_275; +x_273 = lean_ptr_addr(x_254); +lean_dec(x_254); +x_274 = lean_ptr_addr(x_264); +x_275 = lean_usize_dec_eq(x_273, x_274); +if (x_275 == 0) +{ +lean_object* x_276; +lean_dec(x_1); +x_276 = l_Lean_Expr_letE___override(x_251, x_257, x_260, x_264, x_255); +lean_ctor_set(x_262, 0, x_276); +return x_262; +} +else +{ +lean_dec(x_264); +lean_dec(x_260); +lean_dec(x_257); +lean_dec(x_251); +lean_ctor_set(x_262, 0, x_1); +return x_262; +} +} +} +} +else +{ +lean_object* x_277; lean_object* x_278; size_t x_279; size_t x_280; uint8_t x_281; +x_277 = lean_ctor_get(x_262, 0); +x_278 = lean_ctor_get(x_262, 1); +lean_inc(x_278); +lean_inc(x_277); +lean_dec(x_262); +x_279 = lean_ptr_addr(x_252); +lean_dec(x_252); +x_280 = lean_ptr_addr(x_257); +x_281 = lean_usize_dec_eq(x_279, x_280); +if (x_281 == 0) +{ +lean_object* x_282; lean_object* x_283; +lean_dec(x_254); +lean_dec(x_253); +lean_dec(x_1); +x_282 = l_Lean_Expr_letE___override(x_251, x_257, x_260, x_277, x_255); +x_283 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_283, 0, x_282); +lean_ctor_set(x_283, 1, x_278); +return x_283; +} +else +{ +size_t x_284; size_t x_285; uint8_t x_286; +x_284 = lean_ptr_addr(x_253); +lean_dec(x_253); +x_285 = lean_ptr_addr(x_260); +x_286 = lean_usize_dec_eq(x_284, x_285); +if (x_286 == 0) +{ +lean_object* x_287; lean_object* x_288; +lean_dec(x_254); +lean_dec(x_1); +x_287 = l_Lean_Expr_letE___override(x_251, x_257, x_260, x_277, x_255); +x_288 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_288, 0, x_287); +lean_ctor_set(x_288, 1, x_278); +return x_288; +} +else +{ +size_t x_289; size_t x_290; uint8_t x_291; +x_289 = lean_ptr_addr(x_254); +lean_dec(x_254); +x_290 = lean_ptr_addr(x_277); +x_291 = lean_usize_dec_eq(x_289, x_290); +if (x_291 == 0) +{ +lean_object* x_292; lean_object* x_293; +lean_dec(x_1); +x_292 = l_Lean_Expr_letE___override(x_251, x_257, x_260, x_277, x_255); +x_293 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_293, 0, x_292); +lean_ctor_set(x_293, 1, x_278); +return x_293; +} +else +{ +lean_object* x_294; +lean_dec(x_277); +lean_dec(x_260); +lean_dec(x_257); +lean_dec(x_251); +x_294 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_294, 0, x_1); +lean_ctor_set(x_294, 1, x_278); +return x_294; +} +} +} } } case 10: { -lean_object* x_193; lean_object* x_194; uint8_t x_195; -x_193 = lean_ctor_get(x_1, 1); -lean_inc(x_193); -x_194 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_193, x_2); -x_195 = !lean_is_exclusive(x_194); -if (x_195 == 0) +lean_object* x_295; lean_object* x_296; lean_object* x_297; uint8_t x_298; +x_295 = lean_ctor_get(x_1, 0); +lean_inc(x_295); +x_296 = lean_ctor_get(x_1, 1); +lean_inc(x_296); +lean_inc(x_296); +x_297 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_296, x_2); +x_298 = !lean_is_exclusive(x_297); +if (x_298 == 0) +{ +lean_object* x_299; size_t x_300; size_t x_301; uint8_t x_302; +x_299 = lean_ctor_get(x_297, 0); +x_300 = lean_ptr_addr(x_296); +lean_dec(x_296); +x_301 = lean_ptr_addr(x_299); +x_302 = lean_usize_dec_eq(x_300, x_301); +if (x_302 == 0) +{ +lean_object* x_303; +lean_dec(x_1); +x_303 = l_Lean_Expr_mdata___override(x_295, x_299); +lean_ctor_set(x_297, 0, x_303); +return x_297; +} +else +{ +lean_dec(x_299); +lean_dec(x_295); +lean_ctor_set(x_297, 0, x_1); +return x_297; +} +} +else { -lean_object* x_196; lean_object* x_197; -x_196 = lean_ctor_get(x_194, 0); -x_197 = lean_expr_update_mdata(x_1, x_196); -lean_ctor_set(x_194, 0, x_197); -return x_194; +lean_object* x_304; lean_object* x_305; size_t x_306; size_t x_307; uint8_t x_308; +x_304 = lean_ctor_get(x_297, 0); +x_305 = lean_ctor_get(x_297, 1); +lean_inc(x_305); +lean_inc(x_304); +lean_dec(x_297); +x_306 = lean_ptr_addr(x_296); +lean_dec(x_296); +x_307 = lean_ptr_addr(x_304); +x_308 = lean_usize_dec_eq(x_306, x_307); +if (x_308 == 0) +{ +lean_object* x_309; lean_object* x_310; +lean_dec(x_1); +x_309 = l_Lean_Expr_mdata___override(x_295, x_304); +x_310 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_310, 0, x_309); +lean_ctor_set(x_310, 1, x_305); +return x_310; } else { -lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; -x_198 = lean_ctor_get(x_194, 0); -x_199 = lean_ctor_get(x_194, 1); -lean_inc(x_199); -lean_inc(x_198); -lean_dec(x_194); -x_200 = lean_expr_update_mdata(x_1, x_198); -x_201 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_201, 0, x_200); -lean_ctor_set(x_201, 1, x_199); -return x_201; +lean_object* x_311; +lean_dec(x_304); +lean_dec(x_295); +x_311 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_311, 0, x_1); +lean_ctor_set(x_311, 1, x_305); +return x_311; +} } } case 11: { -lean_object* x_202; lean_object* x_203; uint8_t x_204; -x_202 = lean_ctor_get(x_1, 2); -lean_inc(x_202); -x_203 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_202, x_2); -x_204 = !lean_is_exclusive(x_203); -if (x_204 == 0) -{ -lean_object* x_205; lean_object* x_206; -x_205 = lean_ctor_get(x_203, 0); -x_206 = lean_expr_update_proj(x_1, x_205); -lean_ctor_set(x_203, 0, x_206); -return x_203; +lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; uint8_t x_316; +x_312 = lean_ctor_get(x_1, 0); +lean_inc(x_312); +x_313 = lean_ctor_get(x_1, 1); +lean_inc(x_313); +x_314 = lean_ctor_get(x_1, 2); +lean_inc(x_314); +lean_inc(x_314); +x_315 = l_Lean_Meta_AbstractMVars_abstractExprMVars(x_314, x_2); +x_316 = !lean_is_exclusive(x_315); +if (x_316 == 0) +{ +lean_object* x_317; size_t x_318; size_t x_319; uint8_t x_320; +x_317 = lean_ctor_get(x_315, 0); +x_318 = lean_ptr_addr(x_314); +lean_dec(x_314); +x_319 = lean_ptr_addr(x_317); +x_320 = lean_usize_dec_eq(x_318, x_319); +if (x_320 == 0) +{ +lean_object* x_321; +lean_dec(x_1); +x_321 = l_Lean_Expr_proj___override(x_312, x_313, x_317); +lean_ctor_set(x_315, 0, x_321); +return x_315; +} +else +{ +lean_dec(x_317); +lean_dec(x_313); +lean_dec(x_312); +lean_ctor_set(x_315, 0, x_1); +return x_315; +} +} +else +{ +lean_object* x_322; lean_object* x_323; size_t x_324; size_t x_325; uint8_t x_326; +x_322 = lean_ctor_get(x_315, 0); +x_323 = lean_ctor_get(x_315, 1); +lean_inc(x_323); +lean_inc(x_322); +lean_dec(x_315); +x_324 = lean_ptr_addr(x_314); +lean_dec(x_314); +x_325 = lean_ptr_addr(x_322); +x_326 = lean_usize_dec_eq(x_324, x_325); +if (x_326 == 0) +{ +lean_object* x_327; lean_object* x_328; +lean_dec(x_1); +x_327 = l_Lean_Expr_proj___override(x_312, x_313, x_322); +x_328 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_328, 0, x_327); +lean_ctor_set(x_328, 1, x_323); +return x_328; } else { -lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; -x_207 = lean_ctor_get(x_203, 0); -x_208 = lean_ctor_get(x_203, 1); -lean_inc(x_208); -lean_inc(x_207); -lean_dec(x_203); -x_209 = lean_expr_update_proj(x_1, x_207); -x_210 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_210, 0, x_209); -lean_ctor_set(x_210, 1, x_208); -return x_210; +lean_object* x_329; +lean_dec(x_322); +lean_dec(x_313); +lean_dec(x_312); +x_329 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_329, 0, x_1); +lean_ctor_set(x_329, 1, x_323); +return x_329; +} } } default: { -lean_object* x_211; -x_211 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_211, 0, x_1); -lean_ctor_set(x_211, 1, x_2); -return x_211; +lean_object* x_330; +x_330 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_330, 0, x_1); +lean_ctor_set(x_330, 1, x_2); +return x_330; } } } diff --git a/stage0/stdlib/Lean/Meta/AbstractNestedProofs.c b/stage0/stdlib/Lean/Meta/AbstractNestedProofs.c index d6204cb8b25b..95a7c3dde419 100644 --- a/stage0/stdlib/Lean/Meta/AbstractNestedProofs.c +++ b/stage0/stdlib/Lean/Meta/AbstractNestedProofs.c @@ -22,10 +22,10 @@ lean_object* l_Lean_Meta_mkForallFVars(lean_object*, lean_object*, uint8_t, uint lean_object* l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_AbstractNestedProofs_isNonTrivialProof___spec__1(lean_object*, size_t, size_t); static lean_object* l_Lean_Meta_abstractNestedProofs___closed__1; +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); @@ -51,6 +51,7 @@ static lean_object* l___private_Lean_Meta_AbstractNestedProofs_0__Lean_Meta_Abst lean_object* l_Std_mkHashMapImp___rarg(lean_object*); lean_object* l_Std_PersistentArray_set___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_setValue(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); @@ -60,15 +61,14 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_AbstractNestedProofs_0__Lean_Meta LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_AbstractNestedProofs_visit___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AbstractNestedProofs_0__Lean_Meta_AbstractNestedProofs_mkAuxLemma(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_fvarId(lean_object*); static lean_object* l___private_Lean_Meta_AbstractNestedProofs_0__Lean_Meta_AbstractNestedProofs_mkAuxLemma___closed__1; lean_object* l_Lean_LocalDecl_type(lean_object*); lean_object* l_Lean_LocalDecl_value_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLCtx___at_Lean_Meta_AbstractNestedProofs_visit___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_LocalDecl_index(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_AbstractNestedProofs_visit___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_AbstractNestedProofs_visit___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaLetTelescope___at_Lean_Meta_AbstractNestedProofs_visit___spec__6___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*); @@ -90,6 +90,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_AbstractNestedProofs_visit___lambda__1___bo lean_object* l___private_Lean_MonadEnv_0__Lean_mkAuxNameAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Meta_AbstractNestedProofs_visit___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_AbstractNestedProofs_visit___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_setType(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at_Lean_Meta_AbstractNestedProofs_visit___spec__7(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -292,7 +293,7 @@ x_18 = lean_ctor_get(x_7, 1); lean_inc(x_18); lean_dec(x_7); x_19 = lean_unsigned_to_nat(0u); -x_20 = l_Lean_Expr_getAppNumArgsAux(x_1, x_19); +x_20 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_19); x_21 = l_Lean_Meta_AbstractNestedProofs_isNonTrivialProof___closed__1; lean_inc(x_20); x_22 = lean_mk_array(x_20, x_21); @@ -1488,7 +1489,7 @@ x_35 = lean_ctor_get(x_32, 1); lean_inc(x_35); lean_dec(x_32); x_36 = lean_unsigned_to_nat(0u); -x_37 = l_Lean_Expr_getAppNumArgsAux(x_1, x_36); +x_37 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_36); x_38 = l_Lean_Meta_AbstractNestedProofs_isNonTrivialProof___closed__1; lean_inc(x_37); x_39 = lean_mk_array(x_37, x_38); @@ -1686,177 +1687,223 @@ return x_75; } case 10: { -lean_object* x_76; lean_object* x_77; lean_object* x_78; +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; x_76 = lean_ctor_get(x_32, 1); lean_inc(x_76); lean_dec(x_32); -x_77 = lean_ctor_get(x_1, 1); +x_77 = lean_ctor_get(x_1, 0); lean_inc(x_77); +x_78 = lean_ctor_get(x_1, 1); +lean_inc(x_78); lean_inc(x_8); lean_inc(x_3); -x_78 = l_Lean_Meta_AbstractNestedProofs_visit(x_77, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_76); -if (lean_obj_tag(x_78) == 0) +lean_inc(x_78); +x_79 = l_Lean_Meta_AbstractNestedProofs_visit(x_78, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_76); +if (lean_obj_tag(x_79) == 0) { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); +lean_object* x_80; lean_object* x_81; size_t x_82; size_t x_83; uint8_t x_84; +x_80 = lean_ctor_get(x_79, 0); lean_inc(x_80); +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +lean_dec(x_79); +x_82 = lean_ptr_addr(x_78); lean_dec(x_78); +x_83 = lean_ptr_addr(x_80); +x_84 = lean_usize_dec_eq(x_82, x_83); +if (x_84 == 0) +{ +lean_object* x_85; +x_85 = l_Lean_Expr_mdata___override(x_77, x_80); +x_18 = x_85; +x_19 = x_81; +goto block_31; +} +else +{ +lean_dec(x_80); +lean_dec(x_77); lean_inc(x_1); -x_81 = lean_expr_update_mdata(x_1, x_79); -x_18 = x_81; -x_19 = x_80; +x_18 = x_1; +x_19 = x_81; goto block_31; } +} else { -uint8_t x_82; +uint8_t x_86; +lean_dec(x_78); +lean_dec(x_77); lean_dec(x_8); lean_dec(x_3); lean_dec(x_1); -x_82 = !lean_is_exclusive(x_78); -if (x_82 == 0) +x_86 = !lean_is_exclusive(x_79); +if (x_86 == 0) { -return x_78; +return x_79; } else { -lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_83 = lean_ctor_get(x_78, 0); -x_84 = lean_ctor_get(x_78, 1); -lean_inc(x_84); -lean_inc(x_83); -lean_dec(x_78); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -return x_85; +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_79, 0); +x_88 = lean_ctor_get(x_79, 1); +lean_inc(x_88); +lean_inc(x_87); +lean_dec(x_79); +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; } } } case 11: { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_32, 1); -lean_inc(x_86); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_90 = lean_ctor_get(x_32, 1); +lean_inc(x_90); lean_dec(x_32); -x_87 = lean_ctor_get(x_1, 2); -lean_inc(x_87); +x_91 = lean_ctor_get(x_1, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_1, 1); +lean_inc(x_92); +x_93 = lean_ctor_get(x_1, 2); +lean_inc(x_93); lean_inc(x_8); lean_inc(x_3); -x_88 = l_Lean_Meta_AbstractNestedProofs_visit(x_87, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_86); -if (lean_obj_tag(x_88) == 0) +lean_inc(x_93); +x_94 = l_Lean_Meta_AbstractNestedProofs_visit(x_93, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_90); +if (lean_obj_tag(x_94) == 0) { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -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); +lean_object* x_95; lean_object* x_96; size_t x_97; size_t x_98; uint8_t x_99; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +lean_dec(x_94); +x_97 = lean_ptr_addr(x_93); +lean_dec(x_93); +x_98 = lean_ptr_addr(x_95); +x_99 = lean_usize_dec_eq(x_97, x_98); +if (x_99 == 0) +{ +lean_object* x_100; +x_100 = l_Lean_Expr_proj___override(x_91, x_92, x_95); +x_18 = x_100; +x_19 = x_96; +goto block_31; +} +else +{ +lean_dec(x_95); +lean_dec(x_92); +lean_dec(x_91); lean_inc(x_1); -x_91 = lean_expr_update_proj(x_1, x_89); -x_18 = x_91; -x_19 = x_90; +x_18 = x_1; +x_19 = x_96; goto block_31; } +} else { -uint8_t x_92; +uint8_t x_101; +lean_dec(x_93); +lean_dec(x_92); +lean_dec(x_91); lean_dec(x_8); lean_dec(x_3); lean_dec(x_1); -x_92 = !lean_is_exclusive(x_88); -if (x_92 == 0) +x_101 = !lean_is_exclusive(x_94); +if (x_101 == 0) { -return x_88; +return x_94; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_88, 0); -x_94 = lean_ctor_get(x_88, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_88); -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -return x_95; +lean_object* x_102; lean_object* x_103; lean_object* x_104; +x_102 = lean_ctor_get(x_94, 0); +x_103 = lean_ctor_get(x_94, 1); +lean_inc(x_103); +lean_inc(x_102); +lean_dec(x_94); +x_104 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +return x_104; } } } default: { -lean_object* x_96; +lean_object* x_105; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_96 = lean_ctor_get(x_32, 1); -lean_inc(x_96); +x_105 = lean_ctor_get(x_32, 1); +lean_inc(x_105); lean_dec(x_32); lean_inc(x_1); x_18 = x_1; -x_19 = x_96; +x_19 = x_105; goto block_31; } } } else { -lean_object* x_97; lean_object* x_98; -x_97 = lean_ctor_get(x_32, 1); -lean_inc(x_97); +lean_object* x_106; lean_object* x_107; +x_106 = lean_ctor_get(x_32, 1); +lean_inc(x_106); lean_dec(x_32); lean_inc(x_8); lean_inc(x_1); -x_98 = l___private_Lean_Meta_AbstractNestedProofs_0__Lean_Meta_AbstractNestedProofs_mkAuxLemma(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_97); +x_107 = l___private_Lean_Meta_AbstractNestedProofs_0__Lean_Meta_AbstractNestedProofs_mkAuxLemma(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_106); lean_dec(x_4); lean_dec(x_2); -if (lean_obj_tag(x_98) == 0) -{ -lean_object* x_99; lean_object* x_100; -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -x_100 = lean_ctor_get(x_98, 1); -lean_inc(x_100); -lean_dec(x_98); -x_18 = x_99; -x_19 = x_100; +if (lean_obj_tag(x_107) == 0) +{ +lean_object* x_108; lean_object* x_109; +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +x_18 = x_108; +x_19 = x_109; goto block_31; } else { -uint8_t x_101; +uint8_t x_110; lean_dec(x_8); lean_dec(x_3); lean_dec(x_1); -x_101 = !lean_is_exclusive(x_98); -if (x_101 == 0) +x_110 = !lean_is_exclusive(x_107); +if (x_110 == 0) { -return x_98; +return x_107; } else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_102 = lean_ctor_get(x_98, 0); -x_103 = lean_ctor_get(x_98, 1); -lean_inc(x_103); -lean_inc(x_102); -lean_dec(x_98); -x_104 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_104, 0, x_102); -lean_ctor_set(x_104, 1, x_103); -return x_104; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_107, 0); +x_112 = lean_ctor_get(x_107, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_107); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } } else { -uint8_t x_105; +uint8_t x_114; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -1865,23 +1912,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_105 = !lean_is_exclusive(x_32); -if (x_105 == 0) +x_114 = !lean_is_exclusive(x_32); +if (x_114 == 0) { return x_32; } else { -lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_106 = lean_ctor_get(x_32, 0); -x_107 = lean_ctor_get(x_32, 1); -lean_inc(x_107); -lean_inc(x_106); +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_32, 0); +x_116 = lean_ctor_get(x_32, 1); +lean_inc(x_116); +lean_inc(x_115); lean_dec(x_32); -x_108 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_108, 0, x_106); -lean_ctor_set(x_108, 1, x_107); -return x_108; +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } block_31: @@ -1926,7 +1973,7 @@ return x_30; } else { -lean_object* x_109; +lean_object* x_118; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -1935,111 +1982,60 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_109 = lean_ctor_get(x_17, 0); -lean_inc(x_109); +x_118 = lean_ctor_get(x_17, 0); +lean_inc(x_118); lean_dec(x_17); -lean_ctor_set(x_13, 0, x_109); +lean_ctor_set(x_13, 0, x_118); return x_13; } } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = lean_ctor_get(x_13, 0); -x_111 = lean_ctor_get(x_13, 1); -lean_inc(x_111); -lean_inc(x_110); +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_ctor_get(x_13, 0); +x_120 = lean_ctor_get(x_13, 1); +lean_inc(x_120); +lean_inc(x_119); lean_dec(x_13); lean_inc(x_1); -x_112 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_110, x_1); -if (lean_obj_tag(x_112) == 0) +x_121 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_119, x_1); +if (lean_obj_tag(x_121) == 0) { -lean_object* x_113; lean_object* x_114; lean_object* x_126; +lean_object* x_122; lean_object* x_123; lean_object* x_135; lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_1); -x_126 = l_Lean_Meta_AbstractNestedProofs_isNonTrivialProof(x_1, x_5, x_6, x_7, x_8, x_111); -if (lean_obj_tag(x_126) == 0) +x_135 = l_Lean_Meta_AbstractNestedProofs_isNonTrivialProof(x_1, x_5, x_6, x_7, x_8, x_120); +if (lean_obj_tag(x_135) == 0) { -lean_object* x_127; uint8_t x_128; -x_127 = lean_ctor_get(x_126, 0); -lean_inc(x_127); -x_128 = lean_unbox(x_127); -lean_dec(x_127); -if (x_128 == 0) +lean_object* x_136; uint8_t x_137; +x_136 = lean_ctor_get(x_135, 0); +lean_inc(x_136); +x_137 = lean_unbox(x_136); +lean_dec(x_136); +if (x_137 == 0) { switch (lean_obj_tag(x_1)) { case 5: { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; -x_129 = lean_ctor_get(x_126, 1); -lean_inc(x_129); -lean_dec(x_126); -x_130 = lean_unsigned_to_nat(0u); -x_131 = l_Lean_Expr_getAppNumArgsAux(x_1, x_130); -x_132 = l_Lean_Meta_AbstractNestedProofs_isNonTrivialProof___closed__1; -lean_inc(x_131); -x_133 = lean_mk_array(x_131, x_132); -x_134 = lean_unsigned_to_nat(1u); -x_135 = lean_nat_sub(x_131, x_134); -lean_dec(x_131); -lean_inc(x_8); -lean_inc(x_3); -lean_inc(x_1); -x_136 = l_Lean_Expr_withAppAux___at_Lean_Meta_AbstractNestedProofs_visit___spec__2(x_1, x_133, x_135, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_129); -if (lean_obj_tag(x_136) == 0) -{ -lean_object* x_137; lean_object* x_138; -x_137 = lean_ctor_get(x_136, 0); -lean_inc(x_137); -x_138 = lean_ctor_get(x_136, 1); +lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_138 = lean_ctor_get(x_135, 1); lean_inc(x_138); -lean_dec(x_136); -x_113 = x_137; -x_114 = x_138; -goto block_125; -} -else -{ -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; -lean_dec(x_8); -lean_dec(x_3); -lean_dec(x_1); -x_139 = lean_ctor_get(x_136, 0); -lean_inc(x_139); -x_140 = lean_ctor_get(x_136, 1); +lean_dec(x_135); +x_139 = lean_unsigned_to_nat(0u); +x_140 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_139); +x_141 = l_Lean_Meta_AbstractNestedProofs_isNonTrivialProof___closed__1; lean_inc(x_140); -if (lean_is_exclusive(x_136)) { - lean_ctor_release(x_136, 0); - lean_ctor_release(x_136, 1); - x_141 = x_136; -} else { - lean_dec_ref(x_136); - x_141 = lean_box(0); -} -if (lean_is_scalar(x_141)) { - x_142 = lean_alloc_ctor(1, 2, 0); -} else { - x_142 = x_141; -} -lean_ctor_set(x_142, 0, x_139); -lean_ctor_set(x_142, 1, x_140); -return x_142; -} -} -case 6: -{ -lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_143 = lean_ctor_get(x_126, 1); -lean_inc(x_143); -lean_dec(x_126); -x_144 = l_Lean_Meta_AbstractNestedProofs_visit___closed__1; +x_142 = lean_mk_array(x_140, x_141); +x_143 = lean_unsigned_to_nat(1u); +x_144 = lean_nat_sub(x_140, x_143); +lean_dec(x_140); lean_inc(x_8); lean_inc(x_3); lean_inc(x_1); -x_145 = l_Lean_Meta_lambdaLetTelescope___at_Lean_Meta_AbstractNestedProofs_visit___spec__6___rarg(x_1, x_144, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_143); +x_145 = l_Lean_Expr_withAppAux___at_Lean_Meta_AbstractNestedProofs_visit___spec__2(x_1, x_142, x_144, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_138); if (lean_obj_tag(x_145) == 0) { lean_object* x_146; lean_object* x_147; @@ -2048,9 +2044,9 @@ lean_inc(x_146); x_147 = lean_ctor_get(x_145, 1); lean_inc(x_147); lean_dec(x_145); -x_113 = x_146; -x_114 = x_147; -goto block_125; +x_122 = x_146; +x_123 = x_147; +goto block_134; } else { @@ -2080,17 +2076,17 @@ lean_ctor_set(x_151, 1, x_149); return x_151; } } -case 7: +case 6: { lean_object* x_152; lean_object* x_153; lean_object* x_154; -x_152 = lean_ctor_get(x_126, 1); +x_152 = lean_ctor_get(x_135, 1); lean_inc(x_152); -lean_dec(x_126); -x_153 = l_Lean_Meta_AbstractNestedProofs_visit___closed__2; +lean_dec(x_135); +x_153 = l_Lean_Meta_AbstractNestedProofs_visit___closed__1; lean_inc(x_8); lean_inc(x_3); lean_inc(x_1); -x_154 = l_Lean_Meta_forallTelescope___at_Lean_Meta_AbstractNestedProofs_visit___spec__7___rarg(x_1, x_153, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_152); +x_154 = l_Lean_Meta_lambdaLetTelescope___at_Lean_Meta_AbstractNestedProofs_visit___spec__6___rarg(x_1, x_153, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_152); if (lean_obj_tag(x_154) == 0) { lean_object* x_155; lean_object* x_156; @@ -2099,9 +2095,9 @@ lean_inc(x_155); x_156 = lean_ctor_get(x_154, 1); lean_inc(x_156); lean_dec(x_154); -x_113 = x_155; -x_114 = x_156; -goto block_125; +x_122 = x_155; +x_123 = x_156; +goto block_134; } else { @@ -2131,17 +2127,17 @@ lean_ctor_set(x_160, 1, x_158); return x_160; } } -case 8: +case 7: { lean_object* x_161; lean_object* x_162; lean_object* x_163; -x_161 = lean_ctor_get(x_126, 1); +x_161 = lean_ctor_get(x_135, 1); lean_inc(x_161); -lean_dec(x_126); -x_162 = l_Lean_Meta_AbstractNestedProofs_visit___closed__1; +lean_dec(x_135); +x_162 = l_Lean_Meta_AbstractNestedProofs_visit___closed__2; lean_inc(x_8); lean_inc(x_3); lean_inc(x_1); -x_163 = l_Lean_Meta_lambdaLetTelescope___at_Lean_Meta_AbstractNestedProofs_visit___spec__6___rarg(x_1, x_162, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_161); +x_163 = l_Lean_Meta_forallTelescope___at_Lean_Meta_AbstractNestedProofs_visit___spec__7___rarg(x_1, x_162, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_161); if (lean_obj_tag(x_163) == 0) { lean_object* x_164; lean_object* x_165; @@ -2150,9 +2146,9 @@ lean_inc(x_164); x_165 = lean_ctor_get(x_163, 1); lean_inc(x_165); lean_dec(x_163); -x_113 = x_164; -x_114 = x_165; -goto block_125; +x_122 = x_164; +x_123 = x_165; +goto block_134; } else { @@ -2182,185 +2178,282 @@ lean_ctor_set(x_169, 1, x_167); return x_169; } } -case 10: +case 8: { lean_object* x_170; lean_object* x_171; lean_object* x_172; -x_170 = lean_ctor_get(x_126, 1); +x_170 = lean_ctor_get(x_135, 1); lean_inc(x_170); -lean_dec(x_126); -x_171 = lean_ctor_get(x_1, 1); -lean_inc(x_171); +lean_dec(x_135); +x_171 = l_Lean_Meta_AbstractNestedProofs_visit___closed__1; lean_inc(x_8); lean_inc(x_3); -x_172 = l_Lean_Meta_AbstractNestedProofs_visit(x_171, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_170); +lean_inc(x_1); +x_172 = l_Lean_Meta_lambdaLetTelescope___at_Lean_Meta_AbstractNestedProofs_visit___spec__6___rarg(x_1, x_171, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_170); if (lean_obj_tag(x_172) == 0) { -lean_object* x_173; lean_object* x_174; lean_object* x_175; +lean_object* x_173; lean_object* x_174; x_173 = lean_ctor_get(x_172, 0); lean_inc(x_173); x_174 = lean_ctor_get(x_172, 1); lean_inc(x_174); lean_dec(x_172); -lean_inc(x_1); -x_175 = lean_expr_update_mdata(x_1, x_173); -x_113 = x_175; -x_114 = x_174; -goto block_125; +x_122 = x_173; +x_123 = x_174; +goto block_134; } else { -lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_dec(x_8); lean_dec(x_3); lean_dec(x_1); -x_176 = lean_ctor_get(x_172, 0); +x_175 = lean_ctor_get(x_172, 0); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 1); lean_inc(x_176); -x_177 = lean_ctor_get(x_172, 1); -lean_inc(x_177); if (lean_is_exclusive(x_172)) { lean_ctor_release(x_172, 0); lean_ctor_release(x_172, 1); - x_178 = x_172; + x_177 = x_172; } else { lean_dec_ref(x_172); - x_178 = lean_box(0); + x_177 = lean_box(0); } -if (lean_is_scalar(x_178)) { - x_179 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_177)) { + x_178 = lean_alloc_ctor(1, 2, 0); } else { - x_179 = x_178; + x_178 = x_177; } -lean_ctor_set(x_179, 0, x_176); -lean_ctor_set(x_179, 1, x_177); -return x_179; +lean_ctor_set(x_178, 0, x_175); +lean_ctor_set(x_178, 1, x_176); +return x_178; } } -case 11: +case 10: { -lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_180 = lean_ctor_get(x_126, 1); +lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_179 = lean_ctor_get(x_135, 1); +lean_inc(x_179); +lean_dec(x_135); +x_180 = lean_ctor_get(x_1, 0); lean_inc(x_180); -lean_dec(x_126); -x_181 = lean_ctor_get(x_1, 2); +x_181 = lean_ctor_get(x_1, 1); lean_inc(x_181); lean_inc(x_8); lean_inc(x_3); -x_182 = l_Lean_Meta_AbstractNestedProofs_visit(x_181, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_180); +lean_inc(x_181); +x_182 = l_Lean_Meta_AbstractNestedProofs_visit(x_181, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_179); if (lean_obj_tag(x_182) == 0) { -lean_object* x_183; lean_object* x_184; lean_object* x_185; +lean_object* x_183; lean_object* x_184; size_t x_185; size_t x_186; uint8_t x_187; x_183 = lean_ctor_get(x_182, 0); lean_inc(x_183); x_184 = lean_ctor_get(x_182, 1); lean_inc(x_184); lean_dec(x_182); +x_185 = lean_ptr_addr(x_181); +lean_dec(x_181); +x_186 = lean_ptr_addr(x_183); +x_187 = lean_usize_dec_eq(x_185, x_186); +if (x_187 == 0) +{ +lean_object* x_188; +x_188 = l_Lean_Expr_mdata___override(x_180, x_183); +x_122 = x_188; +x_123 = x_184; +goto block_134; +} +else +{ +lean_dec(x_183); +lean_dec(x_180); lean_inc(x_1); -x_185 = lean_expr_update_proj(x_1, x_183); -x_113 = x_185; -x_114 = x_184; -goto block_125; +x_122 = x_1; +x_123 = x_184; +goto block_134; +} } else { -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; +lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; +lean_dec(x_181); +lean_dec(x_180); lean_dec(x_8); lean_dec(x_3); lean_dec(x_1); -x_186 = lean_ctor_get(x_182, 0); -lean_inc(x_186); -x_187 = lean_ctor_get(x_182, 1); -lean_inc(x_187); +x_189 = lean_ctor_get(x_182, 0); +lean_inc(x_189); +x_190 = lean_ctor_get(x_182, 1); +lean_inc(x_190); if (lean_is_exclusive(x_182)) { lean_ctor_release(x_182, 0); lean_ctor_release(x_182, 1); - x_188 = x_182; + x_191 = x_182; } else { lean_dec_ref(x_182); - x_188 = lean_box(0); + x_191 = lean_box(0); } -if (lean_is_scalar(x_188)) { - x_189 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_191)) { + x_192 = lean_alloc_ctor(1, 2, 0); } else { - x_189 = x_188; + x_192 = x_191; } -lean_ctor_set(x_189, 0, x_186); -lean_ctor_set(x_189, 1, x_187); -return x_189; +lean_ctor_set(x_192, 0, x_189); +lean_ctor_set(x_192, 1, x_190); +return x_192; +} +} +case 11: +{ +lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; +x_193 = lean_ctor_get(x_135, 1); +lean_inc(x_193); +lean_dec(x_135); +x_194 = lean_ctor_get(x_1, 0); +lean_inc(x_194); +x_195 = lean_ctor_get(x_1, 1); +lean_inc(x_195); +x_196 = lean_ctor_get(x_1, 2); +lean_inc(x_196); +lean_inc(x_8); +lean_inc(x_3); +lean_inc(x_196); +x_197 = l_Lean_Meta_AbstractNestedProofs_visit(x_196, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_193); +if (lean_obj_tag(x_197) == 0) +{ +lean_object* x_198; lean_object* x_199; size_t x_200; size_t x_201; uint8_t x_202; +x_198 = lean_ctor_get(x_197, 0); +lean_inc(x_198); +x_199 = lean_ctor_get(x_197, 1); +lean_inc(x_199); +lean_dec(x_197); +x_200 = lean_ptr_addr(x_196); +lean_dec(x_196); +x_201 = lean_ptr_addr(x_198); +x_202 = lean_usize_dec_eq(x_200, x_201); +if (x_202 == 0) +{ +lean_object* x_203; +x_203 = l_Lean_Expr_proj___override(x_194, x_195, x_198); +x_122 = x_203; +x_123 = x_199; +goto block_134; +} +else +{ +lean_dec(x_198); +lean_dec(x_195); +lean_dec(x_194); +lean_inc(x_1); +x_122 = x_1; +x_123 = x_199; +goto block_134; +} +} +else +{ +lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; +lean_dec(x_196); +lean_dec(x_195); +lean_dec(x_194); +lean_dec(x_8); +lean_dec(x_3); +lean_dec(x_1); +x_204 = lean_ctor_get(x_197, 0); +lean_inc(x_204); +x_205 = lean_ctor_get(x_197, 1); +lean_inc(x_205); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + lean_ctor_release(x_197, 1); + x_206 = x_197; +} else { + lean_dec_ref(x_197); + x_206 = lean_box(0); +} +if (lean_is_scalar(x_206)) { + x_207 = lean_alloc_ctor(1, 2, 0); +} else { + x_207 = x_206; +} +lean_ctor_set(x_207, 0, x_204); +lean_ctor_set(x_207, 1, x_205); +return x_207; } } default: { -lean_object* x_190; +lean_object* x_208; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_190 = lean_ctor_get(x_126, 1); -lean_inc(x_190); -lean_dec(x_126); +x_208 = lean_ctor_get(x_135, 1); +lean_inc(x_208); +lean_dec(x_135); lean_inc(x_1); -x_113 = x_1; -x_114 = x_190; -goto block_125; +x_122 = x_1; +x_123 = x_208; +goto block_134; } } } else { -lean_object* x_191; lean_object* x_192; -x_191 = lean_ctor_get(x_126, 1); -lean_inc(x_191); -lean_dec(x_126); +lean_object* x_209; lean_object* x_210; +x_209 = lean_ctor_get(x_135, 1); +lean_inc(x_209); +lean_dec(x_135); lean_inc(x_8); lean_inc(x_1); -x_192 = l___private_Lean_Meta_AbstractNestedProofs_0__Lean_Meta_AbstractNestedProofs_mkAuxLemma(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_191); +x_210 = l___private_Lean_Meta_AbstractNestedProofs_0__Lean_Meta_AbstractNestedProofs_mkAuxLemma(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_209); lean_dec(x_4); lean_dec(x_2); -if (lean_obj_tag(x_192) == 0) +if (lean_obj_tag(x_210) == 0) { -lean_object* x_193; lean_object* x_194; -x_193 = lean_ctor_get(x_192, 0); -lean_inc(x_193); -x_194 = lean_ctor_get(x_192, 1); -lean_inc(x_194); -lean_dec(x_192); -x_113 = x_193; -x_114 = x_194; -goto block_125; +lean_object* x_211; lean_object* x_212; +x_211 = lean_ctor_get(x_210, 0); +lean_inc(x_211); +x_212 = lean_ctor_get(x_210, 1); +lean_inc(x_212); +lean_dec(x_210); +x_122 = x_211; +x_123 = x_212; +goto block_134; } else { -lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_dec(x_8); lean_dec(x_3); lean_dec(x_1); -x_195 = lean_ctor_get(x_192, 0); -lean_inc(x_195); -x_196 = lean_ctor_get(x_192, 1); -lean_inc(x_196); -if (lean_is_exclusive(x_192)) { - lean_ctor_release(x_192, 0); - lean_ctor_release(x_192, 1); - x_197 = x_192; +x_213 = lean_ctor_get(x_210, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_210, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_210)) { + lean_ctor_release(x_210, 0); + lean_ctor_release(x_210, 1); + x_215 = x_210; } else { - lean_dec_ref(x_192); - x_197 = lean_box(0); + lean_dec_ref(x_210); + x_215 = lean_box(0); } -if (lean_is_scalar(x_197)) { - x_198 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); } else { - x_198 = x_197; + x_216 = x_215; } -lean_ctor_set(x_198, 0, x_195); -lean_ctor_set(x_198, 1, x_196); -return x_198; +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; } } } else { -lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2369,68 +2462,68 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_199 = lean_ctor_get(x_126, 0); -lean_inc(x_199); -x_200 = lean_ctor_get(x_126, 1); -lean_inc(x_200); -if (lean_is_exclusive(x_126)) { - lean_ctor_release(x_126, 0); - lean_ctor_release(x_126, 1); - x_201 = x_126; +x_217 = lean_ctor_get(x_135, 0); +lean_inc(x_217); +x_218 = lean_ctor_get(x_135, 1); +lean_inc(x_218); +if (lean_is_exclusive(x_135)) { + lean_ctor_release(x_135, 0); + lean_ctor_release(x_135, 1); + x_219 = x_135; } else { - lean_dec_ref(x_126); - x_201 = lean_box(0); + lean_dec_ref(x_135); + x_219 = lean_box(0); } -if (lean_is_scalar(x_201)) { - x_202 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_219)) { + x_220 = lean_alloc_ctor(1, 2, 0); } else { - x_202 = x_201; + x_220 = x_219; } -lean_ctor_set(x_202, 0, x_199); -lean_ctor_set(x_202, 1, x_200); -return x_202; +lean_ctor_set(x_220, 0, x_217); +lean_ctor_set(x_220, 1, x_218); +return x_220; } -block_125: +block_134: { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_115 = lean_st_ref_get(x_8, x_114); +lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_124 = lean_st_ref_get(x_8, x_123); lean_dec(x_8); -x_116 = lean_ctor_get(x_115, 1); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_st_ref_take(x_3, x_116); -x_118 = lean_ctor_get(x_117, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_117, 1); -lean_inc(x_119); -lean_dec(x_117); -lean_inc(x_113); -x_120 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_118, x_1, x_113); -x_121 = lean_st_ref_set(x_3, x_120, x_119); -lean_dec(x_3); -x_122 = lean_ctor_get(x_121, 1); +x_125 = lean_ctor_get(x_124, 1); +lean_inc(x_125); +lean_dec(x_124); +x_126 = lean_st_ref_take(x_3, x_125); +x_127 = lean_ctor_get(x_126, 0); +lean_inc(x_127); +x_128 = lean_ctor_get(x_126, 1); +lean_inc(x_128); +lean_dec(x_126); lean_inc(x_122); -if (lean_is_exclusive(x_121)) { - lean_ctor_release(x_121, 0); - lean_ctor_release(x_121, 1); - x_123 = x_121; +x_129 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_127, x_1, x_122); +x_130 = lean_st_ref_set(x_3, x_129, x_128); +lean_dec(x_3); +x_131 = lean_ctor_get(x_130, 1); +lean_inc(x_131); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_132 = x_130; } else { - lean_dec_ref(x_121); - x_123 = lean_box(0); + lean_dec_ref(x_130); + x_132 = lean_box(0); } -if (lean_is_scalar(x_123)) { - x_124 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_132)) { + x_133 = lean_alloc_ctor(0, 2, 0); } else { - x_124 = x_123; + x_133 = x_132; } -lean_ctor_set(x_124, 0, x_113); -lean_ctor_set(x_124, 1, x_122); -return x_124; +lean_ctor_set(x_133, 0, x_122); +lean_ctor_set(x_133, 1, x_131); +return x_133; } } else { -lean_object* x_203; lean_object* x_204; +lean_object* x_221; lean_object* x_222; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2439,19 +2532,19 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_203 = lean_ctor_get(x_112, 0); -lean_inc(x_203); -lean_dec(x_112); -x_204 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_204, 0, x_203); -lean_ctor_set(x_204, 1, x_111); -return x_204; +x_221 = lean_ctor_get(x_121, 0); +lean_inc(x_221); +lean_dec(x_121); +x_222 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_222, 0, x_221); +lean_ctor_set(x_222, 1, x_120); +return x_222; } } } else { -lean_object* x_205; +lean_object* x_223; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2459,10 +2552,10 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_205 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_205, 0, x_1); -lean_ctor_set(x_205, 1, x_9); -return x_205; +x_223 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_223, 0, x_1); +lean_ctor_set(x_223, 1, x_9); +return x_223; } } } diff --git a/stage0/stdlib/Lean/Meta/AppBuilder.c b/stage0/stdlib/Lean/Meta/AppBuilder.c index 8394457606ce..682cdd4d9160 100644 --- a/stage0/stdlib/Lean/Meta/AppBuilder.c +++ b/stage0/stdlib/Lean/Meta/AppBuilder.c @@ -195,6 +195,7 @@ static lean_object* l_Lean_Meta_mkNoConfusion___closed__2; static lean_object* l_Lean_Meta_mkEqRec___closed__2; static lean_object* l_Lean_Meta_mkNoConfusion___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_mkId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkDecideProof___closed__4; static lean_object* l_Lean_Meta_mkListLit___closed__2; LEAN_EXPORT lean_object* l_List_mapM___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkFun___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -287,7 +288,6 @@ static lean_object* l_Lean_Meta_mkNoConfusion___closed__5; static lean_object* l_Lean_Meta_mkAppM___lambda__1___closed__4; lean_object* l_Lean_Meta_trySynthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAppOptM___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkListLit___closed__3; lean_object* l___private_Lean_Util_Trace_0__Lean_addNode___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -4971,7 +4971,7 @@ static lean_object* _init_l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMAr lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs_loop___closed__10; x_2 = l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs_loop___closed__11; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs_loop___closed__12; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -11496,7 +11496,7 @@ lean_ctor_set(x_52, 0, x_47); lean_ctor_set(x_52, 1, x_32); x_53 = l_Lean_Expr_const___override(x_51, x_52); x_54 = lean_unsigned_to_nat(0u); -x_55 = l_Lean_Expr_getAppNumArgsAux(x_28, x_54); +x_55 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_28, x_54); x_56 = l_Lean_Meta_mkNoConfusion___closed__9; lean_inc(x_55); x_57 = lean_mk_array(x_55, x_56); @@ -11535,7 +11535,7 @@ lean_ctor_set(x_74, 0, x_68); lean_ctor_set(x_74, 1, x_32); x_75 = l_Lean_Expr_const___override(x_73, x_74); x_76 = lean_unsigned_to_nat(0u); -x_77 = l_Lean_Expr_getAppNumArgsAux(x_28, x_76); +x_77 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_28, x_76); x_78 = l_Lean_Meta_mkNoConfusion___closed__9; lean_inc(x_77); x_79 = lean_mk_array(x_77, x_78); @@ -12311,7 +12311,7 @@ x_47 = lean_ctor_get(x_13, 0); lean_inc(x_47); lean_dec(x_13); x_48 = lean_unsigned_to_nat(0u); -x_49 = l_Lean_Expr_getAppNumArgsAux(x_5, x_48); +x_49 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_48); x_50 = l_Lean_Meta_mkNoConfusion___closed__9; lean_inc(x_49); x_51 = lean_mk_array(x_49, x_50); diff --git a/stage0/stdlib/Lean/Meta/Basic.c b/stage0/stdlib/Lean/Meta/Basic.c index 502831de8240..366cef368a5d 100644 --- a/stage0/stdlib/Lean/Meta/Basic.c +++ b/stage0/stdlib/Lean/Meta/Basic.c @@ -48,7 +48,6 @@ static lean_object* l_Lean_Meta_instInhabitedParamInfo___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_etaExpand___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Meta_TransparencyMode_hash(uint8_t); lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__3; lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT uint64_t l_Lean_Meta_InfoCacheKey_instHashableInfoCacheKey(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalInstances___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -94,6 +93,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallMetaTele static lean_object* l_Lean_Meta_instInhabitedSavedState___closed__10; static lean_object* l_Lean_Meta_isExprDefEq___closed__2; static lean_object* l_Lean_Meta_instMonadMetaM___closed__2; +lean_object* l_Lean_Level_succ___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_withIncRecDepth___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_savingCache(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkConstWithFreshMVarLevels(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -123,6 +123,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getP LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_sortFVarIds___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_restore(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_instOrElseMetaM___closed__1; +LEAN_EXPORT uint8_t l_Lean_Meta_ParamInfo_higherOrderOutParam___default; LEAN_EXPORT lean_object* l_Lean_Meta_resetZetaFVarIds___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_saveState___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -212,6 +213,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_checkpointDefEq___at_Lean_Meta_isLevelDefEq LEAN_EXPORT lean_object* l_Lean_Meta_instInhabitedPostponedEntry; LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withNewLocalInstancesImpAux(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_approxDefEqImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isSyntheticMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__10(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -238,7 +240,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_forallMetaBoundedTelescope(lean_object*, le LEAN_EXPORT lean_object* l_Lean_Meta_instMonadEnvMetaM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux_process___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_isClassExpensive_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(uint8_t, uint8_t); +uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(uint8_t, uint8_t); static lean_object* l_Lean_Meta_instAlternativeMetaM___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_setInlineAttribute___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withConfig___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -255,7 +257,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_modifyInferTypeCache(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getPostponed___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_sortFVarIds___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_4_(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getPostponed___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -285,6 +287,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVa LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_liftMkBindingM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___lambda__1___boxed(lean_object*, lean_object*); +lean_object* l_Lean_simpLevelIMax_x27(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_State_mctx___default___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD(lean_object*); static lean_object* l_Lean_Meta_Context_lctx___default___closed__1; @@ -298,7 +301,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate(lean_object*, lean_obj LEAN_EXPORT lean_object* l_Lean_Meta_getConfig___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuickConst_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_throwUnknownFVar___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_normalizeLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_shouldReduceAll(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -381,8 +383,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMCtxImp(le LEAN_EXPORT lean_object* l_Lean_Meta_withNewMCtxDepth___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withNewFVar___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_collectForwardDeps___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__1; -lean_object* lean_level_update_max(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_getLevelMVarDepth___closed__1; uint8_t l_Lean_Level_any(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshMVarId___at_Lean_Meta_mkFreshExprMVarAt___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -394,6 +394,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_Basic LEAN_EXPORT lean_object* l_Lean_Meta_isDefEqStuckExceptionId; LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Trace_0__Lean_addNode___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__13___closed__2; +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_4____closed__2; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkArrow___closed__2; @@ -401,6 +402,7 @@ lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Cache_defEqDefault___default; LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_getDefInfoTemp___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_simpLevelMax_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getLevelMVarDepth___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos(lean_object*); @@ -413,7 +415,6 @@ static lean_object* l_Lean_Meta_instMonadMetaM___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_mapMetaM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_throwIsDefEqStuck___rarg(lean_object*); static lean_object* l_Lean_Meta_instMonadBacktrackSavedStateMetaM___closed__2; static lean_object* l_Lean_Meta_instAddMessageContextMetaM___closed__1; @@ -424,6 +425,7 @@ static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageC lean_object* l_Lean_MetavarContext_MkBinding_elimMVarDeps(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_instMetaEvalMetaM___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_abstractRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); static lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux___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___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp(lean_object*); @@ -451,6 +453,7 @@ LEAN_EXPORT uint8_t l_List_foldr___at___private_Lean_Meta_Basic_0__Lean_Meta_exp LEAN_EXPORT lean_object* l_Lean_Meta_withReducibleAndInstances___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____boxed(lean_object*, lean_object*); lean_object* l_Lean_MetavarContext_elimMVarDeps(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_ParamInfo_isInstImplicit(lean_object*); @@ -467,7 +470,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_instantiateLambda___boxed(lean_object*, lea LEAN_EXPORT lean_object* l_Lean_Meta_resettingSynthInstanceCacheWhen___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); extern lean_object* l_Lean_Expr_instHashableExpr; uint64_t l_Lean_Expr_hash(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_isReadOnlyExprMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__12(uint8_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_abstract_range(lean_object*, lean_object*, lean_object*); @@ -505,13 +507,13 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Cache_whnfAll___default; static lean_object* l_Lean_Meta_getLevelMVarDepth___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_liftMkBindingM(lean_object*); lean_object* l_Lean_printTraces___at_Lean_Core_instMetaEvalCoreM___spec__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withNewLocalInstances(lean_object*); uint64_t lean_uint64_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instMonadEnvMetaM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_approxDefEq___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_orelseMergeErrorsImp(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_instInhabitedSavedState___closed__2; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_withIncRecDepth___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withAtLeastTransparency___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -567,7 +569,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getLevelMVarDepth(lean_object*, lean_object LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateLambdaAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallMetaTelescopeReducing___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__3(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withNewLocalInstancesImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallBoundedTelescopeImp(lean_object*); @@ -579,7 +581,6 @@ size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_Meta_mkLevelStuckErrorMessage___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaMetaTelescope_process___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -633,8 +634,8 @@ lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x LEAN_EXPORT lean_object* l_Lean_Meta_lambdaLetTelescope___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_State_mctx___default___closed__1; extern lean_object* l_Lean_instInhabitedFVarId; +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); -lean_object* lean_level_update_imax(lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withNewBinderInfosImp___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -659,6 +660,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, le lean_object* lean_environment_main_module(lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l_Lean_Meta_instInhabitedState___closed__3; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__4; uint8_t l_Lean_Expr_isMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_abstractRange___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_processPostponed_loop(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -687,6 +689,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_instMonadMCtxMetaM; LEAN_EXPORT lean_object* l_Lean_Meta_throwUnknownFVar___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withAtLeastTransparency___rarg___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getReducibilityStatus___at___private_Lean_Meta_Basic_0__Lean_Meta_getDefInfoTemp___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__1; extern lean_object* l_Lean_Core_instMonadCoreM; LEAN_EXPORT lean_object* l_Lean_Meta_withAtLeastTransparency___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_saveAndResetSynthInstanceCache___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -742,6 +745,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withReducible___rarg(lean_object*, lean_obj LEAN_EXPORT lean_object* l_Lean_Meta_mkFreshExprMVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_processPostponed_loop___lambda__2___closed__2; uint8_t lean_get_reducibility_status(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_fvarsSizeLtMaxFVars___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withAssignableSyntheticOpaque___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalInstancesImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -762,7 +766,8 @@ LEAN_EXPORT lean_object* l_Lean_Meta_throwIsDefEqStuck___boxed(lean_object*, lea static lean_object* l_Lean_Meta_processPostponed_loop___closed__4; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_approxDefEqImp(lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_13474_(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Meta_ParamInfo_dependsOnHigherOrderOutParam___default; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_13494_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instMonadMCtxMetaM___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_resettingSynthInstanceCacheWhen(lean_object*); @@ -773,7 +778,6 @@ static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_Basic_0__L LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_modifyPostponed___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkLambdaFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_level_update_succ(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withMVarContext___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -801,6 +805,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withIncRecDepth___rarg___lambda__1(lean_obj LEAN_EXPORT lean_object* l_Lean_Meta_withTransparency___rarg___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkFreshLevelMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instInhabitedState; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__3; uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_sortFVarIds___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_instMetaEvalMetaM___rarg___closed__7; @@ -1162,6 +1167,22 @@ x_1 = 0; return x_1; } } +static uint8_t _init_l_Lean_Meta_ParamInfo_higherOrderOutParam___default() { +_start: +{ +uint8_t x_1; +x_1 = 0; +return x_1; +} +} +static uint8_t _init_l_Lean_Meta_ParamInfo_dependsOnHigherOrderOutParam___default() { +_start: +{ +uint8_t x_1; +x_1 = 0; +return x_1; +} +} static lean_object* _init_l_Lean_Meta_instInhabitedParamInfo___closed__1() { _start: { @@ -1169,12 +1190,14 @@ uint8_t x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; x_1 = 0; x_2 = 0; x_3 = l_Lean_Meta_ParamInfo_backDeps___default___closed__1; -x_4 = lean_alloc_ctor(0, 1, 4); +x_4 = lean_alloc_ctor(0, 1, 6); lean_ctor_set(x_4, 0, x_3); lean_ctor_set_uint8(x_4, sizeof(void*)*1, x_1); lean_ctor_set_uint8(x_4, sizeof(void*)*1 + 1, x_2); lean_ctor_set_uint8(x_4, sizeof(void*)*1 + 2, x_2); lean_ctor_set_uint8(x_4, sizeof(void*)*1 + 3, x_2); +lean_ctor_set_uint8(x_4, sizeof(void*)*1 + 4, x_2); +lean_ctor_set_uint8(x_4, sizeof(void*)*1 + 5, x_2); return x_4; } } @@ -1325,7 +1348,7 @@ x_1 = l_Lean_Meta_instInhabitedInfoCacheKey___closed__2; return x_1; } } -LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____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_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1362,7 +1385,7 @@ return x_8; } } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; @@ -1372,7 +1395,7 @@ x_5 = lean_ctor_get(x_1, 1); x_6 = lean_ctor_get_uint8(x_2, sizeof(void*)*2); x_7 = lean_ctor_get(x_2, 0); x_8 = lean_ctor_get(x_2, 1); -x_9 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_3, x_6); +x_9 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_3, x_6); if (x_9 == 0) { uint8_t x_10; @@ -1392,28 +1415,28 @@ return x_12; else { uint8_t x_13; -x_13 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_5, x_8); +x_13 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_5, x_8); return x_13; } } } } -LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____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_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____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_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_1, x_2); +x_3 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(x_1, x_2); +x_3 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); @@ -1424,7 +1447,7 @@ static lean_object* _init_l_Lean_Meta_instBEqInfoCacheKey___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____boxed), 2, 0); return x_1; } } @@ -4645,7 +4668,7 @@ lean_dec(x_2); return x_6; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__1() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__1() { _start: { lean_object* x_1; @@ -4653,17 +4676,17 @@ x_1 = lean_mk_string_from_bytes("Meta", 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__1; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__3() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__3() { _start: { lean_object* x_1; @@ -4671,21 +4694,21 @@ x_1 = lean_mk_string_from_bytes("debug", 5); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__4() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__3; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2; x_3 = l_Lean_registerTraceClass(x_2, x_1); if (lean_obj_tag(x_3) == 0) { @@ -4693,7 +4716,7 @@ lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_ctor_get(x_3, 1); lean_inc(x_4); lean_dec(x_3); -x_5 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__4; +x_5 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__4; x_6 = l_Lean_registerTraceClass(x_5, x_4); return x_6; } @@ -7220,7 +7243,7 @@ x_8 = lean_ctor_get(x_6, 0); x_9 = 0; x_10 = lean_unbox(x_8); lean_dec(x_8); -x_11 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_10, x_9); +x_11 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_10, x_9); x_12 = lean_box(x_11); lean_ctor_set(x_6, 0, x_12); return x_6; @@ -7236,7 +7259,7 @@ lean_dec(x_6); x_15 = 0; x_16 = lean_unbox(x_13); lean_dec(x_13); -x_17 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_16, x_15); +x_17 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_16, x_15); x_18 = lean_box(x_17); x_19 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_19, 0, x_18); @@ -7270,7 +7293,7 @@ x_8 = lean_ctor_get(x_6, 0); x_9 = 2; x_10 = lean_unbox(x_8); lean_dec(x_8); -x_11 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_10, x_9); +x_11 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_10, x_9); x_12 = lean_box(x_11); lean_ctor_set(x_6, 0, x_12); return x_6; @@ -7286,7 +7309,7 @@ lean_dec(x_6); x_15 = 2; x_16 = lean_unbox(x_13); lean_dec(x_13); -x_17 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_16, x_15); +x_17 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_16, x_15); x_18 = lean_box(x_17); x_19 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_19, 0, x_18); @@ -27473,205 +27496,391 @@ case 1: lean_object* x_7; lean_object* x_8; uint8_t x_9; x_7 = lean_ctor_get(x_1, 0); lean_inc(x_7); +lean_inc(x_7); x_8 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_7, x_2, x_3, x_4, x_5, x_6); x_9 = !lean_is_exclusive(x_8); if (x_9 == 0) { -lean_object* x_10; lean_object* x_11; +lean_object* x_10; size_t x_11; size_t x_12; uint8_t x_13; x_10 = lean_ctor_get(x_8, 0); -x_11 = lean_level_update_succ(x_1, x_10); -lean_ctor_set(x_8, 0, x_11); +x_11 = lean_ptr_addr(x_7); +lean_dec(x_7); +x_12 = lean_ptr_addr(x_10); +x_13 = lean_usize_dec_eq(x_11, x_12); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_1); +x_14 = l_Lean_Level_succ___override(x_10); +lean_ctor_set(x_8, 0, x_14); return x_8; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_8, 0); -x_13 = lean_ctor_get(x_8, 1); -lean_inc(x_13); -lean_inc(x_12); -lean_dec(x_8); -x_14 = lean_level_update_succ(x_1, 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_13); -return x_15; +lean_dec(x_10); +lean_ctor_set(x_8, 0, x_1); +return x_8; } } -case 2: +else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_16 = lean_ctor_get(x_1, 0); +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; uint8_t x_19; +x_15 = lean_ctor_get(x_8, 0); +x_16 = lean_ctor_get(x_8, 1); lean_inc(x_16); -x_17 = lean_ctor_get(x_1, 1); -lean_inc(x_17); -x_18 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_16, x_2, x_3, x_4, x_5, x_6); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_17, x_2, x_3, x_4, x_5, x_20); -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +lean_inc(x_15); +lean_dec(x_8); +x_17 = lean_ptr_addr(x_7); +lean_dec(x_7); +x_18 = lean_ptr_addr(x_15); +x_19 = lean_usize_dec_eq(x_17, x_18); +if (x_19 == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_21, 0); -x_24 = lean_level_update_max(x_1, x_19, x_23); -lean_ctor_set(x_21, 0, x_24); +lean_object* x_20; lean_object* x_21; +lean_dec(x_1); +x_20 = l_Lean_Level_succ___override(x_15); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_16); return x_21; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_21, 0); -x_26 = lean_ctor_get(x_21, 1); +lean_object* x_22; +lean_dec(x_15); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_1); +lean_ctor_set(x_22, 1, x_16); +return x_22; +} +} +} +case 2: +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_23 = lean_ctor_get(x_1, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_1, 1); +lean_inc(x_24); +lean_inc(x_23); +x_25 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_23, x_2, x_3, x_4, x_5, x_6); +x_26 = lean_ctor_get(x_25, 0); lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_21); -x_27 = lean_level_update_max(x_1, x_19, x_25); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +lean_inc(x_24); +x_28 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_24, x_2, x_3, x_4, x_5, x_27); +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) +{ +lean_object* x_30; size_t x_31; size_t x_32; uint8_t x_33; +x_30 = lean_ctor_get(x_28, 0); +x_31 = lean_ptr_addr(x_23); +lean_dec(x_23); +x_32 = lean_ptr_addr(x_26); +x_33 = lean_usize_dec_eq(x_31, x_32); +if (x_33 == 0) +{ +lean_object* x_34; +lean_dec(x_24); +lean_dec(x_1); +x_34 = l_Lean_mkLevelMax_x27(x_26, x_30); +lean_ctor_set(x_28, 0, x_34); return x_28; } +else +{ +size_t x_35; size_t x_36; uint8_t x_37; +x_35 = lean_ptr_addr(x_24); +lean_dec(x_24); +x_36 = lean_ptr_addr(x_30); +x_37 = lean_usize_dec_eq(x_35, x_36); +if (x_37 == 0) +{ +lean_object* x_38; +lean_dec(x_1); +x_38 = l_Lean_mkLevelMax_x27(x_26, x_30); +lean_ctor_set(x_28, 0, x_38); +return x_28; +} +else +{ +lean_object* x_39; +x_39 = l_Lean_simpLevelMax_x27(x_26, x_30, x_1); +lean_dec(x_1); +lean_dec(x_30); +lean_dec(x_26); +lean_ctor_set(x_28, 0, x_39); +return x_28; +} +} +} +else +{ +lean_object* x_40; lean_object* x_41; size_t x_42; size_t x_43; uint8_t x_44; +x_40 = lean_ctor_get(x_28, 0); +x_41 = lean_ctor_get(x_28, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_28); +x_42 = lean_ptr_addr(x_23); +lean_dec(x_23); +x_43 = lean_ptr_addr(x_26); +x_44 = lean_usize_dec_eq(x_42, x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +lean_dec(x_24); +lean_dec(x_1); +x_45 = l_Lean_mkLevelMax_x27(x_26, x_40); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_41); +return x_46; +} +else +{ +size_t x_47; size_t x_48; uint8_t x_49; +x_47 = lean_ptr_addr(x_24); +lean_dec(x_24); +x_48 = lean_ptr_addr(x_40); +x_49 = lean_usize_dec_eq(x_47, x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; +lean_dec(x_1); +x_50 = l_Lean_mkLevelMax_x27(x_26, x_40); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_41); +return x_51; +} +else +{ +lean_object* x_52; lean_object* x_53; +x_52 = l_Lean_simpLevelMax_x27(x_26, x_40, x_1); +lean_dec(x_1); +lean_dec(x_40); +lean_dec(x_26); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_41); +return x_53; +} +} +} } case 3: { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_29 = lean_ctor_get(x_1, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_1, 1); -lean_inc(x_30); -x_31 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_29, x_2, x_3, x_4, x_5, x_6); -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -x_34 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_30, x_2, x_3, x_4, x_5, x_33); -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; +x_54 = lean_ctor_get(x_1, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_1, 1); +lean_inc(x_55); +lean_inc(x_54); +x_56 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_54, x_2, x_3, x_4, x_5, x_6); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +lean_inc(x_55); +x_59 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_55, x_2, x_3, x_4, x_5, x_58); +x_60 = !lean_is_exclusive(x_59); +if (x_60 == 0) { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_34, 0); -x_37 = lean_level_update_imax(x_1, x_32, x_36); -lean_ctor_set(x_34, 0, x_37); -return x_34; +lean_object* x_61; size_t x_62; size_t x_63; uint8_t x_64; +x_61 = lean_ctor_get(x_59, 0); +x_62 = lean_ptr_addr(x_54); +lean_dec(x_54); +x_63 = lean_ptr_addr(x_57); +x_64 = lean_usize_dec_eq(x_62, x_63); +if (x_64 == 0) +{ +lean_object* x_65; +lean_dec(x_55); +lean_dec(x_1); +x_65 = l_Lean_mkLevelIMax_x27(x_57, x_61); +lean_ctor_set(x_59, 0, x_65); +return x_59; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_38 = lean_ctor_get(x_34, 0); -x_39 = lean_ctor_get(x_34, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_34); -x_40 = lean_level_update_imax(x_1, x_32, x_38); -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_39); -return x_41; +size_t x_66; size_t x_67; uint8_t x_68; +x_66 = lean_ptr_addr(x_55); +lean_dec(x_55); +x_67 = lean_ptr_addr(x_61); +x_68 = lean_usize_dec_eq(x_66, x_67); +if (x_68 == 0) +{ +lean_object* x_69; +lean_dec(x_1); +x_69 = l_Lean_mkLevelIMax_x27(x_57, x_61); +lean_ctor_set(x_59, 0, x_69); +return x_59; +} +else +{ +lean_object* x_70; +x_70 = l_Lean_simpLevelIMax_x27(x_57, x_61, x_1); +lean_dec(x_1); +lean_ctor_set(x_59, 0, x_70); +return x_59; +} +} +} +else +{ +lean_object* x_71; lean_object* x_72; size_t x_73; size_t x_74; uint8_t x_75; +x_71 = lean_ctor_get(x_59, 0); +x_72 = lean_ctor_get(x_59, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_59); +x_73 = lean_ptr_addr(x_54); +lean_dec(x_54); +x_74 = lean_ptr_addr(x_57); +x_75 = lean_usize_dec_eq(x_73, x_74); +if (x_75 == 0) +{ +lean_object* x_76; lean_object* x_77; +lean_dec(x_55); +lean_dec(x_1); +x_76 = l_Lean_mkLevelIMax_x27(x_57, x_71); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_72); +return x_77; +} +else +{ +size_t x_78; size_t x_79; uint8_t x_80; +x_78 = lean_ptr_addr(x_55); +lean_dec(x_55); +x_79 = lean_ptr_addr(x_71); +x_80 = lean_usize_dec_eq(x_78, x_79); +if (x_80 == 0) +{ +lean_object* x_81; lean_object* x_82; +lean_dec(x_1); +x_81 = l_Lean_mkLevelIMax_x27(x_57, x_71); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_72); +return x_82; +} +else +{ +lean_object* x_83; lean_object* x_84; +x_83 = l_Lean_simpLevelIMax_x27(x_57, x_71, x_1); +lean_dec(x_1); +x_84 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_72); +return x_84; +} +} } } case 5: { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_42 = lean_ctor_get(x_1, 0); -lean_inc(x_42); -x_58 = lean_st_ref_get(x_5, x_6); -x_59 = lean_ctor_get(x_58, 1); -lean_inc(x_59); -lean_dec(x_58); -x_60 = lean_st_ref_get(x_3, x_59); -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_60, 1); -lean_inc(x_62); -lean_dec(x_60); -x_63 = lean_ctor_get(x_61, 0); -lean_inc(x_63); -lean_dec(x_61); -x_64 = lean_ctor_get(x_63, 5); -lean_inc(x_64); -lean_dec(x_63); -lean_inc(x_42); -x_65 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_64, x_42); -if (lean_obj_tag(x_65) == 0) +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_85 = lean_ctor_get(x_1, 0); +lean_inc(x_85); +x_101 = lean_st_ref_get(x_5, x_6); +x_102 = lean_ctor_get(x_101, 1); +lean_inc(x_102); +lean_dec(x_101); +x_103 = lean_st_ref_get(x_3, x_102); +x_104 = lean_ctor_get(x_103, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_103, 1); +lean_inc(x_105); +lean_dec(x_103); +x_106 = lean_ctor_get(x_104, 0); +lean_inc(x_106); +lean_dec(x_104); +x_107 = lean_ctor_get(x_106, 5); +lean_inc(x_107); +lean_dec(x_106); +lean_inc(x_85); +x_108 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_107, x_85); +if (lean_obj_tag(x_108) == 0) { -x_43 = x_65; -x_44 = x_62; -goto block_57; +x_86 = x_108; +x_87 = x_105; +goto block_100; } else { -lean_object* x_66; lean_object* x_67; -x_66 = l_Lean_markUsedAssignment___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__2___rarg(x_3, x_4, x_5, x_62); -x_67 = lean_ctor_get(x_66, 1); -lean_inc(x_67); -lean_dec(x_66); -x_43 = x_65; -x_44 = x_67; -goto block_57; +lean_object* x_109; lean_object* x_110; +x_109 = l_Lean_markUsedAssignment___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__2___rarg(x_3, x_4, x_5, x_105); +x_110 = lean_ctor_get(x_109, 1); +lean_inc(x_110); +lean_dec(x_109); +x_86 = x_108; +x_87 = x_110; +goto block_100; } -block_57: +block_100: { -if (lean_obj_tag(x_43) == 0) +if (lean_obj_tag(x_86) == 0) { -lean_object* x_45; -lean_dec(x_42); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_1); -lean_ctor_set(x_45, 1, x_44); -return x_45; +lean_object* x_88; +lean_dec(x_85); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_1); +lean_ctor_set(x_88, 1, x_87); +return x_88; } else { -lean_object* x_46; uint8_t x_47; +lean_object* x_89; uint8_t x_90; lean_dec(x_1); -x_46 = lean_ctor_get(x_43, 0); -lean_inc(x_46); -lean_dec(x_43); -x_47 = l_Lean_Level_hasMVar(x_46); -if (x_47 == 0) +x_89 = lean_ctor_get(x_86, 0); +lean_inc(x_89); +lean_dec(x_86); +x_90 = l_Lean_Level_hasMVar(x_89); +if (x_90 == 0) { -lean_object* x_48; -lean_dec(x_42); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_44); -return x_48; +lean_object* x_91; +lean_dec(x_85); +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_89); +lean_ctor_set(x_91, 1, x_87); +return x_91; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; -x_49 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_46, x_2, x_3, x_4, x_5, x_44); -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_50); -x_52 = l_Lean_assignLevelMVar___at_Lean_Meta_normalizeLevel___spec__2(x_42, x_50, x_2, x_3, x_4, x_5, x_51); -x_53 = !lean_is_exclusive(x_52); -if (x_53 == 0) +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; +x_92 = l_Lean_instantiateLevelMVars___at_Lean_Meta_normalizeLevel___spec__1(x_89, x_2, x_3, x_4, x_5, x_87); +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_inc(x_93); +x_95 = l_Lean_assignLevelMVar___at_Lean_Meta_normalizeLevel___spec__2(x_85, x_93, x_2, x_3, x_4, x_5, x_94); +x_96 = !lean_is_exclusive(x_95); +if (x_96 == 0) { -lean_object* x_54; -x_54 = lean_ctor_get(x_52, 0); -lean_dec(x_54); -lean_ctor_set(x_52, 0, x_50); -return x_52; +lean_object* x_97; +x_97 = lean_ctor_get(x_95, 0); +lean_dec(x_97); +lean_ctor_set(x_95, 0, x_93); +return x_95; } else { -lean_object* x_55; lean_object* x_56; -x_55 = lean_ctor_get(x_52, 1); -lean_inc(x_55); -lean_dec(x_52); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_50); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_98; lean_object* x_99; +x_98 = lean_ctor_get(x_95, 1); +lean_inc(x_98); +lean_dec(x_95); +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_93); +lean_ctor_set(x_99, 1, x_98); +return x_99; } } } @@ -27679,11 +27888,11 @@ return x_56; } default: { -lean_object* x_68; -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_1); -lean_ctor_set(x_68, 1, x_6); -return x_68; +lean_object* x_111; +x_111 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_111, 0, x_1); +lean_ctor_set(x_111, 1, x_6); +return x_111; } } } @@ -36001,7 +36210,7 @@ static lean_object* _init_l___private_Lean_Meta_Basic_0__Lean_Meta_processPostpo _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2; x_2 = l___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -42491,7 +42700,7 @@ static lean_object* _init_l_Lean_Meta_isExprDefEq___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2; x_2 = l_Lean_Meta_isExprDefEq___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -45238,7 +45447,7 @@ lean_dec(x_3); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_13474_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_13494_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -45347,6 +45556,8 @@ l_Lean_Meta_ParamInfo_backDeps___default = _init_l_Lean_Meta_ParamInfo_backDeps_ lean_mark_persistent(l_Lean_Meta_ParamInfo_backDeps___default); l_Lean_Meta_ParamInfo_isProp___default = _init_l_Lean_Meta_ParamInfo_isProp___default(); l_Lean_Meta_ParamInfo_isDecInst___default = _init_l_Lean_Meta_ParamInfo_isDecInst___default(); +l_Lean_Meta_ParamInfo_higherOrderOutParam___default = _init_l_Lean_Meta_ParamInfo_higherOrderOutParam___default(); +l_Lean_Meta_ParamInfo_dependsOnHigherOrderOutParam___default = _init_l_Lean_Meta_ParamInfo_dependsOnHigherOrderOutParam___default(); l_Lean_Meta_instInhabitedParamInfo___closed__1 = _init_l_Lean_Meta_instInhabitedParamInfo___closed__1(); lean_mark_persistent(l_Lean_Meta_instInhabitedParamInfo___closed__1); l_Lean_Meta_instInhabitedParamInfo = _init_l_Lean_Meta_instInhabitedParamInfo(); @@ -45551,15 +45762,15 @@ l_Lean_Meta_throwIsDefEqStuck___rarg___closed__1 = _init_l_Lean_Meta_throwIsDefE lean_mark_persistent(l_Lean_Meta_throwIsDefEqStuck___rarg___closed__1); l_Lean_Meta_throwIsDefEqStuck___rarg___closed__2 = _init_l_Lean_Meta_throwIsDefEqStuck___rarg___closed__2(); lean_mark_persistent(l_Lean_Meta_throwIsDefEqStuck___rarg___closed__2); -l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__1 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__1(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__1); -l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__2); -l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__3 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__3(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__3); -l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__4 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__4(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476____closed__4); -res = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1476_(lean_io_mk_world()); +l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__1 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__1(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__1); +l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__2); +l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__3 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__3(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__3); +l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__4 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__4(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496____closed__4); +res = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_1496_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_throwMaxRecDepthAt___at_Lean_Meta_withIncRecDepth___spec__1___rarg___closed__1 = _init_l_Lean_throwMaxRecDepthAt___at_Lean_Meta_withIncRecDepth___spec__1___rarg___closed__1(); @@ -45720,7 +45931,7 @@ l_Lean_Meta_isExprDefEq___closed__1 = _init_l_Lean_Meta_isExprDefEq___closed__1( lean_mark_persistent(l_Lean_Meta_isExprDefEq___closed__1); l_Lean_Meta_isExprDefEq___closed__2 = _init_l_Lean_Meta_isExprDefEq___closed__2(); lean_mark_persistent(l_Lean_Meta_isExprDefEq___closed__2); -res = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_13474_(lean_io_mk_world()); +res = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_13494_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/CasesOn.c b/stage0/stdlib/Lean/Meta/CasesOn.c index 15a5f3f4e6e8..b59898d731fd 100644 --- a/stage0/stdlib/Lean/Meta/CasesOn.c +++ b/stage0/stdlib/Lean/Meta/CasesOn.c @@ -62,6 +62,7 @@ lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_CasesOnApp_addArg_updateAlts___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_CasesOnApp_addArg_updateAlts___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_CasesOnApp_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Meta_CasesOnApp_addArg___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -84,7 +85,6 @@ static lean_object* l_List_forIn_loop___at_Lean_Meta_toCasesOnApp_x3f___spec__2_ static lean_object* l_Lean_Meta_toCasesOnApp_x3f___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_CasesOnApp_addArg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_CasesOnApp_addArg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_loop___at_Lean_Meta_toCasesOnApp_x3f___spec__2___closed__2; static lean_object* l_List_forIn_loop___at_Lean_Meta_toCasesOnApp_x3f___spec__2___closed__1; @@ -368,7 +368,7 @@ static lean_object* _init_l_Lean_Meta_toCasesOnApp_x3f___lambda__1___closed__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; x_1 = l_Lean_Meta_toCasesOnApp_x3f___lambda__1___closed__2; x_2 = l_Lean_Meta_toCasesOnApp_x3f___lambda__1___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_toCasesOnApp_x3f___lambda__1___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -864,7 +864,7 @@ x_16 = lean_ctor_get(x_12, 0); lean_inc(x_16); lean_dec(x_12); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_2, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_17); x_19 = l_Lean_Meta_toCasesOnApp_x3f___lambda__2___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -925,7 +925,7 @@ x_37 = lean_ctor_get(x_12, 0); lean_inc(x_37); lean_dec(x_12); x_38 = lean_unsigned_to_nat(0u); -x_39 = l_Lean_Expr_getAppNumArgsAux(x_2, x_38); +x_39 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_38); x_40 = l_Lean_Meta_toCasesOnApp_x3f___lambda__2___closed__1; lean_inc(x_39); x_41 = lean_mk_array(x_39, x_40); diff --git a/stage0/stdlib/Lean/Meta/Check.c b/stage0/stdlib/Lean/Meta/Check.c index aa7363db6ae8..a58d739fda52 100644 --- a/stage0/stdlib/Lean/Meta/Check.c +++ b/stage0/stdlib/Lean/Meta/Check.c @@ -95,6 +95,7 @@ LEAN_EXPORT lean_object* l_Std_HashMapImp_moveEntries___at___private_Lean_Meta_C lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Check_0__Lean_Meta_checkAux_checkForall___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_throwLetTypeMismatchMessage___spec__2(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); @@ -126,7 +127,6 @@ lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___privat static lean_object* l_Lean_Meta_addPPExplicitToExposeDiff___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_isTypeCorrect___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at___private_Lean_Meta_Check_0__Lean_Meta_checkAux___spec__1___boxed(lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_addNode___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_equal(lean_object*, lean_object*); @@ -872,7 +872,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Meta_addPPExplicitToE lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Meta_addPPExplicitToExposeDiff_visit___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_Meta_addPPExplicitToExposeDiff_visit___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Meta_addPPExplicitToExposeDiff_visit___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2138,8 +2138,8 @@ else { lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; x_14 = lean_unsigned_to_nat(0u); -x_15 = l_Lean_Expr_getAppNumArgsAux(x_1, x_14); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_2, x_14); +x_15 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_14); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_14); x_17 = lean_nat_dec_eq(x_15, x_16); if (x_17 == 0) { diff --git a/stage0/stdlib/Lean/Meta/Closure.c b/stage0/stdlib/Lean/Meta/Closure.c index 8ca1a8f02aae..7428edddd081 100644 --- a/stage0/stdlib/Lean/Meta/Closure.c +++ b/stage0/stdlib/Lean/Meta/Closure.c @@ -17,7 +17,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_mkBinding(uint8_t, lean_object*, le uint8_t l_Lean_isRecCore(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Closure_collectExprAux___closed__5; static lean_object* l_Lean_Meta_Closure_collectExprAux___closed__18; -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); lean_object* l_Lean_Level_param___override(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); @@ -34,10 +33,11 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_pushFVarArg___boxed(lean_object*, l lean_object* l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldlM___at_Lean_Meta_mkAuxDefinition___spec__8___closed__2; static lean_object* l_Nat_foldRev_loop___at_Lean_Meta_Closure_mkBinding___spec__2___closed__3; +uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_List_foldlM___at_Lean_Meta_mkAuxDefinition___spec__8___closed__4; +lean_object* l_Lean_Level_succ___override(lean_object*); static lean_object* l_Lean_Meta_Closure_collectLevelAux___closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l_Lean_Meta_Closure_collectLevelAux___closed__9; @@ -48,6 +48,7 @@ lean_object* l_panic___at_Lean_LocalDecl_setBinderInfo___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAuxDefinitionFor___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at_Lean_Meta_Closure_collectExprAux___spec__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isCasesOnRecursor(lean_object*, lean_object*); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); uint8_t l_Lean_Level_hasMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_newLocalDecls___default; LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Meta_mkAuxDefinition___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -66,6 +67,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_exprFVarArgs___default; lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at_Lean_Meta_Closure_collectExprAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_nextLevelIdx___default; +uint8_t l_ptrEqList___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_nextExprIdx___default; uint8_t l_Lean_Level_hasParam(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_levelArgs___default; @@ -85,6 +87,7 @@ uint32_t lean_uint32_add(uint32_t, uint32_t); uint8_t lean_expr_has_loose_bvar(lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Closure_mkNewLevelParam___closed__1; +lean_object* l_Lean_simpLevelIMax_x27(lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); lean_object* l_Lean_Expr_FindImpl_findUnsafe_x3f(lean_object*, lean_object*); uint8_t l_Lean_Environment_hasUnsafe(lean_object*, lean_object*); @@ -119,17 +122,19 @@ lean_object* l_Lean_Expr_headBeta(lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshId___at_Lean_Meta_Closure_collectExprAux___spec__2___rarg___boxed(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Level_normalize___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_newLocalDeclsForMVars___default; -lean_object* lean_level_update_max(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_process(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Closure_collectExprAux___closed__6; lean_object* l_Lean_replaceRef(lean_object*, lean_object*); +lean_object* l_Lean_simpLevelMax_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Closure_preprocess___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Closure_State_levelParams___default___closed__1; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_pickNextToProcess_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_name_append_index_after(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_visitedLevel___default; @@ -140,6 +145,7 @@ LEAN_EXPORT uint8_t l_List_foldlM___at_Lean_Meta_mkAuxDefinition___spec__8___lam static lean_object* l_Lean_Meta_Closure_collectExprAux___closed__1; lean_object* lean_expr_abstract_range(lean_object*, lean_object*, lean_object*); lean_object* l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(lean_object*, lean_object*); +lean_object* l_Lean_Expr_sort___override(lean_object*); uint8_t l_Array_contains___at_Lean_registerInternalExceptionId___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Closure_collectExprAux___closed__17; lean_object* l_Array_back___rarg(lean_object*, lean_object*); @@ -168,7 +174,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_mkBinding___boxed(lean_object*, lea LEAN_EXPORT lean_object* l_Lean_Meta_Closure_preprocess___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_resetZetaFVarIds___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_Closure_collectExprAux___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_preprocess___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); lean_object* l_Lean_replaceFVarIdAtLocalDecl(lean_object*, lean_object*, lean_object*); @@ -176,7 +181,6 @@ static lean_object* l_Lean_Meta_Closure_mkNewLevelParam___closed__2; lean_object* l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_visitExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_pushLocalDecl(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_preprocess(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_mkNextUserName___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldRev_loop___at_Lean_Meta_Closure_mkLambda___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -191,10 +195,10 @@ lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); static lean_object* l_List_foldlM___at_Lean_Meta_mkAuxDefinition___spec__8___closed__3; lean_object* l_Lean_Expr_fvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_collectLevelAux___boxed(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_Meta_Closure_collectLevelAux___closed__3; static lean_object* l_Lean_Meta_Closure_collectExprAux___closed__9; LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Meta_Closure_visitLevel___spec__7(lean_object*, lean_object*); -lean_object* lean_level_update_imax(lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MonadEnv_0__Lean_checkUnsupported___at_Lean_Meta_mkAuxDefinition___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_index(lean_object*); @@ -205,7 +209,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_toProcess___default; lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_visitedExpr___default; static lean_object* l_Nat_foldRev_loop___at_Lean_Meta_Closure_mkBinding___spec__2___closed__2; -lean_object* lean_expr_update_sort(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Meta_mkAuxDefinition___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_collectLevelAux(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -230,9 +233,8 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_mkNextUserName___rarg___boxed(lean_ LEAN_EXPORT lean_object* l_Nat_foldRev_loop___at_Lean_Meta_Closure_mkBinding___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_logAt___at_Lean_Meta_mkAuxDefinition___spec__4___closed__1; -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAuxDefinition___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_level_update_succ(lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Meta_mkAuxDefinition___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Meta_Closure_State_visitedLevel___default___spec__1(lean_object*); @@ -240,6 +242,7 @@ LEAN_EXPORT lean_object* l_Lean_mkFreshId___at_Lean_Meta_Closure_collectExprAux_ lean_object* l_Lean_Meta_getMVarDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_pop(lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_throwKernelException___at_Lean_Meta_mkAuxDefinition___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_abstract(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_pickNextToProcessAux(lean_object*, lean_object*, lean_object*, lean_object*); @@ -248,6 +251,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_pickNextToProcess_x3f___boxed(lean_ LEAN_EXPORT lean_object* l_Lean_Meta_mkAuxDefinition___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAuxDefinition___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_instInhabitedToProcessElement; +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Closure_collectExprAux___closed__19; static lean_object* l_Lean_Meta_Closure_collectLevelAux___closed__6; LEAN_EXPORT lean_object* l_Lean_compileDecl___at_Lean_Meta_mkAuxDefinition___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -261,7 +265,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_collectExpr___boxed(lean_object*, l static lean_object* l_Lean_Meta_Closure_State_visitedExpr___default___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Closure_collectLevel(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Declaration_foldExprM___at_Lean_Declaration_hasSorry___spec__1(lean_object*, uint8_t); -lean_object* lean_expr_update_app(lean_object*, lean_object*, lean_object*); uint8_t lean_level_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_State_newLetDecls___default; LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Closure_preprocess___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -275,7 +278,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Closure_collectLevel___boxed(lean_object*, static lean_object* l_Lean_Meta_Closure_collectExprAux___closed__10; extern lean_object* l___private_Lean_MonadEnv_0__Lean_supportedRecursors; LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Meta_mkAuxDefinition___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_const(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_pushToProcess(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_Meta_Closure_visitLevel___spec__8(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Closure_mkValueTypeClosure___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1840,7 +1842,7 @@ static lean_object* _init_l_Lean_Meta_Closure_collectLevelAux___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateSucc!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateSucc!Impl", 48); return x_1; } } @@ -1858,8 +1860,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectLevelAux___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectLevelAux___closed__1; x_2 = l_Lean_Meta_Closure_collectLevelAux___closed__2; -x_3 = lean_unsigned_to_nat(538u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(527u); +x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_Meta_Closure_collectLevelAux___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -1869,7 +1871,7 @@ static lean_object* _init_l_Lean_Meta_Closure_collectLevelAux___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateMax!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateMax!Impl", 47); return x_1; } } @@ -1887,8 +1889,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectLevelAux___closed__7() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectLevelAux___closed__1; x_2 = l_Lean_Meta_Closure_collectLevelAux___closed__5; -x_3 = lean_unsigned_to_nat(547u); -x_4 = lean_unsigned_to_nat(14u); +x_3 = lean_unsigned_to_nat(538u); +x_4 = lean_unsigned_to_nat(19u); x_5 = l_Lean_Meta_Closure_collectLevelAux___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -1898,7 +1900,7 @@ static lean_object* _init_l_Lean_Meta_Closure_collectLevelAux___closed__8() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateIMax!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateIMax!Impl", 48); return x_1; } } @@ -1916,8 +1918,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectLevelAux___closed__10() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectLevelAux___closed__1; x_2 = l_Lean_Meta_Closure_collectLevelAux___closed__8; -x_3 = lean_unsigned_to_nat(556u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(549u); +x_4 = lean_unsigned_to_nat(20u); x_5 = l_Lean_Meta_Closure_collectLevelAux___closed__9; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -1930,626 +1932,637 @@ lean_object* x_9; lean_object* x_10; switch (lean_obj_tag(x_1)) { case 0: { -lean_object* x_17; -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_1); -lean_ctor_set(x_17, 1, x_8); -return x_17; +lean_object* x_22; +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_1); +lean_ctor_set(x_22, 1, x_8); +return x_22; } case 1: { -lean_object* x_18; lean_object* x_19; uint8_t x_53; -x_18 = lean_ctor_get(x_1, 0); -lean_inc(x_18); -x_53 = l_Lean_Level_hasMVar(x_18); -if (x_53 == 0) +lean_object* x_23; lean_object* x_24; uint8_t x_58; +x_23 = lean_ctor_get(x_1, 0); +lean_inc(x_23); +x_58 = l_Lean_Level_hasMVar(x_23); +if (x_58 == 0) { -uint8_t x_54; -x_54 = l_Lean_Level_hasParam(x_18); -if (x_54 == 0) +uint8_t x_59; +x_59 = l_Lean_Level_hasParam(x_23); +if (x_59 == 0) { -x_9 = x_18; +x_9 = x_23; x_10 = x_8; -goto block_16; +goto block_21; } else { -lean_object* x_55; -x_55 = lean_box(0); -x_19 = x_55; -goto block_52; +lean_object* x_60; +x_60 = lean_box(0); +x_24 = x_60; +goto block_57; } } else { -lean_object* x_56; -x_56 = lean_box(0); -x_19 = x_56; -goto block_52; +lean_object* x_61; +x_61 = lean_box(0); +x_24 = x_61; +goto block_57; } -block_52: -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -lean_dec(x_19); -x_20 = lean_st_ref_get(x_7, x_8); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -x_22 = lean_st_ref_get(x_3, x_21); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_ctor_get(x_23, 0); -lean_inc(x_25); -lean_dec(x_23); -lean_inc(x_18); -x_26 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_25, x_18); -if (lean_obj_tag(x_26) == 0) +block_57: { -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_inc(x_18); -x_27 = l_Lean_Meta_Closure_collectLevelAux(x_18, x_2, x_3, x_4, x_5, x_6, x_7, 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_dec(x_24); +x_25 = lean_st_ref_get(x_7, x_8); +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = lean_st_ref_get(x_3, x_26); x_28 = lean_ctor_get(x_27, 0); lean_inc(x_28); x_29 = lean_ctor_get(x_27, 1); lean_inc(x_29); lean_dec(x_27); -x_30 = lean_st_ref_get(x_7, x_29); -x_31 = lean_ctor_get(x_30, 1); -lean_inc(x_31); -lean_dec(x_30); -x_32 = lean_st_ref_take(x_3, x_31); +x_30 = lean_ctor_get(x_28, 0); +lean_inc(x_30); +lean_dec(x_28); +lean_inc(x_23); +x_31 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_30, x_23); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; 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_inc(x_23); +x_32 = l_Lean_Meta_Closure_collectLevelAux(x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_29); x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); x_34 = lean_ctor_get(x_32, 1); lean_inc(x_34); lean_dec(x_32); -x_35 = lean_ctor_get(x_33, 0); -lean_inc(x_35); -lean_inc(x_28); -x_36 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_35, x_18, x_28); -x_37 = lean_ctor_get(x_33, 1); -lean_inc(x_37); -x_38 = lean_ctor_get(x_33, 2); +x_35 = lean_st_ref_get(x_7, x_34); +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +lean_dec(x_35); +x_37 = lean_st_ref_take(x_3, x_36); +x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -x_39 = lean_ctor_get(x_33, 3); +x_39 = lean_ctor_get(x_37, 1); lean_inc(x_39); -x_40 = lean_ctor_get(x_33, 4); +lean_dec(x_37); +x_40 = lean_ctor_get(x_38, 0); lean_inc(x_40); -x_41 = lean_ctor_get(x_33, 5); -lean_inc(x_41); -x_42 = lean_ctor_get(x_33, 6); +lean_inc(x_33); +x_41 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_40, x_23, x_33); +x_42 = lean_ctor_get(x_38, 1); lean_inc(x_42); -x_43 = lean_ctor_get(x_33, 7); +x_43 = lean_ctor_get(x_38, 2); lean_inc(x_43); -x_44 = lean_ctor_get(x_33, 8); +x_44 = lean_ctor_get(x_38, 3); lean_inc(x_44); -x_45 = lean_ctor_get(x_33, 9); +x_45 = lean_ctor_get(x_38, 4); lean_inc(x_45); -x_46 = lean_ctor_get(x_33, 10); +x_46 = lean_ctor_get(x_38, 5); lean_inc(x_46); -x_47 = lean_ctor_get(x_33, 11); +x_47 = lean_ctor_get(x_38, 6); lean_inc(x_47); -lean_dec(x_33); -x_48 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_48, 0, x_36); -lean_ctor_set(x_48, 1, x_37); -lean_ctor_set(x_48, 2, x_38); -lean_ctor_set(x_48, 3, x_39); -lean_ctor_set(x_48, 4, x_40); -lean_ctor_set(x_48, 5, x_41); -lean_ctor_set(x_48, 6, x_42); -lean_ctor_set(x_48, 7, x_43); -lean_ctor_set(x_48, 8, x_44); -lean_ctor_set(x_48, 9, x_45); -lean_ctor_set(x_48, 10, x_46); -lean_ctor_set(x_48, 11, x_47); -x_49 = lean_st_ref_set(x_3, x_48, x_34); -x_50 = lean_ctor_get(x_49, 1); +x_48 = lean_ctor_get(x_38, 7); +lean_inc(x_48); +x_49 = lean_ctor_get(x_38, 8); +lean_inc(x_49); +x_50 = lean_ctor_get(x_38, 9); lean_inc(x_50); -lean_dec(x_49); -x_9 = x_28; -x_10 = x_50; -goto block_16; +x_51 = lean_ctor_get(x_38, 10); +lean_inc(x_51); +x_52 = lean_ctor_get(x_38, 11); +lean_inc(x_52); +lean_dec(x_38); +x_53 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_53, 0, x_41); +lean_ctor_set(x_53, 1, x_42); +lean_ctor_set(x_53, 2, x_43); +lean_ctor_set(x_53, 3, x_44); +lean_ctor_set(x_53, 4, x_45); +lean_ctor_set(x_53, 5, x_46); +lean_ctor_set(x_53, 6, x_47); +lean_ctor_set(x_53, 7, x_48); +lean_ctor_set(x_53, 8, x_49); +lean_ctor_set(x_53, 9, x_50); +lean_ctor_set(x_53, 10, x_51); +lean_ctor_set(x_53, 11, x_52); +x_54 = lean_st_ref_set(x_3, x_53, x_39); +x_55 = lean_ctor_get(x_54, 1); +lean_inc(x_55); +lean_dec(x_54); +x_9 = x_33; +x_10 = x_55; +goto block_21; } else { -lean_object* x_51; -lean_dec(x_18); -x_51 = lean_ctor_get(x_26, 0); -lean_inc(x_51); -lean_dec(x_26); -x_9 = x_51; -x_10 = x_24; -goto block_16; +lean_object* x_56; +lean_dec(x_23); +x_56 = lean_ctor_get(x_31, 0); +lean_inc(x_56); +lean_dec(x_31); +x_9 = x_56; +x_10 = x_29; +goto block_21; } } } case 2: { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_108; uint8_t x_142; -x_57 = lean_ctor_get(x_1, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_1, 1); -lean_inc(x_58); -x_142 = l_Lean_Level_hasMVar(x_57); -if (x_142 == 0) +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_125; uint8_t x_159; +x_62 = lean_ctor_get(x_1, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_1, 1); +lean_inc(x_63); +x_159 = l_Lean_Level_hasMVar(x_62); +if (x_159 == 0) { -uint8_t x_143; -x_143 = l_Lean_Level_hasParam(x_57); -if (x_143 == 0) +uint8_t x_160; +x_160 = l_Lean_Level_hasParam(x_62); +if (x_160 == 0) { -x_59 = x_57; -x_60 = x_8; -goto block_107; +x_64 = x_62; +x_65 = x_8; +goto block_124; } else { -lean_object* x_144; -x_144 = lean_box(0); -x_108 = x_144; -goto block_141; +lean_object* x_161; +x_161 = lean_box(0); +x_125 = x_161; +goto block_158; } } else { -lean_object* x_145; -x_145 = lean_box(0); -x_108 = x_145; -goto block_141; +lean_object* x_162; +x_162 = lean_box(0); +x_125 = x_162; +goto block_158; } -block_107: +block_124: { -lean_object* x_61; lean_object* x_62; lean_object* x_69; uint8_t x_103; -x_103 = l_Lean_Level_hasMVar(x_58); -if (x_103 == 0) +lean_object* x_66; lean_object* x_67; lean_object* x_86; uint8_t x_120; +x_120 = l_Lean_Level_hasMVar(x_63); +if (x_120 == 0) { -uint8_t x_104; -x_104 = l_Lean_Level_hasParam(x_58); -if (x_104 == 0) +uint8_t x_121; +x_121 = l_Lean_Level_hasParam(x_63); +if (x_121 == 0) { -x_61 = x_58; -x_62 = x_60; -goto block_68; +x_66 = x_63; +x_67 = x_65; +goto block_85; } else { -lean_object* x_105; -x_105 = lean_box(0); -x_69 = x_105; -goto block_102; +lean_object* x_122; +x_122 = lean_box(0); +x_86 = x_122; +goto block_119; } } else { -lean_object* x_106; -x_106 = lean_box(0); -x_69 = x_106; -goto block_102; +lean_object* x_123; +x_123 = lean_box(0); +x_86 = x_123; +goto block_119; } -block_68: +block_85: { if (lean_obj_tag(x_1) == 2) { -lean_object* x_63; lean_object* x_64; -x_63 = lean_level_update_max(x_1, x_59, x_61); -x_64 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_62); -return x_64; +lean_object* x_68; lean_object* x_69; size_t x_70; size_t x_71; uint8_t x_72; +x_68 = lean_ctor_get(x_1, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_1, 1); +lean_inc(x_69); +x_70 = lean_ptr_addr(x_68); +lean_dec(x_68); +x_71 = lean_ptr_addr(x_64); +x_72 = lean_usize_dec_eq(x_70, x_71); +if (x_72 == 0) +{ +lean_object* x_73; lean_object* x_74; +lean_dec(x_69); +lean_dec(x_1); +x_73 = l_Lean_mkLevelMax_x27(x_64, x_66); +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_67); +return x_74; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -lean_dec(x_61); -lean_dec(x_59); +size_t x_75; size_t x_76; uint8_t x_77; +x_75 = lean_ptr_addr(x_69); +lean_dec(x_69); +x_76 = lean_ptr_addr(x_66); +x_77 = lean_usize_dec_eq(x_75, x_76); +if (x_77 == 0) +{ +lean_object* x_78; lean_object* x_79; lean_dec(x_1); -x_65 = l_Lean_Meta_Closure_collectLevelAux___closed__7; -x_66 = l_panic___at_Lean_Level_normalize___spec__1(x_65); -x_67 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_62); -return x_67; +x_78 = l_Lean_mkLevelMax_x27(x_64, x_66); +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_67); +return x_79; +} +else +{ +lean_object* x_80; lean_object* x_81; +x_80 = l_Lean_simpLevelMax_x27(x_64, x_66, x_1); +lean_dec(x_1); +lean_dec(x_66); +lean_dec(x_64); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_67); +return x_81; } } -block_102: +} +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_dec(x_69); -x_70 = lean_st_ref_get(x_7, x_60); -x_71 = lean_ctor_get(x_70, 1); -lean_inc(x_71); -lean_dec(x_70); -x_72 = lean_st_ref_get(x_3, x_71); -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 = lean_ctor_get(x_73, 0); -lean_inc(x_75); -lean_dec(x_73); -lean_inc(x_58); -x_76 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_75, x_58); -if (lean_obj_tag(x_76) == 0) +lean_object* x_82; lean_object* x_83; lean_object* x_84; +lean_dec(x_66); +lean_dec(x_64); +lean_dec(x_1); +x_82 = l_Lean_Meta_Closure_collectLevelAux___closed__7; +x_83 = l_panic___at_Lean_Level_normalize___spec__1(x_82); +x_84 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_67); +return x_84; +} +} +block_119: { -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_inc(x_58); -x_77 = l_Lean_Meta_Closure_collectLevelAux(x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_74); -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); -lean_inc(x_79); -lean_dec(x_77); -x_80 = lean_st_ref_get(x_7, x_79); -x_81 = lean_ctor_get(x_80, 1); -lean_inc(x_81); -lean_dec(x_80); -x_82 = lean_st_ref_take(x_3, x_81); -x_83 = lean_ctor_get(x_82, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_82, 1); -lean_inc(x_84); -lean_dec(x_82); -x_85 = lean_ctor_get(x_83, 0); -lean_inc(x_85); -lean_inc(x_78); -x_86 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_85, x_58, x_78); -x_87 = lean_ctor_get(x_83, 1); -lean_inc(x_87); -x_88 = lean_ctor_get(x_83, 2); +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_dec(x_86); +x_87 = lean_st_ref_get(x_7, x_65); +x_88 = lean_ctor_get(x_87, 1); lean_inc(x_88); -x_89 = lean_ctor_get(x_83, 3); -lean_inc(x_89); -x_90 = lean_ctor_get(x_83, 4); +lean_dec(x_87); +x_89 = lean_st_ref_get(x_3, x_88); +x_90 = lean_ctor_get(x_89, 0); lean_inc(x_90); -x_91 = lean_ctor_get(x_83, 5); +x_91 = lean_ctor_get(x_89, 1); lean_inc(x_91); -x_92 = lean_ctor_get(x_83, 6); +lean_dec(x_89); +x_92 = lean_ctor_get(x_90, 0); lean_inc(x_92); -x_93 = lean_ctor_get(x_83, 7); -lean_inc(x_93); -x_94 = lean_ctor_get(x_83, 8); -lean_inc(x_94); -x_95 = lean_ctor_get(x_83, 9); +lean_dec(x_90); +lean_inc(x_63); +x_93 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_92, x_63); +if (lean_obj_tag(x_93) == 0) +{ +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_inc(x_63); +x_94 = l_Lean_Meta_Closure_collectLevelAux(x_63, x_2, x_3, x_4, x_5, x_6, x_7, x_91); +x_95 = lean_ctor_get(x_94, 0); lean_inc(x_95); -x_96 = lean_ctor_get(x_83, 10); +x_96 = lean_ctor_get(x_94, 1); lean_inc(x_96); -x_97 = lean_ctor_get(x_83, 11); -lean_inc(x_97); -lean_dec(x_83); -x_98 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_98, 0, x_86); -lean_ctor_set(x_98, 1, x_87); -lean_ctor_set(x_98, 2, x_88); -lean_ctor_set(x_98, 3, x_89); -lean_ctor_set(x_98, 4, x_90); -lean_ctor_set(x_98, 5, x_91); -lean_ctor_set(x_98, 6, x_92); -lean_ctor_set(x_98, 7, x_93); -lean_ctor_set(x_98, 8, x_94); -lean_ctor_set(x_98, 9, x_95); -lean_ctor_set(x_98, 10, x_96); -lean_ctor_set(x_98, 11, x_97); -x_99 = lean_st_ref_set(x_3, x_98, x_84); -x_100 = lean_ctor_get(x_99, 1); +lean_dec(x_94); +x_97 = lean_st_ref_get(x_7, x_96); +x_98 = lean_ctor_get(x_97, 1); +lean_inc(x_98); +lean_dec(x_97); +x_99 = lean_st_ref_take(x_3, x_98); +x_100 = lean_ctor_get(x_99, 0); lean_inc(x_100); +x_101 = lean_ctor_get(x_99, 1); +lean_inc(x_101); lean_dec(x_99); -x_61 = x_78; -x_62 = x_100; -goto block_68; +x_102 = lean_ctor_get(x_100, 0); +lean_inc(x_102); +lean_inc(x_95); +x_103 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_102, x_63, x_95); +x_104 = lean_ctor_get(x_100, 1); +lean_inc(x_104); +x_105 = lean_ctor_get(x_100, 2); +lean_inc(x_105); +x_106 = lean_ctor_get(x_100, 3); +lean_inc(x_106); +x_107 = lean_ctor_get(x_100, 4); +lean_inc(x_107); +x_108 = lean_ctor_get(x_100, 5); +lean_inc(x_108); +x_109 = lean_ctor_get(x_100, 6); +lean_inc(x_109); +x_110 = lean_ctor_get(x_100, 7); +lean_inc(x_110); +x_111 = lean_ctor_get(x_100, 8); +lean_inc(x_111); +x_112 = lean_ctor_get(x_100, 9); +lean_inc(x_112); +x_113 = lean_ctor_get(x_100, 10); +lean_inc(x_113); +x_114 = lean_ctor_get(x_100, 11); +lean_inc(x_114); +lean_dec(x_100); +x_115 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_115, 0, x_103); +lean_ctor_set(x_115, 1, x_104); +lean_ctor_set(x_115, 2, x_105); +lean_ctor_set(x_115, 3, x_106); +lean_ctor_set(x_115, 4, x_107); +lean_ctor_set(x_115, 5, x_108); +lean_ctor_set(x_115, 6, x_109); +lean_ctor_set(x_115, 7, x_110); +lean_ctor_set(x_115, 8, x_111); +lean_ctor_set(x_115, 9, x_112); +lean_ctor_set(x_115, 10, x_113); +lean_ctor_set(x_115, 11, x_114); +x_116 = lean_st_ref_set(x_3, x_115, x_101); +x_117 = lean_ctor_get(x_116, 1); +lean_inc(x_117); +lean_dec(x_116); +x_66 = x_95; +x_67 = x_117; +goto block_85; } else { -lean_object* x_101; -lean_dec(x_58); -x_101 = lean_ctor_get(x_76, 0); -lean_inc(x_101); -lean_dec(x_76); -x_61 = x_101; -x_62 = x_74; -goto block_68; +lean_object* x_118; +lean_dec(x_63); +x_118 = lean_ctor_get(x_93, 0); +lean_inc(x_118); +lean_dec(x_93); +x_66 = x_118; +x_67 = x_91; +goto block_85; } } } -block_141: -{ -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_dec(x_108); -x_109 = lean_st_ref_get(x_7, x_8); -x_110 = lean_ctor_get(x_109, 1); -lean_inc(x_110); -lean_dec(x_109); -x_111 = lean_st_ref_get(x_3, x_110); -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -x_113 = lean_ctor_get(x_111, 1); -lean_inc(x_113); -lean_dec(x_111); -x_114 = lean_ctor_get(x_112, 0); -lean_inc(x_114); -lean_dec(x_112); -lean_inc(x_57); -x_115 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_114, x_57); -if (lean_obj_tag(x_115) == 0) +block_158: { -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_inc(x_57); -x_116 = l_Lean_Meta_Closure_collectLevelAux(x_57, x_2, x_3, x_4, x_5, x_6, x_7, x_113); -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 = lean_st_ref_get(x_7, x_118); -x_120 = lean_ctor_get(x_119, 1); -lean_inc(x_120); -lean_dec(x_119); -x_121 = lean_st_ref_take(x_3, x_120); -x_122 = lean_ctor_get(x_121, 0); -lean_inc(x_122); -x_123 = lean_ctor_get(x_121, 1); -lean_inc(x_123); -lean_dec(x_121); -x_124 = lean_ctor_get(x_122, 0); -lean_inc(x_124); -lean_inc(x_117); -x_125 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_124, x_57, x_117); -x_126 = lean_ctor_get(x_122, 1); -lean_inc(x_126); -x_127 = lean_ctor_get(x_122, 2); +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_dec(x_125); +x_126 = lean_st_ref_get(x_7, x_8); +x_127 = lean_ctor_get(x_126, 1); lean_inc(x_127); -x_128 = lean_ctor_get(x_122, 3); -lean_inc(x_128); -x_129 = lean_ctor_get(x_122, 4); +lean_dec(x_126); +x_128 = lean_st_ref_get(x_3, x_127); +x_129 = lean_ctor_get(x_128, 0); lean_inc(x_129); -x_130 = lean_ctor_get(x_122, 5); +x_130 = lean_ctor_get(x_128, 1); lean_inc(x_130); -x_131 = lean_ctor_get(x_122, 6); +lean_dec(x_128); +x_131 = lean_ctor_get(x_129, 0); lean_inc(x_131); -x_132 = lean_ctor_get(x_122, 7); -lean_inc(x_132); -x_133 = lean_ctor_get(x_122, 8); -lean_inc(x_133); -x_134 = lean_ctor_get(x_122, 9); +lean_dec(x_129); +lean_inc(x_62); +x_132 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_131, x_62); +if (lean_obj_tag(x_132) == 0) +{ +lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; 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_inc(x_62); +x_133 = l_Lean_Meta_Closure_collectLevelAux(x_62, x_2, x_3, x_4, x_5, x_6, x_7, x_130); +x_134 = lean_ctor_get(x_133, 0); lean_inc(x_134); -x_135 = lean_ctor_get(x_122, 10); +x_135 = lean_ctor_get(x_133, 1); lean_inc(x_135); -x_136 = lean_ctor_get(x_122, 11); -lean_inc(x_136); -lean_dec(x_122); -x_137 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_137, 0, x_125); -lean_ctor_set(x_137, 1, x_126); -lean_ctor_set(x_137, 2, x_127); -lean_ctor_set(x_137, 3, x_128); -lean_ctor_set(x_137, 4, x_129); -lean_ctor_set(x_137, 5, x_130); -lean_ctor_set(x_137, 6, x_131); -lean_ctor_set(x_137, 7, x_132); -lean_ctor_set(x_137, 8, x_133); -lean_ctor_set(x_137, 9, x_134); -lean_ctor_set(x_137, 10, x_135); -lean_ctor_set(x_137, 11, x_136); -x_138 = lean_st_ref_set(x_3, x_137, x_123); -x_139 = lean_ctor_get(x_138, 1); +lean_dec(x_133); +x_136 = lean_st_ref_get(x_7, x_135); +x_137 = lean_ctor_get(x_136, 1); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_st_ref_take(x_3, x_137); +x_139 = lean_ctor_get(x_138, 0); lean_inc(x_139); -lean_dec(x_138); -x_59 = x_117; -x_60 = x_139; -goto block_107; -} -else -{ -lean_object* x_140; -lean_dec(x_57); -x_140 = lean_ctor_get(x_115, 0); +x_140 = lean_ctor_get(x_138, 1); lean_inc(x_140); -lean_dec(x_115); -x_59 = x_140; -x_60 = x_113; -goto block_107; -} -} +lean_dec(x_138); +x_141 = lean_ctor_get(x_139, 0); +lean_inc(x_141); +lean_inc(x_134); +x_142 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_141, x_62, x_134); +x_143 = lean_ctor_get(x_139, 1); +lean_inc(x_143); +x_144 = lean_ctor_get(x_139, 2); +lean_inc(x_144); +x_145 = lean_ctor_get(x_139, 3); +lean_inc(x_145); +x_146 = lean_ctor_get(x_139, 4); +lean_inc(x_146); +x_147 = lean_ctor_get(x_139, 5); +lean_inc(x_147); +x_148 = lean_ctor_get(x_139, 6); +lean_inc(x_148); +x_149 = lean_ctor_get(x_139, 7); +lean_inc(x_149); +x_150 = lean_ctor_get(x_139, 8); +lean_inc(x_150); +x_151 = lean_ctor_get(x_139, 9); +lean_inc(x_151); +x_152 = lean_ctor_get(x_139, 10); +lean_inc(x_152); +x_153 = lean_ctor_get(x_139, 11); +lean_inc(x_153); +lean_dec(x_139); +x_154 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_154, 0, x_142); +lean_ctor_set(x_154, 1, x_143); +lean_ctor_set(x_154, 2, x_144); +lean_ctor_set(x_154, 3, x_145); +lean_ctor_set(x_154, 4, x_146); +lean_ctor_set(x_154, 5, x_147); +lean_ctor_set(x_154, 6, x_148); +lean_ctor_set(x_154, 7, x_149); +lean_ctor_set(x_154, 8, x_150); +lean_ctor_set(x_154, 9, x_151); +lean_ctor_set(x_154, 10, x_152); +lean_ctor_set(x_154, 11, x_153); +x_155 = lean_st_ref_set(x_3, x_154, x_140); +x_156 = lean_ctor_get(x_155, 1); +lean_inc(x_156); +lean_dec(x_155); +x_64 = x_134; +x_65 = x_156; +goto block_124; +} +else +{ +lean_object* x_157; +lean_dec(x_62); +x_157 = lean_ctor_get(x_132, 0); +lean_inc(x_157); +lean_dec(x_132); +x_64 = x_157; +x_65 = x_130; +goto block_124; +} +} } case 3: { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_197; uint8_t x_231; -x_146 = lean_ctor_get(x_1, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_1, 1); -lean_inc(x_147); -x_231 = l_Lean_Level_hasMVar(x_146); -if (x_231 == 0) +lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_226; uint8_t x_260; +x_163 = lean_ctor_get(x_1, 0); +lean_inc(x_163); +x_164 = lean_ctor_get(x_1, 1); +lean_inc(x_164); +x_260 = l_Lean_Level_hasMVar(x_163); +if (x_260 == 0) { -uint8_t x_232; -x_232 = l_Lean_Level_hasParam(x_146); -if (x_232 == 0) +uint8_t x_261; +x_261 = l_Lean_Level_hasParam(x_163); +if (x_261 == 0) { -x_148 = x_146; -x_149 = x_8; -goto block_196; +x_165 = x_163; +x_166 = x_8; +goto block_225; } else { -lean_object* x_233; -x_233 = lean_box(0); -x_197 = x_233; -goto block_230; +lean_object* x_262; +x_262 = lean_box(0); +x_226 = x_262; +goto block_259; } } else { -lean_object* x_234; -x_234 = lean_box(0); -x_197 = x_234; -goto block_230; +lean_object* x_263; +x_263 = lean_box(0); +x_226 = x_263; +goto block_259; } -block_196: +block_225: { -lean_object* x_150; lean_object* x_151; lean_object* x_158; uint8_t x_192; -x_192 = l_Lean_Level_hasMVar(x_147); -if (x_192 == 0) +lean_object* x_167; lean_object* x_168; lean_object* x_187; uint8_t x_221; +x_221 = l_Lean_Level_hasMVar(x_164); +if (x_221 == 0) { -uint8_t x_193; -x_193 = l_Lean_Level_hasParam(x_147); -if (x_193 == 0) +uint8_t x_222; +x_222 = l_Lean_Level_hasParam(x_164); +if (x_222 == 0) { -x_150 = x_147; -x_151 = x_149; -goto block_157; +x_167 = x_164; +x_168 = x_166; +goto block_186; } else { -lean_object* x_194; -x_194 = lean_box(0); -x_158 = x_194; -goto block_191; +lean_object* x_223; +x_223 = lean_box(0); +x_187 = x_223; +goto block_220; } } else { -lean_object* x_195; -x_195 = lean_box(0); -x_158 = x_195; -goto block_191; +lean_object* x_224; +x_224 = lean_box(0); +x_187 = x_224; +goto block_220; } -block_157: +block_186: { if (lean_obj_tag(x_1) == 3) { -lean_object* x_152; lean_object* x_153; -x_152 = lean_level_update_imax(x_1, x_148, x_150); -x_153 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_153, 0, x_152); -lean_ctor_set(x_153, 1, x_151); -return x_153; +lean_object* x_169; lean_object* x_170; size_t x_171; size_t x_172; uint8_t x_173; +x_169 = lean_ctor_get(x_1, 0); +lean_inc(x_169); +x_170 = lean_ctor_get(x_1, 1); +lean_inc(x_170); +x_171 = lean_ptr_addr(x_169); +lean_dec(x_169); +x_172 = lean_ptr_addr(x_165); +x_173 = lean_usize_dec_eq(x_171, x_172); +if (x_173 == 0) +{ +lean_object* x_174; lean_object* x_175; +lean_dec(x_170); +lean_dec(x_1); +x_174 = l_Lean_mkLevelIMax_x27(x_165, x_167); +x_175 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_175, 0, x_174); +lean_ctor_set(x_175, 1, x_168); +return x_175; } else { -lean_object* x_154; lean_object* x_155; lean_object* x_156; -lean_dec(x_150); -lean_dec(x_148); +size_t x_176; size_t x_177; uint8_t x_178; +x_176 = lean_ptr_addr(x_170); +lean_dec(x_170); +x_177 = lean_ptr_addr(x_167); +x_178 = lean_usize_dec_eq(x_176, x_177); +if (x_178 == 0) +{ +lean_object* x_179; lean_object* x_180; lean_dec(x_1); -x_154 = l_Lean_Meta_Closure_collectLevelAux___closed__10; -x_155 = l_panic___at_Lean_Level_normalize___spec__1(x_154); -x_156 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_156, 0, x_155); -lean_ctor_set(x_156, 1, x_151); -return x_156; +x_179 = l_Lean_mkLevelIMax_x27(x_165, x_167); +x_180 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_180, 0, x_179); +lean_ctor_set(x_180, 1, x_168); +return x_180; } -} -block_191: -{ -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -lean_dec(x_158); -x_159 = lean_st_ref_get(x_7, x_149); -x_160 = lean_ctor_get(x_159, 1); -lean_inc(x_160); -lean_dec(x_159); -x_161 = lean_st_ref_get(x_3, x_160); -x_162 = lean_ctor_get(x_161, 0); -lean_inc(x_162); -x_163 = lean_ctor_get(x_161, 1); -lean_inc(x_163); -lean_dec(x_161); -x_164 = lean_ctor_get(x_162, 0); -lean_inc(x_164); -lean_dec(x_162); -lean_inc(x_147); -x_165 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_164, x_147); -if (lean_obj_tag(x_165) == 0) +else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; -lean_inc(x_147); -x_166 = l_Lean_Meta_Closure_collectLevelAux(x_147, x_2, x_3, x_4, x_5, x_6, x_7, x_163); -x_167 = lean_ctor_get(x_166, 0); -lean_inc(x_167); -x_168 = lean_ctor_get(x_166, 1); -lean_inc(x_168); -lean_dec(x_166); -x_169 = lean_st_ref_get(x_7, x_168); -x_170 = lean_ctor_get(x_169, 1); -lean_inc(x_170); -lean_dec(x_169); -x_171 = lean_st_ref_take(x_3, x_170); -x_172 = lean_ctor_get(x_171, 0); -lean_inc(x_172); -x_173 = lean_ctor_get(x_171, 1); -lean_inc(x_173); -lean_dec(x_171); -x_174 = lean_ctor_get(x_172, 0); -lean_inc(x_174); -lean_inc(x_167); -x_175 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_174, x_147, x_167); -x_176 = lean_ctor_get(x_172, 1); -lean_inc(x_176); -x_177 = lean_ctor_get(x_172, 2); -lean_inc(x_177); -x_178 = lean_ctor_get(x_172, 3); -lean_inc(x_178); -x_179 = lean_ctor_get(x_172, 4); -lean_inc(x_179); -x_180 = lean_ctor_get(x_172, 5); -lean_inc(x_180); -x_181 = lean_ctor_get(x_172, 6); -lean_inc(x_181); -x_182 = lean_ctor_get(x_172, 7); -lean_inc(x_182); -x_183 = lean_ctor_get(x_172, 8); -lean_inc(x_183); -x_184 = lean_ctor_get(x_172, 9); -lean_inc(x_184); -x_185 = lean_ctor_get(x_172, 10); -lean_inc(x_185); -x_186 = lean_ctor_get(x_172, 11); -lean_inc(x_186); -lean_dec(x_172); -x_187 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_187, 0, x_175); -lean_ctor_set(x_187, 1, x_176); -lean_ctor_set(x_187, 2, x_177); -lean_ctor_set(x_187, 3, x_178); -lean_ctor_set(x_187, 4, x_179); -lean_ctor_set(x_187, 5, x_180); -lean_ctor_set(x_187, 6, x_181); -lean_ctor_set(x_187, 7, x_182); -lean_ctor_set(x_187, 8, x_183); -lean_ctor_set(x_187, 9, x_184); -lean_ctor_set(x_187, 10, x_185); -lean_ctor_set(x_187, 11, x_186); -x_188 = lean_st_ref_set(x_3, x_187, x_173); -x_189 = lean_ctor_get(x_188, 1); -lean_inc(x_189); -lean_dec(x_188); -x_150 = x_167; -x_151 = x_189; -goto block_157; +lean_object* x_181; lean_object* x_182; +x_181 = l_Lean_simpLevelIMax_x27(x_165, x_167, x_1); +lean_dec(x_1); +x_182 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_182, 0, x_181); +lean_ctor_set(x_182, 1, x_168); +return x_182; +} +} } else { -lean_object* x_190; -lean_dec(x_147); -x_190 = lean_ctor_get(x_165, 0); -lean_inc(x_190); +lean_object* x_183; lean_object* x_184; lean_object* x_185; +lean_dec(x_167); lean_dec(x_165); -x_150 = x_190; -x_151 = x_163; -goto block_157; -} +lean_dec(x_1); +x_183 = l_Lean_Meta_Closure_collectLevelAux___closed__10; +x_184 = l_panic___at_Lean_Level_normalize___spec__1(x_183); +x_185 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_185, 0, x_184); +lean_ctor_set(x_185, 1, x_168); +return x_185; } } -block_230: +block_220: { -lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; -lean_dec(x_197); -x_198 = lean_st_ref_get(x_7, x_8); +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; +lean_dec(x_187); +x_188 = lean_st_ref_get(x_7, x_166); +x_189 = lean_ctor_get(x_188, 1); +lean_inc(x_189); +lean_dec(x_188); +x_190 = lean_st_ref_get(x_3, x_189); +x_191 = lean_ctor_get(x_190, 0); +lean_inc(x_191); +x_192 = lean_ctor_get(x_190, 1); +lean_inc(x_192); +lean_dec(x_190); +x_193 = lean_ctor_get(x_191, 0); +lean_inc(x_193); +lean_dec(x_191); +lean_inc(x_164); +x_194 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_193, x_164); +if (lean_obj_tag(x_194) == 0) +{ +lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; +lean_inc(x_164); +x_195 = l_Lean_Meta_Closure_collectLevelAux(x_164, x_2, x_3, x_4, x_5, x_6, x_7, x_192); +x_196 = lean_ctor_get(x_195, 0); +lean_inc(x_196); +x_197 = lean_ctor_get(x_195, 1); +lean_inc(x_197); +lean_dec(x_195); +x_198 = lean_st_ref_get(x_7, x_197); x_199 = lean_ctor_get(x_198, 1); lean_inc(x_199); lean_dec(x_198); -x_200 = lean_st_ref_get(x_3, x_199); +x_200 = lean_st_ref_take(x_3, x_199); x_201 = lean_ctor_get(x_200, 0); lean_inc(x_201); x_202 = lean_ctor_get(x_200, 1); @@ -2557,119 +2570,214 @@ lean_inc(x_202); lean_dec(x_200); x_203 = lean_ctor_get(x_201, 0); lean_inc(x_203); -lean_dec(x_201); -lean_inc(x_146); -x_204 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_203, x_146); -if (lean_obj_tag(x_204) == 0) -{ -lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; -lean_inc(x_146); -x_205 = l_Lean_Meta_Closure_collectLevelAux(x_146, x_2, x_3, x_4, x_5, x_6, x_7, x_202); -x_206 = lean_ctor_get(x_205, 0); +lean_inc(x_196); +x_204 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_203, x_164, x_196); +x_205 = lean_ctor_get(x_201, 1); +lean_inc(x_205); +x_206 = lean_ctor_get(x_201, 2); lean_inc(x_206); -x_207 = lean_ctor_get(x_205, 1); +x_207 = lean_ctor_get(x_201, 3); lean_inc(x_207); -lean_dec(x_205); -x_208 = lean_st_ref_get(x_7, x_207); -x_209 = lean_ctor_get(x_208, 1); +x_208 = lean_ctor_get(x_201, 4); +lean_inc(x_208); +x_209 = lean_ctor_get(x_201, 5); lean_inc(x_209); -lean_dec(x_208); -x_210 = lean_st_ref_take(x_3, x_209); -x_211 = lean_ctor_get(x_210, 0); +x_210 = lean_ctor_get(x_201, 6); +lean_inc(x_210); +x_211 = lean_ctor_get(x_201, 7); lean_inc(x_211); -x_212 = lean_ctor_get(x_210, 1); +x_212 = lean_ctor_get(x_201, 8); lean_inc(x_212); -lean_dec(x_210); -x_213 = lean_ctor_get(x_211, 0); +x_213 = lean_ctor_get(x_201, 9); lean_inc(x_213); -lean_inc(x_206); -x_214 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_213, x_146, x_206); -x_215 = lean_ctor_get(x_211, 1); +x_214 = lean_ctor_get(x_201, 10); +lean_inc(x_214); +x_215 = lean_ctor_get(x_201, 11); lean_inc(x_215); -x_216 = lean_ctor_get(x_211, 2); -lean_inc(x_216); -x_217 = lean_ctor_get(x_211, 3); -lean_inc(x_217); -x_218 = lean_ctor_get(x_211, 4); +lean_dec(x_201); +x_216 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_216, 0, x_204); +lean_ctor_set(x_216, 1, x_205); +lean_ctor_set(x_216, 2, x_206); +lean_ctor_set(x_216, 3, x_207); +lean_ctor_set(x_216, 4, x_208); +lean_ctor_set(x_216, 5, x_209); +lean_ctor_set(x_216, 6, x_210); +lean_ctor_set(x_216, 7, x_211); +lean_ctor_set(x_216, 8, x_212); +lean_ctor_set(x_216, 9, x_213); +lean_ctor_set(x_216, 10, x_214); +lean_ctor_set(x_216, 11, x_215); +x_217 = lean_st_ref_set(x_3, x_216, x_202); +x_218 = lean_ctor_get(x_217, 1); lean_inc(x_218); -x_219 = lean_ctor_get(x_211, 5); +lean_dec(x_217); +x_167 = x_196; +x_168 = x_218; +goto block_186; +} +else +{ +lean_object* x_219; +lean_dec(x_164); +x_219 = lean_ctor_get(x_194, 0); lean_inc(x_219); -x_220 = lean_ctor_get(x_211, 6); -lean_inc(x_220); -x_221 = lean_ctor_get(x_211, 7); -lean_inc(x_221); -x_222 = lean_ctor_get(x_211, 8); -lean_inc(x_222); -x_223 = lean_ctor_get(x_211, 9); -lean_inc(x_223); -x_224 = lean_ctor_get(x_211, 10); -lean_inc(x_224); -x_225 = lean_ctor_get(x_211, 11); -lean_inc(x_225); -lean_dec(x_211); -x_226 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_226, 0, x_214); -lean_ctor_set(x_226, 1, x_215); -lean_ctor_set(x_226, 2, x_216); -lean_ctor_set(x_226, 3, x_217); -lean_ctor_set(x_226, 4, x_218); -lean_ctor_set(x_226, 5, x_219); -lean_ctor_set(x_226, 6, x_220); -lean_ctor_set(x_226, 7, x_221); -lean_ctor_set(x_226, 8, x_222); -lean_ctor_set(x_226, 9, x_223); -lean_ctor_set(x_226, 10, x_224); -lean_ctor_set(x_226, 11, x_225); -x_227 = lean_st_ref_set(x_3, x_226, x_212); +lean_dec(x_194); +x_167 = x_219; +x_168 = x_192; +goto block_186; +} +} +} +block_259: +{ +lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; +lean_dec(x_226); +x_227 = lean_st_ref_get(x_7, x_8); x_228 = lean_ctor_get(x_227, 1); lean_inc(x_228); lean_dec(x_227); -x_148 = x_206; -x_149 = x_228; -goto block_196; +x_229 = lean_st_ref_get(x_3, x_228); +x_230 = lean_ctor_get(x_229, 0); +lean_inc(x_230); +x_231 = lean_ctor_get(x_229, 1); +lean_inc(x_231); +lean_dec(x_229); +x_232 = lean_ctor_get(x_230, 0); +lean_inc(x_232); +lean_dec(x_230); +lean_inc(x_163); +x_233 = l_Std_HashMapImp_find_x3f___at_Lean_Meta_Closure_visitLevel___spec__1(x_232, x_163); +if (lean_obj_tag(x_233) == 0) +{ +lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; +lean_inc(x_163); +x_234 = l_Lean_Meta_Closure_collectLevelAux(x_163, x_2, x_3, x_4, x_5, x_6, x_7, x_231); +x_235 = lean_ctor_get(x_234, 0); +lean_inc(x_235); +x_236 = lean_ctor_get(x_234, 1); +lean_inc(x_236); +lean_dec(x_234); +x_237 = lean_st_ref_get(x_7, x_236); +x_238 = lean_ctor_get(x_237, 1); +lean_inc(x_238); +lean_dec(x_237); +x_239 = lean_st_ref_take(x_3, x_238); +x_240 = lean_ctor_get(x_239, 0); +lean_inc(x_240); +x_241 = lean_ctor_get(x_239, 1); +lean_inc(x_241); +lean_dec(x_239); +x_242 = lean_ctor_get(x_240, 0); +lean_inc(x_242); +lean_inc(x_235); +x_243 = l_Std_HashMap_insert___at_Lean_Meta_Closure_visitLevel___spec__3(x_242, x_163, x_235); +x_244 = lean_ctor_get(x_240, 1); +lean_inc(x_244); +x_245 = lean_ctor_get(x_240, 2); +lean_inc(x_245); +x_246 = lean_ctor_get(x_240, 3); +lean_inc(x_246); +x_247 = lean_ctor_get(x_240, 4); +lean_inc(x_247); +x_248 = lean_ctor_get(x_240, 5); +lean_inc(x_248); +x_249 = lean_ctor_get(x_240, 6); +lean_inc(x_249); +x_250 = lean_ctor_get(x_240, 7); +lean_inc(x_250); +x_251 = lean_ctor_get(x_240, 8); +lean_inc(x_251); +x_252 = lean_ctor_get(x_240, 9); +lean_inc(x_252); +x_253 = lean_ctor_get(x_240, 10); +lean_inc(x_253); +x_254 = lean_ctor_get(x_240, 11); +lean_inc(x_254); +lean_dec(x_240); +x_255 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_255, 0, x_243); +lean_ctor_set(x_255, 1, x_244); +lean_ctor_set(x_255, 2, x_245); +lean_ctor_set(x_255, 3, x_246); +lean_ctor_set(x_255, 4, x_247); +lean_ctor_set(x_255, 5, x_248); +lean_ctor_set(x_255, 6, x_249); +lean_ctor_set(x_255, 7, x_250); +lean_ctor_set(x_255, 8, x_251); +lean_ctor_set(x_255, 9, x_252); +lean_ctor_set(x_255, 10, x_253); +lean_ctor_set(x_255, 11, x_254); +x_256 = lean_st_ref_set(x_3, x_255, x_241); +x_257 = lean_ctor_get(x_256, 1); +lean_inc(x_257); +lean_dec(x_256); +x_165 = x_235; +x_166 = x_257; +goto block_225; } else { -lean_object* x_229; -lean_dec(x_146); -x_229 = lean_ctor_get(x_204, 0); -lean_inc(x_229); -lean_dec(x_204); -x_148 = x_229; -x_149 = x_202; -goto block_196; +lean_object* x_258; +lean_dec(x_163); +x_258 = lean_ctor_get(x_233, 0); +lean_inc(x_258); +lean_dec(x_233); +x_165 = x_258; +x_166 = x_231; +goto block_225; } } } default: { -lean_object* x_235; -x_235 = l_Lean_Meta_Closure_mkNewLevelParam(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_235; +lean_object* x_264; +x_264 = l_Lean_Meta_Closure_mkNewLevelParam(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_264; } } -block_16: +block_21: { if (lean_obj_tag(x_1) == 1) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_level_update_succ(x_1, x_9); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -return x_12; +lean_object* x_11; size_t x_12; size_t x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +x_12 = lean_ptr_addr(x_11); +lean_dec(x_11); +x_13 = lean_ptr_addr(x_9); +x_14 = lean_usize_dec_eq(x_12, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = l_Lean_Level_succ___override(x_9); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_10); +return x_16; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_17; +lean_dec(x_9); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_17, 1, x_10); +return x_17; +} +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_dec(x_9); lean_dec(x_1); -x_13 = l_Lean_Meta_Closure_collectLevelAux___closed__4; -x_14 = l_panic___at_Lean_Level_normalize___spec__1(x_13); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_10); -return x_15; +x_18 = l_Lean_Meta_Closure_collectLevelAux___closed__4; +x_19 = l_panic___at_Lean_Level_normalize___spec__1(x_18); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_10); +return x_20; } } } @@ -3889,7 +3997,7 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateMData!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateMData!Impl", 47); return x_1; } } @@ -3907,8 +4015,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectExprAux___closed__1; x_2 = l_Lean_Meta_Closure_collectExprAux___closed__2; -x_3 = lean_unsigned_to_nat(1116u); -x_4 = lean_unsigned_to_nat(16u); +x_3 = lean_unsigned_to_nat(1434u); +x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_Meta_Closure_collectExprAux___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -3918,7 +4026,7 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateProj!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateProj!Impl", 46); return x_1; } } @@ -3936,8 +4044,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__7() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectExprAux___closed__1; x_2 = l_Lean_Meta_Closure_collectExprAux___closed__5; -x_3 = lean_unsigned_to_nat(1121u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1445u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Meta_Closure_collectExprAux___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -3947,7 +4055,7 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__8() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateApp!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateApp!Impl", 45); return x_1; } } @@ -3965,8 +4073,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__10() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectExprAux___closed__1; x_2 = l_Lean_Meta_Closure_collectExprAux___closed__8; -x_3 = lean_unsigned_to_nat(1081u); -x_4 = lean_unsigned_to_nat(14u); +x_3 = lean_unsigned_to_nat(1401u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Meta_Closure_collectExprAux___closed__9; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -3994,8 +4102,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__13() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectExprAux___closed__1; x_2 = l_Lean_Meta_Closure_collectExprAux___closed__11; -x_3 = lean_unsigned_to_nat(1149u); -x_4 = lean_unsigned_to_nat(19u); +x_3 = lean_unsigned_to_nat(1491u); +x_4 = lean_unsigned_to_nat(20u); x_5 = l_Lean_Meta_Closure_collectExprAux___closed__12; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -4023,8 +4131,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__16() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectExprAux___closed__1; x_2 = l_Lean_Meta_Closure_collectExprAux___closed__14; -x_3 = lean_unsigned_to_nat(1135u); -x_4 = lean_unsigned_to_nat(23u); +x_3 = lean_unsigned_to_nat(1471u); +x_4 = lean_unsigned_to_nat(24u); x_5 = l_Lean_Meta_Closure_collectExprAux___closed__15; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -4034,7 +4142,7 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__17() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateLet!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateLet!Impl", 45); return x_1; } } @@ -4052,8 +4160,8 @@ static lean_object* _init_l_Lean_Meta_Closure_collectExprAux___closed__19() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Closure_collectExprAux___closed__1; x_2 = l_Lean_Meta_Closure_collectExprAux___closed__17; -x_3 = lean_unsigned_to_nat(1158u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1500u); +x_4 = lean_unsigned_to_nat(22u); x_5 = l_Lean_Meta_Closure_collectExprAux___closed__18; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -4062,708 +4170,708 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Meta_Closure_collectExprAux(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) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_17; lean_object* x_18; +lean_object* x_9; lean_object* x_10; lean_object* x_23; lean_object* x_24; switch (lean_obj_tag(x_1)) { case 1: { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_1, 0); -lean_inc(x_25); +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_1, 0); +lean_inc(x_38); lean_dec(x_1); lean_inc(x_4); -lean_inc(x_25); -x_26 = l_Lean_Meta_getLocalDecl(x_25, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_26) == 0) +lean_inc(x_38); +x_39 = l_Lean_Meta_getLocalDecl(x_38, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_39) == 0) { if (x_2 == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -x_28 = l_Lean_mkFreshFVarId___at_Lean_Meta_Closure_collectExprAux___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_27); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -lean_inc(x_29); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_25); -lean_ctor_set(x_31, 1, x_29); -x_32 = l_Lean_Meta_Closure_pushToProcess(x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_30); +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_41 = l_Lean_mkFreshFVarId___at_Lean_Meta_Closure_collectExprAux___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_40); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +lean_inc(x_42); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_38); +lean_ctor_set(x_44, 1, x_42); +x_45 = l_Lean_Meta_Closure_pushToProcess(x_44, x_2, x_3, x_4, x_5, x_6, x_7, x_43); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) +x_46 = !lean_is_exclusive(x_45); +if (x_46 == 0) { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -lean_dec(x_34); -x_35 = l_Lean_Expr_fvar___override(x_29); -lean_ctor_set(x_32, 0, x_35); -return x_32; +lean_object* x_47; lean_object* x_48; +x_47 = lean_ctor_get(x_45, 0); +lean_dec(x_47); +x_48 = l_Lean_Expr_fvar___override(x_42); +lean_ctor_set(x_45, 0, x_48); +return x_45; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_32, 1); -lean_inc(x_36); -lean_dec(x_32); -x_37 = l_Lean_Expr_fvar___override(x_29); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_36); -return x_38; +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_45, 1); +lean_inc(x_49); +lean_dec(x_45); +x_50 = l_Lean_Expr_fvar___override(x_42); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_49); +return x_51; } } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_26, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_26, 1); -lean_inc(x_40); -lean_dec(x_26); -x_41 = l_Lean_LocalDecl_value_x3f(x_39); +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_39, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_39, 1); +lean_inc(x_53); lean_dec(x_39); -if (lean_obj_tag(x_41) == 0) +x_54 = l_Lean_LocalDecl_value_x3f(x_52); +lean_dec(x_52); +if (lean_obj_tag(x_54) == 0) { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_42 = l_Lean_mkFreshFVarId___at_Lean_Meta_Closure_collectExprAux___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_40); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_inc(x_43); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_25); -lean_ctor_set(x_45, 1, x_43); -x_46 = l_Lean_Meta_Closure_pushToProcess(x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_44); +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; +x_55 = l_Lean_mkFreshFVarId___at_Lean_Meta_Closure_collectExprAux___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_53); +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_56); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_38); +lean_ctor_set(x_58, 1, x_56); +x_59 = l_Lean_Meta_Closure_pushToProcess(x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_57); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +x_60 = !lean_is_exclusive(x_59); +if (x_60 == 0) { -lean_object* x_48; lean_object* x_49; -x_48 = lean_ctor_get(x_46, 0); -lean_dec(x_48); -x_49 = l_Lean_Expr_fvar___override(x_43); -lean_ctor_set(x_46, 0, x_49); -return x_46; +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_59, 0); +lean_dec(x_61); +x_62 = l_Lean_Expr_fvar___override(x_56); +lean_ctor_set(x_59, 0, x_62); +return x_59; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_46, 1); -lean_inc(x_50); -lean_dec(x_46); -x_51 = l_Lean_Expr_fvar___override(x_43); -x_52 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_50); -return x_52; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_59, 1); +lean_inc(x_63); +lean_dec(x_59); +x_64 = l_Lean_Expr_fvar___override(x_56); +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_63); +return x_65; } } else { -lean_object* x_53; lean_object* x_54; -lean_dec(x_25); -x_53 = lean_ctor_get(x_41, 0); -lean_inc(x_53); -lean_dec(x_41); +lean_object* x_66; lean_object* x_67; +lean_dec(x_38); +x_66 = lean_ctor_get(x_54, 0); +lean_inc(x_66); +lean_dec(x_54); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_54 = l_Lean_Meta_Closure_preprocess(x_53, x_2, x_3, x_4, x_5, x_6, x_7, x_40); -if (lean_obj_tag(x_54) == 0) +x_67 = l_Lean_Meta_Closure_preprocess(x_66, x_2, x_3, x_4, x_5, x_6, x_7, x_53); +if (lean_obj_tag(x_67) == 0) { -uint8_t x_55; -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) +uint8_t x_68; +x_68 = !lean_is_exclusive(x_67); +if (x_68 == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_136; -x_56 = lean_ctor_get(x_54, 0); -x_57 = lean_ctor_get(x_54, 1); -x_136 = l_Lean_Expr_hasLevelParam(x_56); -if (x_136 == 0) +lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_149; +x_69 = lean_ctor_get(x_67, 0); +x_70 = lean_ctor_get(x_67, 1); +x_149 = l_Lean_Expr_hasLevelParam(x_69); +if (x_149 == 0) { -uint8_t x_137; -x_137 = l_Lean_Expr_hasFVar(x_56); -if (x_137 == 0) +uint8_t x_150; +x_150 = l_Lean_Expr_hasFVar(x_69); +if (x_150 == 0) { -uint8_t x_138; -x_138 = l_Lean_Expr_hasMVar(x_56); -if (x_138 == 0) +uint8_t x_151; +x_151 = l_Lean_Expr_hasMVar(x_69); +if (x_151 == 0) { lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_54; +return x_67; } else { -lean_object* x_139; -lean_free_object(x_54); -x_139 = lean_box(0); -x_58 = x_139; -goto block_135; +lean_object* x_152; +lean_free_object(x_67); +x_152 = lean_box(0); +x_71 = x_152; +goto block_148; } } else { -lean_object* x_140; -lean_free_object(x_54); -x_140 = lean_box(0); -x_58 = x_140; -goto block_135; +lean_object* x_153; +lean_free_object(x_67); +x_153 = lean_box(0); +x_71 = x_153; +goto block_148; } } else { -lean_object* x_141; -lean_free_object(x_54); -x_141 = lean_box(0); -x_58 = x_141; -goto block_135; +lean_object* x_154; +lean_free_object(x_67); +x_154 = lean_box(0); +x_71 = x_154; +goto block_148; } -block_135: +block_148: { -lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; -lean_dec(x_58); -x_59 = lean_st_ref_get(x_7, x_57); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_st_ref_get(x_3, x_60); -x_62 = !lean_is_exclusive(x_61); -if (x_62 == 0) -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_63 = lean_ctor_get(x_61, 0); -x_64 = lean_ctor_get(x_61, 1); -x_65 = lean_ctor_get(x_63, 1); -lean_inc(x_65); -lean_dec(x_63); -lean_inc(x_56); -x_66 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_65, x_56); -if (lean_obj_tag(x_66) == 0) -{ -lean_object* x_67; -lean_free_object(x_61); -lean_inc(x_7); -lean_inc(x_56); -x_67 = l_Lean_Meta_Closure_collectExprAux(x_56, x_2, x_3, x_4, x_5, x_6, x_7, x_64); -if (lean_obj_tag(x_67) == 0) -{ -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_st_ref_get(x_7, x_69); -lean_dec(x_7); -x_71 = lean_ctor_get(x_70, 1); -lean_inc(x_71); -lean_dec(x_70); -x_72 = lean_st_ref_take(x_3, x_71); -x_73 = lean_ctor_get(x_72, 0); +lean_object* x_72; lean_object* x_73; lean_object* x_74; uint8_t x_75; +lean_dec(x_71); +x_72 = lean_st_ref_get(x_7, x_70); +x_73 = lean_ctor_get(x_72, 1); lean_inc(x_73); -x_74 = lean_ctor_get(x_72, 1); -lean_inc(x_74); lean_dec(x_72); -x_75 = lean_ctor_get(x_73, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_73, 1); -lean_inc(x_76); -lean_inc(x_68); -x_77 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_76, x_56, x_68); -x_78 = lean_ctor_get(x_73, 2); +x_74 = lean_st_ref_get(x_3, x_73); +x_75 = !lean_is_exclusive(x_74); +if (x_75 == 0) +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_76 = lean_ctor_get(x_74, 0); +x_77 = lean_ctor_get(x_74, 1); +x_78 = lean_ctor_get(x_76, 1); lean_inc(x_78); -x_79 = lean_ctor_get(x_73, 3); -lean_inc(x_79); -x_80 = lean_ctor_get(x_73, 4); -lean_inc(x_80); -x_81 = lean_ctor_get(x_73, 5); +lean_dec(x_76); +lean_inc(x_69); +x_79 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_78, x_69); +if (lean_obj_tag(x_79) == 0) +{ +lean_object* x_80; +lean_free_object(x_74); +lean_inc(x_7); +lean_inc(x_69); +x_80 = l_Lean_Meta_Closure_collectExprAux(x_69, x_2, x_3, x_4, x_5, x_6, x_7, x_77); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; 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; uint8_t x_103; +x_81 = lean_ctor_get(x_80, 0); lean_inc(x_81); -x_82 = lean_ctor_get(x_73, 6); +x_82 = lean_ctor_get(x_80, 1); lean_inc(x_82); -x_83 = lean_ctor_get(x_73, 7); -lean_inc(x_83); -x_84 = lean_ctor_get(x_73, 8); +lean_dec(x_80); +x_83 = lean_st_ref_get(x_7, x_82); +lean_dec(x_7); +x_84 = lean_ctor_get(x_83, 1); lean_inc(x_84); -x_85 = lean_ctor_get(x_73, 9); -lean_inc(x_85); -x_86 = lean_ctor_get(x_73, 10); +lean_dec(x_83); +x_85 = lean_st_ref_take(x_3, x_84); +x_86 = lean_ctor_get(x_85, 0); lean_inc(x_86); -x_87 = lean_ctor_get(x_73, 11); +x_87 = lean_ctor_get(x_85, 1); lean_inc(x_87); -lean_dec(x_73); -x_88 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_88, 0, x_75); -lean_ctor_set(x_88, 1, x_77); -lean_ctor_set(x_88, 2, x_78); -lean_ctor_set(x_88, 3, x_79); -lean_ctor_set(x_88, 4, x_80); -lean_ctor_set(x_88, 5, x_81); -lean_ctor_set(x_88, 6, x_82); -lean_ctor_set(x_88, 7, x_83); -lean_ctor_set(x_88, 8, x_84); -lean_ctor_set(x_88, 9, x_85); -lean_ctor_set(x_88, 10, x_86); -lean_ctor_set(x_88, 11, x_87); -x_89 = lean_st_ref_set(x_3, x_88, x_74); -x_90 = !lean_is_exclusive(x_89); -if (x_90 == 0) +lean_dec(x_85); +x_88 = lean_ctor_get(x_86, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_86, 1); +lean_inc(x_89); +lean_inc(x_81); +x_90 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_89, x_69, x_81); +x_91 = lean_ctor_get(x_86, 2); +lean_inc(x_91); +x_92 = lean_ctor_get(x_86, 3); +lean_inc(x_92); +x_93 = lean_ctor_get(x_86, 4); +lean_inc(x_93); +x_94 = lean_ctor_get(x_86, 5); +lean_inc(x_94); +x_95 = lean_ctor_get(x_86, 6); +lean_inc(x_95); +x_96 = lean_ctor_get(x_86, 7); +lean_inc(x_96); +x_97 = lean_ctor_get(x_86, 8); +lean_inc(x_97); +x_98 = lean_ctor_get(x_86, 9); +lean_inc(x_98); +x_99 = lean_ctor_get(x_86, 10); +lean_inc(x_99); +x_100 = lean_ctor_get(x_86, 11); +lean_inc(x_100); +lean_dec(x_86); +x_101 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_101, 0, x_88); +lean_ctor_set(x_101, 1, x_90); +lean_ctor_set(x_101, 2, x_91); +lean_ctor_set(x_101, 3, x_92); +lean_ctor_set(x_101, 4, x_93); +lean_ctor_set(x_101, 5, x_94); +lean_ctor_set(x_101, 6, x_95); +lean_ctor_set(x_101, 7, x_96); +lean_ctor_set(x_101, 8, x_97); +lean_ctor_set(x_101, 9, x_98); +lean_ctor_set(x_101, 10, x_99); +lean_ctor_set(x_101, 11, x_100); +x_102 = lean_st_ref_set(x_3, x_101, x_87); +x_103 = !lean_is_exclusive(x_102); +if (x_103 == 0) { -lean_object* x_91; -x_91 = lean_ctor_get(x_89, 0); -lean_dec(x_91); -lean_ctor_set(x_89, 0, x_68); -return x_89; +lean_object* x_104; +x_104 = lean_ctor_get(x_102, 0); +lean_dec(x_104); +lean_ctor_set(x_102, 0, x_81); +return x_102; } else { -lean_object* x_92; lean_object* x_93; -x_92 = lean_ctor_get(x_89, 1); -lean_inc(x_92); -lean_dec(x_89); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_68); -lean_ctor_set(x_93, 1, x_92); -return x_93; +lean_object* x_105; lean_object* x_106; +x_105 = lean_ctor_get(x_102, 1); +lean_inc(x_105); +lean_dec(x_102); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_81); +lean_ctor_set(x_106, 1, x_105); +return x_106; } } else { -uint8_t x_94; -lean_dec(x_56); +uint8_t x_107; +lean_dec(x_69); lean_dec(x_7); -x_94 = !lean_is_exclusive(x_67); -if (x_94 == 0) +x_107 = !lean_is_exclusive(x_80); +if (x_107 == 0) { -return x_67; +return x_80; } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_95 = lean_ctor_get(x_67, 0); -x_96 = lean_ctor_get(x_67, 1); -lean_inc(x_96); -lean_inc(x_95); -lean_dec(x_67); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set(x_97, 1, x_96); -return x_97; +lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_80, 0); +x_109 = lean_ctor_get(x_80, 1); +lean_inc(x_109); +lean_inc(x_108); +lean_dec(x_80); +x_110 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_110, 0, x_108); +lean_ctor_set(x_110, 1, x_109); +return x_110; } } } else { -lean_object* x_98; -lean_dec(x_56); +lean_object* x_111; +lean_dec(x_69); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_98 = lean_ctor_get(x_66, 0); -lean_inc(x_98); -lean_dec(x_66); -lean_ctor_set(x_61, 0, x_98); -return x_61; +x_111 = lean_ctor_get(x_79, 0); +lean_inc(x_111); +lean_dec(x_79); +lean_ctor_set(x_74, 0, x_111); +return x_74; } } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_99 = lean_ctor_get(x_61, 0); -x_100 = lean_ctor_get(x_61, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_61); -x_101 = lean_ctor_get(x_99, 1); -lean_inc(x_101); -lean_dec(x_99); -lean_inc(x_56); -x_102 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_101, x_56); -if (lean_obj_tag(x_102) == 0) +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_112 = lean_ctor_get(x_74, 0); +x_113 = lean_ctor_get(x_74, 1); +lean_inc(x_113); +lean_inc(x_112); +lean_dec(x_74); +x_114 = lean_ctor_get(x_112, 1); +lean_inc(x_114); +lean_dec(x_112); +lean_inc(x_69); +x_115 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_114, x_69); +if (lean_obj_tag(x_115) == 0) { -lean_object* x_103; +lean_object* x_116; lean_inc(x_7); -lean_inc(x_56); -x_103 = l_Lean_Meta_Closure_collectExprAux(x_56, x_2, x_3, x_4, x_5, x_6, x_7, x_100); -if (lean_obj_tag(x_103) == 0) +lean_inc(x_69); +x_116 = l_Lean_Meta_Closure_collectExprAux(x_69, x_2, x_3, x_4, x_5, x_6, x_7, x_113); +if (lean_obj_tag(x_116) == 0) { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_104 = lean_ctor_get(x_103, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_103, 1); -lean_inc(x_105); -lean_dec(x_103); -x_106 = lean_st_ref_get(x_7, x_105); -lean_dec(x_7); -x_107 = lean_ctor_get(x_106, 1); -lean_inc(x_107); -lean_dec(x_106); -x_108 = lean_st_ref_take(x_3, x_107); -x_109 = lean_ctor_get(x_108, 0); -lean_inc(x_109); -x_110 = lean_ctor_get(x_108, 1); -lean_inc(x_110); -lean_dec(x_108); -x_111 = lean_ctor_get(x_109, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_109, 1); -lean_inc(x_112); -lean_inc(x_104); -x_113 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_112, x_56, x_104); -x_114 = lean_ctor_get(x_109, 2); -lean_inc(x_114); -x_115 = lean_ctor_get(x_109, 3); -lean_inc(x_115); -x_116 = lean_ctor_get(x_109, 4); -lean_inc(x_116); -x_117 = lean_ctor_get(x_109, 5); +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; +x_117 = lean_ctor_get(x_116, 0); lean_inc(x_117); -x_118 = lean_ctor_get(x_109, 6); +x_118 = lean_ctor_get(x_116, 1); lean_inc(x_118); -x_119 = lean_ctor_get(x_109, 7); -lean_inc(x_119); -x_120 = lean_ctor_get(x_109, 8); +lean_dec(x_116); +x_119 = lean_st_ref_get(x_7, x_118); +lean_dec(x_7); +x_120 = lean_ctor_get(x_119, 1); lean_inc(x_120); -x_121 = lean_ctor_get(x_109, 9); -lean_inc(x_121); -x_122 = lean_ctor_get(x_109, 10); +lean_dec(x_119); +x_121 = lean_st_ref_take(x_3, x_120); +x_122 = lean_ctor_get(x_121, 0); lean_inc(x_122); -x_123 = lean_ctor_get(x_109, 11); +x_123 = lean_ctor_get(x_121, 1); lean_inc(x_123); -lean_dec(x_109); -x_124 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_124, 0, x_111); -lean_ctor_set(x_124, 1, x_113); -lean_ctor_set(x_124, 2, x_114); -lean_ctor_set(x_124, 3, x_115); -lean_ctor_set(x_124, 4, x_116); -lean_ctor_set(x_124, 5, x_117); -lean_ctor_set(x_124, 6, x_118); -lean_ctor_set(x_124, 7, x_119); -lean_ctor_set(x_124, 8, x_120); -lean_ctor_set(x_124, 9, x_121); -lean_ctor_set(x_124, 10, x_122); -lean_ctor_set(x_124, 11, x_123); -x_125 = lean_st_ref_set(x_3, x_124, x_110); -x_126 = lean_ctor_get(x_125, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - x_127 = x_125; +lean_dec(x_121); +x_124 = lean_ctor_get(x_122, 0); +lean_inc(x_124); +x_125 = lean_ctor_get(x_122, 1); +lean_inc(x_125); +lean_inc(x_117); +x_126 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_125, x_69, x_117); +x_127 = lean_ctor_get(x_122, 2); +lean_inc(x_127); +x_128 = lean_ctor_get(x_122, 3); +lean_inc(x_128); +x_129 = lean_ctor_get(x_122, 4); +lean_inc(x_129); +x_130 = lean_ctor_get(x_122, 5); +lean_inc(x_130); +x_131 = lean_ctor_get(x_122, 6); +lean_inc(x_131); +x_132 = lean_ctor_get(x_122, 7); +lean_inc(x_132); +x_133 = lean_ctor_get(x_122, 8); +lean_inc(x_133); +x_134 = lean_ctor_get(x_122, 9); +lean_inc(x_134); +x_135 = lean_ctor_get(x_122, 10); +lean_inc(x_135); +x_136 = lean_ctor_get(x_122, 11); +lean_inc(x_136); +lean_dec(x_122); +x_137 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_137, 0, x_124); +lean_ctor_set(x_137, 1, x_126); +lean_ctor_set(x_137, 2, x_127); +lean_ctor_set(x_137, 3, x_128); +lean_ctor_set(x_137, 4, x_129); +lean_ctor_set(x_137, 5, x_130); +lean_ctor_set(x_137, 6, x_131); +lean_ctor_set(x_137, 7, x_132); +lean_ctor_set(x_137, 8, x_133); +lean_ctor_set(x_137, 9, x_134); +lean_ctor_set(x_137, 10, x_135); +lean_ctor_set(x_137, 11, x_136); +x_138 = lean_st_ref_set(x_3, x_137, x_123); +x_139 = lean_ctor_get(x_138, 1); +lean_inc(x_139); +if (lean_is_exclusive(x_138)) { + lean_ctor_release(x_138, 0); + lean_ctor_release(x_138, 1); + x_140 = x_138; } else { - lean_dec_ref(x_125); - x_127 = lean_box(0); + lean_dec_ref(x_138); + x_140 = lean_box(0); } -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_140)) { + x_141 = lean_alloc_ctor(0, 2, 0); } else { - x_128 = x_127; + x_141 = x_140; } -lean_ctor_set(x_128, 0, x_104); -lean_ctor_set(x_128, 1, x_126); -return x_128; +lean_ctor_set(x_141, 0, x_117); +lean_ctor_set(x_141, 1, x_139); +return x_141; } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -lean_dec(x_56); +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +lean_dec(x_69); lean_dec(x_7); -x_129 = lean_ctor_get(x_103, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_103, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_103)) { - lean_ctor_release(x_103, 0); - lean_ctor_release(x_103, 1); - x_131 = x_103; +x_142 = lean_ctor_get(x_116, 0); +lean_inc(x_142); +x_143 = lean_ctor_get(x_116, 1); +lean_inc(x_143); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_144 = x_116; } else { - lean_dec_ref(x_103); - x_131 = lean_box(0); + lean_dec_ref(x_116); + x_144 = lean_box(0); } -if (lean_is_scalar(x_131)) { - x_132 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_144)) { + x_145 = lean_alloc_ctor(1, 2, 0); } else { - x_132 = x_131; + x_145 = x_144; } -lean_ctor_set(x_132, 0, x_129); -lean_ctor_set(x_132, 1, x_130); -return x_132; +lean_ctor_set(x_145, 0, x_142); +lean_ctor_set(x_145, 1, x_143); +return x_145; } } else { -lean_object* x_133; lean_object* x_134; -lean_dec(x_56); +lean_object* x_146; lean_object* x_147; +lean_dec(x_69); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_133 = lean_ctor_get(x_102, 0); -lean_inc(x_133); -lean_dec(x_102); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_133); -lean_ctor_set(x_134, 1, x_100); -return x_134; +x_146 = lean_ctor_get(x_115, 0); +lean_inc(x_146); +lean_dec(x_115); +x_147 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_113); +return x_147; } } } } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; uint8_t x_186; -x_142 = lean_ctor_get(x_54, 0); -x_143 = lean_ctor_get(x_54, 1); -lean_inc(x_143); -lean_inc(x_142); -lean_dec(x_54); -x_186 = l_Lean_Expr_hasLevelParam(x_142); -if (x_186 == 0) +lean_object* x_155; lean_object* x_156; lean_object* x_157; uint8_t x_199; +x_155 = lean_ctor_get(x_67, 0); +x_156 = lean_ctor_get(x_67, 1); +lean_inc(x_156); +lean_inc(x_155); +lean_dec(x_67); +x_199 = l_Lean_Expr_hasLevelParam(x_155); +if (x_199 == 0) { -uint8_t x_187; -x_187 = l_Lean_Expr_hasFVar(x_142); -if (x_187 == 0) +uint8_t x_200; +x_200 = l_Lean_Expr_hasFVar(x_155); +if (x_200 == 0) { -uint8_t x_188; -x_188 = l_Lean_Expr_hasMVar(x_142); -if (x_188 == 0) +uint8_t x_201; +x_201 = l_Lean_Expr_hasMVar(x_155); +if (x_201 == 0) { -lean_object* x_189; +lean_object* x_202; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_189 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_189, 0, x_142); -lean_ctor_set(x_189, 1, x_143); -return x_189; +x_202 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_202, 0, x_155); +lean_ctor_set(x_202, 1, x_156); +return x_202; } else { -lean_object* x_190; -x_190 = lean_box(0); -x_144 = x_190; -goto block_185; +lean_object* x_203; +x_203 = lean_box(0); +x_157 = x_203; +goto block_198; } } else { -lean_object* x_191; -x_191 = lean_box(0); -x_144 = x_191; -goto block_185; +lean_object* x_204; +x_204 = lean_box(0); +x_157 = x_204; +goto block_198; } } else { -lean_object* x_192; -x_192 = lean_box(0); -x_144 = x_192; -goto block_185; +lean_object* x_205; +x_205 = lean_box(0); +x_157 = x_205; +goto block_198; } -block_185: +block_198: { -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_dec(x_144); -x_145 = lean_st_ref_get(x_7, x_143); -x_146 = lean_ctor_get(x_145, 1); -lean_inc(x_146); -lean_dec(x_145); -x_147 = lean_st_ref_get(x_3, x_146); -x_148 = lean_ctor_get(x_147, 0); -lean_inc(x_148); -x_149 = lean_ctor_get(x_147, 1); -lean_inc(x_149); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_150 = x_147; -} else { - lean_dec_ref(x_147); - x_150 = lean_box(0); -} -x_151 = lean_ctor_get(x_148, 1); -lean_inc(x_151); -lean_dec(x_148); -lean_inc(x_142); -x_152 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_151, x_142); -if (lean_obj_tag(x_152) == 0) -{ -lean_object* x_153; -lean_dec(x_150); -lean_inc(x_7); -lean_inc(x_142); -x_153 = l_Lean_Meta_Closure_collectExprAux(x_142, x_2, x_3, x_4, x_5, x_6, x_7, x_149); -if (lean_obj_tag(x_153) == 0) -{ -lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_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); -x_156 = lean_st_ref_get(x_7, x_155); -lean_dec(x_7); -x_157 = lean_ctor_get(x_156, 1); -lean_inc(x_157); -lean_dec(x_156); -x_158 = lean_st_ref_take(x_3, x_157); -x_159 = lean_ctor_get(x_158, 0); +lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_dec(x_157); +x_158 = lean_st_ref_get(x_7, x_156); +x_159 = lean_ctor_get(x_158, 1); lean_inc(x_159); -x_160 = lean_ctor_get(x_158, 1); -lean_inc(x_160); lean_dec(x_158); -x_161 = lean_ctor_get(x_159, 0); +x_160 = lean_st_ref_get(x_3, x_159); +x_161 = lean_ctor_get(x_160, 0); lean_inc(x_161); -x_162 = lean_ctor_get(x_159, 1); +x_162 = lean_ctor_get(x_160, 1); lean_inc(x_162); -lean_inc(x_154); -x_163 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_162, x_142, x_154); -x_164 = lean_ctor_get(x_159, 2); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_163 = x_160; +} else { + lean_dec_ref(x_160); + x_163 = lean_box(0); +} +x_164 = lean_ctor_get(x_161, 1); lean_inc(x_164); -x_165 = lean_ctor_get(x_159, 3); -lean_inc(x_165); -x_166 = lean_ctor_get(x_159, 4); -lean_inc(x_166); -x_167 = lean_ctor_get(x_159, 5); +lean_dec(x_161); +lean_inc(x_155); +x_165 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_164, x_155); +if (lean_obj_tag(x_165) == 0) +{ +lean_object* x_166; +lean_dec(x_163); +lean_inc(x_7); +lean_inc(x_155); +x_166 = l_Lean_Meta_Closure_collectExprAux(x_155, x_2, x_3, x_4, x_5, x_6, x_7, x_162); +if (lean_obj_tag(x_166) == 0) +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +x_167 = lean_ctor_get(x_166, 0); lean_inc(x_167); -x_168 = lean_ctor_get(x_159, 6); +x_168 = lean_ctor_get(x_166, 1); lean_inc(x_168); -x_169 = lean_ctor_get(x_159, 7); -lean_inc(x_169); -x_170 = lean_ctor_get(x_159, 8); +lean_dec(x_166); +x_169 = lean_st_ref_get(x_7, x_168); +lean_dec(x_7); +x_170 = lean_ctor_get(x_169, 1); lean_inc(x_170); -x_171 = lean_ctor_get(x_159, 9); -lean_inc(x_171); -x_172 = lean_ctor_get(x_159, 10); +lean_dec(x_169); +x_171 = lean_st_ref_take(x_3, x_170); +x_172 = lean_ctor_get(x_171, 0); lean_inc(x_172); -x_173 = lean_ctor_get(x_159, 11); +x_173 = lean_ctor_get(x_171, 1); lean_inc(x_173); -lean_dec(x_159); -x_174 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_174, 0, x_161); -lean_ctor_set(x_174, 1, x_163); -lean_ctor_set(x_174, 2, x_164); -lean_ctor_set(x_174, 3, x_165); -lean_ctor_set(x_174, 4, x_166); -lean_ctor_set(x_174, 5, x_167); -lean_ctor_set(x_174, 6, x_168); -lean_ctor_set(x_174, 7, x_169); -lean_ctor_set(x_174, 8, x_170); -lean_ctor_set(x_174, 9, x_171); -lean_ctor_set(x_174, 10, x_172); -lean_ctor_set(x_174, 11, x_173); -x_175 = lean_st_ref_set(x_3, x_174, x_160); -x_176 = lean_ctor_get(x_175, 1); -lean_inc(x_176); -if (lean_is_exclusive(x_175)) { - lean_ctor_release(x_175, 0); - lean_ctor_release(x_175, 1); - x_177 = x_175; +lean_dec(x_171); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 1); +lean_inc(x_175); +lean_inc(x_167); +x_176 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_175, x_155, x_167); +x_177 = lean_ctor_get(x_172, 2); +lean_inc(x_177); +x_178 = lean_ctor_get(x_172, 3); +lean_inc(x_178); +x_179 = lean_ctor_get(x_172, 4); +lean_inc(x_179); +x_180 = lean_ctor_get(x_172, 5); +lean_inc(x_180); +x_181 = lean_ctor_get(x_172, 6); +lean_inc(x_181); +x_182 = lean_ctor_get(x_172, 7); +lean_inc(x_182); +x_183 = lean_ctor_get(x_172, 8); +lean_inc(x_183); +x_184 = lean_ctor_get(x_172, 9); +lean_inc(x_184); +x_185 = lean_ctor_get(x_172, 10); +lean_inc(x_185); +x_186 = lean_ctor_get(x_172, 11); +lean_inc(x_186); +lean_dec(x_172); +x_187 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_187, 0, x_174); +lean_ctor_set(x_187, 1, x_176); +lean_ctor_set(x_187, 2, x_177); +lean_ctor_set(x_187, 3, x_178); +lean_ctor_set(x_187, 4, x_179); +lean_ctor_set(x_187, 5, x_180); +lean_ctor_set(x_187, 6, x_181); +lean_ctor_set(x_187, 7, x_182); +lean_ctor_set(x_187, 8, x_183); +lean_ctor_set(x_187, 9, x_184); +lean_ctor_set(x_187, 10, x_185); +lean_ctor_set(x_187, 11, x_186); +x_188 = lean_st_ref_set(x_3, x_187, x_173); +x_189 = lean_ctor_get(x_188, 1); +lean_inc(x_189); +if (lean_is_exclusive(x_188)) { + lean_ctor_release(x_188, 0); + lean_ctor_release(x_188, 1); + x_190 = x_188; } else { - lean_dec_ref(x_175); - x_177 = lean_box(0); + lean_dec_ref(x_188); + x_190 = lean_box(0); } -if (lean_is_scalar(x_177)) { - x_178 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_190)) { + x_191 = lean_alloc_ctor(0, 2, 0); } else { - x_178 = x_177; + x_191 = x_190; } -lean_ctor_set(x_178, 0, x_154); -lean_ctor_set(x_178, 1, x_176); -return x_178; +lean_ctor_set(x_191, 0, x_167); +lean_ctor_set(x_191, 1, x_189); +return x_191; } else { -lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -lean_dec(x_142); +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +lean_dec(x_155); lean_dec(x_7); -x_179 = lean_ctor_get(x_153, 0); -lean_inc(x_179); -x_180 = lean_ctor_get(x_153, 1); -lean_inc(x_180); -if (lean_is_exclusive(x_153)) { - lean_ctor_release(x_153, 0); - lean_ctor_release(x_153, 1); - x_181 = x_153; +x_192 = lean_ctor_get(x_166, 0); +lean_inc(x_192); +x_193 = lean_ctor_get(x_166, 1); +lean_inc(x_193); +if (lean_is_exclusive(x_166)) { + lean_ctor_release(x_166, 0); + lean_ctor_release(x_166, 1); + x_194 = x_166; } else { - lean_dec_ref(x_153); - x_181 = lean_box(0); + lean_dec_ref(x_166); + x_194 = lean_box(0); } -if (lean_is_scalar(x_181)) { - x_182 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_194)) { + x_195 = lean_alloc_ctor(1, 2, 0); } else { - x_182 = x_181; + x_195 = x_194; } -lean_ctor_set(x_182, 0, x_179); -lean_ctor_set(x_182, 1, x_180); -return x_182; +lean_ctor_set(x_195, 0, x_192); +lean_ctor_set(x_195, 1, x_193); +return x_195; } } else { -lean_object* x_183; lean_object* x_184; -lean_dec(x_142); +lean_object* x_196; lean_object* x_197; +lean_dec(x_155); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_183 = lean_ctor_get(x_152, 0); -lean_inc(x_183); -lean_dec(x_152); -if (lean_is_scalar(x_150)) { - x_184 = lean_alloc_ctor(0, 2, 0); +x_196 = lean_ctor_get(x_165, 0); +lean_inc(x_196); +lean_dec(x_165); +if (lean_is_scalar(x_163)) { + x_197 = lean_alloc_ctor(0, 2, 0); } else { - x_184 = x_150; + x_197 = x_163; } -lean_ctor_set(x_184, 0, x_183); -lean_ctor_set(x_184, 1, x_149); -return x_184; +lean_ctor_set(x_197, 0, x_196); +lean_ctor_set(x_197, 1, x_162); +return x_197; } } } } else { -uint8_t x_193; +uint8_t x_206; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_193 = !lean_is_exclusive(x_54); -if (x_193 == 0) +x_206 = !lean_is_exclusive(x_67); +if (x_206 == 0) { -return x_54; +return x_67; } else { -lean_object* x_194; lean_object* x_195; lean_object* x_196; -x_194 = lean_ctor_get(x_54, 0); -x_195 = lean_ctor_get(x_54, 1); -lean_inc(x_195); -lean_inc(x_194); -lean_dec(x_54); -x_196 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_196, 0, x_194); -lean_ctor_set(x_196, 1, x_195); -return x_196; +lean_object* x_207; lean_object* x_208; lean_object* x_209; +x_207 = lean_ctor_get(x_67, 0); +x_208 = lean_ctor_get(x_67, 1); +lean_inc(x_208); +lean_inc(x_207); +lean_dec(x_67); +x_209 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_209, 0, x_207); +lean_ctor_set(x_209, 1, x_208); +return x_209; } } } @@ -4771,2623 +4879,2981 @@ return x_196; } else { -uint8_t x_197; -lean_dec(x_25); +uint8_t x_210; +lean_dec(x_38); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_197 = !lean_is_exclusive(x_26); -if (x_197 == 0) +x_210 = !lean_is_exclusive(x_39); +if (x_210 == 0) { -return x_26; +return x_39; } else { -lean_object* x_198; lean_object* x_199; lean_object* x_200; -x_198 = lean_ctor_get(x_26, 0); -x_199 = lean_ctor_get(x_26, 1); -lean_inc(x_199); -lean_inc(x_198); -lean_dec(x_26); -x_200 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_200, 0, x_198); -lean_ctor_set(x_200, 1, x_199); -return x_200; +lean_object* x_211; lean_object* x_212; lean_object* x_213; +x_211 = lean_ctor_get(x_39, 0); +x_212 = lean_ctor_get(x_39, 1); +lean_inc(x_212); +lean_inc(x_211); +lean_dec(x_39); +x_213 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_213, 0, x_211); +lean_ctor_set(x_213, 1, x_212); +return x_213; } } } case 2: { -lean_object* x_201; lean_object* x_202; -x_201 = lean_ctor_get(x_1, 0); -lean_inc(x_201); -x_202 = l_Lean_Meta_getMVarDecl(x_201, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_202) == 0) +lean_object* x_214; lean_object* x_215; +x_214 = lean_ctor_get(x_1, 0); +lean_inc(x_214); +x_215 = l_Lean_Meta_getMVarDecl(x_214, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_215) == 0) { -lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; -x_203 = lean_ctor_get(x_202, 0); -lean_inc(x_203); -x_204 = lean_ctor_get(x_202, 1); -lean_inc(x_204); -lean_dec(x_202); -x_205 = lean_ctor_get(x_203, 2); -lean_inc(x_205); -lean_dec(x_203); +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +x_216 = lean_ctor_get(x_215, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_215, 1); +lean_inc(x_217); +lean_dec(x_215); +x_218 = lean_ctor_get(x_216, 2); +lean_inc(x_218); +lean_dec(x_216); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_206 = l_Lean_Meta_Closure_preprocess(x_205, x_2, x_3, x_4, x_5, x_6, x_7, x_204); -if (lean_obj_tag(x_206) == 0) +x_219 = l_Lean_Meta_Closure_preprocess(x_218, x_2, x_3, x_4, x_5, x_6, x_7, x_217); +if (lean_obj_tag(x_219) == 0) { -lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_248; uint8_t x_286; -x_207 = lean_ctor_get(x_206, 0); -lean_inc(x_207); -x_208 = lean_ctor_get(x_206, 1); -lean_inc(x_208); -lean_dec(x_206); -x_286 = l_Lean_Expr_hasLevelParam(x_207); -if (x_286 == 0) +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_261; uint8_t x_299; +x_220 = lean_ctor_get(x_219, 0); +lean_inc(x_220); +x_221 = lean_ctor_get(x_219, 1); +lean_inc(x_221); +lean_dec(x_219); +x_299 = l_Lean_Expr_hasLevelParam(x_220); +if (x_299 == 0) { -uint8_t x_287; -x_287 = l_Lean_Expr_hasFVar(x_207); -if (x_287 == 0) +uint8_t x_300; +x_300 = l_Lean_Expr_hasFVar(x_220); +if (x_300 == 0) { -uint8_t x_288; -x_288 = l_Lean_Expr_hasMVar(x_207); -if (x_288 == 0) +uint8_t x_301; +x_301 = l_Lean_Expr_hasMVar(x_220); +if (x_301 == 0) { -x_209 = x_207; -x_210 = x_208; -goto block_247; +x_222 = x_220; +x_223 = x_221; +goto block_260; } else { -lean_object* x_289; -x_289 = lean_box(0); -x_248 = x_289; -goto block_285; +lean_object* x_302; +x_302 = lean_box(0); +x_261 = x_302; +goto block_298; } } else { -lean_object* x_290; -x_290 = lean_box(0); -x_248 = x_290; -goto block_285; +lean_object* x_303; +x_303 = lean_box(0); +x_261 = x_303; +goto block_298; } } else { -lean_object* x_291; -x_291 = lean_box(0); -x_248 = x_291; -goto block_285; +lean_object* x_304; +x_304 = lean_box(0); +x_261 = x_304; +goto block_298; } -block_247: +block_260: { -lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; uint8_t x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; uint8_t x_241; -x_211 = l_Lean_mkFreshFVarId___at_Lean_Meta_Closure_collectExprAux___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_210); -x_212 = lean_ctor_get(x_211, 0); -lean_inc(x_212); -x_213 = lean_ctor_get(x_211, 1); -lean_inc(x_213); -lean_dec(x_211); -x_214 = l_Lean_Meta_Closure_mkNextUserName___rarg(x_3, x_4, x_5, x_6, x_7, x_213); +lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; uint8_t x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; uint8_t x_254; +x_224 = l_Lean_mkFreshFVarId___at_Lean_Meta_Closure_collectExprAux___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_223); +x_225 = lean_ctor_get(x_224, 0); +lean_inc(x_225); +x_226 = lean_ctor_get(x_224, 1); +lean_inc(x_226); +lean_dec(x_224); +x_227 = l_Lean_Meta_Closure_mkNextUserName___rarg(x_3, x_4, x_5, x_6, x_7, x_226); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_215 = lean_ctor_get(x_214, 0); -lean_inc(x_215); -x_216 = lean_ctor_get(x_214, 1); -lean_inc(x_216); -lean_dec(x_214); -x_217 = lean_st_ref_get(x_7, x_216); -lean_dec(x_7); -x_218 = lean_ctor_get(x_217, 1); -lean_inc(x_218); -lean_dec(x_217); -x_219 = lean_st_ref_take(x_3, x_218); -x_220 = lean_ctor_get(x_219, 0); -lean_inc(x_220); -x_221 = lean_ctor_get(x_219, 1); -lean_inc(x_221); -lean_dec(x_219); -x_222 = lean_ctor_get(x_220, 0); -lean_inc(x_222); -x_223 = lean_ctor_get(x_220, 1); -lean_inc(x_223); -x_224 = lean_ctor_get(x_220, 2); -lean_inc(x_224); -x_225 = lean_ctor_get(x_220, 3); -lean_inc(x_225); -x_226 = lean_ctor_get(x_220, 4); -lean_inc(x_226); -x_227 = lean_ctor_get(x_220, 5); -lean_inc(x_227); -x_228 = lean_ctor_get(x_220, 6); +x_228 = lean_ctor_get(x_227, 0); lean_inc(x_228); -x_229 = lean_unsigned_to_nat(0u); -x_230 = 0; -lean_inc(x_212); -x_231 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_231, 0, x_229); -lean_ctor_set(x_231, 1, x_212); -lean_ctor_set(x_231, 2, x_215); -lean_ctor_set(x_231, 3, x_209); -lean_ctor_set_uint8(x_231, sizeof(void*)*4, x_230); -x_232 = lean_array_push(x_228, x_231); -x_233 = lean_ctor_get(x_220, 7); +x_229 = lean_ctor_get(x_227, 1); +lean_inc(x_229); +lean_dec(x_227); +x_230 = lean_st_ref_get(x_7, x_229); +lean_dec(x_7); +x_231 = lean_ctor_get(x_230, 1); +lean_inc(x_231); +lean_dec(x_230); +x_232 = lean_st_ref_take(x_3, x_231); +x_233 = lean_ctor_get(x_232, 0); lean_inc(x_233); -x_234 = lean_ctor_get(x_220, 8); +x_234 = lean_ctor_get(x_232, 1); lean_inc(x_234); -x_235 = lean_ctor_get(x_220, 9); +lean_dec(x_232); +x_235 = lean_ctor_get(x_233, 0); lean_inc(x_235); -x_236 = lean_array_push(x_235, x_1); -x_237 = lean_ctor_get(x_220, 10); +x_236 = lean_ctor_get(x_233, 1); +lean_inc(x_236); +x_237 = lean_ctor_get(x_233, 2); lean_inc(x_237); -x_238 = lean_ctor_get(x_220, 11); +x_238 = lean_ctor_get(x_233, 3); lean_inc(x_238); -lean_dec(x_220); -x_239 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_239, 0, x_222); -lean_ctor_set(x_239, 1, x_223); -lean_ctor_set(x_239, 2, x_224); -lean_ctor_set(x_239, 3, x_225); -lean_ctor_set(x_239, 4, x_226); -lean_ctor_set(x_239, 5, x_227); -lean_ctor_set(x_239, 6, x_232); -lean_ctor_set(x_239, 7, x_233); -lean_ctor_set(x_239, 8, x_234); -lean_ctor_set(x_239, 9, x_236); -lean_ctor_set(x_239, 10, x_237); -lean_ctor_set(x_239, 11, x_238); -x_240 = lean_st_ref_set(x_3, x_239, x_221); -x_241 = !lean_is_exclusive(x_240); -if (x_241 == 0) -{ -lean_object* x_242; lean_object* x_243; -x_242 = lean_ctor_get(x_240, 0); -lean_dec(x_242); -x_243 = l_Lean_Expr_fvar___override(x_212); -lean_ctor_set(x_240, 0, x_243); -return x_240; +x_239 = lean_ctor_get(x_233, 4); +lean_inc(x_239); +x_240 = lean_ctor_get(x_233, 5); +lean_inc(x_240); +x_241 = lean_ctor_get(x_233, 6); +lean_inc(x_241); +x_242 = lean_unsigned_to_nat(0u); +x_243 = 0; +lean_inc(x_225); +x_244 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_244, 0, x_242); +lean_ctor_set(x_244, 1, x_225); +lean_ctor_set(x_244, 2, x_228); +lean_ctor_set(x_244, 3, x_222); +lean_ctor_set_uint8(x_244, sizeof(void*)*4, x_243); +x_245 = lean_array_push(x_241, x_244); +x_246 = lean_ctor_get(x_233, 7); +lean_inc(x_246); +x_247 = lean_ctor_get(x_233, 8); +lean_inc(x_247); +x_248 = lean_ctor_get(x_233, 9); +lean_inc(x_248); +x_249 = lean_array_push(x_248, x_1); +x_250 = lean_ctor_get(x_233, 10); +lean_inc(x_250); +x_251 = lean_ctor_get(x_233, 11); +lean_inc(x_251); +lean_dec(x_233); +x_252 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_252, 0, x_235); +lean_ctor_set(x_252, 1, x_236); +lean_ctor_set(x_252, 2, x_237); +lean_ctor_set(x_252, 3, x_238); +lean_ctor_set(x_252, 4, x_239); +lean_ctor_set(x_252, 5, x_240); +lean_ctor_set(x_252, 6, x_245); +lean_ctor_set(x_252, 7, x_246); +lean_ctor_set(x_252, 8, x_247); +lean_ctor_set(x_252, 9, x_249); +lean_ctor_set(x_252, 10, x_250); +lean_ctor_set(x_252, 11, x_251); +x_253 = lean_st_ref_set(x_3, x_252, x_234); +x_254 = !lean_is_exclusive(x_253); +if (x_254 == 0) +{ +lean_object* x_255; lean_object* x_256; +x_255 = lean_ctor_get(x_253, 0); +lean_dec(x_255); +x_256 = l_Lean_Expr_fvar___override(x_225); +lean_ctor_set(x_253, 0, x_256); +return x_253; } else { -lean_object* x_244; lean_object* x_245; lean_object* x_246; -x_244 = lean_ctor_get(x_240, 1); -lean_inc(x_244); -lean_dec(x_240); -x_245 = l_Lean_Expr_fvar___override(x_212); -x_246 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_246, 0, x_245); -lean_ctor_set(x_246, 1, x_244); -return x_246; +lean_object* x_257; lean_object* x_258; lean_object* x_259; +x_257 = lean_ctor_get(x_253, 1); +lean_inc(x_257); +lean_dec(x_253); +x_258 = l_Lean_Expr_fvar___override(x_225); +x_259 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_259, 0, x_258); +lean_ctor_set(x_259, 1, x_257); +return x_259; } } -block_285: +block_298: { -lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; -lean_dec(x_248); -x_249 = lean_st_ref_get(x_7, x_208); -x_250 = lean_ctor_get(x_249, 1); -lean_inc(x_250); -lean_dec(x_249); -x_251 = lean_st_ref_get(x_3, x_250); -x_252 = lean_ctor_get(x_251, 0); -lean_inc(x_252); -x_253 = lean_ctor_get(x_251, 1); -lean_inc(x_253); -lean_dec(x_251); -x_254 = lean_ctor_get(x_252, 1); -lean_inc(x_254); -lean_dec(x_252); -lean_inc(x_207); -x_255 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_254, x_207); -if (lean_obj_tag(x_255) == 0) +lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +lean_dec(x_261); +x_262 = lean_st_ref_get(x_7, x_221); +x_263 = lean_ctor_get(x_262, 1); +lean_inc(x_263); +lean_dec(x_262); +x_264 = lean_st_ref_get(x_3, x_263); +x_265 = lean_ctor_get(x_264, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_264, 1); +lean_inc(x_266); +lean_dec(x_264); +x_267 = lean_ctor_get(x_265, 1); +lean_inc(x_267); +lean_dec(x_265); +lean_inc(x_220); +x_268 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_267, x_220); +if (lean_obj_tag(x_268) == 0) { -lean_object* x_256; +lean_object* x_269; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_207); -x_256 = l_Lean_Meta_Closure_collectExprAux(x_207, x_2, x_3, x_4, x_5, x_6, x_7, x_253); -if (lean_obj_tag(x_256) == 0) +lean_inc(x_220); +x_269 = l_Lean_Meta_Closure_collectExprAux(x_220, x_2, x_3, x_4, x_5, x_6, x_7, x_266); +if (lean_obj_tag(x_269) == 0) { -lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; -x_257 = lean_ctor_get(x_256, 0); -lean_inc(x_257); -x_258 = lean_ctor_get(x_256, 1); -lean_inc(x_258); -lean_dec(x_256); -x_259 = lean_st_ref_get(x_7, x_258); -x_260 = lean_ctor_get(x_259, 1); -lean_inc(x_260); -lean_dec(x_259); -x_261 = lean_st_ref_take(x_3, x_260); -x_262 = lean_ctor_get(x_261, 0); -lean_inc(x_262); -x_263 = lean_ctor_get(x_261, 1); -lean_inc(x_263); -lean_dec(x_261); -x_264 = lean_ctor_get(x_262, 0); -lean_inc(x_264); -x_265 = lean_ctor_get(x_262, 1); -lean_inc(x_265); -lean_inc(x_257); -x_266 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_265, x_207, x_257); -x_267 = lean_ctor_get(x_262, 2); -lean_inc(x_267); -x_268 = lean_ctor_get(x_262, 3); -lean_inc(x_268); -x_269 = lean_ctor_get(x_262, 4); -lean_inc(x_269); -x_270 = lean_ctor_get(x_262, 5); +lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; +x_270 = lean_ctor_get(x_269, 0); lean_inc(x_270); -x_271 = lean_ctor_get(x_262, 6); +x_271 = lean_ctor_get(x_269, 1); lean_inc(x_271); -x_272 = lean_ctor_get(x_262, 7); -lean_inc(x_272); -x_273 = lean_ctor_get(x_262, 8); +lean_dec(x_269); +x_272 = lean_st_ref_get(x_7, x_271); +x_273 = lean_ctor_get(x_272, 1); lean_inc(x_273); -x_274 = lean_ctor_get(x_262, 9); -lean_inc(x_274); -x_275 = lean_ctor_get(x_262, 10); +lean_dec(x_272); +x_274 = lean_st_ref_take(x_3, x_273); +x_275 = lean_ctor_get(x_274, 0); lean_inc(x_275); -x_276 = lean_ctor_get(x_262, 11); +x_276 = lean_ctor_get(x_274, 1); lean_inc(x_276); -lean_dec(x_262); -x_277 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_277, 0, x_264); -lean_ctor_set(x_277, 1, x_266); -lean_ctor_set(x_277, 2, x_267); -lean_ctor_set(x_277, 3, x_268); -lean_ctor_set(x_277, 4, x_269); -lean_ctor_set(x_277, 5, x_270); -lean_ctor_set(x_277, 6, x_271); -lean_ctor_set(x_277, 7, x_272); -lean_ctor_set(x_277, 8, x_273); -lean_ctor_set(x_277, 9, x_274); -lean_ctor_set(x_277, 10, x_275); -lean_ctor_set(x_277, 11, x_276); -x_278 = lean_st_ref_set(x_3, x_277, x_263); -x_279 = lean_ctor_get(x_278, 1); -lean_inc(x_279); -lean_dec(x_278); -x_209 = x_257; -x_210 = x_279; -goto block_247; -} -else -{ -uint8_t x_280; -lean_dec(x_207); +lean_dec(x_274); +x_277 = lean_ctor_get(x_275, 0); +lean_inc(x_277); +x_278 = lean_ctor_get(x_275, 1); +lean_inc(x_278); +lean_inc(x_270); +x_279 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_278, x_220, x_270); +x_280 = lean_ctor_get(x_275, 2); +lean_inc(x_280); +x_281 = lean_ctor_get(x_275, 3); +lean_inc(x_281); +x_282 = lean_ctor_get(x_275, 4); +lean_inc(x_282); +x_283 = lean_ctor_get(x_275, 5); +lean_inc(x_283); +x_284 = lean_ctor_get(x_275, 6); +lean_inc(x_284); +x_285 = lean_ctor_get(x_275, 7); +lean_inc(x_285); +x_286 = lean_ctor_get(x_275, 8); +lean_inc(x_286); +x_287 = lean_ctor_get(x_275, 9); +lean_inc(x_287); +x_288 = lean_ctor_get(x_275, 10); +lean_inc(x_288); +x_289 = lean_ctor_get(x_275, 11); +lean_inc(x_289); +lean_dec(x_275); +x_290 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_290, 0, x_277); +lean_ctor_set(x_290, 1, x_279); +lean_ctor_set(x_290, 2, x_280); +lean_ctor_set(x_290, 3, x_281); +lean_ctor_set(x_290, 4, x_282); +lean_ctor_set(x_290, 5, x_283); +lean_ctor_set(x_290, 6, x_284); +lean_ctor_set(x_290, 7, x_285); +lean_ctor_set(x_290, 8, x_286); +lean_ctor_set(x_290, 9, x_287); +lean_ctor_set(x_290, 10, x_288); +lean_ctor_set(x_290, 11, x_289); +x_291 = lean_st_ref_set(x_3, x_290, x_276); +x_292 = lean_ctor_get(x_291, 1); +lean_inc(x_292); +lean_dec(x_291); +x_222 = x_270; +x_223 = x_292; +goto block_260; +} +else +{ +uint8_t x_293; +lean_dec(x_220); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_280 = !lean_is_exclusive(x_256); -if (x_280 == 0) +x_293 = !lean_is_exclusive(x_269); +if (x_293 == 0) { -return x_256; +return x_269; } else { -lean_object* x_281; lean_object* x_282; lean_object* x_283; -x_281 = lean_ctor_get(x_256, 0); -x_282 = lean_ctor_get(x_256, 1); -lean_inc(x_282); -lean_inc(x_281); -lean_dec(x_256); -x_283 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_283, 0, x_281); -lean_ctor_set(x_283, 1, x_282); -return x_283; +lean_object* x_294; lean_object* x_295; lean_object* x_296; +x_294 = lean_ctor_get(x_269, 0); +x_295 = lean_ctor_get(x_269, 1); +lean_inc(x_295); +lean_inc(x_294); +lean_dec(x_269); +x_296 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_296, 0, x_294); +lean_ctor_set(x_296, 1, x_295); +return x_296; } } } else { -lean_object* x_284; -lean_dec(x_207); -x_284 = lean_ctor_get(x_255, 0); -lean_inc(x_284); -lean_dec(x_255); -x_209 = x_284; -x_210 = x_253; -goto block_247; +lean_object* x_297; +lean_dec(x_220); +x_297 = lean_ctor_get(x_268, 0); +lean_inc(x_297); +lean_dec(x_268); +x_222 = x_297; +x_223 = x_266; +goto block_260; } } } else { -uint8_t x_292; +uint8_t x_305; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_292 = !lean_is_exclusive(x_206); -if (x_292 == 0) +x_305 = !lean_is_exclusive(x_219); +if (x_305 == 0) { -return x_206; +return x_219; } else { -lean_object* x_293; lean_object* x_294; lean_object* x_295; -x_293 = lean_ctor_get(x_206, 0); -x_294 = lean_ctor_get(x_206, 1); -lean_inc(x_294); -lean_inc(x_293); -lean_dec(x_206); -x_295 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_295, 0, x_293); -lean_ctor_set(x_295, 1, x_294); -return x_295; +lean_object* x_306; lean_object* x_307; lean_object* x_308; +x_306 = lean_ctor_get(x_219, 0); +x_307 = lean_ctor_get(x_219, 1); +lean_inc(x_307); +lean_inc(x_306); +lean_dec(x_219); +x_308 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_308, 0, x_306); +lean_ctor_set(x_308, 1, x_307); +return x_308; } } } else { -uint8_t x_296; +uint8_t x_309; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_296 = !lean_is_exclusive(x_202); -if (x_296 == 0) +x_309 = !lean_is_exclusive(x_215); +if (x_309 == 0) { -return x_202; +return x_215; } else { -lean_object* x_297; lean_object* x_298; lean_object* x_299; -x_297 = lean_ctor_get(x_202, 0); -x_298 = lean_ctor_get(x_202, 1); -lean_inc(x_298); -lean_inc(x_297); -lean_dec(x_202); -x_299 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_299, 0, x_297); -lean_ctor_set(x_299, 1, x_298); -return x_299; +lean_object* x_310; lean_object* x_311; lean_object* x_312; +x_310 = lean_ctor_get(x_215, 0); +x_311 = lean_ctor_get(x_215, 1); +lean_inc(x_311); +lean_inc(x_310); +lean_dec(x_215); +x_312 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_312, 0, x_310); +lean_ctor_set(x_312, 1, x_311); +return x_312; } } } case 3: { -lean_object* x_300; lean_object* x_301; uint8_t x_302; -x_300 = lean_ctor_get(x_1, 0); -lean_inc(x_300); -x_301 = l_Lean_Meta_Closure_collectLevel(x_300, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_object* x_313; lean_object* x_314; uint8_t x_315; +x_313 = lean_ctor_get(x_1, 0); +lean_inc(x_313); +lean_inc(x_313); +x_314 = l_Lean_Meta_Closure_collectLevel(x_313, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_302 = !lean_is_exclusive(x_301); -if (x_302 == 0) +x_315 = !lean_is_exclusive(x_314); +if (x_315 == 0) +{ +lean_object* x_316; size_t x_317; size_t x_318; uint8_t x_319; +x_316 = lean_ctor_get(x_314, 0); +x_317 = lean_ptr_addr(x_313); +lean_dec(x_313); +x_318 = lean_ptr_addr(x_316); +x_319 = lean_usize_dec_eq(x_317, x_318); +if (x_319 == 0) +{ +lean_object* x_320; +lean_dec(x_1); +x_320 = l_Lean_Expr_sort___override(x_316); +lean_ctor_set(x_314, 0, x_320); +return x_314; +} +else { -lean_object* x_303; lean_object* x_304; -x_303 = lean_ctor_get(x_301, 0); -x_304 = lean_expr_update_sort(x_1, x_303); -lean_ctor_set(x_301, 0, x_304); -return x_301; +lean_dec(x_316); +lean_ctor_set(x_314, 0, x_1); +return x_314; +} } else { -lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; -x_305 = lean_ctor_get(x_301, 0); -x_306 = lean_ctor_get(x_301, 1); -lean_inc(x_306); -lean_inc(x_305); -lean_dec(x_301); -x_307 = lean_expr_update_sort(x_1, x_305); -x_308 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_308, 0, x_307); -lean_ctor_set(x_308, 1, x_306); -return x_308; +lean_object* x_321; lean_object* x_322; size_t x_323; size_t x_324; uint8_t x_325; +x_321 = lean_ctor_get(x_314, 0); +x_322 = lean_ctor_get(x_314, 1); +lean_inc(x_322); +lean_inc(x_321); +lean_dec(x_314); +x_323 = lean_ptr_addr(x_313); +lean_dec(x_313); +x_324 = lean_ptr_addr(x_321); +x_325 = lean_usize_dec_eq(x_323, x_324); +if (x_325 == 0) +{ +lean_object* x_326; lean_object* x_327; +lean_dec(x_1); +x_326 = l_Lean_Expr_sort___override(x_321); +x_327 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_327, 0, x_326); +lean_ctor_set(x_327, 1, x_322); +return x_327; +} +else +{ +lean_object* x_328; +lean_dec(x_321); +x_328 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_328, 0, x_1); +lean_ctor_set(x_328, 1, x_322); +return x_328; +} } } case 4: { -lean_object* x_309; lean_object* x_310; uint8_t x_311; -x_309 = lean_ctor_get(x_1, 1); -lean_inc(x_309); -x_310 = l_List_mapM___at_Lean_Meta_Closure_collectExprAux___spec__3(x_309, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_object* x_329; lean_object* x_330; lean_object* x_331; uint8_t x_332; +x_329 = lean_ctor_get(x_1, 0); +lean_inc(x_329); +x_330 = lean_ctor_get(x_1, 1); +lean_inc(x_330); +lean_inc(x_330); +x_331 = l_List_mapM___at_Lean_Meta_Closure_collectExprAux___spec__3(x_330, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_311 = !lean_is_exclusive(x_310); -if (x_311 == 0) +x_332 = !lean_is_exclusive(x_331); +if (x_332 == 0) +{ +lean_object* x_333; uint8_t x_334; +x_333 = lean_ctor_get(x_331, 0); +x_334 = l_ptrEqList___rarg(x_330, x_333); +lean_dec(x_330); +if (x_334 == 0) { -lean_object* x_312; lean_object* x_313; -x_312 = lean_ctor_get(x_310, 0); -x_313 = lean_expr_update_const(x_1, x_312); -lean_ctor_set(x_310, 0, x_313); -return x_310; +lean_object* x_335; +lean_dec(x_1); +x_335 = l_Lean_Expr_const___override(x_329, x_333); +lean_ctor_set(x_331, 0, x_335); +return x_331; +} +else +{ +lean_dec(x_333); +lean_dec(x_329); +lean_ctor_set(x_331, 0, x_1); +return x_331; +} +} +else +{ +lean_object* x_336; lean_object* x_337; uint8_t x_338; +x_336 = lean_ctor_get(x_331, 0); +x_337 = lean_ctor_get(x_331, 1); +lean_inc(x_337); +lean_inc(x_336); +lean_dec(x_331); +x_338 = l_ptrEqList___rarg(x_330, x_336); +lean_dec(x_330); +if (x_338 == 0) +{ +lean_object* x_339; lean_object* x_340; +lean_dec(x_1); +x_339 = l_Lean_Expr_const___override(x_329, x_336); +x_340 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_340, 0, x_339); +lean_ctor_set(x_340, 1, x_337); +return x_340; } else { -lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; -x_314 = lean_ctor_get(x_310, 0); -x_315 = lean_ctor_get(x_310, 1); -lean_inc(x_315); -lean_inc(x_314); -lean_dec(x_310); -x_316 = lean_expr_update_const(x_1, x_314); -x_317 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_317, 0, x_316); -lean_ctor_set(x_317, 1, x_315); -return x_317; +lean_object* x_341; +lean_dec(x_336); +lean_dec(x_329); +x_341 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_341, 0, x_1); +lean_ctor_set(x_341, 1, x_337); +return x_341; +} } } case 5: { -lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_375; uint8_t x_413; -x_318 = lean_ctor_get(x_1, 0); -lean_inc(x_318); -x_319 = lean_ctor_get(x_1, 1); -lean_inc(x_319); -x_413 = l_Lean_Expr_hasLevelParam(x_318); -if (x_413 == 0) +lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_410; uint8_t x_448; +x_342 = lean_ctor_get(x_1, 0); +lean_inc(x_342); +x_343 = lean_ctor_get(x_1, 1); +lean_inc(x_343); +x_448 = l_Lean_Expr_hasLevelParam(x_342); +if (x_448 == 0) { -uint8_t x_414; -x_414 = l_Lean_Expr_hasFVar(x_318); -if (x_414 == 0) +uint8_t x_449; +x_449 = l_Lean_Expr_hasFVar(x_342); +if (x_449 == 0) { -uint8_t x_415; -x_415 = l_Lean_Expr_hasMVar(x_318); -if (x_415 == 0) +uint8_t x_450; +x_450 = l_Lean_Expr_hasMVar(x_342); +if (x_450 == 0) { -x_320 = x_318; -x_321 = x_8; -goto block_374; +x_344 = x_342; +x_345 = x_8; +goto block_409; } else { -lean_object* x_416; -x_416 = lean_box(0); -x_375 = x_416; -goto block_412; +lean_object* x_451; +x_451 = lean_box(0); +x_410 = x_451; +goto block_447; } } else { -lean_object* x_417; -x_417 = lean_box(0); -x_375 = x_417; -goto block_412; +lean_object* x_452; +x_452 = lean_box(0); +x_410 = x_452; +goto block_447; } } else { -lean_object* x_418; -x_418 = lean_box(0); -x_375 = x_418; -goto block_412; +lean_object* x_453; +x_453 = lean_box(0); +x_410 = x_453; +goto block_447; } -block_374: +block_409: { -lean_object* x_322; lean_object* x_323; lean_object* x_330; uint8_t x_368; -x_368 = l_Lean_Expr_hasLevelParam(x_319); -if (x_368 == 0) +lean_object* x_346; lean_object* x_347; lean_object* x_365; uint8_t x_403; +x_403 = l_Lean_Expr_hasLevelParam(x_343); +if (x_403 == 0) { -uint8_t x_369; -x_369 = l_Lean_Expr_hasFVar(x_319); -if (x_369 == 0) +uint8_t x_404; +x_404 = l_Lean_Expr_hasFVar(x_343); +if (x_404 == 0) { -uint8_t x_370; -x_370 = l_Lean_Expr_hasMVar(x_319); -if (x_370 == 0) +uint8_t x_405; +x_405 = l_Lean_Expr_hasMVar(x_343); +if (x_405 == 0) { lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_322 = x_319; -x_323 = x_321; -goto block_329; +x_346 = x_343; +x_347 = x_345; +goto block_364; } else { -lean_object* x_371; -x_371 = lean_box(0); -x_330 = x_371; -goto block_367; +lean_object* x_406; +x_406 = lean_box(0); +x_365 = x_406; +goto block_402; } } else { -lean_object* x_372; -x_372 = lean_box(0); -x_330 = x_372; -goto block_367; +lean_object* x_407; +x_407 = lean_box(0); +x_365 = x_407; +goto block_402; } } else { -lean_object* x_373; -x_373 = lean_box(0); -x_330 = x_373; -goto block_367; +lean_object* x_408; +x_408 = lean_box(0); +x_365 = x_408; +goto block_402; } -block_329: +block_364: { if (lean_obj_tag(x_1) == 5) { -lean_object* x_324; lean_object* x_325; -x_324 = lean_expr_update_app(x_1, x_320, x_322); -x_325 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_325, 0, x_324); -lean_ctor_set(x_325, 1, x_323); -return x_325; +lean_object* x_348; lean_object* x_349; size_t x_350; size_t x_351; uint8_t x_352; +x_348 = lean_ctor_get(x_1, 0); +lean_inc(x_348); +x_349 = lean_ctor_get(x_1, 1); +lean_inc(x_349); +x_350 = lean_ptr_addr(x_348); +lean_dec(x_348); +x_351 = lean_ptr_addr(x_344); +x_352 = lean_usize_dec_eq(x_350, x_351); +if (x_352 == 0) +{ +lean_object* x_353; lean_object* x_354; +lean_dec(x_349); +lean_dec(x_1); +x_353 = l_Lean_Expr_app___override(x_344, x_346); +x_354 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_354, 0, x_353); +lean_ctor_set(x_354, 1, x_347); +return x_354; } else { -lean_object* x_326; lean_object* x_327; lean_object* x_328; -lean_dec(x_322); -lean_dec(x_320); +size_t x_355; size_t x_356; uint8_t x_357; +x_355 = lean_ptr_addr(x_349); +lean_dec(x_349); +x_356 = lean_ptr_addr(x_346); +x_357 = lean_usize_dec_eq(x_355, x_356); +if (x_357 == 0) +{ +lean_object* x_358; lean_object* x_359; lean_dec(x_1); -x_326 = l_Lean_Meta_Closure_collectExprAux___closed__10; -x_327 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_326); -x_328 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_328, 0, x_327); -lean_ctor_set(x_328, 1, x_323); -return x_328; +x_358 = l_Lean_Expr_app___override(x_344, x_346); +x_359 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_359, 0, x_358); +lean_ctor_set(x_359, 1, x_347); +return x_359; +} +else +{ +lean_object* x_360; +lean_dec(x_346); +lean_dec(x_344); +x_360 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_360, 0, x_1); +lean_ctor_set(x_360, 1, x_347); +return x_360; +} } } -block_367: +else { -lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; -lean_dec(x_330); -x_331 = lean_st_ref_get(x_7, x_321); -x_332 = lean_ctor_get(x_331, 1); -lean_inc(x_332); -lean_dec(x_331); -x_333 = lean_st_ref_get(x_3, x_332); -x_334 = lean_ctor_get(x_333, 0); -lean_inc(x_334); -x_335 = lean_ctor_get(x_333, 1); -lean_inc(x_335); -lean_dec(x_333); -x_336 = lean_ctor_get(x_334, 1); -lean_inc(x_336); -lean_dec(x_334); -lean_inc(x_319); -x_337 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_336, x_319); -if (lean_obj_tag(x_337) == 0) +lean_object* x_361; lean_object* x_362; lean_object* x_363; +lean_dec(x_346); +lean_dec(x_344); +lean_dec(x_1); +x_361 = l_Lean_Meta_Closure_collectExprAux___closed__10; +x_362 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_361); +x_363 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_363, 0, x_362); +lean_ctor_set(x_363, 1, x_347); +return x_363; +} +} +block_402: +{ +lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; +lean_dec(x_365); +x_366 = lean_st_ref_get(x_7, x_345); +x_367 = lean_ctor_get(x_366, 1); +lean_inc(x_367); +lean_dec(x_366); +x_368 = lean_st_ref_get(x_3, x_367); +x_369 = lean_ctor_get(x_368, 0); +lean_inc(x_369); +x_370 = lean_ctor_get(x_368, 1); +lean_inc(x_370); +lean_dec(x_368); +x_371 = lean_ctor_get(x_369, 1); +lean_inc(x_371); +lean_dec(x_369); +lean_inc(x_343); +x_372 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_371, x_343); +if (lean_obj_tag(x_372) == 0) { -lean_object* x_338; +lean_object* x_373; lean_inc(x_7); -lean_inc(x_319); -x_338 = l_Lean_Meta_Closure_collectExprAux(x_319, x_2, x_3, x_4, x_5, x_6, x_7, x_335); -if (lean_obj_tag(x_338) == 0) -{ -lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; -x_339 = lean_ctor_get(x_338, 0); -lean_inc(x_339); -x_340 = lean_ctor_get(x_338, 1); -lean_inc(x_340); -lean_dec(x_338); -x_341 = lean_st_ref_get(x_7, x_340); +lean_inc(x_343); +x_373 = l_Lean_Meta_Closure_collectExprAux(x_343, x_2, x_3, x_4, x_5, x_6, x_7, x_370); +if (lean_obj_tag(x_373) == 0) +{ +lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; +x_374 = lean_ctor_get(x_373, 0); +lean_inc(x_374); +x_375 = lean_ctor_get(x_373, 1); +lean_inc(x_375); +lean_dec(x_373); +x_376 = lean_st_ref_get(x_7, x_375); lean_dec(x_7); -x_342 = lean_ctor_get(x_341, 1); -lean_inc(x_342); -lean_dec(x_341); -x_343 = lean_st_ref_take(x_3, x_342); -x_344 = lean_ctor_get(x_343, 0); -lean_inc(x_344); -x_345 = lean_ctor_get(x_343, 1); -lean_inc(x_345); -lean_dec(x_343); -x_346 = lean_ctor_get(x_344, 0); -lean_inc(x_346); -x_347 = lean_ctor_get(x_344, 1); -lean_inc(x_347); -lean_inc(x_339); -x_348 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_347, x_319, x_339); -x_349 = lean_ctor_get(x_344, 2); -lean_inc(x_349); -x_350 = lean_ctor_get(x_344, 3); -lean_inc(x_350); -x_351 = lean_ctor_get(x_344, 4); -lean_inc(x_351); -x_352 = lean_ctor_get(x_344, 5); -lean_inc(x_352); -x_353 = lean_ctor_get(x_344, 6); -lean_inc(x_353); -x_354 = lean_ctor_get(x_344, 7); -lean_inc(x_354); -x_355 = lean_ctor_get(x_344, 8); -lean_inc(x_355); -x_356 = lean_ctor_get(x_344, 9); -lean_inc(x_356); -x_357 = lean_ctor_get(x_344, 10); -lean_inc(x_357); -x_358 = lean_ctor_get(x_344, 11); -lean_inc(x_358); +x_377 = lean_ctor_get(x_376, 1); +lean_inc(x_377); +lean_dec(x_376); +x_378 = lean_st_ref_take(x_3, x_377); +x_379 = lean_ctor_get(x_378, 0); +lean_inc(x_379); +x_380 = lean_ctor_get(x_378, 1); +lean_inc(x_380); +lean_dec(x_378); +x_381 = lean_ctor_get(x_379, 0); +lean_inc(x_381); +x_382 = lean_ctor_get(x_379, 1); +lean_inc(x_382); +lean_inc(x_374); +x_383 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_382, x_343, x_374); +x_384 = lean_ctor_get(x_379, 2); +lean_inc(x_384); +x_385 = lean_ctor_get(x_379, 3); +lean_inc(x_385); +x_386 = lean_ctor_get(x_379, 4); +lean_inc(x_386); +x_387 = lean_ctor_get(x_379, 5); +lean_inc(x_387); +x_388 = lean_ctor_get(x_379, 6); +lean_inc(x_388); +x_389 = lean_ctor_get(x_379, 7); +lean_inc(x_389); +x_390 = lean_ctor_get(x_379, 8); +lean_inc(x_390); +x_391 = lean_ctor_get(x_379, 9); +lean_inc(x_391); +x_392 = lean_ctor_get(x_379, 10); +lean_inc(x_392); +x_393 = lean_ctor_get(x_379, 11); +lean_inc(x_393); +lean_dec(x_379); +x_394 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_394, 0, x_381); +lean_ctor_set(x_394, 1, x_383); +lean_ctor_set(x_394, 2, x_384); +lean_ctor_set(x_394, 3, x_385); +lean_ctor_set(x_394, 4, x_386); +lean_ctor_set(x_394, 5, x_387); +lean_ctor_set(x_394, 6, x_388); +lean_ctor_set(x_394, 7, x_389); +lean_ctor_set(x_394, 8, x_390); +lean_ctor_set(x_394, 9, x_391); +lean_ctor_set(x_394, 10, x_392); +lean_ctor_set(x_394, 11, x_393); +x_395 = lean_st_ref_set(x_3, x_394, x_380); +x_396 = lean_ctor_get(x_395, 1); +lean_inc(x_396); +lean_dec(x_395); +x_346 = x_374; +x_347 = x_396; +goto block_364; +} +else +{ +uint8_t x_397; lean_dec(x_344); -x_359 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_359, 0, x_346); -lean_ctor_set(x_359, 1, x_348); -lean_ctor_set(x_359, 2, x_349); -lean_ctor_set(x_359, 3, x_350); -lean_ctor_set(x_359, 4, x_351); -lean_ctor_set(x_359, 5, x_352); -lean_ctor_set(x_359, 6, x_353); -lean_ctor_set(x_359, 7, x_354); -lean_ctor_set(x_359, 8, x_355); -lean_ctor_set(x_359, 9, x_356); -lean_ctor_set(x_359, 10, x_357); -lean_ctor_set(x_359, 11, x_358); -x_360 = lean_st_ref_set(x_3, x_359, x_345); -x_361 = lean_ctor_get(x_360, 1); -lean_inc(x_361); -lean_dec(x_360); -x_322 = x_339; -x_323 = x_361; -goto block_329; -} -else -{ -uint8_t x_362; -lean_dec(x_320); -lean_dec(x_319); +lean_dec(x_343); lean_dec(x_7); lean_dec(x_1); -x_362 = !lean_is_exclusive(x_338); -if (x_362 == 0) +x_397 = !lean_is_exclusive(x_373); +if (x_397 == 0) { -return x_338; +return x_373; } else { -lean_object* x_363; lean_object* x_364; lean_object* x_365; -x_363 = lean_ctor_get(x_338, 0); -x_364 = lean_ctor_get(x_338, 1); -lean_inc(x_364); -lean_inc(x_363); -lean_dec(x_338); -x_365 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_365, 0, x_363); -lean_ctor_set(x_365, 1, x_364); -return x_365; +lean_object* x_398; lean_object* x_399; lean_object* x_400; +x_398 = lean_ctor_get(x_373, 0); +x_399 = lean_ctor_get(x_373, 1); +lean_inc(x_399); +lean_inc(x_398); +lean_dec(x_373); +x_400 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_400, 0, x_398); +lean_ctor_set(x_400, 1, x_399); +return x_400; } } } else { -lean_object* x_366; -lean_dec(x_319); +lean_object* x_401; +lean_dec(x_343); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_366 = lean_ctor_get(x_337, 0); -lean_inc(x_366); -lean_dec(x_337); -x_322 = x_366; -x_323 = x_335; -goto block_329; -} -} -} -block_412: -{ -lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; -lean_dec(x_375); -x_376 = lean_st_ref_get(x_7, x_8); -x_377 = lean_ctor_get(x_376, 1); -lean_inc(x_377); -lean_dec(x_376); -x_378 = lean_st_ref_get(x_3, x_377); -x_379 = lean_ctor_get(x_378, 0); -lean_inc(x_379); -x_380 = lean_ctor_get(x_378, 1); -lean_inc(x_380); -lean_dec(x_378); -x_381 = lean_ctor_get(x_379, 1); -lean_inc(x_381); -lean_dec(x_379); -lean_inc(x_318); -x_382 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_381, x_318); -if (lean_obj_tag(x_382) == 0) +x_401 = lean_ctor_get(x_372, 0); +lean_inc(x_401); +lean_dec(x_372); +x_346 = x_401; +x_347 = x_370; +goto block_364; +} +} +} +block_447: +{ +lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; +lean_dec(x_410); +x_411 = lean_st_ref_get(x_7, x_8); +x_412 = lean_ctor_get(x_411, 1); +lean_inc(x_412); +lean_dec(x_411); +x_413 = lean_st_ref_get(x_3, x_412); +x_414 = lean_ctor_get(x_413, 0); +lean_inc(x_414); +x_415 = lean_ctor_get(x_413, 1); +lean_inc(x_415); +lean_dec(x_413); +x_416 = lean_ctor_get(x_414, 1); +lean_inc(x_416); +lean_dec(x_414); +lean_inc(x_342); +x_417 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_416, x_342); +if (lean_obj_tag(x_417) == 0) { -lean_object* x_383; +lean_object* x_418; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_318); -x_383 = l_Lean_Meta_Closure_collectExprAux(x_318, x_2, x_3, x_4, x_5, x_6, x_7, x_380); -if (lean_obj_tag(x_383) == 0) +lean_inc(x_342); +x_418 = l_Lean_Meta_Closure_collectExprAux(x_342, x_2, x_3, x_4, x_5, x_6, x_7, x_415); +if (lean_obj_tag(x_418) == 0) +{ +lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; +x_419 = lean_ctor_get(x_418, 0); +lean_inc(x_419); +x_420 = lean_ctor_get(x_418, 1); +lean_inc(x_420); +lean_dec(x_418); +x_421 = lean_st_ref_get(x_7, x_420); +x_422 = lean_ctor_get(x_421, 1); +lean_inc(x_422); +lean_dec(x_421); +x_423 = lean_st_ref_take(x_3, x_422); +x_424 = lean_ctor_get(x_423, 0); +lean_inc(x_424); +x_425 = lean_ctor_get(x_423, 1); +lean_inc(x_425); +lean_dec(x_423); +x_426 = lean_ctor_get(x_424, 0); +lean_inc(x_426); +x_427 = lean_ctor_get(x_424, 1); +lean_inc(x_427); +lean_inc(x_419); +x_428 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_427, x_342, x_419); +x_429 = lean_ctor_get(x_424, 2); +lean_inc(x_429); +x_430 = lean_ctor_get(x_424, 3); +lean_inc(x_430); +x_431 = lean_ctor_get(x_424, 4); +lean_inc(x_431); +x_432 = lean_ctor_get(x_424, 5); +lean_inc(x_432); +x_433 = lean_ctor_get(x_424, 6); +lean_inc(x_433); +x_434 = lean_ctor_get(x_424, 7); +lean_inc(x_434); +x_435 = lean_ctor_get(x_424, 8); +lean_inc(x_435); +x_436 = lean_ctor_get(x_424, 9); +lean_inc(x_436); +x_437 = lean_ctor_get(x_424, 10); +lean_inc(x_437); +x_438 = lean_ctor_get(x_424, 11); +lean_inc(x_438); +lean_dec(x_424); +x_439 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_439, 0, x_426); +lean_ctor_set(x_439, 1, x_428); +lean_ctor_set(x_439, 2, x_429); +lean_ctor_set(x_439, 3, x_430); +lean_ctor_set(x_439, 4, x_431); +lean_ctor_set(x_439, 5, x_432); +lean_ctor_set(x_439, 6, x_433); +lean_ctor_set(x_439, 7, x_434); +lean_ctor_set(x_439, 8, x_435); +lean_ctor_set(x_439, 9, x_436); +lean_ctor_set(x_439, 10, x_437); +lean_ctor_set(x_439, 11, x_438); +x_440 = lean_st_ref_set(x_3, x_439, x_425); +x_441 = lean_ctor_get(x_440, 1); +lean_inc(x_441); +lean_dec(x_440); +x_344 = x_419; +x_345 = x_441; +goto block_409; +} +else { -lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; -x_384 = lean_ctor_get(x_383, 0); -lean_inc(x_384); -x_385 = lean_ctor_get(x_383, 1); -lean_inc(x_385); -lean_dec(x_383); -x_386 = lean_st_ref_get(x_7, x_385); -x_387 = lean_ctor_get(x_386, 1); -lean_inc(x_387); -lean_dec(x_386); -x_388 = lean_st_ref_take(x_3, x_387); -x_389 = lean_ctor_get(x_388, 0); -lean_inc(x_389); -x_390 = lean_ctor_get(x_388, 1); -lean_inc(x_390); -lean_dec(x_388); -x_391 = lean_ctor_get(x_389, 0); -lean_inc(x_391); -x_392 = lean_ctor_get(x_389, 1); -lean_inc(x_392); -lean_inc(x_384); -x_393 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_392, x_318, x_384); -x_394 = lean_ctor_get(x_389, 2); -lean_inc(x_394); -x_395 = lean_ctor_get(x_389, 3); -lean_inc(x_395); -x_396 = lean_ctor_get(x_389, 4); -lean_inc(x_396); -x_397 = lean_ctor_get(x_389, 5); -lean_inc(x_397); -x_398 = lean_ctor_get(x_389, 6); -lean_inc(x_398); -x_399 = lean_ctor_get(x_389, 7); -lean_inc(x_399); -x_400 = lean_ctor_get(x_389, 8); -lean_inc(x_400); -x_401 = lean_ctor_get(x_389, 9); -lean_inc(x_401); -x_402 = lean_ctor_get(x_389, 10); -lean_inc(x_402); -x_403 = lean_ctor_get(x_389, 11); -lean_inc(x_403); -lean_dec(x_389); -x_404 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_404, 0, x_391); -lean_ctor_set(x_404, 1, x_393); -lean_ctor_set(x_404, 2, x_394); -lean_ctor_set(x_404, 3, x_395); -lean_ctor_set(x_404, 4, x_396); -lean_ctor_set(x_404, 5, x_397); -lean_ctor_set(x_404, 6, x_398); -lean_ctor_set(x_404, 7, x_399); -lean_ctor_set(x_404, 8, x_400); -lean_ctor_set(x_404, 9, x_401); -lean_ctor_set(x_404, 10, x_402); -lean_ctor_set(x_404, 11, x_403); -x_405 = lean_st_ref_set(x_3, x_404, x_390); -x_406 = lean_ctor_get(x_405, 1); -lean_inc(x_406); -lean_dec(x_405); -x_320 = x_384; -x_321 = x_406; -goto block_374; -} -else -{ -uint8_t x_407; -lean_dec(x_319); -lean_dec(x_318); +uint8_t x_442; +lean_dec(x_343); +lean_dec(x_342); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_407 = !lean_is_exclusive(x_383); -if (x_407 == 0) +x_442 = !lean_is_exclusive(x_418); +if (x_442 == 0) { -return x_383; +return x_418; } else { -lean_object* x_408; lean_object* x_409; lean_object* x_410; -x_408 = lean_ctor_get(x_383, 0); -x_409 = lean_ctor_get(x_383, 1); -lean_inc(x_409); -lean_inc(x_408); -lean_dec(x_383); -x_410 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_410, 0, x_408); -lean_ctor_set(x_410, 1, x_409); -return x_410; +lean_object* x_443; lean_object* x_444; lean_object* x_445; +x_443 = lean_ctor_get(x_418, 0); +x_444 = lean_ctor_get(x_418, 1); +lean_inc(x_444); +lean_inc(x_443); +lean_dec(x_418); +x_445 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_445, 0, x_443); +lean_ctor_set(x_445, 1, x_444); +return x_445; } } } else { -lean_object* x_411; -lean_dec(x_318); -x_411 = lean_ctor_get(x_382, 0); -lean_inc(x_411); -lean_dec(x_382); -x_320 = x_411; -x_321 = x_380; -goto block_374; +lean_object* x_446; +lean_dec(x_342); +x_446 = lean_ctor_get(x_417, 0); +lean_inc(x_446); +lean_dec(x_417); +x_344 = x_446; +x_345 = x_415; +goto block_409; } } } case 6: { -lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_477; uint8_t x_515; -x_419 = lean_ctor_get(x_1, 1); -lean_inc(x_419); -x_420 = lean_ctor_get(x_1, 2); -lean_inc(x_420); -x_515 = l_Lean_Expr_hasLevelParam(x_419); -if (x_515 == 0) +lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_528; uint8_t x_566; +x_454 = lean_ctor_get(x_1, 1); +lean_inc(x_454); +x_455 = lean_ctor_get(x_1, 2); +lean_inc(x_455); +x_566 = l_Lean_Expr_hasLevelParam(x_454); +if (x_566 == 0) { -uint8_t x_516; -x_516 = l_Lean_Expr_hasFVar(x_419); -if (x_516 == 0) +uint8_t x_567; +x_567 = l_Lean_Expr_hasFVar(x_454); +if (x_567 == 0) { -uint8_t x_517; -x_517 = l_Lean_Expr_hasMVar(x_419); -if (x_517 == 0) +uint8_t x_568; +x_568 = l_Lean_Expr_hasMVar(x_454); +if (x_568 == 0) { -x_421 = x_419; -x_422 = x_8; -goto block_476; +x_456 = x_454; +x_457 = x_8; +goto block_527; } else { -lean_object* x_518; -x_518 = lean_box(0); -x_477 = x_518; -goto block_514; +lean_object* x_569; +x_569 = lean_box(0); +x_528 = x_569; +goto block_565; } } else { -lean_object* x_519; -x_519 = lean_box(0); -x_477 = x_519; -goto block_514; +lean_object* x_570; +x_570 = lean_box(0); +x_528 = x_570; +goto block_565; } } else { -lean_object* x_520; -x_520 = lean_box(0); -x_477 = x_520; -goto block_514; +lean_object* x_571; +x_571 = lean_box(0); +x_528 = x_571; +goto block_565; } -block_476: +block_527: { -lean_object* x_423; lean_object* x_424; lean_object* x_432; uint8_t x_470; -x_470 = l_Lean_Expr_hasLevelParam(x_420); -if (x_470 == 0) +lean_object* x_458; lean_object* x_459; lean_object* x_483; uint8_t x_521; +x_521 = l_Lean_Expr_hasLevelParam(x_455); +if (x_521 == 0) { -uint8_t x_471; -x_471 = l_Lean_Expr_hasFVar(x_420); -if (x_471 == 0) +uint8_t x_522; +x_522 = l_Lean_Expr_hasFVar(x_455); +if (x_522 == 0) { -uint8_t x_472; -x_472 = l_Lean_Expr_hasMVar(x_420); -if (x_472 == 0) +uint8_t x_523; +x_523 = l_Lean_Expr_hasMVar(x_455); +if (x_523 == 0) { lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_423 = x_420; -x_424 = x_422; -goto block_431; +x_458 = x_455; +x_459 = x_457; +goto block_482; } else { -lean_object* x_473; -x_473 = lean_box(0); -x_432 = x_473; -goto block_469; +lean_object* x_524; +x_524 = lean_box(0); +x_483 = x_524; +goto block_520; } } else { -lean_object* x_474; -x_474 = lean_box(0); -x_432 = x_474; -goto block_469; +lean_object* x_525; +x_525 = lean_box(0); +x_483 = x_525; +goto block_520; } } else { -lean_object* x_475; -x_475 = lean_box(0); -x_432 = x_475; -goto block_469; +lean_object* x_526; +x_526 = lean_box(0); +x_483 = x_526; +goto block_520; } -block_431: +block_482: { if (lean_obj_tag(x_1) == 6) { -uint8_t x_425; lean_object* x_426; lean_object* x_427; -x_425 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_426 = lean_expr_update_lambda(x_1, x_425, x_421, x_423); -x_427 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_427, 0, x_426); -lean_ctor_set(x_427, 1, x_424); -return x_427; +lean_object* x_460; lean_object* x_461; lean_object* x_462; uint8_t x_463; lean_object* x_464; size_t x_465; size_t x_466; uint8_t x_467; +x_460 = lean_ctor_get(x_1, 0); +lean_inc(x_460); +x_461 = lean_ctor_get(x_1, 1); +lean_inc(x_461); +x_462 = lean_ctor_get(x_1, 2); +lean_inc(x_462); +x_463 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_462); +lean_inc(x_461); +lean_inc(x_460); +x_464 = l_Lean_Expr_lam___override(x_460, x_461, x_462, x_463); +x_465 = lean_ptr_addr(x_461); +lean_dec(x_461); +x_466 = lean_ptr_addr(x_456); +x_467 = lean_usize_dec_eq(x_465, x_466); +if (x_467 == 0) +{ +lean_object* x_468; lean_object* x_469; +lean_dec(x_464); +lean_dec(x_462); +x_468 = l_Lean_Expr_lam___override(x_460, x_456, x_458, x_463); +x_469 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_469, 0, x_468); +lean_ctor_set(x_469, 1, x_459); +return x_469; } else { -lean_object* x_428; lean_object* x_429; lean_object* x_430; -lean_dec(x_423); -lean_dec(x_421); +size_t x_470; size_t x_471; uint8_t x_472; +x_470 = lean_ptr_addr(x_462); +lean_dec(x_462); +x_471 = lean_ptr_addr(x_458); +x_472 = lean_usize_dec_eq(x_470, x_471); +if (x_472 == 0) +{ +lean_object* x_473; lean_object* x_474; +lean_dec(x_464); +x_473 = l_Lean_Expr_lam___override(x_460, x_456, x_458, x_463); +x_474 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_474, 0, x_473); +lean_ctor_set(x_474, 1, x_459); +return x_474; +} +else +{ +uint8_t x_475; +x_475 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_463, x_463); +if (x_475 == 0) +{ +lean_object* x_476; lean_object* x_477; +lean_dec(x_464); +x_476 = l_Lean_Expr_lam___override(x_460, x_456, x_458, x_463); +x_477 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_477, 0, x_476); +lean_ctor_set(x_477, 1, x_459); +return x_477; +} +else +{ +lean_object* x_478; +lean_dec(x_460); +lean_dec(x_458); +lean_dec(x_456); +x_478 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_478, 0, x_464); +lean_ctor_set(x_478, 1, x_459); +return x_478; +} +} +} +} +else +{ +lean_object* x_479; lean_object* x_480; lean_object* x_481; +lean_dec(x_458); +lean_dec(x_456); lean_dec(x_1); -x_428 = l_Lean_Meta_Closure_collectExprAux___closed__13; -x_429 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_428); -x_430 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_430, 0, x_429); -lean_ctor_set(x_430, 1, x_424); -return x_430; +x_479 = l_Lean_Meta_Closure_collectExprAux___closed__13; +x_480 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_479); +x_481 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_481, 0, x_480); +lean_ctor_set(x_481, 1, x_459); +return x_481; } } -block_469: +block_520: { -lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; -lean_dec(x_432); -x_433 = lean_st_ref_get(x_7, x_422); -x_434 = lean_ctor_get(x_433, 1); -lean_inc(x_434); -lean_dec(x_433); -x_435 = lean_st_ref_get(x_3, x_434); -x_436 = lean_ctor_get(x_435, 0); -lean_inc(x_436); -x_437 = lean_ctor_get(x_435, 1); -lean_inc(x_437); -lean_dec(x_435); -x_438 = lean_ctor_get(x_436, 1); -lean_inc(x_438); -lean_dec(x_436); -lean_inc(x_420); -x_439 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_438, x_420); -if (lean_obj_tag(x_439) == 0) +lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; +lean_dec(x_483); +x_484 = lean_st_ref_get(x_7, x_457); +x_485 = lean_ctor_get(x_484, 1); +lean_inc(x_485); +lean_dec(x_484); +x_486 = lean_st_ref_get(x_3, x_485); +x_487 = lean_ctor_get(x_486, 0); +lean_inc(x_487); +x_488 = lean_ctor_get(x_486, 1); +lean_inc(x_488); +lean_dec(x_486); +x_489 = lean_ctor_get(x_487, 1); +lean_inc(x_489); +lean_dec(x_487); +lean_inc(x_455); +x_490 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_489, x_455); +if (lean_obj_tag(x_490) == 0) { -lean_object* x_440; +lean_object* x_491; lean_inc(x_7); -lean_inc(x_420); -x_440 = l_Lean_Meta_Closure_collectExprAux(x_420, x_2, x_3, x_4, x_5, x_6, x_7, x_437); -if (lean_obj_tag(x_440) == 0) -{ -lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; -x_441 = lean_ctor_get(x_440, 0); -lean_inc(x_441); -x_442 = lean_ctor_get(x_440, 1); -lean_inc(x_442); -lean_dec(x_440); -x_443 = lean_st_ref_get(x_7, x_442); -lean_dec(x_7); -x_444 = lean_ctor_get(x_443, 1); -lean_inc(x_444); -lean_dec(x_443); -x_445 = lean_st_ref_take(x_3, x_444); -x_446 = lean_ctor_get(x_445, 0); -lean_inc(x_446); -x_447 = lean_ctor_get(x_445, 1); -lean_inc(x_447); -lean_dec(x_445); -x_448 = lean_ctor_get(x_446, 0); -lean_inc(x_448); -x_449 = lean_ctor_get(x_446, 1); -lean_inc(x_449); -lean_inc(x_441); -x_450 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_449, x_420, x_441); -x_451 = lean_ctor_get(x_446, 2); -lean_inc(x_451); -x_452 = lean_ctor_get(x_446, 3); -lean_inc(x_452); -x_453 = lean_ctor_get(x_446, 4); -lean_inc(x_453); -x_454 = lean_ctor_get(x_446, 5); -lean_inc(x_454); -x_455 = lean_ctor_get(x_446, 6); lean_inc(x_455); -x_456 = lean_ctor_get(x_446, 7); -lean_inc(x_456); -x_457 = lean_ctor_get(x_446, 8); -lean_inc(x_457); -x_458 = lean_ctor_get(x_446, 9); -lean_inc(x_458); -x_459 = lean_ctor_get(x_446, 10); -lean_inc(x_459); -x_460 = lean_ctor_get(x_446, 11); -lean_inc(x_460); -lean_dec(x_446); -x_461 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_461, 0, x_448); -lean_ctor_set(x_461, 1, x_450); -lean_ctor_set(x_461, 2, x_451); -lean_ctor_set(x_461, 3, x_452); -lean_ctor_set(x_461, 4, x_453); -lean_ctor_set(x_461, 5, x_454); -lean_ctor_set(x_461, 6, x_455); -lean_ctor_set(x_461, 7, x_456); -lean_ctor_set(x_461, 8, x_457); -lean_ctor_set(x_461, 9, x_458); -lean_ctor_set(x_461, 10, x_459); -lean_ctor_set(x_461, 11, x_460); -x_462 = lean_st_ref_set(x_3, x_461, x_447); -x_463 = lean_ctor_get(x_462, 1); -lean_inc(x_463); -lean_dec(x_462); -x_423 = x_441; -x_424 = x_463; -goto block_431; -} -else +x_491 = l_Lean_Meta_Closure_collectExprAux(x_455, x_2, x_3, x_4, x_5, x_6, x_7, x_488); +if (lean_obj_tag(x_491) == 0) { -uint8_t x_464; -lean_dec(x_421); -lean_dec(x_420); +lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; +x_492 = lean_ctor_get(x_491, 0); +lean_inc(x_492); +x_493 = lean_ctor_get(x_491, 1); +lean_inc(x_493); +lean_dec(x_491); +x_494 = lean_st_ref_get(x_7, x_493); +lean_dec(x_7); +x_495 = lean_ctor_get(x_494, 1); +lean_inc(x_495); +lean_dec(x_494); +x_496 = lean_st_ref_take(x_3, x_495); +x_497 = lean_ctor_get(x_496, 0); +lean_inc(x_497); +x_498 = lean_ctor_get(x_496, 1); +lean_inc(x_498); +lean_dec(x_496); +x_499 = lean_ctor_get(x_497, 0); +lean_inc(x_499); +x_500 = lean_ctor_get(x_497, 1); +lean_inc(x_500); +lean_inc(x_492); +x_501 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_500, x_455, x_492); +x_502 = lean_ctor_get(x_497, 2); +lean_inc(x_502); +x_503 = lean_ctor_get(x_497, 3); +lean_inc(x_503); +x_504 = lean_ctor_get(x_497, 4); +lean_inc(x_504); +x_505 = lean_ctor_get(x_497, 5); +lean_inc(x_505); +x_506 = lean_ctor_get(x_497, 6); +lean_inc(x_506); +x_507 = lean_ctor_get(x_497, 7); +lean_inc(x_507); +x_508 = lean_ctor_get(x_497, 8); +lean_inc(x_508); +x_509 = lean_ctor_get(x_497, 9); +lean_inc(x_509); +x_510 = lean_ctor_get(x_497, 10); +lean_inc(x_510); +x_511 = lean_ctor_get(x_497, 11); +lean_inc(x_511); +lean_dec(x_497); +x_512 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_512, 0, x_499); +lean_ctor_set(x_512, 1, x_501); +lean_ctor_set(x_512, 2, x_502); +lean_ctor_set(x_512, 3, x_503); +lean_ctor_set(x_512, 4, x_504); +lean_ctor_set(x_512, 5, x_505); +lean_ctor_set(x_512, 6, x_506); +lean_ctor_set(x_512, 7, x_507); +lean_ctor_set(x_512, 8, x_508); +lean_ctor_set(x_512, 9, x_509); +lean_ctor_set(x_512, 10, x_510); +lean_ctor_set(x_512, 11, x_511); +x_513 = lean_st_ref_set(x_3, x_512, x_498); +x_514 = lean_ctor_get(x_513, 1); +lean_inc(x_514); +lean_dec(x_513); +x_458 = x_492; +x_459 = x_514; +goto block_482; +} +else +{ +uint8_t x_515; +lean_dec(x_456); +lean_dec(x_455); lean_dec(x_7); lean_dec(x_1); -x_464 = !lean_is_exclusive(x_440); -if (x_464 == 0) +x_515 = !lean_is_exclusive(x_491); +if (x_515 == 0) { -return x_440; +return x_491; } else { -lean_object* x_465; lean_object* x_466; lean_object* x_467; -x_465 = lean_ctor_get(x_440, 0); -x_466 = lean_ctor_get(x_440, 1); -lean_inc(x_466); -lean_inc(x_465); -lean_dec(x_440); -x_467 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_467, 0, x_465); -lean_ctor_set(x_467, 1, x_466); -return x_467; +lean_object* x_516; lean_object* x_517; lean_object* x_518; +x_516 = lean_ctor_get(x_491, 0); +x_517 = lean_ctor_get(x_491, 1); +lean_inc(x_517); +lean_inc(x_516); +lean_dec(x_491); +x_518 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_518, 0, x_516); +lean_ctor_set(x_518, 1, x_517); +return x_518; } } } else { -lean_object* x_468; -lean_dec(x_420); +lean_object* x_519; +lean_dec(x_455); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_468 = lean_ctor_get(x_439, 0); -lean_inc(x_468); -lean_dec(x_439); -x_423 = x_468; -x_424 = x_437; -goto block_431; -} -} -} -block_514: -{ -lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; -lean_dec(x_477); -x_478 = lean_st_ref_get(x_7, x_8); -x_479 = lean_ctor_get(x_478, 1); -lean_inc(x_479); -lean_dec(x_478); -x_480 = lean_st_ref_get(x_3, x_479); -x_481 = lean_ctor_get(x_480, 0); -lean_inc(x_481); -x_482 = lean_ctor_get(x_480, 1); -lean_inc(x_482); -lean_dec(x_480); -x_483 = lean_ctor_get(x_481, 1); -lean_inc(x_483); -lean_dec(x_481); -lean_inc(x_419); -x_484 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_483, x_419); -if (lean_obj_tag(x_484) == 0) +x_519 = lean_ctor_get(x_490, 0); +lean_inc(x_519); +lean_dec(x_490); +x_458 = x_519; +x_459 = x_488; +goto block_482; +} +} +} +block_565: +{ +lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; +lean_dec(x_528); +x_529 = lean_st_ref_get(x_7, x_8); +x_530 = lean_ctor_get(x_529, 1); +lean_inc(x_530); +lean_dec(x_529); +x_531 = lean_st_ref_get(x_3, x_530); +x_532 = lean_ctor_get(x_531, 0); +lean_inc(x_532); +x_533 = lean_ctor_get(x_531, 1); +lean_inc(x_533); +lean_dec(x_531); +x_534 = lean_ctor_get(x_532, 1); +lean_inc(x_534); +lean_dec(x_532); +lean_inc(x_454); +x_535 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_534, x_454); +if (lean_obj_tag(x_535) == 0) { -lean_object* x_485; +lean_object* x_536; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_419); -x_485 = l_Lean_Meta_Closure_collectExprAux(x_419, x_2, x_3, x_4, x_5, x_6, x_7, x_482); -if (lean_obj_tag(x_485) == 0) +lean_inc(x_454); +x_536 = l_Lean_Meta_Closure_collectExprAux(x_454, x_2, x_3, x_4, x_5, x_6, x_7, x_533); +if (lean_obj_tag(x_536) == 0) { -lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; -x_486 = lean_ctor_get(x_485, 0); -lean_inc(x_486); -x_487 = lean_ctor_get(x_485, 1); -lean_inc(x_487); -lean_dec(x_485); -x_488 = lean_st_ref_get(x_7, x_487); -x_489 = lean_ctor_get(x_488, 1); -lean_inc(x_489); -lean_dec(x_488); -x_490 = lean_st_ref_take(x_3, x_489); -x_491 = lean_ctor_get(x_490, 0); -lean_inc(x_491); -x_492 = lean_ctor_get(x_490, 1); -lean_inc(x_492); -lean_dec(x_490); -x_493 = lean_ctor_get(x_491, 0); -lean_inc(x_493); -x_494 = lean_ctor_get(x_491, 1); -lean_inc(x_494); -lean_inc(x_486); -x_495 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_494, x_419, x_486); -x_496 = lean_ctor_get(x_491, 2); -lean_inc(x_496); -x_497 = lean_ctor_get(x_491, 3); -lean_inc(x_497); -x_498 = lean_ctor_get(x_491, 4); -lean_inc(x_498); -x_499 = lean_ctor_get(x_491, 5); -lean_inc(x_499); -x_500 = lean_ctor_get(x_491, 6); -lean_inc(x_500); -x_501 = lean_ctor_get(x_491, 7); -lean_inc(x_501); -x_502 = lean_ctor_get(x_491, 8); -lean_inc(x_502); -x_503 = lean_ctor_get(x_491, 9); -lean_inc(x_503); -x_504 = lean_ctor_get(x_491, 10); -lean_inc(x_504); -x_505 = lean_ctor_get(x_491, 11); -lean_inc(x_505); -lean_dec(x_491); -x_506 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_506, 0, x_493); -lean_ctor_set(x_506, 1, x_495); -lean_ctor_set(x_506, 2, x_496); -lean_ctor_set(x_506, 3, x_497); -lean_ctor_set(x_506, 4, x_498); -lean_ctor_set(x_506, 5, x_499); -lean_ctor_set(x_506, 6, x_500); -lean_ctor_set(x_506, 7, x_501); -lean_ctor_set(x_506, 8, x_502); -lean_ctor_set(x_506, 9, x_503); -lean_ctor_set(x_506, 10, x_504); -lean_ctor_set(x_506, 11, x_505); -x_507 = lean_st_ref_set(x_3, x_506, x_492); -x_508 = lean_ctor_get(x_507, 1); -lean_inc(x_508); -lean_dec(x_507); -x_421 = x_486; -x_422 = x_508; -goto block_476; +lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; +x_537 = lean_ctor_get(x_536, 0); +lean_inc(x_537); +x_538 = lean_ctor_get(x_536, 1); +lean_inc(x_538); +lean_dec(x_536); +x_539 = lean_st_ref_get(x_7, x_538); +x_540 = lean_ctor_get(x_539, 1); +lean_inc(x_540); +lean_dec(x_539); +x_541 = lean_st_ref_take(x_3, x_540); +x_542 = lean_ctor_get(x_541, 0); +lean_inc(x_542); +x_543 = lean_ctor_get(x_541, 1); +lean_inc(x_543); +lean_dec(x_541); +x_544 = lean_ctor_get(x_542, 0); +lean_inc(x_544); +x_545 = lean_ctor_get(x_542, 1); +lean_inc(x_545); +lean_inc(x_537); +x_546 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_545, x_454, x_537); +x_547 = lean_ctor_get(x_542, 2); +lean_inc(x_547); +x_548 = lean_ctor_get(x_542, 3); +lean_inc(x_548); +x_549 = lean_ctor_get(x_542, 4); +lean_inc(x_549); +x_550 = lean_ctor_get(x_542, 5); +lean_inc(x_550); +x_551 = lean_ctor_get(x_542, 6); +lean_inc(x_551); +x_552 = lean_ctor_get(x_542, 7); +lean_inc(x_552); +x_553 = lean_ctor_get(x_542, 8); +lean_inc(x_553); +x_554 = lean_ctor_get(x_542, 9); +lean_inc(x_554); +x_555 = lean_ctor_get(x_542, 10); +lean_inc(x_555); +x_556 = lean_ctor_get(x_542, 11); +lean_inc(x_556); +lean_dec(x_542); +x_557 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_557, 0, x_544); +lean_ctor_set(x_557, 1, x_546); +lean_ctor_set(x_557, 2, x_547); +lean_ctor_set(x_557, 3, x_548); +lean_ctor_set(x_557, 4, x_549); +lean_ctor_set(x_557, 5, x_550); +lean_ctor_set(x_557, 6, x_551); +lean_ctor_set(x_557, 7, x_552); +lean_ctor_set(x_557, 8, x_553); +lean_ctor_set(x_557, 9, x_554); +lean_ctor_set(x_557, 10, x_555); +lean_ctor_set(x_557, 11, x_556); +x_558 = lean_st_ref_set(x_3, x_557, x_543); +x_559 = lean_ctor_get(x_558, 1); +lean_inc(x_559); +lean_dec(x_558); +x_456 = x_537; +x_457 = x_559; +goto block_527; } else { -uint8_t x_509; -lean_dec(x_420); -lean_dec(x_419); +uint8_t x_560; +lean_dec(x_455); +lean_dec(x_454); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_509 = !lean_is_exclusive(x_485); -if (x_509 == 0) +x_560 = !lean_is_exclusive(x_536); +if (x_560 == 0) { -return x_485; +return x_536; } else { -lean_object* x_510; lean_object* x_511; lean_object* x_512; -x_510 = lean_ctor_get(x_485, 0); -x_511 = lean_ctor_get(x_485, 1); -lean_inc(x_511); -lean_inc(x_510); -lean_dec(x_485); -x_512 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_512, 0, x_510); -lean_ctor_set(x_512, 1, x_511); -return x_512; +lean_object* x_561; lean_object* x_562; lean_object* x_563; +x_561 = lean_ctor_get(x_536, 0); +x_562 = lean_ctor_get(x_536, 1); +lean_inc(x_562); +lean_inc(x_561); +lean_dec(x_536); +x_563 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_563, 0, x_561); +lean_ctor_set(x_563, 1, x_562); +return x_563; } } } else { -lean_object* x_513; -lean_dec(x_419); -x_513 = lean_ctor_get(x_484, 0); -lean_inc(x_513); -lean_dec(x_484); -x_421 = x_513; -x_422 = x_482; -goto block_476; +lean_object* x_564; +lean_dec(x_454); +x_564 = lean_ctor_get(x_535, 0); +lean_inc(x_564); +lean_dec(x_535); +x_456 = x_564; +x_457 = x_533; +goto block_527; } } } case 7: { -lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_579; uint8_t x_617; -x_521 = lean_ctor_get(x_1, 1); -lean_inc(x_521); -x_522 = lean_ctor_get(x_1, 2); -lean_inc(x_522); -x_617 = l_Lean_Expr_hasLevelParam(x_521); -if (x_617 == 0) +lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_646; uint8_t x_684; +x_572 = lean_ctor_get(x_1, 1); +lean_inc(x_572); +x_573 = lean_ctor_get(x_1, 2); +lean_inc(x_573); +x_684 = l_Lean_Expr_hasLevelParam(x_572); +if (x_684 == 0) { -uint8_t x_618; -x_618 = l_Lean_Expr_hasFVar(x_521); -if (x_618 == 0) +uint8_t x_685; +x_685 = l_Lean_Expr_hasFVar(x_572); +if (x_685 == 0) { -uint8_t x_619; -x_619 = l_Lean_Expr_hasMVar(x_521); -if (x_619 == 0) +uint8_t x_686; +x_686 = l_Lean_Expr_hasMVar(x_572); +if (x_686 == 0) { -x_523 = x_521; -x_524 = x_8; -goto block_578; +x_574 = x_572; +x_575 = x_8; +goto block_645; } else { -lean_object* x_620; -x_620 = lean_box(0); -x_579 = x_620; -goto block_616; +lean_object* x_687; +x_687 = lean_box(0); +x_646 = x_687; +goto block_683; } } else { -lean_object* x_621; -x_621 = lean_box(0); -x_579 = x_621; -goto block_616; +lean_object* x_688; +x_688 = lean_box(0); +x_646 = x_688; +goto block_683; } } else { -lean_object* x_622; -x_622 = lean_box(0); -x_579 = x_622; -goto block_616; +lean_object* x_689; +x_689 = lean_box(0); +x_646 = x_689; +goto block_683; } -block_578: +block_645: { -lean_object* x_525; lean_object* x_526; lean_object* x_534; uint8_t x_572; -x_572 = l_Lean_Expr_hasLevelParam(x_522); -if (x_572 == 0) +lean_object* x_576; lean_object* x_577; lean_object* x_601; uint8_t x_639; +x_639 = l_Lean_Expr_hasLevelParam(x_573); +if (x_639 == 0) { -uint8_t x_573; -x_573 = l_Lean_Expr_hasFVar(x_522); -if (x_573 == 0) +uint8_t x_640; +x_640 = l_Lean_Expr_hasFVar(x_573); +if (x_640 == 0) { -uint8_t x_574; -x_574 = l_Lean_Expr_hasMVar(x_522); -if (x_574 == 0) +uint8_t x_641; +x_641 = l_Lean_Expr_hasMVar(x_573); +if (x_641 == 0) { lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_525 = x_522; -x_526 = x_524; -goto block_533; +x_576 = x_573; +x_577 = x_575; +goto block_600; } else { -lean_object* x_575; -x_575 = lean_box(0); -x_534 = x_575; -goto block_571; +lean_object* x_642; +x_642 = lean_box(0); +x_601 = x_642; +goto block_638; } } else { -lean_object* x_576; -x_576 = lean_box(0); -x_534 = x_576; -goto block_571; +lean_object* x_643; +x_643 = lean_box(0); +x_601 = x_643; +goto block_638; } } else { -lean_object* x_577; -x_577 = lean_box(0); -x_534 = x_577; -goto block_571; +lean_object* x_644; +x_644 = lean_box(0); +x_601 = x_644; +goto block_638; } -block_533: +block_600: { if (lean_obj_tag(x_1) == 7) { -uint8_t x_527; lean_object* x_528; lean_object* x_529; -x_527 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_528 = lean_expr_update_forall(x_1, x_527, x_523, x_525); -x_529 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_529, 0, x_528); -lean_ctor_set(x_529, 1, x_526); -return x_529; +lean_object* x_578; lean_object* x_579; lean_object* x_580; uint8_t x_581; lean_object* x_582; size_t x_583; size_t x_584; uint8_t x_585; +x_578 = lean_ctor_get(x_1, 0); +lean_inc(x_578); +x_579 = lean_ctor_get(x_1, 1); +lean_inc(x_579); +x_580 = lean_ctor_get(x_1, 2); +lean_inc(x_580); +x_581 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_580); +lean_inc(x_579); +lean_inc(x_578); +x_582 = l_Lean_Expr_forallE___override(x_578, x_579, x_580, x_581); +x_583 = lean_ptr_addr(x_579); +lean_dec(x_579); +x_584 = lean_ptr_addr(x_574); +x_585 = lean_usize_dec_eq(x_583, x_584); +if (x_585 == 0) +{ +lean_object* x_586; lean_object* x_587; +lean_dec(x_582); +lean_dec(x_580); +x_586 = l_Lean_Expr_forallE___override(x_578, x_574, x_576, x_581); +x_587 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_587, 0, x_586); +lean_ctor_set(x_587, 1, x_577); +return x_587; +} +else +{ +size_t x_588; size_t x_589; uint8_t x_590; +x_588 = lean_ptr_addr(x_580); +lean_dec(x_580); +x_589 = lean_ptr_addr(x_576); +x_590 = lean_usize_dec_eq(x_588, x_589); +if (x_590 == 0) +{ +lean_object* x_591; lean_object* x_592; +lean_dec(x_582); +x_591 = l_Lean_Expr_forallE___override(x_578, x_574, x_576, x_581); +x_592 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_592, 0, x_591); +lean_ctor_set(x_592, 1, x_577); +return x_592; +} +else +{ +uint8_t x_593; +x_593 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_581, x_581); +if (x_593 == 0) +{ +lean_object* x_594; lean_object* x_595; +lean_dec(x_582); +x_594 = l_Lean_Expr_forallE___override(x_578, x_574, x_576, x_581); +x_595 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_595, 0, x_594); +lean_ctor_set(x_595, 1, x_577); +return x_595; +} +else +{ +lean_object* x_596; +lean_dec(x_578); +lean_dec(x_576); +lean_dec(x_574); +x_596 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_596, 0, x_582); +lean_ctor_set(x_596, 1, x_577); +return x_596; +} +} +} } else { -lean_object* x_530; lean_object* x_531; lean_object* x_532; -lean_dec(x_525); -lean_dec(x_523); +lean_object* x_597; lean_object* x_598; lean_object* x_599; +lean_dec(x_576); +lean_dec(x_574); lean_dec(x_1); -x_530 = l_Lean_Meta_Closure_collectExprAux___closed__16; -x_531 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_530); -x_532 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_532, 0, x_531); -lean_ctor_set(x_532, 1, x_526); -return x_532; +x_597 = l_Lean_Meta_Closure_collectExprAux___closed__16; +x_598 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_597); +x_599 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_599, 0, x_598); +lean_ctor_set(x_599, 1, x_577); +return x_599; } } -block_571: +block_638: { -lean_object* x_535; lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; -lean_dec(x_534); -x_535 = lean_st_ref_get(x_7, x_524); -x_536 = lean_ctor_get(x_535, 1); -lean_inc(x_536); -lean_dec(x_535); -x_537 = lean_st_ref_get(x_3, x_536); -x_538 = lean_ctor_get(x_537, 0); -lean_inc(x_538); -x_539 = lean_ctor_get(x_537, 1); -lean_inc(x_539); -lean_dec(x_537); -x_540 = lean_ctor_get(x_538, 1); -lean_inc(x_540); -lean_dec(x_538); -lean_inc(x_522); -x_541 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_540, x_522); -if (lean_obj_tag(x_541) == 0) +lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; +lean_dec(x_601); +x_602 = lean_st_ref_get(x_7, x_575); +x_603 = lean_ctor_get(x_602, 1); +lean_inc(x_603); +lean_dec(x_602); +x_604 = lean_st_ref_get(x_3, x_603); +x_605 = lean_ctor_get(x_604, 0); +lean_inc(x_605); +x_606 = lean_ctor_get(x_604, 1); +lean_inc(x_606); +lean_dec(x_604); +x_607 = lean_ctor_get(x_605, 1); +lean_inc(x_607); +lean_dec(x_605); +lean_inc(x_573); +x_608 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_607, x_573); +if (lean_obj_tag(x_608) == 0) { -lean_object* x_542; +lean_object* x_609; lean_inc(x_7); -lean_inc(x_522); -x_542 = l_Lean_Meta_Closure_collectExprAux(x_522, x_2, x_3, x_4, x_5, x_6, x_7, x_539); -if (lean_obj_tag(x_542) == 0) +lean_inc(x_573); +x_609 = l_Lean_Meta_Closure_collectExprAux(x_573, x_2, x_3, x_4, x_5, x_6, x_7, x_606); +if (lean_obj_tag(x_609) == 0) { -lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; -x_543 = lean_ctor_get(x_542, 0); -lean_inc(x_543); -x_544 = lean_ctor_get(x_542, 1); -lean_inc(x_544); -lean_dec(x_542); -x_545 = lean_st_ref_get(x_7, x_544); +lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; +x_610 = lean_ctor_get(x_609, 0); +lean_inc(x_610); +x_611 = lean_ctor_get(x_609, 1); +lean_inc(x_611); +lean_dec(x_609); +x_612 = lean_st_ref_get(x_7, x_611); lean_dec(x_7); -x_546 = lean_ctor_get(x_545, 1); -lean_inc(x_546); -lean_dec(x_545); -x_547 = lean_st_ref_take(x_3, x_546); -x_548 = lean_ctor_get(x_547, 0); -lean_inc(x_548); -x_549 = lean_ctor_get(x_547, 1); -lean_inc(x_549); -lean_dec(x_547); -x_550 = lean_ctor_get(x_548, 0); -lean_inc(x_550); -x_551 = lean_ctor_get(x_548, 1); -lean_inc(x_551); -lean_inc(x_543); -x_552 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_551, x_522, x_543); -x_553 = lean_ctor_get(x_548, 2); -lean_inc(x_553); -x_554 = lean_ctor_get(x_548, 3); -lean_inc(x_554); -x_555 = lean_ctor_get(x_548, 4); -lean_inc(x_555); -x_556 = lean_ctor_get(x_548, 5); -lean_inc(x_556); -x_557 = lean_ctor_get(x_548, 6); -lean_inc(x_557); -x_558 = lean_ctor_get(x_548, 7); -lean_inc(x_558); -x_559 = lean_ctor_get(x_548, 8); -lean_inc(x_559); -x_560 = lean_ctor_get(x_548, 9); -lean_inc(x_560); -x_561 = lean_ctor_get(x_548, 10); -lean_inc(x_561); -x_562 = lean_ctor_get(x_548, 11); -lean_inc(x_562); -lean_dec(x_548); -x_563 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_563, 0, x_550); -lean_ctor_set(x_563, 1, x_552); -lean_ctor_set(x_563, 2, x_553); -lean_ctor_set(x_563, 3, x_554); -lean_ctor_set(x_563, 4, x_555); -lean_ctor_set(x_563, 5, x_556); -lean_ctor_set(x_563, 6, x_557); -lean_ctor_set(x_563, 7, x_558); -lean_ctor_set(x_563, 8, x_559); -lean_ctor_set(x_563, 9, x_560); -lean_ctor_set(x_563, 10, x_561); -lean_ctor_set(x_563, 11, x_562); -x_564 = lean_st_ref_set(x_3, x_563, x_549); -x_565 = lean_ctor_get(x_564, 1); -lean_inc(x_565); -lean_dec(x_564); -x_525 = x_543; -x_526 = x_565; -goto block_533; -} -else -{ -uint8_t x_566; -lean_dec(x_523); -lean_dec(x_522); +x_613 = lean_ctor_get(x_612, 1); +lean_inc(x_613); +lean_dec(x_612); +x_614 = lean_st_ref_take(x_3, x_613); +x_615 = lean_ctor_get(x_614, 0); +lean_inc(x_615); +x_616 = lean_ctor_get(x_614, 1); +lean_inc(x_616); +lean_dec(x_614); +x_617 = lean_ctor_get(x_615, 0); +lean_inc(x_617); +x_618 = lean_ctor_get(x_615, 1); +lean_inc(x_618); +lean_inc(x_610); +x_619 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_618, x_573, x_610); +x_620 = lean_ctor_get(x_615, 2); +lean_inc(x_620); +x_621 = lean_ctor_get(x_615, 3); +lean_inc(x_621); +x_622 = lean_ctor_get(x_615, 4); +lean_inc(x_622); +x_623 = lean_ctor_get(x_615, 5); +lean_inc(x_623); +x_624 = lean_ctor_get(x_615, 6); +lean_inc(x_624); +x_625 = lean_ctor_get(x_615, 7); +lean_inc(x_625); +x_626 = lean_ctor_get(x_615, 8); +lean_inc(x_626); +x_627 = lean_ctor_get(x_615, 9); +lean_inc(x_627); +x_628 = lean_ctor_get(x_615, 10); +lean_inc(x_628); +x_629 = lean_ctor_get(x_615, 11); +lean_inc(x_629); +lean_dec(x_615); +x_630 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_630, 0, x_617); +lean_ctor_set(x_630, 1, x_619); +lean_ctor_set(x_630, 2, x_620); +lean_ctor_set(x_630, 3, x_621); +lean_ctor_set(x_630, 4, x_622); +lean_ctor_set(x_630, 5, x_623); +lean_ctor_set(x_630, 6, x_624); +lean_ctor_set(x_630, 7, x_625); +lean_ctor_set(x_630, 8, x_626); +lean_ctor_set(x_630, 9, x_627); +lean_ctor_set(x_630, 10, x_628); +lean_ctor_set(x_630, 11, x_629); +x_631 = lean_st_ref_set(x_3, x_630, x_616); +x_632 = lean_ctor_get(x_631, 1); +lean_inc(x_632); +lean_dec(x_631); +x_576 = x_610; +x_577 = x_632; +goto block_600; +} +else +{ +uint8_t x_633; +lean_dec(x_574); +lean_dec(x_573); lean_dec(x_7); lean_dec(x_1); -x_566 = !lean_is_exclusive(x_542); -if (x_566 == 0) +x_633 = !lean_is_exclusive(x_609); +if (x_633 == 0) { -return x_542; +return x_609; } else { -lean_object* x_567; lean_object* x_568; lean_object* x_569; -x_567 = lean_ctor_get(x_542, 0); -x_568 = lean_ctor_get(x_542, 1); -lean_inc(x_568); -lean_inc(x_567); -lean_dec(x_542); -x_569 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_569, 0, x_567); -lean_ctor_set(x_569, 1, x_568); -return x_569; +lean_object* x_634; lean_object* x_635; lean_object* x_636; +x_634 = lean_ctor_get(x_609, 0); +x_635 = lean_ctor_get(x_609, 1); +lean_inc(x_635); +lean_inc(x_634); +lean_dec(x_609); +x_636 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_636, 0, x_634); +lean_ctor_set(x_636, 1, x_635); +return x_636; } } } else { -lean_object* x_570; -lean_dec(x_522); +lean_object* x_637; +lean_dec(x_573); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_570 = lean_ctor_get(x_541, 0); -lean_inc(x_570); -lean_dec(x_541); -x_525 = x_570; -x_526 = x_539; -goto block_533; +x_637 = lean_ctor_get(x_608, 0); +lean_inc(x_637); +lean_dec(x_608); +x_576 = x_637; +x_577 = x_606; +goto block_600; } } } -block_616: +block_683: { -lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; -lean_dec(x_579); -x_580 = lean_st_ref_get(x_7, x_8); -x_581 = lean_ctor_get(x_580, 1); -lean_inc(x_581); -lean_dec(x_580); -x_582 = lean_st_ref_get(x_3, x_581); -x_583 = lean_ctor_get(x_582, 0); -lean_inc(x_583); -x_584 = lean_ctor_get(x_582, 1); -lean_inc(x_584); -lean_dec(x_582); -x_585 = lean_ctor_get(x_583, 1); -lean_inc(x_585); -lean_dec(x_583); -lean_inc(x_521); -x_586 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_585, x_521); -if (lean_obj_tag(x_586) == 0) -{ -lean_object* x_587; +lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; +lean_dec(x_646); +x_647 = lean_st_ref_get(x_7, x_8); +x_648 = lean_ctor_get(x_647, 1); +lean_inc(x_648); +lean_dec(x_647); +x_649 = lean_st_ref_get(x_3, x_648); +x_650 = lean_ctor_get(x_649, 0); +lean_inc(x_650); +x_651 = lean_ctor_get(x_649, 1); +lean_inc(x_651); +lean_dec(x_649); +x_652 = lean_ctor_get(x_650, 1); +lean_inc(x_652); +lean_dec(x_650); +lean_inc(x_572); +x_653 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_652, x_572); +if (lean_obj_tag(x_653) == 0) +{ +lean_object* x_654; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_521); -x_587 = l_Lean_Meta_Closure_collectExprAux(x_521, x_2, x_3, x_4, x_5, x_6, x_7, x_584); -if (lean_obj_tag(x_587) == 0) -{ -lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; -x_588 = lean_ctor_get(x_587, 0); -lean_inc(x_588); -x_589 = lean_ctor_get(x_587, 1); -lean_inc(x_589); -lean_dec(x_587); -x_590 = lean_st_ref_get(x_7, x_589); -x_591 = lean_ctor_get(x_590, 1); -lean_inc(x_591); -lean_dec(x_590); -x_592 = lean_st_ref_take(x_3, x_591); -x_593 = lean_ctor_get(x_592, 0); -lean_inc(x_593); -x_594 = lean_ctor_get(x_592, 1); -lean_inc(x_594); -lean_dec(x_592); -x_595 = lean_ctor_get(x_593, 0); -lean_inc(x_595); -x_596 = lean_ctor_get(x_593, 1); -lean_inc(x_596); -lean_inc(x_588); -x_597 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_596, x_521, x_588); -x_598 = lean_ctor_get(x_593, 2); -lean_inc(x_598); -x_599 = lean_ctor_get(x_593, 3); -lean_inc(x_599); -x_600 = lean_ctor_get(x_593, 4); -lean_inc(x_600); -x_601 = lean_ctor_get(x_593, 5); -lean_inc(x_601); -x_602 = lean_ctor_get(x_593, 6); -lean_inc(x_602); -x_603 = lean_ctor_get(x_593, 7); -lean_inc(x_603); -x_604 = lean_ctor_get(x_593, 8); -lean_inc(x_604); -x_605 = lean_ctor_get(x_593, 9); -lean_inc(x_605); -x_606 = lean_ctor_get(x_593, 10); -lean_inc(x_606); -x_607 = lean_ctor_get(x_593, 11); -lean_inc(x_607); -lean_dec(x_593); -x_608 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_608, 0, x_595); -lean_ctor_set(x_608, 1, x_597); -lean_ctor_set(x_608, 2, x_598); -lean_ctor_set(x_608, 3, x_599); -lean_ctor_set(x_608, 4, x_600); -lean_ctor_set(x_608, 5, x_601); -lean_ctor_set(x_608, 6, x_602); -lean_ctor_set(x_608, 7, x_603); -lean_ctor_set(x_608, 8, x_604); -lean_ctor_set(x_608, 9, x_605); -lean_ctor_set(x_608, 10, x_606); -lean_ctor_set(x_608, 11, x_607); -x_609 = lean_st_ref_set(x_3, x_608, x_594); -x_610 = lean_ctor_get(x_609, 1); -lean_inc(x_610); -lean_dec(x_609); -x_523 = x_588; -x_524 = x_610; -goto block_578; +lean_inc(x_572); +x_654 = l_Lean_Meta_Closure_collectExprAux(x_572, x_2, x_3, x_4, x_5, x_6, x_7, x_651); +if (lean_obj_tag(x_654) == 0) +{ +lean_object* x_655; lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; lean_object* x_677; +x_655 = lean_ctor_get(x_654, 0); +lean_inc(x_655); +x_656 = lean_ctor_get(x_654, 1); +lean_inc(x_656); +lean_dec(x_654); +x_657 = lean_st_ref_get(x_7, x_656); +x_658 = lean_ctor_get(x_657, 1); +lean_inc(x_658); +lean_dec(x_657); +x_659 = lean_st_ref_take(x_3, x_658); +x_660 = lean_ctor_get(x_659, 0); +lean_inc(x_660); +x_661 = lean_ctor_get(x_659, 1); +lean_inc(x_661); +lean_dec(x_659); +x_662 = lean_ctor_get(x_660, 0); +lean_inc(x_662); +x_663 = lean_ctor_get(x_660, 1); +lean_inc(x_663); +lean_inc(x_655); +x_664 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_663, x_572, x_655); +x_665 = lean_ctor_get(x_660, 2); +lean_inc(x_665); +x_666 = lean_ctor_get(x_660, 3); +lean_inc(x_666); +x_667 = lean_ctor_get(x_660, 4); +lean_inc(x_667); +x_668 = lean_ctor_get(x_660, 5); +lean_inc(x_668); +x_669 = lean_ctor_get(x_660, 6); +lean_inc(x_669); +x_670 = lean_ctor_get(x_660, 7); +lean_inc(x_670); +x_671 = lean_ctor_get(x_660, 8); +lean_inc(x_671); +x_672 = lean_ctor_get(x_660, 9); +lean_inc(x_672); +x_673 = lean_ctor_get(x_660, 10); +lean_inc(x_673); +x_674 = lean_ctor_get(x_660, 11); +lean_inc(x_674); +lean_dec(x_660); +x_675 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_675, 0, x_662); +lean_ctor_set(x_675, 1, x_664); +lean_ctor_set(x_675, 2, x_665); +lean_ctor_set(x_675, 3, x_666); +lean_ctor_set(x_675, 4, x_667); +lean_ctor_set(x_675, 5, x_668); +lean_ctor_set(x_675, 6, x_669); +lean_ctor_set(x_675, 7, x_670); +lean_ctor_set(x_675, 8, x_671); +lean_ctor_set(x_675, 9, x_672); +lean_ctor_set(x_675, 10, x_673); +lean_ctor_set(x_675, 11, x_674); +x_676 = lean_st_ref_set(x_3, x_675, x_661); +x_677 = lean_ctor_get(x_676, 1); +lean_inc(x_677); +lean_dec(x_676); +x_574 = x_655; +x_575 = x_677; +goto block_645; } else { -uint8_t x_611; -lean_dec(x_522); -lean_dec(x_521); +uint8_t x_678; +lean_dec(x_573); +lean_dec(x_572); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_611 = !lean_is_exclusive(x_587); -if (x_611 == 0) +x_678 = !lean_is_exclusive(x_654); +if (x_678 == 0) { -return x_587; +return x_654; } else { -lean_object* x_612; lean_object* x_613; lean_object* x_614; -x_612 = lean_ctor_get(x_587, 0); -x_613 = lean_ctor_get(x_587, 1); -lean_inc(x_613); -lean_inc(x_612); -lean_dec(x_587); -x_614 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_614, 0, x_612); -lean_ctor_set(x_614, 1, x_613); -return x_614; +lean_object* x_679; lean_object* x_680; lean_object* x_681; +x_679 = lean_ctor_get(x_654, 0); +x_680 = lean_ctor_get(x_654, 1); +lean_inc(x_680); +lean_inc(x_679); +lean_dec(x_654); +x_681 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_681, 0, x_679); +lean_ctor_set(x_681, 1, x_680); +return x_681; } } } else { -lean_object* x_615; -lean_dec(x_521); -x_615 = lean_ctor_get(x_586, 0); -lean_inc(x_615); -lean_dec(x_586); -x_523 = x_615; -x_524 = x_584; -goto block_578; +lean_object* x_682; +lean_dec(x_572); +x_682 = lean_ctor_get(x_653, 0); +lean_inc(x_682); +lean_dec(x_653); +x_574 = x_682; +x_575 = x_651; +goto block_645; } } } case 8: { -lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_728; uint8_t x_766; -x_623 = lean_ctor_get(x_1, 1); -lean_inc(x_623); -x_624 = lean_ctor_get(x_1, 2); -lean_inc(x_624); -x_625 = lean_ctor_get(x_1, 3); -lean_inc(x_625); -x_766 = l_Lean_Expr_hasLevelParam(x_623); -if (x_766 == 0) +lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_814; uint8_t x_852; +x_690 = lean_ctor_get(x_1, 1); +lean_inc(x_690); +x_691 = lean_ctor_get(x_1, 2); +lean_inc(x_691); +x_692 = lean_ctor_get(x_1, 3); +lean_inc(x_692); +x_852 = l_Lean_Expr_hasLevelParam(x_690); +if (x_852 == 0) { -uint8_t x_767; -x_767 = l_Lean_Expr_hasFVar(x_623); -if (x_767 == 0) +uint8_t x_853; +x_853 = l_Lean_Expr_hasFVar(x_690); +if (x_853 == 0) { -uint8_t x_768; -x_768 = l_Lean_Expr_hasMVar(x_623); -if (x_768 == 0) +uint8_t x_854; +x_854 = l_Lean_Expr_hasMVar(x_690); +if (x_854 == 0) { -x_626 = x_623; -x_627 = x_8; -goto block_727; +x_693 = x_690; +x_694 = x_8; +goto block_813; } else { -lean_object* x_769; -x_769 = lean_box(0); -x_728 = x_769; -goto block_765; +lean_object* x_855; +x_855 = lean_box(0); +x_814 = x_855; +goto block_851; } } else { -lean_object* x_770; -x_770 = lean_box(0); -x_728 = x_770; -goto block_765; +lean_object* x_856; +x_856 = lean_box(0); +x_814 = x_856; +goto block_851; } } else { -lean_object* x_771; -x_771 = lean_box(0); -x_728 = x_771; -goto block_765; +lean_object* x_857; +x_857 = lean_box(0); +x_814 = x_857; +goto block_851; } -block_727: +block_813: { -lean_object* x_628; lean_object* x_629; lean_object* x_683; uint8_t x_721; -x_721 = l_Lean_Expr_hasLevelParam(x_624); -if (x_721 == 0) +lean_object* x_695; lean_object* x_696; lean_object* x_769; uint8_t x_807; +x_807 = l_Lean_Expr_hasLevelParam(x_691); +if (x_807 == 0) { -uint8_t x_722; -x_722 = l_Lean_Expr_hasFVar(x_624); -if (x_722 == 0) +uint8_t x_808; +x_808 = l_Lean_Expr_hasFVar(x_691); +if (x_808 == 0) { -uint8_t x_723; -x_723 = l_Lean_Expr_hasMVar(x_624); -if (x_723 == 0) +uint8_t x_809; +x_809 = l_Lean_Expr_hasMVar(x_691); +if (x_809 == 0) { -x_628 = x_624; -x_629 = x_627; -goto block_682; +x_695 = x_691; +x_696 = x_694; +goto block_768; } else { -lean_object* x_724; -x_724 = lean_box(0); -x_683 = x_724; -goto block_720; +lean_object* x_810; +x_810 = lean_box(0); +x_769 = x_810; +goto block_806; } } else { -lean_object* x_725; -x_725 = lean_box(0); -x_683 = x_725; -goto block_720; +lean_object* x_811; +x_811 = lean_box(0); +x_769 = x_811; +goto block_806; } } else { -lean_object* x_726; -x_726 = lean_box(0); -x_683 = x_726; -goto block_720; +lean_object* x_812; +x_812 = lean_box(0); +x_769 = x_812; +goto block_806; } -block_682: +block_768: { -lean_object* x_630; lean_object* x_631; lean_object* x_638; uint8_t x_676; -x_676 = l_Lean_Expr_hasLevelParam(x_625); -if (x_676 == 0) +lean_object* x_697; lean_object* x_698; lean_object* x_724; uint8_t x_762; +x_762 = l_Lean_Expr_hasLevelParam(x_692); +if (x_762 == 0) { -uint8_t x_677; -x_677 = l_Lean_Expr_hasFVar(x_625); -if (x_677 == 0) +uint8_t x_763; +x_763 = l_Lean_Expr_hasFVar(x_692); +if (x_763 == 0) { -uint8_t x_678; -x_678 = l_Lean_Expr_hasMVar(x_625); -if (x_678 == 0) +uint8_t x_764; +x_764 = l_Lean_Expr_hasMVar(x_692); +if (x_764 == 0) { lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_630 = x_625; -x_631 = x_629; -goto block_637; +x_697 = x_692; +x_698 = x_696; +goto block_723; +} +else +{ +lean_object* x_765; +x_765 = lean_box(0); +x_724 = x_765; +goto block_761; +} +} +else +{ +lean_object* x_766; +x_766 = lean_box(0); +x_724 = x_766; +goto block_761; +} +} +else +{ +lean_object* x_767; +x_767 = lean_box(0); +x_724 = x_767; +goto block_761; +} +block_723: +{ +if (lean_obj_tag(x_1) == 8) +{ +lean_object* x_699; lean_object* x_700; lean_object* x_701; lean_object* x_702; uint8_t x_703; size_t x_704; size_t x_705; uint8_t x_706; +x_699 = lean_ctor_get(x_1, 0); +lean_inc(x_699); +x_700 = lean_ctor_get(x_1, 1); +lean_inc(x_700); +x_701 = lean_ctor_get(x_1, 2); +lean_inc(x_701); +x_702 = lean_ctor_get(x_1, 3); +lean_inc(x_702); +x_703 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); +x_704 = lean_ptr_addr(x_700); +lean_dec(x_700); +x_705 = lean_ptr_addr(x_693); +x_706 = lean_usize_dec_eq(x_704, x_705); +if (x_706 == 0) +{ +lean_object* x_707; lean_object* x_708; +lean_dec(x_702); +lean_dec(x_701); +lean_dec(x_1); +x_707 = l_Lean_Expr_letE___override(x_699, x_693, x_695, x_697, x_703); +x_708 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_708, 0, x_707); +lean_ctor_set(x_708, 1, x_698); +return x_708; } else { -lean_object* x_679; -x_679 = lean_box(0); -x_638 = x_679; -goto block_675; +size_t x_709; size_t x_710; uint8_t x_711; +x_709 = lean_ptr_addr(x_701); +lean_dec(x_701); +x_710 = lean_ptr_addr(x_695); +x_711 = lean_usize_dec_eq(x_709, x_710); +if (x_711 == 0) +{ +lean_object* x_712; lean_object* x_713; +lean_dec(x_702); +lean_dec(x_1); +x_712 = l_Lean_Expr_letE___override(x_699, x_693, x_695, x_697, x_703); +x_713 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_713, 0, x_712); +lean_ctor_set(x_713, 1, x_698); +return x_713; } +else +{ +size_t x_714; size_t x_715; uint8_t x_716; +x_714 = lean_ptr_addr(x_702); +lean_dec(x_702); +x_715 = lean_ptr_addr(x_697); +x_716 = lean_usize_dec_eq(x_714, x_715); +if (x_716 == 0) +{ +lean_object* x_717; lean_object* x_718; +lean_dec(x_1); +x_717 = l_Lean_Expr_letE___override(x_699, x_693, x_695, x_697, x_703); +x_718 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_718, 0, x_717); +lean_ctor_set(x_718, 1, x_698); +return x_718; } else { -lean_object* x_680; -x_680 = lean_box(0); -x_638 = x_680; -goto block_675; +lean_object* x_719; +lean_dec(x_699); +lean_dec(x_697); +lean_dec(x_695); +lean_dec(x_693); +x_719 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_719, 0, x_1); +lean_ctor_set(x_719, 1, x_698); +return x_719; } } -else -{ -lean_object* x_681; -x_681 = lean_box(0); -x_638 = x_681; -goto block_675; } -block_637: -{ -if (lean_obj_tag(x_1) == 8) -{ -lean_object* x_632; lean_object* x_633; -x_632 = lean_expr_update_let(x_1, x_626, x_628, x_630); -x_633 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_633, 0, x_632); -lean_ctor_set(x_633, 1, x_631); -return x_633; } else { -lean_object* x_634; lean_object* x_635; lean_object* x_636; -lean_dec(x_630); -lean_dec(x_628); -lean_dec(x_626); +lean_object* x_720; lean_object* x_721; lean_object* x_722; +lean_dec(x_697); +lean_dec(x_695); +lean_dec(x_693); lean_dec(x_1); -x_634 = l_Lean_Meta_Closure_collectExprAux___closed__19; -x_635 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_634); -x_636 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_636, 0, x_635); -lean_ctor_set(x_636, 1, x_631); -return x_636; -} -} -block_675: -{ -lean_object* x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; -lean_dec(x_638); -x_639 = lean_st_ref_get(x_7, x_629); -x_640 = lean_ctor_get(x_639, 1); -lean_inc(x_640); -lean_dec(x_639); -x_641 = lean_st_ref_get(x_3, x_640); -x_642 = lean_ctor_get(x_641, 0); -lean_inc(x_642); -x_643 = lean_ctor_get(x_641, 1); -lean_inc(x_643); -lean_dec(x_641); -x_644 = lean_ctor_get(x_642, 1); -lean_inc(x_644); -lean_dec(x_642); -lean_inc(x_625); -x_645 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_644, x_625); -if (lean_obj_tag(x_645) == 0) +x_720 = l_Lean_Meta_Closure_collectExprAux___closed__19; +x_721 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_720); +x_722 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_722, 0, x_721); +lean_ctor_set(x_722, 1, x_698); +return x_722; +} +} +block_761: +{ +lean_object* x_725; lean_object* x_726; lean_object* x_727; lean_object* x_728; lean_object* x_729; lean_object* x_730; lean_object* x_731; +lean_dec(x_724); +x_725 = lean_st_ref_get(x_7, x_696); +x_726 = lean_ctor_get(x_725, 1); +lean_inc(x_726); +lean_dec(x_725); +x_727 = lean_st_ref_get(x_3, x_726); +x_728 = lean_ctor_get(x_727, 0); +lean_inc(x_728); +x_729 = lean_ctor_get(x_727, 1); +lean_inc(x_729); +lean_dec(x_727); +x_730 = lean_ctor_get(x_728, 1); +lean_inc(x_730); +lean_dec(x_728); +lean_inc(x_692); +x_731 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_730, x_692); +if (lean_obj_tag(x_731) == 0) { -lean_object* x_646; +lean_object* x_732; lean_inc(x_7); -lean_inc(x_625); -x_646 = l_Lean_Meta_Closure_collectExprAux(x_625, x_2, x_3, x_4, x_5, x_6, x_7, x_643); -if (lean_obj_tag(x_646) == 0) +lean_inc(x_692); +x_732 = l_Lean_Meta_Closure_collectExprAux(x_692, x_2, x_3, x_4, x_5, x_6, x_7, x_729); +if (lean_obj_tag(x_732) == 0) { -lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; -x_647 = lean_ctor_get(x_646, 0); -lean_inc(x_647); -x_648 = lean_ctor_get(x_646, 1); -lean_inc(x_648); -lean_dec(x_646); -x_649 = lean_st_ref_get(x_7, x_648); +lean_object* x_733; lean_object* x_734; lean_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; lean_object* x_740; lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; lean_object* x_747; lean_object* x_748; lean_object* x_749; lean_object* x_750; lean_object* x_751; lean_object* x_752; lean_object* x_753; lean_object* x_754; lean_object* x_755; +x_733 = lean_ctor_get(x_732, 0); +lean_inc(x_733); +x_734 = lean_ctor_get(x_732, 1); +lean_inc(x_734); +lean_dec(x_732); +x_735 = lean_st_ref_get(x_7, x_734); lean_dec(x_7); -x_650 = lean_ctor_get(x_649, 1); -lean_inc(x_650); -lean_dec(x_649); -x_651 = lean_st_ref_take(x_3, x_650); -x_652 = lean_ctor_get(x_651, 0); -lean_inc(x_652); -x_653 = lean_ctor_get(x_651, 1); -lean_inc(x_653); -lean_dec(x_651); -x_654 = lean_ctor_get(x_652, 0); -lean_inc(x_654); -x_655 = lean_ctor_get(x_652, 1); -lean_inc(x_655); -lean_inc(x_647); -x_656 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_655, x_625, x_647); -x_657 = lean_ctor_get(x_652, 2); -lean_inc(x_657); -x_658 = lean_ctor_get(x_652, 3); -lean_inc(x_658); -x_659 = lean_ctor_get(x_652, 4); -lean_inc(x_659); -x_660 = lean_ctor_get(x_652, 5); -lean_inc(x_660); -x_661 = lean_ctor_get(x_652, 6); -lean_inc(x_661); -x_662 = lean_ctor_get(x_652, 7); -lean_inc(x_662); -x_663 = lean_ctor_get(x_652, 8); -lean_inc(x_663); -x_664 = lean_ctor_get(x_652, 9); -lean_inc(x_664); -x_665 = lean_ctor_get(x_652, 10); -lean_inc(x_665); -x_666 = lean_ctor_get(x_652, 11); -lean_inc(x_666); -lean_dec(x_652); -x_667 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_667, 0, x_654); -lean_ctor_set(x_667, 1, x_656); -lean_ctor_set(x_667, 2, x_657); -lean_ctor_set(x_667, 3, x_658); -lean_ctor_set(x_667, 4, x_659); -lean_ctor_set(x_667, 5, x_660); -lean_ctor_set(x_667, 6, x_661); -lean_ctor_set(x_667, 7, x_662); -lean_ctor_set(x_667, 8, x_663); -lean_ctor_set(x_667, 9, x_664); -lean_ctor_set(x_667, 10, x_665); -lean_ctor_set(x_667, 11, x_666); -x_668 = lean_st_ref_set(x_3, x_667, x_653); -x_669 = lean_ctor_get(x_668, 1); -lean_inc(x_669); -lean_dec(x_668); -x_630 = x_647; -x_631 = x_669; -goto block_637; +x_736 = lean_ctor_get(x_735, 1); +lean_inc(x_736); +lean_dec(x_735); +x_737 = lean_st_ref_take(x_3, x_736); +x_738 = lean_ctor_get(x_737, 0); +lean_inc(x_738); +x_739 = lean_ctor_get(x_737, 1); +lean_inc(x_739); +lean_dec(x_737); +x_740 = lean_ctor_get(x_738, 0); +lean_inc(x_740); +x_741 = lean_ctor_get(x_738, 1); +lean_inc(x_741); +lean_inc(x_733); +x_742 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_741, x_692, x_733); +x_743 = lean_ctor_get(x_738, 2); +lean_inc(x_743); +x_744 = lean_ctor_get(x_738, 3); +lean_inc(x_744); +x_745 = lean_ctor_get(x_738, 4); +lean_inc(x_745); +x_746 = lean_ctor_get(x_738, 5); +lean_inc(x_746); +x_747 = lean_ctor_get(x_738, 6); +lean_inc(x_747); +x_748 = lean_ctor_get(x_738, 7); +lean_inc(x_748); +x_749 = lean_ctor_get(x_738, 8); +lean_inc(x_749); +x_750 = lean_ctor_get(x_738, 9); +lean_inc(x_750); +x_751 = lean_ctor_get(x_738, 10); +lean_inc(x_751); +x_752 = lean_ctor_get(x_738, 11); +lean_inc(x_752); +lean_dec(x_738); +x_753 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_753, 0, x_740); +lean_ctor_set(x_753, 1, x_742); +lean_ctor_set(x_753, 2, x_743); +lean_ctor_set(x_753, 3, x_744); +lean_ctor_set(x_753, 4, x_745); +lean_ctor_set(x_753, 5, x_746); +lean_ctor_set(x_753, 6, x_747); +lean_ctor_set(x_753, 7, x_748); +lean_ctor_set(x_753, 8, x_749); +lean_ctor_set(x_753, 9, x_750); +lean_ctor_set(x_753, 10, x_751); +lean_ctor_set(x_753, 11, x_752); +x_754 = lean_st_ref_set(x_3, x_753, x_739); +x_755 = lean_ctor_get(x_754, 1); +lean_inc(x_755); +lean_dec(x_754); +x_697 = x_733; +x_698 = x_755; +goto block_723; } else { -uint8_t x_670; -lean_dec(x_628); -lean_dec(x_626); -lean_dec(x_625); +uint8_t x_756; +lean_dec(x_695); +lean_dec(x_693); +lean_dec(x_692); lean_dec(x_7); lean_dec(x_1); -x_670 = !lean_is_exclusive(x_646); -if (x_670 == 0) +x_756 = !lean_is_exclusive(x_732); +if (x_756 == 0) { -return x_646; +return x_732; } else { -lean_object* x_671; lean_object* x_672; lean_object* x_673; -x_671 = lean_ctor_get(x_646, 0); -x_672 = lean_ctor_get(x_646, 1); -lean_inc(x_672); -lean_inc(x_671); -lean_dec(x_646); -x_673 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_673, 0, x_671); -lean_ctor_set(x_673, 1, x_672); -return x_673; +lean_object* x_757; lean_object* x_758; lean_object* x_759; +x_757 = lean_ctor_get(x_732, 0); +x_758 = lean_ctor_get(x_732, 1); +lean_inc(x_758); +lean_inc(x_757); +lean_dec(x_732); +x_759 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_759, 0, x_757); +lean_ctor_set(x_759, 1, x_758); +return x_759; } } } else { -lean_object* x_674; -lean_dec(x_625); +lean_object* x_760; +lean_dec(x_692); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_674 = lean_ctor_get(x_645, 0); -lean_inc(x_674); -lean_dec(x_645); -x_630 = x_674; -x_631 = x_643; -goto block_637; -} -} -} -block_720: -{ -lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; lean_object* x_690; -lean_dec(x_683); -x_684 = lean_st_ref_get(x_7, x_627); -x_685 = lean_ctor_get(x_684, 1); -lean_inc(x_685); -lean_dec(x_684); -x_686 = lean_st_ref_get(x_3, x_685); -x_687 = lean_ctor_get(x_686, 0); -lean_inc(x_687); -x_688 = lean_ctor_get(x_686, 1); -lean_inc(x_688); -lean_dec(x_686); -x_689 = lean_ctor_get(x_687, 1); -lean_inc(x_689); -lean_dec(x_687); -lean_inc(x_624); -x_690 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_689, x_624); -if (lean_obj_tag(x_690) == 0) +x_760 = lean_ctor_get(x_731, 0); +lean_inc(x_760); +lean_dec(x_731); +x_697 = x_760; +x_698 = x_729; +goto block_723; +} +} +} +block_806: +{ +lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; lean_object* x_774; lean_object* x_775; lean_object* x_776; +lean_dec(x_769); +x_770 = lean_st_ref_get(x_7, x_694); +x_771 = lean_ctor_get(x_770, 1); +lean_inc(x_771); +lean_dec(x_770); +x_772 = lean_st_ref_get(x_3, x_771); +x_773 = lean_ctor_get(x_772, 0); +lean_inc(x_773); +x_774 = lean_ctor_get(x_772, 1); +lean_inc(x_774); +lean_dec(x_772); +x_775 = lean_ctor_get(x_773, 1); +lean_inc(x_775); +lean_dec(x_773); +lean_inc(x_691); +x_776 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_775, x_691); +if (lean_obj_tag(x_776) == 0) { -lean_object* x_691; +lean_object* x_777; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_624); -x_691 = l_Lean_Meta_Closure_collectExprAux(x_624, x_2, x_3, x_4, x_5, x_6, x_7, x_688); -if (lean_obj_tag(x_691) == 0) +lean_inc(x_691); +x_777 = l_Lean_Meta_Closure_collectExprAux(x_691, x_2, x_3, x_4, x_5, x_6, x_7, x_774); +if (lean_obj_tag(x_777) == 0) { -lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; lean_object* x_713; lean_object* x_714; -x_692 = lean_ctor_get(x_691, 0); -lean_inc(x_692); -x_693 = lean_ctor_get(x_691, 1); -lean_inc(x_693); +lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_796; lean_object* x_797; lean_object* x_798; lean_object* x_799; lean_object* x_800; +x_778 = lean_ctor_get(x_777, 0); +lean_inc(x_778); +x_779 = lean_ctor_get(x_777, 1); +lean_inc(x_779); +lean_dec(x_777); +x_780 = lean_st_ref_get(x_7, x_779); +x_781 = lean_ctor_get(x_780, 1); +lean_inc(x_781); +lean_dec(x_780); +x_782 = lean_st_ref_take(x_3, x_781); +x_783 = lean_ctor_get(x_782, 0); +lean_inc(x_783); +x_784 = lean_ctor_get(x_782, 1); +lean_inc(x_784); +lean_dec(x_782); +x_785 = lean_ctor_get(x_783, 0); +lean_inc(x_785); +x_786 = lean_ctor_get(x_783, 1); +lean_inc(x_786); +lean_inc(x_778); +x_787 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_786, x_691, x_778); +x_788 = lean_ctor_get(x_783, 2); +lean_inc(x_788); +x_789 = lean_ctor_get(x_783, 3); +lean_inc(x_789); +x_790 = lean_ctor_get(x_783, 4); +lean_inc(x_790); +x_791 = lean_ctor_get(x_783, 5); +lean_inc(x_791); +x_792 = lean_ctor_get(x_783, 6); +lean_inc(x_792); +x_793 = lean_ctor_get(x_783, 7); +lean_inc(x_793); +x_794 = lean_ctor_get(x_783, 8); +lean_inc(x_794); +x_795 = lean_ctor_get(x_783, 9); +lean_inc(x_795); +x_796 = lean_ctor_get(x_783, 10); +lean_inc(x_796); +x_797 = lean_ctor_get(x_783, 11); +lean_inc(x_797); +lean_dec(x_783); +x_798 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_798, 0, x_785); +lean_ctor_set(x_798, 1, x_787); +lean_ctor_set(x_798, 2, x_788); +lean_ctor_set(x_798, 3, x_789); +lean_ctor_set(x_798, 4, x_790); +lean_ctor_set(x_798, 5, x_791); +lean_ctor_set(x_798, 6, x_792); +lean_ctor_set(x_798, 7, x_793); +lean_ctor_set(x_798, 8, x_794); +lean_ctor_set(x_798, 9, x_795); +lean_ctor_set(x_798, 10, x_796); +lean_ctor_set(x_798, 11, x_797); +x_799 = lean_st_ref_set(x_3, x_798, x_784); +x_800 = lean_ctor_get(x_799, 1); +lean_inc(x_800); +lean_dec(x_799); +x_695 = x_778; +x_696 = x_800; +goto block_768; +} +else +{ +uint8_t x_801; +lean_dec(x_693); +lean_dec(x_692); lean_dec(x_691); -x_694 = lean_st_ref_get(x_7, x_693); -x_695 = lean_ctor_get(x_694, 1); -lean_inc(x_695); -lean_dec(x_694); -x_696 = lean_st_ref_take(x_3, x_695); -x_697 = lean_ctor_get(x_696, 0); -lean_inc(x_697); -x_698 = lean_ctor_get(x_696, 1); -lean_inc(x_698); -lean_dec(x_696); -x_699 = lean_ctor_get(x_697, 0); -lean_inc(x_699); -x_700 = lean_ctor_get(x_697, 1); -lean_inc(x_700); -lean_inc(x_692); -x_701 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_700, x_624, x_692); -x_702 = lean_ctor_get(x_697, 2); -lean_inc(x_702); -x_703 = lean_ctor_get(x_697, 3); -lean_inc(x_703); -x_704 = lean_ctor_get(x_697, 4); -lean_inc(x_704); -x_705 = lean_ctor_get(x_697, 5); -lean_inc(x_705); -x_706 = lean_ctor_get(x_697, 6); -lean_inc(x_706); -x_707 = lean_ctor_get(x_697, 7); -lean_inc(x_707); -x_708 = lean_ctor_get(x_697, 8); -lean_inc(x_708); -x_709 = lean_ctor_get(x_697, 9); -lean_inc(x_709); -x_710 = lean_ctor_get(x_697, 10); -lean_inc(x_710); -x_711 = lean_ctor_get(x_697, 11); -lean_inc(x_711); -lean_dec(x_697); -x_712 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_712, 0, x_699); -lean_ctor_set(x_712, 1, x_701); -lean_ctor_set(x_712, 2, x_702); -lean_ctor_set(x_712, 3, x_703); -lean_ctor_set(x_712, 4, x_704); -lean_ctor_set(x_712, 5, x_705); -lean_ctor_set(x_712, 6, x_706); -lean_ctor_set(x_712, 7, x_707); -lean_ctor_set(x_712, 8, x_708); -lean_ctor_set(x_712, 9, x_709); -lean_ctor_set(x_712, 10, x_710); -lean_ctor_set(x_712, 11, x_711); -x_713 = lean_st_ref_set(x_3, x_712, x_698); -x_714 = lean_ctor_get(x_713, 1); -lean_inc(x_714); -lean_dec(x_713); -x_628 = x_692; -x_629 = x_714; -goto block_682; -} -else -{ -uint8_t x_715; -lean_dec(x_626); -lean_dec(x_625); -lean_dec(x_624); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_715 = !lean_is_exclusive(x_691); -if (x_715 == 0) +x_801 = !lean_is_exclusive(x_777); +if (x_801 == 0) { -return x_691; +return x_777; } else { -lean_object* x_716; lean_object* x_717; lean_object* x_718; -x_716 = lean_ctor_get(x_691, 0); -x_717 = lean_ctor_get(x_691, 1); -lean_inc(x_717); -lean_inc(x_716); -lean_dec(x_691); -x_718 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_718, 0, x_716); -lean_ctor_set(x_718, 1, x_717); -return x_718; +lean_object* x_802; lean_object* x_803; lean_object* x_804; +x_802 = lean_ctor_get(x_777, 0); +x_803 = lean_ctor_get(x_777, 1); +lean_inc(x_803); +lean_inc(x_802); +lean_dec(x_777); +x_804 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_804, 0, x_802); +lean_ctor_set(x_804, 1, x_803); +return x_804; } } } else { -lean_object* x_719; -lean_dec(x_624); -x_719 = lean_ctor_get(x_690, 0); -lean_inc(x_719); -lean_dec(x_690); -x_628 = x_719; -x_629 = x_688; -goto block_682; +lean_object* x_805; +lean_dec(x_691); +x_805 = lean_ctor_get(x_776, 0); +lean_inc(x_805); +lean_dec(x_776); +x_695 = x_805; +x_696 = x_774; +goto block_768; } } } -block_765: +block_851: { -lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; lean_object* x_735; -lean_dec(x_728); -x_729 = lean_st_ref_get(x_7, x_8); -x_730 = lean_ctor_get(x_729, 1); -lean_inc(x_730); -lean_dec(x_729); -x_731 = lean_st_ref_get(x_3, x_730); -x_732 = lean_ctor_get(x_731, 0); -lean_inc(x_732); -x_733 = lean_ctor_get(x_731, 1); -lean_inc(x_733); -lean_dec(x_731); -x_734 = lean_ctor_get(x_732, 1); -lean_inc(x_734); -lean_dec(x_732); -lean_inc(x_623); -x_735 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_734, x_623); -if (lean_obj_tag(x_735) == 0) +lean_object* x_815; lean_object* x_816; lean_object* x_817; lean_object* x_818; lean_object* x_819; lean_object* x_820; lean_object* x_821; +lean_dec(x_814); +x_815 = lean_st_ref_get(x_7, x_8); +x_816 = lean_ctor_get(x_815, 1); +lean_inc(x_816); +lean_dec(x_815); +x_817 = lean_st_ref_get(x_3, x_816); +x_818 = lean_ctor_get(x_817, 0); +lean_inc(x_818); +x_819 = lean_ctor_get(x_817, 1); +lean_inc(x_819); +lean_dec(x_817); +x_820 = lean_ctor_get(x_818, 1); +lean_inc(x_820); +lean_dec(x_818); +lean_inc(x_690); +x_821 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_820, x_690); +if (lean_obj_tag(x_821) == 0) { -lean_object* x_736; +lean_object* x_822; lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_623); -x_736 = l_Lean_Meta_Closure_collectExprAux(x_623, x_2, x_3, x_4, x_5, x_6, x_7, x_733); -if (lean_obj_tag(x_736) == 0) +lean_inc(x_690); +x_822 = l_Lean_Meta_Closure_collectExprAux(x_690, x_2, x_3, x_4, x_5, x_6, x_7, x_819); +if (lean_obj_tag(x_822) == 0) { -lean_object* x_737; lean_object* x_738; lean_object* x_739; lean_object* x_740; lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; lean_object* x_747; lean_object* x_748; lean_object* x_749; lean_object* x_750; lean_object* x_751; lean_object* x_752; lean_object* x_753; lean_object* x_754; lean_object* x_755; lean_object* x_756; lean_object* x_757; lean_object* x_758; lean_object* x_759; -x_737 = lean_ctor_get(x_736, 0); -lean_inc(x_737); -x_738 = lean_ctor_get(x_736, 1); -lean_inc(x_738); -lean_dec(x_736); -x_739 = lean_st_ref_get(x_7, x_738); -x_740 = lean_ctor_get(x_739, 1); -lean_inc(x_740); -lean_dec(x_739); -x_741 = lean_st_ref_take(x_3, x_740); -x_742 = lean_ctor_get(x_741, 0); -lean_inc(x_742); -x_743 = lean_ctor_get(x_741, 1); -lean_inc(x_743); -lean_dec(x_741); -x_744 = lean_ctor_get(x_742, 0); -lean_inc(x_744); -x_745 = lean_ctor_get(x_742, 1); -lean_inc(x_745); -lean_inc(x_737); -x_746 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_745, x_623, x_737); -x_747 = lean_ctor_get(x_742, 2); -lean_inc(x_747); -x_748 = lean_ctor_get(x_742, 3); -lean_inc(x_748); -x_749 = lean_ctor_get(x_742, 4); -lean_inc(x_749); -x_750 = lean_ctor_get(x_742, 5); -lean_inc(x_750); -x_751 = lean_ctor_get(x_742, 6); -lean_inc(x_751); -x_752 = lean_ctor_get(x_742, 7); -lean_inc(x_752); -x_753 = lean_ctor_get(x_742, 8); -lean_inc(x_753); -x_754 = lean_ctor_get(x_742, 9); -lean_inc(x_754); -x_755 = lean_ctor_get(x_742, 10); -lean_inc(x_755); -x_756 = lean_ctor_get(x_742, 11); -lean_inc(x_756); -lean_dec(x_742); -x_757 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_757, 0, x_744); -lean_ctor_set(x_757, 1, x_746); -lean_ctor_set(x_757, 2, x_747); -lean_ctor_set(x_757, 3, x_748); -lean_ctor_set(x_757, 4, x_749); -lean_ctor_set(x_757, 5, x_750); -lean_ctor_set(x_757, 6, x_751); -lean_ctor_set(x_757, 7, x_752); -lean_ctor_set(x_757, 8, x_753); -lean_ctor_set(x_757, 9, x_754); -lean_ctor_set(x_757, 10, x_755); -lean_ctor_set(x_757, 11, x_756); -x_758 = lean_st_ref_set(x_3, x_757, x_743); -x_759 = lean_ctor_get(x_758, 1); -lean_inc(x_759); -lean_dec(x_758); -x_626 = x_737; -x_627 = x_759; -goto block_727; -} -else -{ -uint8_t x_760; -lean_dec(x_625); -lean_dec(x_624); -lean_dec(x_623); +lean_object* x_823; lean_object* x_824; lean_object* x_825; lean_object* x_826; lean_object* x_827; lean_object* x_828; lean_object* x_829; lean_object* x_830; lean_object* x_831; lean_object* x_832; lean_object* x_833; lean_object* x_834; lean_object* x_835; lean_object* x_836; lean_object* x_837; lean_object* x_838; lean_object* x_839; lean_object* x_840; lean_object* x_841; lean_object* x_842; lean_object* x_843; lean_object* x_844; lean_object* x_845; +x_823 = lean_ctor_get(x_822, 0); +lean_inc(x_823); +x_824 = lean_ctor_get(x_822, 1); +lean_inc(x_824); +lean_dec(x_822); +x_825 = lean_st_ref_get(x_7, x_824); +x_826 = lean_ctor_get(x_825, 1); +lean_inc(x_826); +lean_dec(x_825); +x_827 = lean_st_ref_take(x_3, x_826); +x_828 = lean_ctor_get(x_827, 0); +lean_inc(x_828); +x_829 = lean_ctor_get(x_827, 1); +lean_inc(x_829); +lean_dec(x_827); +x_830 = lean_ctor_get(x_828, 0); +lean_inc(x_830); +x_831 = lean_ctor_get(x_828, 1); +lean_inc(x_831); +lean_inc(x_823); +x_832 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_831, x_690, x_823); +x_833 = lean_ctor_get(x_828, 2); +lean_inc(x_833); +x_834 = lean_ctor_get(x_828, 3); +lean_inc(x_834); +x_835 = lean_ctor_get(x_828, 4); +lean_inc(x_835); +x_836 = lean_ctor_get(x_828, 5); +lean_inc(x_836); +x_837 = lean_ctor_get(x_828, 6); +lean_inc(x_837); +x_838 = lean_ctor_get(x_828, 7); +lean_inc(x_838); +x_839 = lean_ctor_get(x_828, 8); +lean_inc(x_839); +x_840 = lean_ctor_get(x_828, 9); +lean_inc(x_840); +x_841 = lean_ctor_get(x_828, 10); +lean_inc(x_841); +x_842 = lean_ctor_get(x_828, 11); +lean_inc(x_842); +lean_dec(x_828); +x_843 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_843, 0, x_830); +lean_ctor_set(x_843, 1, x_832); +lean_ctor_set(x_843, 2, x_833); +lean_ctor_set(x_843, 3, x_834); +lean_ctor_set(x_843, 4, x_835); +lean_ctor_set(x_843, 5, x_836); +lean_ctor_set(x_843, 6, x_837); +lean_ctor_set(x_843, 7, x_838); +lean_ctor_set(x_843, 8, x_839); +lean_ctor_set(x_843, 9, x_840); +lean_ctor_set(x_843, 10, x_841); +lean_ctor_set(x_843, 11, x_842); +x_844 = lean_st_ref_set(x_3, x_843, x_829); +x_845 = lean_ctor_get(x_844, 1); +lean_inc(x_845); +lean_dec(x_844); +x_693 = x_823; +x_694 = x_845; +goto block_813; +} +else +{ +uint8_t x_846; +lean_dec(x_692); +lean_dec(x_691); +lean_dec(x_690); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_760 = !lean_is_exclusive(x_736); -if (x_760 == 0) +x_846 = !lean_is_exclusive(x_822); +if (x_846 == 0) { -return x_736; +return x_822; } else { -lean_object* x_761; lean_object* x_762; lean_object* x_763; -x_761 = lean_ctor_get(x_736, 0); -x_762 = lean_ctor_get(x_736, 1); -lean_inc(x_762); -lean_inc(x_761); -lean_dec(x_736); -x_763 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_763, 0, x_761); -lean_ctor_set(x_763, 1, x_762); -return x_763; +lean_object* x_847; lean_object* x_848; lean_object* x_849; +x_847 = lean_ctor_get(x_822, 0); +x_848 = lean_ctor_get(x_822, 1); +lean_inc(x_848); +lean_inc(x_847); +lean_dec(x_822); +x_849 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_849, 0, x_847); +lean_ctor_set(x_849, 1, x_848); +return x_849; } } } else { -lean_object* x_764; -lean_dec(x_623); -x_764 = lean_ctor_get(x_735, 0); -lean_inc(x_764); -lean_dec(x_735); -x_626 = x_764; -x_627 = x_733; -goto block_727; +lean_object* x_850; +lean_dec(x_690); +x_850 = lean_ctor_get(x_821, 0); +lean_inc(x_850); +lean_dec(x_821); +x_693 = x_850; +x_694 = x_819; +goto block_813; } } } case 10: { -lean_object* x_772; lean_object* x_773; uint8_t x_811; -x_772 = lean_ctor_get(x_1, 1); -lean_inc(x_772); -x_811 = l_Lean_Expr_hasLevelParam(x_772); -if (x_811 == 0) +lean_object* x_858; lean_object* x_859; uint8_t x_897; +x_858 = lean_ctor_get(x_1, 1); +lean_inc(x_858); +x_897 = l_Lean_Expr_hasLevelParam(x_858); +if (x_897 == 0) { -uint8_t x_812; -x_812 = l_Lean_Expr_hasFVar(x_772); -if (x_812 == 0) +uint8_t x_898; +x_898 = l_Lean_Expr_hasFVar(x_858); +if (x_898 == 0) { -uint8_t x_813; -x_813 = l_Lean_Expr_hasMVar(x_772); -if (x_813 == 0) +uint8_t x_899; +x_899 = l_Lean_Expr_hasMVar(x_858); +if (x_899 == 0) { lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_9 = x_772; +x_9 = x_858; x_10 = x_8; -goto block_16; +goto block_22; } else { -lean_object* x_814; -x_814 = lean_box(0); -x_773 = x_814; -goto block_810; +lean_object* x_900; +x_900 = lean_box(0); +x_859 = x_900; +goto block_896; } } else { -lean_object* x_815; -x_815 = lean_box(0); -x_773 = x_815; -goto block_810; +lean_object* x_901; +x_901 = lean_box(0); +x_859 = x_901; +goto block_896; } } else { -lean_object* x_816; -x_816 = lean_box(0); -x_773 = x_816; -goto block_810; +lean_object* x_902; +x_902 = lean_box(0); +x_859 = x_902; +goto block_896; } -block_810: +block_896: { -lean_object* x_774; lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; -lean_dec(x_773); -x_774 = lean_st_ref_get(x_7, x_8); -x_775 = lean_ctor_get(x_774, 1); -lean_inc(x_775); -lean_dec(x_774); -x_776 = lean_st_ref_get(x_3, x_775); -x_777 = lean_ctor_get(x_776, 0); -lean_inc(x_777); -x_778 = lean_ctor_get(x_776, 1); -lean_inc(x_778); -lean_dec(x_776); -x_779 = lean_ctor_get(x_777, 1); -lean_inc(x_779); -lean_dec(x_777); -lean_inc(x_772); -x_780 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_779, x_772); -if (lean_obj_tag(x_780) == 0) +lean_object* x_860; lean_object* x_861; lean_object* x_862; lean_object* x_863; lean_object* x_864; lean_object* x_865; lean_object* x_866; +lean_dec(x_859); +x_860 = lean_st_ref_get(x_7, x_8); +x_861 = lean_ctor_get(x_860, 1); +lean_inc(x_861); +lean_dec(x_860); +x_862 = lean_st_ref_get(x_3, x_861); +x_863 = lean_ctor_get(x_862, 0); +lean_inc(x_863); +x_864 = lean_ctor_get(x_862, 1); +lean_inc(x_864); +lean_dec(x_862); +x_865 = lean_ctor_get(x_863, 1); +lean_inc(x_865); +lean_dec(x_863); +lean_inc(x_858); +x_866 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_865, x_858); +if (lean_obj_tag(x_866) == 0) { -lean_object* x_781; +lean_object* x_867; lean_inc(x_7); -lean_inc(x_772); -x_781 = l_Lean_Meta_Closure_collectExprAux(x_772, x_2, x_3, x_4, x_5, x_6, x_7, x_778); -if (lean_obj_tag(x_781) == 0) -{ -lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_796; lean_object* x_797; lean_object* x_798; lean_object* x_799; lean_object* x_800; lean_object* x_801; lean_object* x_802; lean_object* x_803; lean_object* x_804; -x_782 = lean_ctor_get(x_781, 0); -lean_inc(x_782); -x_783 = lean_ctor_get(x_781, 1); -lean_inc(x_783); -lean_dec(x_781); -x_784 = lean_st_ref_get(x_7, x_783); +lean_inc(x_858); +x_867 = l_Lean_Meta_Closure_collectExprAux(x_858, x_2, x_3, x_4, x_5, x_6, x_7, x_864); +if (lean_obj_tag(x_867) == 0) +{ +lean_object* x_868; lean_object* x_869; lean_object* x_870; lean_object* x_871; lean_object* x_872; lean_object* x_873; lean_object* x_874; lean_object* x_875; lean_object* x_876; lean_object* x_877; lean_object* x_878; lean_object* x_879; lean_object* x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; lean_object* x_884; lean_object* x_885; lean_object* x_886; lean_object* x_887; lean_object* x_888; lean_object* x_889; lean_object* x_890; +x_868 = lean_ctor_get(x_867, 0); +lean_inc(x_868); +x_869 = lean_ctor_get(x_867, 1); +lean_inc(x_869); +lean_dec(x_867); +x_870 = lean_st_ref_get(x_7, x_869); lean_dec(x_7); -x_785 = lean_ctor_get(x_784, 1); -lean_inc(x_785); -lean_dec(x_784); -x_786 = lean_st_ref_take(x_3, x_785); -x_787 = lean_ctor_get(x_786, 0); -lean_inc(x_787); -x_788 = lean_ctor_get(x_786, 1); -lean_inc(x_788); -lean_dec(x_786); -x_789 = lean_ctor_get(x_787, 0); -lean_inc(x_789); -x_790 = lean_ctor_get(x_787, 1); -lean_inc(x_790); -lean_inc(x_782); -x_791 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_790, x_772, x_782); -x_792 = lean_ctor_get(x_787, 2); -lean_inc(x_792); -x_793 = lean_ctor_get(x_787, 3); -lean_inc(x_793); -x_794 = lean_ctor_get(x_787, 4); -lean_inc(x_794); -x_795 = lean_ctor_get(x_787, 5); -lean_inc(x_795); -x_796 = lean_ctor_get(x_787, 6); -lean_inc(x_796); -x_797 = lean_ctor_get(x_787, 7); -lean_inc(x_797); -x_798 = lean_ctor_get(x_787, 8); -lean_inc(x_798); -x_799 = lean_ctor_get(x_787, 9); -lean_inc(x_799); -x_800 = lean_ctor_get(x_787, 10); -lean_inc(x_800); -x_801 = lean_ctor_get(x_787, 11); -lean_inc(x_801); -lean_dec(x_787); -x_802 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_802, 0, x_789); -lean_ctor_set(x_802, 1, x_791); -lean_ctor_set(x_802, 2, x_792); -lean_ctor_set(x_802, 3, x_793); -lean_ctor_set(x_802, 4, x_794); -lean_ctor_set(x_802, 5, x_795); -lean_ctor_set(x_802, 6, x_796); -lean_ctor_set(x_802, 7, x_797); -lean_ctor_set(x_802, 8, x_798); -lean_ctor_set(x_802, 9, x_799); -lean_ctor_set(x_802, 10, x_800); -lean_ctor_set(x_802, 11, x_801); -x_803 = lean_st_ref_set(x_3, x_802, x_788); -x_804 = lean_ctor_get(x_803, 1); -lean_inc(x_804); -lean_dec(x_803); -x_9 = x_782; -x_10 = x_804; -goto block_16; -} -else -{ -uint8_t x_805; -lean_dec(x_772); +x_871 = lean_ctor_get(x_870, 1); +lean_inc(x_871); +lean_dec(x_870); +x_872 = lean_st_ref_take(x_3, x_871); +x_873 = lean_ctor_get(x_872, 0); +lean_inc(x_873); +x_874 = lean_ctor_get(x_872, 1); +lean_inc(x_874); +lean_dec(x_872); +x_875 = lean_ctor_get(x_873, 0); +lean_inc(x_875); +x_876 = lean_ctor_get(x_873, 1); +lean_inc(x_876); +lean_inc(x_868); +x_877 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_876, x_858, x_868); +x_878 = lean_ctor_get(x_873, 2); +lean_inc(x_878); +x_879 = lean_ctor_get(x_873, 3); +lean_inc(x_879); +x_880 = lean_ctor_get(x_873, 4); +lean_inc(x_880); +x_881 = lean_ctor_get(x_873, 5); +lean_inc(x_881); +x_882 = lean_ctor_get(x_873, 6); +lean_inc(x_882); +x_883 = lean_ctor_get(x_873, 7); +lean_inc(x_883); +x_884 = lean_ctor_get(x_873, 8); +lean_inc(x_884); +x_885 = lean_ctor_get(x_873, 9); +lean_inc(x_885); +x_886 = lean_ctor_get(x_873, 10); +lean_inc(x_886); +x_887 = lean_ctor_get(x_873, 11); +lean_inc(x_887); +lean_dec(x_873); +x_888 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_888, 0, x_875); +lean_ctor_set(x_888, 1, x_877); +lean_ctor_set(x_888, 2, x_878); +lean_ctor_set(x_888, 3, x_879); +lean_ctor_set(x_888, 4, x_880); +lean_ctor_set(x_888, 5, x_881); +lean_ctor_set(x_888, 6, x_882); +lean_ctor_set(x_888, 7, x_883); +lean_ctor_set(x_888, 8, x_884); +lean_ctor_set(x_888, 9, x_885); +lean_ctor_set(x_888, 10, x_886); +lean_ctor_set(x_888, 11, x_887); +x_889 = lean_st_ref_set(x_3, x_888, x_874); +x_890 = lean_ctor_get(x_889, 1); +lean_inc(x_890); +lean_dec(x_889); +x_9 = x_868; +x_10 = x_890; +goto block_22; +} +else +{ +uint8_t x_891; +lean_dec(x_858); lean_dec(x_7); lean_dec(x_1); -x_805 = !lean_is_exclusive(x_781); -if (x_805 == 0) +x_891 = !lean_is_exclusive(x_867); +if (x_891 == 0) { -return x_781; +return x_867; } else { -lean_object* x_806; lean_object* x_807; lean_object* x_808; -x_806 = lean_ctor_get(x_781, 0); -x_807 = lean_ctor_get(x_781, 1); -lean_inc(x_807); -lean_inc(x_806); -lean_dec(x_781); -x_808 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_808, 0, x_806); -lean_ctor_set(x_808, 1, x_807); -return x_808; +lean_object* x_892; lean_object* x_893; lean_object* x_894; +x_892 = lean_ctor_get(x_867, 0); +x_893 = lean_ctor_get(x_867, 1); +lean_inc(x_893); +lean_inc(x_892); +lean_dec(x_867); +x_894 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_894, 0, x_892); +lean_ctor_set(x_894, 1, x_893); +return x_894; } } } else { -lean_object* x_809; -lean_dec(x_772); +lean_object* x_895; +lean_dec(x_858); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_809 = lean_ctor_get(x_780, 0); -lean_inc(x_809); -lean_dec(x_780); -x_9 = x_809; -x_10 = x_778; -goto block_16; +x_895 = lean_ctor_get(x_866, 0); +lean_inc(x_895); +lean_dec(x_866); +x_9 = x_895; +x_10 = x_864; +goto block_22; } } } case 11: { -lean_object* x_817; lean_object* x_818; uint8_t x_856; -x_817 = lean_ctor_get(x_1, 2); -lean_inc(x_817); -x_856 = l_Lean_Expr_hasLevelParam(x_817); -if (x_856 == 0) +lean_object* x_903; lean_object* x_904; uint8_t x_942; +x_903 = lean_ctor_get(x_1, 2); +lean_inc(x_903); +x_942 = l_Lean_Expr_hasLevelParam(x_903); +if (x_942 == 0) { -uint8_t x_857; -x_857 = l_Lean_Expr_hasFVar(x_817); -if (x_857 == 0) +uint8_t x_943; +x_943 = l_Lean_Expr_hasFVar(x_903); +if (x_943 == 0) { -uint8_t x_858; -x_858 = l_Lean_Expr_hasMVar(x_817); -if (x_858 == 0) +uint8_t x_944; +x_944 = l_Lean_Expr_hasMVar(x_903); +if (x_944 == 0) { lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_17 = x_817; -x_18 = x_8; -goto block_24; +x_23 = x_903; +x_24 = x_8; +goto block_37; } else { -lean_object* x_859; -x_859 = lean_box(0); -x_818 = x_859; -goto block_855; +lean_object* x_945; +x_945 = lean_box(0); +x_904 = x_945; +goto block_941; } } else { -lean_object* x_860; -x_860 = lean_box(0); -x_818 = x_860; -goto block_855; +lean_object* x_946; +x_946 = lean_box(0); +x_904 = x_946; +goto block_941; } } else { -lean_object* x_861; -x_861 = lean_box(0); -x_818 = x_861; -goto block_855; +lean_object* x_947; +x_947 = lean_box(0); +x_904 = x_947; +goto block_941; } -block_855: +block_941: { -lean_object* x_819; lean_object* x_820; lean_object* x_821; lean_object* x_822; lean_object* x_823; lean_object* x_824; lean_object* x_825; -lean_dec(x_818); -x_819 = lean_st_ref_get(x_7, x_8); -x_820 = lean_ctor_get(x_819, 1); -lean_inc(x_820); -lean_dec(x_819); -x_821 = lean_st_ref_get(x_3, x_820); -x_822 = lean_ctor_get(x_821, 0); -lean_inc(x_822); -x_823 = lean_ctor_get(x_821, 1); -lean_inc(x_823); -lean_dec(x_821); -x_824 = lean_ctor_get(x_822, 1); -lean_inc(x_824); -lean_dec(x_822); -lean_inc(x_817); -x_825 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_824, x_817); -if (lean_obj_tag(x_825) == 0) +lean_object* x_905; lean_object* x_906; lean_object* x_907; lean_object* x_908; lean_object* x_909; lean_object* x_910; lean_object* x_911; +lean_dec(x_904); +x_905 = lean_st_ref_get(x_7, x_8); +x_906 = lean_ctor_get(x_905, 1); +lean_inc(x_906); +lean_dec(x_905); +x_907 = lean_st_ref_get(x_3, x_906); +x_908 = lean_ctor_get(x_907, 0); +lean_inc(x_908); +x_909 = lean_ctor_get(x_907, 1); +lean_inc(x_909); +lean_dec(x_907); +x_910 = lean_ctor_get(x_908, 1); +lean_inc(x_910); +lean_dec(x_908); +lean_inc(x_903); +x_911 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_910, x_903); +if (lean_obj_tag(x_911) == 0) { -lean_object* x_826; +lean_object* x_912; lean_inc(x_7); -lean_inc(x_817); -x_826 = l_Lean_Meta_Closure_collectExprAux(x_817, x_2, x_3, x_4, x_5, x_6, x_7, x_823); -if (lean_obj_tag(x_826) == 0) -{ -lean_object* x_827; lean_object* x_828; lean_object* x_829; lean_object* x_830; lean_object* x_831; lean_object* x_832; lean_object* x_833; lean_object* x_834; lean_object* x_835; lean_object* x_836; lean_object* x_837; lean_object* x_838; lean_object* x_839; lean_object* x_840; lean_object* x_841; lean_object* x_842; lean_object* x_843; lean_object* x_844; lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; lean_object* x_849; -x_827 = lean_ctor_get(x_826, 0); -lean_inc(x_827); -x_828 = lean_ctor_get(x_826, 1); -lean_inc(x_828); -lean_dec(x_826); -x_829 = lean_st_ref_get(x_7, x_828); +lean_inc(x_903); +x_912 = l_Lean_Meta_Closure_collectExprAux(x_903, x_2, x_3, x_4, x_5, x_6, x_7, x_909); +if (lean_obj_tag(x_912) == 0) +{ +lean_object* x_913; lean_object* x_914; lean_object* x_915; lean_object* x_916; lean_object* x_917; lean_object* x_918; lean_object* x_919; lean_object* x_920; lean_object* x_921; lean_object* x_922; lean_object* x_923; lean_object* x_924; lean_object* x_925; lean_object* x_926; lean_object* x_927; lean_object* x_928; lean_object* x_929; lean_object* x_930; lean_object* x_931; lean_object* x_932; lean_object* x_933; lean_object* x_934; lean_object* x_935; +x_913 = lean_ctor_get(x_912, 0); +lean_inc(x_913); +x_914 = lean_ctor_get(x_912, 1); +lean_inc(x_914); +lean_dec(x_912); +x_915 = lean_st_ref_get(x_7, x_914); lean_dec(x_7); -x_830 = lean_ctor_get(x_829, 1); -lean_inc(x_830); -lean_dec(x_829); -x_831 = lean_st_ref_take(x_3, x_830); -x_832 = lean_ctor_get(x_831, 0); -lean_inc(x_832); -x_833 = lean_ctor_get(x_831, 1); -lean_inc(x_833); -lean_dec(x_831); -x_834 = lean_ctor_get(x_832, 0); -lean_inc(x_834); -x_835 = lean_ctor_get(x_832, 1); -lean_inc(x_835); -lean_inc(x_827); -x_836 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_835, x_817, x_827); -x_837 = lean_ctor_get(x_832, 2); -lean_inc(x_837); -x_838 = lean_ctor_get(x_832, 3); -lean_inc(x_838); -x_839 = lean_ctor_get(x_832, 4); -lean_inc(x_839); -x_840 = lean_ctor_get(x_832, 5); -lean_inc(x_840); -x_841 = lean_ctor_get(x_832, 6); -lean_inc(x_841); -x_842 = lean_ctor_get(x_832, 7); -lean_inc(x_842); -x_843 = lean_ctor_get(x_832, 8); -lean_inc(x_843); -x_844 = lean_ctor_get(x_832, 9); -lean_inc(x_844); -x_845 = lean_ctor_get(x_832, 10); -lean_inc(x_845); -x_846 = lean_ctor_get(x_832, 11); -lean_inc(x_846); -lean_dec(x_832); -x_847 = lean_alloc_ctor(0, 12, 0); -lean_ctor_set(x_847, 0, x_834); -lean_ctor_set(x_847, 1, x_836); -lean_ctor_set(x_847, 2, x_837); -lean_ctor_set(x_847, 3, x_838); -lean_ctor_set(x_847, 4, x_839); -lean_ctor_set(x_847, 5, x_840); -lean_ctor_set(x_847, 6, x_841); -lean_ctor_set(x_847, 7, x_842); -lean_ctor_set(x_847, 8, x_843); -lean_ctor_set(x_847, 9, x_844); -lean_ctor_set(x_847, 10, x_845); -lean_ctor_set(x_847, 11, x_846); -x_848 = lean_st_ref_set(x_3, x_847, x_833); -x_849 = lean_ctor_get(x_848, 1); -lean_inc(x_849); -lean_dec(x_848); -x_17 = x_827; -x_18 = x_849; -goto block_24; -} -else -{ -uint8_t x_850; -lean_dec(x_817); +x_916 = lean_ctor_get(x_915, 1); +lean_inc(x_916); +lean_dec(x_915); +x_917 = lean_st_ref_take(x_3, x_916); +x_918 = lean_ctor_get(x_917, 0); +lean_inc(x_918); +x_919 = lean_ctor_get(x_917, 1); +lean_inc(x_919); +lean_dec(x_917); +x_920 = lean_ctor_get(x_918, 0); +lean_inc(x_920); +x_921 = lean_ctor_get(x_918, 1); +lean_inc(x_921); +lean_inc(x_913); +x_922 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_921, x_903, x_913); +x_923 = lean_ctor_get(x_918, 2); +lean_inc(x_923); +x_924 = lean_ctor_get(x_918, 3); +lean_inc(x_924); +x_925 = lean_ctor_get(x_918, 4); +lean_inc(x_925); +x_926 = lean_ctor_get(x_918, 5); +lean_inc(x_926); +x_927 = lean_ctor_get(x_918, 6); +lean_inc(x_927); +x_928 = lean_ctor_get(x_918, 7); +lean_inc(x_928); +x_929 = lean_ctor_get(x_918, 8); +lean_inc(x_929); +x_930 = lean_ctor_get(x_918, 9); +lean_inc(x_930); +x_931 = lean_ctor_get(x_918, 10); +lean_inc(x_931); +x_932 = lean_ctor_get(x_918, 11); +lean_inc(x_932); +lean_dec(x_918); +x_933 = lean_alloc_ctor(0, 12, 0); +lean_ctor_set(x_933, 0, x_920); +lean_ctor_set(x_933, 1, x_922); +lean_ctor_set(x_933, 2, x_923); +lean_ctor_set(x_933, 3, x_924); +lean_ctor_set(x_933, 4, x_925); +lean_ctor_set(x_933, 5, x_926); +lean_ctor_set(x_933, 6, x_927); +lean_ctor_set(x_933, 7, x_928); +lean_ctor_set(x_933, 8, x_929); +lean_ctor_set(x_933, 9, x_930); +lean_ctor_set(x_933, 10, x_931); +lean_ctor_set(x_933, 11, x_932); +x_934 = lean_st_ref_set(x_3, x_933, x_919); +x_935 = lean_ctor_get(x_934, 1); +lean_inc(x_935); +lean_dec(x_934); +x_23 = x_913; +x_24 = x_935; +goto block_37; +} +else +{ +uint8_t x_936; +lean_dec(x_903); lean_dec(x_7); lean_dec(x_1); -x_850 = !lean_is_exclusive(x_826); -if (x_850 == 0) +x_936 = !lean_is_exclusive(x_912); +if (x_936 == 0) { -return x_826; +return x_912; } else { -lean_object* x_851; lean_object* x_852; lean_object* x_853; -x_851 = lean_ctor_get(x_826, 0); -x_852 = lean_ctor_get(x_826, 1); -lean_inc(x_852); -lean_inc(x_851); -lean_dec(x_826); -x_853 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_853, 0, x_851); -lean_ctor_set(x_853, 1, x_852); -return x_853; +lean_object* x_937; lean_object* x_938; lean_object* x_939; +x_937 = lean_ctor_get(x_912, 0); +x_938 = lean_ctor_get(x_912, 1); +lean_inc(x_938); +lean_inc(x_937); +lean_dec(x_912); +x_939 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_939, 0, x_937); +lean_ctor_set(x_939, 1, x_938); +return x_939; } } } else { -lean_object* x_854; -lean_dec(x_817); +lean_object* x_940; +lean_dec(x_903); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_854 = lean_ctor_get(x_825, 0); -lean_inc(x_854); -lean_dec(x_825); -x_17 = x_854; -x_18 = x_823; -goto block_24; +x_940 = lean_ctor_get(x_911, 0); +lean_inc(x_940); +lean_dec(x_911); +x_23 = x_940; +x_24 = x_909; +goto block_37; } } } default: { -lean_object* x_862; +lean_object* x_948; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_862 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_862, 0, x_1); -lean_ctor_set(x_862, 1, x_8); -return x_862; +x_948 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_948, 0, x_1); +lean_ctor_set(x_948, 1, x_8); +return x_948; } } -block_16: +block_22: { if (lean_obj_tag(x_1) == 10) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_expr_update_mdata(x_1, x_9); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -return x_12; +lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; uint8_t x_15; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +x_13 = lean_ptr_addr(x_12); +lean_dec(x_12); +x_14 = lean_ptr_addr(x_9); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_1); +x_16 = l_Lean_Expr_mdata___override(x_11, x_9); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_10); +return x_17; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_18; +lean_dec(x_11); +lean_dec(x_9); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_1); +lean_ctor_set(x_18, 1, x_10); +return x_18; +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_9); lean_dec(x_1); -x_13 = l_Lean_Meta_Closure_collectExprAux___closed__4; -x_14 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_13); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_10); -return x_15; +x_19 = l_Lean_Meta_Closure_collectExprAux___closed__4; +x_20 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_19); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_10); +return x_21; } } -block_24: +block_37: { if (lean_obj_tag(x_1) == 11) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_expr_update_proj(x_1, x_17); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -return x_20; +lean_object* x_25; lean_object* x_26; lean_object* x_27; size_t x_28; size_t x_29; uint8_t x_30; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_1, 1); +lean_inc(x_26); +x_27 = lean_ctor_get(x_1, 2); +lean_inc(x_27); +x_28 = lean_ptr_addr(x_27); +lean_dec(x_27); +x_29 = lean_ptr_addr(x_23); +x_30 = lean_usize_dec_eq(x_28, x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +lean_dec(x_1); +x_31 = l_Lean_Expr_proj___override(x_25, x_26, x_23); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_24); +return x_32; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -lean_dec(x_17); +lean_object* x_33; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_1); +lean_ctor_set(x_33, 1, x_24); +return x_33; +} +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_23); lean_dec(x_1); -x_21 = l_Lean_Meta_Closure_collectExprAux___closed__7; -x_22 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_21); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_18); -return x_23; +x_34 = l_Lean_Meta_Closure_collectExprAux___closed__7; +x_35 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_34); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_24); +return x_36; } } } @@ -9888,7 +10354,7 @@ static lean_object* _init_l_Nat_foldRev_loop___at_Lean_Meta_Closure_mkBinding___ 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_Nat_foldRev_loop___at_Lean_Meta_Closure_mkBinding___spec__2___closed__1; x_2 = l_Nat_foldRev_loop___at_Lean_Meta_Closure_mkBinding___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_foldRev_loop___at_Lean_Meta_Closure_mkBinding___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/CongrTheorems.c b/stage0/stdlib/Lean/Meta/CongrTheorems.c index 31d238136eb5..3bb2db6f044a 100644 --- a/stage0/stdlib/Lean/Meta/CongrTheorems.c +++ b/stage0/stdlib/Lean/Meta/CongrTheorems.c @@ -585,7 +585,7 @@ static lean_object* _init_l_Lean_Meta_mkHCongrWithArity_withNewEqs_loop___rarg__ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_mkHCongrWithArity_withNewEqs_loop___rarg___closed__3; x_2 = l_Lean_Meta_mkHCongrWithArity_withNewEqs_loop___rarg___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_mkHCongrWithArity_withNewEqs_loop___rarg___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/DecLevel.c b/stage0/stdlib/Lean/Meta/DecLevel.c index 96b84c1fd51a..1eee220fe078 100644 --- a/stage0/stdlib/Lean/Meta/DecLevel.c +++ b/stage0/stdlib/Lean/Meta/DecLevel.c @@ -37,7 +37,7 @@ static lean_object* l_Lean_addTrace___at___private_Lean_Meta_DecLevel_0__Lean_Me lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l_Lean_addTrace___at___private_Lean_Meta_DecLevel_0__Lean_Meta_decAux_x3f___spec__2___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Meta_DecLevel_0__Lean_Meta_decAux_x3f___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_level_mk_max_simp(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Meta_DecLevel_0__Lean_Meta_decAux_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Meta_DecLevel_0__Lean_Meta_decAux_x3f___spec__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_decLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1045,7 +1045,7 @@ if (x_34 == 0) { lean_object* x_35; lean_object* x_36; x_35 = lean_ctor_get(x_25, 0); -x_36 = lean_level_mk_max_simp(x_23, x_35); +x_36 = l_Lean_mkLevelMax_x27(x_23, x_35); lean_ctor_set(x_25, 0, x_36); return x_24; } @@ -1055,7 +1055,7 @@ lean_object* x_37; lean_object* x_38; lean_object* x_39; x_37 = lean_ctor_get(x_25, 0); lean_inc(x_37); lean_dec(x_25); -x_38 = lean_level_mk_max_simp(x_23, x_37); +x_38 = l_Lean_mkLevelMax_x27(x_23, x_37); x_39 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_39, 0, x_38); lean_ctor_set(x_24, 0, x_39); @@ -1077,7 +1077,7 @@ if (lean_is_exclusive(x_25)) { lean_dec_ref(x_25); x_42 = lean_box(0); } -x_43 = lean_level_mk_max_simp(x_23, x_41); +x_43 = l_Lean_mkLevelMax_x27(x_23, x_41); if (lean_is_scalar(x_42)) { x_44 = lean_alloc_ctor(1, 1, 0); } else { @@ -1250,7 +1250,7 @@ if (x_77 == 0) { lean_object* x_78; lean_object* x_79; x_78 = lean_ctor_get(x_68, 0); -x_79 = lean_level_mk_max_simp(x_66, x_78); +x_79 = l_Lean_mkLevelMax_x27(x_66, x_78); lean_ctor_set(x_68, 0, x_79); return x_67; } @@ -1260,7 +1260,7 @@ lean_object* x_80; lean_object* x_81; lean_object* x_82; x_80 = lean_ctor_get(x_68, 0); lean_inc(x_80); lean_dec(x_68); -x_81 = lean_level_mk_max_simp(x_66, x_80); +x_81 = l_Lean_mkLevelMax_x27(x_66, x_80); x_82 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_82, 0, x_81); lean_ctor_set(x_67, 0, x_82); @@ -1282,7 +1282,7 @@ if (lean_is_exclusive(x_68)) { lean_dec_ref(x_68); x_85 = lean_box(0); } -x_86 = lean_level_mk_max_simp(x_66, x_84); +x_86 = l_Lean_mkLevelMax_x27(x_66, x_84); if (lean_is_scalar(x_85)) { x_87 = lean_alloc_ctor(1, 1, 0); } else { diff --git a/stage0/stdlib/Lean/Meta/DiscrTree.c b/stage0/stdlib/Lean/Meta/DiscrTree.c index a0d24843f640..6fcca28c2e00 100644 --- a/stage0/stdlib/Lean/Meta/DiscrTree.c +++ b/stage0/stdlib/Lean/Meta/DiscrTree.c @@ -230,6 +230,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_ LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_getMatchRoot___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_getStarResult___spec__2___rarg(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_Key_arity(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_instToFormatTrie(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_Meta_DiscrTree_getUnify___spec__21___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -354,7 +355,6 @@ LEAN_EXPORT lean_object* l_Array_binSearchAux___at___private_Lean_Meta_DiscrTree static lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_getKeyArgs___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_getStarResult___rarg(lean_object*); extern lean_object* l_Lean_Meta_DiscrTree_instInhabitedKey; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_getUnifyKeyArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_Meta_DiscrTree_getUnify___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_DiscrTree_getUnify_process___spec__7(lean_object*); @@ -2348,7 +2348,7 @@ else { lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; x_33 = lean_unsigned_to_nat(0u); -x_34 = l_Lean_Expr_getAppNumArgsAux(x_1, x_33); +x_34 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_33); x_35 = lean_unsigned_to_nat(1u); x_36 = lean_nat_dec_eq(x_34, x_35); lean_dec(x_34); @@ -2392,7 +2392,7 @@ else { lean_object* x_13; lean_object* x_14; uint8_t x_15; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); lean_dec(x_1); x_15 = lean_nat_dec_eq(x_14, x_13); lean_dec(x_14); @@ -2403,7 +2403,7 @@ else { lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_1, x_16); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_16); x_18 = lean_unsigned_to_nat(3u); x_19 = lean_nat_dec_eq(x_17, x_18); if (x_19 == 0) @@ -2624,7 +2624,7 @@ else { lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; x_107 = lean_unsigned_to_nat(0u); -x_108 = l_Lean_Expr_getAppNumArgsAux(x_2, x_107); +x_108 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_107); x_109 = lean_unsigned_to_nat(2u); x_110 = lean_nat_dec_eq(x_108, x_109); lean_dec(x_108); @@ -2682,7 +2682,7 @@ else { lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_2, x_16); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_16); lean_dec(x_2); x_18 = lean_unsigned_to_nat(1u); x_19 = lean_nat_dec_eq(x_17, x_18); @@ -2698,7 +2698,7 @@ else { lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_2, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_22); x_24 = lean_unsigned_to_nat(6u); x_25 = lean_nat_dec_eq(x_23, x_24); if (x_25 == 0) @@ -2858,7 +2858,7 @@ else { lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; x_69 = lean_unsigned_to_nat(0u); -x_70 = l_Lean_Expr_getAppNumArgsAux(x_2, x_69); +x_70 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_69); x_71 = lean_unsigned_to_nat(4u); x_72 = lean_nat_dec_eq(x_70, x_71); if (x_72 == 0) @@ -3559,7 +3559,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_ { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_1, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_11); lean_inc(x_12); x_13 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_13, 0, x_2); @@ -3704,7 +3704,7 @@ lean_free_object(x_10); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_12, x_16); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_12, x_16); lean_inc(x_17); x_18 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_18, 0, x_15); @@ -4176,7 +4176,7 @@ lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; x_114 = lean_ctor_get(x_113, 0); lean_inc(x_114); x_115 = lean_unsigned_to_nat(0u); -x_116 = l_Lean_Expr_getAppNumArgsAux(x_111, x_115); +x_116 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_111, x_115); lean_inc(x_116); x_117 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_117, 0, x_114); @@ -8313,7 +8313,7 @@ static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___rarg___closed__4() lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_DiscrTree_insertCore___rarg___closed__1; x_2 = l_Lean_Meta_DiscrTree_insertCore___rarg___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_DiscrTree_insertCore___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -8759,7 +8759,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_ { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Expr_getAppNumArgsAux(x_1, x_9); +x_10 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_9); lean_inc(x_10); x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_2); @@ -8849,7 +8849,7 @@ x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); lean_dec(x_13); x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_11, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_15); lean_inc(x_16); x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_14); @@ -9126,7 +9126,7 @@ x_77 = lean_ctor_get(x_64, 0); lean_inc(x_77); lean_dec(x_64); x_78 = lean_unsigned_to_nat(0u); -x_79 = l_Lean_Expr_getAppNumArgsAux(x_11, x_78); +x_79 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_78); x_80 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_getKeyArgs___closed__3; lean_inc(x_79); x_81 = lean_mk_array(x_79, x_80); @@ -9350,7 +9350,7 @@ x_131 = lean_ctor_get(x_130, 0); lean_inc(x_131); lean_dec(x_130); x_132 = lean_unsigned_to_nat(0u); -x_133 = l_Lean_Expr_getAppNumArgsAux(x_128, x_132); +x_133 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_128, x_132); lean_inc(x_133); x_134 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_134, 0, x_131); @@ -9629,7 +9629,7 @@ x_193 = lean_ctor_get(x_180, 0); lean_inc(x_193); lean_dec(x_180); x_194 = lean_unsigned_to_nat(0u); -x_195 = l_Lean_Expr_getAppNumArgsAux(x_128, x_194); +x_195 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_128, x_194); x_196 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_getKeyArgs___closed__3; lean_inc(x_195); x_197 = lean_mk_array(x_195, x_196); diff --git a/stage0/stdlib/Lean/Meta/ExprDefEq.c b/stage0/stdlib/Lean/Meta/ExprDefEq.c index f6f90902823d..5480faf20e6a 100644 --- a/stage0/stdlib/Lean/Meta/ExprDefEq.c +++ b/stage0/stdlib/Lean/Meta/ExprDefEq.c @@ -22,7 +22,6 @@ static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unstuckMVar___c LEAN_EXPORT lean_object* l_Lean_LocalContext_foldlM___at_Lean_Meta_CheckAssignment_checkMVar___spec__51(lean_object*, lean_object*, lean_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_PersistentArray_anyMAux___at_Lean_Meta_CheckAssignment_checkMVar___spec__47___boxed(lean_object*, lean_object*); lean_object* l_Lean_Meta_getResetPostponed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAuxMVar___boxed(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___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__2; lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); @@ -69,10 +68,10 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Meta_CheckAssignment_checkFVar___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getDelayedMVarAssignment_x3f___at_Lean_Meta_checkAssignment___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isExprDefEqExpensive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_checkAssignmentAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isSynthetic(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_checkAssignment___spec__7(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkCacheKey(lean_object*, lean_object*); static lean_object* l_Lean_Meta_CheckAssignment_check___closed__12; @@ -80,8 +79,8 @@ static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0_ static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__13; LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at_Lean_Meta_CheckAssignment_checkMVar___spec__31(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unfoldBothDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000_(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); @@ -93,7 +92,6 @@ uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1848_(l static lean_object* l_Lean_Meta_isExprDefEqAuxImpl___lambda__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqBindingAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unstuckMVar___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqOnFailure___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignment_process___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__48(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__16(lean_object*, lean_object*, size_t, size_t); @@ -139,8 +137,10 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFV LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processConstApprox___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___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_hasLetDeclsInBetween___closed__1; uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqQuickOther___closed__2; static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__7; +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__2; lean_object* l_Std_PersistentArray_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getStuckMVar_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -161,7 +161,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFV lean_object* l_Lean_Meta_getNumPostponed___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_skipDefEqCache___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__9; extern lean_object* l_Lean_MessageData_nil; static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_assignConst___lambda__2___closed__2; @@ -198,8 +197,10 @@ static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqRight___ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isClass_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_hasLetDeclsInBetween___spec__1___closed__2; +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_Lean_MessageData_ofList(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_hasLetDeclsInBetween___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isTypeCorrect(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_markUsedAssignment___at_Lean_Meta_checkAssignment___spec__5___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_assignConst___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -214,7 +215,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDef LEAN_EXPORT lean_object* l_List_replace___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_collectLetDeclsFrom_visit___spec__6(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignment_process___closed__1; static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__8; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___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_Std_mkHashSetImp___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqProj(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_hasLetDeclsInBetween___closed__2; @@ -230,9 +230,10 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkM static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processConstApprox_go___closed__1; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__32___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignmentFOApprox_loop___lambda__1(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___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processConstApprox_defaultCase___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignment_process___closed__2; -uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(uint8_t, uint8_t); +uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Meta_CheckAssignment_checkApp___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -250,7 +251,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAss LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_checkAssignment___spec__8(lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_isExprMVarAssigned___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_outOfScopeExceptionId; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_withResetUsedAssignment(lean_object*); lean_object* l_Lean_Meta_getPostponed___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -281,6 +281,7 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v lean_object* l_Lean_Meta_mkProjFn(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_is_level_def_eq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__1; size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_checkAssignmentExceptionId; lean_object* l_ReaderT_instMonadLiftReaderT(lean_object*, lean_object*, lean_object*); @@ -326,6 +327,7 @@ uint8_t l_Lean_Option_get___at_Lean_getSanitizeNames___spec__1(lean_object*, lea LEAN_EXPORT lean_object* l_Lean_Meta_isExprDefEqAuxImpl___lambda__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_instantiateMVars___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_collectLetDeclsFrom___spec__1(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___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_hasLetDeclsInBetween___spec__2___boxed(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_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqQuickMVarMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__3; @@ -333,12 +335,13 @@ uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_Meta_isListLevelDefEqAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unfold(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_getCachedResult(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isDefEqBindingDomain(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignment_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__2; lean_object* l_StateRefT_x27_lift(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvar___override(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_CheckAssignment_checkMVar___spec__60(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__2; static lean_object* l_Lean_Meta_isExprDefEqAuxImpl___lambda__2___closed__21; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_addLetDeps___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___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqProj_isDefEqSingleton___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -358,6 +361,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_skipDefEqC lean_object* l_Lean_patternAnnotation_x3f(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqLeft(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isMVarDelayedAssigned___at_Lean_Meta_CheckAssignment_checkApp___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__1; static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqOnFailure___closed__1; lean_object* l_Lean_instantiateMVars___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processConstApprox(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -381,13 +385,16 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_withNestedTracesFin LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_assignConst___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqProj_isDefEqSingleton___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__1; LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at_Lean_Meta_CheckAssignment_checkMVar___spec__38(lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_sameHeadSymbol(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_assignToConstFun___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignment_process___spec__2(lean_object*, lean_object*, size_t, size_t); extern lean_object* l_Lean_instInhabitedProjectionFunctionInfo; uint8_t l_Lean_Expr_hasExprMVar(lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqQuickMVarMVar___spec__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_consumeLet___boxed(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__8(lean_object*, lean_object*, size_t, size_t); @@ -424,6 +431,7 @@ static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unstuckMVar___c static lean_object* l_Lean_Meta_isExprDefEqAuxImpl___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_getCachedResult___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_toCtorIfLit(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_CheckAssignment_checkMVar___spec__58(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at_Lean_Meta_CheckAssignment_checkMVar___spec__47(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__2(lean_object*, lean_object*, size_t, size_t); @@ -442,6 +450,7 @@ static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0_ LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_Meta_CheckAssignment_checkApp___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_Meta_CheckAssignment_checkMVar___spec__43(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__49___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_is_matcher(lean_object*, lean_object*); static lean_object* l_Lean_Meta_CheckAssignment_run___closed__1; extern lean_object* l_Lean_Expr_instHashableExpr; @@ -452,7 +461,6 @@ uint64_t l_Lean_Expr_hash(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_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*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Meta_CheckAssignment_checkMVar___spec__5___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unstuckMVar___closed__3; -static lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__1; LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlMAux___at_Lean_Meta_CheckAssignment_checkMVar___spec__54(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_CheckAssignment_checkMVar___closed__3; lean_object* l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(lean_object*, lean_object*); @@ -479,33 +487,34 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFV lean_object* lean_array_to_list(lean_object*, lean_object*); static lean_object* l_Lean_Meta_isDefEqStringLit___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_expandDelayedAssigned_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_isExprDefEqAuxImpl___lambda__2___closed__4; static lean_object* l_Std_PersistentHashMap_insert___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_cacheResult___spec__1___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_collectLetDeps___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_isExprDefEqAuxImpl___lambda__2___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqProj_isDefEqSingleton(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_addLetDeps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs_processOtherArgs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqBinding___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__3(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___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__10; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignmentFOApproxAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignmentFOApprox_loop___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_findMVarDecl_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_CheckAssignment_instMonadCacheExprCheckAssignmentM___closed__2; extern lean_object* l_Lean_instInhabitedExpr; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_CheckAssignment_checkMVar___spec__60___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_CheckAssignment_checkMVar___closed__5; LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at_Lean_Meta_CheckAssignment_checkMVar___spec__39(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isExprDefEqAuxImpl___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_CheckAssignment_checkMVar___spec__64(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_simpAssignmentArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_modn(size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_checkApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_CheckAssignment_throwOutOfScopeFVar___rarg___closed__2; +static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignmentFOApprox_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqProjInst___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Expr_0__Lean_beqLiteral____x40_Lean_Expr___hyg_31_(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqQuickOther___lambda__2___closed__1; @@ -522,6 +531,7 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_c LEAN_EXPORT lean_object* l_Lean_Meta_whenUndefDo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unfoldReducibeDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_mul(size_t, size_t); +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_checkMaxHeartbeats(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bvar___override(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqLeftRight(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -535,7 +545,7 @@ lean_object* l_Lean_Meta_isExprDefEqAux___boxed(lean_object*, lean_object*, lean static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_CheckAssignment_checkMVar___spec__56___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_skipDefEqCache___closed__1; -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_assignExprMVar___at_Lean_Meta_CheckAssignment_checkMVar___spec__65(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -572,8 +582,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqBin LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processConstApprox_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*); uint8_t l_Lean_Meta_ParamInfo_isExplicit(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqMVarSelf___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_isExprDefEqAuxImpl___lambda__2___closed__11; extern lean_object* l_Lean_Meta_instInhabitedParamInfo; size_t lean_usize_land(size_t, size_t); @@ -611,8 +619,11 @@ lean_object* l_Lean_Expr_fvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_Meta_checkAssignment___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqDelta(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_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1___boxed(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_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__1___closed__1; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__1; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_getCachedResult___spec__2(lean_object*, size_t, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at_Lean_Meta_CheckAssignment_checkMVar___spec__23(lean_object*, lean_object*); @@ -624,11 +635,9 @@ lean_object* l_Lean_LocalDecl_index(lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__26(lean_object*, lean_object*, size_t, size_t); uint8_t l_Lean_MetavarKind_isSyntheticOpaque(uint8_t); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqProjInst(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedTraceElem; lean_object* l___private_Lean_Util_Trace_0__Lean_addNode___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_addAssignmentInfo___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_CheckAssignment_checkFVar___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -666,13 +675,14 @@ lean_object* l_Lean_Name_append(lean_object*, lean_object*); extern lean_object* l_Lean_Meta_instMonadMCtxMetaM; extern lean_object* l_Lean_Core_instMonadCoreM; static lean_object* l_Lean_Meta_isExprDefEqAuxImpl___lambda__2___closed__12; +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unfoldNonProjFnDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAuxMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqApp___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_instantiateForallAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at_Lean_Meta_CheckAssignment_checkMVar___spec__39___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_Meta_CheckAssignment_checkMVar___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs_processOtherArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_CheckAssignmentQuick_check(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_simpAssignmentArg___closed__1; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__49(lean_object*, lean_object*, size_t, size_t); @@ -712,10 +722,12 @@ lean_object* l_Array_ofSubarray___rarg(lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__1; static lean_object* l_Lean_Meta_CheckAssignment_throwCheckAssignmentFailure___rarg___closed__2; lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getStructureCtor(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignmentFOApprox_loop___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instMonadQuotation___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__11; lean_object* l_Lean_Meta_getFunInfoNArgs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MetavarContext_findDecl_x3f(lean_object*, lean_object*); @@ -724,7 +736,6 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_CheckAssignmen LEAN_EXPORT lean_object* l_Lean_Meta_checkAssignment___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__25(lean_object*, lean_object*, size_t, size_t); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unstuckMVar___closed__16; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); @@ -736,9 +747,9 @@ lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMe LEAN_EXPORT lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_Meta_CheckAssignment_checkMVar___spec__53(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at_Lean_Meta_CheckAssignment_checkMVar___spec__46___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_Meta_CheckAssignment_checkMVar___spec__4(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_ExprDefEq___hyg_15529_(lean_object*); +static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_ExprDefEq___hyg_16302_(lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Meta_CheckAssignment_throwCheckAssignmentFailure___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_unstuckMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqQuickOther___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -776,10 +787,12 @@ lean_object* l_Lean_Meta_getTransparency(lean_object*, lean_object*, lean_object uint8_t l_Lean_Expr_isStringLit(lean_object*); static lean_object* l_Lean_Meta_CheckAssignment_check___closed__4; lean_object* lean_array_pop(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_Meta_CheckAssignment_checkMVar___spec__12___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_mkAppRangeAux(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_addLetDeps___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqLeft___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignmentQuick_check_visit___spec__2(lean_object*, lean_object*, size_t, size_t); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); @@ -793,7 +806,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_c LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_consumeLet(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_Meta_CheckAssignment_checkMVar___spec__28(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqLeft___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignmentFOApproxAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_HashSetImp_contains___at___private_Lean_MetavarContext_0__Lean_DependsOn_shouldVisit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isAssignable___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -802,22 +814,23 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_c static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__1; lean_object* l_Lean_Meta_shouldReduceReducibleOnly(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_Meta_CheckAssignment_checkMVar___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDeltaCandidate_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__10; lean_object* l_ReaderT_instMonadReaderT___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_isMVarDelayedAssigned___at_Lean_Meta_CheckAssignment_checkApp___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_reduceNative_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqQuickOther___lambda__2(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__1; lean_object* l_Lean_Meta_whnfD(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_expandDelayedAssigned_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_CheckAssignment_checkMVar___spec__55___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_getCachedResult___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_Meta_CheckAssignment_checkMVar___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addTrace___at_Lean_Meta_CheckAssignment_checkFVar___spec__2___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processConstApprox_go_cont(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_cacheResult___spec__2(lean_object*, size_t, size_t, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__42___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isDefEqNat(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -842,6 +855,7 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v static lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqLeftRight___closed__2; LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Meta_CheckAssignment_checkMVar___spec__45(lean_object*, lean_object*, lean_object*); lean_object* lean_local_ctx_find(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashSet___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_collectLetDeps___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_foldlM___at_Lean_Meta_CheckAssignment_checkMVar___spec__52___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_Meta_checkAssignment___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -886,7 +900,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqMVa lean_object* l_Std_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_collectLetDeps___spec__2(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isSynthetic___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__7___rarg(lean_object*, lean_object*); @@ -910,7 +923,6 @@ lean_object* l_Std_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_o LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_Meta_CheckAssignment_checkMVar___spec__44(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_CheckAssignment_checkMVar___spec__34___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_LocalDecl_isLet(lean_object*); -static lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isAssigned(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_Meta_checkAssignment___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); @@ -1074,7 +1086,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDe lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__10; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__11; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__12; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2212,7 +2224,7 @@ lean_inc(x_11); x_12 = lean_nat_add(x_10, x_11); lean_dec(x_11); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_2, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_13); x_15 = lean_nat_dec_eq(x_12, x_14); lean_dec(x_12); if (x_15 == 0) @@ -4826,426 +4838,6 @@ lean_dec(x_2); return x_7; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass_loop(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; uint8_t x_12; -x_11 = lean_array_get_size(x_1); -x_12 = lean_nat_dec_lt(x_4, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_5); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_10); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; uint8_t x_19; uint8_t x_20; lean_object* x_21; -x_15 = lean_array_fget(x_1, x_4); -x_16 = lean_array_get_size(x_2); -x_17 = lean_nat_dec_lt(x_4, x_16); -lean_dec(x_16); -x_18 = lean_array_get_size(x_3); -x_19 = lean_nat_dec_lt(x_4, x_18); -lean_dec(x_18); -x_20 = l_Lean_Meta_ParamInfo_isExplicit(x_15); -lean_dec(x_15); -if (x_17 == 0) -{ -lean_object* x_87; lean_object* x_88; -x_87 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; -x_88 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_87); -x_21 = x_88; -goto block_86; -} -else -{ -lean_object* x_89; -x_89 = lean_array_fget(x_2, x_4); -x_21 = x_89; -goto block_86; -} -block_86: -{ -lean_object* x_22; -if (x_19 == 0) -{ -lean_object* x_83; lean_object* x_84; -x_83 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; -x_84 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_83); -x_22 = x_84; -goto block_82; -} -else -{ -lean_object* x_85; -x_85 = lean_array_fget(x_3, x_4); -x_22 = x_85; -goto block_82; -} -block_82: -{ -if (x_20 == 0) -{ -uint8_t x_23; lean_object* x_24; lean_object* x_47; -lean_inc(x_21); -x_47 = l_Lean_Meta_isEtaUnassignedMVar(x_21, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_47) == 0) -{ -lean_object* x_48; uint8_t x_49; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_unbox(x_48); -if (x_49 == 0) -{ -lean_object* x_50; lean_object* x_51; -lean_dec(x_48); -x_50 = lean_ctor_get(x_47, 1); -lean_inc(x_50); -lean_dec(x_47); -lean_inc(x_22); -x_51 = l_Lean_Meta_isEtaUnassignedMVar(x_22, x_6, x_7, x_8, x_9, x_50); -if (lean_obj_tag(x_51) == 0) -{ -lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -x_54 = lean_unbox(x_52); -lean_dec(x_52); -x_23 = x_54; -x_24 = x_53; -goto block_46; -} -else -{ -uint8_t x_55; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_55 = !lean_is_exclusive(x_51); -if (x_55 == 0) -{ -return x_51; -} -else -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_51, 0); -x_57 = lean_ctor_get(x_51, 1); -lean_inc(x_57); -lean_inc(x_56); -lean_dec(x_51); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -return x_58; -} -} -} -else -{ -lean_object* x_59; uint8_t x_60; -x_59 = lean_ctor_get(x_47, 1); -lean_inc(x_59); -lean_dec(x_47); -x_60 = lean_unbox(x_48); -lean_dec(x_48); -x_23 = x_60; -x_24 = x_59; -goto block_46; -} -} -else -{ -uint8_t x_61; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_61 = !lean_is_exclusive(x_47); -if (x_61 == 0) -{ -return x_47; -} -else -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_47, 0); -x_63 = lean_ctor_get(x_47, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_47); -x_64 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set(x_64, 1, x_63); -return x_64; -} -} -block_46: -{ -if (x_23 == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -lean_dec(x_22); -lean_dec(x_21); -x_25 = lean_unsigned_to_nat(1u); -x_26 = lean_nat_add(x_4, x_25); -x_27 = lean_array_push(x_5, x_4); -x_4 = x_26; -x_5 = x_27; -x_10 = x_24; -goto _start; -} -else -{ -lean_object* x_29; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_29 = lean_is_expr_def_eq(x_21, x_22, x_6, x_7, x_8, x_9, x_24); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; uint8_t x_31; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_unbox(x_30); -lean_dec(x_30); -if (x_31 == 0) -{ -uint8_t x_32; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_32 = !lean_is_exclusive(x_29); -if (x_32 == 0) -{ -lean_object* x_33; lean_object* x_34; -x_33 = lean_ctor_get(x_29, 0); -lean_dec(x_33); -x_34 = lean_box(0); -lean_ctor_set(x_29, 0, x_34); -return x_29; -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_29, 1); -lean_inc(x_35); -lean_dec(x_29); -x_36 = lean_box(0); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_35); -return x_37; -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_29, 1); -lean_inc(x_38); -lean_dec(x_29); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_nat_add(x_4, x_39); -lean_dec(x_4); -x_4 = x_40; -x_10 = x_38; -goto _start; -} -} -else -{ -uint8_t x_42; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_42 = !lean_is_exclusive(x_29); -if (x_42 == 0) -{ -return x_29; -} -else -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_29, 0); -x_44 = lean_ctor_get(x_29, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_29); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -return x_45; -} -} -} -} -} -else -{ -lean_object* x_65; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_65 = lean_is_expr_def_eq(x_21, x_22, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_65) == 0) -{ -lean_object* x_66; uint8_t x_67; -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_unbox(x_66); -lean_dec(x_66); -if (x_67 == 0) -{ -uint8_t x_68; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_68 = !lean_is_exclusive(x_65); -if (x_68 == 0) -{ -lean_object* x_69; lean_object* x_70; -x_69 = lean_ctor_get(x_65, 0); -lean_dec(x_69); -x_70 = lean_box(0); -lean_ctor_set(x_65, 0, x_70); -return x_65; -} -else -{ -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_65, 1); -lean_inc(x_71); -lean_dec(x_65); -x_72 = lean_box(0); -x_73 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_73, 0, x_72); -lean_ctor_set(x_73, 1, x_71); -return x_73; -} -} -else -{ -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_65, 1); -lean_inc(x_74); -lean_dec(x_65); -x_75 = lean_unsigned_to_nat(1u); -x_76 = lean_nat_add(x_4, x_75); -lean_dec(x_4); -x_4 = x_76; -x_10 = x_74; -goto _start; -} -} -else -{ -uint8_t x_78; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_78 = !lean_is_exclusive(x_65); -if (x_78 == 0) -{ -return x_65; -} -else -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_65, 0); -x_80 = lean_ctor_get(x_65, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_65); -x_81 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_81, 0, x_79); -lean_ctor_set(x_81, 1, x_80); -return x_81; -} -} -} -} -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass_loop___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass_loop(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_11; -} -} -static lean_object* _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(0u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_unsigned_to_nat(0u); -x_10 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__1; -x_11 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass_loop(x_1, x_2, x_3, x_9, x_10, x_4, x_5, x_6, x_7, x_8); -return x_11; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_9; -} -} LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(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: { @@ -5333,1738 +4925,3913 @@ return x_23; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs_processOtherArgs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__1(lean_object* x_1) { _start: { -lean_object* x_10; uint8_t x_11; -x_10 = lean_array_get_size(x_1); -x_11 = lean_nat_dec_lt(x_4, x_10); -lean_dec(x_10); -if (x_11 == 0) +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Meta_instInhabitedParamInfo; +x_3 = lean_panic_fn(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -uint8_t x_12; lean_object* x_13; lean_object* x_14; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_12 = 1; -x_13 = lean_box(x_12); -x_14 = lean_alloc_ctor(0, 2, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_array_push(x_4, x_1); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_2); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_3); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_9); -return x_14; +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_10); +return x_15; } -else +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__1() { +_start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_array_fget(x_1, x_4); -x_16 = lean_array_fget(x_2, x_4); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_17 = lean_is_expr_def_eq(x_15, x_16, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_17) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__2() { +_start: { -lean_object* x_18; uint8_t x_19; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_unbox(x_18); -lean_dec(x_18); -if (x_19 == 0) +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("found messy ", 12); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__3() { +_start: { -uint8_t x_20; -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_1; lean_object* x_2; +x_1 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +uint8_t x_16; +x_16 = lean_nat_dec_le(x_8, x_7); +if (x_16 == 0) +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_unsigned_to_nat(0u); +x_18 = lean_nat_dec_eq(x_6, x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_sub(x_6, x_19); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_20 = !lean_is_exclusive(x_17); -if (x_20 == 0) +x_29 = lean_ctor_get(x_10, 1); +lean_inc(x_29); +lean_dec(x_10); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + x_32 = x_29; +} else { + lean_dec_ref(x_29); + x_32 = lean_box(0); +} +x_33 = lean_nat_dec_lt(x_7, x_4); +x_34 = lean_array_get_size(x_2); +x_35 = lean_nat_dec_lt(x_7, x_34); +lean_dec(x_34); +x_36 = lean_array_get_size(x_3); +x_37 = lean_nat_dec_lt(x_7, x_36); +lean_dec(x_36); +if (x_33 == 0) { -lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_17, 0); -lean_dec(x_21); -x_22 = 0; -x_23 = lean_box(x_22); -lean_ctor_set(x_17, 0, x_23); -return x_17; +lean_object* x_184; lean_object* x_185; +x_184 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_185 = l_panic___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__1(x_184); +x_38 = x_185; +goto block_183; } else { -lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_17, 1); -lean_inc(x_24); -lean_dec(x_17); -x_25 = 0; -x_26 = lean_box(x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; +lean_object* x_186; +x_186 = lean_array_fget(x_1, x_7); +x_38 = x_186; +goto block_183; } +block_28: +{ +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_7); +lean_dec(x_5); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_17, 1); -lean_inc(x_28); -lean_dec(x_17); -x_29 = lean_unsigned_to_nat(1u); -x_30 = lean_nat_add(x_4, x_29); -lean_dec(x_4); -x_3 = lean_box(0); -x_4 = x_30; -x_9 = x_28; +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = lean_nat_add(x_7, x_9); +lean_dec(x_7); +x_6 = x_20; +x_7 = x_26; +x_10 = x_25; +x_15 = x_22; goto _start; } } -else +block_183: { -uint8_t x_32; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_32 = !lean_is_exclusive(x_17); -if (x_32 == 0) +uint8_t x_39; lean_object* x_40; +x_39 = lean_ctor_get_uint8(x_38, sizeof(void*)*1 + 5); +if (x_35 == 0) { -return x_17; +lean_object* x_180; lean_object* x_181; +x_180 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_181 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_180); +x_40 = x_181; +goto block_179; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_17, 0); -x_34 = lean_ctor_get(x_17, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_17); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; -} -} -} -} +lean_object* x_182; +x_182 = lean_array_fget(x_2, x_7); +x_40 = x_182; +goto block_179; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs_processOtherArgs___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +block_179: { -lean_object* x_10; -x_10 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs_processOtherArgs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_2); -lean_dec(x_1); -return x_10; -} -} -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1(lean_object* x_1) { -_start: +lean_object* x_41; +if (x_37 == 0) { -lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Meta_instInhabitedParamInfo; -x_3 = lean_panic_fn(x_2, x_1); -return x_3; +lean_object* x_176; lean_object* x_177; +x_176 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_177 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_176); +x_41 = x_177; +goto block_175; } +else +{ +lean_object* x_178; +x_178 = lean_array_fget(x_3, x_7); +x_41 = x_178; +goto block_175; } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +block_175: { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_4); -if (x_9 == 0) +uint8_t x_42; lean_object* x_43; +if (x_39 == 0) { -lean_object* x_10; uint8_t x_11; -x_10 = lean_ctor_get(x_4, 0); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +uint8_t x_65; +x_65 = lean_ctor_get_uint8(x_38, sizeof(void*)*1 + 4); +if (x_65 == 0) { -uint8_t x_12; uint8_t x_13; uint8_t x_14; -x_12 = lean_ctor_get_uint8(x_10, 5); -x_13 = 1; -x_14 = l_Lean_Meta_TransparencyMode_lt(x_12, x_13); -if (x_14 == 0) +uint8_t x_66; +x_66 = l_Lean_Meta_ParamInfo_isExplicit(x_38); +lean_dec(x_38); +if (x_66 == 0) { -lean_object* x_15; -x_15 = lean_is_expr_def_eq(x_1, x_2, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_15) == 0) +lean_object* x_67; +lean_inc(x_40); +x_67 = l_Lean_Meta_isEtaUnassignedMVar(x_40, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_67) == 0) { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +lean_object* x_68; uint8_t x_69; +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_unbox(x_68); +if (x_69 == 0) { -return x_15; -} -else +lean_object* x_70; lean_object* x_71; +lean_dec(x_68); +x_70 = lean_ctor_get(x_67, 1); +lean_inc(x_70); +lean_dec(x_67); +lean_inc(x_41); +x_71 = l_Lean_Meta_isEtaUnassignedMVar(x_41, x_11, x_12, x_13, x_14, x_70); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_15); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} +lean_object* x_72; lean_object* x_73; uint8_t x_74; +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = lean_unbox(x_72); +lean_dec(x_72); +x_42 = x_74; +x_43 = x_73; +goto block_64; } else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) +uint8_t x_75; +lean_dec(x_41); +lean_dec(x_40); +lean_dec(x_32); +lean_dec(x_31); +lean_dec(x_30); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_7); +lean_dec(x_5); +x_75 = !lean_is_exclusive(x_71); +if (x_75 == 0) { -return x_15; +return x_71; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_15, 0); -x_22 = lean_ctor_get(x_15, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_15); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; -} +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_71, 0); +x_77 = lean_ctor_get(x_71, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_71); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; } } -else -{ -lean_object* x_24; -lean_ctor_set_uint8(x_10, 5, x_13); -x_24 = lean_is_expr_def_eq(x_1, x_2, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_24) == 0) -{ -uint8_t x_25; -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) -{ -return x_24; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_24, 0); -x_27 = lean_ctor_get(x_24, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_24); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; +lean_object* x_79; uint8_t x_80; +x_79 = lean_ctor_get(x_67, 1); +lean_inc(x_79); +lean_dec(x_67); +x_80 = lean_unbox(x_68); +lean_dec(x_68); +x_42 = x_80; +x_43 = x_79; +goto block_64; } } else { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_24); -if (x_29 == 0) +uint8_t x_81; +lean_dec(x_41); +lean_dec(x_40); +lean_dec(x_32); +lean_dec(x_31); +lean_dec(x_30); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_7); +lean_dec(x_5); +x_81 = !lean_is_exclusive(x_67); +if (x_81 == 0) { -return x_24; +return x_67; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_24, 0); -x_31 = lean_ctor_get(x_24, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_24); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; -} +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_67, 0); +x_83 = lean_ctor_get(x_67, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_67); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; } } } else { -uint8_t x_33; uint8_t x_34; uint8_t x_35; uint8_t x_36; uint8_t x_37; uint8_t x_38; uint8_t x_39; 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; -x_33 = lean_ctor_get_uint8(x_10, 0); -x_34 = lean_ctor_get_uint8(x_10, 1); -x_35 = lean_ctor_get_uint8(x_10, 2); -x_36 = lean_ctor_get_uint8(x_10, 3); -x_37 = lean_ctor_get_uint8(x_10, 4); -x_38 = lean_ctor_get_uint8(x_10, 5); -x_39 = lean_ctor_get_uint8(x_10, 6); -x_40 = lean_ctor_get_uint8(x_10, 7); -x_41 = lean_ctor_get_uint8(x_10, 8); -x_42 = lean_ctor_get_uint8(x_10, 9); -x_43 = lean_ctor_get_uint8(x_10, 10); -x_44 = lean_ctor_get_uint8(x_10, 11); -x_45 = lean_ctor_get_uint8(x_10, 12); -x_46 = lean_ctor_get_uint8(x_10, 13); -lean_dec(x_10); -x_47 = 1; -x_48 = l_Lean_Meta_TransparencyMode_lt(x_38, x_47); -if (x_48 == 0) +lean_object* x_85; +lean_dec(x_32); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_85 = lean_is_expr_def_eq(x_40, x_41, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_85) == 0) { -lean_object* x_49; lean_object* x_50; -x_49 = lean_alloc_ctor(0, 0, 14); -lean_ctor_set_uint8(x_49, 0, x_33); -lean_ctor_set_uint8(x_49, 1, x_34); -lean_ctor_set_uint8(x_49, 2, x_35); -lean_ctor_set_uint8(x_49, 3, x_36); -lean_ctor_set_uint8(x_49, 4, x_37); -lean_ctor_set_uint8(x_49, 5, x_38); -lean_ctor_set_uint8(x_49, 6, x_39); -lean_ctor_set_uint8(x_49, 7, x_40); -lean_ctor_set_uint8(x_49, 8, x_41); -lean_ctor_set_uint8(x_49, 9, x_42); -lean_ctor_set_uint8(x_49, 10, x_43); -lean_ctor_set_uint8(x_49, 11, x_44); -lean_ctor_set_uint8(x_49, 12, x_45); -lean_ctor_set_uint8(x_49, 13, x_46); -lean_ctor_set(x_4, 0, x_49); -x_50 = lean_is_expr_def_eq(x_1, x_2, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_50) == 0) +lean_object* x_86; uint8_t x_87; +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +x_87 = lean_unbox(x_86); +lean_dec(x_86); +if (x_87 == 0) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_50)) { - lean_ctor_release(x_50, 0); - lean_ctor_release(x_50, 1); - x_53 = x_50; -} else { - lean_dec_ref(x_50); - x_53 = lean_box(0); -} -if (lean_is_scalar(x_53)) { - x_54 = lean_alloc_ctor(0, 2, 0); -} else { - x_54 = x_53; -} -lean_ctor_set(x_54, 0, x_51); -lean_ctor_set(x_54, 1, x_52); -return x_54; +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_88 = lean_ctor_get(x_85, 1); +lean_inc(x_88); +lean_dec(x_85); +x_89 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_89, 0, x_30); +lean_ctor_set(x_89, 1, x_31); +x_90 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__1; +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_89); +x_92 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_92, 0, x_91); +x_21 = x_92; +x_22 = x_88; +goto block_28; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_55 = lean_ctor_get(x_50, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_50, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_50)) { - lean_ctor_release(x_50, 0); - lean_ctor_release(x_50, 1); - x_57 = x_50; -} else { - lean_dec_ref(x_50); - x_57 = lean_box(0); -} -if (lean_is_scalar(x_57)) { - x_58 = lean_alloc_ctor(1, 2, 0); -} else { - x_58 = x_57; -} -lean_ctor_set(x_58, 0, x_55); -lean_ctor_set(x_58, 1, x_56); -return x_58; +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_93 = lean_ctor_get(x_85, 1); +lean_inc(x_93); +lean_dec(x_85); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_30); +lean_ctor_set(x_94, 1, x_31); +lean_inc(x_5); +x_95 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_95, 0, x_5); +lean_ctor_set(x_95, 1, x_94); +x_96 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_96, 0, x_95); +x_21 = x_96; +x_22 = x_93; +goto block_28; } } else { -lean_object* x_59; lean_object* x_60; -x_59 = lean_alloc_ctor(0, 0, 14); -lean_ctor_set_uint8(x_59, 0, x_33); -lean_ctor_set_uint8(x_59, 1, x_34); -lean_ctor_set_uint8(x_59, 2, x_35); -lean_ctor_set_uint8(x_59, 3, x_36); -lean_ctor_set_uint8(x_59, 4, x_37); -lean_ctor_set_uint8(x_59, 5, x_47); -lean_ctor_set_uint8(x_59, 6, x_39); -lean_ctor_set_uint8(x_59, 7, x_40); -lean_ctor_set_uint8(x_59, 8, x_41); -lean_ctor_set_uint8(x_59, 9, x_42); -lean_ctor_set_uint8(x_59, 10, x_43); -lean_ctor_set_uint8(x_59, 11, x_44); -lean_ctor_set_uint8(x_59, 12, x_45); -lean_ctor_set_uint8(x_59, 13, x_46); -lean_ctor_set(x_4, 0, x_59); -x_60 = lean_is_expr_def_eq(x_1, x_2, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_60) == 0) +uint8_t x_97; +lean_dec(x_31); +lean_dec(x_30); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_7); +lean_dec(x_5); +x_97 = !lean_is_exclusive(x_85); +if (x_97 == 0) { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_60, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_63 = x_60; -} else { - lean_dec_ref(x_60); - x_63 = lean_box(0); -} -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(0, 2, 0); -} else { - x_64 = x_63; -} -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; +return x_85; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_65 = lean_ctor_get(x_60, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_60, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_67 = x_60; -} else { - lean_dec_ref(x_60); - x_67 = lean_box(0); -} -if (lean_is_scalar(x_67)) { - x_68 = lean_alloc_ctor(1, 2, 0); -} else { - x_68 = x_67; -} -lean_ctor_set(x_68, 0, x_65); -lean_ctor_set(x_68, 1, x_66); -return x_68; +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_85, 0); +x_99 = lean_ctor_get(x_85, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_85); +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_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; uint8_t x_75; uint8_t x_76; uint8_t x_77; uint8_t x_78; uint8_t x_79; uint8_t x_80; uint8_t x_81; uint8_t x_82; uint8_t x_83; uint8_t x_84; uint8_t x_85; uint8_t x_86; uint8_t x_87; uint8_t x_88; lean_object* x_89; uint8_t x_90; uint8_t x_91; -x_69 = lean_ctor_get(x_4, 0); -x_70 = lean_ctor_get(x_4, 1); -x_71 = lean_ctor_get(x_4, 2); -x_72 = lean_ctor_get(x_4, 3); -x_73 = lean_ctor_get(x_4, 4); -x_74 = lean_ctor_get(x_4, 5); -lean_inc(x_74); -lean_inc(x_73); -lean_inc(x_72); -lean_inc(x_71); -lean_inc(x_70); -lean_inc(x_69); -lean_dec(x_4); -x_75 = lean_ctor_get_uint8(x_69, 0); -x_76 = lean_ctor_get_uint8(x_69, 1); -x_77 = lean_ctor_get_uint8(x_69, 2); -x_78 = lean_ctor_get_uint8(x_69, 3); -x_79 = lean_ctor_get_uint8(x_69, 4); -x_80 = lean_ctor_get_uint8(x_69, 5); -x_81 = lean_ctor_get_uint8(x_69, 6); -x_82 = lean_ctor_get_uint8(x_69, 7); -x_83 = lean_ctor_get_uint8(x_69, 8); -x_84 = lean_ctor_get_uint8(x_69, 9); -x_85 = lean_ctor_get_uint8(x_69, 10); -x_86 = lean_ctor_get_uint8(x_69, 11); -x_87 = lean_ctor_get_uint8(x_69, 12); -x_88 = lean_ctor_get_uint8(x_69, 13); -if (lean_is_exclusive(x_69)) { - x_89 = x_69; -} else { - lean_dec_ref(x_69); - x_89 = lean_box(0); -} -x_90 = 1; -x_91 = l_Lean_Meta_TransparencyMode_lt(x_80, x_90); -if (x_91 == 0) +lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_127; +lean_dec(x_38); +lean_dec(x_32); +x_101 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__4; +x_124 = lean_st_ref_get(x_14, x_15); +x_125 = lean_ctor_get(x_124, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_125, 3); +lean_inc(x_126); +lean_dec(x_125); +x_127 = lean_ctor_get_uint8(x_126, sizeof(void*)*1); +lean_dec(x_126); +if (x_127 == 0) { -lean_object* x_92; lean_object* x_93; lean_object* x_94; -if (lean_is_scalar(x_89)) { - x_92 = lean_alloc_ctor(0, 0, 14); -} else { - x_92 = x_89; -} -lean_ctor_set_uint8(x_92, 0, x_75); -lean_ctor_set_uint8(x_92, 1, x_76); -lean_ctor_set_uint8(x_92, 2, x_77); -lean_ctor_set_uint8(x_92, 3, x_78); -lean_ctor_set_uint8(x_92, 4, x_79); -lean_ctor_set_uint8(x_92, 5, x_80); -lean_ctor_set_uint8(x_92, 6, x_81); -lean_ctor_set_uint8(x_92, 7, x_82); -lean_ctor_set_uint8(x_92, 8, x_83); -lean_ctor_set_uint8(x_92, 9, x_84); -lean_ctor_set_uint8(x_92, 10, x_85); -lean_ctor_set_uint8(x_92, 11, x_86); -lean_ctor_set_uint8(x_92, 12, x_87); -lean_ctor_set_uint8(x_92, 13, x_88); -x_93 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_70); -lean_ctor_set(x_93, 2, x_71); -lean_ctor_set(x_93, 3, x_72); -lean_ctor_set(x_93, 4, x_73); -lean_ctor_set(x_93, 5, x_74); -x_94 = lean_is_expr_def_eq(x_1, x_2, x_93, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_94) == 0) -{ -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_95 = lean_ctor_get(x_94, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_94, 1); -lean_inc(x_96); -if (lean_is_exclusive(x_94)) { - lean_ctor_release(x_94, 0); - lean_ctor_release(x_94, 1); - x_97 = x_94; -} else { - lean_dec_ref(x_94); - x_97 = lean_box(0); -} -if (lean_is_scalar(x_97)) { - x_98 = lean_alloc_ctor(0, 2, 0); -} else { - x_98 = x_97; -} -lean_ctor_set(x_98, 0, x_95); -lean_ctor_set(x_98, 1, x_96); -return x_98; +lean_object* x_128; uint8_t x_129; +x_128 = lean_ctor_get(x_124, 1); +lean_inc(x_128); +lean_dec(x_124); +x_129 = 0; +x_102 = x_129; +x_103 = x_128; +goto block_123; } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_99 = lean_ctor_get(x_94, 0); -lean_inc(x_99); -x_100 = lean_ctor_get(x_94, 1); -lean_inc(x_100); -if (lean_is_exclusive(x_94)) { - lean_ctor_release(x_94, 0); - lean_ctor_release(x_94, 1); - x_101 = x_94; -} else { - lean_dec_ref(x_94); - x_101 = lean_box(0); -} -if (lean_is_scalar(x_101)) { - x_102 = lean_alloc_ctor(1, 2, 0); -} else { - x_102 = x_101; -} -lean_ctor_set(x_102, 0, x_99); -lean_ctor_set(x_102, 1, x_100); -return x_102; -} +lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; uint8_t x_134; +x_130 = lean_ctor_get(x_124, 1); +lean_inc(x_130); +lean_dec(x_124); +x_131 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__14(x_101, x_11, x_12, x_13, x_14, x_130); +x_132 = lean_ctor_get(x_131, 0); +lean_inc(x_132); +x_133 = lean_ctor_get(x_131, 1); +lean_inc(x_133); +lean_dec(x_131); +x_134 = lean_unbox(x_132); +lean_dec(x_132); +x_102 = x_134; +x_103 = x_133; +goto block_123; } -else +block_123: { -lean_object* x_103; lean_object* x_104; lean_object* x_105; -if (lean_is_scalar(x_89)) { - x_103 = lean_alloc_ctor(0, 0, 14); -} else { - x_103 = x_89; -} -lean_ctor_set_uint8(x_103, 0, x_75); -lean_ctor_set_uint8(x_103, 1, x_76); -lean_ctor_set_uint8(x_103, 2, x_77); -lean_ctor_set_uint8(x_103, 3, x_78); -lean_ctor_set_uint8(x_103, 4, x_79); -lean_ctor_set_uint8(x_103, 5, x_90); -lean_ctor_set_uint8(x_103, 6, x_81); -lean_ctor_set_uint8(x_103, 7, x_82); -lean_ctor_set_uint8(x_103, 8, x_83); -lean_ctor_set_uint8(x_103, 9, x_84); -lean_ctor_set_uint8(x_103, 10, x_85); -lean_ctor_set_uint8(x_103, 11, x_86); -lean_ctor_set_uint8(x_103, 12, x_87); -lean_ctor_set_uint8(x_103, 13, x_88); -x_104 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_70); -lean_ctor_set(x_104, 2, x_71); -lean_ctor_set(x_104, 3, x_72); -lean_ctor_set(x_104, 4, x_73); -lean_ctor_set(x_104, 5, x_74); -x_105 = lean_is_expr_def_eq(x_1, x_2, x_104, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_105) == 0) -{ -lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +if (x_102 == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +lean_dec(x_41); +lean_dec(x_40); +x_104 = lean_box(0); +lean_inc(x_5); +lean_inc(x_7); +x_105 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1(x_7, x_31, x_5, x_30, x_104, x_11, x_12, x_13, x_14, x_103); x_106 = lean_ctor_get(x_105, 0); lean_inc(x_106); x_107 = lean_ctor_get(x_105, 1); lean_inc(x_107); -if (lean_is_exclusive(x_105)) { - lean_ctor_release(x_105, 0); - lean_ctor_release(x_105, 1); - x_108 = x_105; -} else { - lean_dec_ref(x_105); - x_108 = lean_box(0); -} -if (lean_is_scalar(x_108)) { - x_109 = lean_alloc_ctor(0, 2, 0); -} else { - x_109 = x_108; -} -lean_ctor_set(x_109, 0, x_106); -lean_ctor_set(x_109, 1, x_107); -return x_109; +lean_dec(x_105); +x_21 = x_106; +x_22 = x_107; +goto block_28; } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_110 = lean_ctor_get(x_105, 0); -lean_inc(x_110); -x_111 = lean_ctor_get(x_105, 1); -lean_inc(x_111); -if (lean_is_exclusive(x_105)) { - lean_ctor_release(x_105, 0); - lean_ctor_release(x_105, 1); - x_112 = x_105; -} else { - lean_dec_ref(x_105); - x_112 = lean_box(0); -} -if (lean_is_scalar(x_112)) { - x_113 = lean_alloc_ctor(1, 2, 0); -} else { - x_113 = x_112; -} -lean_ctor_set(x_113, 0, x_110); -lean_ctor_set(x_113, 1, x_111); -return x_113; -} +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_108 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_108, 0, x_40); +x_109 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__3; +x_110 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_108); +x_111 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__10; +x_112 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_112, 0, x_110); +lean_ctor_set(x_112, 1, x_111); +x_113 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_113, 0, x_41); +x_114 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +x_115 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__9; +x_116 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +x_117 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__1(x_101, x_116, x_11, x_12, x_13, x_14, x_103); +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_117, 1); +lean_inc(x_119); +lean_dec(x_117); +lean_inc(x_5); +lean_inc(x_7); +x_120 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1(x_7, x_31, x_5, x_30, x_118, x_11, x_12, x_13, x_14, x_119); +lean_dec(x_118); +x_121 = lean_ctor_get(x_120, 0); +lean_inc(x_121); +x_122 = lean_ctor_get(x_120, 1); +lean_inc(x_122); +lean_dec(x_120); +x_21 = x_121; +x_22 = x_122; +goto block_28; } } } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -uint8_t x_15; -x_15 = lean_usize_dec_eq(x_8, x_9); -if (x_15 == 0) +else { -lean_object* x_16; uint8_t x_17; lean_object* x_18; uint8_t x_26; uint8_t x_27; uint8_t x_28; lean_object* x_29; -x_16 = lean_array_uget(x_7, x_8); -x_26 = lean_nat_dec_lt(x_16, x_3); -x_27 = lean_nat_dec_lt(x_16, x_4); -x_28 = lean_nat_dec_lt(x_16, x_6); -if (x_26 == 0) +lean_object* x_135; uint8_t x_136; lean_object* x_137; lean_object* x_164; lean_object* x_165; lean_object* x_166; uint8_t x_167; +lean_dec(x_38); +lean_dec(x_32); +x_135 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__4; +x_164 = lean_st_ref_get(x_14, x_15); +x_165 = lean_ctor_get(x_164, 0); +lean_inc(x_165); +x_166 = lean_ctor_get(x_165, 3); +lean_inc(x_166); +lean_dec(x_165); +x_167 = lean_ctor_get_uint8(x_166, sizeof(void*)*1); +lean_dec(x_166); +if (x_167 == 0) { -lean_object* x_113; lean_object* x_114; -x_113 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; -x_114 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_113); -x_29 = x_114; -goto block_112; +lean_object* x_168; uint8_t x_169; +x_168 = lean_ctor_get(x_164, 1); +lean_inc(x_168); +lean_dec(x_164); +x_169 = 0; +x_136 = x_169; +x_137 = x_168; +goto block_163; } else { -lean_object* x_115; -x_115 = lean_array_fget(x_1, x_16); -x_29 = x_115; -goto block_112; +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; +x_170 = lean_ctor_get(x_164, 1); +lean_inc(x_170); +lean_dec(x_164); +x_171 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__14(x_135, x_11, x_12, x_13, x_14, x_170); +x_172 = lean_ctor_get(x_171, 0); +lean_inc(x_172); +x_173 = lean_ctor_get(x_171, 1); +lean_inc(x_173); +lean_dec(x_171); +x_174 = lean_unbox(x_172); +lean_dec(x_172); +x_136 = x_174; +x_137 = x_173; +goto block_163; } -block_25: +block_163: { -if (x_17 == 0) +if (x_136 == 0) { -size_t x_19; size_t x_20; -x_19 = 1; -x_20 = lean_usize_add(x_8, x_19); -x_8 = x_20; -x_14 = x_18; +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_dec(x_41); +lean_dec(x_40); +x_138 = lean_box(0); +lean_inc(x_5); +lean_inc(x_7); +x_139 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1(x_7, x_31, x_5, x_30, x_138, x_11, x_12, x_13, x_14, x_137); +x_140 = lean_ctor_get(x_139, 0); +lean_inc(x_140); +x_141 = lean_ctor_get(x_139, 1); +lean_inc(x_141); +lean_dec(x_139); +x_142 = lean_ctor_get(x_140, 0); +lean_inc(x_142); +lean_dec(x_140); +x_143 = lean_nat_add(x_7, x_9); +lean_dec(x_7); +x_6 = x_20; +x_7 = x_143; +x_10 = x_142; +x_15 = x_141; goto _start; } else { -uint8_t x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -x_22 = 1; -x_23 = lean_box(x_22); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_18); -return x_24; +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; +x_145 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_145, 0, x_40); +x_146 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__3; +x_147 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_145); +x_148 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___closed__10; +x_149 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_149, 0, x_147); +lean_ctor_set(x_149, 1, x_148); +x_150 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_150, 0, x_41); +x_151 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_151, 0, x_149); +lean_ctor_set(x_151, 1, x_150); +x_152 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__9; +x_153 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_153, 0, x_151); +lean_ctor_set(x_153, 1, x_152); +x_154 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__1(x_135, x_153, x_11, x_12, x_13, x_14, x_137); +x_155 = lean_ctor_get(x_154, 0); +lean_inc(x_155); +x_156 = lean_ctor_get(x_154, 1); +lean_inc(x_156); +lean_dec(x_154); +lean_inc(x_5); +lean_inc(x_7); +x_157 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1(x_7, x_31, x_5, x_30, x_155, x_11, x_12, x_13, x_14, x_156); +lean_dec(x_155); +x_158 = lean_ctor_get(x_157, 0); +lean_inc(x_158); +x_159 = lean_ctor_get(x_157, 1); +lean_inc(x_159); +lean_dec(x_157); +x_160 = lean_ctor_get(x_158, 0); +lean_inc(x_160); +lean_dec(x_158); +x_161 = lean_nat_add(x_7, x_9); +lean_dec(x_7); +x_6 = x_20; +x_7 = x_161; +x_10 = x_160; +x_15 = x_159; +goto _start; +} } } -block_112: +block_64: { -lean_object* x_30; -if (x_27 == 0) +if (x_42 == 0) { -lean_object* x_109; lean_object* x_110; -x_109 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; -x_110 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_109); -x_30 = x_110; -goto block_108; +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +lean_dec(x_41); +lean_dec(x_40); +lean_inc(x_7); +x_44 = lean_array_push(x_31, x_7); +if (lean_is_scalar(x_32)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_32; } -else -{ -lean_object* x_111; -x_111 = lean_array_fget(x_2, x_16); -x_30 = x_111; -goto block_108; +lean_ctor_set(x_45, 0, x_30); +lean_ctor_set(x_45, 1, x_44); +lean_inc(x_5); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_5); +lean_ctor_set(x_46, 1, x_45); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_21 = x_47; +x_22 = x_43; +goto block_28; } -block_108: -{ -if (x_28 == 0) -{ -lean_object* x_31; lean_object* x_32; uint8_t x_33; -lean_dec(x_16); -x_31 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; -x_32 = l_panic___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1(x_31); -x_33 = l_Lean_Meta_ParamInfo_isInstImplicit(x_32); -lean_dec(x_32); -if (x_33 == 0) +else { -lean_object* x_34; lean_object* x_35; -x_34 = lean_box(0); +lean_object* x_48; +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); -x_35 = l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_29, x_30, x_34, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_35) == 0) +x_48 = lean_is_expr_def_eq(x_40, x_41, x_11, x_12, x_13, x_14, x_43); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_36; uint8_t x_37; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_unbox(x_36); -lean_dec(x_36); -if (x_37 == 0) +lean_object* x_49; uint8_t x_50; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_unbox(x_49); +lean_dec(x_49); +if (x_50 == 0) { -lean_object* x_38; uint8_t x_39; -x_38 = lean_ctor_get(x_35, 1); -lean_inc(x_38); -lean_dec(x_35); -x_39 = 1; -x_17 = x_39; -x_18 = x_38; -goto block_25; +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_51 = lean_ctor_get(x_48, 1); +lean_inc(x_51); +lean_dec(x_48); +if (lean_is_scalar(x_32)) { + x_52 = lean_alloc_ctor(0, 2, 0); +} else { + x_52 = x_32; +} +lean_ctor_set(x_52, 0, x_30); +lean_ctor_set(x_52, 1, x_31); +x_53 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__1; +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_52); +x_55 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_55, 0, x_54); +x_21 = x_55; +x_22 = x_51; +goto block_28; } else { -lean_object* x_40; uint8_t x_41; -x_40 = lean_ctor_get(x_35, 1); -lean_inc(x_40); -lean_dec(x_35); -x_41 = 0; -x_17 = x_41; -x_18 = x_40; -goto block_25; +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_56 = lean_ctor_get(x_48, 1); +lean_inc(x_56); +lean_dec(x_48); +if (lean_is_scalar(x_32)) { + x_57 = lean_alloc_ctor(0, 2, 0); +} else { + x_57 = x_32; +} +lean_ctor_set(x_57, 0, x_30); +lean_ctor_set(x_57, 1, x_31); +lean_inc(x_5); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_5); +lean_ctor_set(x_58, 1, x_57); +x_59 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_59, 0, x_58); +x_21 = x_59; +x_22 = x_56; +goto block_28; } } else { -uint8_t x_42; +uint8_t x_60; +lean_dec(x_32); +lean_dec(x_31); +lean_dec(x_30); +lean_dec(x_20); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); -x_42 = !lean_is_exclusive(x_35); -if (x_42 == 0) +lean_dec(x_7); +lean_dec(x_5); +x_60 = !lean_is_exclusive(x_48); +if (x_60 == 0) { -return x_35; +return x_48; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_35, 0); -x_44 = lean_ctor_get(x_35, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_35); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -return x_45; +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_48, 0); +x_62 = lean_ctor_get(x_48, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_48); +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +return x_63; +} +} +} +} } } } -else -{ -lean_object* x_46; -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_29); -x_46 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(x_29, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_46) == 0) -{ -lean_object* x_47; lean_object* x_48; -x_47 = lean_ctor_get(x_46, 1); -lean_inc(x_47); -lean_dec(x_46); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_30); -x_48 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(x_30, x_10, x_11, x_12, x_13, x_47); -if (lean_obj_tag(x_48) == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -lean_dec(x_48); -x_50 = lean_box(0); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_51 = l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_29, x_30, x_50, x_10, x_11, x_12, x_13, x_49); -if (lean_obj_tag(x_51) == 0) -{ -lean_object* x_52; uint8_t x_53; -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_unbox(x_52); -lean_dec(x_52); -if (x_53 == 0) -{ -lean_object* x_54; uint8_t x_55; -x_54 = lean_ctor_get(x_51, 1); -lean_inc(x_54); -lean_dec(x_51); -x_55 = 1; -x_17 = x_55; -x_18 = x_54; -goto block_25; } else { -lean_object* x_56; uint8_t x_57; -x_56 = lean_ctor_get(x_51, 1); -lean_inc(x_56); -lean_dec(x_51); -x_57 = 0; -x_17 = x_57; -x_18 = x_56; -goto block_25; +lean_object* x_187; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_187 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_187, 0, x_10); +lean_ctor_set(x_187, 1, x_15); +return x_187; } } else { -uint8_t x_58; +lean_object* x_188; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); -x_58 = !lean_is_exclusive(x_51); -if (x_58 == 0) +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_188 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_188, 0, x_10); +lean_ctor_set(x_188, 1, x_15); +return x_188; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -return x_51; +lean_object* x_9; lean_object* x_10; +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_1); +lean_ctor_set(x_9, 1, x_2); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; } -else +} +static lean_object* _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__1() { +_start: { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_51, 0); -x_60 = lean_ctor_get(x_51, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_51); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -return x_61; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__1; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___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_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } } +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_array_get_size(x_1); +x_10 = lean_box(0); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_unsigned_to_nat(1u); +x_13 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__3; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_9); +x_14 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2(x_1, x_2, x_3, x_9, x_10, x_9, x_11, x_9, x_12, x_13, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_9); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +x_19 = lean_ctor_get(x_16, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_16, 1); +lean_inc(x_20); +lean_dec(x_16); +x_21 = lean_box(0); +x_22 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___lambda__1(x_20, x_19, x_21, x_4, x_5, x_6, x_7, x_18); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_22; } else { -uint8_t x_62; -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -x_62 = !lean_is_exclusive(x_48); -if (x_62 == 0) +uint8_t x_23; +lean_dec(x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_23 = !lean_is_exclusive(x_14); +if (x_23 == 0) { -return x_48; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_14, 0); +lean_dec(x_24); +x_25 = lean_ctor_get(x_17, 0); +lean_inc(x_25); +lean_dec(x_17); +lean_ctor_set(x_14, 0, x_25); +return x_14; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_48, 0); -x_64 = lean_ctor_get(x_48, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_48); -x_65 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -return x_65; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_14, 1); +lean_inc(x_26); +lean_dec(x_14); +x_27 = lean_ctor_get(x_17, 0); +lean_inc(x_27); +lean_dec(x_17); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +return x_28; } } } else { -uint8_t x_66; -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -x_66 = !lean_is_exclusive(x_46); -if (x_66 == 0) +uint8_t x_29; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_29 = !lean_is_exclusive(x_14); +if (x_29 == 0) { -return x_46; +return x_14; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_46, 0); -x_68 = lean_ctor_get(x_46, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_46); -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_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_14, 0); +x_31 = lean_ctor_get(x_14, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_14); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } } } -else +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_70; uint8_t x_71; -x_70 = lean_array_fget(x_5, x_16); -lean_dec(x_16); -x_71 = l_Lean_Meta_ParamInfo_isInstImplicit(x_70); -lean_dec(x_70); -if (x_71 == 0) +lean_object* x_11; +x_11 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: { -lean_object* x_72; lean_object* x_73; -x_72 = lean_box(0); +lean_object* x_16; +x_16 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; +x_15 = lean_nat_dec_le(x_7, x_6); +if (x_15 == 0) +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_eq(x_5, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_28; lean_object* x_29; uint8_t x_30; +lean_dec(x_9); +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_sub(x_5, x_18); +lean_dec(x_5); +x_28 = lean_nat_dec_lt(x_6, x_3); +x_29 = lean_array_get_size(x_2); +x_30 = lean_nat_dec_lt(x_6, x_29); +lean_dec(x_29); +if (x_28 == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_32 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_31); +if (x_30 == 0) +{ +lean_object* x_33; lean_object* x_34; +x_33 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_31); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); -x_73 = l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_29, x_30, x_72, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_73) == 0) +x_34 = lean_is_expr_def_eq(x_32, x_33, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_74; uint8_t x_75; -x_74 = lean_ctor_get(x_73, 0); -lean_inc(x_74); -x_75 = lean_unbox(x_74); -lean_dec(x_74); -if (x_75 == 0) +lean_object* x_35; uint8_t x_36; +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_unbox(x_35); +lean_dec(x_35); +if (x_36 == 0) { -lean_object* x_76; uint8_t x_77; -x_76 = lean_ctor_get(x_73, 1); -lean_inc(x_76); -lean_dec(x_73); -x_77 = 1; -x_17 = x_77; -x_18 = x_76; -goto block_25; +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_34, 1); +lean_inc(x_37); +lean_dec(x_34); +x_38 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__3; +x_20 = x_38; +x_21 = x_37; +goto block_27; } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_73, 1); -lean_inc(x_78); -lean_dec(x_73); -x_79 = 0; -x_17 = x_79; -x_18 = x_78; -goto block_25; +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_34, 1); +lean_inc(x_39); +lean_dec(x_34); +lean_inc(x_4); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_4); +x_20 = x_40; +x_21 = x_39; +goto block_27; } } else { -uint8_t x_80; +uint8_t x_41; +lean_dec(x_19); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_80 = !lean_is_exclusive(x_73); -if (x_80 == 0) +lean_dec(x_6); +lean_dec(x_4); +x_41 = !lean_is_exclusive(x_34); +if (x_41 == 0) { -return x_73; +return x_34; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_73, 0); -x_82 = lean_ctor_get(x_73, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_73); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -return x_83; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_34, 0); +x_43 = lean_ctor_get(x_34, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_34); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } } } else { -lean_object* x_84; -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_29); -x_84 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(x_29, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_84) == 0) -{ -lean_object* x_85; lean_object* x_86; -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_30); -x_86 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(x_30, x_10, x_11, x_12, x_13, x_85); -if (lean_obj_tag(x_86) == 0) -{ -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_86, 1); -lean_inc(x_87); -lean_dec(x_86); -x_88 = lean_box(0); +lean_object* x_45; lean_object* x_46; +x_45 = lean_array_fget(x_2, x_6); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); -x_89 = l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_29, x_30, x_88, x_10, x_11, x_12, x_13, x_87); -if (lean_obj_tag(x_89) == 0) +x_46 = lean_is_expr_def_eq(x_32, x_45, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_46) == 0) { -lean_object* x_90; uint8_t x_91; -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -x_91 = lean_unbox(x_90); -lean_dec(x_90); -if (x_91 == 0) +lean_object* x_47; uint8_t x_48; +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_unbox(x_47); +lean_dec(x_47); +if (x_48 == 0) { -lean_object* x_92; uint8_t x_93; -x_92 = lean_ctor_get(x_89, 1); -lean_inc(x_92); -lean_dec(x_89); -x_93 = 1; -x_17 = x_93; -x_18 = x_92; -goto block_25; +lean_object* x_49; lean_object* x_50; +x_49 = lean_ctor_get(x_46, 1); +lean_inc(x_49); +lean_dec(x_46); +x_50 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__3; +x_20 = x_50; +x_21 = x_49; +goto block_27; } else { -lean_object* x_94; uint8_t x_95; -x_94 = lean_ctor_get(x_89, 1); -lean_inc(x_94); -lean_dec(x_89); -x_95 = 0; -x_17 = x_95; -x_18 = x_94; -goto block_25; +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_46, 1); +lean_inc(x_51); +lean_dec(x_46); +lean_inc(x_4); +x_52 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_52, 0, x_4); +x_20 = x_52; +x_21 = x_51; +goto block_27; } } else { -uint8_t x_96; +uint8_t x_53; +lean_dec(x_19); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_96 = !lean_is_exclusive(x_89); -if (x_96 == 0) +lean_dec(x_6); +lean_dec(x_4); +x_53 = !lean_is_exclusive(x_46); +if (x_53 == 0) { -return x_89; +return x_46; } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_89, 0); -x_98 = lean_ctor_get(x_89, 1); -lean_inc(x_98); -lean_inc(x_97); -lean_dec(x_89); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_46, 0); +x_55 = lean_ctor_get(x_46, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_46); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +return x_56; } } } -else -{ -uint8_t x_100; -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -x_100 = !lean_is_exclusive(x_86); -if (x_100 == 0) -{ -return x_86; } else { -lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_101 = lean_ctor_get(x_86, 0); -x_102 = lean_ctor_get(x_86, 1); -lean_inc(x_102); -lean_inc(x_101); -lean_dec(x_86); -x_103 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -return x_103; -} -} -} -else +lean_object* x_57; +x_57 = lean_array_fget(x_1, x_6); +if (x_30 == 0) { -uint8_t x_104; -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_13); -lean_dec(x_12); +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_59 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_58); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_60 = lean_is_expr_def_eq(x_57, x_59, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; uint8_t x_62; +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +x_62 = lean_unbox(x_61); +lean_dec(x_61); +if (x_62 == 0) +{ +lean_object* x_63; lean_object* x_64; +x_63 = lean_ctor_get(x_60, 1); +lean_inc(x_63); +lean_dec(x_60); +x_64 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__3; +x_20 = x_64; +x_21 = x_63; +goto block_27; +} +else +{ +lean_object* x_65; lean_object* x_66; +x_65 = lean_ctor_get(x_60, 1); +lean_inc(x_65); +lean_dec(x_60); +lean_inc(x_4); +x_66 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_66, 0, x_4); +x_20 = x_66; +x_21 = x_65; +goto block_27; +} +} +else +{ +uint8_t x_67; +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_104 = !lean_is_exclusive(x_84); -if (x_104 == 0) +lean_dec(x_6); +lean_dec(x_4); +x_67 = !lean_is_exclusive(x_60); +if (x_67 == 0) { -return x_84; +return x_60; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_84, 0); -x_106 = lean_ctor_get(x_84, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_84); -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_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_60, 0); +x_69 = lean_ctor_get(x_60, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_60); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; } } } +else +{ +lean_object* x_71; lean_object* x_72; +x_71 = lean_array_fget(x_2, x_6); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_72 = lean_is_expr_def_eq(x_57, x_71, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_72) == 0) +{ +lean_object* x_73; uint8_t x_74; +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +x_74 = lean_unbox(x_73); +lean_dec(x_73); +if (x_74 == 0) +{ +lean_object* x_75; lean_object* x_76; +x_75 = lean_ctor_get(x_72, 1); +lean_inc(x_75); +lean_dec(x_72); +x_76 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__3; +x_20 = x_76; +x_21 = x_75; +goto block_27; } +else +{ +lean_object* x_77; lean_object* x_78; +x_77 = lean_ctor_get(x_72, 1); +lean_inc(x_77); +lean_dec(x_72); +lean_inc(x_4); +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_4); +x_20 = x_78; +x_21 = x_77; +goto block_27; } } else { -uint8_t x_116; lean_object* x_117; lean_object* x_118; +uint8_t x_79; +lean_dec(x_19); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_116 = 0; -x_117 = lean_box(x_116); -x_118 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_118, 0, x_117); -lean_ctor_set(x_118, 1, x_14); -return x_118; +lean_dec(x_6); +lean_dec(x_4); +x_79 = !lean_is_exclusive(x_72); +if (x_79 == 0) +{ +return x_72; } +else +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_80 = lean_ctor_get(x_72, 0); +x_81 = lean_ctor_get(x_72, 1); +lean_inc(x_81); +lean_inc(x_80); +lean_dec(x_72); +x_82 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +return x_82; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs(lean_object* x_1, lean_object* x_2, 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: +} +} +block_27: { -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_array_get_size(x_2); -x_10 = lean_array_get_size(x_3); -x_11 = lean_nat_dec_eq(x_9, x_10); -if (x_11 == 0) +if (lean_obj_tag(x_20) == 0) { -uint8_t x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_22; lean_object* x_23; +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); -lean_dec(x_1); -x_12 = 0; -x_13 = lean_box(x_12); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_8); -return x_14; +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; } else { -lean_object* x_15; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_9); -x_15 = l_Lean_Meta_getFunInfoNArgs(x_1, x_9, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -lean_dec(x_16); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_19 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass(x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_17); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -if (lean_obj_tag(x_20) == 0) +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_20, 0); +lean_inc(x_24); +lean_dec(x_20); +x_25 = lean_nat_add(x_6, x_8); +lean_dec(x_6); +x_5 = x_19; +x_6 = x_25; +x_9 = x_24; +x_14 = x_21; +goto _start; +} +} +} +else { -uint8_t x_21; -lean_dec(x_18); +lean_object* x_83; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_21 = !lean_is_exclusive(x_19); -if (x_21 == 0) -{ -lean_object* x_22; uint8_t x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_19, 0); -lean_dec(x_22); -x_23 = 0; -x_24 = lean_box(x_23); -lean_ctor_set(x_19, 0, x_24); -return x_19; -} -else -{ -lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_19, 1); -lean_inc(x_25); -lean_dec(x_19); -x_26 = 0; -x_27 = lean_box(x_26); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_25); -return x_28; +x_83 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_83, 0, x_9); +lean_ctor_set(x_83, 1, x_14); +return x_83; } } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_29 = lean_ctor_get(x_19, 1); -lean_inc(x_29); -lean_dec(x_19); -x_30 = lean_ctor_get(x_20, 0); -lean_inc(x_30); -lean_dec(x_20); -x_31 = lean_array_get_size(x_18); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_31); -x_32 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs_processOtherArgs(x_2, x_3, lean_box(0), x_31, x_4, x_5, x_6, x_7, x_29); -if (lean_obj_tag(x_32) == 0) -{ -lean_object* x_33; uint8_t x_34; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_unbox(x_33); -lean_dec(x_33); -if (x_34 == 0) -{ -uint8_t x_35; -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_18); +lean_object* x_84; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_35 = !lean_is_exclusive(x_32); -if (x_35 == 0) +x_84 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_84, 0, x_9); +lean_ctor_set(x_84, 1, x_14); +return x_84; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_36; uint8_t x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_32, 0); -lean_dec(x_36); -x_37 = 0; -x_38 = lean_box(x_37); -lean_ctor_set(x_32, 0, x_38); -return x_32; +uint8_t x_10; lean_object* x_11; uint8_t x_17; +x_17 = !lean_is_exclusive(x_5); +if (x_17 == 0) +{ +lean_object* x_18; uint8_t x_19; +x_18 = lean_ctor_get(x_5, 0); +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) +{ +uint8_t x_20; uint8_t x_21; uint8_t x_22; +x_20 = lean_ctor_get_uint8(x_18, 5); +x_21 = 1; +x_22 = l_Lean_Meta_TransparencyMode_lt(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = lean_is_expr_def_eq(x_1, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_unbox(x_24); +lean_dec(x_24); +x_10 = x_26; +x_11 = x_25; +goto block_16; } else { -lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; -x_39 = lean_ctor_get(x_32, 1); -lean_inc(x_39); -lean_dec(x_32); -x_40 = 0; -x_41 = lean_box(x_40); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_39); -return x_42; -} +uint8_t x_27; +lean_dec(x_3); +x_27 = !lean_is_exclusive(x_23); +if (x_27 == 0) +{ +return x_23; } else { -uint8_t x_43; -x_43 = !lean_is_exclusive(x_32); -if (x_43 == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_23, 0); +x_29 = lean_ctor_get(x_23, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_23); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_44 = lean_ctor_get(x_32, 1); -x_45 = lean_ctor_get(x_32, 0); -lean_dec(x_45); -x_46 = lean_array_get_size(x_30); -x_47 = lean_unsigned_to_nat(0u); -x_48 = lean_nat_dec_lt(x_47, x_46); -if (x_48 == 0) +lean_object* x_31; +lean_ctor_set_uint8(x_18, 5, x_21); +x_31 = lean_is_expr_def_eq(x_1, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_31) == 0) { -uint8_t x_49; lean_object* x_50; -lean_dec(x_46); +lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_18); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_49 = 1; -x_50 = lean_box(x_49); -lean_ctor_set(x_32, 0, x_50); -return x_32; +x_34 = lean_unbox(x_32); +lean_dec(x_32); +x_10 = x_34; +x_11 = x_33; +goto block_16; } else { -uint8_t x_51; -x_51 = lean_nat_dec_le(x_46, x_46); -if (x_51 == 0) +uint8_t x_35; +lean_dec(x_3); +x_35 = !lean_is_exclusive(x_31); +if (x_35 == 0) { -uint8_t x_52; lean_object* x_53; -lean_dec(x_46); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_18); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_52 = 1; -x_53 = lean_box(x_52); -lean_ctor_set(x_32, 0, x_53); -return x_32; +return x_31; } else { -size_t x_54; size_t x_55; lean_object* x_56; -lean_free_object(x_32); -x_54 = 0; -x_55 = lean_usize_of_nat(x_46); -lean_dec(x_46); -x_56 = l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(x_2, x_3, x_9, x_10, x_18, x_31, x_30, x_54, x_55, x_4, x_5, x_6, x_7, x_44); -lean_dec(x_30); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_31, 0); +x_37 = lean_ctor_get(x_31, 1); +lean_inc(x_37); +lean_inc(x_36); lean_dec(x_31); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} +} +} +} +else +{ +uint8_t x_39; 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; uint8_t x_52; uint8_t x_53; uint8_t x_54; +x_39 = lean_ctor_get_uint8(x_18, 0); +x_40 = lean_ctor_get_uint8(x_18, 1); +x_41 = lean_ctor_get_uint8(x_18, 2); +x_42 = lean_ctor_get_uint8(x_18, 3); +x_43 = lean_ctor_get_uint8(x_18, 4); +x_44 = lean_ctor_get_uint8(x_18, 5); +x_45 = lean_ctor_get_uint8(x_18, 6); +x_46 = lean_ctor_get_uint8(x_18, 7); +x_47 = lean_ctor_get_uint8(x_18, 8); +x_48 = lean_ctor_get_uint8(x_18, 9); +x_49 = lean_ctor_get_uint8(x_18, 10); +x_50 = lean_ctor_get_uint8(x_18, 11); +x_51 = lean_ctor_get_uint8(x_18, 12); +x_52 = lean_ctor_get_uint8(x_18, 13); lean_dec(x_18); -lean_dec(x_10); -lean_dec(x_9); +x_53 = 1; +x_54 = l_Lean_Meta_TransparencyMode_lt(x_44, x_53); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; +x_55 = lean_alloc_ctor(0, 0, 14); +lean_ctor_set_uint8(x_55, 0, x_39); +lean_ctor_set_uint8(x_55, 1, x_40); +lean_ctor_set_uint8(x_55, 2, x_41); +lean_ctor_set_uint8(x_55, 3, x_42); +lean_ctor_set_uint8(x_55, 4, x_43); +lean_ctor_set_uint8(x_55, 5, x_44); +lean_ctor_set_uint8(x_55, 6, x_45); +lean_ctor_set_uint8(x_55, 7, x_46); +lean_ctor_set_uint8(x_55, 8, x_47); +lean_ctor_set_uint8(x_55, 9, x_48); +lean_ctor_set_uint8(x_55, 10, x_49); +lean_ctor_set_uint8(x_55, 11, x_50); +lean_ctor_set_uint8(x_55, 12, x_51); +lean_ctor_set_uint8(x_55, 13, x_52); +lean_ctor_set(x_5, 0, x_55); +x_56 = lean_is_expr_def_eq(x_1, x_2, x_5, x_6, x_7, x_8, x_9); if (lean_obj_tag(x_56) == 0) { -lean_object* x_57; uint8_t x_58; +lean_object* x_57; lean_object* x_58; uint8_t x_59; x_57 = lean_ctor_get(x_56, 0); lean_inc(x_57); -x_58 = lean_unbox(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +x_59 = lean_unbox(x_57); lean_dec(x_57); -if (x_58 == 0) -{ -uint8_t x_59; -x_59 = !lean_is_exclusive(x_56); -if (x_59 == 0) -{ -lean_object* x_60; uint8_t x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_56, 0); -lean_dec(x_60); -x_61 = 1; -x_62 = lean_box(x_61); -lean_ctor_set(x_56, 0, x_62); -return x_56; +x_10 = x_59; +x_11 = x_58; +goto block_16; } else { -lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; -x_63 = lean_ctor_get(x_56, 1); -lean_inc(x_63); -lean_dec(x_56); -x_64 = 1; -x_65 = lean_box(x_64); -x_66 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_63); -return x_66; +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +lean_dec(x_3); +x_60 = lean_ctor_get(x_56, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_56, 1); +lean_inc(x_61); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_62 = x_56; +} else { + lean_dec_ref(x_56); + x_62 = lean_box(0); +} +if (lean_is_scalar(x_62)) { + x_63 = lean_alloc_ctor(1, 2, 0); +} else { + x_63 = x_62; +} +lean_ctor_set(x_63, 0, x_60); +lean_ctor_set(x_63, 1, x_61); +return x_63; } } else { -uint8_t x_67; -x_67 = !lean_is_exclusive(x_56); -if (x_67 == 0) +lean_object* x_64; lean_object* x_65; +x_64 = lean_alloc_ctor(0, 0, 14); +lean_ctor_set_uint8(x_64, 0, x_39); +lean_ctor_set_uint8(x_64, 1, x_40); +lean_ctor_set_uint8(x_64, 2, x_41); +lean_ctor_set_uint8(x_64, 3, x_42); +lean_ctor_set_uint8(x_64, 4, x_43); +lean_ctor_set_uint8(x_64, 5, x_53); +lean_ctor_set_uint8(x_64, 6, x_45); +lean_ctor_set_uint8(x_64, 7, x_46); +lean_ctor_set_uint8(x_64, 8, x_47); +lean_ctor_set_uint8(x_64, 9, x_48); +lean_ctor_set_uint8(x_64, 10, x_49); +lean_ctor_set_uint8(x_64, 11, x_50); +lean_ctor_set_uint8(x_64, 12, x_51); +lean_ctor_set_uint8(x_64, 13, x_52); +lean_ctor_set(x_5, 0, x_64); +x_65 = lean_is_expr_def_eq(x_1, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_65) == 0) { -lean_object* x_68; uint8_t x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_56, 0); -lean_dec(x_68); -x_69 = 0; -x_70 = lean_box(x_69); -lean_ctor_set(x_56, 0, x_70); -return x_56; +lean_object* x_66; lean_object* x_67; uint8_t x_68; +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +x_68 = lean_unbox(x_66); +lean_dec(x_66); +x_10 = x_68; +x_11 = x_67; +goto block_16; } else { -lean_object* x_71; uint8_t x_72; lean_object* x_73; lean_object* x_74; -x_71 = lean_ctor_get(x_56, 1); -lean_inc(x_71); -lean_dec(x_56); -x_72 = 0; -x_73 = lean_box(x_72); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_71); -return x_74; +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +lean_dec(x_3); +x_69 = lean_ctor_get(x_65, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_65, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_71 = x_65; +} else { + lean_dec_ref(x_65); + x_71 = lean_box(0); +} +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(1, 2, 0); +} else { + x_72 = x_71; +} +lean_ctor_set(x_72, 0, x_69); +lean_ctor_set(x_72, 1, x_70); +return x_72; } } } -else -{ -uint8_t x_75; -x_75 = !lean_is_exclusive(x_56); -if (x_75 == 0) -{ -return x_56; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_56, 0); -x_77 = lean_ctor_get(x_56, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; uint8_t x_81; uint8_t x_82; uint8_t x_83; uint8_t x_84; uint8_t x_85; uint8_t x_86; uint8_t x_87; uint8_t x_88; uint8_t x_89; uint8_t x_90; uint8_t x_91; uint8_t x_92; lean_object* x_93; uint8_t x_94; uint8_t x_95; +x_73 = lean_ctor_get(x_5, 0); +x_74 = lean_ctor_get(x_5, 1); +x_75 = lean_ctor_get(x_5, 2); +x_76 = lean_ctor_get(x_5, 3); +x_77 = lean_ctor_get(x_5, 4); +x_78 = lean_ctor_get(x_5, 5); +lean_inc(x_78); lean_inc(x_77); lean_inc(x_76); -lean_dec(x_56); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +lean_inc(x_75); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_5); +x_79 = lean_ctor_get_uint8(x_73, 0); +x_80 = lean_ctor_get_uint8(x_73, 1); +x_81 = lean_ctor_get_uint8(x_73, 2); +x_82 = lean_ctor_get_uint8(x_73, 3); +x_83 = lean_ctor_get_uint8(x_73, 4); +x_84 = lean_ctor_get_uint8(x_73, 5); +x_85 = lean_ctor_get_uint8(x_73, 6); +x_86 = lean_ctor_get_uint8(x_73, 7); +x_87 = lean_ctor_get_uint8(x_73, 8); +x_88 = lean_ctor_get_uint8(x_73, 9); +x_89 = lean_ctor_get_uint8(x_73, 10); +x_90 = lean_ctor_get_uint8(x_73, 11); +x_91 = lean_ctor_get_uint8(x_73, 12); +x_92 = lean_ctor_get_uint8(x_73, 13); +if (lean_is_exclusive(x_73)) { + x_93 = x_73; +} else { + lean_dec_ref(x_73); + x_93 = lean_box(0); +} +x_94 = 1; +x_95 = l_Lean_Meta_TransparencyMode_lt(x_84, x_94); +if (x_95 == 0) +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; +if (lean_is_scalar(x_93)) { + x_96 = lean_alloc_ctor(0, 0, 14); +} else { + x_96 = x_93; +} +lean_ctor_set_uint8(x_96, 0, x_79); +lean_ctor_set_uint8(x_96, 1, x_80); +lean_ctor_set_uint8(x_96, 2, x_81); +lean_ctor_set_uint8(x_96, 3, x_82); +lean_ctor_set_uint8(x_96, 4, x_83); +lean_ctor_set_uint8(x_96, 5, x_84); +lean_ctor_set_uint8(x_96, 6, x_85); +lean_ctor_set_uint8(x_96, 7, x_86); +lean_ctor_set_uint8(x_96, 8, x_87); +lean_ctor_set_uint8(x_96, 9, x_88); +lean_ctor_set_uint8(x_96, 10, x_89); +lean_ctor_set_uint8(x_96, 11, x_90); +lean_ctor_set_uint8(x_96, 12, x_91); +lean_ctor_set_uint8(x_96, 13, x_92); +x_97 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_74); +lean_ctor_set(x_97, 2, x_75); +lean_ctor_set(x_97, 3, x_76); +lean_ctor_set(x_97, 4, x_77); +lean_ctor_set(x_97, 5, x_78); +x_98 = lean_is_expr_def_eq(x_1, x_2, x_97, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_98) == 0) +{ +lean_object* x_99; lean_object* x_100; uint8_t x_101; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_98, 1); +lean_inc(x_100); +lean_dec(x_98); +x_101 = lean_unbox(x_99); +lean_dec(x_99); +x_10 = x_101; +x_11 = x_100; +goto block_16; } +else +{ +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_3); +x_102 = lean_ctor_get(x_98, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_98, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_98)) { + lean_ctor_release(x_98, 0); + lean_ctor_release(x_98, 1); + x_104 = x_98; +} else { + lean_dec_ref(x_98); + x_104 = lean_box(0); } +if (lean_is_scalar(x_104)) { + x_105 = lean_alloc_ctor(1, 2, 0); +} else { + x_105 = x_104; } +lean_ctor_set(x_105, 0, x_102); +lean_ctor_set(x_105, 1, x_103); +return x_105; } } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; -x_79 = lean_ctor_get(x_32, 1); -lean_inc(x_79); -lean_dec(x_32); -x_80 = lean_array_get_size(x_30); -x_81 = lean_unsigned_to_nat(0u); -x_82 = lean_nat_dec_lt(x_81, x_80); -if (x_82 == 0) +lean_object* x_106; lean_object* x_107; lean_object* x_108; +if (lean_is_scalar(x_93)) { + x_106 = lean_alloc_ctor(0, 0, 14); +} else { + x_106 = x_93; +} +lean_ctor_set_uint8(x_106, 0, x_79); +lean_ctor_set_uint8(x_106, 1, x_80); +lean_ctor_set_uint8(x_106, 2, x_81); +lean_ctor_set_uint8(x_106, 3, x_82); +lean_ctor_set_uint8(x_106, 4, x_83); +lean_ctor_set_uint8(x_106, 5, x_94); +lean_ctor_set_uint8(x_106, 6, x_85); +lean_ctor_set_uint8(x_106, 7, x_86); +lean_ctor_set_uint8(x_106, 8, x_87); +lean_ctor_set_uint8(x_106, 9, x_88); +lean_ctor_set_uint8(x_106, 10, x_89); +lean_ctor_set_uint8(x_106, 11, x_90); +lean_ctor_set_uint8(x_106, 12, x_91); +lean_ctor_set_uint8(x_106, 13, x_92); +x_107 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set(x_107, 1, x_74); +lean_ctor_set(x_107, 2, x_75); +lean_ctor_set(x_107, 3, x_76); +lean_ctor_set(x_107, 4, x_77); +lean_ctor_set(x_107, 5, x_78); +x_108 = lean_is_expr_def_eq(x_1, x_2, x_107, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_108) == 0) { -uint8_t x_83; lean_object* x_84; lean_object* x_85; -lean_dec(x_80); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_18); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_83 = 1; -x_84 = lean_box(x_83); -x_85 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_85, 0, x_84); -lean_ctor_set(x_85, 1, x_79); -return x_85; +lean_object* x_109; lean_object* x_110; uint8_t x_111; +x_109 = lean_ctor_get(x_108, 0); +lean_inc(x_109); +x_110 = lean_ctor_get(x_108, 1); +lean_inc(x_110); +lean_dec(x_108); +x_111 = lean_unbox(x_109); +lean_dec(x_109); +x_10 = x_111; +x_11 = x_110; +goto block_16; +} +else +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +lean_dec(x_3); +x_112 = lean_ctor_get(x_108, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_108, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_108)) { + lean_ctor_release(x_108, 0); + lean_ctor_release(x_108, 1); + x_114 = x_108; +} else { + lean_dec_ref(x_108); + x_114 = lean_box(0); +} +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); +} else { + x_115 = x_114; +} +lean_ctor_set(x_115, 0, x_112); +lean_ctor_set(x_115, 1, x_113); +return x_115; +} +} +} +block_16: +{ +if (x_10 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_3); +x_12 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__3; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_3); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_11); +return x_15; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_9, x_8); +if (x_16 == 0) +{ +lean_object* x_17; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_10); +lean_ctor_set(x_17, 1, x_15); +return x_17; +} +else +{ +lean_object* x_18; uint8_t x_19; lean_object* x_20; uint8_t x_21; uint8_t x_22; lean_object* x_23; +lean_dec(x_10); +x_18 = lean_array_uget(x_7, x_9); +x_19 = lean_nat_dec_lt(x_18, x_3); +x_20 = lean_array_get_size(x_2); +x_21 = lean_nat_dec_lt(x_18, x_20); +lean_dec(x_20); +x_22 = lean_nat_dec_lt(x_18, x_5); +if (x_19 == 0) +{ +lean_object* x_131; lean_object* x_132; +x_131 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_132 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_131); +x_23 = x_132; +goto block_130; +} +else +{ +lean_object* x_133; +x_133 = lean_array_fget(x_1, x_18); +x_23 = x_133; +goto block_130; +} +block_130: +{ +lean_object* x_24; +if (x_21 == 0) +{ +lean_object* x_127; lean_object* x_128; +x_127 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_128 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_127); +x_24 = x_128; +goto block_126; +} +else +{ +lean_object* x_129; +x_129 = lean_array_fget(x_2, x_18); +x_24 = x_129; +goto block_126; +} +block_126: +{ +if (x_22 == 0) +{ +lean_object* x_25; lean_object* x_26; uint8_t x_27; +lean_dec(x_18); +x_25 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_26 = l_panic___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__1(x_25); +x_27 = l_Lean_Meta_ParamInfo_isInstImplicit(x_26); +lean_dec(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_box(0); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_6); +x_29 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_23, x_24, x_6, x_28, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +if (lean_obj_tag(x_30) == 0) +{ +uint8_t x_31; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_31 = !lean_is_exclusive(x_29); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_29, 0); +lean_dec(x_32); +x_33 = lean_ctor_get(x_30, 0); +lean_inc(x_33); +lean_dec(x_30); +lean_ctor_set(x_29, 0, x_33); +return x_29; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_29, 1); +lean_inc(x_34); +lean_dec(x_29); +x_35 = lean_ctor_get(x_30, 0); +lean_inc(x_35); +lean_dec(x_30); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_34); +return x_36; +} +} +else +{ +lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; +x_37 = lean_ctor_get(x_29, 1); +lean_inc(x_37); +lean_dec(x_29); +x_38 = lean_ctor_get(x_30, 0); +lean_inc(x_38); +lean_dec(x_30); +x_39 = 1; +x_40 = lean_usize_add(x_9, x_39); +x_9 = x_40; +x_10 = x_38; +x_15 = x_37; +goto _start; +} +} +else +{ +uint8_t x_42; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_42 = !lean_is_exclusive(x_29); +if (x_42 == 0) +{ +return x_29; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_29, 0); +x_44 = lean_ctor_get(x_29, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_29); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +else +{ +lean_object* x_46; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_23); +x_46 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(x_23, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_46) == 0) +{ +lean_object* x_47; lean_object* x_48; +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_24); +x_48 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(x_24, x_11, x_12, x_13, x_14, x_47); +if (lean_obj_tag(x_48) == 0) +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = lean_box(0); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_6); +x_51 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_23, x_24, x_6, x_50, x_11, x_12, x_13, x_14, x_49); +if (lean_obj_tag(x_51) == 0) +{ +lean_object* x_52; +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +if (lean_obj_tag(x_52) == 0) +{ +uint8_t x_53; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_53 = !lean_is_exclusive(x_51); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; +x_54 = lean_ctor_get(x_51, 0); +lean_dec(x_54); +x_55 = lean_ctor_get(x_52, 0); +lean_inc(x_55); +lean_dec(x_52); +lean_ctor_set(x_51, 0, x_55); +return x_51; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_51, 1); +lean_inc(x_56); +lean_dec(x_51); +x_57 = lean_ctor_get(x_52, 0); +lean_inc(x_57); +lean_dec(x_52); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_56); +return x_58; +} +} +else +{ +lean_object* x_59; lean_object* x_60; size_t x_61; size_t x_62; +x_59 = lean_ctor_get(x_51, 1); +lean_inc(x_59); +lean_dec(x_51); +x_60 = lean_ctor_get(x_52, 0); +lean_inc(x_60); +lean_dec(x_52); +x_61 = 1; +x_62 = lean_usize_add(x_9, x_61); +x_9 = x_62; +x_10 = x_60; +x_15 = x_59; +goto _start; +} +} +else +{ +uint8_t x_64; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_64 = !lean_is_exclusive(x_51); +if (x_64 == 0) +{ +return x_51; +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_51, 0); +x_66 = lean_ctor_get(x_51, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_51); +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; +} +} +} +else +{ +uint8_t x_68; +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_68 = !lean_is_exclusive(x_48); +if (x_68 == 0) +{ +return x_48; +} +else +{ +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; +} +} +} +else +{ +uint8_t x_72; +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_72 = !lean_is_exclusive(x_46); +if (x_72 == 0) +{ +return x_46; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_46, 0); +x_74 = lean_ctor_get(x_46, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_46); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +return x_75; +} +} +} +} +else +{ +lean_object* x_76; uint8_t x_77; +x_76 = lean_array_fget(x_4, x_18); +lean_dec(x_18); +x_77 = l_Lean_Meta_ParamInfo_isInstImplicit(x_76); +lean_dec(x_76); +if (x_77 == 0) +{ +lean_object* x_78; lean_object* x_79; +x_78 = lean_box(0); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_6); +x_79 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_23, x_24, x_6, x_78, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_79) == 0) +{ +lean_object* x_80; +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +if (lean_obj_tag(x_80) == 0) +{ +uint8_t x_81; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_81 = !lean_is_exclusive(x_79); +if (x_81 == 0) +{ +lean_object* x_82; lean_object* x_83; +x_82 = lean_ctor_get(x_79, 0); +lean_dec(x_82); +x_83 = lean_ctor_get(x_80, 0); +lean_inc(x_83); +lean_dec(x_80); +lean_ctor_set(x_79, 0, x_83); +return x_79; +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_79, 1); +lean_inc(x_84); +lean_dec(x_79); +x_85 = lean_ctor_get(x_80, 0); +lean_inc(x_85); +lean_dec(x_80); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_84); +return x_86; +} +} +else +{ +lean_object* x_87; lean_object* x_88; size_t x_89; size_t x_90; +x_87 = lean_ctor_get(x_79, 1); +lean_inc(x_87); +lean_dec(x_79); +x_88 = lean_ctor_get(x_80, 0); +lean_inc(x_88); +lean_dec(x_80); +x_89 = 1; +x_90 = lean_usize_add(x_9, x_89); +x_9 = x_90; +x_10 = x_88; +x_15 = x_87; +goto _start; +} +} +else +{ +uint8_t x_92; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_92 = !lean_is_exclusive(x_79); +if (x_92 == 0) +{ +return x_79; +} +else +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_79, 0); +x_94 = lean_ctor_get(x_79, 1); +lean_inc(x_94); +lean_inc(x_93); +lean_dec(x_79); +x_95 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_95, 0, x_93); +lean_ctor_set(x_95, 1, x_94); +return x_95; +} +} +} +else +{ +lean_object* x_96; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_23); +x_96 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(x_23, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_96) == 0) +{ +lean_object* x_97; lean_object* x_98; +x_97 = lean_ctor_get(x_96, 1); +lean_inc(x_97); +lean_dec(x_96); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_24); +x_98 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_trySynthPending(x_24, x_11, x_12, x_13, x_14, x_97); +if (lean_obj_tag(x_98) == 0) +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_99 = lean_ctor_get(x_98, 1); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_box(0); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_6); +x_101 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_23, x_24, x_6, x_100, x_11, x_12, x_13, x_14, x_99); +if (lean_obj_tag(x_101) == 0) +{ +lean_object* x_102; +x_102 = lean_ctor_get(x_101, 0); +lean_inc(x_102); +if (lean_obj_tag(x_102) == 0) +{ +uint8_t x_103; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_103 = !lean_is_exclusive(x_101); +if (x_103 == 0) +{ +lean_object* x_104; lean_object* x_105; +x_104 = lean_ctor_get(x_101, 0); +lean_dec(x_104); +x_105 = lean_ctor_get(x_102, 0); +lean_inc(x_105); +lean_dec(x_102); +lean_ctor_set(x_101, 0, x_105); +return x_101; +} +else +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_101, 1); +lean_inc(x_106); +lean_dec(x_101); +x_107 = lean_ctor_get(x_102, 0); +lean_inc(x_107); +lean_dec(x_102); +x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_108, 0, x_107); +lean_ctor_set(x_108, 1, x_106); +return x_108; +} +} +else +{ +lean_object* x_109; lean_object* x_110; size_t x_111; size_t x_112; +x_109 = lean_ctor_get(x_101, 1); +lean_inc(x_109); +lean_dec(x_101); +x_110 = lean_ctor_get(x_102, 0); +lean_inc(x_110); +lean_dec(x_102); +x_111 = 1; +x_112 = lean_usize_add(x_9, x_111); +x_9 = x_112; +x_10 = x_110; +x_15 = x_109; +goto _start; +} +} +else +{ +uint8_t x_114; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_114 = !lean_is_exclusive(x_101); +if (x_114 == 0) +{ +return x_101; +} +else +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_101, 0); +x_116 = lean_ctor_get(x_101, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_101); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; +} +} +} +else +{ +uint8_t x_118; +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_118 = !lean_is_exclusive(x_98); +if (x_118 == 0) +{ +return x_98; +} +else +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_ctor_get(x_98, 0); +x_120 = lean_ctor_get(x_98, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_98); +x_121 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_121, 0, x_119); +lean_ctor_set(x_121, 1, x_120); +return x_121; +} +} +} +else +{ +uint8_t x_122; +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_122 = !lean_is_exclusive(x_96); +if (x_122 == 0) +{ +return x_96; +} +else +{ +lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_123 = lean_ctor_get(x_96, 0); +x_124 = lean_ctor_get(x_96, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_96); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +return x_125; +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +uint8_t x_16; +x_16 = lean_usize_dec_lt(x_9, x_8); +if (x_16 == 0) +{ +lean_object* x_17; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_10); +lean_ctor_set(x_17, 1, x_15); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_28; lean_object* x_29; uint8_t x_33; lean_object* x_34; uint8_t x_35; uint8_t x_36; lean_object* x_37; +lean_dec(x_10); +x_18 = lean_array_uget(x_7, x_9); +x_33 = lean_nat_dec_lt(x_18, x_3); +x_34 = lean_array_get_size(x_2); +x_35 = lean_nat_dec_lt(x_18, x_34); +lean_dec(x_34); +x_36 = lean_nat_dec_lt(x_18, x_5); +if (x_33 == 0) +{ +lean_object* x_199; lean_object* x_200; +x_199 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_200 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_199); +x_37 = x_200; +goto block_198; +} +else +{ +lean_object* x_201; +x_201 = lean_array_fget(x_1, x_18); +x_37 = x_201; +goto block_198; +} +block_27: +{ +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_21 = lean_ctor_get(x_19, 0); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; +} +else +{ +lean_object* x_23; size_t x_24; size_t x_25; +x_23 = lean_ctor_get(x_19, 0); +lean_inc(x_23); +lean_dec(x_19); +x_24 = 1; +x_25 = lean_usize_add(x_9, x_24); +x_9 = x_25; +x_10 = x_23; +x_15 = x_20; +goto _start; +} +} +block_32: +{ +if (x_28 == 0) +{ +lean_object* x_30; +x_30 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__3; +x_19 = x_30; +x_20 = x_29; +goto block_27; +} +else +{ +lean_object* x_31; +lean_inc(x_6); +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_6); +x_19 = x_31; +x_20 = x_29; +goto block_27; +} +} +block_198: +{ +lean_object* x_38; +if (x_35 == 0) +{ +lean_object* x_195; lean_object* x_196; +x_195 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_196 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_195); +x_38 = x_196; +goto block_194; +} +else +{ +lean_object* x_197; +x_197 = lean_array_fget(x_2, x_18); +x_38 = x_197; +goto block_194; +} +block_194: +{ +if (x_36 == 0) +{ +lean_object* x_39; lean_object* x_40; uint8_t x_41; +lean_dec(x_18); +x_39 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__2___closed__13; +x_40 = l_panic___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__1(x_39); +x_41 = l_Lean_Meta_ParamInfo_isInstImplicit(x_40); +lean_dec(x_40); +if (x_41 == 0) +{ +lean_object* x_42; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_42 = lean_is_expr_def_eq(x_37, x_38, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_42) == 0) +{ +lean_object* x_43; uint8_t x_44; +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_unbox(x_43); +lean_dec(x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_42, 1); +lean_inc(x_45); +lean_dec(x_42); +x_46 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__3; +x_19 = x_46; +x_20 = x_45; +goto block_27; +} +else +{ +lean_object* x_47; lean_object* x_48; +x_47 = lean_ctor_get(x_42, 1); +lean_inc(x_47); +lean_dec(x_42); +lean_inc(x_6); +x_48 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_48, 0, x_6); +x_19 = x_48; +x_20 = x_47; +goto block_27; +} +} +else +{ +uint8_t x_49; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_49 = !lean_is_exclusive(x_42); +if (x_49 == 0) +{ +return x_42; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_42, 0); +x_51 = lean_ctor_get(x_42, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_42); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; +} +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; +x_53 = lean_ctor_get(x_11, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_11, 1); +lean_inc(x_54); +x_55 = lean_ctor_get(x_11, 2); +lean_inc(x_55); +x_56 = lean_ctor_get(x_11, 3); +lean_inc(x_56); +x_57 = lean_ctor_get(x_11, 4); +lean_inc(x_57); +x_58 = lean_ctor_get(x_11, 5); +lean_inc(x_58); +x_59 = !lean_is_exclusive(x_53); +if (x_59 == 0) +{ +uint8_t x_60; uint8_t x_61; uint8_t x_62; +x_60 = lean_ctor_get_uint8(x_53, 5); +x_61 = 1; +x_62 = l_Lean_Meta_TransparencyMode_lt(x_60, x_61); +if (x_62 == 0) +{ +lean_object* x_63; lean_object* x_64; +x_63 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_63, 0, x_53); +lean_ctor_set(x_63, 1, x_54); +lean_ctor_set(x_63, 2, x_55); +lean_ctor_set(x_63, 3, x_56); +lean_ctor_set(x_63, 4, x_57); +lean_ctor_set(x_63, 5, x_58); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_64 = lean_is_expr_def_eq(x_37, x_38, x_63, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_64) == 0) +{ +lean_object* x_65; lean_object* x_66; uint8_t x_67; +x_65 = lean_ctor_get(x_64, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_64, 1); +lean_inc(x_66); +lean_dec(x_64); +x_67 = lean_unbox(x_65); +lean_dec(x_65); +x_28 = x_67; +x_29 = x_66; +goto block_32; +} +else +{ +uint8_t x_68; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_68 = !lean_is_exclusive(x_64); +if (x_68 == 0) +{ +return x_64; +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_64, 0); +x_70 = lean_ctor_get(x_64, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_64); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; +} +} +} +else +{ +lean_object* x_72; lean_object* x_73; +lean_ctor_set_uint8(x_53, 5, x_61); +x_72 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_72, 0, x_53); +lean_ctor_set(x_72, 1, x_54); +lean_ctor_set(x_72, 2, x_55); +lean_ctor_set(x_72, 3, x_56); +lean_ctor_set(x_72, 4, x_57); +lean_ctor_set(x_72, 5, x_58); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_73 = lean_is_expr_def_eq(x_37, x_38, x_72, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_73) == 0) +{ +lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_74 = lean_ctor_get(x_73, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_73, 1); +lean_inc(x_75); +lean_dec(x_73); +x_76 = lean_unbox(x_74); +lean_dec(x_74); +x_28 = x_76; +x_29 = x_75; +goto block_32; +} +else +{ +uint8_t x_77; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_77 = !lean_is_exclusive(x_73); +if (x_77 == 0) +{ +return x_73; +} +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_73, 0); +x_79 = lean_ctor_get(x_73, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_73); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +return x_80; +} +} +} +} +else +{ +uint8_t x_81; uint8_t x_82; uint8_t x_83; uint8_t x_84; uint8_t x_85; uint8_t x_86; uint8_t x_87; uint8_t x_88; uint8_t x_89; uint8_t x_90; uint8_t x_91; uint8_t x_92; uint8_t x_93; uint8_t x_94; uint8_t x_95; uint8_t x_96; +x_81 = lean_ctor_get_uint8(x_53, 0); +x_82 = lean_ctor_get_uint8(x_53, 1); +x_83 = lean_ctor_get_uint8(x_53, 2); +x_84 = lean_ctor_get_uint8(x_53, 3); +x_85 = lean_ctor_get_uint8(x_53, 4); +x_86 = lean_ctor_get_uint8(x_53, 5); +x_87 = lean_ctor_get_uint8(x_53, 6); +x_88 = lean_ctor_get_uint8(x_53, 7); +x_89 = lean_ctor_get_uint8(x_53, 8); +x_90 = lean_ctor_get_uint8(x_53, 9); +x_91 = lean_ctor_get_uint8(x_53, 10); +x_92 = lean_ctor_get_uint8(x_53, 11); +x_93 = lean_ctor_get_uint8(x_53, 12); +x_94 = lean_ctor_get_uint8(x_53, 13); +lean_dec(x_53); +x_95 = 1; +x_96 = l_Lean_Meta_TransparencyMode_lt(x_86, x_95); +if (x_96 == 0) +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_alloc_ctor(0, 0, 14); +lean_ctor_set_uint8(x_97, 0, x_81); +lean_ctor_set_uint8(x_97, 1, x_82); +lean_ctor_set_uint8(x_97, 2, x_83); +lean_ctor_set_uint8(x_97, 3, x_84); +lean_ctor_set_uint8(x_97, 4, x_85); +lean_ctor_set_uint8(x_97, 5, x_86); +lean_ctor_set_uint8(x_97, 6, x_87); +lean_ctor_set_uint8(x_97, 7, x_88); +lean_ctor_set_uint8(x_97, 8, x_89); +lean_ctor_set_uint8(x_97, 9, x_90); +lean_ctor_set_uint8(x_97, 10, x_91); +lean_ctor_set_uint8(x_97, 11, x_92); +lean_ctor_set_uint8(x_97, 12, x_93); +lean_ctor_set_uint8(x_97, 13, x_94); +x_98 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_98, 0, x_97); +lean_ctor_set(x_98, 1, x_54); +lean_ctor_set(x_98, 2, x_55); +lean_ctor_set(x_98, 3, x_56); +lean_ctor_set(x_98, 4, x_57); +lean_ctor_set(x_98, 5, x_58); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_99 = lean_is_expr_def_eq(x_37, x_38, x_98, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_99) == 0) +{ +lean_object* x_100; lean_object* x_101; uint8_t x_102; +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_99, 1); +lean_inc(x_101); +lean_dec(x_99); +x_102 = lean_unbox(x_100); +lean_dec(x_100); +x_28 = x_102; +x_29 = x_101; +goto block_32; +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_103 = lean_ctor_get(x_99, 0); +lean_inc(x_103); +x_104 = lean_ctor_get(x_99, 1); +lean_inc(x_104); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_105 = x_99; +} else { + lean_dec_ref(x_99); + x_105 = lean_box(0); +} +if (lean_is_scalar(x_105)) { + x_106 = lean_alloc_ctor(1, 2, 0); +} else { + x_106 = x_105; +} +lean_ctor_set(x_106, 0, x_103); +lean_ctor_set(x_106, 1, x_104); +return x_106; +} +} +else +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_alloc_ctor(0, 0, 14); +lean_ctor_set_uint8(x_107, 0, x_81); +lean_ctor_set_uint8(x_107, 1, x_82); +lean_ctor_set_uint8(x_107, 2, x_83); +lean_ctor_set_uint8(x_107, 3, x_84); +lean_ctor_set_uint8(x_107, 4, x_85); +lean_ctor_set_uint8(x_107, 5, x_95); +lean_ctor_set_uint8(x_107, 6, x_87); +lean_ctor_set_uint8(x_107, 7, x_88); +lean_ctor_set_uint8(x_107, 8, x_89); +lean_ctor_set_uint8(x_107, 9, x_90); +lean_ctor_set_uint8(x_107, 10, x_91); +lean_ctor_set_uint8(x_107, 11, x_92); +lean_ctor_set_uint8(x_107, 12, x_93); +lean_ctor_set_uint8(x_107, 13, x_94); +x_108 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_108, 0, x_107); +lean_ctor_set(x_108, 1, x_54); +lean_ctor_set(x_108, 2, x_55); +lean_ctor_set(x_108, 3, x_56); +lean_ctor_set(x_108, 4, x_57); +lean_ctor_set(x_108, 5, x_58); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_109 = lean_is_expr_def_eq(x_37, x_38, x_108, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_109) == 0) +{ +lean_object* x_110; lean_object* x_111; uint8_t x_112; +x_110 = lean_ctor_get(x_109, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_109, 1); +lean_inc(x_111); +lean_dec(x_109); +x_112 = lean_unbox(x_110); +lean_dec(x_110); +x_28 = x_112; +x_29 = x_111; +goto block_32; +} +else +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_113 = lean_ctor_get(x_109, 0); +lean_inc(x_113); +x_114 = lean_ctor_get(x_109, 1); +lean_inc(x_114); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + lean_ctor_release(x_109, 1); + x_115 = x_109; +} else { + lean_dec_ref(x_109); + x_115 = lean_box(0); +} +if (lean_is_scalar(x_115)) { + x_116 = lean_alloc_ctor(1, 2, 0); +} else { + x_116 = x_115; +} +lean_ctor_set(x_116, 0, x_113); +lean_ctor_set(x_116, 1, x_114); +return x_116; +} +} +} +} +} +else +{ +lean_object* x_117; uint8_t x_118; +x_117 = lean_array_fget(x_4, x_18); +lean_dec(x_18); +x_118 = l_Lean_Meta_ParamInfo_isInstImplicit(x_117); +lean_dec(x_117); +if (x_118 == 0) +{ +lean_object* x_119; +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_119 = lean_is_expr_def_eq(x_37, x_38, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_119) == 0) +{ +lean_object* x_120; uint8_t x_121; +x_120 = lean_ctor_get(x_119, 0); +lean_inc(x_120); +x_121 = lean_unbox(x_120); +lean_dec(x_120); +if (x_121 == 0) +{ +lean_object* x_122; lean_object* x_123; +x_122 = lean_ctor_get(x_119, 1); +lean_inc(x_122); +lean_dec(x_119); +x_123 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___spec__1___lambda__1___closed__3; +x_19 = x_123; +x_20 = x_122; +goto block_27; +} +else +{ +lean_object* x_124; lean_object* x_125; +x_124 = lean_ctor_get(x_119, 1); +lean_inc(x_124); +lean_dec(x_119); +lean_inc(x_6); +x_125 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_125, 0, x_6); +x_19 = x_125; +x_20 = x_124; +goto block_27; +} +} +else +{ +uint8_t x_126; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_126 = !lean_is_exclusive(x_119); +if (x_126 == 0) +{ +return x_119; +} +else +{ +lean_object* x_127; lean_object* x_128; lean_object* x_129; +x_127 = lean_ctor_get(x_119, 0); +x_128 = lean_ctor_get(x_119, 1); +lean_inc(x_128); +lean_inc(x_127); +lean_dec(x_119); +x_129 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_129, 0, x_127); +lean_ctor_set(x_129, 1, x_128); +return x_129; +} +} +} +else +{ +lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; uint8_t x_136; +x_130 = lean_ctor_get(x_11, 0); +lean_inc(x_130); +x_131 = lean_ctor_get(x_11, 1); +lean_inc(x_131); +x_132 = lean_ctor_get(x_11, 2); +lean_inc(x_132); +x_133 = lean_ctor_get(x_11, 3); +lean_inc(x_133); +x_134 = lean_ctor_get(x_11, 4); +lean_inc(x_134); +x_135 = lean_ctor_get(x_11, 5); +lean_inc(x_135); +x_136 = !lean_is_exclusive(x_130); +if (x_136 == 0) +{ +uint8_t x_137; uint8_t x_138; uint8_t x_139; +x_137 = lean_ctor_get_uint8(x_130, 5); +x_138 = 1; +x_139 = l_Lean_Meta_TransparencyMode_lt(x_137, x_138); +if (x_139 == 0) +{ +lean_object* x_140; lean_object* x_141; +x_140 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_140, 0, x_130); +lean_ctor_set(x_140, 1, x_131); +lean_ctor_set(x_140, 2, x_132); +lean_ctor_set(x_140, 3, x_133); +lean_ctor_set(x_140, 4, x_134); +lean_ctor_set(x_140, 5, x_135); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_141 = lean_is_expr_def_eq(x_37, x_38, x_140, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_141) == 0) +{ +lean_object* x_142; lean_object* x_143; uint8_t x_144; +x_142 = lean_ctor_get(x_141, 0); +lean_inc(x_142); +x_143 = lean_ctor_get(x_141, 1); +lean_inc(x_143); +lean_dec(x_141); +x_144 = lean_unbox(x_142); +lean_dec(x_142); +x_28 = x_144; +x_29 = x_143; +goto block_32; +} +else +{ +uint8_t x_145; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_145 = !lean_is_exclusive(x_141); +if (x_145 == 0) +{ +return x_141; +} +else +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; +x_146 = lean_ctor_get(x_141, 0); +x_147 = lean_ctor_get(x_141, 1); +lean_inc(x_147); +lean_inc(x_146); +lean_dec(x_141); +x_148 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_148, 0, x_146); +lean_ctor_set(x_148, 1, x_147); +return x_148; +} +} +} +else +{ +lean_object* x_149; lean_object* x_150; +lean_ctor_set_uint8(x_130, 5, x_138); +x_149 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_149, 0, x_130); +lean_ctor_set(x_149, 1, x_131); +lean_ctor_set(x_149, 2, x_132); +lean_ctor_set(x_149, 3, x_133); +lean_ctor_set(x_149, 4, x_134); +lean_ctor_set(x_149, 5, x_135); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_150 = lean_is_expr_def_eq(x_37, x_38, x_149, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_150) == 0) +{ +lean_object* x_151; lean_object* x_152; uint8_t x_153; +x_151 = lean_ctor_get(x_150, 0); +lean_inc(x_151); +x_152 = lean_ctor_get(x_150, 1); +lean_inc(x_152); +lean_dec(x_150); +x_153 = lean_unbox(x_151); +lean_dec(x_151); +x_28 = x_153; +x_29 = x_152; +goto block_32; +} +else +{ +uint8_t x_154; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_154 = !lean_is_exclusive(x_150); +if (x_154 == 0) +{ +return x_150; +} +else +{ +lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_155 = lean_ctor_get(x_150, 0); +x_156 = lean_ctor_get(x_150, 1); +lean_inc(x_156); +lean_inc(x_155); +lean_dec(x_150); +x_157 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_157, 0, x_155); +lean_ctor_set(x_157, 1, x_156); +return x_157; +} +} +} +} +else +{ +uint8_t x_158; uint8_t x_159; uint8_t x_160; uint8_t x_161; uint8_t x_162; uint8_t x_163; uint8_t x_164; uint8_t x_165; uint8_t x_166; uint8_t x_167; uint8_t x_168; uint8_t x_169; uint8_t x_170; uint8_t x_171; uint8_t x_172; uint8_t x_173; +x_158 = lean_ctor_get_uint8(x_130, 0); +x_159 = lean_ctor_get_uint8(x_130, 1); +x_160 = lean_ctor_get_uint8(x_130, 2); +x_161 = lean_ctor_get_uint8(x_130, 3); +x_162 = lean_ctor_get_uint8(x_130, 4); +x_163 = lean_ctor_get_uint8(x_130, 5); +x_164 = lean_ctor_get_uint8(x_130, 6); +x_165 = lean_ctor_get_uint8(x_130, 7); +x_166 = lean_ctor_get_uint8(x_130, 8); +x_167 = lean_ctor_get_uint8(x_130, 9); +x_168 = lean_ctor_get_uint8(x_130, 10); +x_169 = lean_ctor_get_uint8(x_130, 11); +x_170 = lean_ctor_get_uint8(x_130, 12); +x_171 = lean_ctor_get_uint8(x_130, 13); +lean_dec(x_130); +x_172 = 1; +x_173 = l_Lean_Meta_TransparencyMode_lt(x_163, x_172); +if (x_173 == 0) +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; +x_174 = lean_alloc_ctor(0, 0, 14); +lean_ctor_set_uint8(x_174, 0, x_158); +lean_ctor_set_uint8(x_174, 1, x_159); +lean_ctor_set_uint8(x_174, 2, x_160); +lean_ctor_set_uint8(x_174, 3, x_161); +lean_ctor_set_uint8(x_174, 4, x_162); +lean_ctor_set_uint8(x_174, 5, x_163); +lean_ctor_set_uint8(x_174, 6, x_164); +lean_ctor_set_uint8(x_174, 7, x_165); +lean_ctor_set_uint8(x_174, 8, x_166); +lean_ctor_set_uint8(x_174, 9, x_167); +lean_ctor_set_uint8(x_174, 10, x_168); +lean_ctor_set_uint8(x_174, 11, x_169); +lean_ctor_set_uint8(x_174, 12, x_170); +lean_ctor_set_uint8(x_174, 13, x_171); +x_175 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_175, 0, x_174); +lean_ctor_set(x_175, 1, x_131); +lean_ctor_set(x_175, 2, x_132); +lean_ctor_set(x_175, 3, x_133); +lean_ctor_set(x_175, 4, x_134); +lean_ctor_set(x_175, 5, x_135); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_176 = lean_is_expr_def_eq(x_37, x_38, x_175, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_176) == 0) +{ +lean_object* x_177; lean_object* x_178; uint8_t x_179; +x_177 = lean_ctor_get(x_176, 0); +lean_inc(x_177); +x_178 = lean_ctor_get(x_176, 1); +lean_inc(x_178); +lean_dec(x_176); +x_179 = lean_unbox(x_177); +lean_dec(x_177); +x_28 = x_179; +x_29 = x_178; +goto block_32; +} +else +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_180 = lean_ctor_get(x_176, 0); +lean_inc(x_180); +x_181 = lean_ctor_get(x_176, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_176)) { + lean_ctor_release(x_176, 0); + lean_ctor_release(x_176, 1); + x_182 = x_176; +} else { + lean_dec_ref(x_176); + x_182 = lean_box(0); +} +if (lean_is_scalar(x_182)) { + x_183 = lean_alloc_ctor(1, 2, 0); +} else { + x_183 = x_182; +} +lean_ctor_set(x_183, 0, x_180); +lean_ctor_set(x_183, 1, x_181); +return x_183; +} +} +else +{ +lean_object* x_184; lean_object* x_185; lean_object* x_186; +x_184 = lean_alloc_ctor(0, 0, 14); +lean_ctor_set_uint8(x_184, 0, x_158); +lean_ctor_set_uint8(x_184, 1, x_159); +lean_ctor_set_uint8(x_184, 2, x_160); +lean_ctor_set_uint8(x_184, 3, x_161); +lean_ctor_set_uint8(x_184, 4, x_162); +lean_ctor_set_uint8(x_184, 5, x_172); +lean_ctor_set_uint8(x_184, 6, x_164); +lean_ctor_set_uint8(x_184, 7, x_165); +lean_ctor_set_uint8(x_184, 8, x_166); +lean_ctor_set_uint8(x_184, 9, x_167); +lean_ctor_set_uint8(x_184, 10, x_168); +lean_ctor_set_uint8(x_184, 11, x_169); +lean_ctor_set_uint8(x_184, 12, x_170); +lean_ctor_set_uint8(x_184, 13, x_171); +x_185 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_185, 0, x_184); +lean_ctor_set(x_185, 1, x_131); +lean_ctor_set(x_185, 2, x_132); +lean_ctor_set(x_185, 3, x_133); +lean_ctor_set(x_185, 4, x_134); +lean_ctor_set(x_185, 5, x_135); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_186 = lean_is_expr_def_eq(x_37, x_38, x_185, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_186) == 0) +{ +lean_object* x_187; lean_object* x_188; uint8_t x_189; +x_187 = lean_ctor_get(x_186, 0); +lean_inc(x_187); +x_188 = lean_ctor_get(x_186, 1); +lean_inc(x_188); +lean_dec(x_186); +x_189 = lean_unbox(x_187); +lean_dec(x_187); +x_28 = x_189; +x_29 = x_188; +goto block_32; +} +else +{ +lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +x_190 = lean_ctor_get(x_186, 0); +lean_inc(x_190); +x_191 = lean_ctor_get(x_186, 1); +lean_inc(x_191); +if (lean_is_exclusive(x_186)) { + lean_ctor_release(x_186, 0); + lean_ctor_release(x_186, 1); + x_192 = x_186; +} else { + lean_dec_ref(x_186); + x_192 = lean_box(0); +} +if (lean_is_scalar(x_192)) { + x_193 = lean_alloc_ctor(1, 2, 0); +} else { + x_193 = x_192; +} +lean_ctor_set(x_193, 0, x_190); +lean_ctor_set(x_193, 1, x_191); +return x_193; +} +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___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, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; size_t x_16; lean_object* x_17; +x_15 = lean_array_get_size(x_1); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +lean_inc(x_7); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__3(x_2, x_3, x_4, x_5, x_6, x_7, x_1, x_16, x_8, x_7, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +lean_dec(x_18); +if (lean_obj_tag(x_19) == 0) +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 0); +lean_dec(x_21); +x_22 = 1; +x_23 = lean_box(x_22); +lean_ctor_set(x_17, 0, x_23); +return x_17; +} +else +{ +lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_17, 1); +lean_inc(x_24); +lean_dec(x_17); +x_25 = 1; +x_26 = lean_box(x_25); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_24); +return x_27; +} +} +else +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_17); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_17, 0); +lean_dec(x_29); +x_30 = lean_ctor_get(x_19, 0); +lean_inc(x_30); +lean_dec(x_19); +lean_ctor_set(x_17, 0, x_30); +return x_17; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_17, 1); +lean_inc(x_31); +lean_dec(x_17); +x_32 = lean_ctor_get(x_19, 0); +lean_inc(x_32); +lean_dec(x_19); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +return x_33; +} +} +} +else +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_17); +if (x_34 == 0) +{ +return x_17; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_17, 0); +x_36 = lean_ctor_get(x_17, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_17); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; +lean_dec(x_9); +x_15 = lean_array_get_size(x_1); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc_n(x_7, 2); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(x_2, x_3, x_4, x_5, x_6, x_7, x_1, x_16, x_17, x_7, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_1); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +lean_dec(x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_box(0); +x_23 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__1(x_8, x_2, x_3, x_4, x_5, x_6, x_7, x_17, x_22, x_10, x_11, x_12, x_13, x_21); +lean_dec(x_8); +return x_23; +} +else +{ +uint8_t x_24; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_18, 0); +lean_dec(x_25); +x_26 = lean_ctor_get(x_20, 0); +lean_inc(x_26); +lean_dec(x_20); +lean_ctor_set(x_18, 0, x_26); +return x_18; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_18, 1); +lean_inc(x_27); +lean_dec(x_18); +x_28 = lean_ctor_get(x_20, 0); +lean_inc(x_28); +lean_dec(x_20); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +return x_29; +} +} +} +else +{ +uint8_t x_30; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +x_30 = !lean_is_exclusive(x_18); +if (x_30 == 0) +{ +return x_18; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_18, 0); +x_32 = lean_ctor_get(x_18, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_18); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_4); +x_10 = lean_array_get_size(x_1); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_10); +x_11 = l_Lean_Meta_getFunInfoNArgs(x_2, x_10, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_14); +lean_dec(x_12); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_3); +lean_inc(x_1); +lean_inc(x_14); +x_15 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass(x_14, x_1, x_3, x_5, x_6, x_7, x_8, x_13); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +if (lean_obj_tag(x_16) == 0) +{ +uint8_t x_17; +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_17 = !lean_is_exclusive(x_15); +if (x_17 == 0) +{ +lean_object* x_18; uint8_t x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_15, 0); +lean_dec(x_18); +x_19 = 0; +x_20 = lean_box(x_19); +lean_ctor_set(x_15, 0, x_20); +return x_15; +} +else +{ +lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); +lean_dec(x_15); +x_22 = 0; +x_23 = lean_box(x_22); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_21); +return x_24; +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_25 = lean_ctor_get(x_15, 1); +lean_inc(x_25); +lean_dec(x_15); +x_26 = lean_ctor_get(x_16, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_16, 1); +lean_inc(x_27); +lean_dec(x_16); +x_28 = lean_array_get_size(x_14); +x_29 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__7; +x_30 = lean_unsigned_to_nat(1u); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_28); +lean_inc(x_10); +x_31 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1(x_1, x_3, x_10, x_29, x_10, x_28, x_10, x_30, x_29, x_5, x_6, x_7, x_8, x_25); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +lean_dec(x_32); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_31, 1); +lean_inc(x_34); +lean_dec(x_31); +x_35 = lean_box(0); +x_36 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__2(x_26, x_1, x_3, x_10, x_14, x_28, x_29, x_27, x_35, x_5, x_6, x_7, x_8, x_34); +lean_dec(x_28); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_3); +lean_dec(x_1); +return x_36; } else { -uint8_t x_86; -x_86 = lean_nat_dec_le(x_80, x_80); -if (x_86 == 0) -{ -uint8_t x_87; lean_object* x_88; lean_object* x_89; -lean_dec(x_80); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_18); +uint8_t x_37; +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_14); lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_87 = 1; -x_88 = lean_box(x_87); -x_89 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_79); -return x_89; +lean_dec(x_3); +lean_dec(x_1); +x_37 = !lean_is_exclusive(x_31); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_31, 0); +lean_dec(x_38); +x_39 = lean_ctor_get(x_33, 0); +lean_inc(x_39); +lean_dec(x_33); +lean_ctor_set(x_31, 0, x_39); +return x_31; } else { -size_t x_90; size_t x_91; lean_object* x_92; -x_90 = 0; -x_91 = lean_usize_of_nat(x_80); -lean_dec(x_80); -x_92 = l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(x_2, x_3, x_9, x_10, x_18, x_31, x_30, x_90, x_91, x_4, x_5, x_6, x_7, x_79); -lean_dec(x_30); +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_31, 1); +lean_inc(x_40); lean_dec(x_31); -lean_dec(x_18); -lean_dec(x_10); -lean_dec(x_9); -if (lean_obj_tag(x_92) == 0) -{ -lean_object* x_93; uint8_t x_94; -x_93 = lean_ctor_get(x_92, 0); -lean_inc(x_93); -x_94 = lean_unbox(x_93); -lean_dec(x_93); -if (x_94 == 0) -{ -lean_object* x_95; lean_object* x_96; uint8_t x_97; lean_object* x_98; lean_object* x_99; -x_95 = lean_ctor_get(x_92, 1); -lean_inc(x_95); -if (lean_is_exclusive(x_92)) { - lean_ctor_release(x_92, 0); - lean_ctor_release(x_92, 1); - x_96 = x_92; -} else { - lean_dec_ref(x_92); - x_96 = lean_box(0); +x_41 = lean_ctor_get(x_33, 0); +lean_inc(x_41); +lean_dec(x_33); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +return x_42; } -x_97 = 1; -x_98 = lean_box(x_97); -if (lean_is_scalar(x_96)) { - x_99 = lean_alloc_ctor(0, 2, 0); -} else { - x_99 = x_96; } -lean_ctor_set(x_99, 0, x_98); -lean_ctor_set(x_99, 1, x_95); -return x_99; } else { -lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; -x_100 = lean_ctor_get(x_92, 1); -lean_inc(x_100); -if (lean_is_exclusive(x_92)) { - lean_ctor_release(x_92, 0); - lean_ctor_release(x_92, 1); - x_101 = x_92; -} else { - lean_dec_ref(x_92); - x_101 = lean_box(0); -} -x_102 = 0; -x_103 = lean_box(x_102); -if (lean_is_scalar(x_101)) { - x_104 = lean_alloc_ctor(0, 2, 0); -} else { - x_104 = x_101; -} -lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_100); -return x_104; -} +uint8_t x_43; +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_43 = !lean_is_exclusive(x_31); +if (x_43 == 0) +{ +return x_31; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_105 = lean_ctor_get(x_92, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_92, 1); -lean_inc(x_106); -if (lean_is_exclusive(x_92)) { - lean_ctor_release(x_92, 0); - lean_ctor_release(x_92, 1); - x_107 = x_92; -} else { - lean_dec_ref(x_92); - x_107 = lean_box(0); -} -if (lean_is_scalar(x_107)) { - x_108 = lean_alloc_ctor(1, 2, 0); -} else { - x_108 = x_107; -} -lean_ctor_set(x_108, 0, x_105); -lean_ctor_set(x_108, 1, x_106); -return x_108; -} -} +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_31, 0); +x_45 = lean_ctor_get(x_31, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_31); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } } } } else { -uint8_t x_109; -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_18); +uint8_t x_47; +lean_dec(x_14); lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_109 = !lean_is_exclusive(x_32); -if (x_109 == 0) +lean_dec(x_3); +lean_dec(x_1); +x_47 = !lean_is_exclusive(x_15); +if (x_47 == 0) { -return x_32; +return x_15; } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = lean_ctor_get(x_32, 0); -x_111 = lean_ctor_get(x_32, 1); -lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_32); -x_112 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_112, 0, x_110); -lean_ctor_set(x_112, 1, x_111); -return x_112; -} +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_15, 0); +x_49 = lean_ctor_get(x_15, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_15); +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; } } } else { -uint8_t x_113; -lean_dec(x_18); +uint8_t x_51; lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -x_113 = !lean_is_exclusive(x_19); -if (x_113 == 0) +lean_dec(x_3); +lean_dec(x_1); +x_51 = !lean_is_exclusive(x_11); +if (x_51 == 0) { -return x_19; +return x_11; } else { -lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_114 = lean_ctor_get(x_19, 0); -x_115 = lean_ctor_get(x_19, 1); -lean_inc(x_115); -lean_inc(x_114); -lean_dec(x_19); -x_116 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_116, 0, x_114); -lean_ctor_set(x_116, 1, x_115); -return x_116; +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_11, 0); +x_53 = lean_ctor_get(x_11, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_11); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; } } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -uint8_t x_117; +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_array_get_size(x_2); +x_10 = lean_array_get_size(x_3); +x_11 = lean_nat_dec_eq(x_9, x_10); lean_dec(x_10); lean_dec(x_9); +if (x_11 == 0) +{ +uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_117 = !lean_is_exclusive(x_15); -if (x_117 == 0) -{ -return x_15; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_12 = 0; +x_13 = lean_box(x_12); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_8); +return x_14; } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_15, 0); -x_119 = lean_ctor_get(x_15, 1); -lean_inc(x_119); -lean_inc(x_118); -lean_dec(x_15); -x_120 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_119); -return x_120; +lean_object* x_15; lean_object* x_16; +x_15 = lean_box(0); +x_16 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__3(x_2, x_1, x_3, x_15, x_4, x_5, x_6, x_7, x_8); +return x_16; +} +} } +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_15; } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_9; -x_9 = l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = lean_unbox_usize(x_8); +lean_dec(x_8); +x_17 = lean_unbox_usize(x_9); +lean_dec(x_9); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_16, x_17, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -return x_9; +lean_dec(x_2); +lean_dec(x_1); +return x_18; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -size_t x_15; size_t x_16; lean_object* x_17; -x_15 = lean_unbox_usize(x_8); +size_t x_16; size_t x_17; lean_object* x_18; +x_16 = lean_unbox_usize(x_8); lean_dec(x_8); -x_16 = lean_unbox_usize(x_9); +x_17 = lean_unbox_usize(x_9); lean_dec(x_9); -x_17 = l_Array_anyMUnsafe_any___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_15, x_16, x_10, x_11, x_12, x_13, x_14); +x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_16, x_17, x_10, x_11, x_12, x_13, x_14, x_15); lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_18; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +size_t x_15; lean_object* x_16; +x_15 = lean_unbox_usize(x_8); +lean_dec(x_8); +x_16 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_15, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_9); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_17; +return x_16; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_9; -x_9 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_object* x_15; +x_15 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_9; +return x_15; } } LEAN_EXPORT lean_object* l_Lean_Meta_isDefEqBindingDomain_loop(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { @@ -14816,7 +16583,7 @@ lean_dec(x_5); return x_10; } } -static lean_object* _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__1() { +static lean_object* _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__1() { _start: { lean_object* x_1; @@ -14824,26 +16591,26 @@ x_1 = lean_mk_string_from_bytes("checkAssignment", 15); return x_1; } } -static lean_object* _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__2() { +static lean_object* _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__1; +x_2 = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__2; +x_2 = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__2; x_3 = l_Lean_registerInternalExceptionId(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__1() { +static lean_object* _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__1() { _start: { lean_object* x_1; @@ -14851,21 +16618,21 @@ x_1 = lean_mk_string_from_bytes("outOfScope", 10); return x_1; } } -static lean_object* _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__2() { +static lean_object* _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__1; +x_2 = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__2; +x_2 = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__2; x_3 = l_Lean_registerInternalExceptionId(x_2, x_1); return x_3; } @@ -16386,7 +18153,7 @@ static lean_object* _init_l_Lean_Meta_CheckAssignment_check___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateMData!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateMData!Impl", 47); return x_1; } } @@ -16404,8 +18171,8 @@ static lean_object* _init_l_Lean_Meta_CheckAssignment_check___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_CheckAssignment_check___closed__1; x_2 = l_Lean_Meta_CheckAssignment_check___closed__2; -x_3 = lean_unsigned_to_nat(1116u); -x_4 = lean_unsigned_to_nat(16u); +x_3 = lean_unsigned_to_nat(1434u); +x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_Meta_CheckAssignment_check___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -16415,7 +18182,7 @@ static lean_object* _init_l_Lean_Meta_CheckAssignment_check___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateProj!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateProj!Impl", 46); return x_1; } } @@ -16433,8 +18200,8 @@ static lean_object* _init_l_Lean_Meta_CheckAssignment_check___closed__7() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_CheckAssignment_check___closed__1; x_2 = l_Lean_Meta_CheckAssignment_check___closed__5; -x_3 = lean_unsigned_to_nat(1121u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1445u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Meta_CheckAssignment_check___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -16462,8 +18229,8 @@ static lean_object* _init_l_Lean_Meta_CheckAssignment_check___closed__10() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_CheckAssignment_check___closed__1; x_2 = l_Lean_Meta_CheckAssignment_check___closed__8; -x_3 = lean_unsigned_to_nat(1149u); -x_4 = lean_unsigned_to_nat(19u); +x_3 = lean_unsigned_to_nat(1491u); +x_4 = lean_unsigned_to_nat(20u); x_5 = l_Lean_Meta_CheckAssignment_check___closed__9; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -16491,8 +18258,8 @@ static lean_object* _init_l_Lean_Meta_CheckAssignment_check___closed__13() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_CheckAssignment_check___closed__1; x_2 = l_Lean_Meta_CheckAssignment_check___closed__11; -x_3 = lean_unsigned_to_nat(1135u); -x_4 = lean_unsigned_to_nat(23u); +x_3 = lean_unsigned_to_nat(1471u); +x_4 = lean_unsigned_to_nat(24u); x_5 = l_Lean_Meta_CheckAssignment_check___closed__12; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -16502,7 +18269,7 @@ static lean_object* _init_l_Lean_Meta_CheckAssignment_check___closed__14() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateLet!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateLet!Impl", 45); return x_1; } } @@ -16520,8 +18287,8 @@ static lean_object* _init_l_Lean_Meta_CheckAssignment_check___closed__16() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_CheckAssignment_check___closed__1; x_2 = l_Lean_Meta_CheckAssignment_check___closed__14; -x_3 = lean_unsigned_to_nat(1158u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1500u); +x_4 = lean_unsigned_to_nat(22u); x_5 = l_Lean_Meta_CheckAssignment_check___closed__15; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -16530,59 +18297,59 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_check(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_17; lean_object* x_18; +lean_object* x_9; lean_object* x_10; lean_object* x_23; lean_object* x_24; switch (lean_obj_tag(x_1)) { case 1: { -lean_object* x_25; uint8_t x_48; -x_48 = l_Lean_Expr_hasExprMVar(x_1); -if (x_48 == 0) +lean_object* x_38; uint8_t x_61; +x_61 = l_Lean_Expr_hasExprMVar(x_1); +if (x_61 == 0) { -uint8_t x_49; -x_49 = l_Lean_Expr_hasFVar(x_1); -if (x_49 == 0) +uint8_t x_62; +x_62 = l_Lean_Expr_hasFVar(x_1); +if (x_62 == 0) { -lean_object* x_50; +lean_object* x_63; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_1); -lean_ctor_set(x_50, 1, x_8); -return x_50; +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_1); +lean_ctor_set(x_63, 1, x_8); +return x_63; } else { -lean_object* x_51; -x_51 = lean_box(0); -x_25 = x_51; -goto block_47; +lean_object* x_64; +x_64 = lean_box(0); +x_38 = x_64; +goto block_60; } } else { -lean_object* x_52; -x_52 = lean_box(0); -x_25 = x_52; -goto block_47; +lean_object* x_65; +x_65 = lean_box(0); +x_38 = x_65; +goto block_60; } -block_47: +block_60: { -lean_object* x_26; lean_object* x_27; -lean_dec(x_25); +lean_object* x_39; lean_object* x_40; +lean_dec(x_38); lean_inc(x_1); -x_26 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -if (lean_obj_tag(x_27) == 0) +x_39 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); @@ -16590,47 +18357,47 @@ lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_29 = l_Lean_Meta_CheckAssignment_checkFVar(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_28); -if (lean_obj_tag(x_29) == 0) +x_42 = l_Lean_Meta_CheckAssignment_checkFVar(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_41); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -lean_inc(x_30); -x_32 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_1, x_30, x_2, x_3, x_4, x_5, x_6, x_7, x_31); +lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +lean_inc(x_43); +x_45 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_1, x_43, x_2, x_3, x_4, x_5, x_6, x_7, x_44); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) +x_46 = !lean_is_exclusive(x_45); +if (x_46 == 0) { -lean_object* x_34; -x_34 = lean_ctor_get(x_32, 0); -lean_dec(x_34); -lean_ctor_set(x_32, 0, x_30); -return x_32; +lean_object* x_47; +x_47 = lean_ctor_get(x_45, 0); +lean_dec(x_47); +lean_ctor_set(x_45, 0, x_43); +return x_45; } else { -lean_object* x_35; lean_object* x_36; -x_35 = lean_ctor_get(x_32, 1); -lean_inc(x_35); -lean_dec(x_32); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_30); -lean_ctor_set(x_36, 1, x_35); -return x_36; +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_45, 1); +lean_inc(x_48); +lean_dec(x_45); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_43); +lean_ctor_set(x_49, 1, x_48); +return x_49; } } else { -uint8_t x_37; +uint8_t x_50; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -16638,29 +18405,29 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_37 = !lean_is_exclusive(x_29); -if (x_37 == 0) +x_50 = !lean_is_exclusive(x_42); +if (x_50 == 0) { -return x_29; +return x_42; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_29, 0); -x_39 = lean_ctor_get(x_29, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_29); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_42, 0); +x_52 = lean_ctor_get(x_42, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_42); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; } } } else { -uint8_t x_41; +uint8_t x_54; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -16668,86 +18435,86 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_41 = !lean_is_exclusive(x_26); -if (x_41 == 0) +x_54 = !lean_is_exclusive(x_39); +if (x_54 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_26, 0); -lean_dec(x_42); -x_43 = lean_ctor_get(x_27, 0); -lean_inc(x_43); -lean_dec(x_27); -lean_ctor_set(x_26, 0, x_43); -return x_26; +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_39, 0); +lean_dec(x_55); +x_56 = lean_ctor_get(x_40, 0); +lean_inc(x_56); +lean_dec(x_40); +lean_ctor_set(x_39, 0, x_56); +return x_39; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_26, 1); -lean_inc(x_44); -lean_dec(x_26); -x_45 = lean_ctor_get(x_27, 0); -lean_inc(x_45); -lean_dec(x_27); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -return x_46; +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_39, 1); +lean_inc(x_57); +lean_dec(x_39); +x_58 = lean_ctor_get(x_40, 0); +lean_inc(x_58); +lean_dec(x_40); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_57); +return x_59; } } } } case 2: { -lean_object* x_53; uint8_t x_76; -x_76 = l_Lean_Expr_hasExprMVar(x_1); -if (x_76 == 0) +lean_object* x_66; uint8_t x_89; +x_89 = l_Lean_Expr_hasExprMVar(x_1); +if (x_89 == 0) { -uint8_t x_77; -x_77 = l_Lean_Expr_hasFVar(x_1); -if (x_77 == 0) +uint8_t x_90; +x_90 = l_Lean_Expr_hasFVar(x_1); +if (x_90 == 0) { -lean_object* x_78; +lean_object* x_91; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_78 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_78, 0, x_1); -lean_ctor_set(x_78, 1, x_8); -return x_78; +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_1); +lean_ctor_set(x_91, 1, x_8); +return x_91; } else { -lean_object* x_79; -x_79 = lean_box(0); -x_53 = x_79; -goto block_75; +lean_object* x_92; +x_92 = lean_box(0); +x_66 = x_92; +goto block_88; } } else { -lean_object* x_80; -x_80 = lean_box(0); -x_53 = x_80; -goto block_75; +lean_object* x_93; +x_93 = lean_box(0); +x_66 = x_93; +goto block_88; } -block_75: +block_88: { -lean_object* x_54; lean_object* x_55; -lean_dec(x_53); +lean_object* x_67; lean_object* x_68; +lean_dec(x_66); lean_inc(x_1); -x_54 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -if (lean_obj_tag(x_55) == 0) +x_67 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +if (lean_obj_tag(x_68) == 0) { -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_54, 1); -lean_inc(x_56); -lean_dec(x_54); +lean_object* x_69; lean_object* x_70; +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); @@ -16755,47 +18522,47 @@ lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_57 = l_Lean_Meta_CheckAssignment_checkMVar(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_56); -if (lean_obj_tag(x_57) == 0) +x_70 = l_Lean_Meta_CheckAssignment_checkMVar(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_69); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -lean_inc(x_58); -x_60 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_1, x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_59); +lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +lean_inc(x_71); +x_73 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_1, x_71, x_2, x_3, x_4, x_5, x_6, x_7, x_72); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_61 = !lean_is_exclusive(x_60); -if (x_61 == 0) +x_74 = !lean_is_exclusive(x_73); +if (x_74 == 0) { -lean_object* x_62; -x_62 = lean_ctor_get(x_60, 0); -lean_dec(x_62); -lean_ctor_set(x_60, 0, x_58); -return x_60; +lean_object* x_75; +x_75 = lean_ctor_get(x_73, 0); +lean_dec(x_75); +lean_ctor_set(x_73, 0, x_71); +return x_73; } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_60, 1); -lean_inc(x_63); -lean_dec(x_60); -x_64 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_64, 0, x_58); -lean_ctor_set(x_64, 1, x_63); -return x_64; +lean_object* x_76; lean_object* x_77; +x_76 = lean_ctor_get(x_73, 1); +lean_inc(x_76); +lean_dec(x_73); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_71); +lean_ctor_set(x_77, 1, x_76); +return x_77; } } else { -uint8_t x_65; +uint8_t x_78; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -16803,29 +18570,29 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_57); -if (x_65 == 0) +x_78 = !lean_is_exclusive(x_70); +if (x_78 == 0) { -return x_57; +return x_70; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_57, 0); -x_67 = lean_ctor_get(x_57, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_57); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_70, 0); +x_80 = lean_ctor_get(x_70, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_70); +x_81 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +return x_81; } } } else { -uint8_t x_69; +uint8_t x_82; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -16833,83 +18600,83 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_54); -if (x_69 == 0) +x_82 = !lean_is_exclusive(x_67); +if (x_82 == 0) { -lean_object* x_70; lean_object* x_71; -x_70 = lean_ctor_get(x_54, 0); -lean_dec(x_70); -x_71 = lean_ctor_get(x_55, 0); -lean_inc(x_71); -lean_dec(x_55); -lean_ctor_set(x_54, 0, x_71); -return x_54; +lean_object* x_83; lean_object* x_84; +x_83 = lean_ctor_get(x_67, 0); +lean_dec(x_83); +x_84 = lean_ctor_get(x_68, 0); +lean_inc(x_84); +lean_dec(x_68); +lean_ctor_set(x_67, 0, x_84); +return x_67; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_54, 1); -lean_inc(x_72); -lean_dec(x_54); -x_73 = lean_ctor_get(x_55, 0); -lean_inc(x_73); -lean_dec(x_55); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_72); -return x_74; +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_67, 1); +lean_inc(x_85); +lean_dec(x_67); +x_86 = lean_ctor_get(x_68, 0); +lean_inc(x_86); +lean_dec(x_68); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_85); +return x_87; } } } } case 5: { -lean_object* x_81; -x_81 = l_Lean_Meta_CheckAssignment_checkApp(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_81; +lean_object* x_94; +x_94 = l_Lean_Meta_CheckAssignment_checkApp(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_94; } case 6: { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_116; uint8_t x_132; -x_82 = lean_ctor_get(x_1, 1); -lean_inc(x_82); -x_83 = lean_ctor_get(x_1, 2); -lean_inc(x_83); -x_132 = l_Lean_Expr_hasExprMVar(x_82); -if (x_132 == 0) +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_145; uint8_t x_161; +x_95 = lean_ctor_get(x_1, 1); +lean_inc(x_95); +x_96 = lean_ctor_get(x_1, 2); +lean_inc(x_96); +x_161 = l_Lean_Expr_hasExprMVar(x_95); +if (x_161 == 0) { -uint8_t x_133; -x_133 = l_Lean_Expr_hasFVar(x_82); -if (x_133 == 0) +uint8_t x_162; +x_162 = l_Lean_Expr_hasFVar(x_95); +if (x_162 == 0) { -x_84 = x_82; -x_85 = x_8; -goto block_115; +x_97 = x_95; +x_98 = x_8; +goto block_144; } else { -lean_object* x_134; -x_134 = lean_box(0); -x_116 = x_134; -goto block_131; +lean_object* x_163; +x_163 = lean_box(0); +x_145 = x_163; +goto block_160; } } else { -lean_object* x_135; -x_135 = lean_box(0); -x_116 = x_135; -goto block_131; +lean_object* x_164; +x_164 = lean_box(0); +x_145 = x_164; +goto block_160; } -block_115: +block_144: { -lean_object* x_86; lean_object* x_87; lean_object* x_95; uint8_t x_111; -x_111 = l_Lean_Expr_hasExprMVar(x_83); -if (x_111 == 0) +lean_object* x_99; lean_object* x_100; lean_object* x_124; uint8_t x_140; +x_140 = l_Lean_Expr_hasExprMVar(x_96); +if (x_140 == 0) { -uint8_t x_112; -x_112 = l_Lean_Expr_hasFVar(x_83); -if (x_112 == 0) +uint8_t x_141; +x_141 = l_Lean_Expr_hasFVar(x_96); +if (x_141 == 0) { lean_dec(x_7); lean_dec(x_6); @@ -16917,101 +18684,166 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_86 = x_83; -x_87 = x_85; -goto block_94; +x_99 = x_96; +x_100 = x_98; +goto block_123; } else { -lean_object* x_113; -x_113 = lean_box(0); -x_95 = x_113; -goto block_110; +lean_object* x_142; +x_142 = lean_box(0); +x_124 = x_142; +goto block_139; } } else { -lean_object* x_114; -x_114 = lean_box(0); -x_95 = x_114; -goto block_110; +lean_object* x_143; +x_143 = lean_box(0); +x_124 = x_143; +goto block_139; } -block_94: +block_123: { if (lean_obj_tag(x_1) == 6) { -uint8_t x_88; lean_object* x_89; lean_object* x_90; -x_88 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_89 = lean_expr_update_lambda(x_1, x_88, x_84, x_86); -x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_87); -return x_90; +lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; lean_object* x_105; size_t x_106; size_t x_107; uint8_t x_108; +x_101 = lean_ctor_get(x_1, 0); +lean_inc(x_101); +x_102 = lean_ctor_get(x_1, 1); +lean_inc(x_102); +x_103 = lean_ctor_get(x_1, 2); +lean_inc(x_103); +x_104 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_103); +lean_inc(x_102); +lean_inc(x_101); +x_105 = l_Lean_Expr_lam___override(x_101, x_102, x_103, x_104); +x_106 = lean_ptr_addr(x_102); +lean_dec(x_102); +x_107 = lean_ptr_addr(x_97); +x_108 = lean_usize_dec_eq(x_106, x_107); +if (x_108 == 0) +{ +lean_object* x_109; lean_object* x_110; +lean_dec(x_105); +lean_dec(x_103); +x_109 = l_Lean_Expr_lam___override(x_101, x_97, x_99, x_104); +x_110 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_100); +return x_110; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; -lean_dec(x_86); -lean_dec(x_84); +size_t x_111; size_t x_112; uint8_t x_113; +x_111 = lean_ptr_addr(x_103); +lean_dec(x_103); +x_112 = lean_ptr_addr(x_99); +x_113 = lean_usize_dec_eq(x_111, x_112); +if (x_113 == 0) +{ +lean_object* x_114; lean_object* x_115; +lean_dec(x_105); +x_114 = l_Lean_Expr_lam___override(x_101, x_97, x_99, x_104); +x_115 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_115, 0, x_114); +lean_ctor_set(x_115, 1, x_100); +return x_115; +} +else +{ +uint8_t x_116; +x_116 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_104, x_104); +if (x_116 == 0) +{ +lean_object* x_117; lean_object* x_118; +lean_dec(x_105); +x_117 = l_Lean_Expr_lam___override(x_101, x_97, x_99, x_104); +x_118 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_118, 0, x_117); +lean_ctor_set(x_118, 1, x_100); +return x_118; +} +else +{ +lean_object* x_119; +lean_dec(x_101); +lean_dec(x_99); +lean_dec(x_97); +x_119 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_119, 0, x_105); +lean_ctor_set(x_119, 1, x_100); +return x_119; +} +} +} +} +else +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; +lean_dec(x_99); +lean_dec(x_97); lean_dec(x_1); -x_91 = l_Lean_Meta_CheckAssignment_check___closed__10; -x_92 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_91); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_87); -return x_93; +x_120 = l_Lean_Meta_CheckAssignment_check___closed__10; +x_121 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_120); +x_122 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_122, 0, x_121); +lean_ctor_set(x_122, 1, x_100); +return x_122; } } -block_110: +block_139: { -lean_object* x_96; lean_object* x_97; -lean_dec(x_95); -lean_inc(x_83); -x_96 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_83, x_2, x_3, x_4, x_5, x_6, x_7, x_85); -x_97 = lean_ctor_get(x_96, 0); -lean_inc(x_97); -if (lean_obj_tag(x_97) == 0) +lean_object* x_125; lean_object* x_126; +lean_dec(x_124); +lean_inc(x_96); +x_125 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_96, x_2, x_3, x_4, x_5, x_6, x_7, x_98); +x_126 = lean_ctor_get(x_125, 0); +lean_inc(x_126); +if (lean_obj_tag(x_126) == 0) { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_96, 1); -lean_inc(x_98); -lean_dec(x_96); +lean_object* x_127; lean_object* x_128; +x_127 = lean_ctor_get(x_125, 1); +lean_inc(x_127); +lean_dec(x_125); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_83); -x_99 = l_Lean_Meta_CheckAssignment_check(x_83, x_2, x_3, x_4, x_5, x_6, x_7, x_98); -if (lean_obj_tag(x_99) == 0) +lean_inc(x_96); +x_128 = l_Lean_Meta_CheckAssignment_check(x_96, x_2, x_3, x_4, x_5, x_6, x_7, x_127); +if (lean_obj_tag(x_128) == 0) { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_100 = lean_ctor_get(x_99, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_99, 1); -lean_inc(x_101); -lean_dec(x_99); -lean_inc(x_100); -x_102 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_83, x_100, x_2, x_3, x_4, x_5, x_6, x_7, x_101); +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_129 = lean_ctor_get(x_128, 0); +lean_inc(x_129); +x_130 = lean_ctor_get(x_128, 1); +lean_inc(x_130); +lean_dec(x_128); +lean_inc(x_129); +x_131 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_96, x_129, x_2, x_3, x_4, x_5, x_6, x_7, x_130); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_103 = lean_ctor_get(x_102, 1); -lean_inc(x_103); -lean_dec(x_102); -x_86 = x_100; -x_87 = x_103; -goto block_94; +x_132 = lean_ctor_get(x_131, 1); +lean_inc(x_132); +lean_dec(x_131); +x_99 = x_129; +x_100 = x_132; +goto block_123; } else { -uint8_t x_104; -lean_dec(x_84); -lean_dec(x_83); +uint8_t x_133; +lean_dec(x_97); +lean_dec(x_96); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17019,92 +18851,92 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_104 = !lean_is_exclusive(x_99); -if (x_104 == 0) +x_133 = !lean_is_exclusive(x_128); +if (x_133 == 0) { -return x_99; +return x_128; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_99, 0); -x_106 = lean_ctor_get(x_99, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_99); -x_107 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -return x_107; +lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_134 = lean_ctor_get(x_128, 0); +x_135 = lean_ctor_get(x_128, 1); +lean_inc(x_135); +lean_inc(x_134); +lean_dec(x_128); +x_136 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_136, 0, x_134); +lean_ctor_set(x_136, 1, x_135); +return x_136; } } } else { -lean_object* x_108; lean_object* x_109; -lean_dec(x_83); +lean_object* x_137; lean_object* x_138; +lean_dec(x_96); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_108 = lean_ctor_get(x_96, 1); -lean_inc(x_108); -lean_dec(x_96); -x_109 = lean_ctor_get(x_97, 0); -lean_inc(x_109); -lean_dec(x_97); -x_86 = x_109; -x_87 = x_108; -goto block_94; +x_137 = lean_ctor_get(x_125, 1); +lean_inc(x_137); +lean_dec(x_125); +x_138 = lean_ctor_get(x_126, 0); +lean_inc(x_138); +lean_dec(x_126); +x_99 = x_138; +x_100 = x_137; +goto block_123; } } } -block_131: +block_160: { -lean_object* x_117; lean_object* x_118; -lean_dec(x_116); -lean_inc(x_82); -x_117 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_82, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_118 = lean_ctor_get(x_117, 0); -lean_inc(x_118); -if (lean_obj_tag(x_118) == 0) +lean_object* x_146; lean_object* x_147; +lean_dec(x_145); +lean_inc(x_95); +x_146 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_95, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_147 = lean_ctor_get(x_146, 0); +lean_inc(x_147); +if (lean_obj_tag(x_147) == 0) { -lean_object* x_119; lean_object* x_120; -x_119 = lean_ctor_get(x_117, 1); -lean_inc(x_119); -lean_dec(x_117); +lean_object* x_148; lean_object* x_149; +x_148 = lean_ctor_get(x_146, 1); +lean_inc(x_148); +lean_dec(x_146); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_82); -x_120 = l_Lean_Meta_CheckAssignment_check(x_82, x_2, x_3, x_4, x_5, x_6, x_7, x_119); -if (lean_obj_tag(x_120) == 0) +lean_inc(x_95); +x_149 = l_Lean_Meta_CheckAssignment_check(x_95, x_2, x_3, x_4, x_5, x_6, x_7, x_148); +if (lean_obj_tag(x_149) == 0) { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_121 = lean_ctor_get(x_120, 0); -lean_inc(x_121); -x_122 = lean_ctor_get(x_120, 1); -lean_inc(x_122); -lean_dec(x_120); -lean_inc(x_121); -x_123 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_82, x_121, x_2, x_3, x_4, x_5, x_6, x_7, x_122); -x_124 = lean_ctor_get(x_123, 1); -lean_inc(x_124); -lean_dec(x_123); -x_84 = x_121; -x_85 = x_124; -goto block_115; +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; +x_150 = lean_ctor_get(x_149, 0); +lean_inc(x_150); +x_151 = lean_ctor_get(x_149, 1); +lean_inc(x_151); +lean_dec(x_149); +lean_inc(x_150); +x_152 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_95, x_150, x_2, x_3, x_4, x_5, x_6, x_7, x_151); +x_153 = lean_ctor_get(x_152, 1); +lean_inc(x_153); +lean_dec(x_152); +x_97 = x_150; +x_98 = x_153; +goto block_144; } else { -uint8_t x_125; -lean_dec(x_83); -lean_dec(x_82); +uint8_t x_154; +lean_dec(x_96); +lean_dec(x_95); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17112,84 +18944,84 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_125 = !lean_is_exclusive(x_120); -if (x_125 == 0) +x_154 = !lean_is_exclusive(x_149); +if (x_154 == 0) { -return x_120; +return x_149; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_126 = lean_ctor_get(x_120, 0); -x_127 = lean_ctor_get(x_120, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_120); -x_128 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_128, 0, x_126); -lean_ctor_set(x_128, 1, x_127); -return x_128; +lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_155 = lean_ctor_get(x_149, 0); +x_156 = lean_ctor_get(x_149, 1); +lean_inc(x_156); +lean_inc(x_155); +lean_dec(x_149); +x_157 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_157, 0, x_155); +lean_ctor_set(x_157, 1, x_156); +return x_157; } } } else { -lean_object* x_129; lean_object* x_130; -lean_dec(x_82); -x_129 = lean_ctor_get(x_117, 1); -lean_inc(x_129); -lean_dec(x_117); -x_130 = lean_ctor_get(x_118, 0); -lean_inc(x_130); -lean_dec(x_118); -x_84 = x_130; -x_85 = x_129; -goto block_115; +lean_object* x_158; lean_object* x_159; +lean_dec(x_95); +x_158 = lean_ctor_get(x_146, 1); +lean_inc(x_158); +lean_dec(x_146); +x_159 = lean_ctor_get(x_147, 0); +lean_inc(x_159); +lean_dec(x_147); +x_97 = x_159; +x_98 = x_158; +goto block_144; } } } case 7: { -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_170; uint8_t x_186; -x_136 = lean_ctor_get(x_1, 1); -lean_inc(x_136); -x_137 = lean_ctor_get(x_1, 2); -lean_inc(x_137); -x_186 = l_Lean_Expr_hasExprMVar(x_136); -if (x_186 == 0) +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_215; uint8_t x_231; +x_165 = lean_ctor_get(x_1, 1); +lean_inc(x_165); +x_166 = lean_ctor_get(x_1, 2); +lean_inc(x_166); +x_231 = l_Lean_Expr_hasExprMVar(x_165); +if (x_231 == 0) { -uint8_t x_187; -x_187 = l_Lean_Expr_hasFVar(x_136); -if (x_187 == 0) +uint8_t x_232; +x_232 = l_Lean_Expr_hasFVar(x_165); +if (x_232 == 0) { -x_138 = x_136; -x_139 = x_8; -goto block_169; +x_167 = x_165; +x_168 = x_8; +goto block_214; } else { -lean_object* x_188; -x_188 = lean_box(0); -x_170 = x_188; -goto block_185; +lean_object* x_233; +x_233 = lean_box(0); +x_215 = x_233; +goto block_230; } } else { -lean_object* x_189; -x_189 = lean_box(0); -x_170 = x_189; -goto block_185; +lean_object* x_234; +x_234 = lean_box(0); +x_215 = x_234; +goto block_230; } -block_169: +block_214: { -lean_object* x_140; lean_object* x_141; lean_object* x_149; uint8_t x_165; -x_165 = l_Lean_Expr_hasExprMVar(x_137); -if (x_165 == 0) +lean_object* x_169; lean_object* x_170; lean_object* x_194; uint8_t x_210; +x_210 = l_Lean_Expr_hasExprMVar(x_166); +if (x_210 == 0) { -uint8_t x_166; -x_166 = l_Lean_Expr_hasFVar(x_137); -if (x_166 == 0) +uint8_t x_211; +x_211 = l_Lean_Expr_hasFVar(x_166); +if (x_211 == 0) { lean_dec(x_7); lean_dec(x_6); @@ -17197,101 +19029,166 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_140 = x_137; -x_141 = x_139; -goto block_148; +x_169 = x_166; +x_170 = x_168; +goto block_193; } else { -lean_object* x_167; -x_167 = lean_box(0); -x_149 = x_167; -goto block_164; +lean_object* x_212; +x_212 = lean_box(0); +x_194 = x_212; +goto block_209; } } else { -lean_object* x_168; -x_168 = lean_box(0); -x_149 = x_168; -goto block_164; +lean_object* x_213; +x_213 = lean_box(0); +x_194 = x_213; +goto block_209; } -block_148: +block_193: { if (lean_obj_tag(x_1) == 7) { -uint8_t x_142; lean_object* x_143; lean_object* x_144; -x_142 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_143 = lean_expr_update_forall(x_1, x_142, x_138, x_140); -x_144 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_144, 0, x_143); -lean_ctor_set(x_144, 1, x_141); -return x_144; +lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; lean_object* x_175; size_t x_176; size_t x_177; uint8_t x_178; +x_171 = lean_ctor_get(x_1, 0); +lean_inc(x_171); +x_172 = lean_ctor_get(x_1, 1); +lean_inc(x_172); +x_173 = lean_ctor_get(x_1, 2); +lean_inc(x_173); +x_174 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_173); +lean_inc(x_172); +lean_inc(x_171); +x_175 = l_Lean_Expr_forallE___override(x_171, x_172, x_173, x_174); +x_176 = lean_ptr_addr(x_172); +lean_dec(x_172); +x_177 = lean_ptr_addr(x_167); +x_178 = lean_usize_dec_eq(x_176, x_177); +if (x_178 == 0) +{ +lean_object* x_179; lean_object* x_180; +lean_dec(x_175); +lean_dec(x_173); +x_179 = l_Lean_Expr_forallE___override(x_171, x_167, x_169, x_174); +x_180 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_180, 0, x_179); +lean_ctor_set(x_180, 1, x_170); +return x_180; } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; -lean_dec(x_140); -lean_dec(x_138); +size_t x_181; size_t x_182; uint8_t x_183; +x_181 = lean_ptr_addr(x_173); +lean_dec(x_173); +x_182 = lean_ptr_addr(x_169); +x_183 = lean_usize_dec_eq(x_181, x_182); +if (x_183 == 0) +{ +lean_object* x_184; lean_object* x_185; +lean_dec(x_175); +x_184 = l_Lean_Expr_forallE___override(x_171, x_167, x_169, x_174); +x_185 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_185, 0, x_184); +lean_ctor_set(x_185, 1, x_170); +return x_185; +} +else +{ +uint8_t x_186; +x_186 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_174, x_174); +if (x_186 == 0) +{ +lean_object* x_187; lean_object* x_188; +lean_dec(x_175); +x_187 = l_Lean_Expr_forallE___override(x_171, x_167, x_169, x_174); +x_188 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_188, 0, x_187); +lean_ctor_set(x_188, 1, x_170); +return x_188; +} +else +{ +lean_object* x_189; +lean_dec(x_171); +lean_dec(x_169); +lean_dec(x_167); +x_189 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_189, 0, x_175); +lean_ctor_set(x_189, 1, x_170); +return x_189; +} +} +} +} +else +{ +lean_object* x_190; lean_object* x_191; lean_object* x_192; +lean_dec(x_169); +lean_dec(x_167); lean_dec(x_1); -x_145 = l_Lean_Meta_CheckAssignment_check___closed__13; -x_146 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_145); -x_147 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_147, 0, x_146); -lean_ctor_set(x_147, 1, x_141); -return x_147; +x_190 = l_Lean_Meta_CheckAssignment_check___closed__13; +x_191 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_190); +x_192 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_192, 0, x_191); +lean_ctor_set(x_192, 1, x_170); +return x_192; } } -block_164: +block_209: { -lean_object* x_150; lean_object* x_151; -lean_dec(x_149); -lean_inc(x_137); -x_150 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_137, x_2, x_3, x_4, x_5, x_6, x_7, x_139); -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -if (lean_obj_tag(x_151) == 0) +lean_object* x_195; lean_object* x_196; +lean_dec(x_194); +lean_inc(x_166); +x_195 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_166, x_2, x_3, x_4, x_5, x_6, x_7, x_168); +x_196 = lean_ctor_get(x_195, 0); +lean_inc(x_196); +if (lean_obj_tag(x_196) == 0) { -lean_object* x_152; lean_object* x_153; -x_152 = lean_ctor_get(x_150, 1); -lean_inc(x_152); -lean_dec(x_150); +lean_object* x_197; lean_object* x_198; +x_197 = lean_ctor_get(x_195, 1); +lean_inc(x_197); +lean_dec(x_195); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_137); -x_153 = l_Lean_Meta_CheckAssignment_check(x_137, x_2, x_3, x_4, x_5, x_6, x_7, x_152); -if (lean_obj_tag(x_153) == 0) +lean_inc(x_166); +x_198 = l_Lean_Meta_CheckAssignment_check(x_166, x_2, x_3, x_4, x_5, x_6, x_7, x_197); +if (lean_obj_tag(x_198) == 0) { -lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; -x_154 = lean_ctor_get(x_153, 0); -lean_inc(x_154); -x_155 = lean_ctor_get(x_153, 1); -lean_inc(x_155); -lean_dec(x_153); -lean_inc(x_154); -x_156 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_137, x_154, x_2, x_3, x_4, x_5, x_6, x_7, x_155); +lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; +x_199 = lean_ctor_get(x_198, 0); +lean_inc(x_199); +x_200 = lean_ctor_get(x_198, 1); +lean_inc(x_200); +lean_dec(x_198); +lean_inc(x_199); +x_201 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_166, x_199, x_2, x_3, x_4, x_5, x_6, x_7, x_200); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_157 = lean_ctor_get(x_156, 1); -lean_inc(x_157); -lean_dec(x_156); -x_140 = x_154; -x_141 = x_157; -goto block_148; +x_202 = lean_ctor_get(x_201, 1); +lean_inc(x_202); +lean_dec(x_201); +x_169 = x_199; +x_170 = x_202; +goto block_193; } else { -uint8_t x_158; -lean_dec(x_138); -lean_dec(x_137); +uint8_t x_203; +lean_dec(x_167); +lean_dec(x_166); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17299,92 +19196,92 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_158 = !lean_is_exclusive(x_153); -if (x_158 == 0) +x_203 = !lean_is_exclusive(x_198); +if (x_203 == 0) { -return x_153; +return x_198; } else { -lean_object* x_159; lean_object* x_160; lean_object* x_161; -x_159 = lean_ctor_get(x_153, 0); -x_160 = lean_ctor_get(x_153, 1); -lean_inc(x_160); -lean_inc(x_159); -lean_dec(x_153); -x_161 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_161, 0, x_159); -lean_ctor_set(x_161, 1, x_160); -return x_161; +lean_object* x_204; lean_object* x_205; lean_object* x_206; +x_204 = lean_ctor_get(x_198, 0); +x_205 = lean_ctor_get(x_198, 1); +lean_inc(x_205); +lean_inc(x_204); +lean_dec(x_198); +x_206 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_206, 0, x_204); +lean_ctor_set(x_206, 1, x_205); +return x_206; } } } else { -lean_object* x_162; lean_object* x_163; -lean_dec(x_137); +lean_object* x_207; lean_object* x_208; +lean_dec(x_166); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_162 = lean_ctor_get(x_150, 1); -lean_inc(x_162); -lean_dec(x_150); -x_163 = lean_ctor_get(x_151, 0); -lean_inc(x_163); -lean_dec(x_151); -x_140 = x_163; -x_141 = x_162; -goto block_148; +x_207 = lean_ctor_get(x_195, 1); +lean_inc(x_207); +lean_dec(x_195); +x_208 = lean_ctor_get(x_196, 0); +lean_inc(x_208); +lean_dec(x_196); +x_169 = x_208; +x_170 = x_207; +goto block_193; } } } -block_185: +block_230: { -lean_object* x_171; lean_object* x_172; -lean_dec(x_170); -lean_inc(x_136); -x_171 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_136, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_172 = lean_ctor_get(x_171, 0); -lean_inc(x_172); -if (lean_obj_tag(x_172) == 0) +lean_object* x_216; lean_object* x_217; +lean_dec(x_215); +lean_inc(x_165); +x_216 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_165, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_217 = lean_ctor_get(x_216, 0); +lean_inc(x_217); +if (lean_obj_tag(x_217) == 0) { -lean_object* x_173; lean_object* x_174; -x_173 = lean_ctor_get(x_171, 1); -lean_inc(x_173); -lean_dec(x_171); +lean_object* x_218; lean_object* x_219; +x_218 = lean_ctor_get(x_216, 1); +lean_inc(x_218); +lean_dec(x_216); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_136); -x_174 = l_Lean_Meta_CheckAssignment_check(x_136, x_2, x_3, x_4, x_5, x_6, x_7, x_173); -if (lean_obj_tag(x_174) == 0) +lean_inc(x_165); +x_219 = l_Lean_Meta_CheckAssignment_check(x_165, x_2, x_3, x_4, x_5, x_6, x_7, x_218); +if (lean_obj_tag(x_219) == 0) { -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_175 = lean_ctor_get(x_174, 0); -lean_inc(x_175); -x_176 = lean_ctor_get(x_174, 1); -lean_inc(x_176); -lean_dec(x_174); -lean_inc(x_175); -x_177 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_136, x_175, x_2, x_3, x_4, x_5, x_6, x_7, x_176); -x_178 = lean_ctor_get(x_177, 1); -lean_inc(x_178); -lean_dec(x_177); -x_138 = x_175; -x_139 = x_178; -goto block_169; +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; +x_220 = lean_ctor_get(x_219, 0); +lean_inc(x_220); +x_221 = lean_ctor_get(x_219, 1); +lean_inc(x_221); +lean_dec(x_219); +lean_inc(x_220); +x_222 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_165, x_220, x_2, x_3, x_4, x_5, x_6, x_7, x_221); +x_223 = lean_ctor_get(x_222, 1); +lean_inc(x_223); +lean_dec(x_222); +x_167 = x_220; +x_168 = x_223; +goto block_214; } else { -uint8_t x_179; -lean_dec(x_137); -lean_dec(x_136); +uint8_t x_224; +lean_dec(x_166); +lean_dec(x_165); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17392,115 +19289,115 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_179 = !lean_is_exclusive(x_174); -if (x_179 == 0) +x_224 = !lean_is_exclusive(x_219); +if (x_224 == 0) { -return x_174; +return x_219; } else { -lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_180 = lean_ctor_get(x_174, 0); -x_181 = lean_ctor_get(x_174, 1); -lean_inc(x_181); -lean_inc(x_180); -lean_dec(x_174); -x_182 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_182, 0, x_180); -lean_ctor_set(x_182, 1, x_181); -return x_182; +lean_object* x_225; lean_object* x_226; lean_object* x_227; +x_225 = lean_ctor_get(x_219, 0); +x_226 = lean_ctor_get(x_219, 1); +lean_inc(x_226); +lean_inc(x_225); +lean_dec(x_219); +x_227 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_227, 0, x_225); +lean_ctor_set(x_227, 1, x_226); +return x_227; } } } else { -lean_object* x_183; lean_object* x_184; -lean_dec(x_136); -x_183 = lean_ctor_get(x_171, 1); -lean_inc(x_183); -lean_dec(x_171); -x_184 = lean_ctor_get(x_172, 0); -lean_inc(x_184); -lean_dec(x_172); -x_138 = x_184; -x_139 = x_183; -goto block_169; +lean_object* x_228; lean_object* x_229; +lean_dec(x_165); +x_228 = lean_ctor_get(x_216, 1); +lean_inc(x_228); +lean_dec(x_216); +x_229 = lean_ctor_get(x_217, 0); +lean_inc(x_229); +lean_dec(x_217); +x_167 = x_229; +x_168 = x_228; +goto block_214; } } } case 8: { -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_247; uint8_t x_263; -x_190 = lean_ctor_get(x_1, 1); -lean_inc(x_190); -x_191 = lean_ctor_get(x_1, 2); -lean_inc(x_191); -x_192 = lean_ctor_get(x_1, 3); -lean_inc(x_192); -x_263 = l_Lean_Expr_hasExprMVar(x_190); -if (x_263 == 0) +lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_311; uint8_t x_327; +x_235 = lean_ctor_get(x_1, 1); +lean_inc(x_235); +x_236 = lean_ctor_get(x_1, 2); +lean_inc(x_236); +x_237 = lean_ctor_get(x_1, 3); +lean_inc(x_237); +x_327 = l_Lean_Expr_hasExprMVar(x_235); +if (x_327 == 0) { -uint8_t x_264; -x_264 = l_Lean_Expr_hasFVar(x_190); -if (x_264 == 0) +uint8_t x_328; +x_328 = l_Lean_Expr_hasFVar(x_235); +if (x_328 == 0) { -x_193 = x_190; -x_194 = x_8; -goto block_246; +x_238 = x_235; +x_239 = x_8; +goto block_310; } else { -lean_object* x_265; -x_265 = lean_box(0); -x_247 = x_265; -goto block_262; +lean_object* x_329; +x_329 = lean_box(0); +x_311 = x_329; +goto block_326; } } else { -lean_object* x_266; -x_266 = lean_box(0); -x_247 = x_266; -goto block_262; +lean_object* x_330; +x_330 = lean_box(0); +x_311 = x_330; +goto block_326; } -block_246: +block_310: { -lean_object* x_195; lean_object* x_196; lean_object* x_226; uint8_t x_242; -x_242 = l_Lean_Expr_hasExprMVar(x_191); -if (x_242 == 0) +lean_object* x_240; lean_object* x_241; lean_object* x_290; uint8_t x_306; +x_306 = l_Lean_Expr_hasExprMVar(x_236); +if (x_306 == 0) { -uint8_t x_243; -x_243 = l_Lean_Expr_hasFVar(x_191); -if (x_243 == 0) +uint8_t x_307; +x_307 = l_Lean_Expr_hasFVar(x_236); +if (x_307 == 0) { -x_195 = x_191; -x_196 = x_194; -goto block_225; +x_240 = x_236; +x_241 = x_239; +goto block_289; } else { -lean_object* x_244; -x_244 = lean_box(0); -x_226 = x_244; -goto block_241; +lean_object* x_308; +x_308 = lean_box(0); +x_290 = x_308; +goto block_305; } } else { -lean_object* x_245; -x_245 = lean_box(0); -x_226 = x_245; -goto block_241; +lean_object* x_309; +x_309 = lean_box(0); +x_290 = x_309; +goto block_305; } -block_225: +block_289: { -lean_object* x_197; lean_object* x_198; lean_object* x_205; uint8_t x_221; -x_221 = l_Lean_Expr_hasExprMVar(x_192); -if (x_221 == 0) +lean_object* x_242; lean_object* x_243; lean_object* x_269; uint8_t x_285; +x_285 = l_Lean_Expr_hasExprMVar(x_237); +if (x_285 == 0) { -uint8_t x_222; -x_222 = l_Lean_Expr_hasFVar(x_192); -if (x_222 == 0) +uint8_t x_286; +x_286 = l_Lean_Expr_hasFVar(x_237); +if (x_286 == 0) { lean_dec(x_7); lean_dec(x_6); @@ -17508,102 +19405,171 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_197 = x_192; -x_198 = x_196; -goto block_204; +x_242 = x_237; +x_243 = x_241; +goto block_268; } else { -lean_object* x_223; -x_223 = lean_box(0); -x_205 = x_223; -goto block_220; +lean_object* x_287; +x_287 = lean_box(0); +x_269 = x_287; +goto block_284; } } else { -lean_object* x_224; -x_224 = lean_box(0); -x_205 = x_224; -goto block_220; +lean_object* x_288; +x_288 = lean_box(0); +x_269 = x_288; +goto block_284; } -block_204: +block_268: { if (lean_obj_tag(x_1) == 8) { -lean_object* x_199; lean_object* x_200; -x_199 = lean_expr_update_let(x_1, x_193, x_195, x_197); -x_200 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_200, 0, x_199); -lean_ctor_set(x_200, 1, x_198); -return x_200; +lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; uint8_t x_248; size_t x_249; size_t x_250; uint8_t x_251; +x_244 = lean_ctor_get(x_1, 0); +lean_inc(x_244); +x_245 = lean_ctor_get(x_1, 1); +lean_inc(x_245); +x_246 = lean_ctor_get(x_1, 2); +lean_inc(x_246); +x_247 = lean_ctor_get(x_1, 3); +lean_inc(x_247); +x_248 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); +x_249 = lean_ptr_addr(x_245); +lean_dec(x_245); +x_250 = lean_ptr_addr(x_238); +x_251 = lean_usize_dec_eq(x_249, x_250); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_247); +lean_dec(x_246); +lean_dec(x_1); +x_252 = l_Lean_Expr_letE___override(x_244, x_238, x_240, x_242, x_248); +x_253 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_253, 0, x_252); +lean_ctor_set(x_253, 1, x_243); +return x_253; } else { -lean_object* x_201; lean_object* x_202; lean_object* x_203; -lean_dec(x_197); -lean_dec(x_195); -lean_dec(x_193); +size_t x_254; size_t x_255; uint8_t x_256; +x_254 = lean_ptr_addr(x_246); +lean_dec(x_246); +x_255 = lean_ptr_addr(x_240); +x_256 = lean_usize_dec_eq(x_254, x_255); +if (x_256 == 0) +{ +lean_object* x_257; lean_object* x_258; +lean_dec(x_247); lean_dec(x_1); -x_201 = l_Lean_Meta_CheckAssignment_check___closed__16; -x_202 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_201); -x_203 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_203, 0, x_202); -lean_ctor_set(x_203, 1, x_198); -return x_203; +x_257 = l_Lean_Expr_letE___override(x_244, x_238, x_240, x_242, x_248); +x_258 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_258, 0, x_257); +lean_ctor_set(x_258, 1, x_243); +return x_258; } +else +{ +size_t x_259; size_t x_260; uint8_t x_261; +x_259 = lean_ptr_addr(x_247); +lean_dec(x_247); +x_260 = lean_ptr_addr(x_242); +x_261 = lean_usize_dec_eq(x_259, x_260); +if (x_261 == 0) +{ +lean_object* x_262; lean_object* x_263; +lean_dec(x_1); +x_262 = l_Lean_Expr_letE___override(x_244, x_238, x_240, x_242, x_248); +x_263 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_243); +return x_263; } -block_220: +else { -lean_object* x_206; lean_object* x_207; -lean_dec(x_205); -lean_inc(x_192); -x_206 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_192, x_2, x_3, x_4, x_5, x_6, x_7, x_196); -x_207 = lean_ctor_get(x_206, 0); -lean_inc(x_207); -if (lean_obj_tag(x_207) == 0) +lean_object* x_264; +lean_dec(x_244); +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +x_264 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_264, 0, x_1); +lean_ctor_set(x_264, 1, x_243); +return x_264; +} +} +} +} +else { -lean_object* x_208; lean_object* x_209; -x_208 = lean_ctor_get(x_206, 1); -lean_inc(x_208); -lean_dec(x_206); +lean_object* x_265; lean_object* x_266; lean_object* x_267; +lean_dec(x_242); +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_1); +x_265 = l_Lean_Meta_CheckAssignment_check___closed__16; +x_266 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_265); +x_267 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_267, 0, x_266); +lean_ctor_set(x_267, 1, x_243); +return x_267; +} +} +block_284: +{ +lean_object* x_270; lean_object* x_271; +lean_dec(x_269); +lean_inc(x_237); +x_270 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_237, x_2, x_3, x_4, x_5, x_6, x_7, x_241); +x_271 = lean_ctor_get(x_270, 0); +lean_inc(x_271); +if (lean_obj_tag(x_271) == 0) +{ +lean_object* x_272; lean_object* x_273; +x_272 = lean_ctor_get(x_270, 1); +lean_inc(x_272); +lean_dec(x_270); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_192); -x_209 = l_Lean_Meta_CheckAssignment_check(x_192, x_2, x_3, x_4, x_5, x_6, x_7, x_208); -if (lean_obj_tag(x_209) == 0) -{ -lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; -x_210 = lean_ctor_get(x_209, 0); -lean_inc(x_210); -x_211 = lean_ctor_get(x_209, 1); -lean_inc(x_211); -lean_dec(x_209); -lean_inc(x_210); -x_212 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_192, x_210, x_2, x_3, x_4, x_5, x_6, x_7, x_211); +lean_inc(x_237); +x_273 = l_Lean_Meta_CheckAssignment_check(x_237, x_2, x_3, x_4, x_5, x_6, x_7, x_272); +if (lean_obj_tag(x_273) == 0) +{ +lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; +x_274 = lean_ctor_get(x_273, 0); +lean_inc(x_274); +x_275 = lean_ctor_get(x_273, 1); +lean_inc(x_275); +lean_dec(x_273); +lean_inc(x_274); +x_276 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_237, x_274, x_2, x_3, x_4, x_5, x_6, x_7, x_275); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_213 = lean_ctor_get(x_212, 1); -lean_inc(x_213); -lean_dec(x_212); -x_197 = x_210; -x_198 = x_213; -goto block_204; +x_277 = lean_ctor_get(x_276, 1); +lean_inc(x_277); +lean_dec(x_276); +x_242 = x_274; +x_243 = x_277; +goto block_268; } else { -uint8_t x_214; -lean_dec(x_195); -lean_dec(x_193); -lean_dec(x_192); +uint8_t x_278; +lean_dec(x_240); +lean_dec(x_238); +lean_dec(x_237); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17611,93 +19577,93 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_214 = !lean_is_exclusive(x_209); -if (x_214 == 0) +x_278 = !lean_is_exclusive(x_273); +if (x_278 == 0) { -return x_209; +return x_273; } else { -lean_object* x_215; lean_object* x_216; lean_object* x_217; -x_215 = lean_ctor_get(x_209, 0); -x_216 = lean_ctor_get(x_209, 1); -lean_inc(x_216); -lean_inc(x_215); -lean_dec(x_209); -x_217 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_217, 0, x_215); -lean_ctor_set(x_217, 1, x_216); -return x_217; +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_273, 0); +x_280 = lean_ctor_get(x_273, 1); +lean_inc(x_280); +lean_inc(x_279); +lean_dec(x_273); +x_281 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_281, 0, x_279); +lean_ctor_set(x_281, 1, x_280); +return x_281; } } } else { -lean_object* x_218; lean_object* x_219; -lean_dec(x_192); +lean_object* x_282; lean_object* x_283; +lean_dec(x_237); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_218 = lean_ctor_get(x_206, 1); -lean_inc(x_218); -lean_dec(x_206); -x_219 = lean_ctor_get(x_207, 0); -lean_inc(x_219); -lean_dec(x_207); -x_197 = x_219; -x_198 = x_218; -goto block_204; +x_282 = lean_ctor_get(x_270, 1); +lean_inc(x_282); +lean_dec(x_270); +x_283 = lean_ctor_get(x_271, 0); +lean_inc(x_283); +lean_dec(x_271); +x_242 = x_283; +x_243 = x_282; +goto block_268; } } } -block_241: +block_305: { -lean_object* x_227; lean_object* x_228; -lean_dec(x_226); -lean_inc(x_191); -x_227 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_191, x_2, x_3, x_4, x_5, x_6, x_7, x_194); -x_228 = lean_ctor_get(x_227, 0); -lean_inc(x_228); -if (lean_obj_tag(x_228) == 0) +lean_object* x_291; lean_object* x_292; +lean_dec(x_290); +lean_inc(x_236); +x_291 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_236, x_2, x_3, x_4, x_5, x_6, x_7, x_239); +x_292 = lean_ctor_get(x_291, 0); +lean_inc(x_292); +if (lean_obj_tag(x_292) == 0) { -lean_object* x_229; lean_object* x_230; -x_229 = lean_ctor_get(x_227, 1); -lean_inc(x_229); -lean_dec(x_227); +lean_object* x_293; lean_object* x_294; +x_293 = lean_ctor_get(x_291, 1); +lean_inc(x_293); +lean_dec(x_291); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_191); -x_230 = l_Lean_Meta_CheckAssignment_check(x_191, x_2, x_3, x_4, x_5, x_6, x_7, x_229); -if (lean_obj_tag(x_230) == 0) +lean_inc(x_236); +x_294 = l_Lean_Meta_CheckAssignment_check(x_236, x_2, x_3, x_4, x_5, x_6, x_7, x_293); +if (lean_obj_tag(x_294) == 0) { -lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; -x_231 = lean_ctor_get(x_230, 0); -lean_inc(x_231); -x_232 = lean_ctor_get(x_230, 1); -lean_inc(x_232); -lean_dec(x_230); -lean_inc(x_231); -x_233 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_191, x_231, x_2, x_3, x_4, x_5, x_6, x_7, x_232); -x_234 = lean_ctor_get(x_233, 1); -lean_inc(x_234); -lean_dec(x_233); -x_195 = x_231; -x_196 = x_234; -goto block_225; +lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_295 = lean_ctor_get(x_294, 0); +lean_inc(x_295); +x_296 = lean_ctor_get(x_294, 1); +lean_inc(x_296); +lean_dec(x_294); +lean_inc(x_295); +x_297 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_236, x_295, x_2, x_3, x_4, x_5, x_6, x_7, x_296); +x_298 = lean_ctor_get(x_297, 1); +lean_inc(x_298); +lean_dec(x_297); +x_240 = x_295; +x_241 = x_298; +goto block_289; } else { -uint8_t x_235; -lean_dec(x_193); -lean_dec(x_192); -lean_dec(x_191); +uint8_t x_299; +lean_dec(x_238); +lean_dec(x_237); +lean_dec(x_236); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17705,87 +19671,87 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_235 = !lean_is_exclusive(x_230); -if (x_235 == 0) +x_299 = !lean_is_exclusive(x_294); +if (x_299 == 0) { -return x_230; +return x_294; } else { -lean_object* x_236; lean_object* x_237; lean_object* x_238; -x_236 = lean_ctor_get(x_230, 0); -x_237 = lean_ctor_get(x_230, 1); -lean_inc(x_237); -lean_inc(x_236); -lean_dec(x_230); -x_238 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_238, 0, x_236); -lean_ctor_set(x_238, 1, x_237); -return x_238; +lean_object* x_300; lean_object* x_301; lean_object* x_302; +x_300 = lean_ctor_get(x_294, 0); +x_301 = lean_ctor_get(x_294, 1); +lean_inc(x_301); +lean_inc(x_300); +lean_dec(x_294); +x_302 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_302, 0, x_300); +lean_ctor_set(x_302, 1, x_301); +return x_302; } } } else { -lean_object* x_239; lean_object* x_240; -lean_dec(x_191); -x_239 = lean_ctor_get(x_227, 1); -lean_inc(x_239); -lean_dec(x_227); -x_240 = lean_ctor_get(x_228, 0); -lean_inc(x_240); -lean_dec(x_228); -x_195 = x_240; -x_196 = x_239; -goto block_225; +lean_object* x_303; lean_object* x_304; +lean_dec(x_236); +x_303 = lean_ctor_get(x_291, 1); +lean_inc(x_303); +lean_dec(x_291); +x_304 = lean_ctor_get(x_292, 0); +lean_inc(x_304); +lean_dec(x_292); +x_240 = x_304; +x_241 = x_303; +goto block_289; } } } -block_262: +block_326: { -lean_object* x_248; lean_object* x_249; -lean_dec(x_247); -lean_inc(x_190); -x_248 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_190, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_249 = lean_ctor_get(x_248, 0); -lean_inc(x_249); -if (lean_obj_tag(x_249) == 0) +lean_object* x_312; lean_object* x_313; +lean_dec(x_311); +lean_inc(x_235); +x_312 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_235, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_313 = lean_ctor_get(x_312, 0); +lean_inc(x_313); +if (lean_obj_tag(x_313) == 0) { -lean_object* x_250; lean_object* x_251; -x_250 = lean_ctor_get(x_248, 1); -lean_inc(x_250); -lean_dec(x_248); +lean_object* x_314; lean_object* x_315; +x_314 = lean_ctor_get(x_312, 1); +lean_inc(x_314); +lean_dec(x_312); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_190); -x_251 = l_Lean_Meta_CheckAssignment_check(x_190, x_2, x_3, x_4, x_5, x_6, x_7, x_250); -if (lean_obj_tag(x_251) == 0) +lean_inc(x_235); +x_315 = l_Lean_Meta_CheckAssignment_check(x_235, x_2, x_3, x_4, x_5, x_6, x_7, x_314); +if (lean_obj_tag(x_315) == 0) { -lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; -x_252 = lean_ctor_get(x_251, 0); -lean_inc(x_252); -x_253 = lean_ctor_get(x_251, 1); -lean_inc(x_253); -lean_dec(x_251); -lean_inc(x_252); -x_254 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_190, x_252, x_2, x_3, x_4, x_5, x_6, x_7, x_253); -x_255 = lean_ctor_get(x_254, 1); -lean_inc(x_255); -lean_dec(x_254); -x_193 = x_252; -x_194 = x_255; -goto block_246; +lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; +x_316 = lean_ctor_get(x_315, 0); +lean_inc(x_316); +x_317 = lean_ctor_get(x_315, 1); +lean_inc(x_317); +lean_dec(x_315); +lean_inc(x_316); +x_318 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_235, x_316, x_2, x_3, x_4, x_5, x_6, x_7, x_317); +x_319 = lean_ctor_get(x_318, 1); +lean_inc(x_319); +lean_dec(x_318); +x_238 = x_316; +x_239 = x_319; +goto block_310; } else { -uint8_t x_256; -lean_dec(x_192); -lean_dec(x_191); -lean_dec(x_190); +uint8_t x_320; +lean_dec(x_237); +lean_dec(x_236); +lean_dec(x_235); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17793,53 +19759,53 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_256 = !lean_is_exclusive(x_251); -if (x_256 == 0) +x_320 = !lean_is_exclusive(x_315); +if (x_320 == 0) { -return x_251; +return x_315; } else { -lean_object* x_257; lean_object* x_258; lean_object* x_259; -x_257 = lean_ctor_get(x_251, 0); -x_258 = lean_ctor_get(x_251, 1); -lean_inc(x_258); -lean_inc(x_257); -lean_dec(x_251); -x_259 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_259, 0, x_257); -lean_ctor_set(x_259, 1, x_258); -return x_259; +lean_object* x_321; lean_object* x_322; lean_object* x_323; +x_321 = lean_ctor_get(x_315, 0); +x_322 = lean_ctor_get(x_315, 1); +lean_inc(x_322); +lean_inc(x_321); +lean_dec(x_315); +x_323 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_323, 0, x_321); +lean_ctor_set(x_323, 1, x_322); +return x_323; } } } else { -lean_object* x_260; lean_object* x_261; -lean_dec(x_190); -x_260 = lean_ctor_get(x_248, 1); -lean_inc(x_260); -lean_dec(x_248); -x_261 = lean_ctor_get(x_249, 0); -lean_inc(x_261); -lean_dec(x_249); -x_193 = x_261; -x_194 = x_260; -goto block_246; +lean_object* x_324; lean_object* x_325; +lean_dec(x_235); +x_324 = lean_ctor_get(x_312, 1); +lean_inc(x_324); +lean_dec(x_312); +x_325 = lean_ctor_get(x_313, 0); +lean_inc(x_325); +lean_dec(x_313); +x_238 = x_325; +x_239 = x_324; +goto block_310; } } } case 10: { -lean_object* x_267; lean_object* x_268; uint8_t x_284; -x_267 = lean_ctor_get(x_1, 1); -lean_inc(x_267); -x_284 = l_Lean_Expr_hasExprMVar(x_267); -if (x_284 == 0) +lean_object* x_331; lean_object* x_332; uint8_t x_348; +x_331 = lean_ctor_get(x_1, 1); +lean_inc(x_331); +x_348 = l_Lean_Expr_hasExprMVar(x_331); +if (x_348 == 0) { -uint8_t x_285; -x_285 = l_Lean_Expr_hasFVar(x_267); -if (x_285 == 0) +uint8_t x_349; +x_349 = l_Lean_Expr_hasFVar(x_331); +if (x_349 == 0) { lean_dec(x_7); lean_dec(x_6); @@ -17847,74 +19813,74 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_9 = x_267; +x_9 = x_331; x_10 = x_8; -goto block_16; +goto block_22; } else { -lean_object* x_286; -x_286 = lean_box(0); -x_268 = x_286; -goto block_283; +lean_object* x_350; +x_350 = lean_box(0); +x_332 = x_350; +goto block_347; } } else { -lean_object* x_287; -x_287 = lean_box(0); -x_268 = x_287; -goto block_283; +lean_object* x_351; +x_351 = lean_box(0); +x_332 = x_351; +goto block_347; } -block_283: +block_347: { -lean_object* x_269; lean_object* x_270; -lean_dec(x_268); -lean_inc(x_267); -x_269 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_267, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_270 = lean_ctor_get(x_269, 0); -lean_inc(x_270); -if (lean_obj_tag(x_270) == 0) +lean_object* x_333; lean_object* x_334; +lean_dec(x_332); +lean_inc(x_331); +x_333 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_331, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_334 = lean_ctor_get(x_333, 0); +lean_inc(x_334); +if (lean_obj_tag(x_334) == 0) { -lean_object* x_271; lean_object* x_272; -x_271 = lean_ctor_get(x_269, 1); -lean_inc(x_271); -lean_dec(x_269); +lean_object* x_335; lean_object* x_336; +x_335 = lean_ctor_get(x_333, 1); +lean_inc(x_335); +lean_dec(x_333); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_267); -x_272 = l_Lean_Meta_CheckAssignment_check(x_267, x_2, x_3, x_4, x_5, x_6, x_7, x_271); -if (lean_obj_tag(x_272) == 0) +lean_inc(x_331); +x_336 = l_Lean_Meta_CheckAssignment_check(x_331, x_2, x_3, x_4, x_5, x_6, x_7, x_335); +if (lean_obj_tag(x_336) == 0) { -lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; -x_273 = lean_ctor_get(x_272, 0); -lean_inc(x_273); -x_274 = lean_ctor_get(x_272, 1); -lean_inc(x_274); -lean_dec(x_272); -lean_inc(x_273); -x_275 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_267, x_273, x_2, x_3, x_4, x_5, x_6, x_7, x_274); +lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; +x_337 = lean_ctor_get(x_336, 0); +lean_inc(x_337); +x_338 = lean_ctor_get(x_336, 1); +lean_inc(x_338); +lean_dec(x_336); +lean_inc(x_337); +x_339 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_331, x_337, x_2, x_3, x_4, x_5, x_6, x_7, x_338); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_276 = lean_ctor_get(x_275, 1); -lean_inc(x_276); -lean_dec(x_275); -x_9 = x_273; -x_10 = x_276; -goto block_16; +x_340 = lean_ctor_get(x_339, 1); +lean_inc(x_340); +lean_dec(x_339); +x_9 = x_337; +x_10 = x_340; +goto block_22; } else { -uint8_t x_277; -lean_dec(x_267); +uint8_t x_341; +lean_dec(x_331); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -17922,59 +19888,59 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_277 = !lean_is_exclusive(x_272); -if (x_277 == 0) +x_341 = !lean_is_exclusive(x_336); +if (x_341 == 0) { -return x_272; +return x_336; } else { -lean_object* x_278; lean_object* x_279; lean_object* x_280; -x_278 = lean_ctor_get(x_272, 0); -x_279 = lean_ctor_get(x_272, 1); -lean_inc(x_279); -lean_inc(x_278); -lean_dec(x_272); -x_280 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_280, 0, x_278); -lean_ctor_set(x_280, 1, x_279); -return x_280; +lean_object* x_342; lean_object* x_343; lean_object* x_344; +x_342 = lean_ctor_get(x_336, 0); +x_343 = lean_ctor_get(x_336, 1); +lean_inc(x_343); +lean_inc(x_342); +lean_dec(x_336); +x_344 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_344, 0, x_342); +lean_ctor_set(x_344, 1, x_343); +return x_344; } } } else { -lean_object* x_281; lean_object* x_282; -lean_dec(x_267); +lean_object* x_345; lean_object* x_346; +lean_dec(x_331); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_281 = lean_ctor_get(x_269, 1); -lean_inc(x_281); -lean_dec(x_269); -x_282 = lean_ctor_get(x_270, 0); -lean_inc(x_282); -lean_dec(x_270); -x_9 = x_282; -x_10 = x_281; -goto block_16; +x_345 = lean_ctor_get(x_333, 1); +lean_inc(x_345); +lean_dec(x_333); +x_346 = lean_ctor_get(x_334, 0); +lean_inc(x_346); +lean_dec(x_334); +x_9 = x_346; +x_10 = x_345; +goto block_22; } } } case 11: { -lean_object* x_288; lean_object* x_289; uint8_t x_305; -x_288 = lean_ctor_get(x_1, 2); -lean_inc(x_288); -x_305 = l_Lean_Expr_hasExprMVar(x_288); -if (x_305 == 0) +lean_object* x_352; lean_object* x_353; uint8_t x_369; +x_352 = lean_ctor_get(x_1, 2); +lean_inc(x_352); +x_369 = l_Lean_Expr_hasExprMVar(x_352); +if (x_369 == 0) { -uint8_t x_306; -x_306 = l_Lean_Expr_hasFVar(x_288); -if (x_306 == 0) +uint8_t x_370; +x_370 = l_Lean_Expr_hasFVar(x_352); +if (x_370 == 0) { lean_dec(x_7); lean_dec(x_6); @@ -17982,74 +19948,74 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_17 = x_288; -x_18 = x_8; -goto block_24; +x_23 = x_352; +x_24 = x_8; +goto block_37; } else { -lean_object* x_307; -x_307 = lean_box(0); -x_289 = x_307; -goto block_304; +lean_object* x_371; +x_371 = lean_box(0); +x_353 = x_371; +goto block_368; } } else { -lean_object* x_308; -x_308 = lean_box(0); -x_289 = x_308; -goto block_304; +lean_object* x_372; +x_372 = lean_box(0); +x_353 = x_372; +goto block_368; } -block_304: +block_368: { -lean_object* x_290; lean_object* x_291; -lean_dec(x_289); -lean_inc(x_288); -x_290 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_288, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -x_291 = lean_ctor_get(x_290, 0); -lean_inc(x_291); -if (lean_obj_tag(x_291) == 0) +lean_object* x_354; lean_object* x_355; +lean_dec(x_353); +lean_inc(x_352); +x_354 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_findCached_x3f(x_352, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_355 = lean_ctor_get(x_354, 0); +lean_inc(x_355); +if (lean_obj_tag(x_355) == 0) { -lean_object* x_292; lean_object* x_293; -x_292 = lean_ctor_get(x_290, 1); -lean_inc(x_292); -lean_dec(x_290); +lean_object* x_356; lean_object* x_357; +x_356 = lean_ctor_get(x_354, 1); +lean_inc(x_356); +lean_dec(x_354); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -lean_inc(x_288); -x_293 = l_Lean_Meta_CheckAssignment_check(x_288, x_2, x_3, x_4, x_5, x_6, x_7, x_292); -if (lean_obj_tag(x_293) == 0) +lean_inc(x_352); +x_357 = l_Lean_Meta_CheckAssignment_check(x_352, x_2, x_3, x_4, x_5, x_6, x_7, x_356); +if (lean_obj_tag(x_357) == 0) { -lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; -x_294 = lean_ctor_get(x_293, 0); -lean_inc(x_294); -x_295 = lean_ctor_get(x_293, 1); -lean_inc(x_295); -lean_dec(x_293); -lean_inc(x_294); -x_296 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_288, x_294, x_2, x_3, x_4, x_5, x_6, x_7, x_295); +lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; +x_358 = lean_ctor_get(x_357, 0); +lean_inc(x_358); +x_359 = lean_ctor_get(x_357, 1); +lean_inc(x_359); +lean_dec(x_357); +lean_inc(x_358); +x_360 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_CheckAssignment_cache(x_352, x_358, x_2, x_3, x_4, x_5, x_6, x_7, x_359); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_297 = lean_ctor_get(x_296, 1); -lean_inc(x_297); -lean_dec(x_296); -x_17 = x_294; -x_18 = x_297; -goto block_24; +x_361 = lean_ctor_get(x_360, 1); +lean_inc(x_361); +lean_dec(x_360); +x_23 = x_358; +x_24 = x_361; +goto block_37; } else { -uint8_t x_298; -lean_dec(x_288); +uint8_t x_362; +lean_dec(x_352); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -18057,109 +20023,158 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_298 = !lean_is_exclusive(x_293); -if (x_298 == 0) +x_362 = !lean_is_exclusive(x_357); +if (x_362 == 0) { -return x_293; +return x_357; } else { -lean_object* x_299; lean_object* x_300; lean_object* x_301; -x_299 = lean_ctor_get(x_293, 0); -x_300 = lean_ctor_get(x_293, 1); -lean_inc(x_300); -lean_inc(x_299); -lean_dec(x_293); -x_301 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_301, 0, x_299); -lean_ctor_set(x_301, 1, x_300); -return x_301; +lean_object* x_363; lean_object* x_364; lean_object* x_365; +x_363 = lean_ctor_get(x_357, 0); +x_364 = lean_ctor_get(x_357, 1); +lean_inc(x_364); +lean_inc(x_363); +lean_dec(x_357); +x_365 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_365, 0, x_363); +lean_ctor_set(x_365, 1, x_364); +return x_365; } } } else { -lean_object* x_302; lean_object* x_303; -lean_dec(x_288); +lean_object* x_366; lean_object* x_367; +lean_dec(x_352); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_302 = lean_ctor_get(x_290, 1); -lean_inc(x_302); -lean_dec(x_290); -x_303 = lean_ctor_get(x_291, 0); -lean_inc(x_303); -lean_dec(x_291); -x_17 = x_303; -x_18 = x_302; -goto block_24; +x_366 = lean_ctor_get(x_354, 1); +lean_inc(x_366); +lean_dec(x_354); +x_367 = lean_ctor_get(x_355, 0); +lean_inc(x_367); +lean_dec(x_355); +x_23 = x_367; +x_24 = x_366; +goto block_37; } } } default: { -lean_object* x_309; +lean_object* x_373; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_309 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_309, 0, x_1); -lean_ctor_set(x_309, 1, x_8); -return x_309; +x_373 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_373, 0, x_1); +lean_ctor_set(x_373, 1, x_8); +return x_373; } } -block_16: +block_22: { if (lean_obj_tag(x_1) == 10) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_expr_update_mdata(x_1, x_9); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -return x_12; +lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; uint8_t x_15; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +x_13 = lean_ptr_addr(x_12); +lean_dec(x_12); +x_14 = lean_ptr_addr(x_9); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_1); +x_16 = l_Lean_Expr_mdata___override(x_11, x_9); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_10); +return x_17; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_18; +lean_dec(x_11); +lean_dec(x_9); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_1); +lean_ctor_set(x_18, 1, x_10); +return x_18; +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_9); lean_dec(x_1); -x_13 = l_Lean_Meta_CheckAssignment_check___closed__4; -x_14 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_13); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_10); -return x_15; +x_19 = l_Lean_Meta_CheckAssignment_check___closed__4; +x_20 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_19); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_10); +return x_21; } } -block_24: +block_37: { if (lean_obj_tag(x_1) == 11) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_expr_update_proj(x_1, x_17); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -return x_20; +lean_object* x_25; lean_object* x_26; lean_object* x_27; size_t x_28; size_t x_29; uint8_t x_30; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_1, 1); +lean_inc(x_26); +x_27 = lean_ctor_get(x_1, 2); +lean_inc(x_27); +x_28 = lean_ptr_addr(x_27); +lean_dec(x_27); +x_29 = lean_ptr_addr(x_23); +x_30 = lean_usize_dec_eq(x_28, x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +lean_dec(x_1); +x_31 = l_Lean_Expr_proj___override(x_25, x_26, x_23); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_24); +return x_32; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -lean_dec(x_17); +lean_object* x_33; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_23); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_1); +lean_ctor_set(x_33, 1, x_24); +return x_33; +} +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_23); lean_dec(x_1); -x_21 = l_Lean_Meta_CheckAssignment_check___closed__7; -x_22 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_21); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_18); -return x_23; +x_34 = l_Lean_Meta_CheckAssignment_check___closed__7; +x_35 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_34); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_24); +return x_36; } } } @@ -30133,7 +32148,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_CheckAssignment_checkApp(lean_object* x_1, { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Expr_getAppNumArgsAux(x_1, x_9); +x_10 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_9); x_11 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_inc(x_10); x_12 = lean_mk_array(x_10, x_11); @@ -50036,7 +52051,8 @@ return x_15; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_processAssignmentFOApproxAux(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -if (lean_obj_tag(x_3) == 5) +switch (lean_obj_tag(x_3)) { +case 5: { lean_object* x_9; lean_object* x_10; uint8_t x_11; x_9 = lean_ctor_get(x_3, 0); @@ -50155,21 +52171,31 @@ lean_ctor_set(x_34, 1, x_8); return x_34; } } -else +case 10: +{ +lean_object* x_35; +x_35 = lean_ctor_get(x_3, 1); +lean_inc(x_35); +lean_dec(x_3); +x_3 = x_35; +goto _start; +} +default: { -uint8_t x_35; lean_object* x_36; lean_object* x_37; +uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_35 = 0; -x_36 = lean_box(x_35); -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_8); -return x_37; +x_37 = 0; +x_38 = lean_box(x_37); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_8); +return x_39; +} } } } @@ -54199,7 +56225,7 @@ x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); x_14 = lean_unsigned_to_nat(0u); -x_15 = l_Lean_Expr_getAppNumArgsAux(x_1, x_14); +x_15 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_14); x_16 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_inc(x_15); x_17 = lean_mk_array(x_15, x_16); @@ -57427,7 +59453,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeurist { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_245; lean_object* x_246; lean_object* x_247; uint8_t x_248; x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_1, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_11); x_13 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_inc(x_12); x_14 = lean_mk_array(x_12, x_13); @@ -57436,7 +59462,7 @@ x_16 = lean_nat_sub(x_12, x_15); lean_dec(x_12); lean_inc(x_1); x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_14, x_16); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_2, x_11); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_11); lean_inc(x_18); x_19 = lean_mk_array(x_18, x_13); x_20 = lean_nat_sub(x_18, x_15); @@ -57525,8 +59551,6 @@ x_39 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqLeft___closed__2; x_40 = 1; lean_inc(x_9); x_41 = l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__1(x_1, x_2, x_3, x_4, x_39, x_17, x_21, x_40, x_6, x_7, x_8, x_9, x_38); -lean_dec(x_21); -lean_dec(x_17); if (lean_obj_tag(x_41) == 0) { lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; @@ -57840,8 +59864,6 @@ x_117 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqLeft___closed__2; x_118 = 1; lean_inc(x_9); x_119 = l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__1(x_1, x_2, x_3, x_4, x_117, x_17, x_21, x_118, x_6, x_7, x_8, x_9, x_116); -lean_dec(x_21); -lean_dec(x_17); if (lean_obj_tag(x_119) == 0) { lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; 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; @@ -58071,8 +60093,6 @@ x_176 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqLeft___closed__2; x_177 = 1; lean_inc(x_9); x_178 = l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__1(x_1, x_2, x_3, x_4, x_176, x_17, x_21, x_177, x_6, x_7, x_8, x_9, x_175); -lean_dec(x_21); -lean_dec(x_17); if (lean_obj_tag(x_178) == 0) { lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; @@ -58274,8 +60294,6 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); x_229 = l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__2(x_1, x_2, x_3, x_4, x_227, x_17, x_21, x_228, x_6, x_7, x_8, x_9, x_226); -lean_dec(x_21); -lean_dec(x_17); if (lean_obj_tag(x_229) == 0) { lean_object* x_230; lean_object* x_231; lean_object* x_232; uint8_t x_233; @@ -58581,8 +60599,6 @@ uint8_t x_14; lean_object* x_15; x_14 = lean_unbox(x_8); lean_dec(x_8); x_15 = l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_14, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_7); -lean_dec(x_6); return x_15; } } @@ -58593,8 +60609,6 @@ uint8_t x_14; lean_object* x_15; x_14 = lean_unbox(x_8); lean_dec(x_8); x_15 = l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_tryHeuristic___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_14, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_7); -lean_dec(x_6); return x_15; } } @@ -60467,7 +62481,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_expandDela lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_dec(x_4); x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_1, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_10); x_12 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_inc(x_11); x_13 = lean_mk_array(x_11, x_12); @@ -60824,130 +62838,6 @@ lean_dec(x_5); return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isSynthetic(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -if (lean_obj_tag(x_1) == 2) -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = l_Lean_Meta_getMVarDecl(x_7, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; uint8_t x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_ctor_get_uint8(x_9, sizeof(void*)*7); -lean_dec(x_9); -x_11 = lean_box(x_10); -if (lean_obj_tag(x_11) == 0) -{ -uint8_t x_12; -x_12 = !lean_is_exclusive(x_8); -if (x_12 == 0) -{ -lean_object* x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_8, 0); -lean_dec(x_13); -x_14 = 0; -x_15 = lean_box(x_14); -lean_ctor_set(x_8, 0, x_15); -return x_8; -} -else -{ -lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_8, 1); -lean_inc(x_16); -lean_dec(x_8); -x_17 = 0; -x_18 = lean_box(x_17); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_16); -return x_19; -} -} -else -{ -uint8_t x_20; -lean_dec(x_11); -x_20 = !lean_is_exclusive(x_8); -if (x_20 == 0) -{ -lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_8, 0); -lean_dec(x_21); -x_22 = 1; -x_23 = lean_box(x_22); -lean_ctor_set(x_8, 0, x_23); -return x_8; -} -else -{ -lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_8, 1); -lean_inc(x_24); -lean_dec(x_8); -x_25 = 1; -x_26 = lean_box(x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; -} -} -} -else -{ -uint8_t x_28; -x_28 = !lean_is_exclusive(x_8); -if (x_28 == 0) -{ -return x_8; -} -else -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_8, 0); -x_30 = lean_ctor_get(x_8, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_8); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; -} -} -} -else -{ -uint8_t x_32; lean_object* x_33; lean_object* x_34; -lean_dec(x_1); -x_32 = 0; -x_33 = lean_box(x_32); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_6); -return x_34; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isSynthetic___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isSynthetic(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_7; -} -} LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isAssignable(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: { @@ -62183,6 +64073,7 @@ 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_12 = 0; @@ -62199,6 +64090,7 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); +lean_inc(x_2); lean_inc(x_1); x_15 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); if (lean_obj_tag(x_15) == 0) @@ -62744,15 +64636,6 @@ return x_139; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqMVarSelf___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqMVarSelf(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_3); -return x_9; -} -} LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_consumeLet(lean_object* x_1) { _start: { @@ -64742,7 +66625,7 @@ else lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_dec(x_14); x_126 = lean_unsigned_to_nat(0u); -x_127 = l_Lean_Expr_getAppNumArgsAux(x_1, x_126); +x_127 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_126); x_128 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_inc(x_127); x_129 = lean_mk_array(x_127, x_128); @@ -64750,14 +66633,13 @@ x_130 = lean_unsigned_to_nat(1u); x_131 = lean_nat_sub(x_127, x_130); lean_dec(x_127); x_132 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_129, x_131); -x_133 = l_Lean_Expr_getAppNumArgsAux(x_2, x_126); +x_133 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_126); lean_inc(x_133); x_134 = lean_mk_array(x_133, x_128); x_135 = lean_nat_sub(x_133, x_130); lean_dec(x_133); x_136 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_2, x_134, x_135); x_137 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqMVarSelf(x_13, x_132, x_136, x_3, x_4, x_5, x_6, x_30); -lean_dec(x_136); if (lean_obj_tag(x_137) == 0) { uint8_t x_138; @@ -66849,7 +68731,7 @@ lean_dec(x_25); x_27 = l_Lean_Expr_constLevels_x21(x_3); x_28 = l_Lean_Expr_const___override(x_26, x_27); x_29 = lean_unsigned_to_nat(0u); -x_30 = l_Lean_Expr_getAppNumArgsAux(x_4, x_29); +x_30 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_29); x_31 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_inc(x_30); x_32 = lean_mk_array(x_30, x_31); @@ -67547,7 +69429,7 @@ x_70 = lean_ctor_get(x_65, 1); lean_inc(x_70); lean_dec(x_65); x_71 = lean_unsigned_to_nat(0u); -x_72 = l_Lean_Expr_getAppNumArgsAux(x_1, x_71); +x_72 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_71); x_73 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_inc(x_72); x_74 = lean_mk_array(x_72, x_73); @@ -67555,7 +69437,7 @@ x_75 = lean_unsigned_to_nat(1u); x_76 = lean_nat_sub(x_72, x_75); lean_dec(x_72); x_77 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_74, x_76); -x_78 = l_Lean_Expr_getAppNumArgsAux(x_2, x_71); +x_78 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_71); lean_inc(x_78); x_79 = lean_mk_array(x_78, x_73); x_80 = lean_nat_sub(x_78, x_75); @@ -67566,8 +69448,6 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); x_82 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgs(x_3, x_77, x_81, x_6, x_7, x_8, x_9, x_70); -lean_dec(x_81); -lean_dec(x_77); if (lean_obj_tag(x_82) == 0) { lean_object* x_83; lean_object* x_84; uint8_t x_85; @@ -68115,7 +69995,7 @@ else { lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; lean_object* x_48; x_36 = lean_unsigned_to_nat(0u); -x_37 = l_Lean_Expr_getAppNumArgsAux(x_1, x_36); +x_37 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_36); x_38 = l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqEtaStruct_go___closed__6; lean_inc(x_37); x_39 = lean_mk_array(x_37, x_38); @@ -68124,7 +70004,7 @@ x_41 = lean_nat_sub(x_37, x_40); lean_dec(x_37); lean_inc(x_1); x_42 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_39, x_41); -x_43 = l_Lean_Expr_getAppNumArgsAux(x_2, x_36); +x_43 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_36); lean_inc(x_43); x_44 = lean_mk_array(x_43, x_38); x_45 = lean_nat_sub(x_43, x_40); @@ -68137,8 +70017,6 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); x_48 = l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqApp___spec__2(x_8, x_9, x_42, x_46, x_47, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_46); -lean_dec(x_42); if (lean_obj_tag(x_48) == 0) { lean_object* x_49; uint8_t x_50; @@ -68328,8 +70206,6 @@ uint8_t x_11; lean_object* x_12; x_11 = lean_unbox(x_5); lean_dec(x_5); x_12 = l_Lean_Meta_checkpointDefEq___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqApp___spec__2(x_1, x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_4); -lean_dec(x_3); return x_12; } } @@ -70408,7 +72284,7 @@ x_11 = lean_ctor_get(x_8, 1); x_12 = 3; x_13 = lean_unbox(x_10); lean_dec(x_10); -x_14 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_13, x_12); +x_14 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_13, x_12); if (x_14 == 0) { uint8_t x_15; lean_object* x_16; @@ -70443,7 +72319,7 @@ lean_dec(x_8); x_21 = 3; x_22 = lean_unbox(x_19); lean_dec(x_19); -x_23 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_22, x_21); +x_23 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_22, x_21); if (x_23 == 0) { uint8_t x_24; lean_object* x_25; lean_object* x_26; @@ -83666,7 +85542,7 @@ lean_dec(x_4); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_ExprDefEq___hyg_15529_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_ExprDefEq___hyg_16302_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -83992,8 +85868,18 @@ l_Lean_Meta_isDefEqStringLit___closed__3 = _init_l_Lean_Meta_isDefEqStringLit___ lean_mark_persistent(l_Lean_Meta_isDefEqStringLit___closed__3); l_Lean_Meta_isDefEqStringLit___closed__4 = _init_l_Lean_Meta_isDefEqStringLit___closed__4(); lean_mark_persistent(l_Lean_Meta_isDefEqStringLit___closed__4); +l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__1); +l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__2); +l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__3 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__3(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___spec__2___closed__3); l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__1 = _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__1(); lean_mark_persistent(l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__1); +l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__2 = _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__2); +l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__3 = _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_isDefEqArgsFirstPass___closed__3); l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__1 = _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__1(); lean_mark_persistent(l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__1); l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__2 = _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_checkTypesAndAssign___closed__2(); @@ -84032,20 +85918,20 @@ l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_hasLetDecl lean_mark_persistent(l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_hasLetDeclsInBetween___closed__2); l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_collectLetDeclsFrom___closed__1 = _init_l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_collectLetDeclsFrom___closed__1(); lean_mark_persistent(l___private_Lean_Meta_ExprDefEq_0__Lean_Meta_mkLambdaFVarsWithLetDeps_collectLetDeclsFrom___closed__1); -l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__1 = _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__1(); -lean_mark_persistent(l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__1); -l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__2 = _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__2(); -lean_mark_persistent(l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148____closed__2); -if (builtin) {res = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4148_(lean_io_mk_world()); +l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__1 = _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__1(); +lean_mark_persistent(l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__1); +l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__2 = _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__2(); +lean_mark_persistent(l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000____closed__2); +if (builtin) {res = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5000_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Meta_CheckAssignment_checkAssignmentExceptionId = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Meta_CheckAssignment_checkAssignmentExceptionId); lean_dec_ref(res); -}l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__1 = _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__1(); -lean_mark_persistent(l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__1); -l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__2 = _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__2(); -lean_mark_persistent(l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165____closed__2); -if (builtin) {res = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_4165_(lean_io_mk_world()); +}l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__1 = _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__1(); +lean_mark_persistent(l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__1); +l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__2 = _init_l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__2(); +lean_mark_persistent(l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017____closed__2); +if (builtin) {res = l_Lean_Meta_CheckAssignment_initFn____x40_Lean_Meta_ExprDefEq___hyg_5017_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Meta_CheckAssignment_outOfScopeExceptionId = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Meta_CheckAssignment_outOfScopeExceptionId); @@ -84306,7 +86192,7 @@ l_Lean_Meta_isExprDefEqAuxImpl___closed__1 = _init_l_Lean_Meta_isExprDefEqAuxImp lean_mark_persistent(l_Lean_Meta_isExprDefEqAuxImpl___closed__1); l_Lean_Meta_isExprDefEqAuxImpl___closed__2 = _init_l_Lean_Meta_isExprDefEqAuxImpl___closed__2(); lean_mark_persistent(l_Lean_Meta_isExprDefEqAuxImpl___closed__2); -res = l_Lean_Meta_initFn____x40_Lean_Meta_ExprDefEq___hyg_15529_(lean_io_mk_world()); +res = l_Lean_Meta_initFn____x40_Lean_Meta_ExprDefEq___hyg_16302_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/ExprLens.c b/stage0/stdlib/Lean/Meta/ExprLens.c index 65fc62b1133e..091f894be499 100644 --- a/stage0/stdlib/Lean/Meta/ExprLens.c +++ b/stage0/stdlib/Lean/Meta/ExprLens.c @@ -18,12 +18,12 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_Expr LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Core_viewCoordRaw(lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___closed__5; lean_object* l_Lean_Meta_mkLetFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_viewCoordAux___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_viewBinders___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); +lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Core_numBinders(lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___rarg___lambda__3___closed__1; @@ -31,6 +31,8 @@ static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_foldAncestorsAux___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_foldlM___at_Lean_Core_viewSubexpr___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___closed__14; +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); +uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_viewSubexpr(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_foldAncestors___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -40,11 +42,14 @@ LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_foldlM___at_Lean_Core_viewSubexpr___ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_foldAncestorsAux___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__4(lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_foldAncestorsAux(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_viewCoordAux___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___spec__4(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl(lean_object*, lean_object*); static lean_object* l_Lean_Core_numBinders___rarg___closed__1; lean_object* lean_array_push(lean_object*, lean_object*); +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Core_viewBinders___rarg___lambda__3(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -78,7 +83,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_viewCoordAu LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__11___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_viewCoordAux___spec__1(lean_object*); -lean_object* l_Lean_Expr_updateProj_x21(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); static lean_object* l_Lean_Core_viewBinders___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -99,7 +103,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord__ LEAN_EXPORT lean_object* l_Lean_Core_viewSubexpr(lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_foldAncestorsAux___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_updateMData_x21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_foldAncestorsAux___spec__4(lean_object*); extern lean_object* l_Lean_instInhabitedExpr; @@ -112,7 +115,6 @@ static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg LEAN_EXPORT lean_object* l_Lean_Core_viewBinders___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_replaceSubexpr(lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_size___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__1(lean_object*); lean_object* l_Lean_SubExpr_Pos_head(lean_object*); @@ -123,6 +125,7 @@ LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_foldlM___at_Lean_Core_viewBinders___ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_viewCoordAux___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___closed__19; LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__6(lean_object*, lean_object*, lean_object*); +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_foldAncestorsAux___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -159,7 +162,7 @@ lean_object* l_Lean_throwError___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkForallFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_foldAncestorsAux___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_viewSubexpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -168,6 +171,7 @@ static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___spec__3(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Core_viewCoordRaw___rarg___closed__2; +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -182,7 +186,6 @@ static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_viewCoordAux___at___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_viewAux___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___closed__21; -lean_object* lean_expr_update_app(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLetDeclImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord(lean_object*); static lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___closed__23; @@ -382,7 +385,7 @@ static lean_object* _init_l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord_ _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateApp!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateApp!Impl", 45); return x_1; } } @@ -400,8 +403,8 @@ static lean_object* _init_l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__1; x_2 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__2; -x_3 = lean_unsigned_to_nat(1081u); -x_4 = lean_unsigned_to_nat(14u); +x_3 = lean_unsigned_to_nat(1401u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -412,33 +415,71 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord__ { if (lean_obj_tag(x_2) == 5) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_expr_update_app(x_2, x_3, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_2, 1); +lean_inc(x_8); +x_9 = lean_ptr_addr(x_7); +lean_dec(x_7); +x_10 = lean_ptr_addr(x_3); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_8); +lean_dec(x_2); +x_12 = l_Lean_Expr_app___override(x_3, x_4); +x_13 = lean_apply_2(x_6, lean_box(0), x_12); +return x_13; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +size_t x_14; size_t x_15; uint8_t x_16; +x_14 = lean_ptr_addr(x_8); +lean_dec(x_8); +x_15 = lean_ptr_addr(x_4); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_2); +x_17 = l_Lean_Expr_app___override(x_3, x_4); +x_18 = lean_apply_2(x_6, lean_box(0), x_17); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_4); +lean_dec(x_3); +x_19 = lean_apply_2(x_6, lean_box(0), x_2); +return x_19; +} +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); lean_dec(x_1); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__4; -x_12 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_11); -x_13 = lean_apply_2(x_10, lean_box(0), x_12); -return x_13; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__4; +x_23 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_22); +x_24 = lean_apply_2(x_21, lean_box(0), x_23); +return x_24; } } } @@ -522,7 +563,7 @@ static lean_object* _init_l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord_ _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateLet!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateLet!Impl", 45); return x_1; } } @@ -540,8 +581,8 @@ static lean_object* _init_l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__1; x_2 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__8___closed__1; -x_3 = lean_unsigned_to_nat(1158u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1500u); +x_4 = lean_unsigned_to_nat(22u); x_5 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__8___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -552,34 +593,97 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord__ { if (lean_obj_tag(x_2) == 8) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; size_t x_13; size_t x_14; uint8_t x_15; x_6 = lean_ctor_get(x_1, 0); lean_inc(x_6); lean_dec(x_1); x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_expr_update_let(x_2, x_3, x_5, x_4); -x_9 = lean_apply_2(x_7, lean_box(0), x_8); -return x_9; +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_ctor_get(x_2, 2); +lean_inc(x_10); +x_11 = lean_ctor_get(x_2, 3); +lean_inc(x_11); +x_12 = lean_ctor_get_uint8(x_2, sizeof(void*)*4 + 8); +x_13 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_14 = lean_ptr_addr(x_3); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_2); +x_16 = l_Lean_Expr_letE___override(x_8, x_3, x_5, x_4, x_12); +x_17 = lean_apply_2(x_7, lean_box(0), x_16); +return x_17; +} +else +{ +size_t x_18; size_t x_19; uint8_t x_20; +x_18 = lean_ptr_addr(x_10); +lean_dec(x_10); +x_19 = lean_ptr_addr(x_5); +x_20 = lean_usize_dec_eq(x_18, x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_11); +lean_dec(x_2); +x_21 = l_Lean_Expr_letE___override(x_8, x_3, x_5, x_4, x_12); +x_22 = lean_apply_2(x_7, lean_box(0), x_21); +return x_22; +} +else +{ +size_t x_23; size_t x_24; uint8_t x_25; +x_23 = lean_ptr_addr(x_11); +lean_dec(x_11); +x_24 = lean_ptr_addr(x_4); +x_25 = lean_usize_dec_eq(x_23, x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +lean_dec(x_2); +x_26 = l_Lean_Expr_letE___override(x_8, x_3, x_5, x_4, x_12); +x_27 = lean_apply_2(x_7, lean_box(0), x_26); +return x_27; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_28; +lean_dec(x_8); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_28 = lean_apply_2(x_7, lean_box(0), x_2); +return x_28; +} +} +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +x_29 = lean_ctor_get(x_1, 0); +lean_inc(x_29); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__8___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = lean_apply_2(x_11, lean_box(0), x_13); -return x_14; +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +x_31 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__8___closed__3; +x_32 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_31); +x_33 = lean_apply_2(x_30, lean_box(0), x_32); +return x_33; } } } @@ -588,33 +692,71 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord__ { if (lean_obj_tag(x_2) == 5) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_expr_update_app(x_2, x_4, x_3); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_2, 1); +lean_inc(x_8); +x_9 = lean_ptr_addr(x_7); +lean_dec(x_7); +x_10 = lean_ptr_addr(x_4); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_8); +lean_dec(x_2); +x_12 = l_Lean_Expr_app___override(x_4, x_3); +x_13 = lean_apply_2(x_6, lean_box(0), x_12); +return x_13; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +size_t x_14; size_t x_15; uint8_t x_16; +x_14 = lean_ptr_addr(x_8); +lean_dec(x_8); +x_15 = lean_ptr_addr(x_3); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_2); +x_17 = l_Lean_Expr_app___override(x_4, x_3); +x_18 = lean_apply_2(x_6, lean_box(0), x_17); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_4); +lean_dec(x_3); +x_19 = lean_apply_2(x_6, lean_box(0), x_2); +return x_19; +} +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); lean_dec(x_1); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__4; -x_12 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_11); -x_13 = lean_apply_2(x_10, lean_box(0), x_12); -return x_13; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__4; +x_23 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_22); +x_24 = lean_apply_2(x_21, lean_box(0), x_23); +return x_24; } } } @@ -640,8 +782,8 @@ static lean_object* _init_l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__1; x_2 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__10___closed__1; -x_3 = lean_unsigned_to_nat(1149u); -x_4 = lean_unsigned_to_nat(19u); +x_3 = lean_unsigned_to_nat(1491u); +x_4 = lean_unsigned_to_nat(20u); x_5 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__10___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -652,34 +794,93 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord__ { if (lean_obj_tag(x_2) == 6) { -lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; +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; size_t x_12; size_t x_13; uint8_t x_14; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_8 = lean_expr_update_lambda(x_2, x_7, x_4, x_3); -x_9 = lean_apply_2(x_6, lean_box(0), x_8); -return x_9; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_2, 1); +lean_inc(x_8); +x_9 = lean_ctor_get(x_2, 2); +lean_inc(x_9); +x_10 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_11 = l_Lean_Expr_lam___override(x_7, x_8, x_9, x_10); +x_12 = lean_ptr_addr(x_8); +lean_dec(x_8); +x_13 = lean_ptr_addr(x_4); +x_14 = lean_usize_dec_eq(x_12, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_11); +lean_dec(x_9); +x_15 = l_Lean_Expr_lam___override(x_7, x_4, x_3, x_10); +x_16 = lean_apply_2(x_6, lean_box(0), x_15); +return x_16; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +size_t x_17; size_t x_18; uint8_t x_19; +x_17 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_18 = lean_ptr_addr(x_3); +x_19 = lean_usize_dec_eq(x_17, x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +lean_dec(x_11); +x_20 = l_Lean_Expr_lam___override(x_7, x_4, x_3, x_10); +x_21 = lean_apply_2(x_6, lean_box(0), x_20); +return x_21; +} +else +{ +uint8_t x_22; +x_22 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_10, x_10); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_11); +x_23 = l_Lean_Expr_lam___override(x_7, x_4, x_3, x_10); +x_24 = lean_apply_2(x_6, lean_box(0), x_23); +return x_24; +} +else +{ +lean_object* x_25; +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +x_25 = lean_apply_2(x_6, lean_box(0), x_11); +return x_25; +} +} +} +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__10___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = lean_apply_2(x_11, lean_box(0), x_13); -return x_14; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__10___closed__3; +x_29 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_28); +x_30 = lean_apply_2(x_27, lean_box(0), x_29); +return x_30; } } } @@ -705,8 +906,8 @@ static lean_object* _init_l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__3___closed__1; x_2 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__11___closed__1; -x_3 = lean_unsigned_to_nat(1135u); -x_4 = lean_unsigned_to_nat(23u); +x_3 = lean_unsigned_to_nat(1471u); +x_4 = lean_unsigned_to_nat(24u); x_5 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__11___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -717,34 +918,93 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord__ { if (lean_obj_tag(x_2) == 7) { -lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; +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; size_t x_12; size_t x_13; uint8_t x_14; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_8 = lean_expr_update_forall(x_2, x_7, x_4, x_3); -x_9 = lean_apply_2(x_6, lean_box(0), x_8); -return x_9; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_2, 1); +lean_inc(x_8); +x_9 = lean_ctor_get(x_2, 2); +lean_inc(x_9); +x_10 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_11 = l_Lean_Expr_forallE___override(x_7, x_8, x_9, x_10); +x_12 = lean_ptr_addr(x_8); +lean_dec(x_8); +x_13 = lean_ptr_addr(x_4); +x_14 = lean_usize_dec_eq(x_12, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_11); +lean_dec(x_9); +x_15 = l_Lean_Expr_forallE___override(x_7, x_4, x_3, x_10); +x_16 = lean_apply_2(x_6, lean_box(0), x_15); +return x_16; +} +else +{ +size_t x_17; size_t x_18; uint8_t x_19; +x_17 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_18 = lean_ptr_addr(x_3); +x_19 = lean_usize_dec_eq(x_17, x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +lean_dec(x_11); +x_20 = l_Lean_Expr_forallE___override(x_7, x_4, x_3, x_10); +x_21 = lean_apply_2(x_6, lean_box(0), x_20); +return x_21; +} +else +{ +uint8_t x_22; +x_22 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_10, x_10); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_11); +x_23 = l_Lean_Expr_forallE___override(x_7, x_4, x_3, x_10); +x_24 = lean_apply_2(x_6, lean_box(0), x_23); +return x_24; +} +else +{ +lean_object* x_25; +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +x_25 = lean_apply_2(x_6, lean_box(0), x_11); +return x_25; +} +} +} } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__11___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = lean_apply_2(x_11, lean_box(0), x_13); -return x_14; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__11___closed__3; +x_29 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_28); +x_30 = lean_apply_2(x_27, lean_box(0), x_29); +return x_30; } } } @@ -753,34 +1013,97 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord__ { if (lean_obj_tag(x_2) == 8) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; size_t x_13; size_t x_14; uint8_t x_15; x_6 = lean_ctor_get(x_1, 0); lean_inc(x_6); lean_dec(x_1); x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_expr_update_let(x_2, x_5, x_3, x_4); -x_9 = lean_apply_2(x_7, lean_box(0), x_8); -return x_9; +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_ctor_get(x_2, 2); +lean_inc(x_10); +x_11 = lean_ctor_get(x_2, 3); +lean_inc(x_11); +x_12 = lean_ctor_get_uint8(x_2, sizeof(void*)*4 + 8); +x_13 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_14 = lean_ptr_addr(x_5); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_2); +x_16 = l_Lean_Expr_letE___override(x_8, x_5, x_3, x_4, x_12); +x_17 = lean_apply_2(x_7, lean_box(0), x_16); +return x_17; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +size_t x_18; size_t x_19; uint8_t x_20; +x_18 = lean_ptr_addr(x_10); +lean_dec(x_10); +x_19 = lean_ptr_addr(x_3); +x_20 = lean_usize_dec_eq(x_18, x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_11); +lean_dec(x_2); +x_21 = l_Lean_Expr_letE___override(x_8, x_5, x_3, x_4, x_12); +x_22 = lean_apply_2(x_7, lean_box(0), x_21); +return x_22; +} +else +{ +size_t x_23; size_t x_24; uint8_t x_25; +x_23 = lean_ptr_addr(x_11); +lean_dec(x_11); +x_24 = lean_ptr_addr(x_4); +x_25 = lean_usize_dec_eq(x_23, x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +lean_dec(x_2); +x_26 = l_Lean_Expr_letE___override(x_8, x_5, x_3, x_4, x_12); +x_27 = lean_apply_2(x_7, lean_box(0), x_26); +return x_27; +} +else +{ +lean_object* x_28; +lean_dec(x_8); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_28 = lean_apply_2(x_7, lean_box(0), x_2); +return x_28; +} +} +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +x_29 = lean_ctor_get(x_1, 0); +lean_inc(x_29); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__8___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = lean_apply_2(x_11, lean_box(0), x_13); -return x_14; +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +x_31 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg___lambda__8___closed__3; +x_32 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_31); +x_33 = lean_apply_2(x_30, lean_box(0), x_32); +return x_33; } } } @@ -1047,7 +1370,7 @@ lean_dec(x_17); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); lean_dec(x_18); -x_20 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_20 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_20, 0, x_7); x_21 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_16); x_22 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_20, x_21); @@ -1101,7 +1424,7 @@ lean_dec(x_36); x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); lean_dec(x_37); -x_39 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_39 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_39, 0, x_7); x_40 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg(x_1, x_2, x_3, x_4, x_5, x_14, x_35); x_41 = lean_apply_4(x_38, lean_box(0), lean_box(0), x_39, x_40); @@ -1159,7 +1482,7 @@ lean_dec(x_51); x_53 = lean_ctor_get(x_52, 0); lean_inc(x_53); lean_dec(x_52); -x_54 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_54 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_54, 0, x_7); x_55 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg(x_1, x_2, x_3, x_4, x_5, x_12, x_50); x_56 = lean_apply_4(x_53, lean_box(0), lean_box(0), x_54, x_55); @@ -1289,7 +1612,7 @@ lean_dec(x_89); x_91 = lean_ctor_get(x_90, 0); lean_inc(x_91); lean_dec(x_90); -x_92 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_92 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_92, 0, x_7); x_93 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg(x_1, x_2, x_3, x_4, x_5, x_10, x_88); x_94 = lean_apply_4(x_91, lean_box(0), lean_box(0), x_92, x_93); @@ -1417,7 +1740,7 @@ lean_dec(x_127); x_129 = lean_ctor_get(x_128, 0); lean_inc(x_129); lean_dec(x_128); -x_130 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_130 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_130, 0, x_7); x_131 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___rarg(x_1, x_2, x_3, x_4, x_5, x_8, x_126); x_132 = lean_apply_4(x_129, lean_box(0), lean_box(0), x_130, x_131); @@ -1440,7 +1763,7 @@ lean_dec(x_134); x_136 = lean_ctor_get(x_135, 0); lean_inc(x_136); lean_dec(x_135); -x_137 = lean_alloc_closure((void*)(l_Lean_Expr_updateProj_x21), 2, 1); +x_137 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl), 2, 1); lean_closure_set(x_137, 0, x_7); x_138 = lean_apply_1(x_5, x_133); x_139 = lean_apply_4(x_136, lean_box(0), lean_box(0), x_137, x_138); @@ -1665,7 +1988,7 @@ lean_dec(x_17); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); lean_dec(x_18); -x_20 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_20 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_20, 0, x_7); x_21 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_16); x_22 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_20, x_21); @@ -1719,7 +2042,7 @@ lean_dec(x_36); x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); lean_dec(x_37); -x_39 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_39 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_39, 0, x_7); x_40 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_14, x_35); x_41 = lean_apply_4(x_38, lean_box(0), lean_box(0), x_39, x_40); @@ -1777,7 +2100,7 @@ lean_dec(x_51); x_53 = lean_ctor_get(x_52, 0); lean_inc(x_53); lean_dec(x_52); -x_54 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_54 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_54, 0, x_7); x_55 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_12, x_50); x_56 = lean_apply_4(x_53, lean_box(0), lean_box(0), x_54, x_55); @@ -1907,7 +2230,7 @@ lean_dec(x_89); x_91 = lean_ctor_get(x_90, 0); lean_inc(x_91); lean_dec(x_90); -x_92 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_92 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_92, 0, x_7); x_93 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_10, x_88); x_94 = lean_apply_4(x_91, lean_box(0), lean_box(0), x_92, x_93); @@ -2035,7 +2358,7 @@ lean_dec(x_127); x_129 = lean_ctor_get(x_128, 0); lean_inc(x_129); lean_dec(x_128); -x_130 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_130 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_130, 0, x_7); x_131 = l___private_Lean_Meta_ExprLens_0__Lean_Meta_lensCoord___at___private_Lean_Meta_ExprLens_0__Lean_Meta_lensAux___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_8, x_126); x_132 = lean_apply_4(x_129, lean_box(0), lean_box(0), x_130, x_131); @@ -2058,7 +2381,7 @@ lean_dec(x_134); x_136 = lean_ctor_get(x_135, 0); lean_inc(x_136); lean_dec(x_135); -x_137 = lean_alloc_closure((void*)(l_Lean_Expr_updateProj_x21), 2, 1); +x_137 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl), 2, 1); lean_closure_set(x_137, 0, x_7); x_138 = lean_apply_1(x_5, x_133); x_139 = lean_apply_4(x_136, lean_box(0), lean_box(0), x_137, x_138); diff --git a/stage0/stdlib/Lean/Meta/ExprTraverse.c b/stage0/stdlib/Lean/Meta/ExprTraverse.c index adc83d682048..60640d0c0c20 100644 --- a/stage0/stdlib/Lean/Meta/ExprTraverse.c +++ b/stage0/stdlib/Lean/Meta/ExprTraverse.c @@ -29,9 +29,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprTraverse_0__Lean_Meta_forgetP lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_traverseForallWithPos_visit___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_traverseLambdaWithPos_visit___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ExprTraverse_0__Lean_Meta_forgetPos(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_traverseForallWithPos_visit(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_traverseLambdaWithPos(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); extern lean_object* l_Lean_SubExpr_Pos_root; LEAN_EXPORT lean_object* l_Lean_Meta_traverseLambdaWithPos_visit(lean_object*); @@ -45,10 +47,8 @@ LEAN_EXPORT lean_object* l_Lean_Meta_traverseLambda(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_traverseLambdaWithPos_visit___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_traverseLambdaWithPos___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_traverseLetWithPos___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_updateProj_x21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_traverseChildren(lean_object*); lean_object* l_Lean_Expr_traverseAppWithPos___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_updateMData_x21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_traverseLambdaWithPos_visit___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Meta_traverseLetWithPos_visit___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_traverseLetWithPos_visit___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*); @@ -763,7 +763,7 @@ lean_dec(x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); lean_dec(x_13); -x_15 = lean_alloc_closure((void*)(l_Lean_Expr_updateMData_x21), 2, 1); +x_15 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateMData_x21Impl), 2, 1); lean_closure_set(x_15, 0, x_6); x_16 = lean_apply_2(x_4, x_5, x_11); x_17 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_15, x_16); @@ -785,7 +785,7 @@ lean_dec(x_19); x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); lean_dec(x_20); -x_22 = lean_alloc_closure((void*)(l_Lean_Expr_updateProj_x21), 2, 1); +x_22 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateProj_x21Impl), 2, 1); lean_closure_set(x_22, 0, x_6); x_23 = lean_unsigned_to_nat(0u); x_24 = l_Lean_SubExpr_Pos_push(x_5, x_23); diff --git a/stage0/stdlib/Lean/Meta/ForEachExpr.c b/stage0/stdlib/Lean/Meta/ForEachExpr.c index 0d081aee5057..db0eddf3c62f 100644 --- a/stage0/stdlib/Lean/Meta/ForEachExpr.c +++ b/stage0/stdlib/Lean/Meta/ForEachExpr.c @@ -58,6 +58,7 @@ lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_setMVarUserNamesAt___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); uint64_t l_Lean_Expr_hash(lean_object*); @@ -77,7 +78,6 @@ static lean_object* l_Lean_Meta_ForEachExpr_visit___closed__1; lean_object* l_Lean_MetavarContext_setMVarUserNameTemporarily(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_ForEachExpr_0__Lean_Meta_ForEachExpr_visitBinder___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_resetMVarUserNames___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_setMVarUserNamesAt___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_setMVarUserNamesAt___spec__4___closed__1; uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -2561,7 +2561,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Meta_setMVarUserNames lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Meta_setMVarUserNamesAt___spec__4___closed__2; x_2 = l_Std_Range_forIn_loop___at_Lean_Meta_setMVarUserNamesAt___spec__4___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Meta_setMVarUserNamesAt___spec__4___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2874,7 +2874,7 @@ else { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Lean_Expr_getAppNumArgsAux(x_3, x_12); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_12); x_14 = l_Lean_Meta_setMVarUserNamesAt___lambda__1___closed__1; lean_inc(x_13); x_15 = lean_mk_array(x_13, x_14); diff --git a/stage0/stdlib/Lean/Meta/FunInfo.c b/stage0/stdlib/Lean/Meta/FunInfo.c index 6f5da550305c..b22a0d254f79 100644 --- a/stage0/stdlib/Lean/Meta/FunInfo.c +++ b/stage0/stdlib/Lean/Meta/FunInfo.c @@ -16,6 +16,7 @@ extern "C" { LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_whenHasVar___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__1(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Meta_TransparencyMode_hash(uint8_t); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -29,6 +30,7 @@ lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___ size_t lean_usize_sub(size_t, size_t); lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* l_Nat_decLt___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___closed__1; extern lean_object* l_instInhabitedNat; uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1; @@ -36,93 +38,125 @@ LEAN_EXPORT lean_object* l_Array_contains___at___private_Lean_Meta_FunInfo_0__Le lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* l_Std_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); +lean_object* l_Lean_Meta_isClass_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getFunInfo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__2; lean_object* l_Array_qpartition_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_right(size_t, size_t); -LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l_Lean_levelZero; lean_object* lean_nat_add(lean_object*, lean_object*); static size_t l_Std_PersistentHashMap_findAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__2___closed__1; -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__4; size_t lean_uint64_to_usize(uint64_t); static size_t l_Std_PersistentHashMap_findAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__2___closed__2; +lean_object* l_Lean_Expr_FindImpl_findUnsafe_x3f(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__2(lean_object*, lean_object*); +lean_object* l_Std_RBNode_setBlack___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8(lean_object*); lean_object* lean_array_swap(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_fvarId_x21(lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Std_RBNode_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); +LEAN_EXPORT lean_object* l_Std_RBNode_findCore___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__6(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Expr_hash(lean_object*); +lean_object* l_Lean_Expr_sort___override(lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__1; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__5___closed__1; size_t lean_usize_shift_left(size_t, size_t); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__2; lean_object* l_Lean_Meta_InfoCacheKey_instHashableInfoCacheKey___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_indexOfAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__1___boxed(lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__3; +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__2___boxed(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Array_isEmpty___rarg(lean_object*); size_t lean_usize_mul(size_t, size_t); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__1; -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__2; -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__2; -uint8_t l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__1; +extern lean_object* l_Lean_Meta_instMonadMetaM; +uint8_t l_Lean_Expr_isForall(lean_object*); +lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_whenHasVar___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___closed__1; size_t lean_usize_land(size_t, size_t); +lean_object* l_Lean_getOutParamPositions_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); static lean_object* l_Array_qsort_sort___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__3(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(lean_object*, lean_object*); static lean_object* l_Std_PersistentHashMap_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__4___closed__1; -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_le(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_whenHasVar(lean_object*); +uint8_t l_Std_RBNode_isRed___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_FunInfo_getArity___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_RBNode_findCore___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getFunInfoNArgs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isFVar(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_FunInfo_getArity(lean_object*); lean_object* l_Lean_Meta_getTransparency(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_array(lean_object*, lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__2(lean_object*, size_t, lean_object*); -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__3; LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__5; lean_object* lean_usize_to_nat(size_t); lean_object* l_Lean_Meta_isProp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasFVar(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2___rarg(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___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_indexOfAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps___boxed(lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__4(lean_object*, lean_object*, lean_object*); +lean_object* l_instMonadControlT__1___rarg(lean_object*); lean_object* l_Std_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__1; lean_object* l_Lean_Meta_getFVarLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: @@ -142,7 +176,7 @@ else { lean_object* x_9; uint8_t x_10; x_9 = lean_array_fget(x_1, x_4); -x_10 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(x_5, x_9); +x_10 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(x_5, x_9); lean_dec(x_9); if (x_10 == 0) { @@ -212,7 +246,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_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(x_3, x_11); +x_13 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(x_3, x_11); lean_dec(x_11); if (x_13 == 0) { @@ -423,7 +457,7 @@ else { lean_object* x_17; uint8_t x_18; x_17 = lean_array_fget(x_5, x_2); -x_18 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(x_3, x_17); +x_18 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(x_3, x_17); lean_dec(x_17); if (x_18 == 0) { @@ -520,7 +554,7 @@ if (x_18 == 0) lean_object* x_19; lean_object* x_20; uint8_t x_21; x_19 = lean_ctor_get(x_15, 0); x_20 = lean_ctor_get(x_15, 1); -x_21 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(x_4, x_19); +x_21 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(x_4, x_19); if (x_21 == 0) { lean_object* x_22; lean_object* x_23; lean_object* x_24; @@ -554,7 +588,7 @@ x_27 = lean_ctor_get(x_15, 1); lean_inc(x_27); lean_inc(x_26); lean_dec(x_15); -x_28 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(x_4, x_26); +x_28 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(x_4, x_26); if (x_28 == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; @@ -675,7 +709,7 @@ if (lean_is_exclusive(x_57)) { lean_dec_ref(x_57); x_62 = lean_box(0); } -x_63 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344_(x_4, x_60); +x_63 = l___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364_(x_4, x_60); if (x_63 == 0) { lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; @@ -962,34 +996,34 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfo _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_9 = lean_st_ref_get(x_7, x_8); -x_10 = lean_ctor_get(x_9, 1); +x_9 = l_Lean_Meta_getTransparency(x_4, x_5, x_6, x_7, x_8); +x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); lean_dec(x_9); -x_11 = lean_st_ref_get(x_5, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); +x_12 = lean_st_ref_get(x_7, x_11); +x_13 = lean_ctor_get(x_12, 1); lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Meta_getTransparency(x_4, x_5, x_6, x_7, x_13); +lean_dec(x_12); +x_14 = lean_st_ref_get(x_5, x_13); x_15 = !lean_is_exclusive(x_14); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; x_16 = lean_ctor_get(x_14, 0); x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_12, 1); +x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); -lean_dec(x_12); +lean_dec(x_16); x_19 = lean_ctor_get(x_18, 1); lean_inc(x_19); lean_dec(x_18); x_20 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_20, 0, x_1); lean_ctor_set(x_20, 1, x_2); -x_21 = lean_unbox(x_16); -lean_dec(x_16); +x_21 = lean_unbox(x_10); +lean_dec(x_10); lean_ctor_set_uint8(x_20, sizeof(void*)*2, x_21); lean_inc(x_20); x_22 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__1(x_19, x_20); @@ -1237,17 +1271,17 @@ x_79 = lean_ctor_get(x_14, 1); lean_inc(x_79); lean_inc(x_78); lean_dec(x_14); -x_80 = lean_ctor_get(x_12, 1); +x_80 = lean_ctor_get(x_78, 1); lean_inc(x_80); -lean_dec(x_12); +lean_dec(x_78); x_81 = lean_ctor_get(x_80, 1); lean_inc(x_81); lean_dec(x_80); x_82 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_82, 0, x_1); lean_ctor_set(x_82, 1, x_2); -x_83 = lean_unbox(x_78); -lean_dec(x_78); +x_83 = lean_unbox(x_10); +lean_dec(x_10); lean_ctor_set_uint8(x_82, sizeof(void*)*2, x_83); lean_inc(x_82); x_84 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__1(x_81, x_82); @@ -1986,7 +2020,7 @@ x_8 = lean_unsigned_to_nat(0u); x_9 = lean_nat_dec_eq(x_4, x_8); if (x_9 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; uint8_t x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; lean_object* x_18; +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; uint8_t x_14; lean_object* x_15; uint8_t x_16; uint8_t x_17; uint8_t x_18; uint8_t x_19; lean_object* x_20; x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_sub(x_4, x_10); lean_dec(x_4); @@ -1997,71 +2031,75 @@ x_15 = lean_ctor_get(x_12, 0); lean_inc(x_15); x_16 = lean_ctor_get_uint8(x_12, sizeof(void*)*1 + 2); x_17 = lean_ctor_get_uint8(x_12, sizeof(void*)*1 + 3); -x_18 = lean_nat_add(x_5, x_10); +x_18 = lean_ctor_get_uint8(x_12, sizeof(void*)*1 + 4); +x_19 = lean_ctor_get_uint8(x_12, sizeof(void*)*1 + 5); +x_20 = lean_nat_add(x_5, x_10); if (x_14 == 0) { -uint8_t x_19; -x_19 = l_Array_contains___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__2(x_2, x_5); +uint8_t x_21; +x_21 = l_Array_contains___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__2(x_2, x_5); lean_dec(x_5); -if (x_19 == 0) +if (x_21 == 0) { -lean_object* x_20; +lean_object* x_22; lean_dec(x_15); -x_20 = lean_array_push(x_7, x_12); +x_22 = lean_array_push(x_7, x_12); x_4 = x_11; -x_5 = x_18; +x_5 = x_20; x_6 = lean_box(0); -x_7 = x_20; +x_7 = x_22; goto _start; } else { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_12); -if (x_22 == 0) +uint8_t x_24; +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) { -lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_12, 0); -lean_dec(x_23); -x_24 = 1; -lean_ctor_set_uint8(x_12, sizeof(void*)*1 + 1, x_24); -x_25 = lean_array_push(x_7, x_12); +lean_object* x_25; uint8_t x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_12, 0); +lean_dec(x_25); +x_26 = 1; +lean_ctor_set_uint8(x_12, sizeof(void*)*1 + 1, x_26); +x_27 = lean_array_push(x_7, x_12); x_4 = x_11; -x_5 = x_18; +x_5 = x_20; x_6 = lean_box(0); -x_7 = x_25; +x_7 = x_27; goto _start; } else { -uint8_t x_27; lean_object* x_28; lean_object* x_29; +uint8_t x_29; lean_object* x_30; lean_object* x_31; lean_dec(x_12); -x_27 = 1; -x_28 = lean_alloc_ctor(0, 1, 4); -lean_ctor_set(x_28, 0, x_15); -lean_ctor_set_uint8(x_28, sizeof(void*)*1, x_13); -lean_ctor_set_uint8(x_28, sizeof(void*)*1 + 1, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*1 + 2, x_16); -lean_ctor_set_uint8(x_28, sizeof(void*)*1 + 3, x_17); -x_29 = lean_array_push(x_7, x_28); +x_29 = 1; +x_30 = lean_alloc_ctor(0, 1, 6); +lean_ctor_set(x_30, 0, x_15); +lean_ctor_set_uint8(x_30, sizeof(void*)*1, x_13); +lean_ctor_set_uint8(x_30, sizeof(void*)*1 + 1, x_29); +lean_ctor_set_uint8(x_30, sizeof(void*)*1 + 2, x_16); +lean_ctor_set_uint8(x_30, sizeof(void*)*1 + 3, x_17); +lean_ctor_set_uint8(x_30, sizeof(void*)*1 + 4, x_18); +lean_ctor_set_uint8(x_30, sizeof(void*)*1 + 5, x_19); +x_31 = lean_array_push(x_7, x_30); x_4 = x_11; -x_5 = x_18; +x_5 = x_20; x_6 = lean_box(0); -x_7 = x_29; +x_7 = x_31; goto _start; } } } else { -lean_object* x_31; +lean_object* x_33; lean_dec(x_15); lean_dec(x_5); -x_31 = lean_array_push(x_7, x_12); +x_33 = lean_array_push(x_7, x_12); x_4 = x_11; -x_5 = x_18; +x_5 = x_20; x_6 = lean_box(0); -x_7 = x_31; +x_7 = x_33; goto _start; } } @@ -2117,483 +2155,4598 @@ lean_dec(x_1); return x_3; } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__1() { +LEAN_EXPORT lean_object* l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Decidable", 9); -return x_1; -} -} -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__2() { -_start: +if (lean_obj_tag(x_1) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +lean_object* x_4; uint8_t x_5; lean_object* x_6; +x_4 = lean_box(0); +x_5 = 0; +x_6 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_6, 0, x_4); +lean_ctor_set(x_6, 1, x_2); +lean_ctor_set(x_6, 2, x_3); +lean_ctor_set(x_6, 3, x_4); +lean_ctor_set_uint8(x_6, sizeof(void*)*4, x_5); +return x_6; } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -lean_object* x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; -x_8 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__2; -x_9 = l_Lean_Expr_isAppOf(x_2, x_8); -x_10 = lean_box(x_9); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_7); -return x_11; -} -} -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__1() { -_start: +uint8_t x_7; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +if (x_7 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Init.Util", 9); +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_9 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 1); +x_11 = lean_ctor_get(x_1, 2); +x_12 = lean_ctor_get(x_1, 3); +x_13 = l_Lean_Name_quickCmp(x_2, x_10); +switch (x_13) { +case 0: +{ +lean_object* x_14; uint8_t x_15; +x_14 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_9, x_2, x_3); +x_15 = 0; +lean_ctor_set(x_1, 0, x_14); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_15); return x_1; } -} -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__2() { -_start: +case 1: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("getElem!", 8); +uint8_t x_16; +lean_dec(x_11); +lean_dec(x_10); +x_16 = 0; +lean_ctor_set(x_1, 2, x_3); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_16); return x_1; } -} -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__3() { -_start: +default: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("index out of bounds", 19); +lean_object* x_17; uint8_t x_18; +x_17 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_12, x_2, x_3); +x_18 = 0; +lean_ctor_set(x_1, 3, x_17); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_18); return x_1; } } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__4() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__1; -x_2 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); -x_4 = lean_unsigned_to_nat(36u); -x_5 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__3; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_19 = lean_ctor_get(x_1, 0); +x_20 = lean_ctor_get(x_1, 1); +x_21 = lean_ctor_get(x_1, 2); +x_22 = lean_ctor_get(x_1, 3); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_1); +x_23 = l_Lean_Name_quickCmp(x_2, x_20); +switch (x_23) { +case 0: +{ +lean_object* x_24; uint8_t x_25; lean_object* x_26; +x_24 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_19, x_2, x_3); +x_25 = 0; +x_26 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_20); +lean_ctor_set(x_26, 2, x_21); +lean_ctor_set(x_26, 3, x_22); +lean_ctor_set_uint8(x_26, sizeof(void*)*4, x_25); +return x_26; } +case 1: +{ +uint8_t x_27; lean_object* x_28; +lean_dec(x_21); +lean_dec(x_20); +x_27 = 0; +x_28 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_28, 0, x_19); +lean_ctor_set(x_28, 1, x_2); +lean_ctor_set(x_28, 2, x_3); +lean_ctor_set(x_28, 3, x_22); +lean_ctor_set_uint8(x_28, sizeof(void*)*4, x_27); +return x_28; } -static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__5() { -_start: +default: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___boxed), 7, 0); -return x_1; +lean_object* x_29; uint8_t x_30; lean_object* x_31; +x_29 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_22, x_2, x_3); +x_30 = 0; +x_31 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_31, 0, x_19); +lean_ctor_set(x_31, 1, x_20); +lean_ctor_set(x_31, 2, x_21); +lean_ctor_set(x_31, 3, x_29); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +return x_31; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +} +} +else { -uint8_t x_13; -x_13 = lean_nat_dec_le(x_5, x_4); -if (x_13 == 0) +uint8_t x_32; +x_32 = !lean_is_exclusive(x_1); +if (x_32 == 0) { -lean_object* x_14; uint8_t x_15; -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_nat_dec_eq(x_3, x_14); -if (x_15 == 0) +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_33 = lean_ctor_get(x_1, 0); +x_34 = lean_ctor_get(x_1, 1); +x_35 = lean_ctor_get(x_1, 2); +x_36 = lean_ctor_get(x_1, 3); +x_37 = l_Lean_Name_quickCmp(x_2, x_34); +switch (x_37) { +case 0: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_24; -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_sub(x_3, x_16); -lean_dec(x_3); -x_24 = lean_nat_dec_lt(x_4, x_2); -if (x_24 == 0) +uint8_t x_38; +x_38 = l_Std_RBNode_isRed___rarg(x_33); +if (x_38 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__4; -x_26 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_25); -lean_inc(x_8); -x_27 = l_Lean_Meta_getFVarLocalDecl(x_26, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_27) == 0) +lean_object* x_39; uint8_t x_40; +x_39 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_33, x_2, x_3); +x_40 = 1; +lean_ctor_set(x_1, 0, x_39); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_40); +return x_1; +} +else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = l_Lean_LocalDecl_type(x_28); -lean_inc(x_30); -lean_inc(x_1); -x_31 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(x_1, x_30); -x_32 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(x_7, x_31); -lean_dec(x_7); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_30); -x_33 = l_Lean_Meta_isProp(x_30, x_8, x_9, x_10, x_11, x_29); -if (lean_obj_tag(x_33) == 0) +lean_object* x_41; lean_object* x_42; +x_41 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_33, x_2, x_3); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__5; -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_37 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_30, x_36, x_8, x_9, x_10, x_11, x_35); -if (lean_obj_tag(x_37) == 0) +lean_object* x_43; +x_43 = lean_ctor_get(x_41, 3); +lean_inc(x_43); +if (lean_obj_tag(x_43) == 0) { -lean_object* x_38; lean_object* x_39; uint8_t x_40; uint8_t x_41; lean_object* x_42; uint8_t x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_37, 1); -lean_inc(x_39); -lean_dec(x_37); -x_40 = l_Lean_LocalDecl_binderInfo(x_28); -lean_dec(x_28); -x_41 = 0; -x_42 = lean_alloc_ctor(0, 1, 4); -lean_ctor_set(x_42, 0, x_31); -lean_ctor_set_uint8(x_42, sizeof(void*)*1, x_40); -lean_ctor_set_uint8(x_42, sizeof(void*)*1 + 1, x_41); -x_43 = lean_unbox(x_34); -lean_dec(x_34); -lean_ctor_set_uint8(x_42, sizeof(void*)*1 + 2, x_43); -x_44 = lean_unbox(x_38); -lean_dec(x_38); -lean_ctor_set_uint8(x_42, sizeof(void*)*1 + 3, x_44); -x_45 = lean_array_push(x_32, x_42); -x_46 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_46, 0, x_45); -x_18 = x_46; -x_19 = x_39; -goto block_23; +uint8_t x_44; +x_44 = !lean_is_exclusive(x_41); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; +x_45 = lean_ctor_get(x_41, 3); +lean_dec(x_45); +x_46 = lean_ctor_get(x_41, 0); +lean_dec(x_46); +x_47 = 0; +lean_ctor_set(x_41, 0, x_43); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_47); +x_48 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_48); +return x_1; } else { -uint8_t x_47; -lean_dec(x_34); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_28); -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_4); -lean_dec(x_1); -x_47 = !lean_is_exclusive(x_37); -if (x_47 == 0) +lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; uint8_t x_53; +x_49 = lean_ctor_get(x_41, 1); +x_50 = lean_ctor_get(x_41, 2); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_41); +x_51 = 0; +x_52 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_52, 0, x_43); +lean_ctor_set(x_52, 1, x_49); +lean_ctor_set(x_52, 2, x_50); +lean_ctor_set(x_52, 3, x_43); +lean_ctor_set_uint8(x_52, sizeof(void*)*4, x_51); +x_53 = 1; +lean_ctor_set(x_1, 0, x_52); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_53); +return x_1; +} +} +else { -return x_37; +uint8_t x_54; +x_54 = lean_ctor_get_uint8(x_43, sizeof(void*)*4); +if (x_54 == 0) +{ +uint8_t x_55; +x_55 = !lean_is_exclusive(x_41); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; +x_56 = lean_ctor_get(x_41, 1); +x_57 = lean_ctor_get(x_41, 2); +x_58 = lean_ctor_get(x_41, 3); +lean_dec(x_58); +x_59 = lean_ctor_get(x_41, 0); +lean_dec(x_59); +x_60 = !lean_is_exclusive(x_43); +if (x_60 == 0) +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; uint8_t x_66; +x_61 = lean_ctor_get(x_43, 0); +x_62 = lean_ctor_get(x_43, 1); +x_63 = lean_ctor_get(x_43, 2); +x_64 = lean_ctor_get(x_43, 3); +x_65 = 1; +lean_ctor_set(x_43, 3, x_61); +lean_ctor_set(x_43, 2, x_57); +lean_ctor_set(x_43, 1, x_56); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set_uint8(x_43, sizeof(void*)*4, x_65); +lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 2, x_35); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 0, x_64); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_65); +x_66 = 0; +lean_ctor_set(x_1, 3, x_41); +lean_ctor_set(x_1, 2, x_63); +lean_ctor_set(x_1, 1, x_62); +lean_ctor_set(x_1, 0, x_43); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_66); +return x_1; } 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_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_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; lean_object* x_72; uint8_t x_73; +x_67 = lean_ctor_get(x_43, 0); +x_68 = lean_ctor_get(x_43, 1); +x_69 = lean_ctor_get(x_43, 2); +x_70 = lean_ctor_get(x_43, 3); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_43); +x_71 = 1; +x_72 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_72, 0, x_42); +lean_ctor_set(x_72, 1, x_56); +lean_ctor_set(x_72, 2, x_57); +lean_ctor_set(x_72, 3, x_67); +lean_ctor_set_uint8(x_72, sizeof(void*)*4, x_71); +lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 2, x_35); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 0, x_70); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_71); +x_73 = 0; +lean_ctor_set(x_1, 3, x_41); +lean_ctor_set(x_1, 2, x_69); +lean_ctor_set(x_1, 1, x_68); +lean_ctor_set(x_1, 0, x_72); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_73); +return x_1; +} +} +else +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_74 = lean_ctor_get(x_41, 1); +x_75 = lean_ctor_get(x_41, 2); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_41); +x_76 = lean_ctor_get(x_43, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_43, 1); +lean_inc(x_77); +x_78 = lean_ctor_get(x_43, 2); +lean_inc(x_78); +x_79 = lean_ctor_get(x_43, 3); +lean_inc(x_79); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + lean_ctor_release(x_43, 2); + lean_ctor_release(x_43, 3); + x_80 = x_43; +} else { + lean_dec_ref(x_43); + x_80 = lean_box(0); } +x_81 = 1; +if (lean_is_scalar(x_80)) { + x_82 = lean_alloc_ctor(1, 4, 1); +} else { + x_82 = x_80; +} +lean_ctor_set(x_82, 0, x_42); +lean_ctor_set(x_82, 1, x_74); +lean_ctor_set(x_82, 2, x_75); +lean_ctor_set(x_82, 3, x_76); +lean_ctor_set_uint8(x_82, sizeof(void*)*4, x_81); +x_83 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_83, 0, x_79); +lean_ctor_set(x_83, 1, x_34); +lean_ctor_set(x_83, 2, x_35); +lean_ctor_set(x_83, 3, x_36); +lean_ctor_set_uint8(x_83, sizeof(void*)*4, x_81); +x_84 = 0; +lean_ctor_set(x_1, 3, x_83); +lean_ctor_set(x_1, 2, x_78); +lean_ctor_set(x_1, 1, x_77); +lean_ctor_set(x_1, 0, x_82); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_84); +return x_1; } } else { -uint8_t x_51; -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_28); -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_4); -lean_dec(x_1); -x_51 = !lean_is_exclusive(x_33); -if (x_51 == 0) +uint8_t x_85; +x_85 = !lean_is_exclusive(x_41); +if (x_85 == 0) { -return x_33; +lean_object* x_86; lean_object* x_87; uint8_t x_88; uint8_t x_89; +x_86 = lean_ctor_get(x_41, 3); +lean_dec(x_86); +x_87 = lean_ctor_get(x_41, 0); +lean_dec(x_87); +x_88 = 0; +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_88); +x_89 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_89); +return x_1; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_33, 0); -x_53 = lean_ctor_get(x_33, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_33); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; +lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; uint8_t x_94; +x_90 = lean_ctor_get(x_41, 1); +x_91 = lean_ctor_get(x_41, 2); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_41); +x_92 = 0; +x_93 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_93, 0, x_42); +lean_ctor_set(x_93, 1, x_90); +lean_ctor_set(x_93, 2, x_91); +lean_ctor_set(x_93, 3, x_43); +lean_ctor_set_uint8(x_93, sizeof(void*)*4, x_92); +x_94 = 1; +lean_ctor_set(x_1, 0, x_93); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_94); +return x_1; +} } } } else { -uint8_t x_55; -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_1); -x_55 = !lean_is_exclusive(x_27); -if (x_55 == 0) +uint8_t x_95; +x_95 = lean_ctor_get_uint8(x_42, sizeof(void*)*4); +if (x_95 == 0) +{ +uint8_t x_96; +x_96 = !lean_is_exclusive(x_41); +if (x_96 == 0) +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; uint8_t x_101; +x_97 = lean_ctor_get(x_41, 1); +x_98 = lean_ctor_get(x_41, 2); +x_99 = lean_ctor_get(x_41, 3); +x_100 = lean_ctor_get(x_41, 0); +lean_dec(x_100); +x_101 = !lean_is_exclusive(x_42); +if (x_101 == 0) +{ +uint8_t x_102; uint8_t x_103; +x_102 = 1; +lean_ctor_set_uint8(x_42, sizeof(void*)*4, x_102); +lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 2, x_35); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 0, x_99); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_102); +x_103 = 0; +lean_ctor_set(x_1, 3, x_41); +lean_ctor_set(x_1, 2, x_98); +lean_ctor_set(x_1, 1, x_97); +lean_ctor_set(x_1, 0, x_42); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_103); +return x_1; +} +else { -return x_27; +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; lean_object* x_109; uint8_t x_110; +x_104 = lean_ctor_get(x_42, 0); +x_105 = lean_ctor_get(x_42, 1); +x_106 = lean_ctor_get(x_42, 2); +x_107 = lean_ctor_get(x_42, 3); +lean_inc(x_107); +lean_inc(x_106); +lean_inc(x_105); +lean_inc(x_104); +lean_dec(x_42); +x_108 = 1; +x_109 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_109, 0, x_104); +lean_ctor_set(x_109, 1, x_105); +lean_ctor_set(x_109, 2, x_106); +lean_ctor_set(x_109, 3, x_107); +lean_ctor_set_uint8(x_109, sizeof(void*)*4, x_108); +lean_ctor_set(x_41, 3, x_36); +lean_ctor_set(x_41, 2, x_35); +lean_ctor_set(x_41, 1, x_34); +lean_ctor_set(x_41, 0, x_99); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_108); +x_110 = 0; +lean_ctor_set(x_1, 3, x_41); +lean_ctor_set(x_1, 2, x_98); +lean_ctor_set(x_1, 1, x_97); +lean_ctor_set(x_1, 0, x_109); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_110); +return x_1; +} } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_27, 0); -x_57 = lean_ctor_get(x_27, 1); -lean_inc(x_57); -lean_inc(x_56); -lean_dec(x_27); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -return x_58; +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; +x_111 = lean_ctor_get(x_41, 1); +x_112 = lean_ctor_get(x_41, 2); +x_113 = lean_ctor_get(x_41, 3); +lean_inc(x_113); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_41); +x_114 = lean_ctor_get(x_42, 0); +lean_inc(x_114); +x_115 = lean_ctor_get(x_42, 1); +lean_inc(x_115); +x_116 = lean_ctor_get(x_42, 2); +lean_inc(x_116); +x_117 = lean_ctor_get(x_42, 3); +lean_inc(x_117); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + lean_ctor_release(x_42, 2); + lean_ctor_release(x_42, 3); + x_118 = x_42; +} else { + lean_dec_ref(x_42); + x_118 = lean_box(0); } +x_119 = 1; +if (lean_is_scalar(x_118)) { + x_120 = lean_alloc_ctor(1, 4, 1); +} else { + x_120 = x_118; +} +lean_ctor_set(x_120, 0, x_114); +lean_ctor_set(x_120, 1, x_115); +lean_ctor_set(x_120, 2, x_116); +lean_ctor_set(x_120, 3, x_117); +lean_ctor_set_uint8(x_120, sizeof(void*)*4, x_119); +x_121 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_121, 0, x_113); +lean_ctor_set(x_121, 1, x_34); +lean_ctor_set(x_121, 2, x_35); +lean_ctor_set(x_121, 3, x_36); +lean_ctor_set_uint8(x_121, sizeof(void*)*4, x_119); +x_122 = 0; +lean_ctor_set(x_1, 3, x_121); +lean_ctor_set(x_1, 2, x_112); +lean_ctor_set(x_1, 1, x_111); +lean_ctor_set(x_1, 0, x_120); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_122); +return x_1; } } else { -lean_object* x_59; lean_object* x_60; -x_59 = lean_array_fget(x_1, x_4); -lean_inc(x_8); -x_60 = l_Lean_Meta_getFVarLocalDecl(x_59, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_60) == 0) +lean_object* x_123; +x_123 = lean_ctor_get(x_41, 3); +lean_inc(x_123); +if (lean_obj_tag(x_123) == 0) +{ +uint8_t x_124; +x_124 = !lean_is_exclusive(x_41); +if (x_124 == 0) +{ +lean_object* x_125; lean_object* x_126; uint8_t x_127; uint8_t x_128; +x_125 = lean_ctor_get(x_41, 3); +lean_dec(x_125); +x_126 = lean_ctor_get(x_41, 0); +lean_dec(x_126); +x_127 = 0; +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_127); +x_128 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_128); +return x_1; +} +else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_60, 1); -lean_inc(x_62); -lean_dec(x_60); -x_63 = l_Lean_LocalDecl_type(x_61); -lean_inc(x_63); -lean_inc(x_1); -x_64 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(x_1, x_63); -x_65 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(x_7, x_64); +lean_object* x_129; lean_object* x_130; uint8_t x_131; lean_object* x_132; uint8_t x_133; +x_129 = lean_ctor_get(x_41, 1); +x_130 = lean_ctor_get(x_41, 2); +lean_inc(x_130); +lean_inc(x_129); +lean_dec(x_41); +x_131 = 0; +x_132 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_132, 0, x_42); +lean_ctor_set(x_132, 1, x_129); +lean_ctor_set(x_132, 2, x_130); +lean_ctor_set(x_132, 3, x_123); +lean_ctor_set_uint8(x_132, sizeof(void*)*4, x_131); +x_133 = 1; +lean_ctor_set(x_1, 0, x_132); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_133); +return x_1; +} +} +else +{ +uint8_t x_134; +x_134 = lean_ctor_get_uint8(x_123, sizeof(void*)*4); +if (x_134 == 0) +{ +uint8_t x_135; +lean_free_object(x_1); +x_135 = !lean_is_exclusive(x_41); +if (x_135 == 0) +{ +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; uint8_t x_140; +x_136 = lean_ctor_get(x_41, 1); +x_137 = lean_ctor_get(x_41, 2); +x_138 = lean_ctor_get(x_41, 3); +lean_dec(x_138); +x_139 = lean_ctor_get(x_41, 0); +lean_dec(x_139); +x_140 = !lean_is_exclusive(x_123); +if (x_140 == 0) +{ +lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; uint8_t x_145; uint8_t x_146; +x_141 = lean_ctor_get(x_123, 0); +x_142 = lean_ctor_get(x_123, 1); +x_143 = lean_ctor_get(x_123, 2); +x_144 = lean_ctor_get(x_123, 3); +x_145 = 1; +lean_inc(x_42); +lean_ctor_set(x_123, 3, x_141); +lean_ctor_set(x_123, 2, x_137); +lean_ctor_set(x_123, 1, x_136); +lean_ctor_set(x_123, 0, x_42); +x_146 = !lean_is_exclusive(x_42); +if (x_146 == 0) +{ +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; uint8_t x_151; +x_147 = lean_ctor_get(x_42, 3); +lean_dec(x_147); +x_148 = lean_ctor_get(x_42, 2); +lean_dec(x_148); +x_149 = lean_ctor_get(x_42, 1); +lean_dec(x_149); +x_150 = lean_ctor_get(x_42, 0); +lean_dec(x_150); +lean_ctor_set_uint8(x_123, sizeof(void*)*4, x_145); +lean_ctor_set(x_42, 3, x_36); +lean_ctor_set(x_42, 2, x_35); +lean_ctor_set(x_42, 1, x_34); +lean_ctor_set(x_42, 0, x_144); +lean_ctor_set_uint8(x_42, sizeof(void*)*4, x_145); +x_151 = 0; +lean_ctor_set(x_41, 3, x_42); +lean_ctor_set(x_41, 2, x_143); +lean_ctor_set(x_41, 1, x_142); +lean_ctor_set(x_41, 0, x_123); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_151); +return x_41; +} +else +{ +lean_object* x_152; uint8_t x_153; +lean_dec(x_42); +lean_ctor_set_uint8(x_123, sizeof(void*)*4, x_145); +x_152 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_152, 0, x_144); +lean_ctor_set(x_152, 1, x_34); +lean_ctor_set(x_152, 2, x_35); +lean_ctor_set(x_152, 3, x_36); +lean_ctor_set_uint8(x_152, sizeof(void*)*4, x_145); +x_153 = 0; +lean_ctor_set(x_41, 3, x_152); +lean_ctor_set(x_41, 2, x_143); +lean_ctor_set(x_41, 1, x_142); +lean_ctor_set(x_41, 0, x_123); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_153); +return x_41; +} +} +else +{ +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; uint8_t x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; uint8_t x_162; +x_154 = lean_ctor_get(x_123, 0); +x_155 = lean_ctor_get(x_123, 1); +x_156 = lean_ctor_get(x_123, 2); +x_157 = lean_ctor_get(x_123, 3); +lean_inc(x_157); +lean_inc(x_156); +lean_inc(x_155); +lean_inc(x_154); +lean_dec(x_123); +x_158 = 1; +lean_inc(x_42); +x_159 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_159, 0, x_42); +lean_ctor_set(x_159, 1, x_136); +lean_ctor_set(x_159, 2, x_137); +lean_ctor_set(x_159, 3, x_154); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + lean_ctor_release(x_42, 2); + lean_ctor_release(x_42, 3); + x_160 = x_42; +} else { + lean_dec_ref(x_42); + x_160 = lean_box(0); +} +lean_ctor_set_uint8(x_159, sizeof(void*)*4, x_158); +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(1, 4, 1); +} else { + x_161 = x_160; +} +lean_ctor_set(x_161, 0, x_157); +lean_ctor_set(x_161, 1, x_34); +lean_ctor_set(x_161, 2, x_35); +lean_ctor_set(x_161, 3, x_36); +lean_ctor_set_uint8(x_161, sizeof(void*)*4, x_158); +x_162 = 0; +lean_ctor_set(x_41, 3, x_161); +lean_ctor_set(x_41, 2, x_156); +lean_ctor_set(x_41, 1, x_155); +lean_ctor_set(x_41, 0, x_159); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_162); +return x_41; +} +} +else +{ +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; uint8_t x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; lean_object* x_175; +x_163 = lean_ctor_get(x_41, 1); +x_164 = lean_ctor_get(x_41, 2); +lean_inc(x_164); +lean_inc(x_163); +lean_dec(x_41); +x_165 = lean_ctor_get(x_123, 0); +lean_inc(x_165); +x_166 = lean_ctor_get(x_123, 1); +lean_inc(x_166); +x_167 = lean_ctor_get(x_123, 2); +lean_inc(x_167); +x_168 = lean_ctor_get(x_123, 3); +lean_inc(x_168); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + lean_ctor_release(x_123, 2); + lean_ctor_release(x_123, 3); + x_169 = x_123; +} else { + lean_dec_ref(x_123); + x_169 = lean_box(0); +} +x_170 = 1; +lean_inc(x_42); +if (lean_is_scalar(x_169)) { + x_171 = lean_alloc_ctor(1, 4, 1); +} else { + x_171 = x_169; +} +lean_ctor_set(x_171, 0, x_42); +lean_ctor_set(x_171, 1, x_163); +lean_ctor_set(x_171, 2, x_164); +lean_ctor_set(x_171, 3, x_165); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + lean_ctor_release(x_42, 2); + lean_ctor_release(x_42, 3); + x_172 = x_42; +} else { + lean_dec_ref(x_42); + x_172 = lean_box(0); +} +lean_ctor_set_uint8(x_171, sizeof(void*)*4, x_170); +if (lean_is_scalar(x_172)) { + x_173 = lean_alloc_ctor(1, 4, 1); +} else { + x_173 = x_172; +} +lean_ctor_set(x_173, 0, x_168); +lean_ctor_set(x_173, 1, x_34); +lean_ctor_set(x_173, 2, x_35); +lean_ctor_set(x_173, 3, x_36); +lean_ctor_set_uint8(x_173, sizeof(void*)*4, x_170); +x_174 = 0; +x_175 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_175, 0, x_171); +lean_ctor_set(x_175, 1, x_166); +lean_ctor_set(x_175, 2, x_167); +lean_ctor_set(x_175, 3, x_173); +lean_ctor_set_uint8(x_175, sizeof(void*)*4, x_174); +return x_175; +} +} +else +{ +uint8_t x_176; +x_176 = !lean_is_exclusive(x_41); +if (x_176 == 0) +{ +lean_object* x_177; lean_object* x_178; uint8_t x_179; +x_177 = lean_ctor_get(x_41, 3); +lean_dec(x_177); +x_178 = lean_ctor_get(x_41, 0); +lean_dec(x_178); +x_179 = !lean_is_exclusive(x_42); +if (x_179 == 0) +{ +uint8_t x_180; uint8_t x_181; +lean_ctor_set_uint8(x_42, sizeof(void*)*4, x_134); +x_180 = 0; +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_180); +x_181 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_181); +return x_1; +} +else +{ +lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; uint8_t x_187; uint8_t x_188; +x_182 = lean_ctor_get(x_42, 0); +x_183 = lean_ctor_get(x_42, 1); +x_184 = lean_ctor_get(x_42, 2); +x_185 = lean_ctor_get(x_42, 3); +lean_inc(x_185); +lean_inc(x_184); +lean_inc(x_183); +lean_inc(x_182); +lean_dec(x_42); +x_186 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_186, 0, x_182); +lean_ctor_set(x_186, 1, x_183); +lean_ctor_set(x_186, 2, x_184); +lean_ctor_set(x_186, 3, x_185); +lean_ctor_set_uint8(x_186, sizeof(void*)*4, x_134); +x_187 = 0; +lean_ctor_set(x_41, 0, x_186); +lean_ctor_set_uint8(x_41, sizeof(void*)*4, x_187); +x_188 = 1; +lean_ctor_set(x_1, 0, x_41); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_188); +return x_1; +} +} +else +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; uint8_t x_197; lean_object* x_198; uint8_t x_199; +x_189 = lean_ctor_get(x_41, 1); +x_190 = lean_ctor_get(x_41, 2); +lean_inc(x_190); +lean_inc(x_189); +lean_dec(x_41); +x_191 = lean_ctor_get(x_42, 0); +lean_inc(x_191); +x_192 = lean_ctor_get(x_42, 1); +lean_inc(x_192); +x_193 = lean_ctor_get(x_42, 2); +lean_inc(x_193); +x_194 = lean_ctor_get(x_42, 3); +lean_inc(x_194); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + lean_ctor_release(x_42, 2); + lean_ctor_release(x_42, 3); + x_195 = x_42; +} else { + lean_dec_ref(x_42); + x_195 = lean_box(0); +} +if (lean_is_scalar(x_195)) { + x_196 = lean_alloc_ctor(1, 4, 1); +} else { + x_196 = x_195; +} +lean_ctor_set(x_196, 0, x_191); +lean_ctor_set(x_196, 1, x_192); +lean_ctor_set(x_196, 2, x_193); +lean_ctor_set(x_196, 3, x_194); +lean_ctor_set_uint8(x_196, sizeof(void*)*4, x_134); +x_197 = 0; +x_198 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_198, 0, x_196); +lean_ctor_set(x_198, 1, x_189); +lean_ctor_set(x_198, 2, x_190); +lean_ctor_set(x_198, 3, x_123); +lean_ctor_set_uint8(x_198, sizeof(void*)*4, x_197); +x_199 = 1; +lean_ctor_set(x_1, 0, x_198); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_199); +return x_1; +} +} +} +} +} +} +} +case 1: +{ +uint8_t x_200; +lean_dec(x_35); +lean_dec(x_34); +x_200 = 1; +lean_ctor_set(x_1, 2, x_3); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_200); +return x_1; +} +default: +{ +uint8_t x_201; +x_201 = l_Std_RBNode_isRed___rarg(x_36); +if (x_201 == 0) +{ +lean_object* x_202; uint8_t x_203; +x_202 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_36, x_2, x_3); +x_203 = 1; +lean_ctor_set(x_1, 3, x_202); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_203); +return x_1; +} +else +{ +lean_object* x_204; lean_object* x_205; +x_204 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_36, x_2, x_3); +x_205 = lean_ctor_get(x_204, 0); +lean_inc(x_205); +if (lean_obj_tag(x_205) == 0) +{ +lean_object* x_206; +x_206 = lean_ctor_get(x_204, 3); +lean_inc(x_206); +if (lean_obj_tag(x_206) == 0) +{ +uint8_t x_207; +x_207 = !lean_is_exclusive(x_204); +if (x_207 == 0) +{ +lean_object* x_208; lean_object* x_209; uint8_t x_210; uint8_t x_211; +x_208 = lean_ctor_get(x_204, 3); +lean_dec(x_208); +x_209 = lean_ctor_get(x_204, 0); +lean_dec(x_209); +x_210 = 0; +lean_ctor_set(x_204, 0, x_206); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_210); +x_211 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_211); +return x_1; +} +else +{ +lean_object* x_212; lean_object* x_213; uint8_t x_214; lean_object* x_215; uint8_t x_216; +x_212 = lean_ctor_get(x_204, 1); +x_213 = lean_ctor_get(x_204, 2); +lean_inc(x_213); +lean_inc(x_212); +lean_dec(x_204); +x_214 = 0; +x_215 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_215, 0, x_206); +lean_ctor_set(x_215, 1, x_212); +lean_ctor_set(x_215, 2, x_213); +lean_ctor_set(x_215, 3, x_206); +lean_ctor_set_uint8(x_215, sizeof(void*)*4, x_214); +x_216 = 1; +lean_ctor_set(x_1, 3, x_215); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_216); +return x_1; +} +} +else +{ +uint8_t x_217; +x_217 = lean_ctor_get_uint8(x_206, sizeof(void*)*4); +if (x_217 == 0) +{ +uint8_t x_218; +x_218 = !lean_is_exclusive(x_204); +if (x_218 == 0) +{ +lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; uint8_t x_223; +x_219 = lean_ctor_get(x_204, 1); +x_220 = lean_ctor_get(x_204, 2); +x_221 = lean_ctor_get(x_204, 3); +lean_dec(x_221); +x_222 = lean_ctor_get(x_204, 0); +lean_dec(x_222); +x_223 = !lean_is_exclusive(x_206); +if (x_223 == 0) +{ +lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; uint8_t x_228; uint8_t x_229; +x_224 = lean_ctor_get(x_206, 0); +x_225 = lean_ctor_get(x_206, 1); +x_226 = lean_ctor_get(x_206, 2); +x_227 = lean_ctor_get(x_206, 3); +x_228 = 1; +lean_ctor_set(x_206, 3, x_205); +lean_ctor_set(x_206, 2, x_35); +lean_ctor_set(x_206, 1, x_34); +lean_ctor_set(x_206, 0, x_33); +lean_ctor_set_uint8(x_206, sizeof(void*)*4, x_228); +lean_ctor_set(x_204, 3, x_227); +lean_ctor_set(x_204, 2, x_226); +lean_ctor_set(x_204, 1, x_225); +lean_ctor_set(x_204, 0, x_224); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_228); +x_229 = 0; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set(x_1, 2, x_220); +lean_ctor_set(x_1, 1, x_219); +lean_ctor_set(x_1, 0, x_206); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_229); +return x_1; +} +else +{ +lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; uint8_t x_234; lean_object* x_235; uint8_t x_236; +x_230 = lean_ctor_get(x_206, 0); +x_231 = lean_ctor_get(x_206, 1); +x_232 = lean_ctor_get(x_206, 2); +x_233 = lean_ctor_get(x_206, 3); +lean_inc(x_233); +lean_inc(x_232); +lean_inc(x_231); +lean_inc(x_230); +lean_dec(x_206); +x_234 = 1; +x_235 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_235, 0, x_33); +lean_ctor_set(x_235, 1, x_34); +lean_ctor_set(x_235, 2, x_35); +lean_ctor_set(x_235, 3, x_205); +lean_ctor_set_uint8(x_235, sizeof(void*)*4, x_234); +lean_ctor_set(x_204, 3, x_233); +lean_ctor_set(x_204, 2, x_232); +lean_ctor_set(x_204, 1, x_231); +lean_ctor_set(x_204, 0, x_230); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_234); +x_236 = 0; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set(x_1, 2, x_220); +lean_ctor_set(x_1, 1, x_219); +lean_ctor_set(x_1, 0, x_235); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_236); +return x_1; +} +} +else +{ +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; uint8_t x_244; lean_object* x_245; lean_object* x_246; uint8_t x_247; +x_237 = lean_ctor_get(x_204, 1); +x_238 = lean_ctor_get(x_204, 2); +lean_inc(x_238); +lean_inc(x_237); +lean_dec(x_204); +x_239 = lean_ctor_get(x_206, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_206, 1); +lean_inc(x_240); +x_241 = lean_ctor_get(x_206, 2); +lean_inc(x_241); +x_242 = lean_ctor_get(x_206, 3); +lean_inc(x_242); +if (lean_is_exclusive(x_206)) { + lean_ctor_release(x_206, 0); + lean_ctor_release(x_206, 1); + lean_ctor_release(x_206, 2); + lean_ctor_release(x_206, 3); + x_243 = x_206; +} else { + lean_dec_ref(x_206); + x_243 = lean_box(0); +} +x_244 = 1; +if (lean_is_scalar(x_243)) { + x_245 = lean_alloc_ctor(1, 4, 1); +} else { + x_245 = x_243; +} +lean_ctor_set(x_245, 0, x_33); +lean_ctor_set(x_245, 1, x_34); +lean_ctor_set(x_245, 2, x_35); +lean_ctor_set(x_245, 3, x_205); +lean_ctor_set_uint8(x_245, sizeof(void*)*4, x_244); +x_246 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_246, 0, x_239); +lean_ctor_set(x_246, 1, x_240); +lean_ctor_set(x_246, 2, x_241); +lean_ctor_set(x_246, 3, x_242); +lean_ctor_set_uint8(x_246, sizeof(void*)*4, x_244); +x_247 = 0; +lean_ctor_set(x_1, 3, x_246); +lean_ctor_set(x_1, 2, x_238); +lean_ctor_set(x_1, 1, x_237); +lean_ctor_set(x_1, 0, x_245); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_247); +return x_1; +} +} +else +{ +uint8_t x_248; +x_248 = !lean_is_exclusive(x_204); +if (x_248 == 0) +{ +lean_object* x_249; lean_object* x_250; uint8_t x_251; uint8_t x_252; +x_249 = lean_ctor_get(x_204, 3); +lean_dec(x_249); +x_250 = lean_ctor_get(x_204, 0); +lean_dec(x_250); +x_251 = 0; +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_251); +x_252 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_252); +return x_1; +} +else +{ +lean_object* x_253; lean_object* x_254; uint8_t x_255; lean_object* x_256; uint8_t x_257; +x_253 = lean_ctor_get(x_204, 1); +x_254 = lean_ctor_get(x_204, 2); +lean_inc(x_254); +lean_inc(x_253); +lean_dec(x_204); +x_255 = 0; +x_256 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_256, 0, x_205); +lean_ctor_set(x_256, 1, x_253); +lean_ctor_set(x_256, 2, x_254); +lean_ctor_set(x_256, 3, x_206); +lean_ctor_set_uint8(x_256, sizeof(void*)*4, x_255); +x_257 = 1; +lean_ctor_set(x_1, 3, x_256); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_257); +return x_1; +} +} +} +} +else +{ +uint8_t x_258; +x_258 = lean_ctor_get_uint8(x_205, sizeof(void*)*4); +if (x_258 == 0) +{ +uint8_t x_259; +x_259 = !lean_is_exclusive(x_204); +if (x_259 == 0) +{ +lean_object* x_260; uint8_t x_261; +x_260 = lean_ctor_get(x_204, 0); +lean_dec(x_260); +x_261 = !lean_is_exclusive(x_205); +if (x_261 == 0) +{ +lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; uint8_t x_266; uint8_t x_267; +x_262 = lean_ctor_get(x_205, 0); +x_263 = lean_ctor_get(x_205, 1); +x_264 = lean_ctor_get(x_205, 2); +x_265 = lean_ctor_get(x_205, 3); +x_266 = 1; +lean_ctor_set(x_205, 3, x_262); +lean_ctor_set(x_205, 2, x_35); +lean_ctor_set(x_205, 1, x_34); +lean_ctor_set(x_205, 0, x_33); +lean_ctor_set_uint8(x_205, sizeof(void*)*4, x_266); +lean_ctor_set(x_204, 0, x_265); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_266); +x_267 = 0; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set(x_1, 2, x_264); +lean_ctor_set(x_1, 1, x_263); +lean_ctor_set(x_1, 0, x_205); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_267); +return x_1; +} +else +{ +lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; uint8_t x_272; lean_object* x_273; uint8_t x_274; +x_268 = lean_ctor_get(x_205, 0); +x_269 = lean_ctor_get(x_205, 1); +x_270 = lean_ctor_get(x_205, 2); +x_271 = lean_ctor_get(x_205, 3); +lean_inc(x_271); +lean_inc(x_270); +lean_inc(x_269); +lean_inc(x_268); +lean_dec(x_205); +x_272 = 1; +x_273 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_273, 0, x_33); +lean_ctor_set(x_273, 1, x_34); +lean_ctor_set(x_273, 2, x_35); +lean_ctor_set(x_273, 3, x_268); +lean_ctor_set_uint8(x_273, sizeof(void*)*4, x_272); +lean_ctor_set(x_204, 0, x_271); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_272); +x_274 = 0; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set(x_1, 2, x_270); +lean_ctor_set(x_1, 1, x_269); +lean_ctor_set(x_1, 0, x_273); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_274); +return x_1; +} +} +else +{ +lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; uint8_t x_283; lean_object* x_284; lean_object* x_285; uint8_t x_286; +x_275 = lean_ctor_get(x_204, 1); +x_276 = lean_ctor_get(x_204, 2); +x_277 = lean_ctor_get(x_204, 3); +lean_inc(x_277); +lean_inc(x_276); +lean_inc(x_275); +lean_dec(x_204); +x_278 = lean_ctor_get(x_205, 0); +lean_inc(x_278); +x_279 = lean_ctor_get(x_205, 1); +lean_inc(x_279); +x_280 = lean_ctor_get(x_205, 2); +lean_inc(x_280); +x_281 = lean_ctor_get(x_205, 3); +lean_inc(x_281); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + lean_ctor_release(x_205, 2); + lean_ctor_release(x_205, 3); + x_282 = x_205; +} else { + lean_dec_ref(x_205); + x_282 = lean_box(0); +} +x_283 = 1; +if (lean_is_scalar(x_282)) { + x_284 = lean_alloc_ctor(1, 4, 1); +} else { + x_284 = x_282; +} +lean_ctor_set(x_284, 0, x_33); +lean_ctor_set(x_284, 1, x_34); +lean_ctor_set(x_284, 2, x_35); +lean_ctor_set(x_284, 3, x_278); +lean_ctor_set_uint8(x_284, sizeof(void*)*4, x_283); +x_285 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_285, 0, x_281); +lean_ctor_set(x_285, 1, x_275); +lean_ctor_set(x_285, 2, x_276); +lean_ctor_set(x_285, 3, x_277); +lean_ctor_set_uint8(x_285, sizeof(void*)*4, x_283); +x_286 = 0; +lean_ctor_set(x_1, 3, x_285); +lean_ctor_set(x_1, 2, x_280); +lean_ctor_set(x_1, 1, x_279); +lean_ctor_set(x_1, 0, x_284); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_286); +return x_1; +} +} +else +{ +lean_object* x_287; +x_287 = lean_ctor_get(x_204, 3); +lean_inc(x_287); +if (lean_obj_tag(x_287) == 0) +{ +uint8_t x_288; +x_288 = !lean_is_exclusive(x_204); +if (x_288 == 0) +{ +lean_object* x_289; lean_object* x_290; uint8_t x_291; uint8_t x_292; +x_289 = lean_ctor_get(x_204, 3); +lean_dec(x_289); +x_290 = lean_ctor_get(x_204, 0); +lean_dec(x_290); +x_291 = 0; +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_291); +x_292 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_292); +return x_1; +} +else +{ +lean_object* x_293; lean_object* x_294; uint8_t x_295; lean_object* x_296; uint8_t x_297; +x_293 = lean_ctor_get(x_204, 1); +x_294 = lean_ctor_get(x_204, 2); +lean_inc(x_294); +lean_inc(x_293); +lean_dec(x_204); +x_295 = 0; +x_296 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_296, 0, x_205); +lean_ctor_set(x_296, 1, x_293); +lean_ctor_set(x_296, 2, x_294); +lean_ctor_set(x_296, 3, x_287); +lean_ctor_set_uint8(x_296, sizeof(void*)*4, x_295); +x_297 = 1; +lean_ctor_set(x_1, 3, x_296); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_297); +return x_1; +} +} +else +{ +uint8_t x_298; +x_298 = lean_ctor_get_uint8(x_287, sizeof(void*)*4); +if (x_298 == 0) +{ +uint8_t x_299; +lean_free_object(x_1); +x_299 = !lean_is_exclusive(x_204); +if (x_299 == 0) +{ +lean_object* x_300; lean_object* x_301; uint8_t x_302; +x_300 = lean_ctor_get(x_204, 3); +lean_dec(x_300); +x_301 = lean_ctor_get(x_204, 0); +lean_dec(x_301); +x_302 = !lean_is_exclusive(x_287); +if (x_302 == 0) +{ +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; uint8_t x_307; uint8_t x_308; +x_303 = lean_ctor_get(x_287, 0); +x_304 = lean_ctor_get(x_287, 1); +x_305 = lean_ctor_get(x_287, 2); +x_306 = lean_ctor_get(x_287, 3); +x_307 = 1; +lean_inc(x_205); +lean_ctor_set(x_287, 3, x_205); +lean_ctor_set(x_287, 2, x_35); +lean_ctor_set(x_287, 1, x_34); +lean_ctor_set(x_287, 0, x_33); +x_308 = !lean_is_exclusive(x_205); +if (x_308 == 0) +{ +lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; uint8_t x_313; +x_309 = lean_ctor_get(x_205, 3); +lean_dec(x_309); +x_310 = lean_ctor_get(x_205, 2); +lean_dec(x_310); +x_311 = lean_ctor_get(x_205, 1); +lean_dec(x_311); +x_312 = lean_ctor_get(x_205, 0); +lean_dec(x_312); +lean_ctor_set_uint8(x_287, sizeof(void*)*4, x_307); +lean_ctor_set(x_205, 3, x_306); +lean_ctor_set(x_205, 2, x_305); +lean_ctor_set(x_205, 1, x_304); +lean_ctor_set(x_205, 0, x_303); +lean_ctor_set_uint8(x_205, sizeof(void*)*4, x_307); +x_313 = 0; +lean_ctor_set(x_204, 3, x_205); +lean_ctor_set(x_204, 0, x_287); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_313); +return x_204; +} +else +{ +lean_object* x_314; uint8_t x_315; +lean_dec(x_205); +lean_ctor_set_uint8(x_287, sizeof(void*)*4, x_307); +x_314 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_314, 0, x_303); +lean_ctor_set(x_314, 1, x_304); +lean_ctor_set(x_314, 2, x_305); +lean_ctor_set(x_314, 3, x_306); +lean_ctor_set_uint8(x_314, sizeof(void*)*4, x_307); +x_315 = 0; +lean_ctor_set(x_204, 3, x_314); +lean_ctor_set(x_204, 0, x_287); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_315); +return x_204; +} +} +else +{ +lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; uint8_t x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; uint8_t x_324; +x_316 = lean_ctor_get(x_287, 0); +x_317 = lean_ctor_get(x_287, 1); +x_318 = lean_ctor_get(x_287, 2); +x_319 = lean_ctor_get(x_287, 3); +lean_inc(x_319); +lean_inc(x_318); +lean_inc(x_317); +lean_inc(x_316); +lean_dec(x_287); +x_320 = 1; +lean_inc(x_205); +x_321 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_321, 0, x_33); +lean_ctor_set(x_321, 1, x_34); +lean_ctor_set(x_321, 2, x_35); +lean_ctor_set(x_321, 3, x_205); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + lean_ctor_release(x_205, 2); + lean_ctor_release(x_205, 3); + x_322 = x_205; +} else { + lean_dec_ref(x_205); + x_322 = lean_box(0); +} +lean_ctor_set_uint8(x_321, sizeof(void*)*4, x_320); +if (lean_is_scalar(x_322)) { + x_323 = lean_alloc_ctor(1, 4, 1); +} else { + x_323 = x_322; +} +lean_ctor_set(x_323, 0, x_316); +lean_ctor_set(x_323, 1, x_317); +lean_ctor_set(x_323, 2, x_318); +lean_ctor_set(x_323, 3, x_319); +lean_ctor_set_uint8(x_323, sizeof(void*)*4, x_320); +x_324 = 0; +lean_ctor_set(x_204, 3, x_323); +lean_ctor_set(x_204, 0, x_321); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_324); +return x_204; +} +} +else +{ +lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; uint8_t x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; uint8_t x_336; lean_object* x_337; +x_325 = lean_ctor_get(x_204, 1); +x_326 = lean_ctor_get(x_204, 2); +lean_inc(x_326); +lean_inc(x_325); +lean_dec(x_204); +x_327 = lean_ctor_get(x_287, 0); +lean_inc(x_327); +x_328 = lean_ctor_get(x_287, 1); +lean_inc(x_328); +x_329 = lean_ctor_get(x_287, 2); +lean_inc(x_329); +x_330 = lean_ctor_get(x_287, 3); +lean_inc(x_330); +if (lean_is_exclusive(x_287)) { + lean_ctor_release(x_287, 0); + lean_ctor_release(x_287, 1); + lean_ctor_release(x_287, 2); + lean_ctor_release(x_287, 3); + x_331 = x_287; +} else { + lean_dec_ref(x_287); + x_331 = lean_box(0); +} +x_332 = 1; +lean_inc(x_205); +if (lean_is_scalar(x_331)) { + x_333 = lean_alloc_ctor(1, 4, 1); +} else { + x_333 = x_331; +} +lean_ctor_set(x_333, 0, x_33); +lean_ctor_set(x_333, 1, x_34); +lean_ctor_set(x_333, 2, x_35); +lean_ctor_set(x_333, 3, x_205); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + lean_ctor_release(x_205, 2); + lean_ctor_release(x_205, 3); + x_334 = x_205; +} else { + lean_dec_ref(x_205); + x_334 = lean_box(0); +} +lean_ctor_set_uint8(x_333, sizeof(void*)*4, x_332); +if (lean_is_scalar(x_334)) { + x_335 = lean_alloc_ctor(1, 4, 1); +} else { + x_335 = x_334; +} +lean_ctor_set(x_335, 0, x_327); +lean_ctor_set(x_335, 1, x_328); +lean_ctor_set(x_335, 2, x_329); +lean_ctor_set(x_335, 3, x_330); +lean_ctor_set_uint8(x_335, sizeof(void*)*4, x_332); +x_336 = 0; +x_337 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_337, 0, x_333); +lean_ctor_set(x_337, 1, x_325); +lean_ctor_set(x_337, 2, x_326); +lean_ctor_set(x_337, 3, x_335); +lean_ctor_set_uint8(x_337, sizeof(void*)*4, x_336); +return x_337; +} +} +else +{ +uint8_t x_338; +x_338 = !lean_is_exclusive(x_204); +if (x_338 == 0) +{ +lean_object* x_339; lean_object* x_340; uint8_t x_341; +x_339 = lean_ctor_get(x_204, 3); +lean_dec(x_339); +x_340 = lean_ctor_get(x_204, 0); +lean_dec(x_340); +x_341 = !lean_is_exclusive(x_205); +if (x_341 == 0) +{ +uint8_t x_342; uint8_t x_343; +lean_ctor_set_uint8(x_205, sizeof(void*)*4, x_298); +x_342 = 0; +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_342); +x_343 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_343); +return x_1; +} +else +{ +lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; uint8_t x_349; uint8_t x_350; +x_344 = lean_ctor_get(x_205, 0); +x_345 = lean_ctor_get(x_205, 1); +x_346 = lean_ctor_get(x_205, 2); +x_347 = lean_ctor_get(x_205, 3); +lean_inc(x_347); +lean_inc(x_346); +lean_inc(x_345); +lean_inc(x_344); +lean_dec(x_205); +x_348 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_348, 0, x_344); +lean_ctor_set(x_348, 1, x_345); +lean_ctor_set(x_348, 2, x_346); +lean_ctor_set(x_348, 3, x_347); +lean_ctor_set_uint8(x_348, sizeof(void*)*4, x_298); +x_349 = 0; +lean_ctor_set(x_204, 0, x_348); +lean_ctor_set_uint8(x_204, sizeof(void*)*4, x_349); +x_350 = 1; +lean_ctor_set(x_1, 3, x_204); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_350); +return x_1; +} +} +else +{ +lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; uint8_t x_359; lean_object* x_360; uint8_t x_361; +x_351 = lean_ctor_get(x_204, 1); +x_352 = lean_ctor_get(x_204, 2); +lean_inc(x_352); +lean_inc(x_351); +lean_dec(x_204); +x_353 = lean_ctor_get(x_205, 0); +lean_inc(x_353); +x_354 = lean_ctor_get(x_205, 1); +lean_inc(x_354); +x_355 = lean_ctor_get(x_205, 2); +lean_inc(x_355); +x_356 = lean_ctor_get(x_205, 3); +lean_inc(x_356); +if (lean_is_exclusive(x_205)) { + lean_ctor_release(x_205, 0); + lean_ctor_release(x_205, 1); + lean_ctor_release(x_205, 2); + lean_ctor_release(x_205, 3); + x_357 = x_205; +} else { + lean_dec_ref(x_205); + x_357 = lean_box(0); +} +if (lean_is_scalar(x_357)) { + x_358 = lean_alloc_ctor(1, 4, 1); +} else { + x_358 = x_357; +} +lean_ctor_set(x_358, 0, x_353); +lean_ctor_set(x_358, 1, x_354); +lean_ctor_set(x_358, 2, x_355); +lean_ctor_set(x_358, 3, x_356); +lean_ctor_set_uint8(x_358, sizeof(void*)*4, x_298); +x_359 = 0; +x_360 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_360, 0, x_358); +lean_ctor_set(x_360, 1, x_351); +lean_ctor_set(x_360, 2, x_352); +lean_ctor_set(x_360, 3, x_287); +lean_ctor_set_uint8(x_360, sizeof(void*)*4, x_359); +x_361 = 1; +lean_ctor_set(x_1, 3, x_360); +lean_ctor_set_uint8(x_1, sizeof(void*)*4, x_361); +return x_1; +} +} +} +} +} +} +} +} +} +else +{ +lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; uint8_t x_366; +x_362 = lean_ctor_get(x_1, 0); +x_363 = lean_ctor_get(x_1, 1); +x_364 = lean_ctor_get(x_1, 2); +x_365 = lean_ctor_get(x_1, 3); +lean_inc(x_365); +lean_inc(x_364); +lean_inc(x_363); +lean_inc(x_362); +lean_dec(x_1); +x_366 = l_Lean_Name_quickCmp(x_2, x_363); +switch (x_366) { +case 0: +{ +uint8_t x_367; +x_367 = l_Std_RBNode_isRed___rarg(x_362); +if (x_367 == 0) +{ +lean_object* x_368; uint8_t x_369; lean_object* x_370; +x_368 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_362, x_2, x_3); +x_369 = 1; +x_370 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_370, 0, x_368); +lean_ctor_set(x_370, 1, x_363); +lean_ctor_set(x_370, 2, x_364); +lean_ctor_set(x_370, 3, x_365); +lean_ctor_set_uint8(x_370, sizeof(void*)*4, x_369); +return x_370; +} +else +{ +lean_object* x_371; lean_object* x_372; +x_371 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_362, x_2, x_3); +x_372 = lean_ctor_get(x_371, 0); +lean_inc(x_372); +if (lean_obj_tag(x_372) == 0) +{ +lean_object* x_373; +x_373 = lean_ctor_get(x_371, 3); +lean_inc(x_373); +if (lean_obj_tag(x_373) == 0) +{ +lean_object* x_374; lean_object* x_375; lean_object* x_376; uint8_t x_377; lean_object* x_378; uint8_t x_379; lean_object* x_380; +x_374 = lean_ctor_get(x_371, 1); +lean_inc(x_374); +x_375 = lean_ctor_get(x_371, 2); +lean_inc(x_375); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_376 = x_371; +} else { + lean_dec_ref(x_371); + x_376 = lean_box(0); +} +x_377 = 0; +if (lean_is_scalar(x_376)) { + x_378 = lean_alloc_ctor(1, 4, 1); +} else { + x_378 = x_376; +} +lean_ctor_set(x_378, 0, x_373); +lean_ctor_set(x_378, 1, x_374); +lean_ctor_set(x_378, 2, x_375); +lean_ctor_set(x_378, 3, x_373); +lean_ctor_set_uint8(x_378, sizeof(void*)*4, x_377); +x_379 = 1; +x_380 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_380, 0, x_378); +lean_ctor_set(x_380, 1, x_363); +lean_ctor_set(x_380, 2, x_364); +lean_ctor_set(x_380, 3, x_365); +lean_ctor_set_uint8(x_380, sizeof(void*)*4, x_379); +return x_380; +} +else +{ +uint8_t x_381; +x_381 = lean_ctor_get_uint8(x_373, sizeof(void*)*4); +if (x_381 == 0) +{ +lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; uint8_t x_390; lean_object* x_391; lean_object* x_392; uint8_t x_393; lean_object* x_394; +x_382 = lean_ctor_get(x_371, 1); +lean_inc(x_382); +x_383 = lean_ctor_get(x_371, 2); +lean_inc(x_383); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_384 = x_371; +} else { + lean_dec_ref(x_371); + x_384 = lean_box(0); +} +x_385 = lean_ctor_get(x_373, 0); +lean_inc(x_385); +x_386 = lean_ctor_get(x_373, 1); +lean_inc(x_386); +x_387 = lean_ctor_get(x_373, 2); +lean_inc(x_387); +x_388 = lean_ctor_get(x_373, 3); +lean_inc(x_388); +if (lean_is_exclusive(x_373)) { + lean_ctor_release(x_373, 0); + lean_ctor_release(x_373, 1); + lean_ctor_release(x_373, 2); + lean_ctor_release(x_373, 3); + x_389 = x_373; +} else { + lean_dec_ref(x_373); + x_389 = lean_box(0); +} +x_390 = 1; +if (lean_is_scalar(x_389)) { + x_391 = lean_alloc_ctor(1, 4, 1); +} else { + x_391 = x_389; +} +lean_ctor_set(x_391, 0, x_372); +lean_ctor_set(x_391, 1, x_382); +lean_ctor_set(x_391, 2, x_383); +lean_ctor_set(x_391, 3, x_385); +lean_ctor_set_uint8(x_391, sizeof(void*)*4, x_390); +if (lean_is_scalar(x_384)) { + x_392 = lean_alloc_ctor(1, 4, 1); +} else { + x_392 = x_384; +} +lean_ctor_set(x_392, 0, x_388); +lean_ctor_set(x_392, 1, x_363); +lean_ctor_set(x_392, 2, x_364); +lean_ctor_set(x_392, 3, x_365); +lean_ctor_set_uint8(x_392, sizeof(void*)*4, x_390); +x_393 = 0; +x_394 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_394, 0, x_391); +lean_ctor_set(x_394, 1, x_386); +lean_ctor_set(x_394, 2, x_387); +lean_ctor_set(x_394, 3, x_392); +lean_ctor_set_uint8(x_394, sizeof(void*)*4, x_393); +return x_394; +} +else +{ +lean_object* x_395; lean_object* x_396; lean_object* x_397; uint8_t x_398; lean_object* x_399; uint8_t x_400; lean_object* x_401; +x_395 = lean_ctor_get(x_371, 1); +lean_inc(x_395); +x_396 = lean_ctor_get(x_371, 2); +lean_inc(x_396); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_397 = x_371; +} else { + lean_dec_ref(x_371); + x_397 = lean_box(0); +} +x_398 = 0; +if (lean_is_scalar(x_397)) { + x_399 = lean_alloc_ctor(1, 4, 1); +} else { + x_399 = x_397; +} +lean_ctor_set(x_399, 0, x_372); +lean_ctor_set(x_399, 1, x_395); +lean_ctor_set(x_399, 2, x_396); +lean_ctor_set(x_399, 3, x_373); +lean_ctor_set_uint8(x_399, sizeof(void*)*4, x_398); +x_400 = 1; +x_401 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_401, 0, x_399); +lean_ctor_set(x_401, 1, x_363); +lean_ctor_set(x_401, 2, x_364); +lean_ctor_set(x_401, 3, x_365); +lean_ctor_set_uint8(x_401, sizeof(void*)*4, x_400); +return x_401; +} +} +} +else +{ +uint8_t x_402; +x_402 = lean_ctor_get_uint8(x_372, sizeof(void*)*4); +if (x_402 == 0) +{ +lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; uint8_t x_412; lean_object* x_413; lean_object* x_414; uint8_t x_415; lean_object* x_416; +x_403 = lean_ctor_get(x_371, 1); +lean_inc(x_403); +x_404 = lean_ctor_get(x_371, 2); +lean_inc(x_404); +x_405 = lean_ctor_get(x_371, 3); +lean_inc(x_405); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_406 = x_371; +} else { + lean_dec_ref(x_371); + x_406 = lean_box(0); +} +x_407 = lean_ctor_get(x_372, 0); +lean_inc(x_407); +x_408 = lean_ctor_get(x_372, 1); +lean_inc(x_408); +x_409 = lean_ctor_get(x_372, 2); +lean_inc(x_409); +x_410 = lean_ctor_get(x_372, 3); +lean_inc(x_410); +if (lean_is_exclusive(x_372)) { + lean_ctor_release(x_372, 0); + lean_ctor_release(x_372, 1); + lean_ctor_release(x_372, 2); + lean_ctor_release(x_372, 3); + x_411 = x_372; +} else { + lean_dec_ref(x_372); + x_411 = lean_box(0); +} +x_412 = 1; +if (lean_is_scalar(x_411)) { + x_413 = lean_alloc_ctor(1, 4, 1); +} else { + x_413 = x_411; +} +lean_ctor_set(x_413, 0, x_407); +lean_ctor_set(x_413, 1, x_408); +lean_ctor_set(x_413, 2, x_409); +lean_ctor_set(x_413, 3, x_410); +lean_ctor_set_uint8(x_413, sizeof(void*)*4, x_412); +if (lean_is_scalar(x_406)) { + x_414 = lean_alloc_ctor(1, 4, 1); +} else { + x_414 = x_406; +} +lean_ctor_set(x_414, 0, x_405); +lean_ctor_set(x_414, 1, x_363); +lean_ctor_set(x_414, 2, x_364); +lean_ctor_set(x_414, 3, x_365); +lean_ctor_set_uint8(x_414, sizeof(void*)*4, x_412); +x_415 = 0; +x_416 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_416, 0, x_413); +lean_ctor_set(x_416, 1, x_403); +lean_ctor_set(x_416, 2, x_404); +lean_ctor_set(x_416, 3, x_414); +lean_ctor_set_uint8(x_416, sizeof(void*)*4, x_415); +return x_416; +} +else +{ +lean_object* x_417; +x_417 = lean_ctor_get(x_371, 3); +lean_inc(x_417); +if (lean_obj_tag(x_417) == 0) +{ +lean_object* x_418; lean_object* x_419; lean_object* x_420; uint8_t x_421; lean_object* x_422; uint8_t x_423; lean_object* x_424; +x_418 = lean_ctor_get(x_371, 1); +lean_inc(x_418); +x_419 = lean_ctor_get(x_371, 2); +lean_inc(x_419); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_420 = x_371; +} else { + lean_dec_ref(x_371); + x_420 = lean_box(0); +} +x_421 = 0; +if (lean_is_scalar(x_420)) { + x_422 = lean_alloc_ctor(1, 4, 1); +} else { + x_422 = x_420; +} +lean_ctor_set(x_422, 0, x_372); +lean_ctor_set(x_422, 1, x_418); +lean_ctor_set(x_422, 2, x_419); +lean_ctor_set(x_422, 3, x_417); +lean_ctor_set_uint8(x_422, sizeof(void*)*4, x_421); +x_423 = 1; +x_424 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_424, 0, x_422); +lean_ctor_set(x_424, 1, x_363); +lean_ctor_set(x_424, 2, x_364); +lean_ctor_set(x_424, 3, x_365); +lean_ctor_set_uint8(x_424, sizeof(void*)*4, x_423); +return x_424; +} +else +{ +uint8_t x_425; +x_425 = lean_ctor_get_uint8(x_417, sizeof(void*)*4); +if (x_425 == 0) +{ +lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; uint8_t x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; uint8_t x_438; lean_object* x_439; +x_426 = lean_ctor_get(x_371, 1); +lean_inc(x_426); +x_427 = lean_ctor_get(x_371, 2); +lean_inc(x_427); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_428 = x_371; +} else { + lean_dec_ref(x_371); + x_428 = lean_box(0); +} +x_429 = lean_ctor_get(x_417, 0); +lean_inc(x_429); +x_430 = lean_ctor_get(x_417, 1); +lean_inc(x_430); +x_431 = lean_ctor_get(x_417, 2); +lean_inc(x_431); +x_432 = lean_ctor_get(x_417, 3); +lean_inc(x_432); +if (lean_is_exclusive(x_417)) { + lean_ctor_release(x_417, 0); + lean_ctor_release(x_417, 1); + lean_ctor_release(x_417, 2); + lean_ctor_release(x_417, 3); + x_433 = x_417; +} else { + lean_dec_ref(x_417); + x_433 = lean_box(0); +} +x_434 = 1; +lean_inc(x_372); +if (lean_is_scalar(x_433)) { + x_435 = lean_alloc_ctor(1, 4, 1); +} else { + x_435 = x_433; +} +lean_ctor_set(x_435, 0, x_372); +lean_ctor_set(x_435, 1, x_426); +lean_ctor_set(x_435, 2, x_427); +lean_ctor_set(x_435, 3, x_429); +if (lean_is_exclusive(x_372)) { + lean_ctor_release(x_372, 0); + lean_ctor_release(x_372, 1); + lean_ctor_release(x_372, 2); + lean_ctor_release(x_372, 3); + x_436 = x_372; +} else { + lean_dec_ref(x_372); + x_436 = lean_box(0); +} +lean_ctor_set_uint8(x_435, sizeof(void*)*4, x_434); +if (lean_is_scalar(x_436)) { + x_437 = lean_alloc_ctor(1, 4, 1); +} else { + x_437 = x_436; +} +lean_ctor_set(x_437, 0, x_432); +lean_ctor_set(x_437, 1, x_363); +lean_ctor_set(x_437, 2, x_364); +lean_ctor_set(x_437, 3, x_365); +lean_ctor_set_uint8(x_437, sizeof(void*)*4, x_434); +x_438 = 0; +if (lean_is_scalar(x_428)) { + x_439 = lean_alloc_ctor(1, 4, 1); +} else { + x_439 = x_428; +} +lean_ctor_set(x_439, 0, x_435); +lean_ctor_set(x_439, 1, x_430); +lean_ctor_set(x_439, 2, x_431); +lean_ctor_set(x_439, 3, x_437); +lean_ctor_set_uint8(x_439, sizeof(void*)*4, x_438); +return x_439; +} +else +{ +lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; uint8_t x_449; lean_object* x_450; uint8_t x_451; lean_object* x_452; +x_440 = lean_ctor_get(x_371, 1); +lean_inc(x_440); +x_441 = lean_ctor_get(x_371, 2); +lean_inc(x_441); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + lean_ctor_release(x_371, 2); + lean_ctor_release(x_371, 3); + x_442 = x_371; +} else { + lean_dec_ref(x_371); + x_442 = lean_box(0); +} +x_443 = lean_ctor_get(x_372, 0); +lean_inc(x_443); +x_444 = lean_ctor_get(x_372, 1); +lean_inc(x_444); +x_445 = lean_ctor_get(x_372, 2); +lean_inc(x_445); +x_446 = lean_ctor_get(x_372, 3); +lean_inc(x_446); +if (lean_is_exclusive(x_372)) { + lean_ctor_release(x_372, 0); + lean_ctor_release(x_372, 1); + lean_ctor_release(x_372, 2); + lean_ctor_release(x_372, 3); + x_447 = x_372; +} else { + lean_dec_ref(x_372); + x_447 = lean_box(0); +} +if (lean_is_scalar(x_447)) { + x_448 = lean_alloc_ctor(1, 4, 1); +} else { + x_448 = x_447; +} +lean_ctor_set(x_448, 0, x_443); +lean_ctor_set(x_448, 1, x_444); +lean_ctor_set(x_448, 2, x_445); +lean_ctor_set(x_448, 3, x_446); +lean_ctor_set_uint8(x_448, sizeof(void*)*4, x_425); +x_449 = 0; +if (lean_is_scalar(x_442)) { + x_450 = lean_alloc_ctor(1, 4, 1); +} else { + x_450 = x_442; +} +lean_ctor_set(x_450, 0, x_448); +lean_ctor_set(x_450, 1, x_440); +lean_ctor_set(x_450, 2, x_441); +lean_ctor_set(x_450, 3, x_417); +lean_ctor_set_uint8(x_450, sizeof(void*)*4, x_449); +x_451 = 1; +x_452 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_452, 0, x_450); +lean_ctor_set(x_452, 1, x_363); +lean_ctor_set(x_452, 2, x_364); +lean_ctor_set(x_452, 3, x_365); +lean_ctor_set_uint8(x_452, sizeof(void*)*4, x_451); +return x_452; +} +} +} +} +} +} +case 1: +{ +uint8_t x_453; lean_object* x_454; +lean_dec(x_364); +lean_dec(x_363); +x_453 = 1; +x_454 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_454, 0, x_362); +lean_ctor_set(x_454, 1, x_2); +lean_ctor_set(x_454, 2, x_3); +lean_ctor_set(x_454, 3, x_365); +lean_ctor_set_uint8(x_454, sizeof(void*)*4, x_453); +return x_454; +} +default: +{ +uint8_t x_455; +x_455 = l_Std_RBNode_isRed___rarg(x_365); +if (x_455 == 0) +{ +lean_object* x_456; uint8_t x_457; lean_object* x_458; +x_456 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_365, x_2, x_3); +x_457 = 1; +x_458 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_458, 0, x_362); +lean_ctor_set(x_458, 1, x_363); +lean_ctor_set(x_458, 2, x_364); +lean_ctor_set(x_458, 3, x_456); +lean_ctor_set_uint8(x_458, sizeof(void*)*4, x_457); +return x_458; +} +else +{ +lean_object* x_459; lean_object* x_460; +x_459 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_365, x_2, x_3); +x_460 = lean_ctor_get(x_459, 0); +lean_inc(x_460); +if (lean_obj_tag(x_460) == 0) +{ +lean_object* x_461; +x_461 = lean_ctor_get(x_459, 3); +lean_inc(x_461); +if (lean_obj_tag(x_461) == 0) +{ +lean_object* x_462; lean_object* x_463; lean_object* x_464; uint8_t x_465; lean_object* x_466; uint8_t x_467; lean_object* x_468; +x_462 = lean_ctor_get(x_459, 1); +lean_inc(x_462); +x_463 = lean_ctor_get(x_459, 2); +lean_inc(x_463); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_464 = x_459; +} else { + lean_dec_ref(x_459); + x_464 = lean_box(0); +} +x_465 = 0; +if (lean_is_scalar(x_464)) { + x_466 = lean_alloc_ctor(1, 4, 1); +} else { + x_466 = x_464; +} +lean_ctor_set(x_466, 0, x_461); +lean_ctor_set(x_466, 1, x_462); +lean_ctor_set(x_466, 2, x_463); +lean_ctor_set(x_466, 3, x_461); +lean_ctor_set_uint8(x_466, sizeof(void*)*4, x_465); +x_467 = 1; +x_468 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_468, 0, x_362); +lean_ctor_set(x_468, 1, x_363); +lean_ctor_set(x_468, 2, x_364); +lean_ctor_set(x_468, 3, x_466); +lean_ctor_set_uint8(x_468, sizeof(void*)*4, x_467); +return x_468; +} +else +{ +uint8_t x_469; +x_469 = lean_ctor_get_uint8(x_461, sizeof(void*)*4); +if (x_469 == 0) +{ +lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; uint8_t x_478; lean_object* x_479; lean_object* x_480; uint8_t x_481; lean_object* x_482; +x_470 = lean_ctor_get(x_459, 1); +lean_inc(x_470); +x_471 = lean_ctor_get(x_459, 2); +lean_inc(x_471); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_472 = x_459; +} else { + lean_dec_ref(x_459); + x_472 = lean_box(0); +} +x_473 = lean_ctor_get(x_461, 0); +lean_inc(x_473); +x_474 = lean_ctor_get(x_461, 1); +lean_inc(x_474); +x_475 = lean_ctor_get(x_461, 2); +lean_inc(x_475); +x_476 = lean_ctor_get(x_461, 3); +lean_inc(x_476); +if (lean_is_exclusive(x_461)) { + lean_ctor_release(x_461, 0); + lean_ctor_release(x_461, 1); + lean_ctor_release(x_461, 2); + lean_ctor_release(x_461, 3); + x_477 = x_461; +} else { + lean_dec_ref(x_461); + x_477 = lean_box(0); +} +x_478 = 1; +if (lean_is_scalar(x_477)) { + x_479 = lean_alloc_ctor(1, 4, 1); +} else { + x_479 = x_477; +} +lean_ctor_set(x_479, 0, x_362); +lean_ctor_set(x_479, 1, x_363); +lean_ctor_set(x_479, 2, x_364); +lean_ctor_set(x_479, 3, x_460); +lean_ctor_set_uint8(x_479, sizeof(void*)*4, x_478); +if (lean_is_scalar(x_472)) { + x_480 = lean_alloc_ctor(1, 4, 1); +} else { + x_480 = x_472; +} +lean_ctor_set(x_480, 0, x_473); +lean_ctor_set(x_480, 1, x_474); +lean_ctor_set(x_480, 2, x_475); +lean_ctor_set(x_480, 3, x_476); +lean_ctor_set_uint8(x_480, sizeof(void*)*4, x_478); +x_481 = 0; +x_482 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_482, 0, x_479); +lean_ctor_set(x_482, 1, x_470); +lean_ctor_set(x_482, 2, x_471); +lean_ctor_set(x_482, 3, x_480); +lean_ctor_set_uint8(x_482, sizeof(void*)*4, x_481); +return x_482; +} +else +{ +lean_object* x_483; lean_object* x_484; lean_object* x_485; uint8_t x_486; lean_object* x_487; uint8_t x_488; lean_object* x_489; +x_483 = lean_ctor_get(x_459, 1); +lean_inc(x_483); +x_484 = lean_ctor_get(x_459, 2); +lean_inc(x_484); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_485 = x_459; +} else { + lean_dec_ref(x_459); + x_485 = lean_box(0); +} +x_486 = 0; +if (lean_is_scalar(x_485)) { + x_487 = lean_alloc_ctor(1, 4, 1); +} else { + x_487 = x_485; +} +lean_ctor_set(x_487, 0, x_460); +lean_ctor_set(x_487, 1, x_483); +lean_ctor_set(x_487, 2, x_484); +lean_ctor_set(x_487, 3, x_461); +lean_ctor_set_uint8(x_487, sizeof(void*)*4, x_486); +x_488 = 1; +x_489 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_489, 0, x_362); +lean_ctor_set(x_489, 1, x_363); +lean_ctor_set(x_489, 2, x_364); +lean_ctor_set(x_489, 3, x_487); +lean_ctor_set_uint8(x_489, sizeof(void*)*4, x_488); +return x_489; +} +} +} +else +{ +uint8_t x_490; +x_490 = lean_ctor_get_uint8(x_460, sizeof(void*)*4); +if (x_490 == 0) +{ +lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; uint8_t x_500; lean_object* x_501; lean_object* x_502; uint8_t x_503; lean_object* x_504; +x_491 = lean_ctor_get(x_459, 1); +lean_inc(x_491); +x_492 = lean_ctor_get(x_459, 2); +lean_inc(x_492); +x_493 = lean_ctor_get(x_459, 3); +lean_inc(x_493); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_494 = x_459; +} else { + lean_dec_ref(x_459); + x_494 = lean_box(0); +} +x_495 = lean_ctor_get(x_460, 0); +lean_inc(x_495); +x_496 = lean_ctor_get(x_460, 1); +lean_inc(x_496); +x_497 = lean_ctor_get(x_460, 2); +lean_inc(x_497); +x_498 = lean_ctor_get(x_460, 3); +lean_inc(x_498); +if (lean_is_exclusive(x_460)) { + lean_ctor_release(x_460, 0); + lean_ctor_release(x_460, 1); + lean_ctor_release(x_460, 2); + lean_ctor_release(x_460, 3); + x_499 = x_460; +} else { + lean_dec_ref(x_460); + x_499 = lean_box(0); +} +x_500 = 1; +if (lean_is_scalar(x_499)) { + x_501 = lean_alloc_ctor(1, 4, 1); +} else { + x_501 = x_499; +} +lean_ctor_set(x_501, 0, x_362); +lean_ctor_set(x_501, 1, x_363); +lean_ctor_set(x_501, 2, x_364); +lean_ctor_set(x_501, 3, x_495); +lean_ctor_set_uint8(x_501, sizeof(void*)*4, x_500); +if (lean_is_scalar(x_494)) { + x_502 = lean_alloc_ctor(1, 4, 1); +} else { + x_502 = x_494; +} +lean_ctor_set(x_502, 0, x_498); +lean_ctor_set(x_502, 1, x_491); +lean_ctor_set(x_502, 2, x_492); +lean_ctor_set(x_502, 3, x_493); +lean_ctor_set_uint8(x_502, sizeof(void*)*4, x_500); +x_503 = 0; +x_504 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_504, 0, x_501); +lean_ctor_set(x_504, 1, x_496); +lean_ctor_set(x_504, 2, x_497); +lean_ctor_set(x_504, 3, x_502); +lean_ctor_set_uint8(x_504, sizeof(void*)*4, x_503); +return x_504; +} +else +{ +lean_object* x_505; +x_505 = lean_ctor_get(x_459, 3); +lean_inc(x_505); +if (lean_obj_tag(x_505) == 0) +{ +lean_object* x_506; lean_object* x_507; lean_object* x_508; uint8_t x_509; lean_object* x_510; uint8_t x_511; lean_object* x_512; +x_506 = lean_ctor_get(x_459, 1); +lean_inc(x_506); +x_507 = lean_ctor_get(x_459, 2); +lean_inc(x_507); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_508 = x_459; +} else { + lean_dec_ref(x_459); + x_508 = lean_box(0); +} +x_509 = 0; +if (lean_is_scalar(x_508)) { + x_510 = lean_alloc_ctor(1, 4, 1); +} else { + x_510 = x_508; +} +lean_ctor_set(x_510, 0, x_460); +lean_ctor_set(x_510, 1, x_506); +lean_ctor_set(x_510, 2, x_507); +lean_ctor_set(x_510, 3, x_505); +lean_ctor_set_uint8(x_510, sizeof(void*)*4, x_509); +x_511 = 1; +x_512 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_512, 0, x_362); +lean_ctor_set(x_512, 1, x_363); +lean_ctor_set(x_512, 2, x_364); +lean_ctor_set(x_512, 3, x_510); +lean_ctor_set_uint8(x_512, sizeof(void*)*4, x_511); +return x_512; +} +else +{ +uint8_t x_513; +x_513 = lean_ctor_get_uint8(x_505, sizeof(void*)*4); +if (x_513 == 0) +{ +lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; uint8_t x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; uint8_t x_526; lean_object* x_527; +x_514 = lean_ctor_get(x_459, 1); +lean_inc(x_514); +x_515 = lean_ctor_get(x_459, 2); +lean_inc(x_515); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_516 = x_459; +} else { + lean_dec_ref(x_459); + x_516 = lean_box(0); +} +x_517 = lean_ctor_get(x_505, 0); +lean_inc(x_517); +x_518 = lean_ctor_get(x_505, 1); +lean_inc(x_518); +x_519 = lean_ctor_get(x_505, 2); +lean_inc(x_519); +x_520 = lean_ctor_get(x_505, 3); +lean_inc(x_520); +if (lean_is_exclusive(x_505)) { + lean_ctor_release(x_505, 0); + lean_ctor_release(x_505, 1); + lean_ctor_release(x_505, 2); + lean_ctor_release(x_505, 3); + x_521 = x_505; +} else { + lean_dec_ref(x_505); + x_521 = lean_box(0); +} +x_522 = 1; +lean_inc(x_460); +if (lean_is_scalar(x_521)) { + x_523 = lean_alloc_ctor(1, 4, 1); +} else { + x_523 = x_521; +} +lean_ctor_set(x_523, 0, x_362); +lean_ctor_set(x_523, 1, x_363); +lean_ctor_set(x_523, 2, x_364); +lean_ctor_set(x_523, 3, x_460); +if (lean_is_exclusive(x_460)) { + lean_ctor_release(x_460, 0); + lean_ctor_release(x_460, 1); + lean_ctor_release(x_460, 2); + lean_ctor_release(x_460, 3); + x_524 = x_460; +} else { + lean_dec_ref(x_460); + x_524 = lean_box(0); +} +lean_ctor_set_uint8(x_523, sizeof(void*)*4, x_522); +if (lean_is_scalar(x_524)) { + x_525 = lean_alloc_ctor(1, 4, 1); +} else { + x_525 = x_524; +} +lean_ctor_set(x_525, 0, x_517); +lean_ctor_set(x_525, 1, x_518); +lean_ctor_set(x_525, 2, x_519); +lean_ctor_set(x_525, 3, x_520); +lean_ctor_set_uint8(x_525, sizeof(void*)*4, x_522); +x_526 = 0; +if (lean_is_scalar(x_516)) { + x_527 = lean_alloc_ctor(1, 4, 1); +} else { + x_527 = x_516; +} +lean_ctor_set(x_527, 0, x_523); +lean_ctor_set(x_527, 1, x_514); +lean_ctor_set(x_527, 2, x_515); +lean_ctor_set(x_527, 3, x_525); +lean_ctor_set_uint8(x_527, sizeof(void*)*4, x_526); +return x_527; +} +else +{ +lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; uint8_t x_537; lean_object* x_538; uint8_t x_539; lean_object* x_540; +x_528 = lean_ctor_get(x_459, 1); +lean_inc(x_528); +x_529 = lean_ctor_get(x_459, 2); +lean_inc(x_529); +if (lean_is_exclusive(x_459)) { + lean_ctor_release(x_459, 0); + lean_ctor_release(x_459, 1); + lean_ctor_release(x_459, 2); + lean_ctor_release(x_459, 3); + x_530 = x_459; +} else { + lean_dec_ref(x_459); + x_530 = lean_box(0); +} +x_531 = lean_ctor_get(x_460, 0); +lean_inc(x_531); +x_532 = lean_ctor_get(x_460, 1); +lean_inc(x_532); +x_533 = lean_ctor_get(x_460, 2); +lean_inc(x_533); +x_534 = lean_ctor_get(x_460, 3); +lean_inc(x_534); +if (lean_is_exclusive(x_460)) { + lean_ctor_release(x_460, 0); + lean_ctor_release(x_460, 1); + lean_ctor_release(x_460, 2); + lean_ctor_release(x_460, 3); + x_535 = x_460; +} else { + lean_dec_ref(x_460); + x_535 = lean_box(0); +} +if (lean_is_scalar(x_535)) { + x_536 = lean_alloc_ctor(1, 4, 1); +} else { + x_536 = x_535; +} +lean_ctor_set(x_536, 0, x_531); +lean_ctor_set(x_536, 1, x_532); +lean_ctor_set(x_536, 2, x_533); +lean_ctor_set(x_536, 3, x_534); +lean_ctor_set_uint8(x_536, sizeof(void*)*4, x_513); +x_537 = 0; +if (lean_is_scalar(x_530)) { + x_538 = lean_alloc_ctor(1, 4, 1); +} else { + x_538 = x_530; +} +lean_ctor_set(x_538, 0, x_536); +lean_ctor_set(x_538, 1, x_528); +lean_ctor_set(x_538, 2, x_529); +lean_ctor_set(x_538, 3, x_505); +lean_ctor_set_uint8(x_538, sizeof(void*)*4, x_537); +x_539 = 1; +x_540 = lean_alloc_ctor(1, 4, 1); +lean_ctor_set(x_540, 0, x_362); +lean_ctor_set(x_540, 1, x_363); +lean_ctor_set(x_540, 2, x_364); +lean_ctor_set(x_540, 3, x_538); +lean_ctor_set_uint8(x_540, sizeof(void*)*4, x_539); +return x_540; +} +} +} +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = l_Std_RBNode_isRed___rarg(x_1); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_1, x_2, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +x_6 = l_Std_RBNode_ins___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(x_1, x_2, x_3); +x_7 = l_Std_RBNode_setBlack___rarg(x_6); +return x_7; +} +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Init.Util", 9); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("getElem!", 8); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("index out of bounds", 19); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__1; +x_2 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__2; +x_3 = lean_unsigned_to_nat(69u); +x_4 = lean_unsigned_to_nat(36u); +x_5 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +uint8_t x_16; +x_16 = lean_nat_dec_le(x_8, x_7); +if (x_16 == 0) +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_unsigned_to_nat(0u); +x_18 = lean_nat_dec_eq(x_6, x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_81; +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_sub(x_6, x_19); +lean_dec(x_6); +x_27 = lean_ctor_get(x_10, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_10, 1); +lean_inc(x_28); +if (lean_is_exclusive(x_10)) { + lean_ctor_release(x_10, 0); + lean_ctor_release(x_10, 1); + x_29 = x_10; +} else { + lean_dec_ref(x_10); + x_29 = lean_box(0); +} +x_81 = l_Array_contains___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__2(x_3, x_7); +if (x_81 == 0) +{ +lean_object* x_82; lean_object* x_83; +lean_dec(x_29); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_27); +lean_ctor_set(x_82, 1, x_28); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_82); +x_21 = x_83; +x_22 = x_15; +goto block_26; +} +else +{ +uint8_t x_84; +x_84 = lean_nat_dec_lt(x_7, x_5); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; +x_85 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4; +x_86 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_85); +x_30 = x_86; +goto block_80; +} +else +{ +lean_object* x_87; +x_87 = lean_array_fget(x_4, x_7); +x_30 = x_87; +goto block_80; +} +} +block_26: +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_nat_add(x_7, x_9); +lean_dec(x_7); +x_6 = x_20; +x_7 = x_24; +x_10 = x_23; +x_15 = x_22; +goto _start; +} +block_80: +{ +lean_object* x_31; +x_31 = l_Array_indexOfAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__1(x_1, x_30, x_17); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_30); +if (lean_is_scalar(x_29)) { + x_32 = lean_alloc_ctor(0, 2, 0); +} else { + x_32 = x_29; +} +lean_ctor_set(x_32, 0, x_27); +lean_ctor_set(x_32, 1, x_28); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_32); +x_21 = x_33; +x_22 = x_15; +goto block_26; +} +else +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_31, 0); +lean_inc(x_34); +lean_dec(x_31); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_30); +x_35 = lean_infer_type(x_30, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_35) == 0) +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_38 = lean_whnf(x_36, x_11, x_12, x_13, x_14, x_37); +if (lean_obj_tag(x_38) == 0) +{ +lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = l_Lean_Expr_isForall(x_39); +lean_dec(x_39); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +lean_dec(x_34); +lean_dec(x_30); +if (lean_is_scalar(x_29)) { + x_42 = lean_alloc_ctor(0, 2, 0); +} else { + x_42 = x_29; +} +lean_ctor_set(x_42, 0, x_27); +lean_ctor_set(x_42, 1, x_28); +x_43 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_43, 0, x_42); +x_21 = x_43; +x_22 = x_40; +goto block_26; +} +else +{ +lean_object* x_44; uint8_t x_45; lean_object* x_46; +x_44 = lean_array_get_size(x_28); +x_45 = lean_nat_dec_lt(x_34, x_44); +lean_dec(x_44); +x_46 = l_Lean_Expr_fvarId_x21(x_30); +if (x_45 == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_dec(x_34); +x_47 = lean_box(0); +x_48 = l_Std_RBNode_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(x_27, x_46, x_47); +if (lean_is_scalar(x_29)) { + x_49 = lean_alloc_ctor(0, 2, 0); +} else { + x_49 = x_29; +} +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_28); +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +x_21 = x_50; +x_22 = x_40; +goto block_26; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_51 = lean_array_fget(x_28, x_34); +x_52 = lean_box(0); +x_53 = lean_array_fset(x_28, x_34, x_52); +x_54 = !lean_is_exclusive(x_51); +if (x_54 == 0) +{ +uint8_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_55 = 1; +lean_ctor_set_uint8(x_51, sizeof(void*)*1 + 4, x_55); +x_56 = lean_array_fset(x_53, x_34, x_51); +lean_dec(x_34); +x_57 = l_Std_RBNode_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(x_27, x_46, x_52); +if (lean_is_scalar(x_29)) { + x_58 = lean_alloc_ctor(0, 2, 0); +} else { + x_58 = x_29; +} +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_56); +x_59 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_59, 0, x_58); +x_21 = x_59; +x_22 = x_40; +goto block_26; +} +else +{ +uint8_t x_60; uint8_t x_61; lean_object* 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; lean_object* x_70; lean_object* x_71; +x_60 = lean_ctor_get_uint8(x_51, sizeof(void*)*1); +x_61 = lean_ctor_get_uint8(x_51, sizeof(void*)*1 + 1); +x_62 = lean_ctor_get(x_51, 0); +x_63 = lean_ctor_get_uint8(x_51, sizeof(void*)*1 + 2); +x_64 = lean_ctor_get_uint8(x_51, sizeof(void*)*1 + 3); +x_65 = lean_ctor_get_uint8(x_51, sizeof(void*)*1 + 5); +lean_inc(x_62); +lean_dec(x_51); +x_66 = 1; +x_67 = lean_alloc_ctor(0, 1, 6); +lean_ctor_set(x_67, 0, x_62); +lean_ctor_set_uint8(x_67, sizeof(void*)*1, x_60); +lean_ctor_set_uint8(x_67, sizeof(void*)*1 + 1, x_61); +lean_ctor_set_uint8(x_67, sizeof(void*)*1 + 2, x_63); +lean_ctor_set_uint8(x_67, sizeof(void*)*1 + 3, x_64); +lean_ctor_set_uint8(x_67, sizeof(void*)*1 + 4, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*1 + 5, x_65); +x_68 = lean_array_fset(x_53, x_34, x_67); +lean_dec(x_34); +x_69 = l_Std_RBNode_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(x_27, x_46, x_52); +if (lean_is_scalar(x_29)) { + x_70 = lean_alloc_ctor(0, 2, 0); +} else { + x_70 = x_29; +} +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_68); +x_71 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_71, 0, x_70); +x_21 = x_71; +x_22 = x_40; +goto block_26; +} +} +} +} +else +{ +uint8_t x_72; +lean_dec(x_34); +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_7); +x_72 = !lean_is_exclusive(x_38); +if (x_72 == 0) +{ +return x_38; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_38, 0); +x_74 = lean_ctor_get(x_38, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_38); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +return x_75; +} +} +} +else +{ +uint8_t x_76; +lean_dec(x_34); +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_7); +x_76 = !lean_is_exclusive(x_35); +if (x_76 == 0) +{ +return x_35; +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_35, 0); +x_78 = lean_ctor_get(x_35, 1); +lean_inc(x_78); +lean_inc(x_77); +lean_dec(x_35); +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; +} +} +} +} +} +else +{ +lean_object* x_88; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_7); +lean_dec(x_6); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_10); +lean_ctor_set(x_88, 1, x_15); +return x_88; +} +} +else +{ +lean_object* x_89; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_7); +lean_dec(x_6); +x_89 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_89, 0, x_10); +lean_ctor_set(x_89, 1, x_15); +return x_89; +} +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; +x_15 = lean_nat_dec_le(x_7, x_6); +if (x_15 == 0) +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_eq(x_5, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_80; +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_sub(x_5, x_18); +lean_dec(x_5); +x_26 = lean_ctor_get(x_9, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_9, 1); +lean_inc(x_27); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + lean_ctor_release(x_9, 1); + x_28 = x_9; +} else { + lean_dec_ref(x_9); + x_28 = lean_box(0); +} +x_80 = l_Array_contains___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__2(x_2, x_6); +if (x_80 == 0) +{ +lean_object* x_81; lean_object* x_82; +lean_dec(x_28); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_26); +lean_ctor_set(x_81, 1, x_27); +x_82 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_82, 0, x_81); +x_20 = x_82; +x_21 = x_14; +goto block_25; +} +else +{ +uint8_t x_83; +x_83 = lean_nat_dec_lt(x_6, x_4); +if (x_83 == 0) +{ +lean_object* x_84; lean_object* x_85; +x_84 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4; +x_85 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_84); +x_29 = x_85; +goto block_79; +} +else +{ +lean_object* x_86; +x_86 = lean_array_fget(x_3, x_6); +x_29 = x_86; +goto block_79; +} +} +block_25: +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_nat_add(x_6, x_8); +lean_dec(x_6); +x_5 = x_19; +x_6 = x_23; +x_9 = x_22; +x_14 = x_21; +goto _start; +} +block_79: +{ +lean_object* x_30; +x_30 = l_Array_indexOfAux___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps_visit___spec__1(x_1, x_29, x_16); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; +lean_dec(x_29); +if (lean_is_scalar(x_28)) { + x_31 = lean_alloc_ctor(0, 2, 0); +} else { + x_31 = x_28; +} +lean_ctor_set(x_31, 0, x_26); +lean_ctor_set(x_31, 1, x_27); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +x_20 = x_32; +x_21 = x_14; +goto block_25; +} +else +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_30, 0); +lean_inc(x_33); +lean_dec(x_30); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_29); +x_34 = lean_infer_type(x_29, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_37 = lean_whnf(x_35, x_10, x_11, x_12, x_13, x_36); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = l_Lean_Expr_isForall(x_38); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_33); +lean_dec(x_29); +if (lean_is_scalar(x_28)) { + x_41 = lean_alloc_ctor(0, 2, 0); +} else { + x_41 = x_28; +} +lean_ctor_set(x_41, 0, x_26); +lean_ctor_set(x_41, 1, x_27); +x_42 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_42, 0, x_41); +x_20 = x_42; +x_21 = x_39; +goto block_25; +} +else +{ +lean_object* x_43; uint8_t x_44; lean_object* x_45; +x_43 = lean_array_get_size(x_27); +x_44 = lean_nat_dec_lt(x_33, x_43); +lean_dec(x_43); +x_45 = l_Lean_Expr_fvarId_x21(x_29); +if (x_44 == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +lean_dec(x_33); +x_46 = lean_box(0); +x_47 = l_Std_RBNode_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(x_26, x_45, x_46); +if (lean_is_scalar(x_28)) { + x_48 = lean_alloc_ctor(0, 2, 0); +} else { + x_48 = x_28; +} +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_27); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +x_20 = x_49; +x_21 = x_39; +goto block_25; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_array_fget(x_27, x_33); +x_51 = lean_box(0); +x_52 = lean_array_fset(x_27, x_33, x_51); +x_53 = !lean_is_exclusive(x_50); +if (x_53 == 0) +{ +uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_54 = 1; +lean_ctor_set_uint8(x_50, sizeof(void*)*1 + 4, x_54); +x_55 = lean_array_fset(x_52, x_33, x_50); +lean_dec(x_33); +x_56 = l_Std_RBNode_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(x_26, x_45, x_51); +if (lean_is_scalar(x_28)) { + x_57 = lean_alloc_ctor(0, 2, 0); +} else { + x_57 = x_28; +} +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_55); +x_58 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_58, 0, x_57); +x_20 = x_58; +x_21 = x_39; +goto block_25; +} +else +{ +uint8_t x_59; uint8_t x_60; lean_object* x_61; uint8_t x_62; uint8_t x_63; uint8_t x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_59 = lean_ctor_get_uint8(x_50, sizeof(void*)*1); +x_60 = lean_ctor_get_uint8(x_50, sizeof(void*)*1 + 1); +x_61 = lean_ctor_get(x_50, 0); +x_62 = lean_ctor_get_uint8(x_50, sizeof(void*)*1 + 2); +x_63 = lean_ctor_get_uint8(x_50, sizeof(void*)*1 + 3); +x_64 = lean_ctor_get_uint8(x_50, sizeof(void*)*1 + 5); +lean_inc(x_61); +lean_dec(x_50); +x_65 = 1; +x_66 = lean_alloc_ctor(0, 1, 6); +lean_ctor_set(x_66, 0, x_61); +lean_ctor_set_uint8(x_66, sizeof(void*)*1, x_59); +lean_ctor_set_uint8(x_66, sizeof(void*)*1 + 1, x_60); +lean_ctor_set_uint8(x_66, sizeof(void*)*1 + 2, x_62); +lean_ctor_set_uint8(x_66, sizeof(void*)*1 + 3, x_63); +lean_ctor_set_uint8(x_66, sizeof(void*)*1 + 4, x_65); +lean_ctor_set_uint8(x_66, sizeof(void*)*1 + 5, x_64); +x_67 = lean_array_fset(x_52, x_33, x_66); +lean_dec(x_33); +x_68 = l_Std_RBNode_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(x_26, x_45, x_51); +if (lean_is_scalar(x_28)) { + x_69 = lean_alloc_ctor(0, 2, 0); +} else { + x_69 = x_28; +} +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_67); +x_70 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_70, 0, x_69); +x_20 = x_70; +x_21 = x_39; +goto block_25; +} +} +} +} +else +{ +uint8_t x_71; +lean_dec(x_33); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +x_71 = !lean_is_exclusive(x_37); +if (x_71 == 0) +{ +return x_37; +} +else +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_72 = lean_ctor_get(x_37, 0); +x_73 = lean_ctor_get(x_37, 1); +lean_inc(x_73); +lean_inc(x_72); +lean_dec(x_37); +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set(x_74, 1, x_73); +return x_74; +} +} +} +else +{ +uint8_t x_75; +lean_dec(x_33); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +x_75 = !lean_is_exclusive(x_34); +if (x_75 == 0) +{ +return x_34; +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_34, 0); +x_77 = lean_ctor_get(x_34, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_34); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; +} +} +} +} +} +else +{ +lean_object* x_87; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_9); +lean_ctor_set(x_87, 1, x_14); +return x_87; +} +} +else +{ +lean_object* x_88; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_9); +lean_ctor_set(x_88, 1, x_14); +return x_88; +} +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_findCore___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__5(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_4 = lean_ctor_get(x_1, 0); +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_1, 2); +x_7 = lean_ctor_get(x_1, 3); +x_8 = l_Lean_Name_quickCmp(x_2, x_5); +switch (x_8) { +case 0: +{ +x_1 = x_4; +goto _start; +} +case 1: +{ +lean_object* x_10; lean_object* x_11; +lean_inc(x_6); +lean_inc(x_5); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_5); +lean_ctor_set(x_10, 1, x_6); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; +} +default: +{ +x_1 = x_7; +goto _start; +} +} +} +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Decidable", 9); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; +x_8 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__2; +x_9 = l_Lean_Expr_isAppOf(x_2, x_8); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_7); +return x_11; +} +} +LEAN_EXPORT uint8_t l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; +x_3 = l_Lean_Expr_isFVar(x_2); +if (x_3 == 0) +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = 0; +return x_4; +} +else +{ +lean_object* x_5; lean_object* x_6; +x_5 = l_Lean_Expr_fvarId_x21(x_2); +x_6 = l_Std_RBNode_findCore___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__5(x_1, x_5); +lean_dec(x_5); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_7; +x_7 = 0; +return x_7; +} +else +{ +uint8_t x_8; +lean_dec(x_6); +x_8 = 1; +return x_8; +} +} +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___boxed), 7, 0); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_levelZero; +x_2 = l_Lean_Expr_sort___override(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; +x_15 = lean_nat_dec_le(x_7, x_6); +if (x_15 == 0) +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_eq(x_5, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_131; +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_sub(x_5, x_18); +lean_dec(x_5); +x_26 = lean_ctor_get(x_9, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_9, 1); +lean_inc(x_27); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + lean_ctor_release(x_9, 1); + x_28 = x_9; +} else { + lean_dec_ref(x_9); + x_28 = lean_box(0); +} +x_131 = lean_nat_dec_lt(x_6, x_4); +if (x_131 == 0) +{ +lean_object* x_132; lean_object* x_133; +x_132 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4; +x_133 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_132); +x_29 = x_133; +goto block_130; +} +else +{ +lean_object* x_134; +x_134 = lean_array_fget(x_2, x_6); +x_29 = x_134; +goto block_130; +} +block_25: +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_nat_add(x_6, x_8); +lean_dec(x_6); +x_5 = x_19; +x_6 = x_23; +x_9 = x_22; +x_14 = x_21; +goto _start; +} +block_130: +{ +lean_object* x_30; +lean_inc(x_10); +x_30 = l_Lean_Meta_getFVarLocalDecl(x_29, x_10, x_11, x_12, x_13, x_14); +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; uint8_t x_36; uint8_t x_37; lean_object* x_38; lean_object* x_99; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = l_Lean_LocalDecl_type(x_31); +lean_inc(x_33); +lean_inc(x_2); +x_34 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(x_2, x_33); +x_35 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(x_27, x_34); +lean_dec(x_27); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_33); +x_99 = l_Lean_Meta_isProp(x_33, x_10, x_11, x_12, x_13, x_32); +if (lean_obj_tag(x_26) == 0) +{ +if (lean_obj_tag(x_99) == 0) +{ +lean_object* x_100; lean_object* x_101; uint8_t x_102; uint8_t x_103; +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_99, 1); +lean_inc(x_101); +lean_dec(x_99); +x_102 = 0; +x_103 = lean_unbox(x_100); +lean_dec(x_100); +x_36 = x_102; +x_37 = x_103; +x_38 = x_101; +goto block_98; +} +else +{ +uint8_t x_104; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_31); +lean_dec(x_28); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_104 = !lean_is_exclusive(x_99); +if (x_104 == 0) +{ +return x_99; +} +else +{ +lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_105 = lean_ctor_get(x_99, 0); +x_106 = lean_ctor_get(x_99, 1); +lean_inc(x_106); +lean_inc(x_105); +lean_dec(x_99); +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 +{ +lean_object* x_108; lean_object* x_109; +lean_inc(x_26); +x_108 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__2___boxed), 2, 1); +lean_closure_set(x_108, 0, x_26); +lean_inc(x_33); +x_109 = l_Lean_Expr_FindImpl_findUnsafe_x3f(x_108, x_33); +if (lean_obj_tag(x_109) == 0) +{ +if (lean_obj_tag(x_99) == 0) +{ +lean_object* x_110; lean_object* x_111; uint8_t x_112; uint8_t x_113; +x_110 = lean_ctor_get(x_99, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_99, 1); +lean_inc(x_111); +lean_dec(x_99); +x_112 = 0; +x_113 = lean_unbox(x_110); +lean_dec(x_110); +x_36 = x_112; +x_37 = x_113; +x_38 = x_111; +goto block_98; +} +else +{ +uint8_t x_114; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_31); +lean_dec(x_28); +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_114 = !lean_is_exclusive(x_99); +if (x_114 == 0) +{ +return x_99; +} +else +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_99, 0); +x_116 = lean_ctor_get(x_99, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_99); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; +} +} +} +else +{ +lean_dec(x_109); +if (lean_obj_tag(x_99) == 0) +{ +lean_object* x_118; lean_object* x_119; uint8_t x_120; uint8_t x_121; +x_118 = lean_ctor_get(x_99, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_99, 1); +lean_inc(x_119); +lean_dec(x_99); +x_120 = 1; +x_121 = lean_unbox(x_118); +lean_dec(x_118); +x_36 = x_120; +x_37 = x_121; +x_38 = x_119; +goto block_98; +} +else +{ +uint8_t x_122; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_31); +lean_dec(x_28); +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_122 = !lean_is_exclusive(x_99); +if (x_122 == 0) +{ +return x_99; +} +else +{ +lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_123 = lean_ctor_get(x_99, 0); +x_124 = lean_ctor_get(x_99, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_99); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +return x_125; +} +} +} +} +block_98: +{ +lean_object* x_39; lean_object* x_40; +x_39 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__1; +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_33); +x_40 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_33, x_39, x_10, x_11, x_12, x_13, x_38); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; lean_object* x_42; uint8_t x_43; uint8_t x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; uint8_t x_48; uint8_t x_49; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = l_Lean_LocalDecl_binderInfo(x_31); +lean_dec(x_31); +x_44 = 0; +x_45 = lean_alloc_ctor(0, 1, 6); +lean_ctor_set(x_45, 0, x_34); +lean_ctor_set_uint8(x_45, sizeof(void*)*1, x_43); +lean_ctor_set_uint8(x_45, sizeof(void*)*1 + 1, x_44); +lean_ctor_set_uint8(x_45, sizeof(void*)*1 + 2, x_37); +x_46 = lean_unbox(x_41); +lean_dec(x_41); +lean_ctor_set_uint8(x_45, sizeof(void*)*1 + 3, x_46); +lean_ctor_set_uint8(x_45, sizeof(void*)*1 + 4, x_44); +lean_ctor_set_uint8(x_45, sizeof(void*)*1 + 5, x_36); +x_47 = lean_array_push(x_35, x_45); +x_48 = 3; +x_49 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_43, x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; +lean_dec(x_33); +if (lean_is_scalar(x_28)) { + x_50 = lean_alloc_ctor(0, 2, 0); +} else { + x_50 = x_28; +} +lean_ctor_set(x_50, 0, x_26); +lean_ctor_set(x_50, 1, x_47); +x_51 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_51, 0, x_50); +x_20 = x_51; +x_21 = x_42; +goto block_25; +} +else +{ +lean_object* x_52; +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_33); +x_52 = l_Lean_Meta_isClass_x3f(x_33, x_10, x_11, x_12, x_13, x_42); +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_53; +x_53 = lean_ctor_get(x_52, 0); +lean_inc(x_53); +if (lean_obj_tag(x_53) == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; +lean_dec(x_33); +x_54 = lean_ctor_get(x_52, 1); +lean_inc(x_54); +lean_dec(x_52); +if (lean_is_scalar(x_28)) { + x_55 = lean_alloc_ctor(0, 2, 0); +} else { + x_55 = x_28; +} +lean_ctor_set(x_55, 0, x_26); +lean_ctor_set(x_55, 1, x_47); +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_55); +x_20 = x_56; +x_21 = x_54; +goto block_25; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_57 = lean_ctor_get(x_52, 1); +lean_inc(x_57); +lean_dec(x_52); +x_58 = lean_ctor_get(x_53, 0); +lean_inc(x_58); +lean_dec(x_53); +x_59 = lean_st_ref_get(x_13, x_57); +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = lean_ctor_get(x_60, 0); +lean_inc(x_62); +lean_dec(x_60); +x_63 = l_Lean_getOutParamPositions_x3f(x_62, x_58); +if (lean_obj_tag(x_63) == 0) +{ +lean_object* x_64; lean_object* x_65; +lean_dec(x_33); +if (lean_is_scalar(x_28)) { + x_64 = lean_alloc_ctor(0, 2, 0); +} else { + x_64 = x_28; +} +lean_ctor_set(x_64, 0, x_26); +lean_ctor_set(x_64, 1, x_47); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_20 = x_65; +x_21 = x_61; +goto block_25; +} +else +{ +lean_object* x_66; uint8_t x_67; +x_66 = lean_ctor_get(x_63, 0); +lean_inc(x_66); +lean_dec(x_63); +x_67 = l_Array_isEmpty___rarg(x_66); +if (x_67 == 0) +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_68 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_33, x_16); +x_69 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__2; +lean_inc(x_68); +x_70 = lean_mk_array(x_68, x_69); +x_71 = lean_nat_sub(x_68, x_18); +lean_dec(x_68); +x_72 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_33, x_70, x_71); +x_73 = lean_array_get_size(x_72); +if (lean_is_scalar(x_28)) { + x_74 = lean_alloc_ctor(0, 2, 0); +} else { + x_74 = x_28; +} +lean_ctor_set(x_74, 0, x_26); +lean_ctor_set(x_74, 1, x_47); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_73); +x_75 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__4(x_2, x_66, x_72, x_73, x_73, x_16, x_73, x_18, x_74, x_10, x_11, x_12, x_13, x_61); +lean_dec(x_73); +lean_dec(x_72); +lean_dec(x_66); +if (lean_obj_tag(x_75) == 0) +{ +lean_object* x_76; lean_object* x_77; uint8_t x_78; +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_75, 1); +lean_inc(x_77); +lean_dec(x_75); +x_78 = !lean_is_exclusive(x_76); +if (x_78 == 0) +{ +lean_object* x_79; +x_79 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_79, 0, x_76); +x_20 = x_79; +x_21 = x_77; +goto block_25; +} +else +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_76, 0); +x_81 = lean_ctor_get(x_76, 1); +lean_inc(x_81); +lean_inc(x_80); +lean_dec(x_76); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_82); +x_20 = x_83; +x_21 = x_77; +goto block_25; +} +} +else +{ +uint8_t x_84; +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_84 = !lean_is_exclusive(x_75); +if (x_84 == 0) +{ +return x_75; +} +else +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_75, 0); +x_86 = lean_ctor_get(x_75, 1); +lean_inc(x_86); +lean_inc(x_85); +lean_dec(x_75); +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +return x_87; +} +} +} +else +{ +lean_object* x_88; lean_object* x_89; +lean_dec(x_66); +lean_dec(x_33); +if (lean_is_scalar(x_28)) { + x_88 = lean_alloc_ctor(0, 2, 0); +} else { + x_88 = x_28; +} +lean_ctor_set(x_88, 0, x_26); +lean_ctor_set(x_88, 1, x_47); +x_89 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_89, 0, x_88); +x_20 = x_89; +x_21 = x_61; +goto block_25; +} +} +} +} +else +{ +uint8_t x_90; +lean_dec(x_47); +lean_dec(x_33); +lean_dec(x_28); +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_90 = !lean_is_exclusive(x_52); +if (x_90 == 0) +{ +return x_52; +} +else +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_52, 0); +x_92 = lean_ctor_get(x_52, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_52); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +return x_93; +} +} +} +} +else +{ +uint8_t x_94; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_31); +lean_dec(x_28); +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_94 = !lean_is_exclusive(x_40); +if (x_94 == 0) +{ +return x_40; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_40, 0); +x_96 = lean_ctor_get(x_40, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_40); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; +} +} +} +} +else +{ +uint8_t x_126; +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_126 = !lean_is_exclusive(x_30); +if (x_126 == 0) +{ +return x_30; +} +else +{ +lean_object* x_127; lean_object* x_128; lean_object* x_129; +x_127 = lean_ctor_get(x_30, 0); +x_128 = lean_ctor_get(x_30, 1); +lean_inc(x_128); +lean_inc(x_127); +lean_dec(x_30); +x_129 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_129, 0, x_127); +lean_ctor_set(x_129, 1, x_128); +return x_129; +} +} +} +} +else +{ +lean_object* x_135; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_135 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_135, 0, x_9); +lean_ctor_set(x_135, 1, x_14); +return x_135; +} +} +else +{ +lean_object* x_136; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_136 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_136, 0, x_9); +lean_ctor_set(x_136, 1, x_14); +return x_136; +} +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; +x_14 = lean_nat_dec_le(x_6, x_5); +if (x_14 == 0) +{ +lean_object* x_15; uint8_t x_16; +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_nat_dec_eq(x_4, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_130; +x_17 = lean_unsigned_to_nat(1u); +x_18 = lean_nat_sub(x_4, x_17); +lean_dec(x_4); +x_25 = lean_ctor_get(x_8, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_8, 1); +lean_inc(x_26); +if (lean_is_exclusive(x_8)) { + lean_ctor_release(x_8, 0); + lean_ctor_release(x_8, 1); + x_27 = x_8; +} else { + lean_dec_ref(x_8); + x_27 = lean_box(0); +} +x_130 = lean_nat_dec_lt(x_5, x_3); +if (x_130 == 0) +{ +lean_object* x_131; lean_object* x_132; +x_131 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4; +x_132 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_131); +x_28 = x_132; +goto block_129; +} +else +{ +lean_object* x_133; +x_133 = lean_array_fget(x_2, x_5); +x_28 = x_133; +goto block_129; +} +block_24: +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_19, 0); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_nat_add(x_5, x_7); +lean_dec(x_5); +x_4 = x_18; +x_5 = x_22; +x_8 = x_21; +x_13 = x_20; +goto _start; +} +block_129: +{ +lean_object* x_29; +lean_inc(x_9); +x_29 = l_Lean_Meta_getFVarLocalDecl(x_28, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; uint8_t x_36; lean_object* x_37; lean_object* x_98; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = l_Lean_LocalDecl_type(x_30); +lean_inc(x_32); +lean_inc(x_2); +x_33 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(x_2, x_32); +x_34 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(x_26, x_33); +lean_dec(x_26); +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_63); -x_66 = l_Lean_Meta_isProp(x_63, x_8, x_9, x_10, x_11, x_62); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_32); +x_98 = l_Lean_Meta_isProp(x_32, x_9, x_10, x_11, x_12, x_31); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__5; +if (lean_obj_tag(x_98) == 0) +{ +lean_object* x_99; lean_object* x_100; uint8_t x_101; uint8_t x_102; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_98, 1); +lean_inc(x_100); +lean_dec(x_98); +x_101 = 0; +x_102 = lean_unbox(x_99); +lean_dec(x_99); +x_35 = x_101; +x_36 = x_102; +x_37 = x_100; +goto block_97; +} +else +{ +uint8_t x_103; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); +lean_dec(x_30); +lean_dec(x_27); +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_2); +x_103 = !lean_is_exclusive(x_98); +if (x_103 == 0) +{ +return x_98; +} +else +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_104 = lean_ctor_get(x_98, 0); +x_105 = lean_ctor_get(x_98, 1); +lean_inc(x_105); +lean_inc(x_104); +lean_dec(x_98); +x_106 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_106, 0, x_104); +lean_ctor_set(x_106, 1, x_105); +return x_106; +} +} +} +else +{ +lean_object* x_107; lean_object* x_108; +lean_inc(x_25); +x_107 = lean_alloc_closure((void*)(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__2___boxed), 2, 1); +lean_closure_set(x_107, 0, x_25); +lean_inc(x_32); +x_108 = l_Lean_Expr_FindImpl_findUnsafe_x3f(x_107, x_32); +if (lean_obj_tag(x_108) == 0) +{ +if (lean_obj_tag(x_98) == 0) +{ +lean_object* x_109; lean_object* x_110; uint8_t x_111; uint8_t x_112; +x_109 = lean_ctor_get(x_98, 0); +lean_inc(x_109); +x_110 = lean_ctor_get(x_98, 1); +lean_inc(x_110); +lean_dec(x_98); +x_111 = 0; +x_112 = lean_unbox(x_109); +lean_dec(x_109); +x_35 = x_111; +x_36 = x_112; +x_37 = x_110; +goto block_97; +} +else +{ +uint8_t x_113; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); +lean_dec(x_30); +lean_dec(x_27); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_2); +x_113 = !lean_is_exclusive(x_98); +if (x_113 == 0) +{ +return x_98; +} +else +{ +lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_114 = lean_ctor_get(x_98, 0); +x_115 = lean_ctor_get(x_98, 1); +lean_inc(x_115); +lean_inc(x_114); +lean_dec(x_98); +x_116 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +return x_116; +} +} +} +else +{ +lean_dec(x_108); +if (lean_obj_tag(x_98) == 0) +{ +lean_object* x_117; lean_object* x_118; uint8_t x_119; uint8_t x_120; +x_117 = lean_ctor_get(x_98, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_98, 1); +lean_inc(x_118); +lean_dec(x_98); +x_119 = 1; +x_120 = lean_unbox(x_117); +lean_dec(x_117); +x_35 = x_119; +x_36 = x_120; +x_37 = x_118; +goto block_97; +} +else +{ +uint8_t x_121; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); +lean_dec(x_30); +lean_dec(x_27); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_2); +x_121 = !lean_is_exclusive(x_98); +if (x_121 == 0) +{ +return x_98; +} +else +{ +lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_98, 0); +x_123 = lean_ctor_get(x_98, 1); +lean_inc(x_123); +lean_inc(x_122); +lean_dec(x_98); +x_124 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_124, 0, x_122); +lean_ctor_set(x_124, 1, x_123); +return x_124; +} +} +} +} +block_97: +{ +lean_object* x_38; lean_object* x_39; +x_38 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__1; +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_70 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_63, x_69, x_8, x_9, x_10, x_11, x_68); -if (lean_obj_tag(x_70) == 0) +lean_inc(x_32); +x_39 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_32, x_38, x_9, x_10, x_11, x_12, x_37); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_71; lean_object* x_72; uint8_t x_73; uint8_t x_74; lean_object* x_75; uint8_t x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; -x_71 = lean_ctor_get(x_70, 0); -lean_inc(x_71); -x_72 = lean_ctor_get(x_70, 1); -lean_inc(x_72); -lean_dec(x_70); -x_73 = l_Lean_LocalDecl_binderInfo(x_61); -lean_dec(x_61); -x_74 = 0; -x_75 = lean_alloc_ctor(0, 1, 4); -lean_ctor_set(x_75, 0, x_64); -lean_ctor_set_uint8(x_75, sizeof(void*)*1, x_73); -lean_ctor_set_uint8(x_75, sizeof(void*)*1 + 1, x_74); -x_76 = lean_unbox(x_67); -lean_dec(x_67); -lean_ctor_set_uint8(x_75, sizeof(void*)*1 + 2, x_76); -x_77 = lean_unbox(x_71); -lean_dec(x_71); -lean_ctor_set_uint8(x_75, sizeof(void*)*1 + 3, x_77); -x_78 = lean_array_push(x_65, x_75); -x_79 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_79, 0, x_78); -x_18 = x_79; -x_19 = x_72; -goto block_23; +lean_object* x_40; lean_object* x_41; uint8_t x_42; uint8_t x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); +x_42 = l_Lean_LocalDecl_binderInfo(x_30); +lean_dec(x_30); +x_43 = 0; +x_44 = lean_alloc_ctor(0, 1, 6); +lean_ctor_set(x_44, 0, x_33); +lean_ctor_set_uint8(x_44, sizeof(void*)*1, x_42); +lean_ctor_set_uint8(x_44, sizeof(void*)*1 + 1, x_43); +lean_ctor_set_uint8(x_44, sizeof(void*)*1 + 2, x_36); +x_45 = lean_unbox(x_40); +lean_dec(x_40); +lean_ctor_set_uint8(x_44, sizeof(void*)*1 + 3, x_45); +lean_ctor_set_uint8(x_44, sizeof(void*)*1 + 4, x_43); +lean_ctor_set_uint8(x_44, sizeof(void*)*1 + 5, x_35); +x_46 = lean_array_push(x_34, x_44); +x_47 = 3; +x_48 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_42, x_47); +if (x_48 == 0) +{ +lean_object* x_49; lean_object* x_50; +lean_dec(x_32); +if (lean_is_scalar(x_27)) { + x_49 = lean_alloc_ctor(0, 2, 0); +} else { + x_49 = x_27; +} +lean_ctor_set(x_49, 0, x_25); +lean_ctor_set(x_49, 1, x_46); +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +x_19 = x_50; +x_20 = x_41; +goto block_24; +} +else +{ +lean_object* x_51; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_32); +x_51 = l_Lean_Meta_isClass_x3f(x_32, x_9, x_10, x_11, x_12, x_41); +if (lean_obj_tag(x_51) == 0) +{ +lean_object* x_52; +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_dec(x_32); +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); +if (lean_is_scalar(x_27)) { + x_54 = lean_alloc_ctor(0, 2, 0); +} else { + x_54 = x_27; +} +lean_ctor_set(x_54, 0, x_25); +lean_ctor_set(x_54, 1, x_46); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_54); +x_19 = x_55; +x_20 = x_53; +goto block_24; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_56 = lean_ctor_get(x_51, 1); +lean_inc(x_56); +lean_dec(x_51); +x_57 = lean_ctor_get(x_52, 0); +lean_inc(x_57); +lean_dec(x_52); +x_58 = lean_st_ref_get(x_12, 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_61 = lean_ctor_get(x_59, 0); +lean_inc(x_61); +lean_dec(x_59); +x_62 = l_Lean_getOutParamPositions_x3f(x_61, x_57); +if (lean_obj_tag(x_62) == 0) +{ +lean_object* x_63; lean_object* x_64; +lean_dec(x_32); +if (lean_is_scalar(x_27)) { + x_63 = lean_alloc_ctor(0, 2, 0); +} else { + x_63 = x_27; +} +lean_ctor_set(x_63, 0, x_25); +lean_ctor_set(x_63, 1, x_46); +x_64 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_64, 0, x_63); +x_19 = x_64; +x_20 = x_60; +goto block_24; } else { -uint8_t x_80; +lean_object* x_65; uint8_t x_66; +x_65 = lean_ctor_get(x_62, 0); +lean_inc(x_65); +lean_dec(x_62); +x_66 = l_Array_isEmpty___rarg(x_65); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_67 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_32, x_15); +x_68 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__2; +lean_inc(x_67); +x_69 = lean_mk_array(x_67, x_68); +x_70 = lean_nat_sub(x_67, x_17); lean_dec(x_67); +x_71 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_32, x_69, x_70); +x_72 = lean_array_get_size(x_71); +if (lean_is_scalar(x_27)) { + x_73 = lean_alloc_ctor(0, 2, 0); +} else { + x_73 = x_27; +} +lean_ctor_set(x_73, 0, x_25); +lean_ctor_set(x_73, 1, x_46); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_72); +x_74 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__4(x_2, x_65, x_71, x_72, x_72, x_15, x_72, x_17, x_73, x_9, x_10, x_11, x_12, x_60); +lean_dec(x_72); +lean_dec(x_71); lean_dec(x_65); -lean_dec(x_64); -lean_dec(x_61); -lean_dec(x_17); +if (lean_obj_tag(x_74) == 0) +{ +lean_object* x_75; lean_object* x_76; uint8_t x_77; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); +x_77 = !lean_is_exclusive(x_75); +if (x_77 == 0) +{ +lean_object* x_78; +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_75); +x_19 = x_78; +x_20 = x_76; +goto block_24; +} +else +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_79 = lean_ctor_get(x_75, 0); +x_80 = lean_ctor_get(x_75, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_75); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +x_82 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_82, 0, x_81); +x_19 = x_82; +x_20 = x_76; +goto block_24; +} +} +else +{ +uint8_t x_83; +lean_dec(x_18); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_4); -lean_dec(x_1); -x_80 = !lean_is_exclusive(x_70); -if (x_80 == 0) +lean_dec(x_5); +lean_dec(x_2); +x_83 = !lean_is_exclusive(x_74); +if (x_83 == 0) { -return x_70; +return x_74; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_70, 0); -x_82 = lean_ctor_get(x_70, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_70); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -return x_83; +lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_74, 0); +x_85 = lean_ctor_get(x_74, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_74); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +return x_86; } } } else { -uint8_t x_84; +lean_object* x_87; lean_object* x_88; lean_dec(x_65); -lean_dec(x_64); -lean_dec(x_63); -lean_dec(x_61); -lean_dec(x_17); +lean_dec(x_32); +if (lean_is_scalar(x_27)) { + x_87 = lean_alloc_ctor(0, 2, 0); +} else { + x_87 = x_27; +} +lean_ctor_set(x_87, 0, x_25); +lean_ctor_set(x_87, 1, x_46); +x_88 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_88, 0, x_87); +x_19 = x_88; +x_20 = x_60; +goto block_24; +} +} +} +} +else +{ +uint8_t x_89; +lean_dec(x_46); +lean_dec(x_32); +lean_dec(x_27); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_4); -lean_dec(x_1); -x_84 = !lean_is_exclusive(x_66); -if (x_84 == 0) +lean_dec(x_5); +lean_dec(x_2); +x_89 = !lean_is_exclusive(x_51); +if (x_89 == 0) { -return x_66; +return x_51; } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_85 = lean_ctor_get(x_66, 0); -x_86 = lean_ctor_get(x_66, 1); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_66); -x_87 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_87, 0, x_85); -lean_ctor_set(x_87, 1, x_86); -return x_87; +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_51, 0); +x_91 = lean_ctor_get(x_51, 1); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_51); +x_92 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_91); +return x_92; +} +} +} +} +else +{ +uint8_t x_93; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); +lean_dec(x_30); +lean_dec(x_27); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_2); +x_93 = !lean_is_exclusive(x_39); +if (x_93 == 0) +{ +return x_39; +} +else +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_39, 0); +x_95 = lean_ctor_get(x_39, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_39); +x_96 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +return x_96; +} } } } else { -uint8_t x_88; -lean_dec(x_17); +uint8_t x_125; +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_1); -x_88 = !lean_is_exclusive(x_60); -if (x_88 == 0) +lean_dec(x_5); +lean_dec(x_2); +x_125 = !lean_is_exclusive(x_29); +if (x_125 == 0) { -return x_60; +return x_29; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_60, 0); -x_90 = lean_ctor_get(x_60, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_60); -x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_90); -return x_91; -} +lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_126 = lean_ctor_get(x_29, 0); +x_127 = lean_ctor_get(x_29, 1); +lean_inc(x_127); +lean_inc(x_126); +lean_dec(x_29); +x_128 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_128, 0, x_126); +lean_ctor_set(x_128, 1, x_127); +return x_128; } } -block_23: -{ -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_18, 0); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_nat_add(x_4, x_6); -lean_dec(x_4); -x_3 = x_17; -x_4 = x_21; -x_7 = x_20; -x_12 = x_19; -goto _start; } } else { -lean_object* x_92; +lean_object* x_134; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_92 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_92, 0, x_7); -lean_ctor_set(x_92, 1, x_12); -return x_92; +lean_dec(x_2); +x_134 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_134, 0, x_8); +lean_ctor_set(x_134, 1, x_13); +return x_134; } } else { -lean_object* x_93; +lean_object* x_135; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_7); -lean_ctor_set(x_93, 1, x_12); -return x_93; +lean_dec(x_2); +x_135 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_135, 0, x_8); +lean_ctor_set(x_135, 1, x_13); +return x_135; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; @@ -2644,85 +6797,103 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2___rarg), 8, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8___rarg), 8, 0); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___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) { +static lean_object* _init_l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___closed__1() { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_array_get_size(x_1); -x_9 = lean_unsigned_to_nat(0u); -x_10 = lean_unsigned_to_nat(1u); -x_11 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___closed__1; -lean_inc(x_8); -lean_inc(x_1); -x_12 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(x_1, x_8, x_8, x_9, x_8, x_10, x_11, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_8); -if (lean_obj_tag(x_12) == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___closed__1; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_array_get_size(x_2); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_unsigned_to_nat(1u); +x_12 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___closed__1; +lean_inc(x_9); +lean_inc(x_2); +x_13 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__7(x_1, x_2, x_9, x_9, x_10, x_9, x_11, x_12, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_9); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(x_1, x_2); -x_16 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(x_14, x_15); -lean_dec(x_14); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -lean_ctor_set(x_12, 0, x_17); -return x_12; +uint8_t x_14; +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(x_2, x_3); +x_18 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(x_16, x_17); +lean_dec(x_16); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +lean_ctor_set(x_13, 0, x_19); +return x_13; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_18 = lean_ctor_get(x_12, 0); -x_19 = lean_ctor_get(x_12, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_12); -x_20 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(x_1, x_2); -x_21 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(x_18, x_20); -lean_dec(x_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_19); -return x_23; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_13, 0); +x_21 = lean_ctor_get(x_13, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_13); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps(x_2, x_3); +x_24 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_updateHasFwdDeps(x_22, x_23); +lean_dec(x_22); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_21); +return x_26; } } else { -uint8_t x_24; +uint8_t x_27; +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_24 = !lean_is_exclusive(x_12); -if (x_24 == 0) +x_27 = !lean_is_exclusive(x_13); +if (x_27 == 0) { -return x_12; +return x_13; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_12, 0); -x_26 = lean_ctor_get(x_12, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_12); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_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; } } } @@ -2730,35 +6901,41 @@ return x_27; static lean_object* _init_l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1), 7, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Meta_instMonadMetaM; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = lean_ctor_get(x_2, 1); +lean_inc(x_3); +lean_dec(x_2); +x_4 = l_instMonadControlT__1___rarg(x_3); +return x_4; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_8 = lean_st_ref_get(x_6, x_7); -x_9 = lean_ctor_get(x_8, 1); +x_8 = l_Lean_Meta_getTransparency(x_3, x_4, x_5, x_6, x_7); +x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); lean_dec(x_8); -x_10 = lean_st_ref_get(x_4, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); +x_11 = lean_st_ref_get(x_6, x_10); +x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Meta_getTransparency(x_3, x_4, x_5, x_6, x_12); +lean_dec(x_11); +x_13 = lean_st_ref_get(x_4, x_12); x_14 = !lean_is_exclusive(x_13); if (x_14 == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; x_15 = lean_ctor_get(x_13, 0); x_16 = lean_ctor_get(x_13, 1); -x_17 = lean_ctor_get(x_11, 1); +x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); -lean_dec(x_11); +lean_dec(x_15); x_18 = lean_ctor_get(x_17, 1); lean_inc(x_18); lean_dec(x_17); @@ -2767,8 +6944,8 @@ lean_inc(x_1); x_19 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_19, 0, x_1); lean_ctor_set(x_19, 1, x_2); -x_20 = lean_unbox(x_15); -lean_dec(x_15); +x_20 = lean_unbox(x_9); +lean_dec(x_9); lean_ctor_set_uint8(x_19, sizeof(void*)*2, x_20); lean_inc(x_19); x_21 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__1(x_18, x_19); @@ -2783,30 +6960,29 @@ lean_inc(x_3); x_22 = lean_infer_type(x_1, x_3, x_4, x_5, x_6, x_16); if (lean_obj_tag(x_22) == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = lean_ctor_get(x_3, 0); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 0); +x_24 = lean_ctor_get(x_22, 1); lean_inc(x_24); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); lean_dec(x_22); -x_26 = !lean_is_exclusive(x_3); -if (x_26 == 0) +x_25 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1; +x_26 = lean_alloc_closure((void*)(l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___boxed), 8, 1); +lean_closure_set(x_26, 0, x_25); +x_27 = !lean_is_exclusive(x_3); +if (x_27 == 0) { -lean_object* x_27; uint8_t x_28; -x_27 = lean_ctor_get(x_3, 0); -lean_dec(x_27); -x_28 = !lean_is_exclusive(x_23); -if (x_28 == 0) +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_3, 0); +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) { -uint8_t x_29; lean_object* x_30; lean_object* x_31; -x_29 = 1; -lean_ctor_set_uint8(x_23, 5, x_29); -x_30 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1; +uint8_t x_30; lean_object* x_31; +x_30 = 1; +lean_ctor_set_uint8(x_28, 5, x_30); lean_inc(x_6); lean_inc(x_4); -x_31 = l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2___rarg(x_24, x_2, x_30, x_3, x_4, x_5, x_6, x_25); +x_31 = l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8___rarg(x_23, x_2, x_26, x_3, x_4, x_5, x_6, x_24); if (lean_obj_tag(x_31) == 0) { lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; @@ -3022,21 +7198,21 @@ return x_84; } else { -uint8_t x_85; uint8_t x_86; uint8_t x_87; uint8_t x_88; uint8_t x_89; uint8_t x_90; uint8_t x_91; uint8_t x_92; uint8_t x_93; uint8_t x_94; uint8_t x_95; uint8_t x_96; uint8_t x_97; uint8_t x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_85 = lean_ctor_get_uint8(x_23, 0); -x_86 = lean_ctor_get_uint8(x_23, 1); -x_87 = lean_ctor_get_uint8(x_23, 2); -x_88 = lean_ctor_get_uint8(x_23, 3); -x_89 = lean_ctor_get_uint8(x_23, 4); -x_90 = lean_ctor_get_uint8(x_23, 6); -x_91 = lean_ctor_get_uint8(x_23, 7); -x_92 = lean_ctor_get_uint8(x_23, 8); -x_93 = lean_ctor_get_uint8(x_23, 9); -x_94 = lean_ctor_get_uint8(x_23, 10); -x_95 = lean_ctor_get_uint8(x_23, 11); -x_96 = lean_ctor_get_uint8(x_23, 12); -x_97 = lean_ctor_get_uint8(x_23, 13); -lean_dec(x_23); +uint8_t x_85; uint8_t x_86; uint8_t x_87; uint8_t x_88; uint8_t x_89; uint8_t x_90; uint8_t x_91; uint8_t x_92; uint8_t x_93; uint8_t x_94; uint8_t x_95; uint8_t x_96; uint8_t x_97; uint8_t x_98; lean_object* x_99; lean_object* x_100; +x_85 = lean_ctor_get_uint8(x_28, 0); +x_86 = lean_ctor_get_uint8(x_28, 1); +x_87 = lean_ctor_get_uint8(x_28, 2); +x_88 = lean_ctor_get_uint8(x_28, 3); +x_89 = lean_ctor_get_uint8(x_28, 4); +x_90 = lean_ctor_get_uint8(x_28, 6); +x_91 = lean_ctor_get_uint8(x_28, 7); +x_92 = lean_ctor_get_uint8(x_28, 8); +x_93 = lean_ctor_get_uint8(x_28, 9); +x_94 = lean_ctor_get_uint8(x_28, 10); +x_95 = lean_ctor_get_uint8(x_28, 11); +x_96 = lean_ctor_get_uint8(x_28, 12); +x_97 = lean_ctor_get_uint8(x_28, 13); +lean_dec(x_28); x_98 = 1; x_99 = lean_alloc_ctor(0, 0, 14); lean_ctor_set_uint8(x_99, 0, x_85); @@ -3054,150 +7230,150 @@ lean_ctor_set_uint8(x_99, 11, x_95); lean_ctor_set_uint8(x_99, 12, x_96); lean_ctor_set_uint8(x_99, 13, x_97); lean_ctor_set(x_3, 0, x_99); -x_100 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1; lean_inc(x_6); lean_inc(x_4); -x_101 = l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2___rarg(x_24, x_2, x_100, x_3, x_4, x_5, x_6, x_25); -if (lean_obj_tag(x_101) == 0) +x_100 = l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8___rarg(x_23, x_2, x_26, x_3, x_4, x_5, x_6, x_24); +if (lean_obj_tag(x_100) == 0) { -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_102 = lean_ctor_get(x_101, 0); +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; 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; +x_101 = lean_ctor_get(x_100, 0); +lean_inc(x_101); +x_102 = lean_ctor_get(x_100, 1); lean_inc(x_102); -x_103 = lean_ctor_get(x_101, 1); -lean_inc(x_103); -lean_dec(x_101); -x_104 = lean_st_ref_get(x_6, x_103); +lean_dec(x_100); +x_103 = lean_st_ref_get(x_6, x_102); lean_dec(x_6); -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -lean_dec(x_104); -x_106 = lean_st_ref_take(x_4, x_105); -x_107 = lean_ctor_get(x_106, 0); +x_104 = lean_ctor_get(x_103, 1); +lean_inc(x_104); +lean_dec(x_103); +x_105 = lean_st_ref_take(x_4, x_104); +x_106 = lean_ctor_get(x_105, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_106, 1); lean_inc(x_107); -x_108 = lean_ctor_get(x_107, 1); +x_108 = lean_ctor_get(x_105, 1); lean_inc(x_108); -x_109 = lean_ctor_get(x_106, 1); +lean_dec(x_105); +x_109 = lean_ctor_get(x_106, 0); lean_inc(x_109); -lean_dec(x_106); -x_110 = lean_ctor_get(x_107, 0); +x_110 = lean_ctor_get(x_106, 2); lean_inc(x_110); -x_111 = lean_ctor_get(x_107, 2); +x_111 = lean_ctor_get(x_106, 3); lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 3); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - lean_ctor_release(x_107, 2); - lean_ctor_release(x_107, 3); - x_113 = x_107; +if (lean_is_exclusive(x_106)) { + lean_ctor_release(x_106, 0); + lean_ctor_release(x_106, 1); + lean_ctor_release(x_106, 2); + lean_ctor_release(x_106, 3); + x_112 = x_106; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_106); + x_112 = lean_box(0); } -x_114 = lean_ctor_get(x_108, 0); +x_113 = lean_ctor_get(x_107, 0); +lean_inc(x_113); +x_114 = lean_ctor_get(x_107, 2); lean_inc(x_114); -x_115 = lean_ctor_get(x_108, 2); +x_115 = lean_ctor_get(x_107, 3); lean_inc(x_115); -x_116 = lean_ctor_get(x_108, 3); +x_116 = lean_ctor_get(x_107, 4); lean_inc(x_116); -x_117 = lean_ctor_get(x_108, 4); +x_117 = lean_ctor_get(x_107, 5); lean_inc(x_117); -x_118 = lean_ctor_get(x_108, 5); +x_118 = lean_ctor_get(x_107, 6); lean_inc(x_118); -x_119 = lean_ctor_get(x_108, 6); +x_119 = lean_ctor_get(x_107, 1); lean_inc(x_119); -x_120 = lean_ctor_get(x_108, 1); -lean_inc(x_120); -if (lean_is_exclusive(x_108)) { - lean_ctor_release(x_108, 0); - lean_ctor_release(x_108, 1); - lean_ctor_release(x_108, 2); - lean_ctor_release(x_108, 3); - lean_ctor_release(x_108, 4); - lean_ctor_release(x_108, 5); - lean_ctor_release(x_108, 6); - x_121 = x_108; -} else { - lean_dec_ref(x_108); - x_121 = lean_box(0); -} -lean_inc(x_102); -x_122 = l_Std_PersistentHashMap_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__4(x_120, x_19, x_102); -if (lean_is_scalar(x_121)) { - x_123 = lean_alloc_ctor(0, 7, 0); +if (lean_is_exclusive(x_107)) { + lean_ctor_release(x_107, 0); + lean_ctor_release(x_107, 1); + lean_ctor_release(x_107, 2); + lean_ctor_release(x_107, 3); + lean_ctor_release(x_107, 4); + lean_ctor_release(x_107, 5); + lean_ctor_release(x_107, 6); + x_120 = x_107; } else { - x_123 = x_121; + lean_dec_ref(x_107); + x_120 = lean_box(0); } -lean_ctor_set(x_123, 0, x_114); -lean_ctor_set(x_123, 1, x_122); -lean_ctor_set(x_123, 2, x_115); -lean_ctor_set(x_123, 3, x_116); -lean_ctor_set(x_123, 4, x_117); -lean_ctor_set(x_123, 5, x_118); -lean_ctor_set(x_123, 6, x_119); -if (lean_is_scalar(x_113)) { - x_124 = lean_alloc_ctor(0, 4, 0); +lean_inc(x_101); +x_121 = l_Std_PersistentHashMap_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__4(x_119, x_19, x_101); +if (lean_is_scalar(x_120)) { + x_122 = lean_alloc_ctor(0, 7, 0); +} else { + x_122 = x_120; +} +lean_ctor_set(x_122, 0, x_113); +lean_ctor_set(x_122, 1, x_121); +lean_ctor_set(x_122, 2, x_114); +lean_ctor_set(x_122, 3, x_115); +lean_ctor_set(x_122, 4, x_116); +lean_ctor_set(x_122, 5, x_117); +lean_ctor_set(x_122, 6, x_118); +if (lean_is_scalar(x_112)) { + x_123 = lean_alloc_ctor(0, 4, 0); } else { - x_124 = x_113; + x_123 = x_112; } -lean_ctor_set(x_124, 0, x_110); -lean_ctor_set(x_124, 1, x_123); -lean_ctor_set(x_124, 2, x_111); -lean_ctor_set(x_124, 3, x_112); -x_125 = lean_st_ref_set(x_4, x_124, x_109); +lean_ctor_set(x_123, 0, x_109); +lean_ctor_set(x_123, 1, x_122); +lean_ctor_set(x_123, 2, x_110); +lean_ctor_set(x_123, 3, x_111); +x_124 = lean_st_ref_set(x_4, x_123, x_108); lean_dec(x_4); -x_126 = lean_ctor_get(x_125, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_125)) { - lean_ctor_release(x_125, 0); - lean_ctor_release(x_125, 1); - x_127 = x_125; +x_125 = lean_ctor_get(x_124, 1); +lean_inc(x_125); +if (lean_is_exclusive(x_124)) { + lean_ctor_release(x_124, 0); + lean_ctor_release(x_124, 1); + x_126 = x_124; } else { - lean_dec_ref(x_125); - x_127 = lean_box(0); + lean_dec_ref(x_124); + x_126 = lean_box(0); } -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_126)) { + x_127 = lean_alloc_ctor(0, 2, 0); } else { - x_128 = x_127; + x_127 = x_126; } -lean_ctor_set(x_128, 0, x_102); -lean_ctor_set(x_128, 1, x_126); -return x_128; +lean_ctor_set(x_127, 0, x_101); +lean_ctor_set(x_127, 1, x_125); +return x_127; } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_dec(x_19); lean_dec(x_6); lean_dec(x_4); -x_129 = lean_ctor_get(x_101, 0); +x_128 = lean_ctor_get(x_100, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_100, 1); lean_inc(x_129); -x_130 = lean_ctor_get(x_101, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_131 = x_101; +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + x_130 = x_100; } else { - lean_dec_ref(x_101); - x_131 = lean_box(0); + lean_dec_ref(x_100); + x_130 = lean_box(0); } -if (lean_is_scalar(x_131)) { - x_132 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_130)) { + x_131 = lean_alloc_ctor(1, 2, 0); } else { - x_132 = x_131; + x_131 = x_130; } -lean_ctor_set(x_132, 0, x_129); -lean_ctor_set(x_132, 1, x_130); -return x_132; +lean_ctor_set(x_131, 0, x_128); +lean_ctor_set(x_131, 1, x_129); +return x_131; } } } else { -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; uint8_t x_138; uint8_t x_139; uint8_t x_140; uint8_t x_141; uint8_t x_142; uint8_t x_143; uint8_t x_144; uint8_t x_145; uint8_t x_146; uint8_t x_147; uint8_t x_148; uint8_t x_149; uint8_t x_150; lean_object* x_151; uint8_t x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; +lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; uint8_t x_138; uint8_t x_139; uint8_t x_140; uint8_t x_141; uint8_t x_142; uint8_t x_143; uint8_t x_144; uint8_t x_145; uint8_t x_146; uint8_t x_147; uint8_t x_148; uint8_t x_149; uint8_t x_150; lean_object* x_151; uint8_t x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; +x_132 = lean_ctor_get(x_3, 0); x_133 = lean_ctor_get(x_3, 1); x_134 = lean_ctor_get(x_3, 2); x_135 = lean_ctor_get(x_3, 3); @@ -3208,24 +7384,25 @@ lean_inc(x_136); lean_inc(x_135); lean_inc(x_134); lean_inc(x_133); +lean_inc(x_132); lean_dec(x_3); -x_138 = lean_ctor_get_uint8(x_23, 0); -x_139 = lean_ctor_get_uint8(x_23, 1); -x_140 = lean_ctor_get_uint8(x_23, 2); -x_141 = lean_ctor_get_uint8(x_23, 3); -x_142 = lean_ctor_get_uint8(x_23, 4); -x_143 = lean_ctor_get_uint8(x_23, 6); -x_144 = lean_ctor_get_uint8(x_23, 7); -x_145 = lean_ctor_get_uint8(x_23, 8); -x_146 = lean_ctor_get_uint8(x_23, 9); -x_147 = lean_ctor_get_uint8(x_23, 10); -x_148 = lean_ctor_get_uint8(x_23, 11); -x_149 = lean_ctor_get_uint8(x_23, 12); -x_150 = lean_ctor_get_uint8(x_23, 13); -if (lean_is_exclusive(x_23)) { - x_151 = x_23; -} else { - lean_dec_ref(x_23); +x_138 = lean_ctor_get_uint8(x_132, 0); +x_139 = lean_ctor_get_uint8(x_132, 1); +x_140 = lean_ctor_get_uint8(x_132, 2); +x_141 = lean_ctor_get_uint8(x_132, 3); +x_142 = lean_ctor_get_uint8(x_132, 4); +x_143 = lean_ctor_get_uint8(x_132, 6); +x_144 = lean_ctor_get_uint8(x_132, 7); +x_145 = lean_ctor_get_uint8(x_132, 8); +x_146 = lean_ctor_get_uint8(x_132, 9); +x_147 = lean_ctor_get_uint8(x_132, 10); +x_148 = lean_ctor_get_uint8(x_132, 11); +x_149 = lean_ctor_get_uint8(x_132, 12); +x_150 = lean_ctor_get_uint8(x_132, 13); +if (lean_is_exclusive(x_132)) { + x_151 = x_132; +} else { + lean_dec_ref(x_132); x_151 = lean_box(0); } x_152 = 1; @@ -3255,179 +7432,178 @@ lean_ctor_set(x_154, 2, x_134); lean_ctor_set(x_154, 3, x_135); lean_ctor_set(x_154, 4, x_136); lean_ctor_set(x_154, 5, x_137); -x_155 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1; lean_inc(x_6); lean_inc(x_4); -x_156 = l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2___rarg(x_24, x_2, x_155, x_154, x_4, x_5, x_6, x_25); -if (lean_obj_tag(x_156) == 0) +x_155 = l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8___rarg(x_23, x_2, x_26, x_154, x_4, x_5, x_6, x_24); +if (lean_obj_tag(x_155) == 0) { -lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_157 = lean_ctor_get(x_156, 0); +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_156 = lean_ctor_get(x_155, 0); +lean_inc(x_156); +x_157 = lean_ctor_get(x_155, 1); lean_inc(x_157); -x_158 = lean_ctor_get(x_156, 1); -lean_inc(x_158); -lean_dec(x_156); -x_159 = lean_st_ref_get(x_6, x_158); +lean_dec(x_155); +x_158 = lean_st_ref_get(x_6, x_157); lean_dec(x_6); -x_160 = lean_ctor_get(x_159, 1); -lean_inc(x_160); -lean_dec(x_159); -x_161 = lean_st_ref_take(x_4, x_160); -x_162 = lean_ctor_get(x_161, 0); +x_159 = lean_ctor_get(x_158, 1); +lean_inc(x_159); +lean_dec(x_158); +x_160 = lean_st_ref_take(x_4, x_159); +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_161, 1); lean_inc(x_162); -x_163 = lean_ctor_get(x_162, 1); +x_163 = lean_ctor_get(x_160, 1); lean_inc(x_163); -x_164 = lean_ctor_get(x_161, 1); +lean_dec(x_160); +x_164 = lean_ctor_get(x_161, 0); lean_inc(x_164); -lean_dec(x_161); -x_165 = lean_ctor_get(x_162, 0); +x_165 = lean_ctor_get(x_161, 2); lean_inc(x_165); -x_166 = lean_ctor_get(x_162, 2); +x_166 = lean_ctor_get(x_161, 3); lean_inc(x_166); -x_167 = lean_ctor_get(x_162, 3); -lean_inc(x_167); -if (lean_is_exclusive(x_162)) { - lean_ctor_release(x_162, 0); - lean_ctor_release(x_162, 1); - lean_ctor_release(x_162, 2); - lean_ctor_release(x_162, 3); - x_168 = x_162; +if (lean_is_exclusive(x_161)) { + lean_ctor_release(x_161, 0); + lean_ctor_release(x_161, 1); + lean_ctor_release(x_161, 2); + lean_ctor_release(x_161, 3); + x_167 = x_161; } else { - lean_dec_ref(x_162); - x_168 = lean_box(0); + lean_dec_ref(x_161); + x_167 = lean_box(0); } -x_169 = lean_ctor_get(x_163, 0); +x_168 = lean_ctor_get(x_162, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_162, 2); lean_inc(x_169); -x_170 = lean_ctor_get(x_163, 2); +x_170 = lean_ctor_get(x_162, 3); lean_inc(x_170); -x_171 = lean_ctor_get(x_163, 3); +x_171 = lean_ctor_get(x_162, 4); lean_inc(x_171); -x_172 = lean_ctor_get(x_163, 4); +x_172 = lean_ctor_get(x_162, 5); lean_inc(x_172); -x_173 = lean_ctor_get(x_163, 5); +x_173 = lean_ctor_get(x_162, 6); lean_inc(x_173); -x_174 = lean_ctor_get(x_163, 6); +x_174 = lean_ctor_get(x_162, 1); lean_inc(x_174); -x_175 = lean_ctor_get(x_163, 1); -lean_inc(x_175); -if (lean_is_exclusive(x_163)) { - lean_ctor_release(x_163, 0); - lean_ctor_release(x_163, 1); - lean_ctor_release(x_163, 2); - lean_ctor_release(x_163, 3); - lean_ctor_release(x_163, 4); - lean_ctor_release(x_163, 5); - lean_ctor_release(x_163, 6); - x_176 = x_163; -} else { - lean_dec_ref(x_163); - x_176 = lean_box(0); +if (lean_is_exclusive(x_162)) { + lean_ctor_release(x_162, 0); + lean_ctor_release(x_162, 1); + lean_ctor_release(x_162, 2); + lean_ctor_release(x_162, 3); + lean_ctor_release(x_162, 4); + lean_ctor_release(x_162, 5); + lean_ctor_release(x_162, 6); + x_175 = x_162; +} else { + lean_dec_ref(x_162); + x_175 = lean_box(0); } -lean_inc(x_157); -x_177 = l_Std_PersistentHashMap_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__4(x_175, x_19, x_157); -if (lean_is_scalar(x_176)) { - x_178 = lean_alloc_ctor(0, 7, 0); +lean_inc(x_156); +x_176 = l_Std_PersistentHashMap_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__4(x_174, x_19, x_156); +if (lean_is_scalar(x_175)) { + x_177 = lean_alloc_ctor(0, 7, 0); +} else { + x_177 = x_175; +} +lean_ctor_set(x_177, 0, x_168); +lean_ctor_set(x_177, 1, x_176); +lean_ctor_set(x_177, 2, x_169); +lean_ctor_set(x_177, 3, x_170); +lean_ctor_set(x_177, 4, x_171); +lean_ctor_set(x_177, 5, x_172); +lean_ctor_set(x_177, 6, x_173); +if (lean_is_scalar(x_167)) { + x_178 = lean_alloc_ctor(0, 4, 0); } else { - x_178 = x_176; + x_178 = x_167; } -lean_ctor_set(x_178, 0, x_169); +lean_ctor_set(x_178, 0, x_164); lean_ctor_set(x_178, 1, x_177); -lean_ctor_set(x_178, 2, x_170); -lean_ctor_set(x_178, 3, x_171); -lean_ctor_set(x_178, 4, x_172); -lean_ctor_set(x_178, 5, x_173); -lean_ctor_set(x_178, 6, x_174); -if (lean_is_scalar(x_168)) { - x_179 = lean_alloc_ctor(0, 4, 0); -} else { - x_179 = x_168; -} -lean_ctor_set(x_179, 0, x_165); -lean_ctor_set(x_179, 1, x_178); -lean_ctor_set(x_179, 2, x_166); -lean_ctor_set(x_179, 3, x_167); -x_180 = lean_st_ref_set(x_4, x_179, x_164); +lean_ctor_set(x_178, 2, x_165); +lean_ctor_set(x_178, 3, x_166); +x_179 = lean_st_ref_set(x_4, x_178, x_163); lean_dec(x_4); -x_181 = lean_ctor_get(x_180, 1); -lean_inc(x_181); -if (lean_is_exclusive(x_180)) { - lean_ctor_release(x_180, 0); - lean_ctor_release(x_180, 1); - x_182 = x_180; +x_180 = lean_ctor_get(x_179, 1); +lean_inc(x_180); +if (lean_is_exclusive(x_179)) { + lean_ctor_release(x_179, 0); + lean_ctor_release(x_179, 1); + x_181 = x_179; } else { - lean_dec_ref(x_180); - x_182 = lean_box(0); + lean_dec_ref(x_179); + x_181 = lean_box(0); } -if (lean_is_scalar(x_182)) { - x_183 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_181)) { + x_182 = lean_alloc_ctor(0, 2, 0); } else { - x_183 = x_182; + x_182 = x_181; } -lean_ctor_set(x_183, 0, x_157); -lean_ctor_set(x_183, 1, x_181); -return x_183; +lean_ctor_set(x_182, 0, x_156); +lean_ctor_set(x_182, 1, x_180); +return x_182; } else { -lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_dec(x_19); lean_dec(x_6); lean_dec(x_4); -x_184 = lean_ctor_get(x_156, 0); +x_183 = lean_ctor_get(x_155, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_155, 1); lean_inc(x_184); -x_185 = lean_ctor_get(x_156, 1); -lean_inc(x_185); -if (lean_is_exclusive(x_156)) { - lean_ctor_release(x_156, 0); - lean_ctor_release(x_156, 1); - x_186 = x_156; +if (lean_is_exclusive(x_155)) { + lean_ctor_release(x_155, 0); + lean_ctor_release(x_155, 1); + x_185 = x_155; } else { - lean_dec_ref(x_156); - x_186 = lean_box(0); + lean_dec_ref(x_155); + x_185 = lean_box(0); } -if (lean_is_scalar(x_186)) { - x_187 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_185)) { + x_186 = lean_alloc_ctor(1, 2, 0); } else { - x_187 = x_186; + x_186 = x_185; } -lean_ctor_set(x_187, 0, x_184); -lean_ctor_set(x_187, 1, x_185); -return x_187; +lean_ctor_set(x_186, 0, x_183); +lean_ctor_set(x_186, 1, x_184); +return x_186; } } } else { -uint8_t x_188; +uint8_t x_187; lean_dec(x_19); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_188 = !lean_is_exclusive(x_22); -if (x_188 == 0) +x_187 = !lean_is_exclusive(x_22); +if (x_187 == 0) { return x_22; } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_189 = lean_ctor_get(x_22, 0); -x_190 = lean_ctor_get(x_22, 1); -lean_inc(x_190); +lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_188 = lean_ctor_get(x_22, 0); +x_189 = lean_ctor_get(x_22, 1); lean_inc(x_189); +lean_inc(x_188); lean_dec(x_22); -x_191 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_191, 0, x_189); -lean_ctor_set(x_191, 1, x_190); -return x_191; +x_190 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_190, 0, x_188); +lean_ctor_set(x_190, 1, x_189); +return x_190; } } } else { -lean_object* x_192; +lean_object* x_191; lean_dec(x_19); lean_dec(x_6); lean_dec(x_5); @@ -3435,65 +7611,68 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_192 = lean_ctor_get(x_21, 0); -lean_inc(x_192); +x_191 = lean_ctor_get(x_21, 0); +lean_inc(x_191); lean_dec(x_21); -lean_ctor_set(x_13, 0, x_192); +lean_ctor_set(x_13, 0, x_191); return x_13; } } else { -lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; uint8_t x_198; lean_object* x_199; -x_193 = lean_ctor_get(x_13, 0); -x_194 = lean_ctor_get(x_13, 1); -lean_inc(x_194); +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; uint8_t x_197; lean_object* x_198; +x_192 = lean_ctor_get(x_13, 0); +x_193 = lean_ctor_get(x_13, 1); lean_inc(x_193); +lean_inc(x_192); lean_dec(x_13); -x_195 = lean_ctor_get(x_11, 1); +x_194 = lean_ctor_get(x_192, 1); +lean_inc(x_194); +lean_dec(x_192); +x_195 = lean_ctor_get(x_194, 1); lean_inc(x_195); -lean_dec(x_11); -x_196 = lean_ctor_get(x_195, 1); -lean_inc(x_196); -lean_dec(x_195); +lean_dec(x_194); lean_inc(x_2); lean_inc(x_1); -x_197 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_197, 0, x_1); -lean_ctor_set(x_197, 1, x_2); -x_198 = lean_unbox(x_193); -lean_dec(x_193); -lean_ctor_set_uint8(x_197, sizeof(void*)*2, x_198); -lean_inc(x_197); -x_199 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__1(x_196, x_197); -if (lean_obj_tag(x_199) == 0) +x_196 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_196, 0, x_1); +lean_ctor_set(x_196, 1, x_2); +x_197 = lean_unbox(x_9); +lean_dec(x_9); +lean_ctor_set_uint8(x_196, sizeof(void*)*2, x_197); +lean_inc(x_196); +x_198 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__1(x_195, x_196); +if (lean_obj_tag(x_198) == 0) { -lean_object* x_200; +lean_object* x_199; lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_200 = lean_infer_type(x_1, x_3, x_4, x_5, x_6, x_194); -if (lean_obj_tag(x_200) == 0) +x_199 = lean_infer_type(x_1, x_3, x_4, x_5, x_6, x_193); +if (lean_obj_tag(x_199) == 0) { -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; uint8_t x_210; uint8_t x_211; uint8_t x_212; uint8_t x_213; uint8_t x_214; uint8_t x_215; uint8_t x_216; uint8_t x_217; uint8_t x_218; uint8_t x_219; uint8_t x_220; uint8_t x_221; uint8_t x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; -x_201 = lean_ctor_get(x_3, 0); +lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; uint8_t x_211; uint8_t x_212; uint8_t x_213; uint8_t x_214; uint8_t x_215; uint8_t x_216; uint8_t x_217; uint8_t x_218; uint8_t x_219; uint8_t x_220; uint8_t x_221; uint8_t x_222; uint8_t x_223; lean_object* x_224; uint8_t x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_200 = lean_ctor_get(x_199, 0); +lean_inc(x_200); +x_201 = lean_ctor_get(x_199, 1); lean_inc(x_201); -x_202 = lean_ctor_get(x_200, 0); -lean_inc(x_202); -x_203 = lean_ctor_get(x_200, 1); -lean_inc(x_203); -lean_dec(x_200); -x_204 = lean_ctor_get(x_3, 1); +lean_dec(x_199); +x_202 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1; +x_203 = lean_alloc_closure((void*)(l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___boxed), 8, 1); +lean_closure_set(x_203, 0, x_202); +x_204 = lean_ctor_get(x_3, 0); lean_inc(x_204); -x_205 = lean_ctor_get(x_3, 2); +x_205 = lean_ctor_get(x_3, 1); lean_inc(x_205); -x_206 = lean_ctor_get(x_3, 3); +x_206 = lean_ctor_get(x_3, 2); lean_inc(x_206); -x_207 = lean_ctor_get(x_3, 4); +x_207 = lean_ctor_get(x_3, 3); lean_inc(x_207); -x_208 = lean_ctor_get(x_3, 5); +x_208 = lean_ctor_get(x_3, 4); lean_inc(x_208); +x_209 = lean_ctor_get(x_3, 5); +lean_inc(x_209); if (lean_is_exclusive(x_3)) { lean_ctor_release(x_3, 0); lean_ctor_release(x_3, 1); @@ -3501,65 +7680,64 @@ if (lean_is_exclusive(x_3)) { lean_ctor_release(x_3, 3); lean_ctor_release(x_3, 4); lean_ctor_release(x_3, 5); - x_209 = x_3; + x_210 = x_3; } else { lean_dec_ref(x_3); - x_209 = lean_box(0); -} -x_210 = lean_ctor_get_uint8(x_201, 0); -x_211 = lean_ctor_get_uint8(x_201, 1); -x_212 = lean_ctor_get_uint8(x_201, 2); -x_213 = lean_ctor_get_uint8(x_201, 3); -x_214 = lean_ctor_get_uint8(x_201, 4); -x_215 = lean_ctor_get_uint8(x_201, 6); -x_216 = lean_ctor_get_uint8(x_201, 7); -x_217 = lean_ctor_get_uint8(x_201, 8); -x_218 = lean_ctor_get_uint8(x_201, 9); -x_219 = lean_ctor_get_uint8(x_201, 10); -x_220 = lean_ctor_get_uint8(x_201, 11); -x_221 = lean_ctor_get_uint8(x_201, 12); -x_222 = lean_ctor_get_uint8(x_201, 13); -if (lean_is_exclusive(x_201)) { - x_223 = x_201; -} else { - lean_dec_ref(x_201); - x_223 = lean_box(0); -} -x_224 = 1; -if (lean_is_scalar(x_223)) { - x_225 = lean_alloc_ctor(0, 0, 14); -} else { - x_225 = x_223; -} -lean_ctor_set_uint8(x_225, 0, x_210); -lean_ctor_set_uint8(x_225, 1, x_211); -lean_ctor_set_uint8(x_225, 2, x_212); -lean_ctor_set_uint8(x_225, 3, x_213); -lean_ctor_set_uint8(x_225, 4, x_214); -lean_ctor_set_uint8(x_225, 5, x_224); -lean_ctor_set_uint8(x_225, 6, x_215); -lean_ctor_set_uint8(x_225, 7, x_216); -lean_ctor_set_uint8(x_225, 8, x_217); -lean_ctor_set_uint8(x_225, 9, x_218); -lean_ctor_set_uint8(x_225, 10, x_219); -lean_ctor_set_uint8(x_225, 11, x_220); -lean_ctor_set_uint8(x_225, 12, x_221); -lean_ctor_set_uint8(x_225, 13, x_222); -if (lean_is_scalar(x_209)) { - x_226 = lean_alloc_ctor(0, 6, 0); -} else { - x_226 = x_209; -} -lean_ctor_set(x_226, 0, x_225); -lean_ctor_set(x_226, 1, x_204); -lean_ctor_set(x_226, 2, x_205); -lean_ctor_set(x_226, 3, x_206); -lean_ctor_set(x_226, 4, x_207); -lean_ctor_set(x_226, 5, x_208); -x_227 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1; + x_210 = lean_box(0); +} +x_211 = lean_ctor_get_uint8(x_204, 0); +x_212 = lean_ctor_get_uint8(x_204, 1); +x_213 = lean_ctor_get_uint8(x_204, 2); +x_214 = lean_ctor_get_uint8(x_204, 3); +x_215 = lean_ctor_get_uint8(x_204, 4); +x_216 = lean_ctor_get_uint8(x_204, 6); +x_217 = lean_ctor_get_uint8(x_204, 7); +x_218 = lean_ctor_get_uint8(x_204, 8); +x_219 = lean_ctor_get_uint8(x_204, 9); +x_220 = lean_ctor_get_uint8(x_204, 10); +x_221 = lean_ctor_get_uint8(x_204, 11); +x_222 = lean_ctor_get_uint8(x_204, 12); +x_223 = lean_ctor_get_uint8(x_204, 13); +if (lean_is_exclusive(x_204)) { + x_224 = x_204; +} else { + lean_dec_ref(x_204); + x_224 = lean_box(0); +} +x_225 = 1; +if (lean_is_scalar(x_224)) { + x_226 = lean_alloc_ctor(0, 0, 14); +} else { + x_226 = x_224; +} +lean_ctor_set_uint8(x_226, 0, x_211); +lean_ctor_set_uint8(x_226, 1, x_212); +lean_ctor_set_uint8(x_226, 2, x_213); +lean_ctor_set_uint8(x_226, 3, x_214); +lean_ctor_set_uint8(x_226, 4, x_215); +lean_ctor_set_uint8(x_226, 5, x_225); +lean_ctor_set_uint8(x_226, 6, x_216); +lean_ctor_set_uint8(x_226, 7, x_217); +lean_ctor_set_uint8(x_226, 8, x_218); +lean_ctor_set_uint8(x_226, 9, x_219); +lean_ctor_set_uint8(x_226, 10, x_220); +lean_ctor_set_uint8(x_226, 11, x_221); +lean_ctor_set_uint8(x_226, 12, x_222); +lean_ctor_set_uint8(x_226, 13, x_223); +if (lean_is_scalar(x_210)) { + x_227 = lean_alloc_ctor(0, 6, 0); +} else { + x_227 = x_210; +} +lean_ctor_set(x_227, 0, x_226); +lean_ctor_set(x_227, 1, x_205); +lean_ctor_set(x_227, 2, x_206); +lean_ctor_set(x_227, 3, x_207); +lean_ctor_set(x_227, 4, x_208); +lean_ctor_set(x_227, 5, x_209); lean_inc(x_6); lean_inc(x_4); -x_228 = l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__2___rarg(x_202, x_2, x_227, x_226, x_4, x_5, x_6, x_203); +x_228 = l_Lean_Meta_forallBoundedTelescope___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__8___rarg(x_200, x_2, x_203, x_227, x_4, x_5, x_6, x_201); if (lean_obj_tag(x_228) == 0) { lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; @@ -3625,7 +7803,7 @@ if (lean_is_exclusive(x_235)) { x_248 = lean_box(0); } lean_inc(x_229); -x_249 = l_Std_PersistentHashMap_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__4(x_247, x_197, x_229); +x_249 = l_Std_PersistentHashMap_insert___at___private_Lean_Meta_FunInfo_0__Lean_Meta_checkFunInfoCache___spec__4(x_247, x_196, x_229); if (lean_is_scalar(x_248)) { x_250 = lean_alloc_ctor(0, 7, 0); } else { @@ -3671,7 +7849,7 @@ return x_255; else { lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; -lean_dec(x_197); +lean_dec(x_196); lean_dec(x_6); lean_dec(x_4); x_256 = lean_ctor_get(x_228, 0); @@ -3699,22 +7877,22 @@ return x_259; else { lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; -lean_dec(x_197); +lean_dec(x_196); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_260 = lean_ctor_get(x_200, 0); +x_260 = lean_ctor_get(x_199, 0); lean_inc(x_260); -x_261 = lean_ctor_get(x_200, 1); +x_261 = lean_ctor_get(x_199, 1); lean_inc(x_261); -if (lean_is_exclusive(x_200)) { - lean_ctor_release(x_200, 0); - lean_ctor_release(x_200, 1); - x_262 = x_200; +if (lean_is_exclusive(x_199)) { + lean_ctor_release(x_199, 0); + lean_ctor_release(x_199, 1); + x_262 = x_199; } else { - lean_dec_ref(x_200); + lean_dec_ref(x_199); x_262 = lean_box(0); } if (lean_is_scalar(x_262)) { @@ -3730,29 +7908,68 @@ return x_263; else { lean_object* x_264; lean_object* x_265; -lean_dec(x_197); +lean_dec(x_196); 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_264 = lean_ctor_get(x_199, 0); +x_264 = lean_ctor_get(x_198, 0); lean_inc(x_264); -lean_dec(x_199); +lean_dec(x_198); x_265 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_265, 0, x_264); -lean_ctor_set(x_265, 1, x_194); +lean_ctor_set(x_265, 1, x_193); return x_265; } } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +lean_object* x_16; +x_16 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Std_RBNode_findCore___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__5___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_RBNode_findCore___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__5(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -3762,15 +7979,48 @@ lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__2___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__2(x_1, x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; -x_13 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_14; +x_14 = l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -return x_13; +lean_dec(x_3); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_1); +return x_9; } } LEAN_EXPORT lean_object* l_Lean_Meta_getFunInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -3837,20 +8087,24 @@ l_Array_qsort_sort___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___s lean_mark_persistent(l_Array_qsort_sort___at___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___spec__1___closed__1); l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___closed__1 = _init_l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___closed__1(); lean_mark_persistent(l___private_Lean_Meta_FunInfo_0__Lean_Meta_collectDeps___closed__1); -l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__1(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__1); -l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__2(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___lambda__1___closed__2); -l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__1(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__1); -l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__2(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__2); -l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__3 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__3(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__3); -l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__4 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__4(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__4); -l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__5 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__5(); -lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__1___closed__5); +l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__1); +l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__2); +l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__3 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__3(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__3); +l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__3___closed__4); +l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__1); +l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___lambda__1___closed__2); +l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__1 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__1); +l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__2 = _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_loop___at___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___spec__6___closed__2); +l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___closed__1 = _init_l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___lambda__1___closed__1); l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1 = _init_l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1(); lean_mark_persistent(l___private_Lean_Meta_FunInfo_0__Lean_Meta_getFunInfoAux___closed__1); return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/GetConst.c b/stage0/stdlib/Lean/Meta/GetConst.c index 97c4f3cad923..469f897850bb 100644 --- a/stage0/stdlib/Lean/Meta/GetConst.c +++ b/stage0/stdlib/Lean/Meta/GetConst.c @@ -21,7 +21,7 @@ lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getConstNoEx_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isReducible___at___private_Lean_Meta_GetConst_0__Lean_Meta_canUnfoldDefault___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getConst_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(uint8_t, uint8_t); +uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(uint8_t, uint8_t); lean_object* l_Lean_ConstantInfo_name(lean_object*); LEAN_EXPORT lean_object* l_Lean_getReducibilityStatus___at___private_Lean_Meta_GetConst_0__Lean_Meta_canUnfoldDefault___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_GetConst_0__Lean_Meta_canUnfoldDefault(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -315,7 +315,7 @@ x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); lean_dec(x_38); x_40 = 3; -x_41 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_6, x_40); +x_41 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_6, x_40); if (x_41 == 0) { uint8_t x_42; lean_object* x_43; @@ -360,7 +360,7 @@ x_51 = lean_ctor_get(x_49, 0); lean_inc(x_51); lean_dec(x_49); x_52 = 3; -x_53 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_6, x_52); +x_53 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_6, x_52); if (x_53 == 0) { uint8_t x_54; lean_object* x_55; lean_object* x_56; diff --git a/stage0/stdlib/Lean/Meta/IndPredBelow.c b/stage0/stdlib/Lean/Meta/IndPredBelow.c index 42f0f289783e..4c91242e1974 100644 --- a/stage0/stdlib/Lean/Meta/IndPredBelow.c +++ b/stage0/stdlib/Lean/Meta/IndPredBelow.c @@ -52,7 +52,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___at_Lean_Meta_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher_convertToBelow___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_numLevelParams(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_proveBrecOn_induction___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -84,6 +83,7 @@ static lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveName___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkContext_motiveName___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_cases_on(lean_object*, lean_object*); static lean_object* l_Array_mapIdxM_map___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__3___lambda__2___closed__7; +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_findBelowIdx___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__7(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); @@ -251,6 +251,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Meta_IndPredBelow_mkCto LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_IndPredBelow_mkBelowMatcher___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_mkCtorType_rebuild___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addDecl___at_Lean_Meta_IndPredBelow_mkBelow___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addHeaderVars___spec__3(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -348,7 +349,6 @@ lean_object* l_Lean_throwKernelException___at_Lean_Meta_evalExprCore___spec__3(l LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_IndPredBelow_mkInductiveType___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at_Lean_Meta_IndPredBelow_backwardsChaining___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__6___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceOptions(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkBelow___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -368,6 +368,7 @@ lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); +size_t lean_ptr_addr(lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_checkCount___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -383,7 +384,6 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_IndPredBelow_mkBelowMatcher_tran static lean_object* l_Lean_Meta_IndPredBelow_proveBrecOn_closeGoal___closed__2; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lean_Meta_IndPredBelow_mkBelow___closed__4; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_mkCasesOn___at_Lean_Meta_IndPredBelow_mkBelow___spec__1___closed__12; extern lean_object* l_Lean_Meta_Match_instInhabitedPattern; LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkBelowMatcher_addBelowPattern___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -515,6 +515,7 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_IndPredBelow_back LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_IndPredBelow_mkCtorType_addMotives___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_proveBrecOn_applyCtors___spec__4(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_findBelowIdx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_IndPredBelow_mkContext_addMotives___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); @@ -2077,7 +2078,7 @@ static lean_object* _init_l_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars___ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars___closed__1; x_2 = l_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_IndPredBelow_mkCtorType_replaceTempVars___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4491,7 +4492,7 @@ lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean x_10 = lean_ctor_get(x_4, 5); lean_inc(x_10); x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_10, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_10, x_11); x_13 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_12); x_14 = lean_mk_array(x_12, x_13); @@ -4818,7 +4819,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_mkMotiveBinder___la { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_7, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_7, x_13); x_15 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -5318,7 +5319,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_IndPredBelow_mkCtorType_mkBelowBinder___lam { lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Lean_Expr_getAppNumArgsAux(x_6, x_12); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_6, x_12); x_14 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_13); x_15 = lean_mk_array(x_13, x_14); @@ -6923,7 +6924,7 @@ case 5: { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_16, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_16, x_17); x_19 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -6956,35 +6957,57 @@ return x_29; } case 10: { -lean_object* x_30; lean_object* x_31; -x_30 = lean_ctor_get(x_16, 1); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_16, 0); lean_inc(x_30); +x_31 = lean_ctor_get(x_16, 1); +lean_inc(x_31); 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_31); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_31 = l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_31) == 0) +x_32 = l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2(x_1, x_2, x_3, x_4, x_5, x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); +lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; uint8_t x_37; +x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = lean_ptr_addr(x_31); lean_dec(x_31); -x_34 = lean_expr_update_mdata(x_16, x_32); -x_35 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3(x_1, x_2, x_3, x_4, x_5, x_34, x_7, x_8, x_9, x_10, x_11, x_12, x_33); -return x_35; +x_36 = lean_ptr_addr(x_33); +x_37 = lean_usize_dec_eq(x_35, x_36); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; +lean_dec(x_16); +x_38 = l_Lean_Expr_mdata___override(x_30, x_33); +x_39 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3(x_1, x_2, x_3, x_4, x_5, x_38, x_7, x_8, x_9, x_10, x_11, x_12, x_34); +return x_39; } else { -uint8_t x_36; +lean_object* x_40; +lean_dec(x_33); +lean_dec(x_30); +x_40 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3(x_1, x_2, x_3, x_4, x_5, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_34); +return x_40; +} +} +else +{ +uint8_t x_41; +lean_dec(x_31); +lean_dec(x_30); lean_dec(x_16); lean_dec(x_12); lean_dec(x_11); @@ -6996,57 +7019,83 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_36 = !lean_is_exclusive(x_31); -if (x_36 == 0) +x_41 = !lean_is_exclusive(x_32); +if (x_41 == 0) { -return x_31; +return x_32; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_31, 0); -x_38 = lean_ctor_get(x_31, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_31); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_32, 0); +x_43 = lean_ctor_get(x_32, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_32); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } } } case 11: { -lean_object* x_40; lean_object* x_41; -x_40 = lean_ctor_get(x_16, 2); -lean_inc(x_40); +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_45 = lean_ctor_get(x_16, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_16, 1); +lean_inc(x_46); +x_47 = lean_ctor_get(x_16, 2); +lean_inc(x_47); 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_47); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_41 = l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2(x_1, x_2, x_3, x_4, x_5, x_40, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_41) == 0) +x_48 = l_Lean_Meta_transform_visit___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__2(x_1, x_2, x_3, x_4, x_5, x_47, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = lean_expr_update_proj(x_16, x_42); -x_45 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3(x_1, x_2, x_3, x_4, x_5, x_44, x_7, x_8, x_9, x_10, x_11, x_12, x_43); -return x_45; +lean_object* x_49; lean_object* x_50; size_t x_51; size_t x_52; uint8_t x_53; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_ptr_addr(x_47); +lean_dec(x_47); +x_52 = lean_ptr_addr(x_49); +x_53 = lean_usize_dec_eq(x_51, x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; +lean_dec(x_16); +x_54 = l_Lean_Expr_proj___override(x_45, x_46, x_49); +x_55 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3(x_1, x_2, x_3, x_4, x_5, x_54, x_7, x_8, x_9, x_10, x_11, x_12, x_50); +return x_55; } else { -uint8_t x_46; +lean_object* x_56; +lean_dec(x_49); +lean_dec(x_46); +lean_dec(x_45); +x_56 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3(x_1, x_2, x_3, x_4, x_5, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_50); +return x_56; +} +} +else +{ +uint8_t x_57; +lean_dec(x_47); +lean_dec(x_46); +lean_dec(x_45); lean_dec(x_16); lean_dec(x_12); lean_dec(x_11); @@ -7058,31 +7107,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_46 = !lean_is_exclusive(x_41); -if (x_46 == 0) +x_57 = !lean_is_exclusive(x_48); +if (x_57 == 0) { -return x_41; +return x_48; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_41, 0); -x_48 = lean_ctor_get(x_41, 1); -lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_41); -x_49 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); -return x_49; +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_48, 0); +x_59 = lean_ctor_get(x_48, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_48); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; } } } default: { -lean_object* x_50; -x_50 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3(x_1, x_2, x_3, x_4, x_5, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_50; +lean_object* x_61; +x_61 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_IndPredBelow_mkCtorType_checkCount___spec__3(x_1, x_2, x_3, x_4, x_5, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_61; } } } @@ -12811,7 +12860,7 @@ x_16 = l_Lean_instInhabitedExpr; x_17 = l_Array_back___rarg(x_16, x_3); lean_dec(x_3); x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_17, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_17, x_18); x_20 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_19); x_21 = lean_mk_array(x_19, x_20); @@ -12866,7 +12915,7 @@ lean_inc(x_21); x_22 = lean_ctor_get(x_20, 1); lean_inc(x_22); lean_dec(x_20); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_21, x_12); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_21, x_12); x_24 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -15481,7 +15530,7 @@ x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_11, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_13); x_15 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -17166,7 +17215,7 @@ x_39 = lean_ctor_get(x_37, 1); lean_inc(x_39); lean_dec(x_37); x_40 = lean_unsigned_to_nat(0u); -x_41 = l_Lean_Expr_getAppNumArgsAux(x_38, x_40); +x_41 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_38, x_40); x_42 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_41); x_43 = lean_mk_array(x_41, x_42); @@ -25137,7 +25186,7 @@ x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); x_19 = lean_unsigned_to_nat(0u); -x_20 = l_Lean_Expr_getAppNumArgsAux(x_17, x_19); +x_20 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_17, x_19); x_21 = l_Lean_Meta_IndPredBelow_mkContext_motiveType___lambda__1___closed__1; lean_inc(x_20); x_22 = lean_mk_array(x_20, x_21); diff --git a/stage0/stdlib/Lean/Meta/InferType.c b/stage0/stdlib/Lean/Meta/InferType.c index 50e3a9640f27..17baef86c886 100644 --- a/stage0/stdlib/Lean/Meta/InferType.c +++ b/stage0/stdlib/Lean/Meta/InferType.c @@ -13,22 +13,22 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_throwUnknownMVar___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux___rarg(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFreshLevelMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_throwTypeExcepted___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); +lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_assignExprMVar___at_Lean_Meta_getLevel___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkForallFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(lean_object*); +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferLambdaType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_withLocalDecl_x27(lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); lean_object* l_Lean_Level_succ___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_instantiateBetaRevRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferMVarType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -47,6 +47,7 @@ size_t lean_usize_sub(size_t, size_t); lean_object* lean_environment_find(lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_isArrowType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_throwFunctionExpected(lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_inferTypeImp_infer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -65,6 +66,7 @@ lean_object* l_Std_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_InferType_0__Lean_Meta_inferProjType___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_lift_loose_bvars(lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_Std_PersistentHashMap_insert___at_Lean_assignExprMVar___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Expr_0__Lean_Expr_withAppRevAux___at_Lean_Expr_instantiateBetaRevRange_visit___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_right(size_t, size_t); @@ -117,10 +119,11 @@ lean_object* l_Std_mkHashMapImp___rarg(lean_object*); lean_object* l_instInhabited___rarg(lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Expr_instantiateBetaRevRange_visit___spec__10___closed__2; static lean_object* l_panic___at_Lean_Expr_instantiateBetaRevRange_visit___spec__10___closed__1; -lean_object* lean_level_mk_imax_simp(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Expr_instantiateBetaRevRange_visit___spec__7___at_Lean_Expr_instantiateBetaRevRange_visit___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Expr_instantiateBetaRevRange_visit___spec__2(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Expr_instantiateBetaRevRange_visit___closed__4; LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Expr_instantiateBetaRevRange_visit___spec__2___boxed(lean_object*, lean_object*); uint64_t l_Lean_Expr_hash(lean_object*); @@ -147,7 +150,6 @@ size_t lean_usize_mul(size_t, size_t); lean_object* l_Lean_Expr_bvar___override(lean_object*); static lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferProjType___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_throwTypeExcepted(lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_throwIncorrectNumberOfLevels___rarg___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferForallType___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_inferFVarType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -157,7 +159,6 @@ static lean_object* l_Lean_Expr_instantiateBetaRevRange_visit___closed__13; size_t lean_usize_of_nat(lean_object*); lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_throwFunctionExpected___rarg___closed__3; -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_throwFunctionExpected___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_throwFunctionExpected___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -173,9 +174,9 @@ lean_object* lean_local_ctx_mk_local_decl(lean_object*, lean_object*, lean_objec LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); static lean_object* l_Lean_Meta_throwUnknownMVar___rarg___closed__3; +size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Expr_instantiateBetaRevRange_visit___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isTypeQuick(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Meta_abstractRange___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_equal(lean_object*, lean_object*); @@ -206,7 +207,6 @@ lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_InferType_0__Lean_Meta_isPropQuickApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Meta_throwFunctionExpected___rarg___closed__4; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_throwUnknownMVar___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -223,6 +223,7 @@ lean_object* lean_mk_array(lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_mkAppRangeAux(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instHashableNat___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Expr_instantiateBetaRevRange___spec__1(lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_throwUnknownMVar___spec__1(lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); static lean_object* l_Lean_Expr_instantiateBetaRevRange_visit___closed__5; @@ -1059,7 +1060,7 @@ static lean_object* _init_l_Lean_Expr_instantiateBetaRevRange_visit___closed__7( lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Expr_instantiateBetaRevRange_visit___closed__4; x_2 = l_Lean_Expr_instantiateBetaRevRange_visit___closed__5; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Expr_instantiateBetaRevRange_visit___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1390,7 +1391,7 @@ case 5: { lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; x_76 = lean_unsigned_to_nat(0u); -x_77 = l_Lean_Expr_getAppNumArgsAux(x_4, x_76); +x_77 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_76); x_78 = lean_mk_empty_array_with_capacity(x_77); lean_dec(x_77); x_79 = l_Lean_Expr_instantiateBetaRevRange_visit___closed__1; @@ -1425,290 +1426,777 @@ return x_89; } case 6: { -lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; -x_90 = lean_ctor_get(x_4, 1); +lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; uint8_t x_100; +x_90 = lean_ctor_get(x_4, 0); lean_inc(x_90); -x_91 = lean_ctor_get(x_4, 2); +x_91 = lean_ctor_get(x_4, 1); lean_inc(x_91); -x_92 = lean_ctor_get_uint8(x_4, sizeof(void*)*3 + 8); +x_92 = lean_ctor_get(x_4, 2); +lean_inc(x_92); +x_93 = lean_ctor_get_uint8(x_4, sizeof(void*)*3 + 8); +lean_dec(x_4); lean_inc(x_5); -x_93 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_90, x_5, x_6); -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_93, 1); +lean_inc(x_91); +x_94 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_91, x_5, x_6); +x_95 = lean_ctor_get(x_94, 0); lean_inc(x_95); -lean_dec(x_93); -x_96 = lean_unsigned_to_nat(1u); -x_97 = lean_nat_add(x_5, x_96); -lean_dec(x_5); -x_98 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_91, x_97, x_95); -x_99 = !lean_is_exclusive(x_98); -if (x_99 == 0) -{ -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_100 = lean_ctor_get(x_98, 0); -x_101 = lean_ctor_get(x_98, 1); -x_102 = lean_expr_update_lambda(x_4, x_92, x_94, x_100); -lean_inc(x_102); -x_103 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_101, x_9, x_102); -lean_ctor_set(x_98, 1, x_103); -lean_ctor_set(x_98, 0, x_102); -return x_98; +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +lean_dec(x_94); +x_97 = lean_unsigned_to_nat(1u); +x_98 = lean_nat_add(x_5, x_97); +lean_dec(x_5); +lean_inc(x_92); +x_99 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_92, x_98, x_96); +x_100 = !lean_is_exclusive(x_99); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; size_t x_104; size_t x_105; uint8_t x_106; +x_101 = lean_ctor_get(x_99, 0); +x_102 = lean_ctor_get(x_99, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_inc(x_90); +x_103 = l_Lean_Expr_lam___override(x_90, x_91, x_92, x_93); +x_104 = lean_ptr_addr(x_91); +lean_dec(x_91); +x_105 = lean_ptr_addr(x_95); +x_106 = lean_usize_dec_eq(x_104, x_105); +if (x_106 == 0) +{ +lean_object* x_107; lean_object* x_108; +lean_dec(x_103); +lean_dec(x_92); +x_107 = l_Lean_Expr_lam___override(x_90, x_95, x_101, x_93); +lean_inc(x_107); +x_108 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_102, x_9, x_107); +lean_ctor_set(x_99, 1, x_108); +lean_ctor_set(x_99, 0, x_107); +return x_99; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_104 = lean_ctor_get(x_98, 0); -x_105 = lean_ctor_get(x_98, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_98); -x_106 = lean_expr_update_lambda(x_4, x_92, x_94, x_104); -lean_inc(x_106); -x_107 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_105, x_9, x_106); -x_108 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_108, 0, x_106); -lean_ctor_set(x_108, 1, x_107); -return x_108; +size_t x_109; size_t x_110; uint8_t x_111; +x_109 = lean_ptr_addr(x_92); +lean_dec(x_92); +x_110 = lean_ptr_addr(x_101); +x_111 = lean_usize_dec_eq(x_109, x_110); +if (x_111 == 0) +{ +lean_object* x_112; lean_object* x_113; +lean_dec(x_103); +x_112 = l_Lean_Expr_lam___override(x_90, x_95, x_101, x_93); +lean_inc(x_112); +x_113 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_102, x_9, x_112); +lean_ctor_set(x_99, 1, x_113); +lean_ctor_set(x_99, 0, x_112); +return x_99; +} +else +{ +uint8_t x_114; +x_114 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_93, x_93); +if (x_114 == 0) +{ +lean_object* x_115; lean_object* x_116; +lean_dec(x_103); +x_115 = l_Lean_Expr_lam___override(x_90, x_95, x_101, x_93); +lean_inc(x_115); +x_116 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_102, x_9, x_115); +lean_ctor_set(x_99, 1, x_116); +lean_ctor_set(x_99, 0, x_115); +return x_99; +} +else +{ +lean_object* x_117; +lean_dec(x_101); +lean_dec(x_95); +lean_dec(x_90); +lean_inc(x_103); +x_117 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_102, x_9, x_103); +lean_ctor_set(x_99, 1, x_117); +lean_ctor_set(x_99, 0, x_103); +return x_99; +} +} +} +} +else +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; size_t x_121; size_t x_122; uint8_t x_123; +x_118 = lean_ctor_get(x_99, 0); +x_119 = lean_ctor_get(x_99, 1); +lean_inc(x_119); +lean_inc(x_118); +lean_dec(x_99); +lean_inc(x_92); +lean_inc(x_91); +lean_inc(x_90); +x_120 = l_Lean_Expr_lam___override(x_90, x_91, x_92, x_93); +x_121 = lean_ptr_addr(x_91); +lean_dec(x_91); +x_122 = lean_ptr_addr(x_95); +x_123 = lean_usize_dec_eq(x_121, x_122); +if (x_123 == 0) +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; +lean_dec(x_120); +lean_dec(x_92); +x_124 = l_Lean_Expr_lam___override(x_90, x_95, x_118, x_93); +lean_inc(x_124); +x_125 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_119, x_9, x_124); +x_126 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +return x_126; +} +else +{ +size_t x_127; size_t x_128; uint8_t x_129; +x_127 = lean_ptr_addr(x_92); +lean_dec(x_92); +x_128 = lean_ptr_addr(x_118); +x_129 = lean_usize_dec_eq(x_127, x_128); +if (x_129 == 0) +{ +lean_object* x_130; lean_object* x_131; lean_object* x_132; +lean_dec(x_120); +x_130 = l_Lean_Expr_lam___override(x_90, x_95, x_118, x_93); +lean_inc(x_130); +x_131 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_119, x_9, x_130); +x_132 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_132, 0, x_130); +lean_ctor_set(x_132, 1, x_131); +return x_132; +} +else +{ +uint8_t x_133; +x_133 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_93, x_93); +if (x_133 == 0) +{ +lean_object* x_134; lean_object* x_135; lean_object* x_136; +lean_dec(x_120); +x_134 = l_Lean_Expr_lam___override(x_90, x_95, x_118, x_93); +lean_inc(x_134); +x_135 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_119, x_9, x_134); +x_136 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_136, 0, x_134); +lean_ctor_set(x_136, 1, x_135); +return x_136; +} +else +{ +lean_object* x_137; lean_object* x_138; +lean_dec(x_118); +lean_dec(x_95); +lean_dec(x_90); +lean_inc(x_120); +x_137 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_119, x_9, x_120); +x_138 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_138, 0, x_120); +lean_ctor_set(x_138, 1, x_137); +return x_138; +} +} +} } } case 7: { -lean_object* x_109; lean_object* x_110; uint8_t x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; uint8_t x_118; -x_109 = lean_ctor_get(x_4, 1); -lean_inc(x_109); -x_110 = lean_ctor_get(x_4, 2); -lean_inc(x_110); -x_111 = lean_ctor_get_uint8(x_4, sizeof(void*)*3 + 8); +lean_object* x_139; lean_object* x_140; lean_object* x_141; uint8_t x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; uint8_t x_149; +x_139 = lean_ctor_get(x_4, 0); +lean_inc(x_139); +x_140 = lean_ctor_get(x_4, 1); +lean_inc(x_140); +x_141 = lean_ctor_get(x_4, 2); +lean_inc(x_141); +x_142 = lean_ctor_get_uint8(x_4, sizeof(void*)*3 + 8); +lean_dec(x_4); lean_inc(x_5); -x_112 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_109, x_5, x_6); -x_113 = lean_ctor_get(x_112, 0); -lean_inc(x_113); -x_114 = lean_ctor_get(x_112, 1); -lean_inc(x_114); -lean_dec(x_112); -x_115 = lean_unsigned_to_nat(1u); -x_116 = lean_nat_add(x_5, x_115); -lean_dec(x_5); -x_117 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_110, x_116, x_114); -x_118 = !lean_is_exclusive(x_117); -if (x_118 == 0) -{ -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_119 = lean_ctor_get(x_117, 0); -x_120 = lean_ctor_get(x_117, 1); -x_121 = lean_expr_update_forall(x_4, x_111, x_113, x_119); -lean_inc(x_121); -x_122 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_120, x_9, x_121); -lean_ctor_set(x_117, 1, x_122); -lean_ctor_set(x_117, 0, x_121); -return x_117; +lean_inc(x_140); +x_143 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_140, x_5, x_6); +x_144 = lean_ctor_get(x_143, 0); +lean_inc(x_144); +x_145 = lean_ctor_get(x_143, 1); +lean_inc(x_145); +lean_dec(x_143); +x_146 = lean_unsigned_to_nat(1u); +x_147 = lean_nat_add(x_5, x_146); +lean_dec(x_5); +lean_inc(x_141); +x_148 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_141, x_147, x_145); +x_149 = !lean_is_exclusive(x_148); +if (x_149 == 0) +{ +lean_object* x_150; lean_object* x_151; lean_object* x_152; size_t x_153; size_t x_154; uint8_t x_155; +x_150 = lean_ctor_get(x_148, 0); +x_151 = lean_ctor_get(x_148, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_inc(x_139); +x_152 = l_Lean_Expr_forallE___override(x_139, x_140, x_141, x_142); +x_153 = lean_ptr_addr(x_140); +lean_dec(x_140); +x_154 = lean_ptr_addr(x_144); +x_155 = lean_usize_dec_eq(x_153, x_154); +if (x_155 == 0) +{ +lean_object* x_156; lean_object* x_157; +lean_dec(x_152); +lean_dec(x_141); +x_156 = l_Lean_Expr_forallE___override(x_139, x_144, x_150, x_142); +lean_inc(x_156); +x_157 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_151, x_9, x_156); +lean_ctor_set(x_148, 1, x_157); +lean_ctor_set(x_148, 0, x_156); +return x_148; } else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_123 = lean_ctor_get(x_117, 0); -x_124 = lean_ctor_get(x_117, 1); -lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_117); -x_125 = lean_expr_update_forall(x_4, x_111, x_113, x_123); -lean_inc(x_125); -x_126 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_124, x_9, x_125); -x_127 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_127, 0, x_125); -lean_ctor_set(x_127, 1, x_126); -return x_127; +size_t x_158; size_t x_159; uint8_t x_160; +x_158 = lean_ptr_addr(x_141); +lean_dec(x_141); +x_159 = lean_ptr_addr(x_150); +x_160 = lean_usize_dec_eq(x_158, x_159); +if (x_160 == 0) +{ +lean_object* x_161; lean_object* x_162; +lean_dec(x_152); +x_161 = l_Lean_Expr_forallE___override(x_139, x_144, x_150, x_142); +lean_inc(x_161); +x_162 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_151, x_9, x_161); +lean_ctor_set(x_148, 1, x_162); +lean_ctor_set(x_148, 0, x_161); +return x_148; +} +else +{ +uint8_t x_163; +x_163 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_142, x_142); +if (x_163 == 0) +{ +lean_object* x_164; lean_object* x_165; +lean_dec(x_152); +x_164 = l_Lean_Expr_forallE___override(x_139, x_144, x_150, x_142); +lean_inc(x_164); +x_165 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_151, x_9, x_164); +lean_ctor_set(x_148, 1, x_165); +lean_ctor_set(x_148, 0, x_164); +return x_148; +} +else +{ +lean_object* x_166; +lean_dec(x_150); +lean_dec(x_144); +lean_dec(x_139); +lean_inc(x_152); +x_166 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_151, x_9, x_152); +lean_ctor_set(x_148, 1, x_166); +lean_ctor_set(x_148, 0, x_152); +return x_148; +} +} +} +} +else +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; size_t x_170; size_t x_171; uint8_t x_172; +x_167 = lean_ctor_get(x_148, 0); +x_168 = lean_ctor_get(x_148, 1); +lean_inc(x_168); +lean_inc(x_167); +lean_dec(x_148); +lean_inc(x_141); +lean_inc(x_140); +lean_inc(x_139); +x_169 = l_Lean_Expr_forallE___override(x_139, x_140, x_141, x_142); +x_170 = lean_ptr_addr(x_140); +lean_dec(x_140); +x_171 = lean_ptr_addr(x_144); +x_172 = lean_usize_dec_eq(x_170, x_171); +if (x_172 == 0) +{ +lean_object* x_173; lean_object* x_174; lean_object* x_175; +lean_dec(x_169); +lean_dec(x_141); +x_173 = l_Lean_Expr_forallE___override(x_139, x_144, x_167, x_142); +lean_inc(x_173); +x_174 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_168, x_9, x_173); +x_175 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_175, 0, x_173); +lean_ctor_set(x_175, 1, x_174); +return x_175; +} +else +{ +size_t x_176; size_t x_177; uint8_t x_178; +x_176 = lean_ptr_addr(x_141); +lean_dec(x_141); +x_177 = lean_ptr_addr(x_167); +x_178 = lean_usize_dec_eq(x_176, x_177); +if (x_178 == 0) +{ +lean_object* x_179; lean_object* x_180; lean_object* x_181; +lean_dec(x_169); +x_179 = l_Lean_Expr_forallE___override(x_139, x_144, x_167, x_142); +lean_inc(x_179); +x_180 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_168, x_9, x_179); +x_181 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_181, 0, x_179); +lean_ctor_set(x_181, 1, x_180); +return x_181; +} +else +{ +uint8_t x_182; +x_182 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_142, x_142); +if (x_182 == 0) +{ +lean_object* x_183; lean_object* x_184; lean_object* x_185; +lean_dec(x_169); +x_183 = l_Lean_Expr_forallE___override(x_139, x_144, x_167, x_142); +lean_inc(x_183); +x_184 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_168, x_9, x_183); +x_185 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_185, 0, x_183); +lean_ctor_set(x_185, 1, x_184); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; +lean_dec(x_167); +lean_dec(x_144); +lean_dec(x_139); +lean_inc(x_169); +x_186 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_168, x_9, x_169); +x_187 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_187, 0, x_169); +lean_ctor_set(x_187, 1, x_186); +return x_187; +} +} +} } } case 8: { -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; uint8_t x_140; -x_128 = lean_ctor_get(x_4, 1); -lean_inc(x_128); -x_129 = lean_ctor_get(x_4, 2); -lean_inc(x_129); -x_130 = lean_ctor_get(x_4, 3); -lean_inc(x_130); +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; uint8_t x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; uint8_t x_202; +x_188 = lean_ctor_get(x_4, 0); +lean_inc(x_188); +x_189 = lean_ctor_get(x_4, 1); +lean_inc(x_189); +x_190 = lean_ctor_get(x_4, 2); +lean_inc(x_190); +x_191 = lean_ctor_get(x_4, 3); +lean_inc(x_191); +x_192 = lean_ctor_get_uint8(x_4, sizeof(void*)*4 + 8); lean_inc(x_5); -x_131 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_128, x_5, x_6); -x_132 = lean_ctor_get(x_131, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_131, 1); -lean_inc(x_133); -lean_dec(x_131); +lean_inc(x_189); +x_193 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_189, x_5, x_6); +x_194 = lean_ctor_get(x_193, 0); +lean_inc(x_194); +x_195 = lean_ctor_get(x_193, 1); +lean_inc(x_195); +lean_dec(x_193); lean_inc(x_5); -x_134 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_129, x_5, x_133); -x_135 = lean_ctor_get(x_134, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_134, 1); -lean_inc(x_136); -lean_dec(x_134); -x_137 = lean_unsigned_to_nat(1u); -x_138 = lean_nat_add(x_5, x_137); +lean_inc(x_190); +x_196 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_190, x_5, x_195); +x_197 = lean_ctor_get(x_196, 0); +lean_inc(x_197); +x_198 = lean_ctor_get(x_196, 1); +lean_inc(x_198); +lean_dec(x_196); +x_199 = lean_unsigned_to_nat(1u); +x_200 = lean_nat_add(x_5, x_199); lean_dec(x_5); -x_139 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_130, x_138, x_136); -x_140 = !lean_is_exclusive(x_139); -if (x_140 == 0) +lean_inc(x_191); +x_201 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_191, x_200, x_198); +x_202 = !lean_is_exclusive(x_201); +if (x_202 == 0) { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_141 = lean_ctor_get(x_139, 0); -x_142 = lean_ctor_get(x_139, 1); -x_143 = lean_expr_update_let(x_4, x_132, x_135, x_141); -lean_inc(x_143); -x_144 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_142, x_9, x_143); -lean_ctor_set(x_139, 1, x_144); -lean_ctor_set(x_139, 0, x_143); -return x_139; +lean_object* x_203; lean_object* x_204; size_t x_205; size_t x_206; uint8_t x_207; +x_203 = lean_ctor_get(x_201, 0); +x_204 = lean_ctor_get(x_201, 1); +x_205 = lean_ptr_addr(x_189); +lean_dec(x_189); +x_206 = lean_ptr_addr(x_194); +x_207 = lean_usize_dec_eq(x_205, x_206); +if (x_207 == 0) +{ +lean_object* x_208; lean_object* x_209; +lean_dec(x_191); +lean_dec(x_190); +lean_dec(x_4); +x_208 = l_Lean_Expr_letE___override(x_188, x_194, x_197, x_203, x_192); +lean_inc(x_208); +x_209 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_204, x_9, x_208); +lean_ctor_set(x_201, 1, x_209); +lean_ctor_set(x_201, 0, x_208); +return x_201; } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -x_145 = lean_ctor_get(x_139, 0); -x_146 = lean_ctor_get(x_139, 1); -lean_inc(x_146); -lean_inc(x_145); -lean_dec(x_139); -x_147 = lean_expr_update_let(x_4, x_132, x_135, x_145); -lean_inc(x_147); -x_148 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_146, x_9, x_147); -x_149 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_149, 0, x_147); -lean_ctor_set(x_149, 1, x_148); -return x_149; +size_t x_210; size_t x_211; uint8_t x_212; +x_210 = lean_ptr_addr(x_190); +lean_dec(x_190); +x_211 = lean_ptr_addr(x_197); +x_212 = lean_usize_dec_eq(x_210, x_211); +if (x_212 == 0) +{ +lean_object* x_213; lean_object* x_214; +lean_dec(x_191); +lean_dec(x_4); +x_213 = l_Lean_Expr_letE___override(x_188, x_194, x_197, x_203, x_192); +lean_inc(x_213); +x_214 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_204, x_9, x_213); +lean_ctor_set(x_201, 1, x_214); +lean_ctor_set(x_201, 0, x_213); +return x_201; +} +else +{ +size_t x_215; size_t x_216; uint8_t x_217; +x_215 = lean_ptr_addr(x_191); +lean_dec(x_191); +x_216 = lean_ptr_addr(x_203); +x_217 = lean_usize_dec_eq(x_215, x_216); +if (x_217 == 0) +{ +lean_object* x_218; lean_object* x_219; +lean_dec(x_4); +x_218 = l_Lean_Expr_letE___override(x_188, x_194, x_197, x_203, x_192); +lean_inc(x_218); +x_219 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_204, x_9, x_218); +lean_ctor_set(x_201, 1, x_219); +lean_ctor_set(x_201, 0, x_218); +return x_201; +} +else +{ +lean_object* x_220; +lean_dec(x_203); +lean_dec(x_197); +lean_dec(x_194); +lean_dec(x_188); +lean_inc(x_4); +x_220 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_204, x_9, x_4); +lean_ctor_set(x_201, 1, x_220); +lean_ctor_set(x_201, 0, x_4); +return x_201; +} +} +} +} +else +{ +lean_object* x_221; lean_object* x_222; size_t x_223; size_t x_224; uint8_t x_225; +x_221 = lean_ctor_get(x_201, 0); +x_222 = lean_ctor_get(x_201, 1); +lean_inc(x_222); +lean_inc(x_221); +lean_dec(x_201); +x_223 = lean_ptr_addr(x_189); +lean_dec(x_189); +x_224 = lean_ptr_addr(x_194); +x_225 = lean_usize_dec_eq(x_223, x_224); +if (x_225 == 0) +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; +lean_dec(x_191); +lean_dec(x_190); +lean_dec(x_4); +x_226 = l_Lean_Expr_letE___override(x_188, x_194, x_197, x_221, x_192); +lean_inc(x_226); +x_227 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_222, x_9, x_226); +x_228 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_228, 0, x_226); +lean_ctor_set(x_228, 1, x_227); +return x_228; +} +else +{ +size_t x_229; size_t x_230; uint8_t x_231; +x_229 = lean_ptr_addr(x_190); +lean_dec(x_190); +x_230 = lean_ptr_addr(x_197); +x_231 = lean_usize_dec_eq(x_229, x_230); +if (x_231 == 0) +{ +lean_object* x_232; lean_object* x_233; lean_object* x_234; +lean_dec(x_191); +lean_dec(x_4); +x_232 = l_Lean_Expr_letE___override(x_188, x_194, x_197, x_221, x_192); +lean_inc(x_232); +x_233 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_222, x_9, x_232); +x_234 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_234, 0, x_232); +lean_ctor_set(x_234, 1, x_233); +return x_234; +} +else +{ +size_t x_235; size_t x_236; uint8_t x_237; +x_235 = lean_ptr_addr(x_191); +lean_dec(x_191); +x_236 = lean_ptr_addr(x_221); +x_237 = lean_usize_dec_eq(x_235, x_236); +if (x_237 == 0) +{ +lean_object* x_238; lean_object* x_239; lean_object* x_240; +lean_dec(x_4); +x_238 = l_Lean_Expr_letE___override(x_188, x_194, x_197, x_221, x_192); +lean_inc(x_238); +x_239 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_222, x_9, x_238); +x_240 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_240, 0, x_238); +lean_ctor_set(x_240, 1, x_239); +return x_240; +} +else +{ +lean_object* x_241; lean_object* x_242; +lean_dec(x_221); +lean_dec(x_197); +lean_dec(x_194); +lean_dec(x_188); +lean_inc(x_4); +x_241 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_222, x_9, x_4); +x_242 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_242, 0, x_4); +lean_ctor_set(x_242, 1, x_241); +return x_242; +} +} +} } } case 9: { -lean_object* x_150; lean_object* x_151; uint8_t x_152; +lean_object* x_243; lean_object* x_244; uint8_t x_245; lean_dec(x_5); lean_dec(x_4); -x_150 = l_Lean_Expr_instantiateBetaRevRange_visit___closed__15; -x_151 = l_panic___at_Lean_Expr_instantiateBetaRevRange_visit___spec__10(x_150, x_6); -x_152 = !lean_is_exclusive(x_151); -if (x_152 == 0) +x_243 = l_Lean_Expr_instantiateBetaRevRange_visit___closed__15; +x_244 = l_panic___at_Lean_Expr_instantiateBetaRevRange_visit___spec__10(x_243, x_6); +x_245 = !lean_is_exclusive(x_244); +if (x_245 == 0) { -lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_153 = lean_ctor_get(x_151, 0); -x_154 = lean_ctor_get(x_151, 1); -lean_inc(x_153); -x_155 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_154, x_9, x_153); -lean_ctor_set(x_151, 1, x_155); -return x_151; +lean_object* x_246; lean_object* x_247; lean_object* x_248; +x_246 = lean_ctor_get(x_244, 0); +x_247 = lean_ctor_get(x_244, 1); +lean_inc(x_246); +x_248 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_247, x_9, x_246); +lean_ctor_set(x_244, 1, x_248); +return x_244; } else { -lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_156 = lean_ctor_get(x_151, 0); -x_157 = lean_ctor_get(x_151, 1); -lean_inc(x_157); -lean_inc(x_156); -lean_dec(x_151); -lean_inc(x_156); -x_158 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_157, x_9, x_156); -x_159 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_159, 0, x_156); -lean_ctor_set(x_159, 1, x_158); -return x_159; +lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; +x_249 = lean_ctor_get(x_244, 0); +x_250 = lean_ctor_get(x_244, 1); +lean_inc(x_250); +lean_inc(x_249); +lean_dec(x_244); +lean_inc(x_249); +x_251 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_250, x_9, x_249); +x_252 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_252, 0, x_249); +lean_ctor_set(x_252, 1, x_251); +return x_252; } } case 10: { -lean_object* x_160; lean_object* x_161; uint8_t x_162; -x_160 = lean_ctor_get(x_4, 1); -lean_inc(x_160); -x_161 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_160, x_5, x_6); -x_162 = !lean_is_exclusive(x_161); -if (x_162 == 0) -{ -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_163 = lean_ctor_get(x_161, 0); -x_164 = lean_ctor_get(x_161, 1); -x_165 = lean_expr_update_mdata(x_4, x_163); -lean_inc(x_165); -x_166 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_164, x_9, x_165); -lean_ctor_set(x_161, 1, x_166); -lean_ctor_set(x_161, 0, x_165); -return x_161; +lean_object* x_253; lean_object* x_254; lean_object* x_255; uint8_t x_256; +x_253 = lean_ctor_get(x_4, 0); +lean_inc(x_253); +x_254 = lean_ctor_get(x_4, 1); +lean_inc(x_254); +lean_inc(x_254); +x_255 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_254, x_5, x_6); +x_256 = !lean_is_exclusive(x_255); +if (x_256 == 0) +{ +lean_object* x_257; lean_object* x_258; size_t x_259; size_t x_260; uint8_t x_261; +x_257 = lean_ctor_get(x_255, 0); +x_258 = lean_ctor_get(x_255, 1); +x_259 = lean_ptr_addr(x_254); +lean_dec(x_254); +x_260 = lean_ptr_addr(x_257); +x_261 = lean_usize_dec_eq(x_259, x_260); +if (x_261 == 0) +{ +lean_object* x_262; lean_object* x_263; +lean_dec(x_4); +x_262 = l_Lean_Expr_mdata___override(x_253, x_257); +lean_inc(x_262); +x_263 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_258, x_9, x_262); +lean_ctor_set(x_255, 1, x_263); +lean_ctor_set(x_255, 0, x_262); +return x_255; +} +else +{ +lean_object* x_264; +lean_dec(x_257); +lean_dec(x_253); +lean_inc(x_4); +x_264 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_258, x_9, x_4); +lean_ctor_set(x_255, 1, x_264); +lean_ctor_set(x_255, 0, x_4); +return x_255; +} } else { -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; -x_167 = lean_ctor_get(x_161, 0); -x_168 = lean_ctor_get(x_161, 1); -lean_inc(x_168); -lean_inc(x_167); -lean_dec(x_161); -x_169 = lean_expr_update_mdata(x_4, x_167); -lean_inc(x_169); -x_170 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_168, x_9, x_169); -x_171 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_171, 0, x_169); -lean_ctor_set(x_171, 1, x_170); -return x_171; +lean_object* x_265; lean_object* x_266; size_t x_267; size_t x_268; uint8_t x_269; +x_265 = lean_ctor_get(x_255, 0); +x_266 = lean_ctor_get(x_255, 1); +lean_inc(x_266); +lean_inc(x_265); +lean_dec(x_255); +x_267 = lean_ptr_addr(x_254); +lean_dec(x_254); +x_268 = lean_ptr_addr(x_265); +x_269 = lean_usize_dec_eq(x_267, x_268); +if (x_269 == 0) +{ +lean_object* x_270; lean_object* x_271; lean_object* x_272; +lean_dec(x_4); +x_270 = l_Lean_Expr_mdata___override(x_253, x_265); +lean_inc(x_270); +x_271 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_266, x_9, x_270); +x_272 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_272, 0, x_270); +lean_ctor_set(x_272, 1, x_271); +return x_272; +} +else +{ +lean_object* x_273; lean_object* x_274; +lean_dec(x_265); +lean_dec(x_253); +lean_inc(x_4); +x_273 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_266, x_9, x_4); +x_274 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_274, 0, x_4); +lean_ctor_set(x_274, 1, x_273); +return x_274; +} } } default: { -lean_object* x_172; lean_object* x_173; uint8_t x_174; -x_172 = lean_ctor_get(x_4, 2); -lean_inc(x_172); -x_173 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_172, x_5, x_6); -x_174 = !lean_is_exclusive(x_173); -if (x_174 == 0) +lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; uint8_t x_279; +x_275 = lean_ctor_get(x_4, 0); +lean_inc(x_275); +x_276 = lean_ctor_get(x_4, 1); +lean_inc(x_276); +x_277 = lean_ctor_get(x_4, 2); +lean_inc(x_277); +lean_inc(x_277); +x_278 = l_Lean_Expr_instantiateBetaRevRange_visit(x_1, x_2, x_3, x_277, x_5, x_6); +x_279 = !lean_is_exclusive(x_278); +if (x_279 == 0) +{ +lean_object* x_280; lean_object* x_281; size_t x_282; size_t x_283; uint8_t x_284; +x_280 = lean_ctor_get(x_278, 0); +x_281 = lean_ctor_get(x_278, 1); +x_282 = lean_ptr_addr(x_277); +lean_dec(x_277); +x_283 = lean_ptr_addr(x_280); +x_284 = lean_usize_dec_eq(x_282, x_283); +if (x_284 == 0) { -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_175 = lean_ctor_get(x_173, 0); -x_176 = lean_ctor_get(x_173, 1); -x_177 = lean_expr_update_proj(x_4, x_175); -lean_inc(x_177); -x_178 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_176, x_9, x_177); -lean_ctor_set(x_173, 1, x_178); -lean_ctor_set(x_173, 0, x_177); -return x_173; +lean_object* x_285; lean_object* x_286; +lean_dec(x_4); +x_285 = l_Lean_Expr_proj___override(x_275, x_276, x_280); +lean_inc(x_285); +x_286 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_281, x_9, x_285); +lean_ctor_set(x_278, 1, x_286); +lean_ctor_set(x_278, 0, x_285); +return x_278; } else { -lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_179 = lean_ctor_get(x_173, 0); -x_180 = lean_ctor_get(x_173, 1); -lean_inc(x_180); -lean_inc(x_179); -lean_dec(x_173); -x_181 = lean_expr_update_proj(x_4, x_179); -lean_inc(x_181); -x_182 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_180, x_9, x_181); -x_183 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_183, 0, x_181); -lean_ctor_set(x_183, 1, x_182); -return x_183; +lean_object* x_287; +lean_dec(x_280); +lean_dec(x_276); +lean_dec(x_275); +lean_inc(x_4); +x_287 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_281, x_9, x_4); +lean_ctor_set(x_278, 1, x_287); +lean_ctor_set(x_278, 0, x_4); +return x_278; +} +} +else +{ +lean_object* x_288; lean_object* x_289; size_t x_290; size_t x_291; uint8_t x_292; +x_288 = lean_ctor_get(x_278, 0); +x_289 = lean_ctor_get(x_278, 1); +lean_inc(x_289); +lean_inc(x_288); +lean_dec(x_278); +x_290 = lean_ptr_addr(x_277); +lean_dec(x_277); +x_291 = lean_ptr_addr(x_288); +x_292 = lean_usize_dec_eq(x_290, x_291); +if (x_292 == 0) +{ +lean_object* x_293; lean_object* x_294; lean_object* x_295; +lean_dec(x_4); +x_293 = l_Lean_Expr_proj___override(x_275, x_276, x_288); +lean_inc(x_293); +x_294 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_289, x_9, x_293); +x_295 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_295, 0, x_293); +lean_ctor_set(x_295, 1, x_294); +return x_295; +} +else +{ +lean_object* x_296; lean_object* x_297; +lean_dec(x_288); +lean_dec(x_276); +lean_dec(x_275); +lean_inc(x_4); +x_296 = l_Std_HashMap_insert___at_Lean_Expr_instantiateBetaRevRange_visit___spec__3(x_289, x_9, x_4); +x_297 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_297, 0, x_4); +lean_ctor_set(x_297, 1, x_296); +return x_297; +} } } } } else { -lean_object* x_184; lean_object* x_185; +lean_object* x_298; lean_object* x_299; lean_dec(x_9); lean_dec(x_5); lean_dec(x_4); -x_184 = lean_ctor_get(x_10, 0); -lean_inc(x_184); +x_298 = lean_ctor_get(x_10, 0); +lean_inc(x_298); lean_dec(x_10); -x_185 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_185, 0, x_184); -lean_ctor_set(x_185, 1, x_6); -return x_185; +x_299 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_299, 0, x_298); +lean_ctor_set(x_299, 1, x_6); +return x_299; } } else { -lean_object* x_186; +lean_object* x_300; lean_dec(x_5); -x_186 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_186, 0, x_4); -lean_ctor_set(x_186, 1, x_6); -return x_186; +x_300 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_300, 0, x_4); +lean_ctor_set(x_300, 1, x_6); +return x_300; } } } @@ -2952,7 +3440,7 @@ lean_dec(x_54); x_57 = lean_ctor_get(x_31, 1); lean_inc(x_57); lean_dec(x_31); -x_58 = l_Lean_Expr_getAppNumArgsAux(x_13, x_34); +x_58 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_13, x_34); x_59 = l___private_Lean_Meta_InferType_0__Lean_Meta_inferProjType___closed__1; lean_inc(x_58); x_60 = lean_mk_array(x_58, x_59); @@ -4031,7 +4519,7 @@ lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -x_20 = lean_level_mk_imax_simp(x_18, x_4); +x_20 = l_Lean_mkLevelIMax_x27(x_18, x_4); x_2 = x_12; x_4 = x_20; x_9 = x_19; @@ -7438,7 +7926,7 @@ lean_inc(x_170); x_171 = l_Lean_Expr_getAppFn(x_170); lean_dec(x_170); x_172 = lean_unsigned_to_nat(0u); -x_173 = l_Lean_Expr_getAppNumArgsAux(x_1, x_172); +x_173 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_172); x_174 = l___private_Lean_Meta_InferType_0__Lean_Meta_inferProjType___closed__1; lean_inc(x_173); x_175 = lean_mk_array(x_173, x_174); diff --git a/stage0/stdlib/Lean/Meta/Injective.c b/stage0/stdlib/Lean/Meta/Injective.c index 28c118fc80a4..b6e009775bae 100644 --- a/stage0/stdlib/Lean/Meta/Injective.c +++ b/stage0/stdlib/Lean/Meta/Injective.c @@ -95,6 +95,7 @@ lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheoremTypeCore_x3f_mkArgs2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheoremTypeCore_x3f_mkArgs2___closed__3; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Injective_0__Lean_Meta_throwInjectiveTheoremFailure___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveTheoremTypeCore_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Injective_0__Lean_Meta_injTheoremFailureHeader___closed__2; @@ -133,7 +134,6 @@ static lean_object* l___private_Lean_Meta_Injective_0__Lean_Meta_mkInjectiveEqTh lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_Meta_substEqs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Std_Format_initFn____x40_Lean_Data_Format___hyg_57____spec__1(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Meta_assumptionCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Injective___hyg_1685_(lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -324,7 +324,7 @@ else { lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_1, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_10); x_12 = lean_nat_sub(x_11, x_10); lean_dec(x_11); x_13 = lean_unsigned_to_nat(1u); diff --git a/stage0/stdlib/Lean/Meta/Instances.c b/stage0/stdlib/Lean/Meta/Instances.c index ed81d1b5ff71..ac74b1b632aa 100644 --- a/stage0/stdlib/Lean/Meta/Instances.c +++ b/stage0/stdlib/Lean/Meta/Instances.c @@ -1804,7 +1804,7 @@ static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addIns lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addInstanceEntry___spec__1___closed__1; x_2 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addInstanceEntry___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addInstanceEntry___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/KAbstract.c b/stage0/stdlib/Lean/Meta/KAbstract.c index a12eed066a29..17f41c331de9 100644 --- a/stage0/stdlib/Lean/Meta/KAbstract.c +++ b/stage0/stdlib/Lean/Meta/KAbstract.c @@ -13,19 +13,21 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* lean_mk_empty_array_with_capacity(lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); +uint8_t lean_usize_dec_eq(size_t, size_t); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); lean_object* lean_nat_add(lean_object*, lean_object*); uint8_t l_Lean_Occurrences_contains(lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_kabstract_visit___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* l_Lean_Expr_toHeadIndex(lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); +size_t lean_ptr_addr(lean_object*); lean_object* l___private_Lean_HeadIndex_0__Lean_Expr_headNumArgsAux(lean_object*, lean_object*); uint8_t l___private_Lean_HeadIndex_0__Lean_beqHeadIndex____x40_Lean_HeadIndex___hyg_66_(lean_object*, lean_object*); uint8_t l___private_Lean_Data_Occurrences_0__Lean_beqOccurrences____x40_Lean_Data_Occurrences___hyg_32_(lean_object*, lean_object*); @@ -33,150 +35,227 @@ LEAN_EXPORT lean_object* l_Lean_Meta_kabstract_visit(lean_object*, lean_object*, lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isFVar(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); lean_object* lean_expr_abstract(lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_app(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_kabstract(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_kabstract___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_kabstract___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_kabstract_visit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_13; uint8_t x_142; -x_142 = l_Lean_Expr_hasLooseBVars(x_5); -if (x_142 == 0) +lean_object* x_13; uint8_t x_250; +x_250 = l_Lean_Expr_hasLooseBVars(x_5); +if (x_250 == 0) { -lean_object* x_143; uint8_t x_144; +lean_object* x_251; uint8_t x_252; lean_inc(x_5); -x_143 = l_Lean_Expr_toHeadIndex(x_5); -x_144 = l___private_Lean_HeadIndex_0__Lean_beqHeadIndex____x40_Lean_HeadIndex___hyg_66_(x_143, x_3); -lean_dec(x_143); -if (x_144 == 0) +x_251 = l_Lean_Expr_toHeadIndex(x_5); +x_252 = l___private_Lean_HeadIndex_0__Lean_beqHeadIndex____x40_Lean_HeadIndex___hyg_66_(x_251, x_3); +lean_dec(x_251); +if (x_252 == 0) { -lean_object* x_145; -x_145 = lean_box(0); -x_13 = x_145; -goto block_141; +lean_object* x_253; +x_253 = lean_box(0); +x_13 = x_253; +goto block_249; } else { -lean_object* x_146; lean_object* x_147; uint8_t x_148; -x_146 = lean_unsigned_to_nat(0u); -x_147 = l___private_Lean_HeadIndex_0__Lean_Expr_headNumArgsAux(x_5, x_146); -x_148 = lean_nat_dec_eq(x_147, x_4); -lean_dec(x_147); -if (x_148 == 0) +lean_object* x_254; lean_object* x_255; uint8_t x_256; +x_254 = lean_unsigned_to_nat(0u); +x_255 = l___private_Lean_HeadIndex_0__Lean_Expr_headNumArgsAux(x_5, x_254); +x_256 = lean_nat_dec_eq(x_255, x_4); +lean_dec(x_255); +if (x_256 == 0) { -lean_object* x_149; -x_149 = lean_box(0); -x_13 = x_149; -goto block_141; +lean_object* x_257; +x_257 = lean_box(0); +x_13 = x_257; +goto block_249; } else { -lean_object* x_150; +lean_object* x_258; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_1); lean_inc(x_5); -x_150 = l_Lean_Meta_isExprDefEq(x_5, x_1, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_150) == 0) +x_258 = l_Lean_Meta_isExprDefEq(x_5, x_1, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_258) == 0) { -lean_object* x_151; uint8_t x_152; -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -x_152 = lean_unbox(x_151); -lean_dec(x_151); -if (x_152 == 0) +lean_object* x_259; uint8_t x_260; +x_259 = lean_ctor_get(x_258, 0); +lean_inc(x_259); +x_260 = lean_unbox(x_259); +lean_dec(x_259); +if (x_260 == 0) { switch (lean_obj_tag(x_5)) { case 5: { -lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_153 = lean_ctor_get(x_150, 1); -lean_inc(x_153); -lean_dec(x_150); -x_154 = lean_ctor_get(x_5, 0); -lean_inc(x_154); -x_155 = lean_ctor_get(x_5, 1); -lean_inc(x_155); +lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; +x_261 = lean_ctor_get(x_258, 1); +lean_inc(x_261); +lean_dec(x_258); +x_262 = lean_ctor_get(x_5, 0); +lean_inc(x_262); +x_263 = lean_ctor_get(x_5, 1); +lean_inc(x_263); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_262); lean_inc(x_1); -x_156 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_154, x_6, x_7, x_8, x_9, x_10, x_11, x_153); -if (lean_obj_tag(x_156) == 0) +x_264 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_262, x_6, x_7, x_8, x_9, x_10, x_11, x_261); +if (lean_obj_tag(x_264) == 0) +{ +lean_object* x_265; lean_object* x_266; lean_object* x_267; +x_265 = lean_ctor_get(x_264, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_264, 1); +lean_inc(x_266); +lean_dec(x_264); +lean_inc(x_263); +x_267 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_263, x_6, x_7, x_8, x_9, x_10, x_11, x_266); +if (lean_obj_tag(x_267) == 0) +{ +uint8_t x_268; +x_268 = !lean_is_exclusive(x_267); +if (x_268 == 0) +{ +lean_object* x_269; size_t x_270; size_t x_271; uint8_t x_272; +x_269 = lean_ctor_get(x_267, 0); +x_270 = lean_ptr_addr(x_262); +lean_dec(x_262); +x_271 = lean_ptr_addr(x_265); +x_272 = lean_usize_dec_eq(x_270, x_271); +if (x_272 == 0) +{ +lean_object* x_273; +lean_dec(x_263); +lean_dec(x_5); +x_273 = l_Lean_Expr_app___override(x_265, x_269); +lean_ctor_set(x_267, 0, x_273); +return x_267; +} +else { -lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_157 = lean_ctor_get(x_156, 0); -lean_inc(x_157); -x_158 = lean_ctor_get(x_156, 1); -lean_inc(x_158); -lean_dec(x_156); -x_159 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_155, x_6, x_7, x_8, x_9, x_10, x_11, x_158); -if (lean_obj_tag(x_159) == 0) +size_t x_274; size_t x_275; uint8_t x_276; +x_274 = lean_ptr_addr(x_263); +lean_dec(x_263); +x_275 = lean_ptr_addr(x_269); +x_276 = lean_usize_dec_eq(x_274, x_275); +if (x_276 == 0) { -uint8_t x_160; -x_160 = !lean_is_exclusive(x_159); -if (x_160 == 0) +lean_object* x_277; +lean_dec(x_5); +x_277 = l_Lean_Expr_app___override(x_265, x_269); +lean_ctor_set(x_267, 0, x_277); +return x_267; +} +else { -lean_object* x_161; lean_object* x_162; -x_161 = lean_ctor_get(x_159, 0); -x_162 = lean_expr_update_app(x_5, x_157, x_161); -lean_ctor_set(x_159, 0, x_162); -return x_159; +lean_dec(x_269); +lean_dec(x_265); +lean_ctor_set(x_267, 0, x_5); +return x_267; +} +} } else { -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_163 = lean_ctor_get(x_159, 0); -x_164 = lean_ctor_get(x_159, 1); -lean_inc(x_164); -lean_inc(x_163); -lean_dec(x_159); -x_165 = lean_expr_update_app(x_5, x_157, x_163); -x_166 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_166, 0, x_165); -lean_ctor_set(x_166, 1, x_164); -return x_166; +lean_object* x_278; lean_object* x_279; size_t x_280; size_t x_281; uint8_t x_282; +x_278 = lean_ctor_get(x_267, 0); +x_279 = lean_ctor_get(x_267, 1); +lean_inc(x_279); +lean_inc(x_278); +lean_dec(x_267); +x_280 = lean_ptr_addr(x_262); +lean_dec(x_262); +x_281 = lean_ptr_addr(x_265); +x_282 = lean_usize_dec_eq(x_280, x_281); +if (x_282 == 0) +{ +lean_object* x_283; lean_object* x_284; +lean_dec(x_263); +lean_dec(x_5); +x_283 = l_Lean_Expr_app___override(x_265, x_278); +x_284 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_284, 0, x_283); +lean_ctor_set(x_284, 1, x_279); +return x_284; } +else +{ +size_t x_285; size_t x_286; uint8_t x_287; +x_285 = lean_ptr_addr(x_263); +lean_dec(x_263); +x_286 = lean_ptr_addr(x_278); +x_287 = lean_usize_dec_eq(x_285, x_286); +if (x_287 == 0) +{ +lean_object* x_288; lean_object* x_289; +lean_dec(x_5); +x_288 = l_Lean_Expr_app___override(x_265, x_278); +x_289 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_289, 0, x_288); +lean_ctor_set(x_289, 1, x_279); +return x_289; } else { -uint8_t x_167; -lean_dec(x_157); +lean_object* x_290; +lean_dec(x_278); +lean_dec(x_265); +x_290 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_290, 0, x_5); +lean_ctor_set(x_290, 1, x_279); +return x_290; +} +} +} +} +else +{ +uint8_t x_291; +lean_dec(x_265); +lean_dec(x_263); +lean_dec(x_262); lean_dec(x_5); -x_167 = !lean_is_exclusive(x_159); -if (x_167 == 0) +x_291 = !lean_is_exclusive(x_267); +if (x_291 == 0) { -return x_159; +return x_267; } else { -lean_object* x_168; lean_object* x_169; lean_object* x_170; -x_168 = lean_ctor_get(x_159, 0); -x_169 = lean_ctor_get(x_159, 1); -lean_inc(x_169); -lean_inc(x_168); -lean_dec(x_159); -x_170 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_170, 0, x_168); -lean_ctor_set(x_170, 1, x_169); -return x_170; +lean_object* x_292; lean_object* x_293; lean_object* x_294; +x_292 = lean_ctor_get(x_267, 0); +x_293 = lean_ctor_get(x_267, 1); +lean_inc(x_293); +lean_inc(x_292); +lean_dec(x_267); +x_294 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_294, 0, x_292); +lean_ctor_set(x_294, 1, x_293); +return x_294; } } } else { -uint8_t x_171; -lean_dec(x_155); +uint8_t x_295; +lean_dec(x_263); +lean_dec(x_262); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -184,356 +263,716 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_171 = !lean_is_exclusive(x_156); -if (x_171 == 0) +x_295 = !lean_is_exclusive(x_264); +if (x_295 == 0) { -return x_156; +return x_264; } else { -lean_object* x_172; lean_object* x_173; lean_object* x_174; -x_172 = lean_ctor_get(x_156, 0); -x_173 = lean_ctor_get(x_156, 1); -lean_inc(x_173); -lean_inc(x_172); -lean_dec(x_156); -x_174 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_174, 0, x_172); -lean_ctor_set(x_174, 1, x_173); -return x_174; +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_264, 0); +x_297 = lean_ctor_get(x_264, 1); +lean_inc(x_297); +lean_inc(x_296); +lean_dec(x_264); +x_298 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_298, 0, x_296); +lean_ctor_set(x_298, 1, x_297); +return x_298; } } } case 6: { -lean_object* x_175; lean_object* x_176; lean_object* x_177; uint8_t x_178; lean_object* x_179; -x_175 = lean_ctor_get(x_150, 1); -lean_inc(x_175); -lean_dec(x_150); -x_176 = lean_ctor_get(x_5, 1); -lean_inc(x_176); -x_177 = lean_ctor_get(x_5, 2); -lean_inc(x_177); -x_178 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; uint8_t x_303; lean_object* x_304; +x_299 = lean_ctor_get(x_258, 1); +lean_inc(x_299); +lean_dec(x_258); +x_300 = lean_ctor_get(x_5, 0); +lean_inc(x_300); +x_301 = lean_ctor_get(x_5, 1); +lean_inc(x_301); +x_302 = lean_ctor_get(x_5, 2); +lean_inc(x_302); +x_303 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_301); lean_inc(x_1); -x_179 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_176, x_6, x_7, x_8, x_9, x_10, x_11, x_175); -if (lean_obj_tag(x_179) == 0) -{ -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; -x_180 = lean_ctor_get(x_179, 0); -lean_inc(x_180); -x_181 = lean_ctor_get(x_179, 1); -lean_inc(x_181); -lean_dec(x_179); -x_182 = lean_unsigned_to_nat(1u); -x_183 = lean_nat_add(x_6, x_182); +x_304 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_301, x_6, x_7, x_8, x_9, x_10, x_11, x_299); +if (lean_obj_tag(x_304) == 0) +{ +lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; +x_305 = lean_ctor_get(x_304, 0); +lean_inc(x_305); +x_306 = lean_ctor_get(x_304, 1); +lean_inc(x_306); +lean_dec(x_304); +x_307 = lean_unsigned_to_nat(1u); +x_308 = lean_nat_add(x_6, x_307); lean_dec(x_6); -x_184 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_177, x_183, x_7, x_8, x_9, x_10, x_11, x_181); -if (lean_obj_tag(x_184) == 0) +lean_inc(x_302); +x_309 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_302, x_308, x_7, x_8, x_9, x_10, x_11, x_306); +if (lean_obj_tag(x_309) == 0) { -uint8_t x_185; -x_185 = !lean_is_exclusive(x_184); -if (x_185 == 0) +uint8_t x_310; +x_310 = !lean_is_exclusive(x_309); +if (x_310 == 0) { -lean_object* x_186; lean_object* x_187; -x_186 = lean_ctor_get(x_184, 0); -x_187 = lean_expr_update_lambda(x_5, x_178, x_180, x_186); -lean_ctor_set(x_184, 0, x_187); -return x_184; +lean_object* x_311; lean_object* x_312; size_t x_313; size_t x_314; uint8_t x_315; +x_311 = lean_ctor_get(x_309, 0); +lean_inc(x_302); +lean_inc(x_301); +lean_inc(x_300); +x_312 = l_Lean_Expr_lam___override(x_300, x_301, x_302, x_303); +x_313 = lean_ptr_addr(x_301); +lean_dec(x_301); +x_314 = lean_ptr_addr(x_305); +x_315 = lean_usize_dec_eq(x_313, x_314); +if (x_315 == 0) +{ +lean_object* x_316; +lean_dec(x_312); +lean_dec(x_302); +x_316 = l_Lean_Expr_lam___override(x_300, x_305, x_311, x_303); +lean_ctor_set(x_309, 0, x_316); +return x_309; } else { -lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_188 = lean_ctor_get(x_184, 0); -x_189 = lean_ctor_get(x_184, 1); -lean_inc(x_189); -lean_inc(x_188); -lean_dec(x_184); -x_190 = lean_expr_update_lambda(x_5, x_178, x_180, x_188); -x_191 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_191, 0, x_190); -lean_ctor_set(x_191, 1, x_189); -return x_191; +size_t x_317; size_t x_318; uint8_t x_319; +x_317 = lean_ptr_addr(x_302); +lean_dec(x_302); +x_318 = lean_ptr_addr(x_311); +x_319 = lean_usize_dec_eq(x_317, x_318); +if (x_319 == 0) +{ +lean_object* x_320; +lean_dec(x_312); +x_320 = l_Lean_Expr_lam___override(x_300, x_305, x_311, x_303); +lean_ctor_set(x_309, 0, x_320); +return x_309; } +else +{ +uint8_t x_321; +x_321 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_303, x_303); +if (x_321 == 0) +{ +lean_object* x_322; +lean_dec(x_312); +x_322 = l_Lean_Expr_lam___override(x_300, x_305, x_311, x_303); +lean_ctor_set(x_309, 0, x_322); +return x_309; } else { -uint8_t x_192; -lean_dec(x_180); -lean_dec(x_5); -x_192 = !lean_is_exclusive(x_184); -if (x_192 == 0) +lean_dec(x_311); +lean_dec(x_305); +lean_dec(x_300); +lean_ctor_set(x_309, 0, x_312); +return x_309; +} +} +} +} +else { -return x_184; +lean_object* x_323; lean_object* x_324; lean_object* x_325; size_t x_326; size_t x_327; uint8_t x_328; +x_323 = lean_ctor_get(x_309, 0); +x_324 = lean_ctor_get(x_309, 1); +lean_inc(x_324); +lean_inc(x_323); +lean_dec(x_309); +lean_inc(x_302); +lean_inc(x_301); +lean_inc(x_300); +x_325 = l_Lean_Expr_lam___override(x_300, x_301, x_302, x_303); +x_326 = lean_ptr_addr(x_301); +lean_dec(x_301); +x_327 = lean_ptr_addr(x_305); +x_328 = lean_usize_dec_eq(x_326, x_327); +if (x_328 == 0) +{ +lean_object* x_329; lean_object* x_330; +lean_dec(x_325); +lean_dec(x_302); +x_329 = l_Lean_Expr_lam___override(x_300, x_305, x_323, x_303); +x_330 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_330, 0, x_329); +lean_ctor_set(x_330, 1, x_324); +return x_330; } else { -lean_object* x_193; lean_object* x_194; lean_object* x_195; -x_193 = lean_ctor_get(x_184, 0); -x_194 = lean_ctor_get(x_184, 1); -lean_inc(x_194); -lean_inc(x_193); -lean_dec(x_184); -x_195 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_195, 0, x_193); -lean_ctor_set(x_195, 1, x_194); -return x_195; +size_t x_331; size_t x_332; uint8_t x_333; +x_331 = lean_ptr_addr(x_302); +lean_dec(x_302); +x_332 = lean_ptr_addr(x_323); +x_333 = lean_usize_dec_eq(x_331, x_332); +if (x_333 == 0) +{ +lean_object* x_334; lean_object* x_335; +lean_dec(x_325); +x_334 = l_Lean_Expr_lam___override(x_300, x_305, x_323, x_303); +x_335 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_335, 0, x_334); +lean_ctor_set(x_335, 1, x_324); +return x_335; +} +else +{ +uint8_t x_336; +x_336 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_303, x_303); +if (x_336 == 0) +{ +lean_object* x_337; lean_object* x_338; +lean_dec(x_325); +x_337 = l_Lean_Expr_lam___override(x_300, x_305, x_323, x_303); +x_338 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_338, 0, x_337); +lean_ctor_set(x_338, 1, x_324); +return x_338; +} +else +{ +lean_object* x_339; +lean_dec(x_323); +lean_dec(x_305); +lean_dec(x_300); +x_339 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_339, 0, x_325); +lean_ctor_set(x_339, 1, x_324); +return x_339; +} +} +} +} +} +else +{ +uint8_t x_340; +lean_dec(x_305); +lean_dec(x_302); +lean_dec(x_301); +lean_dec(x_300); +x_340 = !lean_is_exclusive(x_309); +if (x_340 == 0) +{ +return x_309; +} +else +{ +lean_object* x_341; lean_object* x_342; lean_object* x_343; +x_341 = lean_ctor_get(x_309, 0); +x_342 = lean_ctor_get(x_309, 1); +lean_inc(x_342); +lean_inc(x_341); +lean_dec(x_309); +x_343 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_343, 0, x_341); +lean_ctor_set(x_343, 1, x_342); +return x_343; } } } else { -uint8_t x_196; -lean_dec(x_177); +uint8_t x_344; +lean_dec(x_302); +lean_dec(x_301); +lean_dec(x_300); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_196 = !lean_is_exclusive(x_179); -if (x_196 == 0) +x_344 = !lean_is_exclusive(x_304); +if (x_344 == 0) { -return x_179; +return x_304; } else { -lean_object* x_197; lean_object* x_198; lean_object* x_199; -x_197 = lean_ctor_get(x_179, 0); -x_198 = lean_ctor_get(x_179, 1); -lean_inc(x_198); -lean_inc(x_197); -lean_dec(x_179); -x_199 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_199, 0, x_197); -lean_ctor_set(x_199, 1, x_198); -return x_199; +lean_object* x_345; lean_object* x_346; lean_object* x_347; +x_345 = lean_ctor_get(x_304, 0); +x_346 = lean_ctor_get(x_304, 1); +lean_inc(x_346); +lean_inc(x_345); +lean_dec(x_304); +x_347 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_347, 0, x_345); +lean_ctor_set(x_347, 1, x_346); +return x_347; } } } case 7: { -lean_object* x_200; lean_object* x_201; lean_object* x_202; uint8_t x_203; lean_object* x_204; -x_200 = lean_ctor_get(x_150, 1); -lean_inc(x_200); -lean_dec(x_150); -x_201 = lean_ctor_get(x_5, 1); -lean_inc(x_201); -x_202 = lean_ctor_get(x_5, 2); -lean_inc(x_202); -x_203 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; uint8_t x_352; lean_object* x_353; +x_348 = lean_ctor_get(x_258, 1); +lean_inc(x_348); +lean_dec(x_258); +x_349 = lean_ctor_get(x_5, 0); +lean_inc(x_349); +x_350 = lean_ctor_get(x_5, 1); +lean_inc(x_350); +x_351 = lean_ctor_get(x_5, 2); +lean_inc(x_351); +x_352 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_350); lean_inc(x_1); -x_204 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_201, x_6, x_7, x_8, x_9, x_10, x_11, x_200); -if (lean_obj_tag(x_204) == 0) -{ -lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; -x_205 = lean_ctor_get(x_204, 0); -lean_inc(x_205); -x_206 = lean_ctor_get(x_204, 1); -lean_inc(x_206); -lean_dec(x_204); -x_207 = lean_unsigned_to_nat(1u); -x_208 = lean_nat_add(x_6, x_207); +x_353 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_350, x_6, x_7, x_8, x_9, x_10, x_11, x_348); +if (lean_obj_tag(x_353) == 0) +{ +lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; +x_354 = lean_ctor_get(x_353, 0); +lean_inc(x_354); +x_355 = lean_ctor_get(x_353, 1); +lean_inc(x_355); +lean_dec(x_353); +x_356 = lean_unsigned_to_nat(1u); +x_357 = lean_nat_add(x_6, x_356); lean_dec(x_6); -x_209 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_202, x_208, x_7, x_8, x_9, x_10, x_11, x_206); -if (lean_obj_tag(x_209) == 0) +lean_inc(x_351); +x_358 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_351, x_357, x_7, x_8, x_9, x_10, x_11, x_355); +if (lean_obj_tag(x_358) == 0) +{ +uint8_t x_359; +x_359 = !lean_is_exclusive(x_358); +if (x_359 == 0) +{ +lean_object* x_360; lean_object* x_361; size_t x_362; size_t x_363; uint8_t x_364; +x_360 = lean_ctor_get(x_358, 0); +lean_inc(x_351); +lean_inc(x_350); +lean_inc(x_349); +x_361 = l_Lean_Expr_forallE___override(x_349, x_350, x_351, x_352); +x_362 = lean_ptr_addr(x_350); +lean_dec(x_350); +x_363 = lean_ptr_addr(x_354); +x_364 = lean_usize_dec_eq(x_362, x_363); +if (x_364 == 0) +{ +lean_object* x_365; +lean_dec(x_361); +lean_dec(x_351); +x_365 = l_Lean_Expr_forallE___override(x_349, x_354, x_360, x_352); +lean_ctor_set(x_358, 0, x_365); +return x_358; +} +else { -uint8_t x_210; -x_210 = !lean_is_exclusive(x_209); -if (x_210 == 0) +size_t x_366; size_t x_367; uint8_t x_368; +x_366 = lean_ptr_addr(x_351); +lean_dec(x_351); +x_367 = lean_ptr_addr(x_360); +x_368 = lean_usize_dec_eq(x_366, x_367); +if (x_368 == 0) { -lean_object* x_211; lean_object* x_212; -x_211 = lean_ctor_get(x_209, 0); -x_212 = lean_expr_update_forall(x_5, x_203, x_205, x_211); -lean_ctor_set(x_209, 0, x_212); -return x_209; +lean_object* x_369; +lean_dec(x_361); +x_369 = l_Lean_Expr_forallE___override(x_349, x_354, x_360, x_352); +lean_ctor_set(x_358, 0, x_369); +return x_358; } else { -lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; -x_213 = lean_ctor_get(x_209, 0); -x_214 = lean_ctor_get(x_209, 1); -lean_inc(x_214); -lean_inc(x_213); -lean_dec(x_209); -x_215 = lean_expr_update_forall(x_5, x_203, x_205, x_213); -x_216 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_216, 0, x_215); -lean_ctor_set(x_216, 1, x_214); -return x_216; +uint8_t x_370; +x_370 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_352, x_352); +if (x_370 == 0) +{ +lean_object* x_371; +lean_dec(x_361); +x_371 = l_Lean_Expr_forallE___override(x_349, x_354, x_360, x_352); +lean_ctor_set(x_358, 0, x_371); +return x_358; +} +else +{ +lean_dec(x_360); +lean_dec(x_354); +lean_dec(x_349); +lean_ctor_set(x_358, 0, x_361); +return x_358; +} +} } } else { -uint8_t x_217; -lean_dec(x_205); -lean_dec(x_5); -x_217 = !lean_is_exclusive(x_209); -if (x_217 == 0) +lean_object* x_372; lean_object* x_373; lean_object* x_374; size_t x_375; size_t x_376; uint8_t x_377; +x_372 = lean_ctor_get(x_358, 0); +x_373 = lean_ctor_get(x_358, 1); +lean_inc(x_373); +lean_inc(x_372); +lean_dec(x_358); +lean_inc(x_351); +lean_inc(x_350); +lean_inc(x_349); +x_374 = l_Lean_Expr_forallE___override(x_349, x_350, x_351, x_352); +x_375 = lean_ptr_addr(x_350); +lean_dec(x_350); +x_376 = lean_ptr_addr(x_354); +x_377 = lean_usize_dec_eq(x_375, x_376); +if (x_377 == 0) +{ +lean_object* x_378; lean_object* x_379; +lean_dec(x_374); +lean_dec(x_351); +x_378 = l_Lean_Expr_forallE___override(x_349, x_354, x_372, x_352); +x_379 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_379, 0, x_378); +lean_ctor_set(x_379, 1, x_373); +return x_379; +} +else +{ +size_t x_380; size_t x_381; uint8_t x_382; +x_380 = lean_ptr_addr(x_351); +lean_dec(x_351); +x_381 = lean_ptr_addr(x_372); +x_382 = lean_usize_dec_eq(x_380, x_381); +if (x_382 == 0) { -return x_209; +lean_object* x_383; lean_object* x_384; +lean_dec(x_374); +x_383 = l_Lean_Expr_forallE___override(x_349, x_354, x_372, x_352); +x_384 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_384, 0, x_383); +lean_ctor_set(x_384, 1, x_373); +return x_384; } else { -lean_object* x_218; lean_object* x_219; lean_object* x_220; -x_218 = lean_ctor_get(x_209, 0); -x_219 = lean_ctor_get(x_209, 1); -lean_inc(x_219); -lean_inc(x_218); -lean_dec(x_209); -x_220 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_220, 0, x_218); -lean_ctor_set(x_220, 1, x_219); -return x_220; +uint8_t x_385; +x_385 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_352, x_352); +if (x_385 == 0) +{ +lean_object* x_386; lean_object* x_387; +lean_dec(x_374); +x_386 = l_Lean_Expr_forallE___override(x_349, x_354, x_372, x_352); +x_387 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_387, 0, x_386); +lean_ctor_set(x_387, 1, x_373); +return x_387; +} +else +{ +lean_object* x_388; +lean_dec(x_372); +lean_dec(x_354); +lean_dec(x_349); +x_388 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_388, 0, x_374); +lean_ctor_set(x_388, 1, x_373); +return x_388; +} +} } } } else { -uint8_t x_221; -lean_dec(x_202); +uint8_t x_389; +lean_dec(x_354); +lean_dec(x_351); +lean_dec(x_350); +lean_dec(x_349); +x_389 = !lean_is_exclusive(x_358); +if (x_389 == 0) +{ +return x_358; +} +else +{ +lean_object* x_390; lean_object* x_391; lean_object* x_392; +x_390 = lean_ctor_get(x_358, 0); +x_391 = lean_ctor_get(x_358, 1); +lean_inc(x_391); +lean_inc(x_390); +lean_dec(x_358); +x_392 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_392, 0, x_390); +lean_ctor_set(x_392, 1, x_391); +return x_392; +} +} +} +else +{ +uint8_t x_393; +lean_dec(x_351); +lean_dec(x_350); +lean_dec(x_349); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_221 = !lean_is_exclusive(x_204); -if (x_221 == 0) +x_393 = !lean_is_exclusive(x_353); +if (x_393 == 0) { -return x_204; +return x_353; } else { -lean_object* x_222; lean_object* x_223; lean_object* x_224; -x_222 = lean_ctor_get(x_204, 0); -x_223 = lean_ctor_get(x_204, 1); -lean_inc(x_223); -lean_inc(x_222); -lean_dec(x_204); -x_224 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_224, 0, x_222); -lean_ctor_set(x_224, 1, x_223); -return x_224; +lean_object* x_394; lean_object* x_395; lean_object* x_396; +x_394 = lean_ctor_get(x_353, 0); +x_395 = lean_ctor_get(x_353, 1); +lean_inc(x_395); +lean_inc(x_394); +lean_dec(x_353); +x_396 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_396, 0, x_394); +lean_ctor_set(x_396, 1, x_395); +return x_396; } } } case 8: { -lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; -x_225 = lean_ctor_get(x_150, 1); -lean_inc(x_225); -lean_dec(x_150); -x_226 = lean_ctor_get(x_5, 1); -lean_inc(x_226); -x_227 = lean_ctor_get(x_5, 2); -lean_inc(x_227); -x_228 = lean_ctor_get(x_5, 3); -lean_inc(x_228); +lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; uint8_t x_402; lean_object* x_403; +x_397 = lean_ctor_get(x_258, 1); +lean_inc(x_397); +lean_dec(x_258); +x_398 = lean_ctor_get(x_5, 0); +lean_inc(x_398); +x_399 = lean_ctor_get(x_5, 1); +lean_inc(x_399); +x_400 = lean_ctor_get(x_5, 2); +lean_inc(x_400); +x_401 = lean_ctor_get(x_5, 3); +lean_inc(x_401); +x_402 = lean_ctor_get_uint8(x_5, sizeof(void*)*4 + 8); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_399); lean_inc(x_1); -x_229 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_226, x_6, x_7, x_8, x_9, x_10, x_11, x_225); -if (lean_obj_tag(x_229) == 0) -{ -lean_object* x_230; lean_object* x_231; lean_object* x_232; -x_230 = lean_ctor_get(x_229, 0); -lean_inc(x_230); -x_231 = lean_ctor_get(x_229, 1); -lean_inc(x_231); -lean_dec(x_229); +x_403 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_399, x_6, x_7, x_8, x_9, x_10, x_11, x_397); +if (lean_obj_tag(x_403) == 0) +{ +lean_object* x_404; lean_object* x_405; lean_object* x_406; +x_404 = lean_ctor_get(x_403, 0); +lean_inc(x_404); +x_405 = lean_ctor_get(x_403, 1); +lean_inc(x_405); +lean_dec(x_403); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_400); lean_inc(x_1); -x_232 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_227, x_6, x_7, x_8, x_9, x_10, x_11, x_231); -if (lean_obj_tag(x_232) == 0) -{ -lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; -x_233 = lean_ctor_get(x_232, 0); -lean_inc(x_233); -x_234 = lean_ctor_get(x_232, 1); -lean_inc(x_234); -lean_dec(x_232); -x_235 = lean_unsigned_to_nat(1u); -x_236 = lean_nat_add(x_6, x_235); +x_406 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_400, x_6, x_7, x_8, x_9, x_10, x_11, x_405); +if (lean_obj_tag(x_406) == 0) +{ +lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; +x_407 = lean_ctor_get(x_406, 0); +lean_inc(x_407); +x_408 = lean_ctor_get(x_406, 1); +lean_inc(x_408); +lean_dec(x_406); +x_409 = lean_unsigned_to_nat(1u); +x_410 = lean_nat_add(x_6, x_409); lean_dec(x_6); -x_237 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_228, x_236, x_7, x_8, x_9, x_10, x_11, x_234); -if (lean_obj_tag(x_237) == 0) +lean_inc(x_401); +x_411 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_401, x_410, x_7, x_8, x_9, x_10, x_11, x_408); +if (lean_obj_tag(x_411) == 0) +{ +uint8_t x_412; +x_412 = !lean_is_exclusive(x_411); +if (x_412 == 0) +{ +lean_object* x_413; size_t x_414; size_t x_415; uint8_t x_416; +x_413 = lean_ctor_get(x_411, 0); +x_414 = lean_ptr_addr(x_399); +lean_dec(x_399); +x_415 = lean_ptr_addr(x_404); +x_416 = lean_usize_dec_eq(x_414, x_415); +if (x_416 == 0) +{ +lean_object* x_417; +lean_dec(x_401); +lean_dec(x_400); +lean_dec(x_5); +x_417 = l_Lean_Expr_letE___override(x_398, x_404, x_407, x_413, x_402); +lean_ctor_set(x_411, 0, x_417); +return x_411; +} +else { -uint8_t x_238; -x_238 = !lean_is_exclusive(x_237); -if (x_238 == 0) +size_t x_418; size_t x_419; uint8_t x_420; +x_418 = lean_ptr_addr(x_400); +lean_dec(x_400); +x_419 = lean_ptr_addr(x_407); +x_420 = lean_usize_dec_eq(x_418, x_419); +if (x_420 == 0) { -lean_object* x_239; lean_object* x_240; -x_239 = lean_ctor_get(x_237, 0); -x_240 = lean_expr_update_let(x_5, x_230, x_233, x_239); -lean_ctor_set(x_237, 0, x_240); -return x_237; +lean_object* x_421; +lean_dec(x_401); +lean_dec(x_5); +x_421 = l_Lean_Expr_letE___override(x_398, x_404, x_407, x_413, x_402); +lean_ctor_set(x_411, 0, x_421); +return x_411; } else { -lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; -x_241 = lean_ctor_get(x_237, 0); -x_242 = lean_ctor_get(x_237, 1); -lean_inc(x_242); -lean_inc(x_241); -lean_dec(x_237); -x_243 = lean_expr_update_let(x_5, x_230, x_233, x_241); -x_244 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_244, 0, x_243); -lean_ctor_set(x_244, 1, x_242); -return x_244; +size_t x_422; size_t x_423; uint8_t x_424; +x_422 = lean_ptr_addr(x_401); +lean_dec(x_401); +x_423 = lean_ptr_addr(x_413); +x_424 = lean_usize_dec_eq(x_422, x_423); +if (x_424 == 0) +{ +lean_object* x_425; +lean_dec(x_5); +x_425 = l_Lean_Expr_letE___override(x_398, x_404, x_407, x_413, x_402); +lean_ctor_set(x_411, 0, x_425); +return x_411; +} +else +{ +lean_dec(x_413); +lean_dec(x_407); +lean_dec(x_404); +lean_dec(x_398); +lean_ctor_set(x_411, 0, x_5); +return x_411; +} +} } } else { -uint8_t x_245; -lean_dec(x_233); -lean_dec(x_230); +lean_object* x_426; lean_object* x_427; size_t x_428; size_t x_429; uint8_t x_430; +x_426 = lean_ctor_get(x_411, 0); +x_427 = lean_ctor_get(x_411, 1); +lean_inc(x_427); +lean_inc(x_426); +lean_dec(x_411); +x_428 = lean_ptr_addr(x_399); +lean_dec(x_399); +x_429 = lean_ptr_addr(x_404); +x_430 = lean_usize_dec_eq(x_428, x_429); +if (x_430 == 0) +{ +lean_object* x_431; lean_object* x_432; +lean_dec(x_401); +lean_dec(x_400); lean_dec(x_5); -x_245 = !lean_is_exclusive(x_237); -if (x_245 == 0) +x_431 = l_Lean_Expr_letE___override(x_398, x_404, x_407, x_426, x_402); +x_432 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_432, 0, x_431); +lean_ctor_set(x_432, 1, x_427); +return x_432; +} +else { -return x_237; +size_t x_433; size_t x_434; uint8_t x_435; +x_433 = lean_ptr_addr(x_400); +lean_dec(x_400); +x_434 = lean_ptr_addr(x_407); +x_435 = lean_usize_dec_eq(x_433, x_434); +if (x_435 == 0) +{ +lean_object* x_436; lean_object* x_437; +lean_dec(x_401); +lean_dec(x_5); +x_436 = l_Lean_Expr_letE___override(x_398, x_404, x_407, x_426, x_402); +x_437 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_437, 0, x_436); +lean_ctor_set(x_437, 1, x_427); +return x_437; } else { -lean_object* x_246; lean_object* x_247; lean_object* x_248; -x_246 = lean_ctor_get(x_237, 0); -x_247 = lean_ctor_get(x_237, 1); -lean_inc(x_247); -lean_inc(x_246); -lean_dec(x_237); -x_248 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_248, 0, x_246); -lean_ctor_set(x_248, 1, x_247); -return x_248; +size_t x_438; size_t x_439; uint8_t x_440; +x_438 = lean_ptr_addr(x_401); +lean_dec(x_401); +x_439 = lean_ptr_addr(x_426); +x_440 = lean_usize_dec_eq(x_438, x_439); +if (x_440 == 0) +{ +lean_object* x_441; lean_object* x_442; +lean_dec(x_5); +x_441 = l_Lean_Expr_letE___override(x_398, x_404, x_407, x_426, x_402); +x_442 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_442, 0, x_441); +lean_ctor_set(x_442, 1, x_427); +return x_442; +} +else +{ +lean_object* x_443; +lean_dec(x_426); +lean_dec(x_407); +lean_dec(x_404); +lean_dec(x_398); +x_443 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_443, 0, x_5); +lean_ctor_set(x_443, 1, x_427); +return x_443; +} +} } } } else { -uint8_t x_249; -lean_dec(x_230); -lean_dec(x_228); +uint8_t x_444; +lean_dec(x_407); +lean_dec(x_404); +lean_dec(x_401); +lean_dec(x_400); +lean_dec(x_399); +lean_dec(x_398); +lean_dec(x_5); +x_444 = !lean_is_exclusive(x_411); +if (x_444 == 0) +{ +return x_411; +} +else +{ +lean_object* x_445; lean_object* x_446; lean_object* x_447; +x_445 = lean_ctor_get(x_411, 0); +x_446 = lean_ctor_get(x_411, 1); +lean_inc(x_446); +lean_inc(x_445); +lean_dec(x_411); +x_447 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_447, 0, x_445); +lean_ctor_set(x_447, 1, x_446); +return x_447; +} +} +} +else +{ +uint8_t x_448; +lean_dec(x_404); +lean_dec(x_401); +lean_dec(x_400); +lean_dec(x_399); +lean_dec(x_398); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -541,31 +980,33 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_249 = !lean_is_exclusive(x_232); -if (x_249 == 0) +x_448 = !lean_is_exclusive(x_406); +if (x_448 == 0) { -return x_232; +return x_406; } else { -lean_object* x_250; lean_object* x_251; lean_object* x_252; -x_250 = lean_ctor_get(x_232, 0); -x_251 = lean_ctor_get(x_232, 1); -lean_inc(x_251); -lean_inc(x_250); -lean_dec(x_232); -x_252 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_252, 0, x_250); -lean_ctor_set(x_252, 1, x_251); -return x_252; +lean_object* x_449; lean_object* x_450; lean_object* x_451; +x_449 = lean_ctor_get(x_406, 0); +x_450 = lean_ctor_get(x_406, 1); +lean_inc(x_450); +lean_inc(x_449); +lean_dec(x_406); +x_451 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_451, 0, x_449); +lean_ctor_set(x_451, 1, x_450); +return x_451; } } } else { -uint8_t x_253; -lean_dec(x_228); -lean_dec(x_227); +uint8_t x_452; +lean_dec(x_401); +lean_dec(x_400); +lean_dec(x_399); +lean_dec(x_398); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -573,293 +1014,454 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_253 = !lean_is_exclusive(x_229); -if (x_253 == 0) +x_452 = !lean_is_exclusive(x_403); +if (x_452 == 0) { -return x_229; +return x_403; } else { -lean_object* x_254; lean_object* x_255; lean_object* x_256; -x_254 = lean_ctor_get(x_229, 0); -x_255 = lean_ctor_get(x_229, 1); -lean_inc(x_255); -lean_inc(x_254); -lean_dec(x_229); -x_256 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_256, 0, x_254); -lean_ctor_set(x_256, 1, x_255); -return x_256; +lean_object* x_453; lean_object* x_454; lean_object* x_455; +x_453 = lean_ctor_get(x_403, 0); +x_454 = lean_ctor_get(x_403, 1); +lean_inc(x_454); +lean_inc(x_453); +lean_dec(x_403); +x_455 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_455, 0, x_453); +lean_ctor_set(x_455, 1, x_454); +return x_455; } } } case 10: { -lean_object* x_257; lean_object* x_258; lean_object* x_259; -x_257 = lean_ctor_get(x_150, 1); -lean_inc(x_257); -lean_dec(x_150); -x_258 = lean_ctor_get(x_5, 1); -lean_inc(x_258); -x_259 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_258, x_6, x_7, x_8, x_9, x_10, x_11, x_257); -if (lean_obj_tag(x_259) == 0) +lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; +x_456 = lean_ctor_get(x_258, 1); +lean_inc(x_456); +lean_dec(x_258); +x_457 = lean_ctor_get(x_5, 0); +lean_inc(x_457); +x_458 = lean_ctor_get(x_5, 1); +lean_inc(x_458); +lean_inc(x_458); +x_459 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_458, x_6, x_7, x_8, x_9, x_10, x_11, x_456); +if (lean_obj_tag(x_459) == 0) +{ +uint8_t x_460; +x_460 = !lean_is_exclusive(x_459); +if (x_460 == 0) +{ +lean_object* x_461; size_t x_462; size_t x_463; uint8_t x_464; +x_461 = lean_ctor_get(x_459, 0); +x_462 = lean_ptr_addr(x_458); +lean_dec(x_458); +x_463 = lean_ptr_addr(x_461); +x_464 = lean_usize_dec_eq(x_462, x_463); +if (x_464 == 0) +{ +lean_object* x_465; +lean_dec(x_5); +x_465 = l_Lean_Expr_mdata___override(x_457, x_461); +lean_ctor_set(x_459, 0, x_465); +return x_459; +} +else { -uint8_t x_260; -x_260 = !lean_is_exclusive(x_259); -if (x_260 == 0) +lean_dec(x_461); +lean_dec(x_457); +lean_ctor_set(x_459, 0, x_5); +return x_459; +} +} +else { -lean_object* x_261; lean_object* x_262; -x_261 = lean_ctor_get(x_259, 0); -x_262 = lean_expr_update_mdata(x_5, x_261); -lean_ctor_set(x_259, 0, x_262); -return x_259; +lean_object* x_466; lean_object* x_467; size_t x_468; size_t x_469; uint8_t x_470; +x_466 = lean_ctor_get(x_459, 0); +x_467 = lean_ctor_get(x_459, 1); +lean_inc(x_467); +lean_inc(x_466); +lean_dec(x_459); +x_468 = lean_ptr_addr(x_458); +lean_dec(x_458); +x_469 = lean_ptr_addr(x_466); +x_470 = lean_usize_dec_eq(x_468, x_469); +if (x_470 == 0) +{ +lean_object* x_471; lean_object* x_472; +lean_dec(x_5); +x_471 = l_Lean_Expr_mdata___override(x_457, x_466); +x_472 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_472, 0, x_471); +lean_ctor_set(x_472, 1, x_467); +return x_472; } else { -lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; -x_263 = lean_ctor_get(x_259, 0); -x_264 = lean_ctor_get(x_259, 1); -lean_inc(x_264); -lean_inc(x_263); -lean_dec(x_259); -x_265 = lean_expr_update_mdata(x_5, x_263); -x_266 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_266, 0, x_265); -lean_ctor_set(x_266, 1, x_264); -return x_266; +lean_object* x_473; +lean_dec(x_466); +lean_dec(x_457); +x_473 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_473, 0, x_5); +lean_ctor_set(x_473, 1, x_467); +return x_473; +} } } else { -uint8_t x_267; +uint8_t x_474; +lean_dec(x_458); +lean_dec(x_457); lean_dec(x_5); -x_267 = !lean_is_exclusive(x_259); -if (x_267 == 0) +x_474 = !lean_is_exclusive(x_459); +if (x_474 == 0) { -return x_259; +return x_459; } else { -lean_object* x_268; lean_object* x_269; lean_object* x_270; -x_268 = lean_ctor_get(x_259, 0); -x_269 = lean_ctor_get(x_259, 1); -lean_inc(x_269); -lean_inc(x_268); -lean_dec(x_259); -x_270 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_270, 0, x_268); -lean_ctor_set(x_270, 1, x_269); -return x_270; +lean_object* x_475; lean_object* x_476; lean_object* x_477; +x_475 = lean_ctor_get(x_459, 0); +x_476 = lean_ctor_get(x_459, 1); +lean_inc(x_476); +lean_inc(x_475); +lean_dec(x_459); +x_477 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_477, 0, x_475); +lean_ctor_set(x_477, 1, x_476); +return x_477; } } } case 11: { -lean_object* x_271; lean_object* x_272; lean_object* x_273; -x_271 = lean_ctor_get(x_150, 1); -lean_inc(x_271); -lean_dec(x_150); -x_272 = lean_ctor_get(x_5, 2); -lean_inc(x_272); -x_273 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_272, x_6, x_7, x_8, x_9, x_10, x_11, x_271); -if (lean_obj_tag(x_273) == 0) +lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; +x_478 = lean_ctor_get(x_258, 1); +lean_inc(x_478); +lean_dec(x_258); +x_479 = lean_ctor_get(x_5, 0); +lean_inc(x_479); +x_480 = lean_ctor_get(x_5, 1); +lean_inc(x_480); +x_481 = lean_ctor_get(x_5, 2); +lean_inc(x_481); +lean_inc(x_481); +x_482 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_481, x_6, x_7, x_8, x_9, x_10, x_11, x_478); +if (lean_obj_tag(x_482) == 0) +{ +uint8_t x_483; +x_483 = !lean_is_exclusive(x_482); +if (x_483 == 0) +{ +lean_object* x_484; size_t x_485; size_t x_486; uint8_t x_487; +x_484 = lean_ctor_get(x_482, 0); +x_485 = lean_ptr_addr(x_481); +lean_dec(x_481); +x_486 = lean_ptr_addr(x_484); +x_487 = lean_usize_dec_eq(x_485, x_486); +if (x_487 == 0) +{ +lean_object* x_488; +lean_dec(x_5); +x_488 = l_Lean_Expr_proj___override(x_479, x_480, x_484); +lean_ctor_set(x_482, 0, x_488); +return x_482; +} +else +{ +lean_dec(x_484); +lean_dec(x_480); +lean_dec(x_479); +lean_ctor_set(x_482, 0, x_5); +return x_482; +} +} +else { -uint8_t x_274; -x_274 = !lean_is_exclusive(x_273); -if (x_274 == 0) +lean_object* x_489; lean_object* x_490; size_t x_491; size_t x_492; uint8_t x_493; +x_489 = lean_ctor_get(x_482, 0); +x_490 = lean_ctor_get(x_482, 1); +lean_inc(x_490); +lean_inc(x_489); +lean_dec(x_482); +x_491 = lean_ptr_addr(x_481); +lean_dec(x_481); +x_492 = lean_ptr_addr(x_489); +x_493 = lean_usize_dec_eq(x_491, x_492); +if (x_493 == 0) { -lean_object* x_275; lean_object* x_276; -x_275 = lean_ctor_get(x_273, 0); -x_276 = lean_expr_update_proj(x_5, x_275); -lean_ctor_set(x_273, 0, x_276); -return x_273; +lean_object* x_494; lean_object* x_495; +lean_dec(x_5); +x_494 = l_Lean_Expr_proj___override(x_479, x_480, x_489); +x_495 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_495, 0, x_494); +lean_ctor_set(x_495, 1, x_490); +return x_495; } else { -lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; -x_277 = lean_ctor_get(x_273, 0); -x_278 = lean_ctor_get(x_273, 1); -lean_inc(x_278); -lean_inc(x_277); -lean_dec(x_273); -x_279 = lean_expr_update_proj(x_5, x_277); -x_280 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_280, 0, x_279); -lean_ctor_set(x_280, 1, x_278); -return x_280; +lean_object* x_496; +lean_dec(x_489); +lean_dec(x_480); +lean_dec(x_479); +x_496 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_496, 0, x_5); +lean_ctor_set(x_496, 1, x_490); +return x_496; +} } } else { -uint8_t x_281; +uint8_t x_497; +lean_dec(x_481); +lean_dec(x_480); +lean_dec(x_479); lean_dec(x_5); -x_281 = !lean_is_exclusive(x_273); -if (x_281 == 0) +x_497 = !lean_is_exclusive(x_482); +if (x_497 == 0) { -return x_273; +return x_482; } else { -lean_object* x_282; lean_object* x_283; lean_object* x_284; -x_282 = lean_ctor_get(x_273, 0); -x_283 = lean_ctor_get(x_273, 1); -lean_inc(x_283); -lean_inc(x_282); -lean_dec(x_273); -x_284 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_284, 0, x_282); -lean_ctor_set(x_284, 1, x_283); -return x_284; +lean_object* x_498; lean_object* x_499; lean_object* x_500; +x_498 = lean_ctor_get(x_482, 0); +x_499 = lean_ctor_get(x_482, 1); +lean_inc(x_499); +lean_inc(x_498); +lean_dec(x_482); +x_500 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_500, 0, x_498); +lean_ctor_set(x_500, 1, x_499); +return x_500; } } } default: { -uint8_t x_285; +uint8_t x_501; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_1); -x_285 = !lean_is_exclusive(x_150); -if (x_285 == 0) +x_501 = !lean_is_exclusive(x_258); +if (x_501 == 0) { -lean_object* x_286; -x_286 = lean_ctor_get(x_150, 0); -lean_dec(x_286); -lean_ctor_set(x_150, 0, x_5); -return x_150; +lean_object* x_502; +x_502 = lean_ctor_get(x_258, 0); +lean_dec(x_502); +lean_ctor_set(x_258, 0, x_5); +return x_258; } else { -lean_object* x_287; lean_object* x_288; -x_287 = lean_ctor_get(x_150, 1); -lean_inc(x_287); -lean_dec(x_150); -x_288 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_288, 0, x_5); -lean_ctor_set(x_288, 1, x_287); -return x_288; +lean_object* x_503; lean_object* x_504; +x_503 = lean_ctor_get(x_258, 1); +lean_inc(x_503); +lean_dec(x_258); +x_504 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_504, 0, x_5); +lean_ctor_set(x_504, 1, x_503); +return x_504; } } } } else { -lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; uint8_t x_300; -x_289 = lean_ctor_get(x_150, 1); -lean_inc(x_289); -lean_dec(x_150); -x_290 = lean_st_ref_get(x_11, x_289); -x_291 = lean_ctor_get(x_290, 1); -lean_inc(x_291); -lean_dec(x_290); -x_292 = lean_st_ref_get(x_7, x_291); -x_293 = lean_ctor_get(x_292, 0); -lean_inc(x_293); -x_294 = lean_ctor_get(x_292, 1); -lean_inc(x_294); -lean_dec(x_292); -x_295 = lean_unsigned_to_nat(1u); -x_296 = lean_nat_add(x_293, x_295); -x_297 = lean_st_ref_get(x_11, x_294); -x_298 = lean_ctor_get(x_297, 1); -lean_inc(x_298); -lean_dec(x_297); -x_299 = lean_st_ref_set(x_7, x_296, x_298); -x_300 = !lean_is_exclusive(x_299); -if (x_300 == 0) -{ -lean_object* x_301; lean_object* x_302; uint8_t x_303; -x_301 = lean_ctor_get(x_299, 1); -x_302 = lean_ctor_get(x_299, 0); -lean_dec(x_302); -x_303 = l_Lean_Occurrences_contains(x_2, x_293); -lean_dec(x_293); -if (x_303 == 0) +lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; uint8_t x_516; +x_505 = lean_ctor_get(x_258, 1); +lean_inc(x_505); +lean_dec(x_258); +x_506 = lean_st_ref_get(x_11, x_505); +x_507 = lean_ctor_get(x_506, 1); +lean_inc(x_507); +lean_dec(x_506); +x_508 = lean_st_ref_get(x_7, x_507); +x_509 = lean_ctor_get(x_508, 0); +lean_inc(x_509); +x_510 = lean_ctor_get(x_508, 1); +lean_inc(x_510); +lean_dec(x_508); +x_511 = lean_unsigned_to_nat(1u); +x_512 = lean_nat_add(x_509, x_511); +x_513 = lean_st_ref_get(x_11, x_510); +x_514 = lean_ctor_get(x_513, 1); +lean_inc(x_514); +lean_dec(x_513); +x_515 = lean_st_ref_set(x_7, x_512, x_514); +x_516 = !lean_is_exclusive(x_515); +if (x_516 == 0) +{ +lean_object* x_517; lean_object* x_518; uint8_t x_519; +x_517 = lean_ctor_get(x_515, 1); +x_518 = lean_ctor_get(x_515, 0); +lean_dec(x_518); +x_519 = l_Lean_Occurrences_contains(x_2, x_509); +lean_dec(x_509); +if (x_519 == 0) { switch (lean_obj_tag(x_5)) { case 5: { -lean_object* x_304; lean_object* x_305; lean_object* x_306; -lean_free_object(x_299); -x_304 = lean_ctor_get(x_5, 0); -lean_inc(x_304); -x_305 = lean_ctor_get(x_5, 1); -lean_inc(x_305); +lean_object* x_520; lean_object* x_521; lean_object* x_522; +lean_free_object(x_515); +x_520 = lean_ctor_get(x_5, 0); +lean_inc(x_520); +x_521 = lean_ctor_get(x_5, 1); +lean_inc(x_521); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_520); lean_inc(x_1); -x_306 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_304, x_6, x_7, x_8, x_9, x_10, x_11, x_301); -if (lean_obj_tag(x_306) == 0) -{ -lean_object* x_307; lean_object* x_308; lean_object* x_309; -x_307 = lean_ctor_get(x_306, 0); -lean_inc(x_307); -x_308 = lean_ctor_get(x_306, 1); -lean_inc(x_308); -lean_dec(x_306); -x_309 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_305, x_6, x_7, x_8, x_9, x_10, x_11, x_308); -if (lean_obj_tag(x_309) == 0) +x_522 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_520, x_6, x_7, x_8, x_9, x_10, x_11, x_517); +if (lean_obj_tag(x_522) == 0) +{ +lean_object* x_523; lean_object* x_524; lean_object* x_525; +x_523 = lean_ctor_get(x_522, 0); +lean_inc(x_523); +x_524 = lean_ctor_get(x_522, 1); +lean_inc(x_524); +lean_dec(x_522); +lean_inc(x_521); +x_525 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_521, x_6, x_7, x_8, x_9, x_10, x_11, x_524); +if (lean_obj_tag(x_525) == 0) +{ +uint8_t x_526; +x_526 = !lean_is_exclusive(x_525); +if (x_526 == 0) +{ +lean_object* x_527; size_t x_528; size_t x_529; uint8_t x_530; +x_527 = lean_ctor_get(x_525, 0); +x_528 = lean_ptr_addr(x_520); +lean_dec(x_520); +x_529 = lean_ptr_addr(x_523); +x_530 = lean_usize_dec_eq(x_528, x_529); +if (x_530 == 0) +{ +lean_object* x_531; +lean_dec(x_521); +lean_dec(x_5); +x_531 = l_Lean_Expr_app___override(x_523, x_527); +lean_ctor_set(x_525, 0, x_531); +return x_525; +} +else { -uint8_t x_310; -x_310 = !lean_is_exclusive(x_309); -if (x_310 == 0) +size_t x_532; size_t x_533; uint8_t x_534; +x_532 = lean_ptr_addr(x_521); +lean_dec(x_521); +x_533 = lean_ptr_addr(x_527); +x_534 = lean_usize_dec_eq(x_532, x_533); +if (x_534 == 0) { -lean_object* x_311; lean_object* x_312; -x_311 = lean_ctor_get(x_309, 0); -x_312 = lean_expr_update_app(x_5, x_307, x_311); -lean_ctor_set(x_309, 0, x_312); -return x_309; +lean_object* x_535; +lean_dec(x_5); +x_535 = l_Lean_Expr_app___override(x_523, x_527); +lean_ctor_set(x_525, 0, x_535); +return x_525; } else { -lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; -x_313 = lean_ctor_get(x_309, 0); -x_314 = lean_ctor_get(x_309, 1); -lean_inc(x_314); -lean_inc(x_313); -lean_dec(x_309); -x_315 = lean_expr_update_app(x_5, x_307, x_313); -x_316 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_316, 0, x_315); -lean_ctor_set(x_316, 1, x_314); -return x_316; +lean_dec(x_527); +lean_dec(x_523); +lean_ctor_set(x_525, 0, x_5); +return x_525; +} } } else { -uint8_t x_317; -lean_dec(x_307); +lean_object* x_536; lean_object* x_537; size_t x_538; size_t x_539; uint8_t x_540; +x_536 = lean_ctor_get(x_525, 0); +x_537 = lean_ctor_get(x_525, 1); +lean_inc(x_537); +lean_inc(x_536); +lean_dec(x_525); +x_538 = lean_ptr_addr(x_520); +lean_dec(x_520); +x_539 = lean_ptr_addr(x_523); +x_540 = lean_usize_dec_eq(x_538, x_539); +if (x_540 == 0) +{ +lean_object* x_541; lean_object* x_542; +lean_dec(x_521); lean_dec(x_5); -x_317 = !lean_is_exclusive(x_309); -if (x_317 == 0) +x_541 = l_Lean_Expr_app___override(x_523, x_536); +x_542 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_542, 0, x_541); +lean_ctor_set(x_542, 1, x_537); +return x_542; +} +else { -return x_309; +size_t x_543; size_t x_544; uint8_t x_545; +x_543 = lean_ptr_addr(x_521); +lean_dec(x_521); +x_544 = lean_ptr_addr(x_536); +x_545 = lean_usize_dec_eq(x_543, x_544); +if (x_545 == 0) +{ +lean_object* x_546; lean_object* x_547; +lean_dec(x_5); +x_546 = l_Lean_Expr_app___override(x_523, x_536); +x_547 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_547, 0, x_546); +lean_ctor_set(x_547, 1, x_537); +return x_547; } else { -lean_object* x_318; lean_object* x_319; lean_object* x_320; -x_318 = lean_ctor_get(x_309, 0); -x_319 = lean_ctor_get(x_309, 1); -lean_inc(x_319); -lean_inc(x_318); -lean_dec(x_309); -x_320 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_320, 0, x_318); -lean_ctor_set(x_320, 1, x_319); -return x_320; +lean_object* x_548; +lean_dec(x_536); +lean_dec(x_523); +x_548 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_548, 0, x_5); +lean_ctor_set(x_548, 1, x_537); +return x_548; +} } } } else { -uint8_t x_321; -lean_dec(x_305); +uint8_t x_549; +lean_dec(x_523); +lean_dec(x_521); +lean_dec(x_520); +lean_dec(x_5); +x_549 = !lean_is_exclusive(x_525); +if (x_549 == 0) +{ +return x_525; +} +else +{ +lean_object* x_550; lean_object* x_551; lean_object* x_552; +x_550 = lean_ctor_get(x_525, 0); +x_551 = lean_ctor_get(x_525, 1); +lean_inc(x_551); +lean_inc(x_550); +lean_dec(x_525); +x_552 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_552, 0, x_550); +lean_ctor_set(x_552, 1, x_551); +return x_552; +} +} +} +else +{ +uint8_t x_553; +lean_dec(x_521); +lean_dec(x_520); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -867,347 +1469,707 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_321 = !lean_is_exclusive(x_306); -if (x_321 == 0) +x_553 = !lean_is_exclusive(x_522); +if (x_553 == 0) { -return x_306; +return x_522; } else { -lean_object* x_322; lean_object* x_323; lean_object* x_324; -x_322 = lean_ctor_get(x_306, 0); -x_323 = lean_ctor_get(x_306, 1); -lean_inc(x_323); -lean_inc(x_322); -lean_dec(x_306); -x_324 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_324, 0, x_322); -lean_ctor_set(x_324, 1, x_323); -return x_324; +lean_object* x_554; lean_object* x_555; lean_object* x_556; +x_554 = lean_ctor_get(x_522, 0); +x_555 = lean_ctor_get(x_522, 1); +lean_inc(x_555); +lean_inc(x_554); +lean_dec(x_522); +x_556 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_556, 0, x_554); +lean_ctor_set(x_556, 1, x_555); +return x_556; } } } case 6: { -lean_object* x_325; lean_object* x_326; uint8_t x_327; lean_object* x_328; -lean_free_object(x_299); -x_325 = lean_ctor_get(x_5, 1); -lean_inc(x_325); -x_326 = lean_ctor_get(x_5, 2); -lean_inc(x_326); -x_327 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_object* x_557; lean_object* x_558; lean_object* x_559; uint8_t x_560; lean_object* x_561; +lean_free_object(x_515); +x_557 = lean_ctor_get(x_5, 0); +lean_inc(x_557); +x_558 = lean_ctor_get(x_5, 1); +lean_inc(x_558); +x_559 = lean_ctor_get(x_5, 2); +lean_inc(x_559); +x_560 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_558); lean_inc(x_1); -x_328 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_325, x_6, x_7, x_8, x_9, x_10, x_11, x_301); -if (lean_obj_tag(x_328) == 0) -{ -lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; -x_329 = lean_ctor_get(x_328, 0); -lean_inc(x_329); -x_330 = lean_ctor_get(x_328, 1); -lean_inc(x_330); -lean_dec(x_328); -x_331 = lean_nat_add(x_6, x_295); +x_561 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_558, x_6, x_7, x_8, x_9, x_10, x_11, x_517); +if (lean_obj_tag(x_561) == 0) +{ +lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; +x_562 = lean_ctor_get(x_561, 0); +lean_inc(x_562); +x_563 = lean_ctor_get(x_561, 1); +lean_inc(x_563); +lean_dec(x_561); +x_564 = lean_nat_add(x_6, x_511); lean_dec(x_6); -x_332 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_326, x_331, x_7, x_8, x_9, x_10, x_11, x_330); -if (lean_obj_tag(x_332) == 0) +lean_inc(x_559); +x_565 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_559, x_564, x_7, x_8, x_9, x_10, x_11, x_563); +if (lean_obj_tag(x_565) == 0) { -uint8_t x_333; -x_333 = !lean_is_exclusive(x_332); -if (x_333 == 0) +uint8_t x_566; +x_566 = !lean_is_exclusive(x_565); +if (x_566 == 0) { -lean_object* x_334; lean_object* x_335; -x_334 = lean_ctor_get(x_332, 0); -x_335 = lean_expr_update_lambda(x_5, x_327, x_329, x_334); -lean_ctor_set(x_332, 0, x_335); -return x_332; +lean_object* x_567; lean_object* x_568; size_t x_569; size_t x_570; uint8_t x_571; +x_567 = lean_ctor_get(x_565, 0); +lean_inc(x_559); +lean_inc(x_558); +lean_inc(x_557); +x_568 = l_Lean_Expr_lam___override(x_557, x_558, x_559, x_560); +x_569 = lean_ptr_addr(x_558); +lean_dec(x_558); +x_570 = lean_ptr_addr(x_562); +x_571 = lean_usize_dec_eq(x_569, x_570); +if (x_571 == 0) +{ +lean_object* x_572; +lean_dec(x_568); +lean_dec(x_559); +x_572 = l_Lean_Expr_lam___override(x_557, x_562, x_567, x_560); +lean_ctor_set(x_565, 0, x_572); +return x_565; } else { -lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; -x_336 = lean_ctor_get(x_332, 0); -x_337 = lean_ctor_get(x_332, 1); -lean_inc(x_337); -lean_inc(x_336); -lean_dec(x_332); -x_338 = lean_expr_update_lambda(x_5, x_327, x_329, x_336); -x_339 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_339, 0, x_338); -lean_ctor_set(x_339, 1, x_337); -return x_339; +size_t x_573; size_t x_574; uint8_t x_575; +x_573 = lean_ptr_addr(x_559); +lean_dec(x_559); +x_574 = lean_ptr_addr(x_567); +x_575 = lean_usize_dec_eq(x_573, x_574); +if (x_575 == 0) +{ +lean_object* x_576; +lean_dec(x_568); +x_576 = l_Lean_Expr_lam___override(x_557, x_562, x_567, x_560); +lean_ctor_set(x_565, 0, x_576); +return x_565; } +else +{ +uint8_t x_577; +x_577 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_560, x_560); +if (x_577 == 0) +{ +lean_object* x_578; +lean_dec(x_568); +x_578 = l_Lean_Expr_lam___override(x_557, x_562, x_567, x_560); +lean_ctor_set(x_565, 0, x_578); +return x_565; } else { -uint8_t x_340; -lean_dec(x_329); -lean_dec(x_5); -x_340 = !lean_is_exclusive(x_332); -if (x_340 == 0) +lean_dec(x_567); +lean_dec(x_562); +lean_dec(x_557); +lean_ctor_set(x_565, 0, x_568); +return x_565; +} +} +} +} +else +{ +lean_object* x_579; lean_object* x_580; lean_object* x_581; size_t x_582; size_t x_583; uint8_t x_584; +x_579 = lean_ctor_get(x_565, 0); +x_580 = lean_ctor_get(x_565, 1); +lean_inc(x_580); +lean_inc(x_579); +lean_dec(x_565); +lean_inc(x_559); +lean_inc(x_558); +lean_inc(x_557); +x_581 = l_Lean_Expr_lam___override(x_557, x_558, x_559, x_560); +x_582 = lean_ptr_addr(x_558); +lean_dec(x_558); +x_583 = lean_ptr_addr(x_562); +x_584 = lean_usize_dec_eq(x_582, x_583); +if (x_584 == 0) +{ +lean_object* x_585; lean_object* x_586; +lean_dec(x_581); +lean_dec(x_559); +x_585 = l_Lean_Expr_lam___override(x_557, x_562, x_579, x_560); +x_586 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_586, 0, x_585); +lean_ctor_set(x_586, 1, x_580); +return x_586; +} +else +{ +size_t x_587; size_t x_588; uint8_t x_589; +x_587 = lean_ptr_addr(x_559); +lean_dec(x_559); +x_588 = lean_ptr_addr(x_579); +x_589 = lean_usize_dec_eq(x_587, x_588); +if (x_589 == 0) { -return x_332; +lean_object* x_590; lean_object* x_591; +lean_dec(x_581); +x_590 = l_Lean_Expr_lam___override(x_557, x_562, x_579, x_560); +x_591 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_591, 0, x_590); +lean_ctor_set(x_591, 1, x_580); +return x_591; } else { -lean_object* x_341; lean_object* x_342; lean_object* x_343; -x_341 = lean_ctor_get(x_332, 0); -x_342 = lean_ctor_get(x_332, 1); -lean_inc(x_342); -lean_inc(x_341); -lean_dec(x_332); -x_343 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_343, 0, x_341); -lean_ctor_set(x_343, 1, x_342); -return x_343; +uint8_t x_592; +x_592 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_560, x_560); +if (x_592 == 0) +{ +lean_object* x_593; lean_object* x_594; +lean_dec(x_581); +x_593 = l_Lean_Expr_lam___override(x_557, x_562, x_579, x_560); +x_594 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_594, 0, x_593); +lean_ctor_set(x_594, 1, x_580); +return x_594; +} +else +{ +lean_object* x_595; +lean_dec(x_579); +lean_dec(x_562); +lean_dec(x_557); +x_595 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_595, 0, x_581); +lean_ctor_set(x_595, 1, x_580); +return x_595; +} +} } } } else { -uint8_t x_344; -lean_dec(x_326); +uint8_t x_596; +lean_dec(x_562); +lean_dec(x_559); +lean_dec(x_558); +lean_dec(x_557); +x_596 = !lean_is_exclusive(x_565); +if (x_596 == 0) +{ +return x_565; +} +else +{ +lean_object* x_597; lean_object* x_598; lean_object* x_599; +x_597 = lean_ctor_get(x_565, 0); +x_598 = lean_ctor_get(x_565, 1); +lean_inc(x_598); +lean_inc(x_597); +lean_dec(x_565); +x_599 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_599, 0, x_597); +lean_ctor_set(x_599, 1, x_598); +return x_599; +} +} +} +else +{ +uint8_t x_600; +lean_dec(x_559); +lean_dec(x_558); +lean_dec(x_557); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_344 = !lean_is_exclusive(x_328); -if (x_344 == 0) +x_600 = !lean_is_exclusive(x_561); +if (x_600 == 0) { -return x_328; +return x_561; } else { -lean_object* x_345; lean_object* x_346; lean_object* x_347; -x_345 = lean_ctor_get(x_328, 0); -x_346 = lean_ctor_get(x_328, 1); -lean_inc(x_346); -lean_inc(x_345); -lean_dec(x_328); -x_347 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_347, 0, x_345); -lean_ctor_set(x_347, 1, x_346); -return x_347; +lean_object* x_601; lean_object* x_602; lean_object* x_603; +x_601 = lean_ctor_get(x_561, 0); +x_602 = lean_ctor_get(x_561, 1); +lean_inc(x_602); +lean_inc(x_601); +lean_dec(x_561); +x_603 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_603, 0, x_601); +lean_ctor_set(x_603, 1, x_602); +return x_603; } } } case 7: { -lean_object* x_348; lean_object* x_349; uint8_t x_350; lean_object* x_351; -lean_free_object(x_299); -x_348 = lean_ctor_get(x_5, 1); -lean_inc(x_348); -x_349 = lean_ctor_get(x_5, 2); -lean_inc(x_349); -x_350 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_object* x_604; lean_object* x_605; lean_object* x_606; uint8_t x_607; lean_object* x_608; +lean_free_object(x_515); +x_604 = lean_ctor_get(x_5, 0); +lean_inc(x_604); +x_605 = lean_ctor_get(x_5, 1); +lean_inc(x_605); +x_606 = lean_ctor_get(x_5, 2); +lean_inc(x_606); +x_607 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_605); lean_inc(x_1); -x_351 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_348, x_6, x_7, x_8, x_9, x_10, x_11, x_301); -if (lean_obj_tag(x_351) == 0) -{ -lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; -x_352 = lean_ctor_get(x_351, 0); -lean_inc(x_352); -x_353 = lean_ctor_get(x_351, 1); -lean_inc(x_353); -lean_dec(x_351); -x_354 = lean_nat_add(x_6, x_295); +x_608 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_605, x_6, x_7, x_8, x_9, x_10, x_11, x_517); +if (lean_obj_tag(x_608) == 0) +{ +lean_object* x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; +x_609 = lean_ctor_get(x_608, 0); +lean_inc(x_609); +x_610 = lean_ctor_get(x_608, 1); +lean_inc(x_610); +lean_dec(x_608); +x_611 = lean_nat_add(x_6, x_511); lean_dec(x_6); -x_355 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_349, x_354, x_7, x_8, x_9, x_10, x_11, x_353); -if (lean_obj_tag(x_355) == 0) +lean_inc(x_606); +x_612 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_606, x_611, x_7, x_8, x_9, x_10, x_11, x_610); +if (lean_obj_tag(x_612) == 0) +{ +uint8_t x_613; +x_613 = !lean_is_exclusive(x_612); +if (x_613 == 0) +{ +lean_object* x_614; lean_object* x_615; size_t x_616; size_t x_617; uint8_t x_618; +x_614 = lean_ctor_get(x_612, 0); +lean_inc(x_606); +lean_inc(x_605); +lean_inc(x_604); +x_615 = l_Lean_Expr_forallE___override(x_604, x_605, x_606, x_607); +x_616 = lean_ptr_addr(x_605); +lean_dec(x_605); +x_617 = lean_ptr_addr(x_609); +x_618 = lean_usize_dec_eq(x_616, x_617); +if (x_618 == 0) +{ +lean_object* x_619; +lean_dec(x_615); +lean_dec(x_606); +x_619 = l_Lean_Expr_forallE___override(x_604, x_609, x_614, x_607); +lean_ctor_set(x_612, 0, x_619); +return x_612; +} +else +{ +size_t x_620; size_t x_621; uint8_t x_622; +x_620 = lean_ptr_addr(x_606); +lean_dec(x_606); +x_621 = lean_ptr_addr(x_614); +x_622 = lean_usize_dec_eq(x_620, x_621); +if (x_622 == 0) +{ +lean_object* x_623; +lean_dec(x_615); +x_623 = l_Lean_Expr_forallE___override(x_604, x_609, x_614, x_607); +lean_ctor_set(x_612, 0, x_623); +return x_612; +} +else { -uint8_t x_356; -x_356 = !lean_is_exclusive(x_355); -if (x_356 == 0) +uint8_t x_624; +x_624 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_607, x_607); +if (x_624 == 0) { -lean_object* x_357; lean_object* x_358; -x_357 = lean_ctor_get(x_355, 0); -x_358 = lean_expr_update_forall(x_5, x_350, x_352, x_357); -lean_ctor_set(x_355, 0, x_358); -return x_355; +lean_object* x_625; +lean_dec(x_615); +x_625 = l_Lean_Expr_forallE___override(x_604, x_609, x_614, x_607); +lean_ctor_set(x_612, 0, x_625); +return x_612; } else { -lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; -x_359 = lean_ctor_get(x_355, 0); -x_360 = lean_ctor_get(x_355, 1); -lean_inc(x_360); -lean_inc(x_359); -lean_dec(x_355); -x_361 = lean_expr_update_forall(x_5, x_350, x_352, x_359); -x_362 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_362, 0, x_361); -lean_ctor_set(x_362, 1, x_360); -return x_362; +lean_dec(x_614); +lean_dec(x_609); +lean_dec(x_604); +lean_ctor_set(x_612, 0, x_615); +return x_612; +} +} } } else { -uint8_t x_363; -lean_dec(x_352); -lean_dec(x_5); -x_363 = !lean_is_exclusive(x_355); -if (x_363 == 0) +lean_object* x_626; lean_object* x_627; lean_object* x_628; size_t x_629; size_t x_630; uint8_t x_631; +x_626 = lean_ctor_get(x_612, 0); +x_627 = lean_ctor_get(x_612, 1); +lean_inc(x_627); +lean_inc(x_626); +lean_dec(x_612); +lean_inc(x_606); +lean_inc(x_605); +lean_inc(x_604); +x_628 = l_Lean_Expr_forallE___override(x_604, x_605, x_606, x_607); +x_629 = lean_ptr_addr(x_605); +lean_dec(x_605); +x_630 = lean_ptr_addr(x_609); +x_631 = lean_usize_dec_eq(x_629, x_630); +if (x_631 == 0) +{ +lean_object* x_632; lean_object* x_633; +lean_dec(x_628); +lean_dec(x_606); +x_632 = l_Lean_Expr_forallE___override(x_604, x_609, x_626, x_607); +x_633 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_633, 0, x_632); +lean_ctor_set(x_633, 1, x_627); +return x_633; +} +else +{ +size_t x_634; size_t x_635; uint8_t x_636; +x_634 = lean_ptr_addr(x_606); +lean_dec(x_606); +x_635 = lean_ptr_addr(x_626); +x_636 = lean_usize_dec_eq(x_634, x_635); +if (x_636 == 0) +{ +lean_object* x_637; lean_object* x_638; +lean_dec(x_628); +x_637 = l_Lean_Expr_forallE___override(x_604, x_609, x_626, x_607); +x_638 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_638, 0, x_637); +lean_ctor_set(x_638, 1, x_627); +return x_638; +} +else +{ +uint8_t x_639; +x_639 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_607, x_607); +if (x_639 == 0) { -return x_355; +lean_object* x_640; lean_object* x_641; +lean_dec(x_628); +x_640 = l_Lean_Expr_forallE___override(x_604, x_609, x_626, x_607); +x_641 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_641, 0, x_640); +lean_ctor_set(x_641, 1, x_627); +return x_641; } else { -lean_object* x_364; lean_object* x_365; lean_object* x_366; -x_364 = lean_ctor_get(x_355, 0); -x_365 = lean_ctor_get(x_355, 1); -lean_inc(x_365); -lean_inc(x_364); -lean_dec(x_355); -x_366 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_366, 0, x_364); -lean_ctor_set(x_366, 1, x_365); -return x_366; +lean_object* x_642; +lean_dec(x_626); +lean_dec(x_609); +lean_dec(x_604); +x_642 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_642, 0, x_628); +lean_ctor_set(x_642, 1, x_627); +return x_642; +} +} } } } else { -uint8_t x_367; -lean_dec(x_349); +uint8_t x_643; +lean_dec(x_609); +lean_dec(x_606); +lean_dec(x_605); +lean_dec(x_604); +x_643 = !lean_is_exclusive(x_612); +if (x_643 == 0) +{ +return x_612; +} +else +{ +lean_object* x_644; lean_object* x_645; lean_object* x_646; +x_644 = lean_ctor_get(x_612, 0); +x_645 = lean_ctor_get(x_612, 1); +lean_inc(x_645); +lean_inc(x_644); +lean_dec(x_612); +x_646 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_646, 0, x_644); +lean_ctor_set(x_646, 1, x_645); +return x_646; +} +} +} +else +{ +uint8_t x_647; +lean_dec(x_606); +lean_dec(x_605); +lean_dec(x_604); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_367 = !lean_is_exclusive(x_351); -if (x_367 == 0) +x_647 = !lean_is_exclusive(x_608); +if (x_647 == 0) { -return x_351; +return x_608; } else { -lean_object* x_368; lean_object* x_369; lean_object* x_370; -x_368 = lean_ctor_get(x_351, 0); -x_369 = lean_ctor_get(x_351, 1); -lean_inc(x_369); -lean_inc(x_368); -lean_dec(x_351); -x_370 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_370, 0, x_368); -lean_ctor_set(x_370, 1, x_369); -return x_370; +lean_object* x_648; lean_object* x_649; lean_object* x_650; +x_648 = lean_ctor_get(x_608, 0); +x_649 = lean_ctor_get(x_608, 1); +lean_inc(x_649); +lean_inc(x_648); +lean_dec(x_608); +x_650 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_650, 0, x_648); +lean_ctor_set(x_650, 1, x_649); +return x_650; } } } case 8: { -lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; -lean_free_object(x_299); -x_371 = lean_ctor_get(x_5, 1); -lean_inc(x_371); -x_372 = lean_ctor_get(x_5, 2); -lean_inc(x_372); -x_373 = lean_ctor_get(x_5, 3); -lean_inc(x_373); +lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; uint8_t x_655; lean_object* x_656; +lean_free_object(x_515); +x_651 = lean_ctor_get(x_5, 0); +lean_inc(x_651); +x_652 = lean_ctor_get(x_5, 1); +lean_inc(x_652); +x_653 = lean_ctor_get(x_5, 2); +lean_inc(x_653); +x_654 = lean_ctor_get(x_5, 3); +lean_inc(x_654); +x_655 = lean_ctor_get_uint8(x_5, sizeof(void*)*4 + 8); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_652); lean_inc(x_1); -x_374 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_371, x_6, x_7, x_8, x_9, x_10, x_11, x_301); -if (lean_obj_tag(x_374) == 0) -{ -lean_object* x_375; lean_object* x_376; lean_object* x_377; -x_375 = lean_ctor_get(x_374, 0); -lean_inc(x_375); -x_376 = lean_ctor_get(x_374, 1); -lean_inc(x_376); -lean_dec(x_374); +x_656 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_652, x_6, x_7, x_8, x_9, x_10, x_11, x_517); +if (lean_obj_tag(x_656) == 0) +{ +lean_object* x_657; lean_object* x_658; lean_object* x_659; +x_657 = lean_ctor_get(x_656, 0); +lean_inc(x_657); +x_658 = lean_ctor_get(x_656, 1); +lean_inc(x_658); +lean_dec(x_656); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_653); lean_inc(x_1); -x_377 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_372, x_6, x_7, x_8, x_9, x_10, x_11, x_376); -if (lean_obj_tag(x_377) == 0) -{ -lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; -x_378 = lean_ctor_get(x_377, 0); -lean_inc(x_378); -x_379 = lean_ctor_get(x_377, 1); -lean_inc(x_379); -lean_dec(x_377); -x_380 = lean_nat_add(x_6, x_295); +x_659 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_653, x_6, x_7, x_8, x_9, x_10, x_11, x_658); +if (lean_obj_tag(x_659) == 0) +{ +lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; +x_660 = lean_ctor_get(x_659, 0); +lean_inc(x_660); +x_661 = lean_ctor_get(x_659, 1); +lean_inc(x_661); +lean_dec(x_659); +x_662 = lean_nat_add(x_6, x_511); lean_dec(x_6); -x_381 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_373, x_380, x_7, x_8, x_9, x_10, x_11, x_379); -if (lean_obj_tag(x_381) == 0) +lean_inc(x_654); +x_663 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_654, x_662, x_7, x_8, x_9, x_10, x_11, x_661); +if (lean_obj_tag(x_663) == 0) +{ +uint8_t x_664; +x_664 = !lean_is_exclusive(x_663); +if (x_664 == 0) +{ +lean_object* x_665; size_t x_666; size_t x_667; uint8_t x_668; +x_665 = lean_ctor_get(x_663, 0); +x_666 = lean_ptr_addr(x_652); +lean_dec(x_652); +x_667 = lean_ptr_addr(x_657); +x_668 = lean_usize_dec_eq(x_666, x_667); +if (x_668 == 0) +{ +lean_object* x_669; +lean_dec(x_654); +lean_dec(x_653); +lean_dec(x_5); +x_669 = l_Lean_Expr_letE___override(x_651, x_657, x_660, x_665, x_655); +lean_ctor_set(x_663, 0, x_669); +return x_663; +} +else { -uint8_t x_382; -x_382 = !lean_is_exclusive(x_381); -if (x_382 == 0) +size_t x_670; size_t x_671; uint8_t x_672; +x_670 = lean_ptr_addr(x_653); +lean_dec(x_653); +x_671 = lean_ptr_addr(x_660); +x_672 = lean_usize_dec_eq(x_670, x_671); +if (x_672 == 0) { -lean_object* x_383; lean_object* x_384; -x_383 = lean_ctor_get(x_381, 0); -x_384 = lean_expr_update_let(x_5, x_375, x_378, x_383); -lean_ctor_set(x_381, 0, x_384); -return x_381; +lean_object* x_673; +lean_dec(x_654); +lean_dec(x_5); +x_673 = l_Lean_Expr_letE___override(x_651, x_657, x_660, x_665, x_655); +lean_ctor_set(x_663, 0, x_673); +return x_663; } else { -lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; -x_385 = lean_ctor_get(x_381, 0); -x_386 = lean_ctor_get(x_381, 1); -lean_inc(x_386); -lean_inc(x_385); -lean_dec(x_381); -x_387 = lean_expr_update_let(x_5, x_375, x_378, x_385); -x_388 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_388, 0, x_387); -lean_ctor_set(x_388, 1, x_386); -return x_388; +size_t x_674; size_t x_675; uint8_t x_676; +x_674 = lean_ptr_addr(x_654); +lean_dec(x_654); +x_675 = lean_ptr_addr(x_665); +x_676 = lean_usize_dec_eq(x_674, x_675); +if (x_676 == 0) +{ +lean_object* x_677; +lean_dec(x_5); +x_677 = l_Lean_Expr_letE___override(x_651, x_657, x_660, x_665, x_655); +lean_ctor_set(x_663, 0, x_677); +return x_663; +} +else +{ +lean_dec(x_665); +lean_dec(x_660); +lean_dec(x_657); +lean_dec(x_651); +lean_ctor_set(x_663, 0, x_5); +return x_663; +} +} } } else { -uint8_t x_389; -lean_dec(x_378); -lean_dec(x_375); +lean_object* x_678; lean_object* x_679; size_t x_680; size_t x_681; uint8_t x_682; +x_678 = lean_ctor_get(x_663, 0); +x_679 = lean_ctor_get(x_663, 1); +lean_inc(x_679); +lean_inc(x_678); +lean_dec(x_663); +x_680 = lean_ptr_addr(x_652); +lean_dec(x_652); +x_681 = lean_ptr_addr(x_657); +x_682 = lean_usize_dec_eq(x_680, x_681); +if (x_682 == 0) +{ +lean_object* x_683; lean_object* x_684; +lean_dec(x_654); +lean_dec(x_653); lean_dec(x_5); -x_389 = !lean_is_exclusive(x_381); -if (x_389 == 0) +x_683 = l_Lean_Expr_letE___override(x_651, x_657, x_660, x_678, x_655); +x_684 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_684, 0, x_683); +lean_ctor_set(x_684, 1, x_679); +return x_684; +} +else { -return x_381; +size_t x_685; size_t x_686; uint8_t x_687; +x_685 = lean_ptr_addr(x_653); +lean_dec(x_653); +x_686 = lean_ptr_addr(x_660); +x_687 = lean_usize_dec_eq(x_685, x_686); +if (x_687 == 0) +{ +lean_object* x_688; lean_object* x_689; +lean_dec(x_654); +lean_dec(x_5); +x_688 = l_Lean_Expr_letE___override(x_651, x_657, x_660, x_678, x_655); +x_689 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_689, 0, x_688); +lean_ctor_set(x_689, 1, x_679); +return x_689; } else { -lean_object* x_390; lean_object* x_391; lean_object* x_392; -x_390 = lean_ctor_get(x_381, 0); -x_391 = lean_ctor_get(x_381, 1); -lean_inc(x_391); -lean_inc(x_390); -lean_dec(x_381); -x_392 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_392, 0, x_390); -lean_ctor_set(x_392, 1, x_391); -return x_392; +size_t x_690; size_t x_691; uint8_t x_692; +x_690 = lean_ptr_addr(x_654); +lean_dec(x_654); +x_691 = lean_ptr_addr(x_678); +x_692 = lean_usize_dec_eq(x_690, x_691); +if (x_692 == 0) +{ +lean_object* x_693; lean_object* x_694; +lean_dec(x_5); +x_693 = l_Lean_Expr_letE___override(x_651, x_657, x_660, x_678, x_655); +x_694 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_694, 0, x_693); +lean_ctor_set(x_694, 1, x_679); +return x_694; +} +else +{ +lean_object* x_695; +lean_dec(x_678); +lean_dec(x_660); +lean_dec(x_657); +lean_dec(x_651); +x_695 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_695, 0, x_5); +lean_ctor_set(x_695, 1, x_679); +return x_695; +} +} +} +} +} +else +{ +uint8_t x_696; +lean_dec(x_660); +lean_dec(x_657); +lean_dec(x_654); +lean_dec(x_653); +lean_dec(x_652); +lean_dec(x_651); +lean_dec(x_5); +x_696 = !lean_is_exclusive(x_663); +if (x_696 == 0) +{ +return x_663; +} +else +{ +lean_object* x_697; lean_object* x_698; lean_object* x_699; +x_697 = lean_ctor_get(x_663, 0); +x_698 = lean_ctor_get(x_663, 1); +lean_inc(x_698); +lean_inc(x_697); +lean_dec(x_663); +x_699 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_699, 0, x_697); +lean_ctor_set(x_699, 1, x_698); +return x_699; } } } else { -uint8_t x_393; -lean_dec(x_375); -lean_dec(x_373); +uint8_t x_700; +lean_dec(x_657); +lean_dec(x_654); +lean_dec(x_653); +lean_dec(x_652); +lean_dec(x_651); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -1215,31 +2177,33 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_393 = !lean_is_exclusive(x_377); -if (x_393 == 0) +x_700 = !lean_is_exclusive(x_659); +if (x_700 == 0) { -return x_377; +return x_659; } else { -lean_object* x_394; lean_object* x_395; lean_object* x_396; -x_394 = lean_ctor_get(x_377, 0); -x_395 = lean_ctor_get(x_377, 1); -lean_inc(x_395); -lean_inc(x_394); -lean_dec(x_377); -x_396 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_396, 0, x_394); -lean_ctor_set(x_396, 1, x_395); -return x_396; +lean_object* x_701; lean_object* x_702; lean_object* x_703; +x_701 = lean_ctor_get(x_659, 0); +x_702 = lean_ctor_get(x_659, 1); +lean_inc(x_702); +lean_inc(x_701); +lean_dec(x_659); +x_703 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_703, 0, x_701); +lean_ctor_set(x_703, 1, x_702); +return x_703; } } } else { -uint8_t x_397; -lean_dec(x_373); -lean_dec(x_372); +uint8_t x_704; +lean_dec(x_654); +lean_dec(x_653); +lean_dec(x_652); +lean_dec(x_651); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -1247,139 +2211,224 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_397 = !lean_is_exclusive(x_374); -if (x_397 == 0) +x_704 = !lean_is_exclusive(x_656); +if (x_704 == 0) { -return x_374; +return x_656; } else { -lean_object* x_398; lean_object* x_399; lean_object* x_400; -x_398 = lean_ctor_get(x_374, 0); -x_399 = lean_ctor_get(x_374, 1); -lean_inc(x_399); -lean_inc(x_398); -lean_dec(x_374); -x_400 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_400, 0, x_398); -lean_ctor_set(x_400, 1, x_399); -return x_400; +lean_object* x_705; lean_object* x_706; lean_object* x_707; +x_705 = lean_ctor_get(x_656, 0); +x_706 = lean_ctor_get(x_656, 1); +lean_inc(x_706); +lean_inc(x_705); +lean_dec(x_656); +x_707 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_707, 0, x_705); +lean_ctor_set(x_707, 1, x_706); +return x_707; } } } case 10: { -lean_object* x_401; lean_object* x_402; -lean_free_object(x_299); -x_401 = lean_ctor_get(x_5, 1); -lean_inc(x_401); -x_402 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_401, x_6, x_7, x_8, x_9, x_10, x_11, x_301); -if (lean_obj_tag(x_402) == 0) +lean_object* x_708; lean_object* x_709; lean_object* x_710; +lean_free_object(x_515); +x_708 = lean_ctor_get(x_5, 0); +lean_inc(x_708); +x_709 = lean_ctor_get(x_5, 1); +lean_inc(x_709); +lean_inc(x_709); +x_710 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_709, x_6, x_7, x_8, x_9, x_10, x_11, x_517); +if (lean_obj_tag(x_710) == 0) +{ +uint8_t x_711; +x_711 = !lean_is_exclusive(x_710); +if (x_711 == 0) +{ +lean_object* x_712; size_t x_713; size_t x_714; uint8_t x_715; +x_712 = lean_ctor_get(x_710, 0); +x_713 = lean_ptr_addr(x_709); +lean_dec(x_709); +x_714 = lean_ptr_addr(x_712); +x_715 = lean_usize_dec_eq(x_713, x_714); +if (x_715 == 0) +{ +lean_object* x_716; +lean_dec(x_5); +x_716 = l_Lean_Expr_mdata___override(x_708, x_712); +lean_ctor_set(x_710, 0, x_716); +return x_710; +} +else { -uint8_t x_403; -x_403 = !lean_is_exclusive(x_402); -if (x_403 == 0) +lean_dec(x_712); +lean_dec(x_708); +lean_ctor_set(x_710, 0, x_5); +return x_710; +} +} +else +{ +lean_object* x_717; lean_object* x_718; size_t x_719; size_t x_720; uint8_t x_721; +x_717 = lean_ctor_get(x_710, 0); +x_718 = lean_ctor_get(x_710, 1); +lean_inc(x_718); +lean_inc(x_717); +lean_dec(x_710); +x_719 = lean_ptr_addr(x_709); +lean_dec(x_709); +x_720 = lean_ptr_addr(x_717); +x_721 = lean_usize_dec_eq(x_719, x_720); +if (x_721 == 0) { -lean_object* x_404; lean_object* x_405; -x_404 = lean_ctor_get(x_402, 0); -x_405 = lean_expr_update_mdata(x_5, x_404); -lean_ctor_set(x_402, 0, x_405); -return x_402; +lean_object* x_722; lean_object* x_723; +lean_dec(x_5); +x_722 = l_Lean_Expr_mdata___override(x_708, x_717); +x_723 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_723, 0, x_722); +lean_ctor_set(x_723, 1, x_718); +return x_723; } else { -lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; -x_406 = lean_ctor_get(x_402, 0); -x_407 = lean_ctor_get(x_402, 1); -lean_inc(x_407); -lean_inc(x_406); -lean_dec(x_402); -x_408 = lean_expr_update_mdata(x_5, x_406); -x_409 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_409, 0, x_408); -lean_ctor_set(x_409, 1, x_407); -return x_409; +lean_object* x_724; +lean_dec(x_717); +lean_dec(x_708); +x_724 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_724, 0, x_5); +lean_ctor_set(x_724, 1, x_718); +return x_724; +} } } else { -uint8_t x_410; +uint8_t x_725; +lean_dec(x_709); +lean_dec(x_708); lean_dec(x_5); -x_410 = !lean_is_exclusive(x_402); -if (x_410 == 0) +x_725 = !lean_is_exclusive(x_710); +if (x_725 == 0) { -return x_402; +return x_710; } else { -lean_object* x_411; lean_object* x_412; lean_object* x_413; -x_411 = lean_ctor_get(x_402, 0); -x_412 = lean_ctor_get(x_402, 1); -lean_inc(x_412); -lean_inc(x_411); -lean_dec(x_402); -x_413 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_413, 0, x_411); -lean_ctor_set(x_413, 1, x_412); -return x_413; +lean_object* x_726; lean_object* x_727; lean_object* x_728; +x_726 = lean_ctor_get(x_710, 0); +x_727 = lean_ctor_get(x_710, 1); +lean_inc(x_727); +lean_inc(x_726); +lean_dec(x_710); +x_728 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_728, 0, x_726); +lean_ctor_set(x_728, 1, x_727); +return x_728; } } } case 11: { -lean_object* x_414; lean_object* x_415; -lean_free_object(x_299); -x_414 = lean_ctor_get(x_5, 2); -lean_inc(x_414); -x_415 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_414, x_6, x_7, x_8, x_9, x_10, x_11, x_301); -if (lean_obj_tag(x_415) == 0) +lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; +lean_free_object(x_515); +x_729 = lean_ctor_get(x_5, 0); +lean_inc(x_729); +x_730 = lean_ctor_get(x_5, 1); +lean_inc(x_730); +x_731 = lean_ctor_get(x_5, 2); +lean_inc(x_731); +lean_inc(x_731); +x_732 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_731, x_6, x_7, x_8, x_9, x_10, x_11, x_517); +if (lean_obj_tag(x_732) == 0) +{ +uint8_t x_733; +x_733 = !lean_is_exclusive(x_732); +if (x_733 == 0) +{ +lean_object* x_734; size_t x_735; size_t x_736; uint8_t x_737; +x_734 = lean_ctor_get(x_732, 0); +x_735 = lean_ptr_addr(x_731); +lean_dec(x_731); +x_736 = lean_ptr_addr(x_734); +x_737 = lean_usize_dec_eq(x_735, x_736); +if (x_737 == 0) +{ +lean_object* x_738; +lean_dec(x_5); +x_738 = l_Lean_Expr_proj___override(x_729, x_730, x_734); +lean_ctor_set(x_732, 0, x_738); +return x_732; +} +else +{ +lean_dec(x_734); +lean_dec(x_730); +lean_dec(x_729); +lean_ctor_set(x_732, 0, x_5); +return x_732; +} +} +else { -uint8_t x_416; -x_416 = !lean_is_exclusive(x_415); -if (x_416 == 0) +lean_object* x_739; lean_object* x_740; size_t x_741; size_t x_742; uint8_t x_743; +x_739 = lean_ctor_get(x_732, 0); +x_740 = lean_ctor_get(x_732, 1); +lean_inc(x_740); +lean_inc(x_739); +lean_dec(x_732); +x_741 = lean_ptr_addr(x_731); +lean_dec(x_731); +x_742 = lean_ptr_addr(x_739); +x_743 = lean_usize_dec_eq(x_741, x_742); +if (x_743 == 0) { -lean_object* x_417; lean_object* x_418; -x_417 = lean_ctor_get(x_415, 0); -x_418 = lean_expr_update_proj(x_5, x_417); -lean_ctor_set(x_415, 0, x_418); -return x_415; +lean_object* x_744; lean_object* x_745; +lean_dec(x_5); +x_744 = l_Lean_Expr_proj___override(x_729, x_730, x_739); +x_745 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_745, 0, x_744); +lean_ctor_set(x_745, 1, x_740); +return x_745; } else { -lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; -x_419 = lean_ctor_get(x_415, 0); -x_420 = lean_ctor_get(x_415, 1); -lean_inc(x_420); -lean_inc(x_419); -lean_dec(x_415); -x_421 = lean_expr_update_proj(x_5, x_419); -x_422 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_422, 0, x_421); -lean_ctor_set(x_422, 1, x_420); -return x_422; +lean_object* x_746; +lean_dec(x_739); +lean_dec(x_730); +lean_dec(x_729); +x_746 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_746, 0, x_5); +lean_ctor_set(x_746, 1, x_740); +return x_746; +} } } else { -uint8_t x_423; +uint8_t x_747; +lean_dec(x_731); +lean_dec(x_730); +lean_dec(x_729); lean_dec(x_5); -x_423 = !lean_is_exclusive(x_415); -if (x_423 == 0) +x_747 = !lean_is_exclusive(x_732); +if (x_747 == 0) { -return x_415; +return x_732; } else { -lean_object* x_424; lean_object* x_425; lean_object* x_426; -x_424 = lean_ctor_get(x_415, 0); -x_425 = lean_ctor_get(x_415, 1); -lean_inc(x_425); -lean_inc(x_424); -lean_dec(x_415); -x_426 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_426, 0, x_424); -lean_ctor_set(x_426, 1, x_425); -return x_426; +lean_object* x_748; lean_object* x_749; lean_object* x_750; +x_748 = lean_ctor_get(x_732, 0); +x_749 = lean_ctor_get(x_732, 1); +lean_inc(x_749); +lean_inc(x_748); +lean_dec(x_732); +x_750 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_750, 0, x_748); +lean_ctor_set(x_750, 1, x_749); +return x_750; } } } @@ -1391,115 +2440,166 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_1); -lean_ctor_set(x_299, 0, x_5); -return x_299; +lean_ctor_set(x_515, 0, x_5); +return x_515; } } } else { -lean_object* x_427; +lean_object* x_751; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_5); lean_dec(x_1); -x_427 = l_Lean_Expr_bvar___override(x_6); -lean_ctor_set(x_299, 0, x_427); -return x_299; +x_751 = l_Lean_Expr_bvar___override(x_6); +lean_ctor_set(x_515, 0, x_751); +return x_515; } } else { -lean_object* x_428; uint8_t x_429; -x_428 = lean_ctor_get(x_299, 1); -lean_inc(x_428); -lean_dec(x_299); -x_429 = l_Lean_Occurrences_contains(x_2, x_293); -lean_dec(x_293); -if (x_429 == 0) +lean_object* x_752; uint8_t x_753; +x_752 = lean_ctor_get(x_515, 1); +lean_inc(x_752); +lean_dec(x_515); +x_753 = l_Lean_Occurrences_contains(x_2, x_509); +lean_dec(x_509); +if (x_753 == 0) { switch (lean_obj_tag(x_5)) { case 5: { -lean_object* x_430; lean_object* x_431; lean_object* x_432; -x_430 = lean_ctor_get(x_5, 0); -lean_inc(x_430); -x_431 = lean_ctor_get(x_5, 1); -lean_inc(x_431); +lean_object* x_754; lean_object* x_755; lean_object* x_756; +x_754 = lean_ctor_get(x_5, 0); +lean_inc(x_754); +x_755 = lean_ctor_get(x_5, 1); +lean_inc(x_755); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_754); lean_inc(x_1); -x_432 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_430, x_6, x_7, x_8, x_9, x_10, x_11, x_428); -if (lean_obj_tag(x_432) == 0) -{ -lean_object* x_433; lean_object* x_434; lean_object* x_435; -x_433 = lean_ctor_get(x_432, 0); -lean_inc(x_433); -x_434 = lean_ctor_get(x_432, 1); -lean_inc(x_434); -lean_dec(x_432); -x_435 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_431, x_6, x_7, x_8, x_9, x_10, x_11, x_434); -if (lean_obj_tag(x_435) == 0) -{ -lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; -x_436 = lean_ctor_get(x_435, 0); -lean_inc(x_436); -x_437 = lean_ctor_get(x_435, 1); -lean_inc(x_437); -if (lean_is_exclusive(x_435)) { - lean_ctor_release(x_435, 0); - lean_ctor_release(x_435, 1); - x_438 = x_435; +x_756 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_754, x_6, x_7, x_8, x_9, x_10, x_11, x_752); +if (lean_obj_tag(x_756) == 0) +{ +lean_object* x_757; lean_object* x_758; lean_object* x_759; +x_757 = lean_ctor_get(x_756, 0); +lean_inc(x_757); +x_758 = lean_ctor_get(x_756, 1); +lean_inc(x_758); +lean_dec(x_756); +lean_inc(x_755); +x_759 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_755, x_6, x_7, x_8, x_9, x_10, x_11, x_758); +if (lean_obj_tag(x_759) == 0) +{ +lean_object* x_760; lean_object* x_761; lean_object* x_762; size_t x_763; size_t x_764; uint8_t x_765; +x_760 = lean_ctor_get(x_759, 0); +lean_inc(x_760); +x_761 = lean_ctor_get(x_759, 1); +lean_inc(x_761); +if (lean_is_exclusive(x_759)) { + lean_ctor_release(x_759, 0); + lean_ctor_release(x_759, 1); + x_762 = x_759; +} else { + lean_dec_ref(x_759); + x_762 = lean_box(0); +} +x_763 = lean_ptr_addr(x_754); +lean_dec(x_754); +x_764 = lean_ptr_addr(x_757); +x_765 = lean_usize_dec_eq(x_763, x_764); +if (x_765 == 0) +{ +lean_object* x_766; lean_object* x_767; +lean_dec(x_755); +lean_dec(x_5); +x_766 = l_Lean_Expr_app___override(x_757, x_760); +if (lean_is_scalar(x_762)) { + x_767 = lean_alloc_ctor(0, 2, 0); +} else { + x_767 = x_762; +} +lean_ctor_set(x_767, 0, x_766); +lean_ctor_set(x_767, 1, x_761); +return x_767; +} +else +{ +size_t x_768; size_t x_769; uint8_t x_770; +x_768 = lean_ptr_addr(x_755); +lean_dec(x_755); +x_769 = lean_ptr_addr(x_760); +x_770 = lean_usize_dec_eq(x_768, x_769); +if (x_770 == 0) +{ +lean_object* x_771; lean_object* x_772; +lean_dec(x_5); +x_771 = l_Lean_Expr_app___override(x_757, x_760); +if (lean_is_scalar(x_762)) { + x_772 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_435); - x_438 = lean_box(0); + x_772 = x_762; } -x_439 = lean_expr_update_app(x_5, x_433, x_436); -if (lean_is_scalar(x_438)) { - x_440 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_772, 0, x_771); +lean_ctor_set(x_772, 1, x_761); +return x_772; +} +else +{ +lean_object* x_773; +lean_dec(x_760); +lean_dec(x_757); +if (lean_is_scalar(x_762)) { + x_773 = lean_alloc_ctor(0, 2, 0); } else { - x_440 = x_438; + x_773 = x_762; +} +lean_ctor_set(x_773, 0, x_5); +lean_ctor_set(x_773, 1, x_761); +return x_773; +} } -lean_ctor_set(x_440, 0, x_439); -lean_ctor_set(x_440, 1, x_437); -return x_440; } else { -lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; -lean_dec(x_433); +lean_object* x_774; lean_object* x_775; lean_object* x_776; lean_object* x_777; +lean_dec(x_757); +lean_dec(x_755); +lean_dec(x_754); lean_dec(x_5); -x_441 = lean_ctor_get(x_435, 0); -lean_inc(x_441); -x_442 = lean_ctor_get(x_435, 1); -lean_inc(x_442); -if (lean_is_exclusive(x_435)) { - lean_ctor_release(x_435, 0); - lean_ctor_release(x_435, 1); - x_443 = x_435; +x_774 = lean_ctor_get(x_759, 0); +lean_inc(x_774); +x_775 = lean_ctor_get(x_759, 1); +lean_inc(x_775); +if (lean_is_exclusive(x_759)) { + lean_ctor_release(x_759, 0); + lean_ctor_release(x_759, 1); + x_776 = x_759; } else { - lean_dec_ref(x_435); - x_443 = lean_box(0); + lean_dec_ref(x_759); + x_776 = lean_box(0); } -if (lean_is_scalar(x_443)) { - x_444 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_776)) { + x_777 = lean_alloc_ctor(1, 2, 0); } else { - x_444 = x_443; + x_777 = x_776; } -lean_ctor_set(x_444, 0, x_441); -lean_ctor_set(x_444, 1, x_442); -return x_444; +lean_ctor_set(x_777, 0, x_774); +lean_ctor_set(x_777, 1, x_775); +return x_777; } } else { -lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; -lean_dec(x_431); +lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; +lean_dec(x_755); +lean_dec(x_754); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -1507,350 +2607,591 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_445 = lean_ctor_get(x_432, 0); -lean_inc(x_445); -x_446 = lean_ctor_get(x_432, 1); -lean_inc(x_446); -if (lean_is_exclusive(x_432)) { - lean_ctor_release(x_432, 0); - lean_ctor_release(x_432, 1); - x_447 = x_432; +x_778 = lean_ctor_get(x_756, 0); +lean_inc(x_778); +x_779 = lean_ctor_get(x_756, 1); +lean_inc(x_779); +if (lean_is_exclusive(x_756)) { + lean_ctor_release(x_756, 0); + lean_ctor_release(x_756, 1); + x_780 = x_756; } else { - lean_dec_ref(x_432); - x_447 = lean_box(0); + lean_dec_ref(x_756); + x_780 = lean_box(0); } -if (lean_is_scalar(x_447)) { - x_448 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_780)) { + x_781 = lean_alloc_ctor(1, 2, 0); } else { - x_448 = x_447; + x_781 = x_780; } -lean_ctor_set(x_448, 0, x_445); -lean_ctor_set(x_448, 1, x_446); -return x_448; +lean_ctor_set(x_781, 0, x_778); +lean_ctor_set(x_781, 1, x_779); +return x_781; } } case 6: { -lean_object* x_449; lean_object* x_450; uint8_t x_451; lean_object* x_452; -x_449 = lean_ctor_get(x_5, 1); -lean_inc(x_449); -x_450 = lean_ctor_get(x_5, 2); -lean_inc(x_450); -x_451 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_object* x_782; lean_object* x_783; lean_object* x_784; uint8_t x_785; lean_object* x_786; +x_782 = lean_ctor_get(x_5, 0); +lean_inc(x_782); +x_783 = lean_ctor_get(x_5, 1); +lean_inc(x_783); +x_784 = lean_ctor_get(x_5, 2); +lean_inc(x_784); +x_785 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_783); lean_inc(x_1); -x_452 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_449, x_6, x_7, x_8, x_9, x_10, x_11, x_428); -if (lean_obj_tag(x_452) == 0) -{ -lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; -x_453 = lean_ctor_get(x_452, 0); -lean_inc(x_453); -x_454 = lean_ctor_get(x_452, 1); -lean_inc(x_454); -lean_dec(x_452); -x_455 = lean_nat_add(x_6, x_295); +x_786 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_783, x_6, x_7, x_8, x_9, x_10, x_11, x_752); +if (lean_obj_tag(x_786) == 0) +{ +lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; +x_787 = lean_ctor_get(x_786, 0); +lean_inc(x_787); +x_788 = lean_ctor_get(x_786, 1); +lean_inc(x_788); +lean_dec(x_786); +x_789 = lean_nat_add(x_6, x_511); lean_dec(x_6); -x_456 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_450, x_455, x_7, x_8, x_9, x_10, x_11, x_454); -if (lean_obj_tag(x_456) == 0) +lean_inc(x_784); +x_790 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_784, x_789, x_7, x_8, x_9, x_10, x_11, x_788); +if (lean_obj_tag(x_790) == 0) +{ +lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; size_t x_795; size_t x_796; uint8_t x_797; +x_791 = lean_ctor_get(x_790, 0); +lean_inc(x_791); +x_792 = lean_ctor_get(x_790, 1); +lean_inc(x_792); +if (lean_is_exclusive(x_790)) { + lean_ctor_release(x_790, 0); + lean_ctor_release(x_790, 1); + x_793 = x_790; +} else { + lean_dec_ref(x_790); + x_793 = lean_box(0); +} +lean_inc(x_784); +lean_inc(x_783); +lean_inc(x_782); +x_794 = l_Lean_Expr_lam___override(x_782, x_783, x_784, x_785); +x_795 = lean_ptr_addr(x_783); +lean_dec(x_783); +x_796 = lean_ptr_addr(x_787); +x_797 = lean_usize_dec_eq(x_795, x_796); +if (x_797 == 0) +{ +lean_object* x_798; lean_object* x_799; +lean_dec(x_794); +lean_dec(x_784); +x_798 = l_Lean_Expr_lam___override(x_782, x_787, x_791, x_785); +if (lean_is_scalar(x_793)) { + x_799 = lean_alloc_ctor(0, 2, 0); +} else { + x_799 = x_793; +} +lean_ctor_set(x_799, 0, x_798); +lean_ctor_set(x_799, 1, x_792); +return x_799; +} +else { -lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; -x_457 = lean_ctor_get(x_456, 0); -lean_inc(x_457); -x_458 = lean_ctor_get(x_456, 1); -lean_inc(x_458); -if (lean_is_exclusive(x_456)) { - lean_ctor_release(x_456, 0); - lean_ctor_release(x_456, 1); - x_459 = x_456; +size_t x_800; size_t x_801; uint8_t x_802; +x_800 = lean_ptr_addr(x_784); +lean_dec(x_784); +x_801 = lean_ptr_addr(x_791); +x_802 = lean_usize_dec_eq(x_800, x_801); +if (x_802 == 0) +{ +lean_object* x_803; lean_object* x_804; +lean_dec(x_794); +x_803 = l_Lean_Expr_lam___override(x_782, x_787, x_791, x_785); +if (lean_is_scalar(x_793)) { + x_804 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_456); - x_459 = lean_box(0); + x_804 = x_793; +} +lean_ctor_set(x_804, 0, x_803); +lean_ctor_set(x_804, 1, x_792); +return x_804; } -x_460 = lean_expr_update_lambda(x_5, x_451, x_453, x_457); -if (lean_is_scalar(x_459)) { - x_461 = lean_alloc_ctor(0, 2, 0); +else +{ +uint8_t x_805; +x_805 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_785, x_785); +if (x_805 == 0) +{ +lean_object* x_806; lean_object* x_807; +lean_dec(x_794); +x_806 = l_Lean_Expr_lam___override(x_782, x_787, x_791, x_785); +if (lean_is_scalar(x_793)) { + x_807 = lean_alloc_ctor(0, 2, 0); } else { - x_461 = x_459; + x_807 = x_793; } -lean_ctor_set(x_461, 0, x_460); -lean_ctor_set(x_461, 1, x_458); -return x_461; +lean_ctor_set(x_807, 0, x_806); +lean_ctor_set(x_807, 1, x_792); +return x_807; } else { -lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; -lean_dec(x_453); -lean_dec(x_5); -x_462 = lean_ctor_get(x_456, 0); -lean_inc(x_462); -x_463 = lean_ctor_get(x_456, 1); -lean_inc(x_463); -if (lean_is_exclusive(x_456)) { - lean_ctor_release(x_456, 0); - lean_ctor_release(x_456, 1); - x_464 = x_456; +lean_object* x_808; +lean_dec(x_791); +lean_dec(x_787); +lean_dec(x_782); +if (lean_is_scalar(x_793)) { + x_808 = lean_alloc_ctor(0, 2, 0); +} else { + x_808 = x_793; +} +lean_ctor_set(x_808, 0, x_794); +lean_ctor_set(x_808, 1, x_792); +return x_808; +} +} +} +} +else +{ +lean_object* x_809; lean_object* x_810; lean_object* x_811; lean_object* x_812; +lean_dec(x_787); +lean_dec(x_784); +lean_dec(x_783); +lean_dec(x_782); +x_809 = lean_ctor_get(x_790, 0); +lean_inc(x_809); +x_810 = lean_ctor_get(x_790, 1); +lean_inc(x_810); +if (lean_is_exclusive(x_790)) { + lean_ctor_release(x_790, 0); + lean_ctor_release(x_790, 1); + x_811 = x_790; } else { - lean_dec_ref(x_456); - x_464 = lean_box(0); + lean_dec_ref(x_790); + x_811 = lean_box(0); } -if (lean_is_scalar(x_464)) { - x_465 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_811)) { + x_812 = lean_alloc_ctor(1, 2, 0); } else { - x_465 = x_464; + x_812 = x_811; } -lean_ctor_set(x_465, 0, x_462); -lean_ctor_set(x_465, 1, x_463); -return x_465; +lean_ctor_set(x_812, 0, x_809); +lean_ctor_set(x_812, 1, x_810); +return x_812; } } else { -lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; -lean_dec(x_450); +lean_object* x_813; lean_object* x_814; lean_object* x_815; lean_object* x_816; +lean_dec(x_784); +lean_dec(x_783); +lean_dec(x_782); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_466 = lean_ctor_get(x_452, 0); -lean_inc(x_466); -x_467 = lean_ctor_get(x_452, 1); -lean_inc(x_467); -if (lean_is_exclusive(x_452)) { - lean_ctor_release(x_452, 0); - lean_ctor_release(x_452, 1); - x_468 = x_452; +x_813 = lean_ctor_get(x_786, 0); +lean_inc(x_813); +x_814 = lean_ctor_get(x_786, 1); +lean_inc(x_814); +if (lean_is_exclusive(x_786)) { + lean_ctor_release(x_786, 0); + lean_ctor_release(x_786, 1); + x_815 = x_786; } else { - lean_dec_ref(x_452); - x_468 = lean_box(0); + lean_dec_ref(x_786); + x_815 = lean_box(0); } -if (lean_is_scalar(x_468)) { - x_469 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_815)) { + x_816 = lean_alloc_ctor(1, 2, 0); } else { - x_469 = x_468; + x_816 = x_815; } -lean_ctor_set(x_469, 0, x_466); -lean_ctor_set(x_469, 1, x_467); -return x_469; +lean_ctor_set(x_816, 0, x_813); +lean_ctor_set(x_816, 1, x_814); +return x_816; } } case 7: { -lean_object* x_470; lean_object* x_471; uint8_t x_472; lean_object* x_473; -x_470 = lean_ctor_get(x_5, 1); -lean_inc(x_470); -x_471 = lean_ctor_get(x_5, 2); -lean_inc(x_471); -x_472 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_object* x_817; lean_object* x_818; lean_object* x_819; uint8_t x_820; lean_object* x_821; +x_817 = lean_ctor_get(x_5, 0); +lean_inc(x_817); +x_818 = lean_ctor_get(x_5, 1); +lean_inc(x_818); +x_819 = lean_ctor_get(x_5, 2); +lean_inc(x_819); +x_820 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_818); lean_inc(x_1); -x_473 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_470, x_6, x_7, x_8, x_9, x_10, x_11, x_428); -if (lean_obj_tag(x_473) == 0) -{ -lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; -x_474 = lean_ctor_get(x_473, 0); -lean_inc(x_474); -x_475 = lean_ctor_get(x_473, 1); -lean_inc(x_475); -lean_dec(x_473); -x_476 = lean_nat_add(x_6, x_295); +x_821 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_818, x_6, x_7, x_8, x_9, x_10, x_11, x_752); +if (lean_obj_tag(x_821) == 0) +{ +lean_object* x_822; lean_object* x_823; lean_object* x_824; lean_object* x_825; +x_822 = lean_ctor_get(x_821, 0); +lean_inc(x_822); +x_823 = lean_ctor_get(x_821, 1); +lean_inc(x_823); +lean_dec(x_821); +x_824 = lean_nat_add(x_6, x_511); lean_dec(x_6); -x_477 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_471, x_476, x_7, x_8, x_9, x_10, x_11, x_475); -if (lean_obj_tag(x_477) == 0) +lean_inc(x_819); +x_825 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_819, x_824, x_7, x_8, x_9, x_10, x_11, x_823); +if (lean_obj_tag(x_825) == 0) +{ +lean_object* x_826; lean_object* x_827; lean_object* x_828; lean_object* x_829; size_t x_830; size_t x_831; uint8_t x_832; +x_826 = lean_ctor_get(x_825, 0); +lean_inc(x_826); +x_827 = lean_ctor_get(x_825, 1); +lean_inc(x_827); +if (lean_is_exclusive(x_825)) { + lean_ctor_release(x_825, 0); + lean_ctor_release(x_825, 1); + x_828 = x_825; +} else { + lean_dec_ref(x_825); + x_828 = lean_box(0); +} +lean_inc(x_819); +lean_inc(x_818); +lean_inc(x_817); +x_829 = l_Lean_Expr_forallE___override(x_817, x_818, x_819, x_820); +x_830 = lean_ptr_addr(x_818); +lean_dec(x_818); +x_831 = lean_ptr_addr(x_822); +x_832 = lean_usize_dec_eq(x_830, x_831); +if (x_832 == 0) +{ +lean_object* x_833; lean_object* x_834; +lean_dec(x_829); +lean_dec(x_819); +x_833 = l_Lean_Expr_forallE___override(x_817, x_822, x_826, x_820); +if (lean_is_scalar(x_828)) { + x_834 = lean_alloc_ctor(0, 2, 0); +} else { + x_834 = x_828; +} +lean_ctor_set(x_834, 0, x_833); +lean_ctor_set(x_834, 1, x_827); +return x_834; +} +else { -lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; -x_478 = lean_ctor_get(x_477, 0); -lean_inc(x_478); -x_479 = lean_ctor_get(x_477, 1); -lean_inc(x_479); -if (lean_is_exclusive(x_477)) { - lean_ctor_release(x_477, 0); - lean_ctor_release(x_477, 1); - x_480 = x_477; +size_t x_835; size_t x_836; uint8_t x_837; +x_835 = lean_ptr_addr(x_819); +lean_dec(x_819); +x_836 = lean_ptr_addr(x_826); +x_837 = lean_usize_dec_eq(x_835, x_836); +if (x_837 == 0) +{ +lean_object* x_838; lean_object* x_839; +lean_dec(x_829); +x_838 = l_Lean_Expr_forallE___override(x_817, x_822, x_826, x_820); +if (lean_is_scalar(x_828)) { + x_839 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_477); - x_480 = lean_box(0); + x_839 = x_828; +} +lean_ctor_set(x_839, 0, x_838); +lean_ctor_set(x_839, 1, x_827); +return x_839; } -x_481 = lean_expr_update_forall(x_5, x_472, x_474, x_478); -if (lean_is_scalar(x_480)) { - x_482 = lean_alloc_ctor(0, 2, 0); +else +{ +uint8_t x_840; +x_840 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_820, x_820); +if (x_840 == 0) +{ +lean_object* x_841; lean_object* x_842; +lean_dec(x_829); +x_841 = l_Lean_Expr_forallE___override(x_817, x_822, x_826, x_820); +if (lean_is_scalar(x_828)) { + x_842 = lean_alloc_ctor(0, 2, 0); } else { - x_482 = x_480; + x_842 = x_828; } -lean_ctor_set(x_482, 0, x_481); -lean_ctor_set(x_482, 1, x_479); -return x_482; +lean_ctor_set(x_842, 0, x_841); +lean_ctor_set(x_842, 1, x_827); +return x_842; } else { -lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; -lean_dec(x_474); -lean_dec(x_5); -x_483 = lean_ctor_get(x_477, 0); -lean_inc(x_483); -x_484 = lean_ctor_get(x_477, 1); -lean_inc(x_484); -if (lean_is_exclusive(x_477)) { - lean_ctor_release(x_477, 0); - lean_ctor_release(x_477, 1); - x_485 = x_477; +lean_object* x_843; +lean_dec(x_826); +lean_dec(x_822); +lean_dec(x_817); +if (lean_is_scalar(x_828)) { + x_843 = lean_alloc_ctor(0, 2, 0); +} else { + x_843 = x_828; +} +lean_ctor_set(x_843, 0, x_829); +lean_ctor_set(x_843, 1, x_827); +return x_843; +} +} +} +} +else +{ +lean_object* x_844; lean_object* x_845; lean_object* x_846; lean_object* x_847; +lean_dec(x_822); +lean_dec(x_819); +lean_dec(x_818); +lean_dec(x_817); +x_844 = lean_ctor_get(x_825, 0); +lean_inc(x_844); +x_845 = lean_ctor_get(x_825, 1); +lean_inc(x_845); +if (lean_is_exclusive(x_825)) { + lean_ctor_release(x_825, 0); + lean_ctor_release(x_825, 1); + x_846 = x_825; } else { - lean_dec_ref(x_477); - x_485 = lean_box(0); + lean_dec_ref(x_825); + x_846 = lean_box(0); } -if (lean_is_scalar(x_485)) { - x_486 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_846)) { + x_847 = lean_alloc_ctor(1, 2, 0); } else { - x_486 = x_485; + x_847 = x_846; } -lean_ctor_set(x_486, 0, x_483); -lean_ctor_set(x_486, 1, x_484); -return x_486; +lean_ctor_set(x_847, 0, x_844); +lean_ctor_set(x_847, 1, x_845); +return x_847; } } else { -lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; -lean_dec(x_471); +lean_object* x_848; lean_object* x_849; lean_object* x_850; lean_object* x_851; +lean_dec(x_819); +lean_dec(x_818); +lean_dec(x_817); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_487 = lean_ctor_get(x_473, 0); -lean_inc(x_487); -x_488 = lean_ctor_get(x_473, 1); -lean_inc(x_488); -if (lean_is_exclusive(x_473)) { - lean_ctor_release(x_473, 0); - lean_ctor_release(x_473, 1); - x_489 = x_473; +x_848 = lean_ctor_get(x_821, 0); +lean_inc(x_848); +x_849 = lean_ctor_get(x_821, 1); +lean_inc(x_849); +if (lean_is_exclusive(x_821)) { + lean_ctor_release(x_821, 0); + lean_ctor_release(x_821, 1); + x_850 = x_821; } else { - lean_dec_ref(x_473); - x_489 = lean_box(0); + lean_dec_ref(x_821); + x_850 = lean_box(0); } -if (lean_is_scalar(x_489)) { - x_490 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_850)) { + x_851 = lean_alloc_ctor(1, 2, 0); } else { - x_490 = x_489; + x_851 = x_850; } -lean_ctor_set(x_490, 0, x_487); -lean_ctor_set(x_490, 1, x_488); -return x_490; +lean_ctor_set(x_851, 0, x_848); +lean_ctor_set(x_851, 1, x_849); +return x_851; } } case 8: { -lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; -x_491 = lean_ctor_get(x_5, 1); -lean_inc(x_491); -x_492 = lean_ctor_get(x_5, 2); -lean_inc(x_492); -x_493 = lean_ctor_get(x_5, 3); -lean_inc(x_493); +lean_object* x_852; lean_object* x_853; lean_object* x_854; lean_object* x_855; uint8_t x_856; lean_object* x_857; +x_852 = lean_ctor_get(x_5, 0); +lean_inc(x_852); +x_853 = lean_ctor_get(x_5, 1); +lean_inc(x_853); +x_854 = lean_ctor_get(x_5, 2); +lean_inc(x_854); +x_855 = lean_ctor_get(x_5, 3); +lean_inc(x_855); +x_856 = lean_ctor_get_uint8(x_5, sizeof(void*)*4 + 8); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_853); lean_inc(x_1); -x_494 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_491, x_6, x_7, x_8, x_9, x_10, x_11, x_428); -if (lean_obj_tag(x_494) == 0) -{ -lean_object* x_495; lean_object* x_496; lean_object* x_497; -x_495 = lean_ctor_get(x_494, 0); -lean_inc(x_495); -x_496 = lean_ctor_get(x_494, 1); -lean_inc(x_496); -lean_dec(x_494); +x_857 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_853, x_6, x_7, x_8, x_9, x_10, x_11, x_752); +if (lean_obj_tag(x_857) == 0) +{ +lean_object* x_858; lean_object* x_859; lean_object* x_860; +x_858 = lean_ctor_get(x_857, 0); +lean_inc(x_858); +x_859 = lean_ctor_get(x_857, 1); +lean_inc(x_859); +lean_dec(x_857); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_854); lean_inc(x_1); -x_497 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_492, x_6, x_7, x_8, x_9, x_10, x_11, x_496); -if (lean_obj_tag(x_497) == 0) -{ -lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; -x_498 = lean_ctor_get(x_497, 0); -lean_inc(x_498); -x_499 = lean_ctor_get(x_497, 1); -lean_inc(x_499); -lean_dec(x_497); -x_500 = lean_nat_add(x_6, x_295); +x_860 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_854, x_6, x_7, x_8, x_9, x_10, x_11, x_859); +if (lean_obj_tag(x_860) == 0) +{ +lean_object* x_861; lean_object* x_862; lean_object* x_863; lean_object* x_864; +x_861 = lean_ctor_get(x_860, 0); +lean_inc(x_861); +x_862 = lean_ctor_get(x_860, 1); +lean_inc(x_862); +lean_dec(x_860); +x_863 = lean_nat_add(x_6, x_511); lean_dec(x_6); -x_501 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_493, x_500, x_7, x_8, x_9, x_10, x_11, x_499); -if (lean_obj_tag(x_501) == 0) +lean_inc(x_855); +x_864 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_855, x_863, x_7, x_8, x_9, x_10, x_11, x_862); +if (lean_obj_tag(x_864) == 0) +{ +lean_object* x_865; lean_object* x_866; lean_object* x_867; size_t x_868; size_t x_869; uint8_t x_870; +x_865 = lean_ctor_get(x_864, 0); +lean_inc(x_865); +x_866 = lean_ctor_get(x_864, 1); +lean_inc(x_866); +if (lean_is_exclusive(x_864)) { + lean_ctor_release(x_864, 0); + lean_ctor_release(x_864, 1); + x_867 = x_864; +} else { + lean_dec_ref(x_864); + x_867 = lean_box(0); +} +x_868 = lean_ptr_addr(x_853); +lean_dec(x_853); +x_869 = lean_ptr_addr(x_858); +x_870 = lean_usize_dec_eq(x_868, x_869); +if (x_870 == 0) +{ +lean_object* x_871; lean_object* x_872; +lean_dec(x_855); +lean_dec(x_854); +lean_dec(x_5); +x_871 = l_Lean_Expr_letE___override(x_852, x_858, x_861, x_865, x_856); +if (lean_is_scalar(x_867)) { + x_872 = lean_alloc_ctor(0, 2, 0); +} else { + x_872 = x_867; +} +lean_ctor_set(x_872, 0, x_871); +lean_ctor_set(x_872, 1, x_866); +return x_872; +} +else { -lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; -x_502 = lean_ctor_get(x_501, 0); -lean_inc(x_502); -x_503 = lean_ctor_get(x_501, 1); -lean_inc(x_503); -if (lean_is_exclusive(x_501)) { - lean_ctor_release(x_501, 0); - lean_ctor_release(x_501, 1); - x_504 = x_501; +size_t x_873; size_t x_874; uint8_t x_875; +x_873 = lean_ptr_addr(x_854); +lean_dec(x_854); +x_874 = lean_ptr_addr(x_861); +x_875 = lean_usize_dec_eq(x_873, x_874); +if (x_875 == 0) +{ +lean_object* x_876; lean_object* x_877; +lean_dec(x_855); +lean_dec(x_5); +x_876 = l_Lean_Expr_letE___override(x_852, x_858, x_861, x_865, x_856); +if (lean_is_scalar(x_867)) { + x_877 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_501); - x_504 = lean_box(0); + x_877 = x_867; } -x_505 = lean_expr_update_let(x_5, x_495, x_498, x_502); -if (lean_is_scalar(x_504)) { - x_506 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_877, 0, x_876); +lean_ctor_set(x_877, 1, x_866); +return x_877; +} +else +{ +size_t x_878; size_t x_879; uint8_t x_880; +x_878 = lean_ptr_addr(x_855); +lean_dec(x_855); +x_879 = lean_ptr_addr(x_865); +x_880 = lean_usize_dec_eq(x_878, x_879); +if (x_880 == 0) +{ +lean_object* x_881; lean_object* x_882; +lean_dec(x_5); +x_881 = l_Lean_Expr_letE___override(x_852, x_858, x_861, x_865, x_856); +if (lean_is_scalar(x_867)) { + x_882 = lean_alloc_ctor(0, 2, 0); +} else { + x_882 = x_867; +} +lean_ctor_set(x_882, 0, x_881); +lean_ctor_set(x_882, 1, x_866); +return x_882; +} +else +{ +lean_object* x_883; +lean_dec(x_865); +lean_dec(x_861); +lean_dec(x_858); +lean_dec(x_852); +if (lean_is_scalar(x_867)) { + x_883 = lean_alloc_ctor(0, 2, 0); } else { - x_506 = x_504; + x_883 = x_867; +} +lean_ctor_set(x_883, 0, x_5); +lean_ctor_set(x_883, 1, x_866); +return x_883; +} +} } -lean_ctor_set(x_506, 0, x_505); -lean_ctor_set(x_506, 1, x_503); -return x_506; } else { -lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; -lean_dec(x_498); -lean_dec(x_495); +lean_object* x_884; lean_object* x_885; lean_object* x_886; lean_object* x_887; +lean_dec(x_861); +lean_dec(x_858); +lean_dec(x_855); +lean_dec(x_854); +lean_dec(x_853); +lean_dec(x_852); lean_dec(x_5); -x_507 = lean_ctor_get(x_501, 0); -lean_inc(x_507); -x_508 = lean_ctor_get(x_501, 1); -lean_inc(x_508); -if (lean_is_exclusive(x_501)) { - lean_ctor_release(x_501, 0); - lean_ctor_release(x_501, 1); - x_509 = x_501; +x_884 = lean_ctor_get(x_864, 0); +lean_inc(x_884); +x_885 = lean_ctor_get(x_864, 1); +lean_inc(x_885); +if (lean_is_exclusive(x_864)) { + lean_ctor_release(x_864, 0); + lean_ctor_release(x_864, 1); + x_886 = x_864; } else { - lean_dec_ref(x_501); - x_509 = lean_box(0); + lean_dec_ref(x_864); + x_886 = lean_box(0); } -if (lean_is_scalar(x_509)) { - x_510 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_886)) { + x_887 = lean_alloc_ctor(1, 2, 0); } else { - x_510 = x_509; + x_887 = x_886; } -lean_ctor_set(x_510, 0, x_507); -lean_ctor_set(x_510, 1, x_508); -return x_510; +lean_ctor_set(x_887, 0, x_884); +lean_ctor_set(x_887, 1, x_885); +return x_887; } } else { -lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; -lean_dec(x_495); -lean_dec(x_493); +lean_object* x_888; lean_object* x_889; lean_object* x_890; lean_object* x_891; +lean_dec(x_858); +lean_dec(x_855); +lean_dec(x_854); +lean_dec(x_853); +lean_dec(x_852); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -1858,33 +3199,35 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_511 = lean_ctor_get(x_497, 0); -lean_inc(x_511); -x_512 = lean_ctor_get(x_497, 1); -lean_inc(x_512); -if (lean_is_exclusive(x_497)) { - lean_ctor_release(x_497, 0); - lean_ctor_release(x_497, 1); - x_513 = x_497; +x_888 = lean_ctor_get(x_860, 0); +lean_inc(x_888); +x_889 = lean_ctor_get(x_860, 1); +lean_inc(x_889); +if (lean_is_exclusive(x_860)) { + lean_ctor_release(x_860, 0); + lean_ctor_release(x_860, 1); + x_890 = x_860; } else { - lean_dec_ref(x_497); - x_513 = lean_box(0); + lean_dec_ref(x_860); + x_890 = lean_box(0); } -if (lean_is_scalar(x_513)) { - x_514 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_890)) { + x_891 = lean_alloc_ctor(1, 2, 0); } else { - x_514 = x_513; + x_891 = x_890; } -lean_ctor_set(x_514, 0, x_511); -lean_ctor_set(x_514, 1, x_512); -return x_514; +lean_ctor_set(x_891, 0, x_888); +lean_ctor_set(x_891, 1, x_889); +return x_891; } } else { -lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; -lean_dec(x_493); -lean_dec(x_492); +lean_object* x_892; lean_object* x_893; lean_object* x_894; lean_object* x_895; +lean_dec(x_855); +lean_dec(x_854); +lean_dec(x_853); +lean_dec(x_852); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -1892,179 +3235,239 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_515 = lean_ctor_get(x_494, 0); -lean_inc(x_515); -x_516 = lean_ctor_get(x_494, 1); -lean_inc(x_516); -if (lean_is_exclusive(x_494)) { - lean_ctor_release(x_494, 0); - lean_ctor_release(x_494, 1); - x_517 = x_494; +x_892 = lean_ctor_get(x_857, 0); +lean_inc(x_892); +x_893 = lean_ctor_get(x_857, 1); +lean_inc(x_893); +if (lean_is_exclusive(x_857)) { + lean_ctor_release(x_857, 0); + lean_ctor_release(x_857, 1); + x_894 = x_857; } else { - lean_dec_ref(x_494); - x_517 = lean_box(0); + lean_dec_ref(x_857); + x_894 = lean_box(0); } -if (lean_is_scalar(x_517)) { - x_518 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_894)) { + x_895 = lean_alloc_ctor(1, 2, 0); } else { - x_518 = x_517; + x_895 = x_894; } -lean_ctor_set(x_518, 0, x_515); -lean_ctor_set(x_518, 1, x_516); -return x_518; +lean_ctor_set(x_895, 0, x_892); +lean_ctor_set(x_895, 1, x_893); +return x_895; } } case 10: { -lean_object* x_519; lean_object* x_520; -x_519 = lean_ctor_get(x_5, 1); -lean_inc(x_519); -x_520 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_519, x_6, x_7, x_8, x_9, x_10, x_11, x_428); -if (lean_obj_tag(x_520) == 0) +lean_object* x_896; lean_object* x_897; lean_object* x_898; +x_896 = lean_ctor_get(x_5, 0); +lean_inc(x_896); +x_897 = lean_ctor_get(x_5, 1); +lean_inc(x_897); +lean_inc(x_897); +x_898 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_897, x_6, x_7, x_8, x_9, x_10, x_11, x_752); +if (lean_obj_tag(x_898) == 0) +{ +lean_object* x_899; lean_object* x_900; lean_object* x_901; size_t x_902; size_t x_903; uint8_t x_904; +x_899 = lean_ctor_get(x_898, 0); +lean_inc(x_899); +x_900 = lean_ctor_get(x_898, 1); +lean_inc(x_900); +if (lean_is_exclusive(x_898)) { + lean_ctor_release(x_898, 0); + lean_ctor_release(x_898, 1); + x_901 = x_898; +} else { + lean_dec_ref(x_898); + x_901 = lean_box(0); +} +x_902 = lean_ptr_addr(x_897); +lean_dec(x_897); +x_903 = lean_ptr_addr(x_899); +x_904 = lean_usize_dec_eq(x_902, x_903); +if (x_904 == 0) { -lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; -x_521 = lean_ctor_get(x_520, 0); -lean_inc(x_521); -x_522 = lean_ctor_get(x_520, 1); -lean_inc(x_522); -if (lean_is_exclusive(x_520)) { - lean_ctor_release(x_520, 0); - lean_ctor_release(x_520, 1); - x_523 = x_520; +lean_object* x_905; lean_object* x_906; +lean_dec(x_5); +x_905 = l_Lean_Expr_mdata___override(x_896, x_899); +if (lean_is_scalar(x_901)) { + x_906 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_520); - x_523 = lean_box(0); + x_906 = x_901; } -x_524 = lean_expr_update_mdata(x_5, x_521); -if (lean_is_scalar(x_523)) { - x_525 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_906, 0, x_905); +lean_ctor_set(x_906, 1, x_900); +return x_906; +} +else +{ +lean_object* x_907; +lean_dec(x_899); +lean_dec(x_896); +if (lean_is_scalar(x_901)) { + x_907 = lean_alloc_ctor(0, 2, 0); } else { - x_525 = x_523; + x_907 = x_901; +} +lean_ctor_set(x_907, 0, x_5); +lean_ctor_set(x_907, 1, x_900); +return x_907; } -lean_ctor_set(x_525, 0, x_524); -lean_ctor_set(x_525, 1, x_522); -return x_525; } else { -lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; +lean_object* x_908; lean_object* x_909; lean_object* x_910; lean_object* x_911; +lean_dec(x_897); +lean_dec(x_896); lean_dec(x_5); -x_526 = lean_ctor_get(x_520, 0); -lean_inc(x_526); -x_527 = lean_ctor_get(x_520, 1); -lean_inc(x_527); -if (lean_is_exclusive(x_520)) { - lean_ctor_release(x_520, 0); - lean_ctor_release(x_520, 1); - x_528 = x_520; +x_908 = lean_ctor_get(x_898, 0); +lean_inc(x_908); +x_909 = lean_ctor_get(x_898, 1); +lean_inc(x_909); +if (lean_is_exclusive(x_898)) { + lean_ctor_release(x_898, 0); + lean_ctor_release(x_898, 1); + x_910 = x_898; } else { - lean_dec_ref(x_520); - x_528 = lean_box(0); + lean_dec_ref(x_898); + x_910 = lean_box(0); } -if (lean_is_scalar(x_528)) { - x_529 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_910)) { + x_911 = lean_alloc_ctor(1, 2, 0); } else { - x_529 = x_528; + x_911 = x_910; } -lean_ctor_set(x_529, 0, x_526); -lean_ctor_set(x_529, 1, x_527); -return x_529; +lean_ctor_set(x_911, 0, x_908); +lean_ctor_set(x_911, 1, x_909); +return x_911; } } case 11: { -lean_object* x_530; lean_object* x_531; -x_530 = lean_ctor_get(x_5, 2); -lean_inc(x_530); -x_531 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_530, x_6, x_7, x_8, x_9, x_10, x_11, x_428); -if (lean_obj_tag(x_531) == 0) -{ -lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; -x_532 = lean_ctor_get(x_531, 0); -lean_inc(x_532); -x_533 = lean_ctor_get(x_531, 1); -lean_inc(x_533); -if (lean_is_exclusive(x_531)) { - lean_ctor_release(x_531, 0); - lean_ctor_release(x_531, 1); - x_534 = x_531; +lean_object* x_912; lean_object* x_913; lean_object* x_914; lean_object* x_915; +x_912 = lean_ctor_get(x_5, 0); +lean_inc(x_912); +x_913 = lean_ctor_get(x_5, 1); +lean_inc(x_913); +x_914 = lean_ctor_get(x_5, 2); +lean_inc(x_914); +lean_inc(x_914); +x_915 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_914, x_6, x_7, x_8, x_9, x_10, x_11, x_752); +if (lean_obj_tag(x_915) == 0) +{ +lean_object* x_916; lean_object* x_917; lean_object* x_918; size_t x_919; size_t x_920; uint8_t x_921; +x_916 = lean_ctor_get(x_915, 0); +lean_inc(x_916); +x_917 = lean_ctor_get(x_915, 1); +lean_inc(x_917); +if (lean_is_exclusive(x_915)) { + lean_ctor_release(x_915, 0); + lean_ctor_release(x_915, 1); + x_918 = x_915; +} else { + lean_dec_ref(x_915); + x_918 = lean_box(0); +} +x_919 = lean_ptr_addr(x_914); +lean_dec(x_914); +x_920 = lean_ptr_addr(x_916); +x_921 = lean_usize_dec_eq(x_919, x_920); +if (x_921 == 0) +{ +lean_object* x_922; lean_object* x_923; +lean_dec(x_5); +x_922 = l_Lean_Expr_proj___override(x_912, x_913, x_916); +if (lean_is_scalar(x_918)) { + x_923 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_531); - x_534 = lean_box(0); + x_923 = x_918; +} +lean_ctor_set(x_923, 0, x_922); +lean_ctor_set(x_923, 1, x_917); +return x_923; } -x_535 = lean_expr_update_proj(x_5, x_532); -if (lean_is_scalar(x_534)) { - x_536 = lean_alloc_ctor(0, 2, 0); +else +{ +lean_object* x_924; +lean_dec(x_916); +lean_dec(x_913); +lean_dec(x_912); +if (lean_is_scalar(x_918)) { + x_924 = lean_alloc_ctor(0, 2, 0); } else { - x_536 = x_534; + x_924 = x_918; +} +lean_ctor_set(x_924, 0, x_5); +lean_ctor_set(x_924, 1, x_917); +return x_924; } -lean_ctor_set(x_536, 0, x_535); -lean_ctor_set(x_536, 1, x_533); -return x_536; } else { -lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; +lean_object* x_925; lean_object* x_926; lean_object* x_927; lean_object* x_928; +lean_dec(x_914); +lean_dec(x_913); +lean_dec(x_912); lean_dec(x_5); -x_537 = lean_ctor_get(x_531, 0); -lean_inc(x_537); -x_538 = lean_ctor_get(x_531, 1); -lean_inc(x_538); -if (lean_is_exclusive(x_531)) { - lean_ctor_release(x_531, 0); - lean_ctor_release(x_531, 1); - x_539 = x_531; +x_925 = lean_ctor_get(x_915, 0); +lean_inc(x_925); +x_926 = lean_ctor_get(x_915, 1); +lean_inc(x_926); +if (lean_is_exclusive(x_915)) { + lean_ctor_release(x_915, 0); + lean_ctor_release(x_915, 1); + x_927 = x_915; } else { - lean_dec_ref(x_531); - x_539 = lean_box(0); + lean_dec_ref(x_915); + x_927 = lean_box(0); } -if (lean_is_scalar(x_539)) { - x_540 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_927)) { + x_928 = lean_alloc_ctor(1, 2, 0); } else { - x_540 = x_539; + x_928 = x_927; } -lean_ctor_set(x_540, 0, x_537); -lean_ctor_set(x_540, 1, x_538); -return x_540; +lean_ctor_set(x_928, 0, x_925); +lean_ctor_set(x_928, 1, x_926); +return x_928; } } default: { -lean_object* x_541; +lean_object* x_929; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_1); -x_541 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_541, 0, x_5); -lean_ctor_set(x_541, 1, x_428); -return x_541; +x_929 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_929, 0, x_5); +lean_ctor_set(x_929, 1, x_752); +return x_929; } } } else { -lean_object* x_542; lean_object* x_543; +lean_object* x_930; lean_object* x_931; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_5); lean_dec(x_1); -x_542 = l_Lean_Expr_bvar___override(x_6); -x_543 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_543, 0, x_542); -lean_ctor_set(x_543, 1, x_428); -return x_543; +x_930 = l_Lean_Expr_bvar___override(x_6); +x_931 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_931, 0, x_930); +lean_ctor_set(x_931, 1, x_752); +return x_931; } } } } else { -uint8_t x_544; +uint8_t x_932; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2072,23 +3475,23 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_544 = !lean_is_exclusive(x_150); -if (x_544 == 0) +x_932 = !lean_is_exclusive(x_258); +if (x_932 == 0) { -return x_150; +return x_258; } else { -lean_object* x_545; lean_object* x_546; lean_object* x_547; -x_545 = lean_ctor_get(x_150, 0); -x_546 = lean_ctor_get(x_150, 1); -lean_inc(x_546); -lean_inc(x_545); -lean_dec(x_150); -x_547 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_547, 0, x_545); -lean_ctor_set(x_547, 1, x_546); -return x_547; +lean_object* x_933; lean_object* x_934; lean_object* x_935; +x_933 = lean_ctor_get(x_258, 0); +x_934 = lean_ctor_get(x_258, 1); +lean_inc(x_934); +lean_inc(x_933); +lean_dec(x_258); +x_935 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_935, 0, x_933); +lean_ctor_set(x_935, 1, x_934); +return x_935; } } } @@ -2099,431 +3502,867 @@ else switch (lean_obj_tag(x_5)) { case 5: { -lean_object* x_548; lean_object* x_549; lean_object* x_550; -x_548 = lean_ctor_get(x_5, 0); -lean_inc(x_548); -x_549 = lean_ctor_get(x_5, 1); -lean_inc(x_549); +lean_object* x_936; lean_object* x_937; lean_object* x_938; +x_936 = lean_ctor_get(x_5, 0); +lean_inc(x_936); +x_937 = lean_ctor_get(x_5, 1); +lean_inc(x_937); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_936); lean_inc(x_1); -x_550 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_548, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_550) == 0) +x_938 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_936, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_938) == 0) +{ +lean_object* x_939; lean_object* x_940; lean_object* x_941; +x_939 = lean_ctor_get(x_938, 0); +lean_inc(x_939); +x_940 = lean_ctor_get(x_938, 1); +lean_inc(x_940); +lean_dec(x_938); +lean_inc(x_937); +x_941 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_937, x_6, x_7, x_8, x_9, x_10, x_11, x_940); +if (lean_obj_tag(x_941) == 0) +{ +uint8_t x_942; +x_942 = !lean_is_exclusive(x_941); +if (x_942 == 0) +{ +lean_object* x_943; size_t x_944; size_t x_945; uint8_t x_946; +x_943 = lean_ctor_get(x_941, 0); +x_944 = lean_ptr_addr(x_936); +lean_dec(x_936); +x_945 = lean_ptr_addr(x_939); +x_946 = lean_usize_dec_eq(x_944, x_945); +if (x_946 == 0) +{ +lean_object* x_947; +lean_dec(x_937); +lean_dec(x_5); +x_947 = l_Lean_Expr_app___override(x_939, x_943); +lean_ctor_set(x_941, 0, x_947); +return x_941; +} +else { -lean_object* x_551; lean_object* x_552; lean_object* x_553; -x_551 = lean_ctor_get(x_550, 0); -lean_inc(x_551); -x_552 = lean_ctor_get(x_550, 1); -lean_inc(x_552); -lean_dec(x_550); -x_553 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_549, x_6, x_7, x_8, x_9, x_10, x_11, x_552); -if (lean_obj_tag(x_553) == 0) +size_t x_948; size_t x_949; uint8_t x_950; +x_948 = lean_ptr_addr(x_937); +lean_dec(x_937); +x_949 = lean_ptr_addr(x_943); +x_950 = lean_usize_dec_eq(x_948, x_949); +if (x_950 == 0) { -uint8_t x_554; -x_554 = !lean_is_exclusive(x_553); -if (x_554 == 0) +lean_object* x_951; +lean_dec(x_5); +x_951 = l_Lean_Expr_app___override(x_939, x_943); +lean_ctor_set(x_941, 0, x_951); +return x_941; +} +else { -lean_object* x_555; lean_object* x_556; -x_555 = lean_ctor_get(x_553, 0); -x_556 = lean_expr_update_app(x_5, x_551, x_555); -lean_ctor_set(x_553, 0, x_556); -return x_553; +lean_dec(x_943); +lean_dec(x_939); +lean_ctor_set(x_941, 0, x_5); +return x_941; +} +} } else { -lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; -x_557 = lean_ctor_get(x_553, 0); -x_558 = lean_ctor_get(x_553, 1); -lean_inc(x_558); -lean_inc(x_557); -lean_dec(x_553); -x_559 = lean_expr_update_app(x_5, x_551, x_557); -x_560 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_560, 0, x_559); -lean_ctor_set(x_560, 1, x_558); -return x_560; +lean_object* x_952; lean_object* x_953; size_t x_954; size_t x_955; uint8_t x_956; +x_952 = lean_ctor_get(x_941, 0); +x_953 = lean_ctor_get(x_941, 1); +lean_inc(x_953); +lean_inc(x_952); +lean_dec(x_941); +x_954 = lean_ptr_addr(x_936); +lean_dec(x_936); +x_955 = lean_ptr_addr(x_939); +x_956 = lean_usize_dec_eq(x_954, x_955); +if (x_956 == 0) +{ +lean_object* x_957; lean_object* x_958; +lean_dec(x_937); +lean_dec(x_5); +x_957 = l_Lean_Expr_app___override(x_939, x_952); +x_958 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_958, 0, x_957); +lean_ctor_set(x_958, 1, x_953); +return x_958; +} +else +{ +size_t x_959; size_t x_960; uint8_t x_961; +x_959 = lean_ptr_addr(x_937); +lean_dec(x_937); +x_960 = lean_ptr_addr(x_952); +x_961 = lean_usize_dec_eq(x_959, x_960); +if (x_961 == 0) +{ +lean_object* x_962; lean_object* x_963; +lean_dec(x_5); +x_962 = l_Lean_Expr_app___override(x_939, x_952); +x_963 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_963, 0, x_962); +lean_ctor_set(x_963, 1, x_953); +return x_963; +} +else +{ +lean_object* x_964; +lean_dec(x_952); +lean_dec(x_939); +x_964 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_964, 0, x_5); +lean_ctor_set(x_964, 1, x_953); +return x_964; +} +} } } else { -uint8_t x_561; -lean_dec(x_551); +uint8_t x_965; +lean_dec(x_939); +lean_dec(x_937); +lean_dec(x_936); lean_dec(x_5); -x_561 = !lean_is_exclusive(x_553); -if (x_561 == 0) +x_965 = !lean_is_exclusive(x_941); +if (x_965 == 0) { -return x_553; +return x_941; } else { -lean_object* x_562; lean_object* x_563; lean_object* x_564; -x_562 = lean_ctor_get(x_553, 0); -x_563 = lean_ctor_get(x_553, 1); -lean_inc(x_563); -lean_inc(x_562); -lean_dec(x_553); -x_564 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_564, 0, x_562); -lean_ctor_set(x_564, 1, x_563); -return x_564; +lean_object* x_966; lean_object* x_967; lean_object* x_968; +x_966 = lean_ctor_get(x_941, 0); +x_967 = lean_ctor_get(x_941, 1); +lean_inc(x_967); +lean_inc(x_966); +lean_dec(x_941); +x_968 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_968, 0, x_966); +lean_ctor_set(x_968, 1, x_967); +return x_968; +} +} +} +else +{ +uint8_t x_969; +lean_dec(x_937); +lean_dec(x_936); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_969 = !lean_is_exclusive(x_938); +if (x_969 == 0) +{ +return x_938; +} +else +{ +lean_object* x_970; lean_object* x_971; lean_object* x_972; +x_970 = lean_ctor_get(x_938, 0); +x_971 = lean_ctor_get(x_938, 1); +lean_inc(x_971); +lean_inc(x_970); +lean_dec(x_938); +x_972 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_972, 0, x_970); +lean_ctor_set(x_972, 1, x_971); +return x_972; +} +} +} +case 6: +{ +lean_object* x_973; lean_object* x_974; lean_object* x_975; uint8_t x_976; lean_object* x_977; +x_973 = lean_ctor_get(x_5, 0); +lean_inc(x_973); +x_974 = lean_ctor_get(x_5, 1); +lean_inc(x_974); +x_975 = lean_ctor_get(x_5, 2); +lean_inc(x_975); +x_976 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_6); +lean_inc(x_974); +lean_inc(x_1); +x_977 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_974, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_977) == 0) +{ +lean_object* x_978; lean_object* x_979; lean_object* x_980; lean_object* x_981; lean_object* x_982; +x_978 = lean_ctor_get(x_977, 0); +lean_inc(x_978); +x_979 = lean_ctor_get(x_977, 1); +lean_inc(x_979); +lean_dec(x_977); +x_980 = lean_unsigned_to_nat(1u); +x_981 = lean_nat_add(x_6, x_980); +lean_dec(x_6); +lean_inc(x_975); +x_982 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_975, x_981, x_7, x_8, x_9, x_10, x_11, x_979); +if (lean_obj_tag(x_982) == 0) +{ +uint8_t x_983; +x_983 = !lean_is_exclusive(x_982); +if (x_983 == 0) +{ +lean_object* x_984; lean_object* x_985; size_t x_986; size_t x_987; uint8_t x_988; +x_984 = lean_ctor_get(x_982, 0); +lean_inc(x_975); +lean_inc(x_974); +lean_inc(x_973); +x_985 = l_Lean_Expr_lam___override(x_973, x_974, x_975, x_976); +x_986 = lean_ptr_addr(x_974); +lean_dec(x_974); +x_987 = lean_ptr_addr(x_978); +x_988 = lean_usize_dec_eq(x_986, x_987); +if (x_988 == 0) +{ +lean_object* x_989; +lean_dec(x_985); +lean_dec(x_975); +x_989 = l_Lean_Expr_lam___override(x_973, x_978, x_984, x_976); +lean_ctor_set(x_982, 0, x_989); +return x_982; +} +else +{ +size_t x_990; size_t x_991; uint8_t x_992; +x_990 = lean_ptr_addr(x_975); +lean_dec(x_975); +x_991 = lean_ptr_addr(x_984); +x_992 = lean_usize_dec_eq(x_990, x_991); +if (x_992 == 0) +{ +lean_object* x_993; +lean_dec(x_985); +x_993 = l_Lean_Expr_lam___override(x_973, x_978, x_984, x_976); +lean_ctor_set(x_982, 0, x_993); +return x_982; +} +else +{ +uint8_t x_994; +x_994 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_976, x_976); +if (x_994 == 0) +{ +lean_object* x_995; +lean_dec(x_985); +x_995 = l_Lean_Expr_lam___override(x_973, x_978, x_984, x_976); +lean_ctor_set(x_982, 0, x_995); +return x_982; +} +else +{ +lean_dec(x_984); +lean_dec(x_978); +lean_dec(x_973); +lean_ctor_set(x_982, 0, x_985); +return x_982; +} +} +} +} +else +{ +lean_object* x_996; lean_object* x_997; lean_object* x_998; size_t x_999; size_t x_1000; uint8_t x_1001; +x_996 = lean_ctor_get(x_982, 0); +x_997 = lean_ctor_get(x_982, 1); +lean_inc(x_997); +lean_inc(x_996); +lean_dec(x_982); +lean_inc(x_975); +lean_inc(x_974); +lean_inc(x_973); +x_998 = l_Lean_Expr_lam___override(x_973, x_974, x_975, x_976); +x_999 = lean_ptr_addr(x_974); +lean_dec(x_974); +x_1000 = lean_ptr_addr(x_978); +x_1001 = lean_usize_dec_eq(x_999, x_1000); +if (x_1001 == 0) +{ +lean_object* x_1002; lean_object* x_1003; +lean_dec(x_998); +lean_dec(x_975); +x_1002 = l_Lean_Expr_lam___override(x_973, x_978, x_996, x_976); +x_1003 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1003, 0, x_1002); +lean_ctor_set(x_1003, 1, x_997); +return x_1003; +} +else +{ +size_t x_1004; size_t x_1005; uint8_t x_1006; +x_1004 = lean_ptr_addr(x_975); +lean_dec(x_975); +x_1005 = lean_ptr_addr(x_996); +x_1006 = lean_usize_dec_eq(x_1004, x_1005); +if (x_1006 == 0) +{ +lean_object* x_1007; lean_object* x_1008; +lean_dec(x_998); +x_1007 = l_Lean_Expr_lam___override(x_973, x_978, x_996, x_976); +x_1008 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1008, 0, x_1007); +lean_ctor_set(x_1008, 1, x_997); +return x_1008; +} +else +{ +uint8_t x_1009; +x_1009 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_976, x_976); +if (x_1009 == 0) +{ +lean_object* x_1010; lean_object* x_1011; +lean_dec(x_998); +x_1010 = l_Lean_Expr_lam___override(x_973, x_978, x_996, x_976); +x_1011 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1011, 0, x_1010); +lean_ctor_set(x_1011, 1, x_997); +return x_1011; +} +else +{ +lean_object* x_1012; +lean_dec(x_996); +lean_dec(x_978); +lean_dec(x_973); +x_1012 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1012, 0, x_998); +lean_ctor_set(x_1012, 1, x_997); +return x_1012; +} +} +} +} +} +else +{ +uint8_t x_1013; +lean_dec(x_978); +lean_dec(x_975); +lean_dec(x_974); +lean_dec(x_973); +x_1013 = !lean_is_exclusive(x_982); +if (x_1013 == 0) +{ +return x_982; +} +else +{ +lean_object* x_1014; lean_object* x_1015; lean_object* x_1016; +x_1014 = lean_ctor_get(x_982, 0); +x_1015 = lean_ctor_get(x_982, 1); +lean_inc(x_1015); +lean_inc(x_1014); +lean_dec(x_982); +x_1016 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1016, 0, x_1014); +lean_ctor_set(x_1016, 1, x_1015); +return x_1016; } } } else { -uint8_t x_565; -lean_dec(x_549); +uint8_t x_1017; +lean_dec(x_975); +lean_dec(x_974); +lean_dec(x_973); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_565 = !lean_is_exclusive(x_550); -if (x_565 == 0) +x_1017 = !lean_is_exclusive(x_977); +if (x_1017 == 0) { -return x_550; +return x_977; } else { -lean_object* x_566; lean_object* x_567; lean_object* x_568; -x_566 = lean_ctor_get(x_550, 0); -x_567 = lean_ctor_get(x_550, 1); -lean_inc(x_567); -lean_inc(x_566); -lean_dec(x_550); -x_568 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_568, 0, x_566); -lean_ctor_set(x_568, 1, x_567); -return x_568; +lean_object* x_1018; lean_object* x_1019; lean_object* x_1020; +x_1018 = lean_ctor_get(x_977, 0); +x_1019 = lean_ctor_get(x_977, 1); +lean_inc(x_1019); +lean_inc(x_1018); +lean_dec(x_977); +x_1020 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1020, 0, x_1018); +lean_ctor_set(x_1020, 1, x_1019); +return x_1020; } } } -case 6: +case 7: { -lean_object* x_569; lean_object* x_570; uint8_t x_571; lean_object* x_572; -x_569 = lean_ctor_get(x_5, 1); -lean_inc(x_569); -x_570 = lean_ctor_get(x_5, 2); -lean_inc(x_570); -x_571 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_object* x_1021; lean_object* x_1022; lean_object* x_1023; uint8_t x_1024; lean_object* x_1025; +x_1021 = lean_ctor_get(x_5, 0); +lean_inc(x_1021); +x_1022 = lean_ctor_get(x_5, 1); +lean_inc(x_1022); +x_1023 = lean_ctor_get(x_5, 2); +lean_inc(x_1023); +x_1024 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_1022); lean_inc(x_1); -x_572 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_569, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_572) == 0) -{ -lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_577; -x_573 = lean_ctor_get(x_572, 0); -lean_inc(x_573); -x_574 = lean_ctor_get(x_572, 1); -lean_inc(x_574); -lean_dec(x_572); -x_575 = lean_unsigned_to_nat(1u); -x_576 = lean_nat_add(x_6, x_575); +x_1025 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_1022, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_1025) == 0) +{ +lean_object* x_1026; lean_object* x_1027; lean_object* x_1028; lean_object* x_1029; lean_object* x_1030; +x_1026 = lean_ctor_get(x_1025, 0); +lean_inc(x_1026); +x_1027 = lean_ctor_get(x_1025, 1); +lean_inc(x_1027); +lean_dec(x_1025); +x_1028 = lean_unsigned_to_nat(1u); +x_1029 = lean_nat_add(x_6, x_1028); lean_dec(x_6); -x_577 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_570, x_576, x_7, x_8, x_9, x_10, x_11, x_574); -if (lean_obj_tag(x_577) == 0) -{ -uint8_t x_578; -x_578 = !lean_is_exclusive(x_577); -if (x_578 == 0) -{ -lean_object* x_579; lean_object* x_580; -x_579 = lean_ctor_get(x_577, 0); -x_580 = lean_expr_update_lambda(x_5, x_571, x_573, x_579); -lean_ctor_set(x_577, 0, x_580); -return x_577; +lean_inc(x_1023); +x_1030 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_1023, x_1029, x_7, x_8, x_9, x_10, x_11, x_1027); +if (lean_obj_tag(x_1030) == 0) +{ +uint8_t x_1031; +x_1031 = !lean_is_exclusive(x_1030); +if (x_1031 == 0) +{ +lean_object* x_1032; lean_object* x_1033; size_t x_1034; size_t x_1035; uint8_t x_1036; +x_1032 = lean_ctor_get(x_1030, 0); +lean_inc(x_1023); +lean_inc(x_1022); +lean_inc(x_1021); +x_1033 = l_Lean_Expr_forallE___override(x_1021, x_1022, x_1023, x_1024); +x_1034 = lean_ptr_addr(x_1022); +lean_dec(x_1022); +x_1035 = lean_ptr_addr(x_1026); +x_1036 = lean_usize_dec_eq(x_1034, x_1035); +if (x_1036 == 0) +{ +lean_object* x_1037; +lean_dec(x_1033); +lean_dec(x_1023); +x_1037 = l_Lean_Expr_forallE___override(x_1021, x_1026, x_1032, x_1024); +lean_ctor_set(x_1030, 0, x_1037); +return x_1030; } else { -lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; -x_581 = lean_ctor_get(x_577, 0); -x_582 = lean_ctor_get(x_577, 1); -lean_inc(x_582); -lean_inc(x_581); -lean_dec(x_577); -x_583 = lean_expr_update_lambda(x_5, x_571, x_573, x_581); -x_584 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_584, 0, x_583); -lean_ctor_set(x_584, 1, x_582); -return x_584; -} +size_t x_1038; size_t x_1039; uint8_t x_1040; +x_1038 = lean_ptr_addr(x_1023); +lean_dec(x_1023); +x_1039 = lean_ptr_addr(x_1032); +x_1040 = lean_usize_dec_eq(x_1038, x_1039); +if (x_1040 == 0) +{ +lean_object* x_1041; +lean_dec(x_1033); +x_1041 = l_Lean_Expr_forallE___override(x_1021, x_1026, x_1032, x_1024); +lean_ctor_set(x_1030, 0, x_1041); +return x_1030; } else { -uint8_t x_585; -lean_dec(x_573); -lean_dec(x_5); -x_585 = !lean_is_exclusive(x_577); -if (x_585 == 0) +uint8_t x_1042; +x_1042 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_1024, x_1024); +if (x_1042 == 0) { -return x_577; +lean_object* x_1043; +lean_dec(x_1033); +x_1043 = l_Lean_Expr_forallE___override(x_1021, x_1026, x_1032, x_1024); +lean_ctor_set(x_1030, 0, x_1043); +return x_1030; } else { -lean_object* x_586; lean_object* x_587; lean_object* x_588; -x_586 = lean_ctor_get(x_577, 0); -x_587 = lean_ctor_get(x_577, 1); -lean_inc(x_587); -lean_inc(x_586); -lean_dec(x_577); -x_588 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_588, 0, x_586); -lean_ctor_set(x_588, 1, x_587); -return x_588; +lean_dec(x_1032); +lean_dec(x_1026); +lean_dec(x_1021); +lean_ctor_set(x_1030, 0, x_1033); +return x_1030; +} } } } else { -uint8_t x_589; -lean_dec(x_570); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_589 = !lean_is_exclusive(x_572); -if (x_589 == 0) +lean_object* x_1044; lean_object* x_1045; lean_object* x_1046; size_t x_1047; size_t x_1048; uint8_t x_1049; +x_1044 = lean_ctor_get(x_1030, 0); +x_1045 = lean_ctor_get(x_1030, 1); +lean_inc(x_1045); +lean_inc(x_1044); +lean_dec(x_1030); +lean_inc(x_1023); +lean_inc(x_1022); +lean_inc(x_1021); +x_1046 = l_Lean_Expr_forallE___override(x_1021, x_1022, x_1023, x_1024); +x_1047 = lean_ptr_addr(x_1022); +lean_dec(x_1022); +x_1048 = lean_ptr_addr(x_1026); +x_1049 = lean_usize_dec_eq(x_1047, x_1048); +if (x_1049 == 0) { -return x_572; +lean_object* x_1050; lean_object* x_1051; +lean_dec(x_1046); +lean_dec(x_1023); +x_1050 = l_Lean_Expr_forallE___override(x_1021, x_1026, x_1044, x_1024); +x_1051 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1051, 0, x_1050); +lean_ctor_set(x_1051, 1, x_1045); +return x_1051; } else { -lean_object* x_590; lean_object* x_591; lean_object* x_592; -x_590 = lean_ctor_get(x_572, 0); -x_591 = lean_ctor_get(x_572, 1); -lean_inc(x_591); -lean_inc(x_590); -lean_dec(x_572); -x_592 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_592, 0, x_590); -lean_ctor_set(x_592, 1, x_591); -return x_592; -} -} -} -case 7: -{ -lean_object* x_593; lean_object* x_594; uint8_t x_595; lean_object* x_596; -x_593 = lean_ctor_get(x_5, 1); -lean_inc(x_593); -x_594 = lean_ctor_get(x_5, 2); -lean_inc(x_594); -x_595 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_6); -lean_inc(x_1); -x_596 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_593, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_596) == 0) +size_t x_1052; size_t x_1053; uint8_t x_1054; +x_1052 = lean_ptr_addr(x_1023); +lean_dec(x_1023); +x_1053 = lean_ptr_addr(x_1044); +x_1054 = lean_usize_dec_eq(x_1052, x_1053); +if (x_1054 == 0) { -lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; -x_597 = lean_ctor_get(x_596, 0); -lean_inc(x_597); -x_598 = lean_ctor_get(x_596, 1); -lean_inc(x_598); -lean_dec(x_596); -x_599 = lean_unsigned_to_nat(1u); -x_600 = lean_nat_add(x_6, x_599); -lean_dec(x_6); -x_601 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_594, x_600, x_7, x_8, x_9, x_10, x_11, x_598); -if (lean_obj_tag(x_601) == 0) +lean_object* x_1055; lean_object* x_1056; +lean_dec(x_1046); +x_1055 = l_Lean_Expr_forallE___override(x_1021, x_1026, x_1044, x_1024); +x_1056 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1056, 0, x_1055); +lean_ctor_set(x_1056, 1, x_1045); +return x_1056; +} +else { -uint8_t x_602; -x_602 = !lean_is_exclusive(x_601); -if (x_602 == 0) +uint8_t x_1057; +x_1057 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_1024, x_1024); +if (x_1057 == 0) { -lean_object* x_603; lean_object* x_604; -x_603 = lean_ctor_get(x_601, 0); -x_604 = lean_expr_update_forall(x_5, x_595, x_597, x_603); -lean_ctor_set(x_601, 0, x_604); -return x_601; +lean_object* x_1058; lean_object* x_1059; +lean_dec(x_1046); +x_1058 = l_Lean_Expr_forallE___override(x_1021, x_1026, x_1044, x_1024); +x_1059 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1059, 0, x_1058); +lean_ctor_set(x_1059, 1, x_1045); +return x_1059; } else { -lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; -x_605 = lean_ctor_get(x_601, 0); -x_606 = lean_ctor_get(x_601, 1); -lean_inc(x_606); -lean_inc(x_605); -lean_dec(x_601); -x_607 = lean_expr_update_forall(x_5, x_595, x_597, x_605); -x_608 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_608, 0, x_607); -lean_ctor_set(x_608, 1, x_606); -return x_608; +lean_object* x_1060; +lean_dec(x_1044); +lean_dec(x_1026); +lean_dec(x_1021); +x_1060 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1060, 0, x_1046); +lean_ctor_set(x_1060, 1, x_1045); +return x_1060; +} +} +} } } else { -uint8_t x_609; -lean_dec(x_597); -lean_dec(x_5); -x_609 = !lean_is_exclusive(x_601); -if (x_609 == 0) +uint8_t x_1061; +lean_dec(x_1026); +lean_dec(x_1023); +lean_dec(x_1022); +lean_dec(x_1021); +x_1061 = !lean_is_exclusive(x_1030); +if (x_1061 == 0) { -return x_601; +return x_1030; } else { -lean_object* x_610; lean_object* x_611; lean_object* x_612; -x_610 = lean_ctor_get(x_601, 0); -x_611 = lean_ctor_get(x_601, 1); -lean_inc(x_611); -lean_inc(x_610); -lean_dec(x_601); -x_612 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_612, 0, x_610); -lean_ctor_set(x_612, 1, x_611); -return x_612; +lean_object* x_1062; lean_object* x_1063; lean_object* x_1064; +x_1062 = lean_ctor_get(x_1030, 0); +x_1063 = lean_ctor_get(x_1030, 1); +lean_inc(x_1063); +lean_inc(x_1062); +lean_dec(x_1030); +x_1064 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1064, 0, x_1062); +lean_ctor_set(x_1064, 1, x_1063); +return x_1064; } } } else { -uint8_t x_613; -lean_dec(x_594); +uint8_t x_1065; +lean_dec(x_1023); +lean_dec(x_1022); +lean_dec(x_1021); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_613 = !lean_is_exclusive(x_596); -if (x_613 == 0) +x_1065 = !lean_is_exclusive(x_1025); +if (x_1065 == 0) { -return x_596; +return x_1025; } else { -lean_object* x_614; lean_object* x_615; lean_object* x_616; -x_614 = lean_ctor_get(x_596, 0); -x_615 = lean_ctor_get(x_596, 1); -lean_inc(x_615); -lean_inc(x_614); -lean_dec(x_596); -x_616 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_616, 0, x_614); -lean_ctor_set(x_616, 1, x_615); -return x_616; +lean_object* x_1066; lean_object* x_1067; lean_object* x_1068; +x_1066 = lean_ctor_get(x_1025, 0); +x_1067 = lean_ctor_get(x_1025, 1); +lean_inc(x_1067); +lean_inc(x_1066); +lean_dec(x_1025); +x_1068 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1068, 0, x_1066); +lean_ctor_set(x_1068, 1, x_1067); +return x_1068; } } } case 8: { -lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; -x_617 = lean_ctor_get(x_5, 1); -lean_inc(x_617); -x_618 = lean_ctor_get(x_5, 2); -lean_inc(x_618); -x_619 = lean_ctor_get(x_5, 3); -lean_inc(x_619); +lean_object* x_1069; lean_object* x_1070; lean_object* x_1071; lean_object* x_1072; uint8_t x_1073; lean_object* x_1074; +x_1069 = lean_ctor_get(x_5, 0); +lean_inc(x_1069); +x_1070 = lean_ctor_get(x_5, 1); +lean_inc(x_1070); +x_1071 = lean_ctor_get(x_5, 2); +lean_inc(x_1071); +x_1072 = lean_ctor_get(x_5, 3); +lean_inc(x_1072); +x_1073 = lean_ctor_get_uint8(x_5, sizeof(void*)*4 + 8); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_1070); lean_inc(x_1); -x_620 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_617, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_620) == 0) -{ -lean_object* x_621; lean_object* x_622; lean_object* x_623; -x_621 = lean_ctor_get(x_620, 0); -lean_inc(x_621); -x_622 = lean_ctor_get(x_620, 1); -lean_inc(x_622); -lean_dec(x_620); +x_1074 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_1070, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_1074) == 0) +{ +lean_object* x_1075; lean_object* x_1076; lean_object* x_1077; +x_1075 = lean_ctor_get(x_1074, 0); +lean_inc(x_1075); +x_1076 = lean_ctor_get(x_1074, 1); +lean_inc(x_1076); +lean_dec(x_1074); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_1071); lean_inc(x_1); -x_623 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_618, x_6, x_7, x_8, x_9, x_10, x_11, x_622); -if (lean_obj_tag(x_623) == 0) -{ -lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; -x_624 = lean_ctor_get(x_623, 0); -lean_inc(x_624); -x_625 = lean_ctor_get(x_623, 1); -lean_inc(x_625); -lean_dec(x_623); -x_626 = lean_unsigned_to_nat(1u); -x_627 = lean_nat_add(x_6, x_626); +x_1077 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_1071, x_6, x_7, x_8, x_9, x_10, x_11, x_1076); +if (lean_obj_tag(x_1077) == 0) +{ +lean_object* x_1078; lean_object* x_1079; lean_object* x_1080; lean_object* x_1081; lean_object* x_1082; +x_1078 = lean_ctor_get(x_1077, 0); +lean_inc(x_1078); +x_1079 = lean_ctor_get(x_1077, 1); +lean_inc(x_1079); +lean_dec(x_1077); +x_1080 = lean_unsigned_to_nat(1u); +x_1081 = lean_nat_add(x_6, x_1080); lean_dec(x_6); -x_628 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_619, x_627, x_7, x_8, x_9, x_10, x_11, x_625); -if (lean_obj_tag(x_628) == 0) +lean_inc(x_1072); +x_1082 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_1072, x_1081, x_7, x_8, x_9, x_10, x_11, x_1079); +if (lean_obj_tag(x_1082) == 0) +{ +uint8_t x_1083; +x_1083 = !lean_is_exclusive(x_1082); +if (x_1083 == 0) +{ +lean_object* x_1084; size_t x_1085; size_t x_1086; uint8_t x_1087; +x_1084 = lean_ctor_get(x_1082, 0); +x_1085 = lean_ptr_addr(x_1070); +lean_dec(x_1070); +x_1086 = lean_ptr_addr(x_1075); +x_1087 = lean_usize_dec_eq(x_1085, x_1086); +if (x_1087 == 0) +{ +lean_object* x_1088; +lean_dec(x_1072); +lean_dec(x_1071); +lean_dec(x_5); +x_1088 = l_Lean_Expr_letE___override(x_1069, x_1075, x_1078, x_1084, x_1073); +lean_ctor_set(x_1082, 0, x_1088); +return x_1082; +} +else { -uint8_t x_629; -x_629 = !lean_is_exclusive(x_628); -if (x_629 == 0) +size_t x_1089; size_t x_1090; uint8_t x_1091; +x_1089 = lean_ptr_addr(x_1071); +lean_dec(x_1071); +x_1090 = lean_ptr_addr(x_1078); +x_1091 = lean_usize_dec_eq(x_1089, x_1090); +if (x_1091 == 0) { -lean_object* x_630; lean_object* x_631; -x_630 = lean_ctor_get(x_628, 0); -x_631 = lean_expr_update_let(x_5, x_621, x_624, x_630); -lean_ctor_set(x_628, 0, x_631); -return x_628; +lean_object* x_1092; +lean_dec(x_1072); +lean_dec(x_5); +x_1092 = l_Lean_Expr_letE___override(x_1069, x_1075, x_1078, x_1084, x_1073); +lean_ctor_set(x_1082, 0, x_1092); +return x_1082; } else { -lean_object* x_632; lean_object* x_633; lean_object* x_634; lean_object* x_635; -x_632 = lean_ctor_get(x_628, 0); -x_633 = lean_ctor_get(x_628, 1); -lean_inc(x_633); -lean_inc(x_632); -lean_dec(x_628); -x_634 = lean_expr_update_let(x_5, x_621, x_624, x_632); -x_635 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_635, 0, x_634); -lean_ctor_set(x_635, 1, x_633); -return x_635; +size_t x_1093; size_t x_1094; uint8_t x_1095; +x_1093 = lean_ptr_addr(x_1072); +lean_dec(x_1072); +x_1094 = lean_ptr_addr(x_1084); +x_1095 = lean_usize_dec_eq(x_1093, x_1094); +if (x_1095 == 0) +{ +lean_object* x_1096; +lean_dec(x_5); +x_1096 = l_Lean_Expr_letE___override(x_1069, x_1075, x_1078, x_1084, x_1073); +lean_ctor_set(x_1082, 0, x_1096); +return x_1082; +} +else +{ +lean_dec(x_1084); +lean_dec(x_1078); +lean_dec(x_1075); +lean_dec(x_1069); +lean_ctor_set(x_1082, 0, x_5); +return x_1082; +} +} } } else { -uint8_t x_636; -lean_dec(x_624); -lean_dec(x_621); +lean_object* x_1097; lean_object* x_1098; size_t x_1099; size_t x_1100; uint8_t x_1101; +x_1097 = lean_ctor_get(x_1082, 0); +x_1098 = lean_ctor_get(x_1082, 1); +lean_inc(x_1098); +lean_inc(x_1097); +lean_dec(x_1082); +x_1099 = lean_ptr_addr(x_1070); +lean_dec(x_1070); +x_1100 = lean_ptr_addr(x_1075); +x_1101 = lean_usize_dec_eq(x_1099, x_1100); +if (x_1101 == 0) +{ +lean_object* x_1102; lean_object* x_1103; +lean_dec(x_1072); +lean_dec(x_1071); lean_dec(x_5); -x_636 = !lean_is_exclusive(x_628); -if (x_636 == 0) +x_1102 = l_Lean_Expr_letE___override(x_1069, x_1075, x_1078, x_1097, x_1073); +x_1103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1103, 0, x_1102); +lean_ctor_set(x_1103, 1, x_1098); +return x_1103; +} +else +{ +size_t x_1104; size_t x_1105; uint8_t x_1106; +x_1104 = lean_ptr_addr(x_1071); +lean_dec(x_1071); +x_1105 = lean_ptr_addr(x_1078); +x_1106 = lean_usize_dec_eq(x_1104, x_1105); +if (x_1106 == 0) +{ +lean_object* x_1107; lean_object* x_1108; +lean_dec(x_1072); +lean_dec(x_5); +x_1107 = l_Lean_Expr_letE___override(x_1069, x_1075, x_1078, x_1097, x_1073); +x_1108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1108, 0, x_1107); +lean_ctor_set(x_1108, 1, x_1098); +return x_1108; +} +else +{ +size_t x_1109; size_t x_1110; uint8_t x_1111; +x_1109 = lean_ptr_addr(x_1072); +lean_dec(x_1072); +x_1110 = lean_ptr_addr(x_1097); +x_1111 = lean_usize_dec_eq(x_1109, x_1110); +if (x_1111 == 0) { -return x_628; +lean_object* x_1112; lean_object* x_1113; +lean_dec(x_5); +x_1112 = l_Lean_Expr_letE___override(x_1069, x_1075, x_1078, x_1097, x_1073); +x_1113 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1113, 0, x_1112); +lean_ctor_set(x_1113, 1, x_1098); +return x_1113; } else { -lean_object* x_637; lean_object* x_638; lean_object* x_639; -x_637 = lean_ctor_get(x_628, 0); -x_638 = lean_ctor_get(x_628, 1); -lean_inc(x_638); -lean_inc(x_637); -lean_dec(x_628); -x_639 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_639, 0, x_637); -lean_ctor_set(x_639, 1, x_638); -return x_639; +lean_object* x_1114; +lean_dec(x_1097); +lean_dec(x_1078); +lean_dec(x_1075); +lean_dec(x_1069); +x_1114 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1114, 0, x_5); +lean_ctor_set(x_1114, 1, x_1098); +return x_1114; +} +} +} +} +} +else +{ +uint8_t x_1115; +lean_dec(x_1078); +lean_dec(x_1075); +lean_dec(x_1072); +lean_dec(x_1071); +lean_dec(x_1070); +lean_dec(x_1069); +lean_dec(x_5); +x_1115 = !lean_is_exclusive(x_1082); +if (x_1115 == 0) +{ +return x_1082; +} +else +{ +lean_object* x_1116; lean_object* x_1117; lean_object* x_1118; +x_1116 = lean_ctor_get(x_1082, 0); +x_1117 = lean_ctor_get(x_1082, 1); +lean_inc(x_1117); +lean_inc(x_1116); +lean_dec(x_1082); +x_1118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1118, 0, x_1116); +lean_ctor_set(x_1118, 1, x_1117); +return x_1118; } } } else { -uint8_t x_640; -lean_dec(x_621); -lean_dec(x_619); +uint8_t x_1119; +lean_dec(x_1075); +lean_dec(x_1072); +lean_dec(x_1071); +lean_dec(x_1070); +lean_dec(x_1069); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2531,31 +4370,33 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_640 = !lean_is_exclusive(x_623); -if (x_640 == 0) +x_1119 = !lean_is_exclusive(x_1077); +if (x_1119 == 0) { -return x_623; +return x_1077; } else { -lean_object* x_641; lean_object* x_642; lean_object* x_643; -x_641 = lean_ctor_get(x_623, 0); -x_642 = lean_ctor_get(x_623, 1); -lean_inc(x_642); -lean_inc(x_641); -lean_dec(x_623); -x_643 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_643, 0, x_641); -lean_ctor_set(x_643, 1, x_642); -return x_643; +lean_object* x_1120; lean_object* x_1121; lean_object* x_1122; +x_1120 = lean_ctor_get(x_1077, 0); +x_1121 = lean_ctor_get(x_1077, 1); +lean_inc(x_1121); +lean_inc(x_1120); +lean_dec(x_1077); +x_1122 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1122, 0, x_1120); +lean_ctor_set(x_1122, 1, x_1121); +return x_1122; } } } else { -uint8_t x_644; -lean_dec(x_619); -lean_dec(x_618); +uint8_t x_1123; +lean_dec(x_1072); +lean_dec(x_1071); +lean_dec(x_1070); +lean_dec(x_1069); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2563,157 +4404,242 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_644 = !lean_is_exclusive(x_620); -if (x_644 == 0) +x_1123 = !lean_is_exclusive(x_1074); +if (x_1123 == 0) { -return x_620; +return x_1074; } else { -lean_object* x_645; lean_object* x_646; lean_object* x_647; -x_645 = lean_ctor_get(x_620, 0); -x_646 = lean_ctor_get(x_620, 1); -lean_inc(x_646); -lean_inc(x_645); -lean_dec(x_620); -x_647 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_647, 0, x_645); -lean_ctor_set(x_647, 1, x_646); -return x_647; +lean_object* x_1124; lean_object* x_1125; lean_object* x_1126; +x_1124 = lean_ctor_get(x_1074, 0); +x_1125 = lean_ctor_get(x_1074, 1); +lean_inc(x_1125); +lean_inc(x_1124); +lean_dec(x_1074); +x_1126 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1126, 0, x_1124); +lean_ctor_set(x_1126, 1, x_1125); +return x_1126; } } } case 10: { -lean_object* x_648; lean_object* x_649; -x_648 = lean_ctor_get(x_5, 1); -lean_inc(x_648); -x_649 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_648, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_649) == 0) +lean_object* x_1127; lean_object* x_1128; lean_object* x_1129; +x_1127 = lean_ctor_get(x_5, 0); +lean_inc(x_1127); +x_1128 = lean_ctor_get(x_5, 1); +lean_inc(x_1128); +lean_inc(x_1128); +x_1129 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_1128, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_1129) == 0) +{ +uint8_t x_1130; +x_1130 = !lean_is_exclusive(x_1129); +if (x_1130 == 0) +{ +lean_object* x_1131; size_t x_1132; size_t x_1133; uint8_t x_1134; +x_1131 = lean_ctor_get(x_1129, 0); +x_1132 = lean_ptr_addr(x_1128); +lean_dec(x_1128); +x_1133 = lean_ptr_addr(x_1131); +x_1134 = lean_usize_dec_eq(x_1132, x_1133); +if (x_1134 == 0) +{ +lean_object* x_1135; +lean_dec(x_5); +x_1135 = l_Lean_Expr_mdata___override(x_1127, x_1131); +lean_ctor_set(x_1129, 0, x_1135); +return x_1129; +} +else +{ +lean_dec(x_1131); +lean_dec(x_1127); +lean_ctor_set(x_1129, 0, x_5); +return x_1129; +} +} +else { -uint8_t x_650; -x_650 = !lean_is_exclusive(x_649); -if (x_650 == 0) +lean_object* x_1136; lean_object* x_1137; size_t x_1138; size_t x_1139; uint8_t x_1140; +x_1136 = lean_ctor_get(x_1129, 0); +x_1137 = lean_ctor_get(x_1129, 1); +lean_inc(x_1137); +lean_inc(x_1136); +lean_dec(x_1129); +x_1138 = lean_ptr_addr(x_1128); +lean_dec(x_1128); +x_1139 = lean_ptr_addr(x_1136); +x_1140 = lean_usize_dec_eq(x_1138, x_1139); +if (x_1140 == 0) { -lean_object* x_651; lean_object* x_652; -x_651 = lean_ctor_get(x_649, 0); -x_652 = lean_expr_update_mdata(x_5, x_651); -lean_ctor_set(x_649, 0, x_652); -return x_649; +lean_object* x_1141; lean_object* x_1142; +lean_dec(x_5); +x_1141 = l_Lean_Expr_mdata___override(x_1127, x_1136); +x_1142 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1142, 0, x_1141); +lean_ctor_set(x_1142, 1, x_1137); +return x_1142; } else { -lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; -x_653 = lean_ctor_get(x_649, 0); -x_654 = lean_ctor_get(x_649, 1); -lean_inc(x_654); -lean_inc(x_653); -lean_dec(x_649); -x_655 = lean_expr_update_mdata(x_5, x_653); -x_656 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_656, 0, x_655); -lean_ctor_set(x_656, 1, x_654); -return x_656; +lean_object* x_1143; +lean_dec(x_1136); +lean_dec(x_1127); +x_1143 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1143, 0, x_5); +lean_ctor_set(x_1143, 1, x_1137); +return x_1143; +} } } else { -uint8_t x_657; +uint8_t x_1144; +lean_dec(x_1128); +lean_dec(x_1127); lean_dec(x_5); -x_657 = !lean_is_exclusive(x_649); -if (x_657 == 0) +x_1144 = !lean_is_exclusive(x_1129); +if (x_1144 == 0) { -return x_649; +return x_1129; } else { -lean_object* x_658; lean_object* x_659; lean_object* x_660; -x_658 = lean_ctor_get(x_649, 0); -x_659 = lean_ctor_get(x_649, 1); -lean_inc(x_659); -lean_inc(x_658); -lean_dec(x_649); -x_660 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_660, 0, x_658); -lean_ctor_set(x_660, 1, x_659); -return x_660; +lean_object* x_1145; lean_object* x_1146; lean_object* x_1147; +x_1145 = lean_ctor_get(x_1129, 0); +x_1146 = lean_ctor_get(x_1129, 1); +lean_inc(x_1146); +lean_inc(x_1145); +lean_dec(x_1129); +x_1147 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1147, 0, x_1145); +lean_ctor_set(x_1147, 1, x_1146); +return x_1147; } } } case 11: { -lean_object* x_661; lean_object* x_662; -x_661 = lean_ctor_get(x_5, 2); -lean_inc(x_661); -x_662 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_661, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_662) == 0) +lean_object* x_1148; lean_object* x_1149; lean_object* x_1150; lean_object* x_1151; +x_1148 = lean_ctor_get(x_5, 0); +lean_inc(x_1148); +x_1149 = lean_ctor_get(x_5, 1); +lean_inc(x_1149); +x_1150 = lean_ctor_get(x_5, 2); +lean_inc(x_1150); +lean_inc(x_1150); +x_1151 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_1150, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_1151) == 0) +{ +uint8_t x_1152; +x_1152 = !lean_is_exclusive(x_1151); +if (x_1152 == 0) +{ +lean_object* x_1153; size_t x_1154; size_t x_1155; uint8_t x_1156; +x_1153 = lean_ctor_get(x_1151, 0); +x_1154 = lean_ptr_addr(x_1150); +lean_dec(x_1150); +x_1155 = lean_ptr_addr(x_1153); +x_1156 = lean_usize_dec_eq(x_1154, x_1155); +if (x_1156 == 0) +{ +lean_object* x_1157; +lean_dec(x_5); +x_1157 = l_Lean_Expr_proj___override(x_1148, x_1149, x_1153); +lean_ctor_set(x_1151, 0, x_1157); +return x_1151; +} +else +{ +lean_dec(x_1153); +lean_dec(x_1149); +lean_dec(x_1148); +lean_ctor_set(x_1151, 0, x_5); +return x_1151; +} +} +else { -uint8_t x_663; -x_663 = !lean_is_exclusive(x_662); -if (x_663 == 0) +lean_object* x_1158; lean_object* x_1159; size_t x_1160; size_t x_1161; uint8_t x_1162; +x_1158 = lean_ctor_get(x_1151, 0); +x_1159 = lean_ctor_get(x_1151, 1); +lean_inc(x_1159); +lean_inc(x_1158); +lean_dec(x_1151); +x_1160 = lean_ptr_addr(x_1150); +lean_dec(x_1150); +x_1161 = lean_ptr_addr(x_1158); +x_1162 = lean_usize_dec_eq(x_1160, x_1161); +if (x_1162 == 0) { -lean_object* x_664; lean_object* x_665; -x_664 = lean_ctor_get(x_662, 0); -x_665 = lean_expr_update_proj(x_5, x_664); -lean_ctor_set(x_662, 0, x_665); -return x_662; +lean_object* x_1163; lean_object* x_1164; +lean_dec(x_5); +x_1163 = l_Lean_Expr_proj___override(x_1148, x_1149, x_1158); +x_1164 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1164, 0, x_1163); +lean_ctor_set(x_1164, 1, x_1159); +return x_1164; } else { -lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; -x_666 = lean_ctor_get(x_662, 0); -x_667 = lean_ctor_get(x_662, 1); -lean_inc(x_667); -lean_inc(x_666); -lean_dec(x_662); -x_668 = lean_expr_update_proj(x_5, x_666); -x_669 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_669, 0, x_668); -lean_ctor_set(x_669, 1, x_667); -return x_669; +lean_object* x_1165; +lean_dec(x_1158); +lean_dec(x_1149); +lean_dec(x_1148); +x_1165 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1165, 0, x_5); +lean_ctor_set(x_1165, 1, x_1159); +return x_1165; +} } } else { -uint8_t x_670; +uint8_t x_1166; +lean_dec(x_1150); +lean_dec(x_1149); +lean_dec(x_1148); lean_dec(x_5); -x_670 = !lean_is_exclusive(x_662); -if (x_670 == 0) +x_1166 = !lean_is_exclusive(x_1151); +if (x_1166 == 0) { -return x_662; +return x_1151; } else { -lean_object* x_671; lean_object* x_672; lean_object* x_673; -x_671 = lean_ctor_get(x_662, 0); -x_672 = lean_ctor_get(x_662, 1); -lean_inc(x_672); -lean_inc(x_671); -lean_dec(x_662); -x_673 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_673, 0, x_671); -lean_ctor_set(x_673, 1, x_672); -return x_673; +lean_object* x_1167; lean_object* x_1168; lean_object* x_1169; +x_1167 = lean_ctor_get(x_1151, 0); +x_1168 = lean_ctor_get(x_1151, 1); +lean_inc(x_1168); +lean_inc(x_1167); +lean_dec(x_1151); +x_1169 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1169, 0, x_1167); +lean_ctor_set(x_1169, 1, x_1168); +return x_1169; } } } default: { -lean_object* x_674; +lean_object* x_1170; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_1); -x_674 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_674, 0, x_5); -lean_ctor_set(x_674, 1, x_12); -return x_674; +x_1170 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1170, 0, x_5); +lean_ctor_set(x_1170, 1, x_12); +return x_1170; } } } -block_141: +block_249: { lean_dec(x_13); switch (lean_obj_tag(x_5)) { @@ -2729,421 +4655,857 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_14); lean_inc(x_1); x_16 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_14, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_16) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_18); -if (lean_obj_tag(x_19) == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_15); +x_19 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_18); +if (lean_obj_tag(x_19) == 0) +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) +{ +lean_object* x_21; size_t x_22; size_t x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_19, 0); +x_22 = lean_ptr_addr(x_14); +lean_dec(x_14); +x_23 = lean_ptr_addr(x_17); +x_24 = lean_usize_dec_eq(x_22, x_23); +if (x_24 == 0) +{ +lean_object* x_25; +lean_dec(x_15); +lean_dec(x_5); +x_25 = l_Lean_Expr_app___override(x_17, x_21); +lean_ctor_set(x_19, 0, x_25); +return x_19; +} +else +{ +size_t x_26; size_t x_27; uint8_t x_28; +x_26 = lean_ptr_addr(x_15); +lean_dec(x_15); +x_27 = lean_ptr_addr(x_21); +x_28 = lean_usize_dec_eq(x_26, x_27); +if (x_28 == 0) +{ +lean_object* x_29; +lean_dec(x_5); +x_29 = l_Lean_Expr_app___override(x_17, x_21); +lean_ctor_set(x_19, 0, x_29); +return x_19; +} +else +{ +lean_dec(x_21); +lean_dec(x_17); +lean_ctor_set(x_19, 0, x_5); +return x_19; +} +} +} +else +{ +lean_object* x_30; lean_object* x_31; size_t x_32; size_t x_33; uint8_t x_34; +x_30 = lean_ctor_get(x_19, 0); +x_31 = lean_ctor_get(x_19, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_19); +x_32 = lean_ptr_addr(x_14); +lean_dec(x_14); +x_33 = lean_ptr_addr(x_17); +x_34 = lean_usize_dec_eq(x_32, x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +lean_dec(x_15); +lean_dec(x_5); +x_35 = l_Lean_Expr_app___override(x_17, x_30); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_31); +return x_36; +} +else +{ +size_t x_37; size_t x_38; uint8_t x_39; +x_37 = lean_ptr_addr(x_15); +lean_dec(x_15); +x_38 = lean_ptr_addr(x_30); +x_39 = lean_usize_dec_eq(x_37, x_38); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; +lean_dec(x_5); +x_40 = l_Lean_Expr_app___override(x_17, x_30); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_31); +return x_41; +} +else +{ +lean_object* x_42; +lean_dec(x_30); +lean_dec(x_17); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_5); +lean_ctor_set(x_42, 1, x_31); +return x_42; +} +} +} +} +else +{ +uint8_t x_43; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_5); +x_43 = !lean_is_exclusive(x_19); +if (x_43 == 0) +{ +return x_19; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_19, 0); +x_45 = lean_ctor_get(x_19, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_19); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; +} +} +} +else +{ +uint8_t x_47; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_47 = !lean_is_exclusive(x_16); +if (x_47 == 0) +{ +return x_16; +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_16, 0); +x_49 = lean_ctor_get(x_16, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_16); +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; +} +} +} +case 6: +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; +x_51 = lean_ctor_get(x_5, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_5, 1); +lean_inc(x_52); +x_53 = lean_ctor_get(x_5, 2); +lean_inc(x_53); +x_54 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_6); +lean_inc(x_52); +lean_inc(x_1); +x_55 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_52, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_55) == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +lean_dec(x_55); +x_58 = lean_unsigned_to_nat(1u); +x_59 = lean_nat_add(x_6, x_58); +lean_dec(x_6); +lean_inc(x_53); +x_60 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_53, x_59, x_7, x_8, x_9, x_10, x_11, x_57); +if (lean_obj_tag(x_60) == 0) +{ +uint8_t x_61; +x_61 = !lean_is_exclusive(x_60); +if (x_61 == 0) +{ +lean_object* x_62; lean_object* x_63; size_t x_64; size_t x_65; uint8_t x_66; +x_62 = lean_ctor_get(x_60, 0); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +x_63 = l_Lean_Expr_lam___override(x_51, x_52, x_53, x_54); +x_64 = lean_ptr_addr(x_52); +lean_dec(x_52); +x_65 = lean_ptr_addr(x_56); +x_66 = lean_usize_dec_eq(x_64, x_65); +if (x_66 == 0) +{ +lean_object* x_67; +lean_dec(x_63); +lean_dec(x_53); +x_67 = l_Lean_Expr_lam___override(x_51, x_56, x_62, x_54); +lean_ctor_set(x_60, 0, x_67); +return x_60; +} +else +{ +size_t x_68; size_t x_69; uint8_t x_70; +x_68 = lean_ptr_addr(x_53); +lean_dec(x_53); +x_69 = lean_ptr_addr(x_62); +x_70 = lean_usize_dec_eq(x_68, x_69); +if (x_70 == 0) +{ +lean_object* x_71; +lean_dec(x_63); +x_71 = l_Lean_Expr_lam___override(x_51, x_56, x_62, x_54); +lean_ctor_set(x_60, 0, x_71); +return x_60; +} +else +{ +uint8_t x_72; +x_72 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_54, x_54); +if (x_72 == 0) +{ +lean_object* x_73; +lean_dec(x_63); +x_73 = l_Lean_Expr_lam___override(x_51, x_56, x_62, x_54); +lean_ctor_set(x_60, 0, x_73); +return x_60; +} +else +{ +lean_dec(x_62); +lean_dec(x_56); +lean_dec(x_51); +lean_ctor_set(x_60, 0, x_63); +return x_60; +} +} +} +} +else +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; size_t x_77; size_t x_78; uint8_t x_79; +x_74 = lean_ctor_get(x_60, 0); +x_75 = lean_ctor_get(x_60, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_60); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +x_76 = l_Lean_Expr_lam___override(x_51, x_52, x_53, x_54); +x_77 = lean_ptr_addr(x_52); +lean_dec(x_52); +x_78 = lean_ptr_addr(x_56); +x_79 = lean_usize_dec_eq(x_77, x_78); +if (x_79 == 0) +{ +lean_object* x_80; lean_object* x_81; +lean_dec(x_76); +lean_dec(x_53); +x_80 = l_Lean_Expr_lam___override(x_51, x_56, x_74, x_54); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_75); +return x_81; +} +else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +size_t x_82; size_t x_83; uint8_t x_84; +x_82 = lean_ptr_addr(x_53); +lean_dec(x_53); +x_83 = lean_ptr_addr(x_74); +x_84 = lean_usize_dec_eq(x_82, x_83); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; +lean_dec(x_76); +x_85 = l_Lean_Expr_lam___override(x_51, x_56, x_74, x_54); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_75); +return x_86; +} +else { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_expr_update_app(x_5, x_17, x_21); -lean_ctor_set(x_19, 0, x_22); -return x_19; +uint8_t x_87; +x_87 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_54, x_54); +if (x_87 == 0) +{ +lean_object* x_88; lean_object* x_89; +lean_dec(x_76); +x_88 = l_Lean_Expr_lam___override(x_51, x_56, x_74, x_54); +x_89 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_89, 0, x_88); +lean_ctor_set(x_89, 1, x_75); +return x_89; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_19, 0); -x_24 = lean_ctor_get(x_19, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_19); -x_25 = lean_expr_update_app(x_5, x_17, x_23); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -return x_26; +lean_object* x_90; +lean_dec(x_74); +lean_dec(x_56); +lean_dec(x_51); +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_76); +lean_ctor_set(x_90, 1, x_75); +return x_90; +} +} +} } } else { -uint8_t x_27; -lean_dec(x_17); -lean_dec(x_5); -x_27 = !lean_is_exclusive(x_19); -if (x_27 == 0) +uint8_t x_91; +lean_dec(x_56); +lean_dec(x_53); +lean_dec(x_52); +lean_dec(x_51); +x_91 = !lean_is_exclusive(x_60); +if (x_91 == 0) { -return x_19; +return x_60; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_19, 0); -x_29 = lean_ctor_get(x_19, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_19); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_92 = lean_ctor_get(x_60, 0); +x_93 = lean_ctor_get(x_60, 1); +lean_inc(x_93); +lean_inc(x_92); +lean_dec(x_60); +x_94 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_93); +return x_94; } } } else { -uint8_t x_31; -lean_dec(x_15); +uint8_t x_95; +lean_dec(x_53); +lean_dec(x_52); +lean_dec(x_51); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_31 = !lean_is_exclusive(x_16); -if (x_31 == 0) +x_95 = !lean_is_exclusive(x_55); +if (x_95 == 0) { -return x_16; +return x_55; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_16, 0); -x_33 = lean_ctor_get(x_16, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_16); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_55, 0); +x_97 = lean_ctor_get(x_55, 1); +lean_inc(x_97); +lean_inc(x_96); +lean_dec(x_55); +x_98 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_97); +return x_98; } } } -case 6: +case 7: { -lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; -x_35 = lean_ctor_get(x_5, 1); -lean_inc(x_35); -x_36 = lean_ctor_get(x_5, 2); -lean_inc(x_36); -x_37 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; +x_99 = lean_ctor_get(x_5, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_5, 1); +lean_inc(x_100); +x_101 = lean_ctor_get(x_5, 2); +lean_inc(x_101); +x_102 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); +lean_dec(x_5); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_100); lean_inc(x_1); -x_38 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_35, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_38) == 0) -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_39 = lean_ctor_get(x_38, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_38, 1); -lean_inc(x_40); -lean_dec(x_38); -x_41 = lean_unsigned_to_nat(1u); -x_42 = lean_nat_add(x_6, x_41); +x_103 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_100, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_103) == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_104 = lean_ctor_get(x_103, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_103, 1); +lean_inc(x_105); +lean_dec(x_103); +x_106 = lean_unsigned_to_nat(1u); +x_107 = lean_nat_add(x_6, x_106); lean_dec(x_6); -x_43 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_36, x_42, x_7, x_8, x_9, x_10, x_11, x_40); -if (lean_obj_tag(x_43) == 0) +lean_inc(x_101); +x_108 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_101, x_107, x_7, x_8, x_9, x_10, x_11, x_105); +if (lean_obj_tag(x_108) == 0) { -uint8_t x_44; -x_44 = !lean_is_exclusive(x_43); -if (x_44 == 0) +uint8_t x_109; +x_109 = !lean_is_exclusive(x_108); +if (x_109 == 0) { -lean_object* x_45; lean_object* x_46; -x_45 = lean_ctor_get(x_43, 0); -x_46 = lean_expr_update_lambda(x_5, x_37, x_39, x_45); -lean_ctor_set(x_43, 0, x_46); -return x_43; +lean_object* x_110; lean_object* x_111; size_t x_112; size_t x_113; uint8_t x_114; +x_110 = lean_ctor_get(x_108, 0); +lean_inc(x_101); +lean_inc(x_100); +lean_inc(x_99); +x_111 = l_Lean_Expr_forallE___override(x_99, x_100, x_101, x_102); +x_112 = lean_ptr_addr(x_100); +lean_dec(x_100); +x_113 = lean_ptr_addr(x_104); +x_114 = lean_usize_dec_eq(x_112, x_113); +if (x_114 == 0) +{ +lean_object* x_115; +lean_dec(x_111); +lean_dec(x_101); +x_115 = l_Lean_Expr_forallE___override(x_99, x_104, x_110, x_102); +lean_ctor_set(x_108, 0, x_115); +return x_108; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_47 = lean_ctor_get(x_43, 0); -x_48 = lean_ctor_get(x_43, 1); -lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_43); -x_49 = lean_expr_update_lambda(x_5, x_37, x_39, x_47); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_48); -return x_50; -} +size_t x_116; size_t x_117; uint8_t x_118; +x_116 = lean_ptr_addr(x_101); +lean_dec(x_101); +x_117 = lean_ptr_addr(x_110); +x_118 = lean_usize_dec_eq(x_116, x_117); +if (x_118 == 0) +{ +lean_object* x_119; +lean_dec(x_111); +x_119 = l_Lean_Expr_forallE___override(x_99, x_104, x_110, x_102); +lean_ctor_set(x_108, 0, x_119); +return x_108; } else { -uint8_t x_51; -lean_dec(x_39); -lean_dec(x_5); -x_51 = !lean_is_exclusive(x_43); -if (x_51 == 0) +uint8_t x_120; +x_120 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_102, x_102); +if (x_120 == 0) { -return x_43; +lean_object* x_121; +lean_dec(x_111); +x_121 = l_Lean_Expr_forallE___override(x_99, x_104, x_110, x_102); +lean_ctor_set(x_108, 0, x_121); +return x_108; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_43, 0); -x_53 = lean_ctor_get(x_43, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_43); -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_110); +lean_dec(x_104); +lean_dec(x_99); +lean_ctor_set(x_108, 0, x_111); +return x_108; +} } } } else { -uint8_t x_55; -lean_dec(x_36); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_55 = !lean_is_exclusive(x_38); -if (x_55 == 0) -{ -return x_38; +lean_object* x_122; lean_object* x_123; lean_object* x_124; size_t x_125; size_t x_126; uint8_t x_127; +x_122 = lean_ctor_get(x_108, 0); +x_123 = lean_ctor_get(x_108, 1); +lean_inc(x_123); +lean_inc(x_122); +lean_dec(x_108); +lean_inc(x_101); +lean_inc(x_100); +lean_inc(x_99); +x_124 = l_Lean_Expr_forallE___override(x_99, x_100, x_101, x_102); +x_125 = lean_ptr_addr(x_100); +lean_dec(x_100); +x_126 = lean_ptr_addr(x_104); +x_127 = lean_usize_dec_eq(x_125, x_126); +if (x_127 == 0) +{ +lean_object* x_128; lean_object* x_129; +lean_dec(x_124); +lean_dec(x_101); +x_128 = l_Lean_Expr_forallE___override(x_99, x_104, x_122, x_102); +x_129 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_129, 0, x_128); +lean_ctor_set(x_129, 1, x_123); +return x_129; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_38, 0); -x_57 = lean_ctor_get(x_38, 1); -lean_inc(x_57); -lean_inc(x_56); -lean_dec(x_38); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -return x_58; -} -} -} -case 7: +size_t x_130; size_t x_131; uint8_t x_132; +x_130 = lean_ptr_addr(x_101); +lean_dec(x_101); +x_131 = lean_ptr_addr(x_122); +x_132 = lean_usize_dec_eq(x_130, x_131); +if (x_132 == 0) { -lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; -x_59 = lean_ctor_get(x_5, 1); -lean_inc(x_59); -x_60 = lean_ctor_get(x_5, 2); -lean_inc(x_60); -x_61 = lean_ctor_get_uint8(x_5, sizeof(void*)*3 + 8); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_6); -lean_inc(x_1); -x_62 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_59, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_62) == 0) -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_63 = lean_ctor_get(x_62, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_62, 1); -lean_inc(x_64); -lean_dec(x_62); -x_65 = lean_unsigned_to_nat(1u); -x_66 = lean_nat_add(x_6, x_65); -lean_dec(x_6); -x_67 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_60, x_66, x_7, x_8, x_9, x_10, x_11, x_64); -if (lean_obj_tag(x_67) == 0) +lean_object* x_133; lean_object* x_134; +lean_dec(x_124); +x_133 = l_Lean_Expr_forallE___override(x_99, x_104, x_122, x_102); +x_134 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_134, 0, x_133); +lean_ctor_set(x_134, 1, x_123); +return x_134; +} +else { -uint8_t x_68; -x_68 = !lean_is_exclusive(x_67); -if (x_68 == 0) +uint8_t x_135; +x_135 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_102, x_102); +if (x_135 == 0) { -lean_object* x_69; lean_object* x_70; -x_69 = lean_ctor_get(x_67, 0); -x_70 = lean_expr_update_forall(x_5, x_61, x_63, x_69); -lean_ctor_set(x_67, 0, x_70); -return x_67; +lean_object* x_136; lean_object* x_137; +lean_dec(x_124); +x_136 = l_Lean_Expr_forallE___override(x_99, x_104, x_122, x_102); +x_137 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set(x_137, 1, x_123); +return x_137; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_71 = lean_ctor_get(x_67, 0); -x_72 = lean_ctor_get(x_67, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_67); -x_73 = lean_expr_update_forall(x_5, x_61, x_63, x_71); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_72); -return x_74; +lean_object* x_138; +lean_dec(x_122); +lean_dec(x_104); +lean_dec(x_99); +x_138 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_138, 0, x_124); +lean_ctor_set(x_138, 1, x_123); +return x_138; +} +} +} } } else { -uint8_t x_75; -lean_dec(x_63); -lean_dec(x_5); -x_75 = !lean_is_exclusive(x_67); -if (x_75 == 0) +uint8_t x_139; +lean_dec(x_104); +lean_dec(x_101); +lean_dec(x_100); +lean_dec(x_99); +x_139 = !lean_is_exclusive(x_108); +if (x_139 == 0) { -return x_67; +return x_108; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_67, 0); -x_77 = lean_ctor_get(x_67, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_67); -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_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_108, 0); +x_141 = lean_ctor_get(x_108, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_108); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } } else { -uint8_t x_79; -lean_dec(x_60); +uint8_t x_143; +lean_dec(x_101); +lean_dec(x_100); +lean_dec(x_99); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_79 = !lean_is_exclusive(x_62); -if (x_79 == 0) +x_143 = !lean_is_exclusive(x_103); +if (x_143 == 0) { -return x_62; +return x_103; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_80 = lean_ctor_get(x_62, 0); -x_81 = lean_ctor_get(x_62, 1); -lean_inc(x_81); -lean_inc(x_80); -lean_dec(x_62); -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -return x_82; +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_103, 0); +x_145 = lean_ctor_get(x_103, 1); +lean_inc(x_145); +lean_inc(x_144); +lean_dec(x_103); +x_146 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +return x_146; } } } case 8: { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_83 = lean_ctor_get(x_5, 1); -lean_inc(x_83); -x_84 = lean_ctor_get(x_5, 2); -lean_inc(x_84); -x_85 = lean_ctor_get(x_5, 3); -lean_inc(x_85); +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; uint8_t x_151; lean_object* x_152; +x_147 = lean_ctor_get(x_5, 0); +lean_inc(x_147); +x_148 = lean_ctor_get(x_5, 1); +lean_inc(x_148); +x_149 = lean_ctor_get(x_5, 2); +lean_inc(x_149); +x_150 = lean_ctor_get(x_5, 3); +lean_inc(x_150); +x_151 = lean_ctor_get_uint8(x_5, sizeof(void*)*4 + 8); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_148); lean_inc(x_1); -x_86 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_83, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_86) == 0) +x_152 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_148, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_152) == 0) { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); -lean_inc(x_88); -lean_dec(x_86); +lean_object* x_153; lean_object* x_154; lean_object* x_155; +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +x_154 = lean_ctor_get(x_152, 1); +lean_inc(x_154); +lean_dec(x_152); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); +lean_inc(x_149); lean_inc(x_1); -x_89 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_84, x_6, x_7, x_8, x_9, x_10, x_11, x_88); -if (lean_obj_tag(x_89) == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_89, 1); -lean_inc(x_91); -lean_dec(x_89); -x_92 = lean_unsigned_to_nat(1u); -x_93 = lean_nat_add(x_6, x_92); +x_155 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_149, x_6, x_7, x_8, x_9, x_10, x_11, x_154); +if (lean_obj_tag(x_155) == 0) +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; +x_156 = lean_ctor_get(x_155, 0); +lean_inc(x_156); +x_157 = lean_ctor_get(x_155, 1); +lean_inc(x_157); +lean_dec(x_155); +x_158 = lean_unsigned_to_nat(1u); +x_159 = lean_nat_add(x_6, x_158); lean_dec(x_6); -x_94 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_85, x_93, x_7, x_8, x_9, x_10, x_11, x_91); -if (lean_obj_tag(x_94) == 0) +lean_inc(x_150); +x_160 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_150, x_159, x_7, x_8, x_9, x_10, x_11, x_157); +if (lean_obj_tag(x_160) == 0) +{ +uint8_t x_161; +x_161 = !lean_is_exclusive(x_160); +if (x_161 == 0) +{ +lean_object* x_162; size_t x_163; size_t x_164; uint8_t x_165; +x_162 = lean_ctor_get(x_160, 0); +x_163 = lean_ptr_addr(x_148); +lean_dec(x_148); +x_164 = lean_ptr_addr(x_153); +x_165 = lean_usize_dec_eq(x_163, x_164); +if (x_165 == 0) +{ +lean_object* x_166; +lean_dec(x_150); +lean_dec(x_149); +lean_dec(x_5); +x_166 = l_Lean_Expr_letE___override(x_147, x_153, x_156, x_162, x_151); +lean_ctor_set(x_160, 0, x_166); +return x_160; +} +else { -uint8_t x_95; -x_95 = !lean_is_exclusive(x_94); -if (x_95 == 0) +size_t x_167; size_t x_168; uint8_t x_169; +x_167 = lean_ptr_addr(x_149); +lean_dec(x_149); +x_168 = lean_ptr_addr(x_156); +x_169 = lean_usize_dec_eq(x_167, x_168); +if (x_169 == 0) { -lean_object* x_96; lean_object* x_97; -x_96 = lean_ctor_get(x_94, 0); -x_97 = lean_expr_update_let(x_5, x_87, x_90, x_96); -lean_ctor_set(x_94, 0, x_97); -return x_94; +lean_object* x_170; +lean_dec(x_150); +lean_dec(x_5); +x_170 = l_Lean_Expr_letE___override(x_147, x_153, x_156, x_162, x_151); +lean_ctor_set(x_160, 0, x_170); +return x_160; } else { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_98 = lean_ctor_get(x_94, 0); -x_99 = lean_ctor_get(x_94, 1); -lean_inc(x_99); -lean_inc(x_98); -lean_dec(x_94); -x_100 = lean_expr_update_let(x_5, x_87, x_90, x_98); -x_101 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_101, 0, x_100); -lean_ctor_set(x_101, 1, x_99); -return x_101; +size_t x_171; size_t x_172; uint8_t x_173; +x_171 = lean_ptr_addr(x_150); +lean_dec(x_150); +x_172 = lean_ptr_addr(x_162); +x_173 = lean_usize_dec_eq(x_171, x_172); +if (x_173 == 0) +{ +lean_object* x_174; +lean_dec(x_5); +x_174 = l_Lean_Expr_letE___override(x_147, x_153, x_156, x_162, x_151); +lean_ctor_set(x_160, 0, x_174); +return x_160; +} +else +{ +lean_dec(x_162); +lean_dec(x_156); +lean_dec(x_153); +lean_dec(x_147); +lean_ctor_set(x_160, 0, x_5); +return x_160; +} +} } } else { -uint8_t x_102; -lean_dec(x_90); -lean_dec(x_87); +lean_object* x_175; lean_object* x_176; size_t x_177; size_t x_178; uint8_t x_179; +x_175 = lean_ctor_get(x_160, 0); +x_176 = lean_ctor_get(x_160, 1); +lean_inc(x_176); +lean_inc(x_175); +lean_dec(x_160); +x_177 = lean_ptr_addr(x_148); +lean_dec(x_148); +x_178 = lean_ptr_addr(x_153); +x_179 = lean_usize_dec_eq(x_177, x_178); +if (x_179 == 0) +{ +lean_object* x_180; lean_object* x_181; +lean_dec(x_150); +lean_dec(x_149); lean_dec(x_5); -x_102 = !lean_is_exclusive(x_94); -if (x_102 == 0) +x_180 = l_Lean_Expr_letE___override(x_147, x_153, x_156, x_175, x_151); +x_181 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_181, 0, x_180); +lean_ctor_set(x_181, 1, x_176); +return x_181; +} +else { -return x_94; +size_t x_182; size_t x_183; uint8_t x_184; +x_182 = lean_ptr_addr(x_149); +lean_dec(x_149); +x_183 = lean_ptr_addr(x_156); +x_184 = lean_usize_dec_eq(x_182, x_183); +if (x_184 == 0) +{ +lean_object* x_185; lean_object* x_186; +lean_dec(x_150); +lean_dec(x_5); +x_185 = l_Lean_Expr_letE___override(x_147, x_153, x_156, x_175, x_151); +x_186 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_186, 0, x_185); +lean_ctor_set(x_186, 1, x_176); +return x_186; } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_103 = lean_ctor_get(x_94, 0); -x_104 = lean_ctor_get(x_94, 1); -lean_inc(x_104); -lean_inc(x_103); -lean_dec(x_94); -x_105 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_104); -return x_105; +size_t x_187; size_t x_188; uint8_t x_189; +x_187 = lean_ptr_addr(x_150); +lean_dec(x_150); +x_188 = lean_ptr_addr(x_175); +x_189 = lean_usize_dec_eq(x_187, x_188); +if (x_189 == 0) +{ +lean_object* x_190; lean_object* x_191; +lean_dec(x_5); +x_190 = l_Lean_Expr_letE___override(x_147, x_153, x_156, x_175, x_151); +x_191 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_191, 0, x_190); +lean_ctor_set(x_191, 1, x_176); +return x_191; +} +else +{ +lean_object* x_192; +lean_dec(x_175); +lean_dec(x_156); +lean_dec(x_153); +lean_dec(x_147); +x_192 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_192, 0, x_5); +lean_ctor_set(x_192, 1, x_176); +return x_192; +} +} +} +} +} +else +{ +uint8_t x_193; +lean_dec(x_156); +lean_dec(x_153); +lean_dec(x_150); +lean_dec(x_149); +lean_dec(x_148); +lean_dec(x_147); +lean_dec(x_5); +x_193 = !lean_is_exclusive(x_160); +if (x_193 == 0) +{ +return x_160; +} +else +{ +lean_object* x_194; lean_object* x_195; lean_object* x_196; +x_194 = lean_ctor_get(x_160, 0); +x_195 = lean_ctor_get(x_160, 1); +lean_inc(x_195); +lean_inc(x_194); +lean_dec(x_160); +x_196 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_196, 0, x_194); +lean_ctor_set(x_196, 1, x_195); +return x_196; } } } else { -uint8_t x_106; -lean_dec(x_87); -lean_dec(x_85); +uint8_t x_197; +lean_dec(x_153); +lean_dec(x_150); +lean_dec(x_149); +lean_dec(x_148); +lean_dec(x_147); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -3151,31 +5513,33 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_106 = !lean_is_exclusive(x_89); -if (x_106 == 0) +x_197 = !lean_is_exclusive(x_155); +if (x_197 == 0) { -return x_89; +return x_155; } else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_107 = lean_ctor_get(x_89, 0); -x_108 = lean_ctor_get(x_89, 1); -lean_inc(x_108); -lean_inc(x_107); -lean_dec(x_89); -x_109 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_109, 0, x_107); -lean_ctor_set(x_109, 1, x_108); -return x_109; +lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_198 = lean_ctor_get(x_155, 0); +x_199 = lean_ctor_get(x_155, 1); +lean_inc(x_199); +lean_inc(x_198); +lean_dec(x_155); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_198); +lean_ctor_set(x_200, 1, x_199); +return x_200; } } } else { -uint8_t x_110; -lean_dec(x_85); -lean_dec(x_84); +uint8_t x_201; +lean_dec(x_150); +lean_dec(x_149); +lean_dec(x_148); +lean_dec(x_147); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -3183,153 +5547,238 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_110 = !lean_is_exclusive(x_86); -if (x_110 == 0) +x_201 = !lean_is_exclusive(x_152); +if (x_201 == 0) { -return x_86; +return x_152; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_111 = lean_ctor_get(x_86, 0); -x_112 = lean_ctor_get(x_86, 1); -lean_inc(x_112); -lean_inc(x_111); -lean_dec(x_86); -x_113 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_113, 0, x_111); -lean_ctor_set(x_113, 1, x_112); -return x_113; +lean_object* x_202; lean_object* x_203; lean_object* x_204; +x_202 = lean_ctor_get(x_152, 0); +x_203 = lean_ctor_get(x_152, 1); +lean_inc(x_203); +lean_inc(x_202); +lean_dec(x_152); +x_204 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_204, 0, x_202); +lean_ctor_set(x_204, 1, x_203); +return x_204; } } } case 10: { -lean_object* x_114; lean_object* x_115; -x_114 = lean_ctor_get(x_5, 1); -lean_inc(x_114); -x_115 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_114, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_115) == 0) +lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_205 = lean_ctor_get(x_5, 0); +lean_inc(x_205); +x_206 = lean_ctor_get(x_5, 1); +lean_inc(x_206); +lean_inc(x_206); +x_207 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_206, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_207) == 0) +{ +uint8_t x_208; +x_208 = !lean_is_exclusive(x_207); +if (x_208 == 0) +{ +lean_object* x_209; size_t x_210; size_t x_211; uint8_t x_212; +x_209 = lean_ctor_get(x_207, 0); +x_210 = lean_ptr_addr(x_206); +lean_dec(x_206); +x_211 = lean_ptr_addr(x_209); +x_212 = lean_usize_dec_eq(x_210, x_211); +if (x_212 == 0) +{ +lean_object* x_213; +lean_dec(x_5); +x_213 = l_Lean_Expr_mdata___override(x_205, x_209); +lean_ctor_set(x_207, 0, x_213); +return x_207; +} +else { -uint8_t x_116; -x_116 = !lean_is_exclusive(x_115); -if (x_116 == 0) +lean_dec(x_209); +lean_dec(x_205); +lean_ctor_set(x_207, 0, x_5); +return x_207; +} +} +else { -lean_object* x_117; lean_object* x_118; -x_117 = lean_ctor_get(x_115, 0); -x_118 = lean_expr_update_mdata(x_5, x_117); -lean_ctor_set(x_115, 0, x_118); -return x_115; +lean_object* x_214; lean_object* x_215; size_t x_216; size_t x_217; uint8_t x_218; +x_214 = lean_ctor_get(x_207, 0); +x_215 = lean_ctor_get(x_207, 1); +lean_inc(x_215); +lean_inc(x_214); +lean_dec(x_207); +x_216 = lean_ptr_addr(x_206); +lean_dec(x_206); +x_217 = lean_ptr_addr(x_214); +x_218 = lean_usize_dec_eq(x_216, x_217); +if (x_218 == 0) +{ +lean_object* x_219; lean_object* x_220; +lean_dec(x_5); +x_219 = l_Lean_Expr_mdata___override(x_205, x_214); +x_220 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_220, 0, x_219); +lean_ctor_set(x_220, 1, x_215); +return x_220; } else { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_119 = lean_ctor_get(x_115, 0); -x_120 = lean_ctor_get(x_115, 1); -lean_inc(x_120); -lean_inc(x_119); -lean_dec(x_115); -x_121 = lean_expr_update_mdata(x_5, x_119); -x_122 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_122, 0, x_121); -lean_ctor_set(x_122, 1, x_120); -return x_122; +lean_object* x_221; +lean_dec(x_214); +lean_dec(x_205); +x_221 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_221, 0, x_5); +lean_ctor_set(x_221, 1, x_215); +return x_221; +} } } else { -uint8_t x_123; +uint8_t x_222; +lean_dec(x_206); +lean_dec(x_205); lean_dec(x_5); -x_123 = !lean_is_exclusive(x_115); -if (x_123 == 0) +x_222 = !lean_is_exclusive(x_207); +if (x_222 == 0) { -return x_115; +return x_207; } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_124 = lean_ctor_get(x_115, 0); -x_125 = lean_ctor_get(x_115, 1); -lean_inc(x_125); -lean_inc(x_124); -lean_dec(x_115); -x_126 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_126, 0, x_124); -lean_ctor_set(x_126, 1, x_125); -return x_126; +lean_object* x_223; lean_object* x_224; lean_object* x_225; +x_223 = lean_ctor_get(x_207, 0); +x_224 = lean_ctor_get(x_207, 1); +lean_inc(x_224); +lean_inc(x_223); +lean_dec(x_207); +x_225 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_225, 0, x_223); +lean_ctor_set(x_225, 1, x_224); +return x_225; } } } case 11: { -lean_object* x_127; lean_object* x_128; -x_127 = lean_ctor_get(x_5, 2); -lean_inc(x_127); -x_128 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_127, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_128) == 0) +lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; +x_226 = lean_ctor_get(x_5, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_5, 1); +lean_inc(x_227); +x_228 = lean_ctor_get(x_5, 2); +lean_inc(x_228); +lean_inc(x_228); +x_229 = l_Lean_Meta_kabstract_visit(x_1, x_2, x_3, x_4, x_228, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_229) == 0) +{ +uint8_t x_230; +x_230 = !lean_is_exclusive(x_229); +if (x_230 == 0) +{ +lean_object* x_231; size_t x_232; size_t x_233; uint8_t x_234; +x_231 = lean_ctor_get(x_229, 0); +x_232 = lean_ptr_addr(x_228); +lean_dec(x_228); +x_233 = lean_ptr_addr(x_231); +x_234 = lean_usize_dec_eq(x_232, x_233); +if (x_234 == 0) +{ +lean_object* x_235; +lean_dec(x_5); +x_235 = l_Lean_Expr_proj___override(x_226, x_227, x_231); +lean_ctor_set(x_229, 0, x_235); +return x_229; +} +else +{ +lean_dec(x_231); +lean_dec(x_227); +lean_dec(x_226); +lean_ctor_set(x_229, 0, x_5); +return x_229; +} +} +else { -uint8_t x_129; -x_129 = !lean_is_exclusive(x_128); -if (x_129 == 0) +lean_object* x_236; lean_object* x_237; size_t x_238; size_t x_239; uint8_t x_240; +x_236 = lean_ctor_get(x_229, 0); +x_237 = lean_ctor_get(x_229, 1); +lean_inc(x_237); +lean_inc(x_236); +lean_dec(x_229); +x_238 = lean_ptr_addr(x_228); +lean_dec(x_228); +x_239 = lean_ptr_addr(x_236); +x_240 = lean_usize_dec_eq(x_238, x_239); +if (x_240 == 0) { -lean_object* x_130; lean_object* x_131; -x_130 = lean_ctor_get(x_128, 0); -x_131 = lean_expr_update_proj(x_5, x_130); -lean_ctor_set(x_128, 0, x_131); -return x_128; +lean_object* x_241; lean_object* x_242; +lean_dec(x_5); +x_241 = l_Lean_Expr_proj___override(x_226, x_227, x_236); +x_242 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_242, 0, x_241); +lean_ctor_set(x_242, 1, x_237); +return x_242; } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_132 = lean_ctor_get(x_128, 0); -x_133 = lean_ctor_get(x_128, 1); -lean_inc(x_133); -lean_inc(x_132); -lean_dec(x_128); -x_134 = lean_expr_update_proj(x_5, x_132); -x_135 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_135, 0, x_134); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_object* x_243; +lean_dec(x_236); +lean_dec(x_227); +lean_dec(x_226); +x_243 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_243, 0, x_5); +lean_ctor_set(x_243, 1, x_237); +return x_243; +} } } else { -uint8_t x_136; +uint8_t x_244; +lean_dec(x_228); +lean_dec(x_227); +lean_dec(x_226); lean_dec(x_5); -x_136 = !lean_is_exclusive(x_128); -if (x_136 == 0) +x_244 = !lean_is_exclusive(x_229); +if (x_244 == 0) { -return x_128; +return x_229; } else { -lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_137 = lean_ctor_get(x_128, 0); -x_138 = lean_ctor_get(x_128, 1); -lean_inc(x_138); -lean_inc(x_137); -lean_dec(x_128); -x_139 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); -return x_139; +lean_object* x_245; lean_object* x_246; lean_object* x_247; +x_245 = lean_ctor_get(x_229, 0); +x_246 = lean_ctor_get(x_229, 1); +lean_inc(x_246); +lean_inc(x_245); +lean_dec(x_229); +x_247 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_247, 0, x_245); +lean_ctor_set(x_247, 1, x_246); +return x_247; } } } default: { -lean_object* x_140; +lean_object* x_248; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_1); -x_140 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_140, 0, x_5); -lean_ctor_set(x_140, 1, x_12); -return x_140; +x_248 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_248, 0, x_5); +lean_ctor_set(x_248, 1, x_12); +return x_248; } } } diff --git a/stage0/stdlib/Lean/Meta/LevelDefEq.c b/stage0/stdlib/Lean/Meta/LevelDefEq.c index 9bf28f9d7795..0b89267926d7 100644 --- a/stage0/stdlib/Lean/Meta/LevelDefEq.c +++ b/stage0/stdlib/Lean/Meta/LevelDefEq.c @@ -60,7 +60,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_LevelDefEq_0__Lean_Meta_postponeI LEAN_EXPORT lean_object* l___private_Lean_Meta_LevelDefEq_0__Lean_Meta_solve(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_LevelDefEq_0__Lean_Meta_solveSelfMax(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_level_mk_max_simp(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_LevelDefEq_0__Lean_Meta_mkMaxArgsDiff___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_throwIsDefEqStuck___rarg(lean_object*); lean_object* l_instInhabited___rarg(lean_object*, lean_object*); @@ -224,7 +224,7 @@ lean_dec(x_8); if (x_9 == 0) { lean_object* x_10; -x_10 = lean_level_mk_max_simp(x_3, x_2); +x_10 = l_Lean_mkLevelMax_x27(x_3, x_2); return x_10; } else @@ -236,7 +236,7 @@ return x_3; default: { lean_object* x_11; -x_11 = lean_level_mk_max_simp(x_3, x_2); +x_11 = l_Lean_mkLevelMax_x27(x_3, x_2); return x_11; } } diff --git a/stage0/stdlib/Lean/Meta/Match/Basic.c b/stage0/stdlib/Lean/Meta/Match/Basic.c index 5874cbf7cb5d..1e3c98166623 100644 --- a/stage0/stdlib/Lean/Meta/Match/Basic.c +++ b/stage0/stdlib/Lean/Meta/Match/Basic.c @@ -119,6 +119,7 @@ LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Meta_Match_Pattern_applyFVarS LEAN_EXPORT lean_object* l_Lean_Meta_Match_isNamedPattern_x3f(lean_object*); static lean_object* l_Lean_Meta_Match_Pattern_toMessageData___closed__4; LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_Match_Problem_toMessageData___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_Pattern_toMessageData___closed__8; LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_Match_instantiatePatternMVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkArrayLit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -181,7 +182,6 @@ LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_Match_Pattern_toExpr_visit__ lean_object* l_List_redLength___rarg(lean_object*); static lean_object* l_Lean_Meta_Match_toPattern___closed__3; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_instInhabitedPattern; LEAN_EXPORT lean_object* l_Lean_instantiateLocalDeclMVars___at_Lean_Meta_Match_instantiateAltLHSMVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_find_x3f___rarg(lean_object*, lean_object*); @@ -311,7 +311,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Match_isNamedPattern_x3f(lean_object* x_1) lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; x_2 = l_Lean_Expr_consumeMData(x_1); x_3 = lean_unsigned_to_nat(0u); -x_4 = l_Lean_Expr_getAppNumArgsAux(x_2, x_3); +x_4 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_3); x_5 = lean_unsigned_to_nat(4u); x_6 = lean_nat_dec_eq(x_4, x_5); lean_dec(x_4); @@ -7094,7 +7094,7 @@ x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); lean_dec(x_31); x_33 = lean_unsigned_to_nat(0u); -x_34 = l_Lean_Expr_getAppNumArgsAux(x_1, x_33); +x_34 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_33); x_35 = l_Lean_Meta_Match_toPattern___closed__3; lean_inc(x_34); x_36 = lean_mk_array(x_34, x_35); @@ -7274,7 +7274,7 @@ x_78 = lean_ctor_get(x_9, 0); lean_inc(x_78); lean_dec(x_9); x_79 = lean_unsigned_to_nat(0u); -x_80 = l_Lean_Expr_getAppNumArgsAux(x_78, x_79); +x_80 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_78, x_79); x_81 = lean_unsigned_to_nat(2u); x_82 = lean_nat_sub(x_80, x_81); x_83 = lean_unsigned_to_nat(1u); diff --git a/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c b/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c index 631aa327df24..84675457f05d 100644 --- a/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c +++ b/stage0/stdlib/Lean/Meta/Match/CaseArraySizes.c @@ -1503,7 +1503,7 @@ static lean_object* _init_l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___sp lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___closed__1; x_2 = l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Array_mapIdxM_map___at_Lean_Meta_caseArraySizes___spec__3___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Match/Match.c b/stage0/stdlib/Lean/Meta/Match/Match.c index 048d15979edd..8b4cc9ca1640 100644 --- a/stage0/stdlib/Lean/Meta/Match/Match.c +++ b/stage0/stdlib/Lean/Meta/Match/Match.c @@ -91,6 +91,7 @@ lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isArrayLitTransition___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__13(lean_object*, lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7; LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__10___lambda__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__2(lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); @@ -98,7 +99,6 @@ LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Meta_Match_processInaccessibl static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process_search___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoArrayLit_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isArrayLitTransition___boxed(lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__4___closed__1; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Match_processInaccessibleAsCtor___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -166,6 +166,7 @@ uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNumPatterns(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__8(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_constructorApp_x3f(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__6; @@ -178,7 +179,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Match_MkMatcherInput_collectDependencies(le static lean_object* l_Lean_Meta_Match_Unify_assign___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasValPattern___boxed(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_getMkMatcherInputInContext___spec__5___lambda__1___closed__1; -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__17(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__15___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___lambda__2___boxed(lean_object**); @@ -197,6 +197,7 @@ uint8_t l_Lean_Expr_isEq(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__13; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__12(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasNatValPattern(lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__5; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__6___closed__4; LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__7(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofList(lean_object*); @@ -213,7 +214,6 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__4; lean_object* l_Std_AssocList_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isFirstPatternVar___boxed(lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__5; LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_inLocalDecls(lean_object*, lean_object*); lean_object* l_Std_mkHashSetImp___rarg(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___closed__10; @@ -291,7 +291,7 @@ lean_object* l_Lean_mkAppN(lean_object*, lean_object*); static lean_object* l_List_filterMapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processNonVariable___spec__1___closed__2; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___closed__3; size_t lean_uint64_to_usize(uint64_t); -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Match_Match___hyg_13855_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Match_Match___hyg_13851_(lean_object*); lean_object* l_Lean_Expr_FindImpl_findUnsafe_x3f(lean_object*, lean_object*); uint8_t l_Lean_Environment_hasUnsafe(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -329,6 +329,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor(lean_object LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_unify_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* l_Lean_Meta_withMVarContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts(lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__6; static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___closed__1; lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Match_withMkMatcherInput___spec__3(lean_object*); @@ -377,19 +378,18 @@ LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasArra static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkRawNatLit(lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___closed__2; lean_object* l_Lean_Meta_mkHasTypeButIsExpectedMsg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getArrayArgType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoArrayLit___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_getUElimPos_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___closed__9; static lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandNatValuePattern___spec__1___closed__3; +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__4; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwInductiveTypeExpected___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Match_Match_0__Lean_Meta_updateAlts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_moveToFront___boxed(lean_object*, lean_object*); @@ -397,13 +397,13 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_ex LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___closed__4; lean_object* l_Lean_Meta_FVarSubst_apply(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__4; static lean_object* l_List_forIn_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes___spec__2___closed__1; LEAN_EXPORT lean_object* l_List_replace___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___spec__8(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isNatValueTransition___spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__5; lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__3(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__1; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___closed__4; static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__1___closed__1; static lean_object* l_Lean_Meta_Match_Unify_unify___closed__2; @@ -425,7 +425,6 @@ lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__20___closed__2; LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasValPattern(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__10(lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__8; lean_object* lean_name_append_index_after(lean_object*, lean_object*); static lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandNatValuePattern___spec__1___closed__5; lean_object* l_Std_RBNode_findCore___at_Lean_Meta_removeUnused___spec__1(lean_object*, lean_object*); @@ -441,19 +440,21 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCa LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processVariable___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__16___boxed(lean_object**); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__8; LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_List_moveToFront___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process_tryToProcess___closed__3; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___closed__1; lean_object* l_Nat_repr(lean_object*); static lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_getMkMatcherInputInContext___spec__2(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_withMkMatcherInput(lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__1; LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__9(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkArrayLit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_replace___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___spec__8___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____lambda__1(uint8_t, uint8_t); lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasNatValPattern___spec__1(uint8_t, lean_object*); static lean_object* l_List_filterMapM_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processNonVariable___spec__2___closed__1; @@ -462,7 +463,9 @@ lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Meta_Match_mkMatcher___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_matcherExt; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__1; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__17___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____lambda__1___boxed(lean_object*, lean_object*); extern lean_object* l_Lean_Expr_instHashableExpr; LEAN_EXPORT lean_object* l_Lean_Meta_Match_Unify_assign(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__12___boxed(lean_object**); @@ -470,7 +473,6 @@ LEAN_EXPORT lean_object* l_List_foldr___at___private_Lean_Meta_Match_Match_0__Le uint64_t l_Lean_Expr_hash(lean_object*); uint8_t l_Array_contains___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getMajorPosDepElim___spec__4(lean_object*, lean_object*); static lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandNatValuePattern___spec__1___closed__7; -LEAN_EXPORT uint8_t l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____lambda__1(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__20___closed__1; @@ -487,7 +489,6 @@ lean_object* l_Lean_LocalContext_getFVar_x21(lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withEqs_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process_tryToProcess___closed__4; -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__2; LEAN_EXPORT lean_object* l_List_filterTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoCtor_x3f___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isConstructorTransition___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -497,6 +498,7 @@ lean_object* lean_array_to_list(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_InfoCacheKey_instHashableInfoCacheKey___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__2; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_getUElimPos_x3f___closed__2; LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isFirstPatternVar(lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Match_Unify_occurs___lambda__1(lean_object*, lean_object*); @@ -545,6 +547,7 @@ LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Matc LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__11___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isVariableTransition___spec__1(uint8_t, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__4; LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_moveToFront___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_checkNextPatternTypes___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -557,11 +560,9 @@ static lean_object* l_Lean_Meta_Match_getMkMatcherInputInContext___lambda__3___c LEAN_EXPORT lean_object* l_Lean_Meta_MatcherApp_addArg_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_processInaccessibleAsCtor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_expandVarIntoCtor_x3f___lambda__2___closed__4; -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__4; static lean_object* l_Lean_Meta_Match_Unify_assign___closed__1; LEAN_EXPORT lean_object* l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasValPattern___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isValueTransition___spec__1(uint8_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__5___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_mkMinorType___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -573,9 +574,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher__ lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_mkMinorType___lambda__2(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__2; size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Match_withMkMatcherInput___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__9; lean_object* l_Lean_mkSimpleThunkType(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processVariable(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__7(size_t, size_t, lean_object*); @@ -594,12 +595,12 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Matc LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwInductiveTypeExpected___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasNonTrivialExample___spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___closed__1; +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__9; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___lambda__1___closed__2; size_t lean_usize_land(size_t, size_t); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withAlts_loop___rarg___lambda__1___closed__5; lean_object* l_Lean_LocalDecl_fvarId(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_List_moveToFront___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__2; lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceOptions(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasCtorPattern(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException(lean_object*); @@ -641,7 +642,6 @@ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_isNatValueTransition___boxed(lean_object*); lean_object* l_Lean_Option_register___at_Std_Format_initFn____x40_Lean_Data_Format___hyg_57____spec__1(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Match_getMkMatcherInputInContext___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__4(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwNonSupported___lambda__1___closed__2; @@ -711,7 +711,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Match_processInaccessi LEAN_EXPORT uint8_t l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_hasValPattern___spec__1(uint8_t, lean_object*); static lean_object* l_Lean_addTrace___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___spec__1___closed__2; static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__3___closed__2; -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processSkipInaccessible(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process_checkVarDeps___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -720,6 +719,7 @@ LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Meta_Match_Match_0_ static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withEqs_go___rarg___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_updateAlts___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withEqs_go___rarg___closed__1; +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__6; static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__10; LEAN_EXPORT lean_object* l_Array_indexOfAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_getUElimPos_x3f___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); @@ -730,7 +730,6 @@ static lean_object* l_Lean_Meta_MatcherApp_addArg___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Nat_foldAux___at_Lean_Meta_Match_mkMatcher___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__8___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_traceState(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processArrayLit___spec__5(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_mkMatcher___lambda__5___closed__2; @@ -861,6 +860,7 @@ lean_object* l_Lean_Meta_setInlineAttribute(lean_object*, uint8_t, lean_object*, LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__6(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_compileDecl___at_Lean_Meta_mkAuxDefinition___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__5; lean_object* l_Lean_CollectFVars_State_addDependencies(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashSetImp_expand___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processLeaf___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process_tryToProcess(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -868,6 +868,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_wi lean_object* l_Lean_Expr_getAppFn(lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processConstructor___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__3(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__3; static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Match_getMkMatcherInputInContext___spec__5___closed__1; lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Match_mkMatcherAuxDefinition___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -905,7 +906,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_mo static lean_object* l_Lean_Meta_Match_Unify_assign___closed__6; LEAN_EXPORT uint8_t l_List_foldr___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_inLocalDecls___spec__1(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__3; uint8_t lean_level_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_mkMatcher___lambda__6___boxed(lean_object**); lean_object* l_EStateM_pure___rarg(lean_object*, lean_object*); @@ -946,8 +946,8 @@ lean_object* l_Lean_Meta_Match_Alt_applyFVarSubst(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_List_moveToFront_loop___spec__1(lean_object*); static lean_object* l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_throwCasesException___rarg___closed__12; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Meta_Match_withCleanLCtxFor___spec__11(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840_(lean_object*); static lean_object* l_Array_mapIdxM_map___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_processValue___spec__10___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Match_withMkMatcherInput___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_process_tryToProcess___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1139,7 +1139,7 @@ static lean_object* _init_l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_w lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withEqs_go___rarg___closed__1; x_2 = l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withEqs_go___rarg___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_withEqs_go___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -23178,7 +23178,7 @@ lean_dec(x_2); return x_7; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__1() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__1() { _start: { lean_object* x_1; @@ -23186,17 +23186,17 @@ x_1 = lean_mk_string_from_bytes("bootstrap", 9); return x_1; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__2() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__1; +x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__3() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__3() { _start: { lean_object* x_1; @@ -23204,17 +23204,17 @@ x_1 = lean_mk_string_from_bytes("genMatcherCode", 14); return x_1; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__4() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__2; -x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__3; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__2; +x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__5() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__5() { _start: { lean_object* x_1; @@ -23222,13 +23222,13 @@ x_1 = lean_mk_string_from_bytes("disable code generation for auxiliary matcher f return x_1; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__6() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__6() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 1; -x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__1; -x_3 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__5; +x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__1; +x_3 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__5; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -23237,17 +23237,17 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__4; -x_3 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__6; +x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__4; +x_3 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__6; x_4 = l_Lean_Option_register___at_Std_Format_initFn____x40_Lean_Data_Format___hyg_57____spec__1(x_2, x_3, x_1); return x_4; } } -LEAN_EXPORT uint8_t l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____lambda__1(uint8_t x_1, uint8_t x_2) { +LEAN_EXPORT uint8_t l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____lambda__1(uint8_t x_1, uint8_t x_2) { _start: { if (x_1 == 0) @@ -23271,37 +23271,37 @@ return x_2; } } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__1() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____lambda__1___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____lambda__1___boxed), 2, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__2() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__1; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__1; x_2 = lean_alloc_closure((void*)(l_instBEq___rarg), 3, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__3() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Expr_instBEqExpr; -x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__2; +x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__2; x_3 = lean_alloc_closure((void*)(l_instBEqProd___rarg), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__4() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__4() { _start: { lean_object* x_1; @@ -23309,19 +23309,19 @@ x_1 = lean_alloc_closure((void*)(l_instHashableBool___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__5() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Expr_instHashableExpr; -x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__4; +x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__4; x_3 = lean_alloc_closure((void*)(l_instHashableProd___rarg___boxed), 3, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__6() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__6() { _start: { lean_object* x_1; @@ -23329,21 +23329,21 @@ x_1 = l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); return x_1; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__6; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__6; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__8() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -23351,26 +23351,26 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__9() { +static lean_object* _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__8; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__8; x_2 = lean_alloc_closure((void*)(l_EStateM_pure___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__9; +x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__9; x_3 = l_Lean_EnvExtensionInterfaceUnsafe_registerExt___rarg(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____lambda__1___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; @@ -23378,7 +23378,7 @@ x_3 = lean_unbox(x_1); lean_dec(x_1); x_4 = lean_unbox(x_2); lean_dec(x_2); -x_5 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____lambda__1(x_3, x_4); +x_5 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____lambda__1(x_3, x_4); x_6 = lean_box(x_5); return x_6; } @@ -24551,7 +24551,7 @@ static lean_object* _init_l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__2__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -24574,7 +24574,7 @@ static lean_object* _init_l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__2__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -24594,7 +24594,7 @@ static lean_object* _init_l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__2__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -24606,7 +24606,7 @@ static lean_object* _init_l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__2__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -24640,7 +24640,7 @@ static lean_object* _init_l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__2__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -25143,8 +25143,8 @@ static lean_object* _init_l_Lean_Meta_Match_mkMatcherAuxDefinition___lambda__4__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__3; -x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__5; +x_1 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__3; +x_2 = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__5; x_3 = l_Std_PersistentHashMap_instInhabitedPersistentHashMap___rarg(x_1, x_2); return x_3; } @@ -29859,7 +29859,7 @@ x_56 = lean_ctor_get(x_8, 0); lean_inc(x_56); lean_dec(x_8); x_57 = lean_unsigned_to_nat(0u); -x_58 = l_Lean_Expr_getAppNumArgsAux(x_1, x_57); +x_58 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_57); x_59 = l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__5(x_9, x_10, x_11, x_12); lean_dec(x_9); x_60 = lean_alloc_ctor(0, 5, 0); @@ -30866,7 +30866,7 @@ x_56 = lean_ctor_get(x_8, 0); lean_inc(x_56); lean_dec(x_8); x_57 = lean_unsigned_to_nat(0u); -x_58 = l_Lean_Expr_getAppNumArgsAux(x_1, x_57); +x_58 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_57); x_59 = l_Array_mapMUnsafe_map___at_Lean_Meta_Match_mkMatcher___spec__15(x_9, x_10, x_11, x_12); lean_dec(x_9); x_60 = lean_alloc_ctor(0, 5, 0); @@ -33579,7 +33579,7 @@ goto block_19; block_19: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_13 = l_Lean_Expr_getAppNumArgsAux(x_2, x_9); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_9); x_14 = l_Array_mapMUnsafe_map___at_Lean_Meta_Match_getMkMatcherInputInContext___spec__5___lambda__1___closed__1; lean_inc(x_13); x_15 = lean_mk_array(x_13, x_14); @@ -34817,7 +34817,7 @@ if (x_20 == 0) lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; x_21 = lean_ctor_get(x_11, 0); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_1, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_22); x_24 = l_Array_mapMUnsafe_map___at_Lean_Meta_Match_getMkMatcherInputInContext___spec__5___lambda__1___closed__1; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -34927,7 +34927,7 @@ x_57 = lean_ctor_get(x_11, 0); lean_inc(x_57); lean_dec(x_11); x_58 = lean_unsigned_to_nat(0u); -x_59 = l_Lean_Expr_getAppNumArgsAux(x_1, x_58); +x_59 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_58); x_60 = l_Array_mapMUnsafe_map___at_Lean_Meta_Match_getMkMatcherInputInContext___spec__5___lambda__1___closed__1; lean_inc(x_59); x_61 = lean_mk_array(x_59, x_60); @@ -35050,7 +35050,7 @@ if (lean_is_exclusive(x_11)) { x_97 = lean_box(0); } x_98 = lean_unsigned_to_nat(0u); -x_99 = l_Lean_Expr_getAppNumArgsAux(x_1, x_98); +x_99 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_98); x_100 = l_Array_mapMUnsafe_map___at_Lean_Meta_Match_getMkMatcherInputInContext___spec__5___lambda__1___closed__1; lean_inc(x_99); x_101 = lean_mk_array(x_99, x_100); @@ -37000,7 +37000,7 @@ return x_21; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Match_Match___hyg_13855_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Match_Match___hyg_13851_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -37486,42 +37486,42 @@ l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_getUElimPos_x3f___closed__1 lean_mark_persistent(l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_getUElimPos_x3f___closed__1); l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_getUElimPos_x3f___closed__2 = _init_l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_getUElimPos_x3f___closed__2(); lean_mark_persistent(l___private_Lean_Meta_Match_Match_0__Lean_Meta_Match_getUElimPos_x3f___closed__2); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__1 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__1(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__1); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__2 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__2(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__2); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__3 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__3(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__3); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__4 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__4(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__4); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__5 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__5(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__5); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__6 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__6(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815____closed__6); -if (builtin) {res = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9815_(lean_io_mk_world()); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__1 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__1(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__1); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__2 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__2(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__2); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__3 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__3(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__3); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__4 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__4(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__4); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__5 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__5(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__5); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__6 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__6(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811____closed__6); +if (builtin) {res = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9811_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Meta_Match_bootstrap_genMatcherCode = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Meta_Match_bootstrap_genMatcherCode); lean_dec_ref(res); -}l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__1 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__1(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__1); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__2 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__2(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__2); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__3 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__3(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__3); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__4 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__4(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__4); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__5 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__5(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__5); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__6 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__6(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__6); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__7); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__8 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__8(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__8); -l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__9 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__9(); -lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844____closed__9); -if (builtin) {res = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9844_(lean_io_mk_world()); +}l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__1 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__1(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__1); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__2 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__2(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__2); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__3 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__3(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__3); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__4 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__4(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__4); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__5 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__5(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__5); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__6 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__6(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__6); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__7); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__8 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__8(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__8); +l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__9 = _init_l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__9(); +lean_mark_persistent(l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840____closed__9); +if (builtin) {res = l_Lean_Meta_Match_initFn____x40_Lean_Meta_Match_Match___hyg_9840_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Meta_Match_matcherExt = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Meta_Match_matcherExt); @@ -37658,7 +37658,7 @@ l_Lean_Meta_MatcherApp_addArg___lambda__4___closed__3 = _init_l_Lean_Meta_Matche lean_mark_persistent(l_Lean_Meta_MatcherApp_addArg___lambda__4___closed__3); l_Lean_Meta_MatcherApp_addArg___lambda__4___closed__4 = _init_l_Lean_Meta_MatcherApp_addArg___lambda__4___closed__4(); lean_mark_persistent(l_Lean_Meta_MatcherApp_addArg___lambda__4___closed__4); -res = l_Lean_Meta_initFn____x40_Lean_Meta_Match_Match___hyg_13855_(lean_io_mk_world()); +res = l_Lean_Meta_initFn____x40_Lean_Meta_Match_Match___hyg_13851_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/Match/MatchEqs.c b/stage0/stdlib/Lean/Meta/Match/MatchEqs.c index a06e8970c5f2..7f550c86245f 100644 --- a/stage0/stdlib/Lean/Meta/Match/MatchEqs.c +++ b/stage0/stdlib/Lean/Meta/Match/MatchEqs.c @@ -68,7 +68,6 @@ LEAN_EXPORT lean_object* l_Std_RBNode_find___at___private_Lean_Meta_Match_MatchE static lean_object* l_Lean_Meta_casesOnStuckLHS___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Std_RBNode_insert___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_mkMap___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_simpH_x3f___lambda__3___closed__7; -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__13(lean_object*, lean_object*); static lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_isCastEqRec___spec__2___closed__1; @@ -105,6 +104,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match static lean_object* l_Lean_Meta_Match_proveCondEqThm___closed__3; lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertCastEqRec___spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_Meta_Match_getEquationsForImpl___spec__2(lean_object*, size_t, lean_object*); @@ -340,6 +340,7 @@ lean_object* l_Lean_Meta_Match_isNamedPattern_x3f(lean_object*); static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_substSomeVar___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__12___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_proveSubgoal___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_proveCondEqThm_go___lambda__2___closed__2; static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_proveSubgoal___closed__3; @@ -448,7 +449,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Match_proveCondEqThm_go(lean_object*, lean_ static lean_object* l_Lean_Meta_Match_forallAltTelescope_go___rarg___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_SimpH_contradiction___closed__1; -lean_object* lean_expr_update_proj(lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertCastEqRec___spec__8___lambda__6___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_proveSubgoalLoop___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertCastEqRec___spec__3___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -496,6 +496,7 @@ static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_simp static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___lambda__2___closed__4; lean_object* l_Lean_Expr_fvar___override(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_isCastEqRec___lambda__2(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*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_proveCondEqThm___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_SimpH_processNextEq___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_unfoldNamedPattern___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -508,7 +509,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_Match lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_SimpH_processNextEq___lambda__2___closed__2; static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertCastEqRec___closed__2; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertCastEqRec___spec__6___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertCastEqRec___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern uint8_t l_instInhabitedBool; @@ -655,6 +655,7 @@ static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Match_MatchE static lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_proveSubgoal___closed__4; LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertCastEqRec___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__11___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonadReaderT___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_substSomeVar___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -790,7 +791,7 @@ static lean_object* _init_l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___lambda__1__ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___lambda__1___closed__1; x_2 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -907,7 +908,7 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean x_12 = l_Lean_Expr_constName_x21(x_7); lean_dec(x_7); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -1221,7 +1222,7 @@ lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean x_80 = l_Lean_Expr_constName_x21(x_7); lean_dec(x_7); x_81 = lean_unsigned_to_nat(0u); -x_82 = l_Lean_Expr_getAppNumArgsAux(x_1, x_81); +x_82 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_81); x_83 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___closed__1; lean_inc(x_82); x_84 = lean_mk_array(x_82, x_83); @@ -20693,7 +20694,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match { lean_object* x_10; 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; size_t x_21; lean_object* x_22; size_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_1, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_10); x_12 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___closed__1; lean_inc(x_11); x_13 = lean_mk_array(x_11, x_12); @@ -20775,7 +20776,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_dec(x_2); x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_1, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_10); x_12 = lean_unsigned_to_nat(6u); x_13 = lean_nat_dec_lt(x_12, x_11); lean_dec(x_11); @@ -28493,7 +28494,7 @@ x_16 = lean_ctor_get(x_10, 1); lean_inc(x_16); lean_dec(x_10); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_2, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_17); x_19 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -30594,7 +30595,7 @@ case 5: { lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_17, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_17, x_18); x_20 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___closed__1; lean_inc(x_19); x_21 = lean_mk_array(x_19, x_20); @@ -30627,9 +30628,11 @@ return x_30; } case 10: { -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_17, 1); +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_17, 0); lean_inc(x_31); +x_32 = lean_ctor_get(x_17, 1); +lean_inc(x_32); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -30637,26 +30640,46 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); +lean_inc(x_32); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_32 = l_Lean_Meta_transform_visit___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__7(x_1, x_2, x_3, x_4, x_5, x_31, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_32) == 0) +x_33 = l_Lean_Meta_transform_visit___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__7(x_1, x_2, x_3, x_4, x_5, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); +lean_object* x_34; lean_object* x_35; size_t x_36; size_t x_37; uint8_t x_38; +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_ptr_addr(x_32); lean_dec(x_32); -x_35 = lean_expr_update_mdata(x_17, x_33); -x_36 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__8(x_1, x_2, x_3, x_4, x_5, x_35, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_34); -return x_36; +x_37 = lean_ptr_addr(x_34); +x_38 = lean_usize_dec_eq(x_36, x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +lean_dec(x_17); +x_39 = l_Lean_Expr_mdata___override(x_31, x_34); +x_40 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__8(x_1, x_2, x_3, x_4, x_5, x_39, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_35); +return x_40; } else { -uint8_t x_37; +lean_object* x_41; +lean_dec(x_34); +lean_dec(x_31); +x_41 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__8(x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_35); +return x_41; +} +} +else +{ +uint8_t x_42; +lean_dec(x_32); +lean_dec(x_31); lean_dec(x_17); lean_dec(x_13); lean_dec(x_12); @@ -30669,31 +30692,35 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_37 = !lean_is_exclusive(x_32); -if (x_37 == 0) +x_42 = !lean_is_exclusive(x_33); +if (x_42 == 0) { -return x_32; +return x_33; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_32, 0); -x_39 = lean_ctor_get(x_32, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_32); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_33, 0); +x_44 = lean_ctor_get(x_33, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_33); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } case 11: { -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_17, 2); -lean_inc(x_41); +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_46 = lean_ctor_get(x_17, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_17, 1); +lean_inc(x_47); +x_48 = lean_ctor_get(x_17, 2); +lean_inc(x_48); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -30701,26 +30728,48 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); +lean_inc(x_48); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_42 = l_Lean_Meta_transform_visit___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__7(x_1, x_2, x_3, x_4, x_5, x_41, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_42) == 0) +x_49 = l_Lean_Meta_transform_visit___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__7(x_1, x_2, x_3, x_4, x_5, x_48, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_49) == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_expr_update_proj(x_17, x_43); -x_46 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__8(x_1, x_2, x_3, x_4, x_5, x_45, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_44); -return x_46; +lean_object* x_50; lean_object* x_51; size_t x_52; size_t x_53; uint8_t x_54; +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = lean_ptr_addr(x_48); +lean_dec(x_48); +x_53 = lean_ptr_addr(x_50); +x_54 = lean_usize_dec_eq(x_52, x_53); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; +lean_dec(x_17); +x_55 = l_Lean_Expr_proj___override(x_46, x_47, x_50); +x_56 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__8(x_1, x_2, x_3, x_4, x_5, x_55, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_51); +return x_56; } else { -uint8_t x_47; +lean_object* x_57; +lean_dec(x_50); +lean_dec(x_47); +lean_dec(x_46); +x_57 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__8(x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_51); +return x_57; +} +} +else +{ +uint8_t x_58; +lean_dec(x_48); +lean_dec(x_47); +lean_dec(x_46); lean_dec(x_17); lean_dec(x_13); lean_dec(x_12); @@ -30733,31 +30782,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_47 = !lean_is_exclusive(x_42); -if (x_47 == 0) +x_58 = !lean_is_exclusive(x_49); +if (x_58 == 0) { -return x_42; +return x_49; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_42, 0); -x_49 = lean_ctor_get(x_42, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_42); -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_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_49, 0); +x_60 = lean_ctor_get(x_49, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_49); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } } default: { -lean_object* x_51; -x_51 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__8(x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_51; +lean_object* x_62; +x_62 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_convertTemplate___spec__8(x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_62; } } } @@ -31284,7 +31333,7 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_array_get_size(x_1); x_15 = lean_unsigned_to_nat(0u); x_16 = l_Array_toSubarray___rarg(x_1, x_15, x_14); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_2, x_15); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_15); x_18 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___closed__1; lean_inc(x_17); x_19 = lean_mk_array(x_17, x_18); @@ -31502,7 +31551,7 @@ lean_dec(x_6); x_14 = l___private_Lean_Meta_Match_MatchEqs_0__Lean_Meta_Match_mkSplitterProof_trimFalseTrail(x_1); x_15 = lean_array_get_size(x_14); x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_2, x_16); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_16); x_18 = lean_nat_dec_le(x_15, x_17); lean_dec(x_17); lean_dec(x_15); @@ -35208,7 +35257,7 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_Match_M { 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; size_t x_35; size_t x_36; lean_object* x_37; x_27 = lean_unsigned_to_nat(0u); -x_28 = l_Lean_Expr_getAppNumArgsAux(x_21, x_27); +x_28 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_21, x_27); x_29 = l_Lean_Meta_casesOnStuckLHS_findFVar_x3f___closed__1; lean_inc(x_28); x_30 = lean_mk_array(x_28, x_29); diff --git a/stage0/stdlib/Lean/Meta/Match/MatcherInfo.c b/stage0/stdlib/Lean/Meta/Match/MatcherInfo.c index f2e4557dbdc3..fc2226647f33 100644 --- a/stage0/stdlib/Lean/Meta/Match/MatcherInfo.c +++ b/stage0/stdlib/Lean/Meta/Match/MatcherInfo.c @@ -81,6 +81,7 @@ lean_object* l_Std_mkHashMapImp___rarg(lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Match_Extension_State_addEntry___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_Extension_State_map___default___closed__1; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Match_Extension_State_switch(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_Meta_Match_Extension_getMatcherInfo_x3f___spec__5(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_addMatcherInfo___closed__2; @@ -128,7 +129,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getMatcherInfo_x3f(lean_object*); lean_object* l_List_redLength___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_matchMatcherApp_x3f(lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Meta_Match_Extension_State_addEntry___spec__6(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Match_Extension_initFn____x40_Lean_Meta_Match_MatcherInfo___hyg_311____closed__4; lean_object* lean_list_to_array(lean_object*, lean_object*); @@ -2517,7 +2517,7 @@ lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint x_10 = lean_ctor_get(x_7, 0); x_11 = l_Lean_Meta_Match_MatcherInfo_arity(x_10); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Lean_Expr_getAppNumArgsAux(x_2, x_12); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_12); x_14 = lean_nat_dec_le(x_11, x_13); lean_dec(x_13); lean_dec(x_11); @@ -2542,7 +2542,7 @@ lean_inc(x_16); lean_dec(x_7); x_17 = l_Lean_Meta_Match_MatcherInfo_arity(x_16); x_18 = lean_unsigned_to_nat(0u); -x_19 = l_Lean_Expr_getAppNumArgsAux(x_2, x_18); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_18); x_20 = lean_nat_dec_le(x_17, x_19); lean_dec(x_19); lean_dec(x_17); @@ -2692,7 +2692,7 @@ static lean_object* _init_l_Lean_Meta_matchMatcherApp_x3f___rarg___lambda__1___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_Lean_Meta_matchMatcherApp_x3f___rarg___lambda__1___closed__2; x_2 = l_Lean_Meta_matchMatcherApp_x3f___rarg___lambda__1___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_matchMatcherApp_x3f___rarg___lambda__1___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2727,7 +2727,7 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_11 = lean_ctor_get(x_5, 0); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Lean_Expr_getAppNumArgsAux(x_2, x_12); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_12); x_14 = l_Lean_Meta_matchMatcherApp_x3f___rarg___lambda__1___closed__1; lean_inc(x_13); x_15 = lean_mk_array(x_13, x_14); @@ -2851,7 +2851,7 @@ x_54 = lean_ctor_get(x_5, 0); lean_inc(x_54); lean_dec(x_5); x_55 = lean_unsigned_to_nat(0u); -x_56 = l_Lean_Expr_getAppNumArgsAux(x_2, x_55); +x_56 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_55); x_57 = l_Lean_Meta_matchMatcherApp_x3f___rarg___lambda__1___closed__1; lean_inc(x_56); x_58 = lean_mk_array(x_56, x_57); diff --git a/stage0/stdlib/Lean/Meta/Offset.c b/stage0/stdlib/Lean/Meta/Offset.c index 69421edf25d6..232e0ef7d754 100644 --- a/stage0/stdlib/Lean/Meta/Offset.c +++ b/stage0/stdlib/Lean/Meta/Offset.c @@ -39,6 +39,7 @@ static lean_object* l_Lean_Meta_isNatProjInst___closed__19; lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l_Lean_Meta_isNatProjInst___closed__2; static lean_object* l_Lean_Meta_isNatProjInst___closed__23; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_isNatProjInst___closed__21; LEAN_EXPORT lean_object* l_Lean_Meta_isDefEqOffset(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Offset_0__Lean_Meta_withInstantiatedMVars___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -57,7 +58,6 @@ static lean_object* l_Lean_Meta_evalNat_visit___closed__6; lean_object* l_Lean_Meta_unfoldProjInst_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_isNatProjInst___closed__6; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Offset_0__Lean_Meta_mkOffset(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_evalNat_visit___closed__4; static lean_object* l_Lean_Meta_isNatProjInst___closed__3; @@ -863,7 +863,7 @@ x_25 = lean_ctor_get(x_7, 0); lean_inc(x_25); lean_dec(x_7); x_26 = lean_unsigned_to_nat(0u); -x_27 = l_Lean_Expr_getAppNumArgsAux(x_1, x_26); +x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_26); x_224 = l_Lean_Meta_evalNat_visit___closed__7; x_225 = lean_name_eq(x_25, x_224); if (x_225 == 0) @@ -2240,7 +2240,7 @@ x_27 = lean_ctor_get(x_9, 0); lean_inc(x_27); lean_dec(x_9); x_28 = lean_unsigned_to_nat(0u); -x_29 = l_Lean_Expr_getAppNumArgsAux(x_1, x_28); +x_29 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_28); x_175 = l_Lean_Meta_evalNat_visit___closed__7; x_176 = lean_name_eq(x_27, x_175); if (x_176 == 0) @@ -3308,7 +3308,7 @@ x_25 = lean_ctor_get(x_7, 0); lean_inc(x_25); lean_dec(x_7); x_26 = lean_unsigned_to_nat(0u); -x_27 = l_Lean_Expr_getAppNumArgsAux(x_1, x_26); +x_27 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_26); x_64 = l_Lean_Meta_evalNat_visit___closed__7; x_65 = lean_name_eq(x_25, x_64); if (x_65 == 0) diff --git a/stage0/stdlib/Lean/Meta/RecursorInfo.c b/stage0/stdlib/Lean/Meta/RecursorInfo.c index a92c842858e5..61bd9c4f2f2e 100644 --- a/stage0/stdlib/Lean/Meta/RecursorInfo.c +++ b/stage0/stdlib/Lean/Meta/RecursorInfo.c @@ -171,6 +171,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_RecursorInfo static lean_object* l_Lean_Meta_RecursorInfo_instToStringRecursorInfo___closed__4; lean_object* l_Lean_ConstantInfo_name(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_RecursorInfo_0__Lean_Meta_mkRecursorInfoForKernelRec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); @@ -239,7 +240,6 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_RecursorInfo lean_object* l_List_redLength___rarg(lean_object*); static lean_object* l___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getProduceMotiveAndRecursive___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Attribute_Recursor_getMajorPos___closed__6; static lean_object* l___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getMajorPosDepElim___closed__5; static lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getParamsPos___spec__2___closed__7; @@ -3798,7 +3798,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_Recurs lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getParamsPos___spec__2___closed__4; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getParamsPos___spec__2___closed__5; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getParamsPos___spec__2___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -5489,7 +5489,7 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at___private_Lean_Meta_Recurso { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_5, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_11); x_13 = l_Std_Range_forIn_loop___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getProduceMotiveAndRecursive___spec__3___lambda__1___closed__1; lean_inc(x_12); x_14 = lean_mk_array(x_12, x_13); @@ -6834,7 +6834,7 @@ x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_18, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_18, x_20); x_22 = l_Std_Range_forIn_loop___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getProduceMotiveAndRecursive___spec__3___lambda__1___closed__1; lean_inc(x_21); x_23 = lean_mk_array(x_21, x_22); @@ -8928,7 +8928,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_RecursorInfo_0__Lean_Meta_mkRecur { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_5, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_11); x_13 = l_Std_Range_forIn_loop___at___private_Lean_Meta_RecursorInfo_0__Lean_Meta_getProduceMotiveAndRecursive___spec__3___lambda__1___closed__1; lean_inc(x_12); x_14 = lean_mk_array(x_12, x_13); diff --git a/stage0/stdlib/Lean/Meta/Reduce.c b/stage0/stdlib/Lean/Meta/Reduce.c index 60a7a4a9f18c..ffe899e716ae 100644 --- a/stage0/stdlib/Lean/Meta/Reduce.c +++ b/stage0/stdlib/Lean/Meta/Reduce.c @@ -59,6 +59,7 @@ LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_Meta_reduce_visit__ lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_reduce_visit___lambda__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_reduce_visit___lambda__4___closed__4; lean_object* lean_st_mk_ref(lean_object*, lean_object*); @@ -83,7 +84,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_reduce___boxed(lean_object*, lean_object*, LEAN_EXPORT lean_object* l_Lean_Meta_reduce_visit___lambda__4(lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_contains___at_Lean_Meta_reduce_visit___spec__11___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Meta_reduce_visit___spec__10(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___at_Lean_Meta_reduce_visit___spec__6___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -1436,7 +1436,7 @@ static lean_object* _init_l_Lean_Meta_reduce_visit___lambda__4___closed__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; x_1 = l_Lean_Meta_reduce_visit___lambda__4___closed__2; x_2 = l_Lean_Meta_reduce_visit___lambda__4___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_reduce_visit___lambda__4___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1618,7 +1618,7 @@ x_20 = lean_ctor_get(x_18, 1); lean_inc(x_20); lean_dec(x_18); x_21 = lean_unsigned_to_nat(0u); -x_22 = l_Lean_Expr_getAppNumArgsAux(x_15, x_21); +x_22 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_15, x_21); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); diff --git a/stage0/stdlib/Lean/Meta/ReduceEval.c b/stage0/stdlib/Lean/Meta/ReduceEval.c index 462ca3c0b783..b78a12c1e98f 100644 --- a/stage0/stdlib/Lean/Meta/ReduceEval.c +++ b/stage0/stdlib/Lean/Meta/ReduceEval.c @@ -36,6 +36,7 @@ lean_object* lean_nat_sub(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ReduceEval_0__Lean_Meta_evalName___closed__6; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_ReduceEval_0__Lean_Meta_throwFailedToEval___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_ReduceEval_0__Lean_Meta_evalName___closed__4; static lean_object* l___private_Lean_Meta_ReduceEval_0__Lean_Meta_evalName___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_instReduceEvalOption(lean_object*); @@ -47,7 +48,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_instReduceEvalOption___rarg(lean_object*, l lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instReduceEvalString(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_reduceEval___at___private_Lean_Meta_ReduceEval_0__Lean_Meta_evalName___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_ReduceEval_0__Lean_Meta_throwFailedToEval___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -889,7 +889,7 @@ x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); lean_dec(x_12); x_14 = lean_unsigned_to_nat(0u); -x_15 = l_Lean_Expr_getAppNumArgsAux(x_10, x_14); +x_15 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_10, x_14); x_16 = l_Lean_Meta_instReduceEvalOption___rarg___closed__4; x_17 = lean_name_eq(x_13, x_16); if (x_17 == 0) @@ -1135,7 +1135,7 @@ x_62 = lean_ctor_get(x_61, 0); lean_inc(x_62); lean_dec(x_61); x_63 = lean_unsigned_to_nat(0u); -x_64 = l_Lean_Expr_getAppNumArgsAux(x_59, x_63); +x_64 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_59, x_63); x_65 = l_Lean_Meta_instReduceEvalOption___rarg___closed__4; x_66 = lean_name_eq(x_62, x_65); if (x_66 == 0) @@ -3588,7 +3588,7 @@ x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); lean_dec(x_11); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_9, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_13); x_83 = l___private_Lean_Meta_ReduceEval_0__Lean_Meta_evalName___closed__10; x_84 = lean_name_eq(x_12, x_83); if (x_84 == 0) @@ -3936,7 +3936,7 @@ x_93 = lean_ctor_get(x_92, 0); lean_inc(x_93); lean_dec(x_92); x_94 = lean_unsigned_to_nat(0u); -x_95 = l_Lean_Expr_getAppNumArgsAux(x_90, x_94); +x_95 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_90, x_94); x_160 = l___private_Lean_Meta_ReduceEval_0__Lean_Meta_evalName___closed__10; x_161 = lean_name_eq(x_93, x_160); if (x_161 == 0) diff --git a/stage0/stdlib/Lean/Meta/SizeOf.c b/stage0/stdlib/Lean/Meta/SizeOf.c index 2ab33a381018..086ae54b5728 100644 --- a/stage0/stdlib/Lean/Meta/SizeOf.c +++ b/stage0/stdlib/Lean/Meta/SizeOf.c @@ -208,6 +208,7 @@ LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_SizeOf_0__Le LEAN_EXPORT lean_object* l_Lean_logAt___at___private_Lean_Meta_SizeOf_0__Lean_Meta_SizeOfSpecNested_mkSizeOfAuxLemma___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_SizeOf_0__Lean_Meta_SizeOfSpecNested_mkSizeOfAuxLemmaProof___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_SizeOf_0__Lean_Meta_mkSizeOfMinors_loop___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_setEnv___at___private_Lean_Meta_SizeOf_0__Lean_Meta_SizeOfSpecNested_mkSizeOfAuxLemma___spec__5___closed__3; lean_object* l_Std_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkSizeOfFn___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -318,7 +319,6 @@ static lean_object* l___private_Lean_Meta_SizeOf_0__Lean_Meta_mkSizeOfSpecTheore lean_object* lean_name_append_after(lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Std_Format_initFn____x40_Lean_Data_Format___hyg_57____spec__1(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_SizeOf_0__Lean_Meta_SizeOfSpecNested_mkMinorProof___lambda__1___closed__6; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_mkSizeOfInstances___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwKernelException___at_Lean_Meta_mkSizeOfFn___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2596,7 +2596,7 @@ static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Meta_Size lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_SizeOf_0__Lean_Meta_mkSizeOfMinors_loop___spec__1___closed__2; x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_SizeOf_0__Lean_Meta_mkSizeOfMinors_loop___spec__1___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Array_forInUnsafe_loop___at___private_Lean_Meta_SizeOf_0__Lean_Meta_mkSizeOfMinors_loop___spec__1___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -7826,7 +7826,7 @@ x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); lean_dec(x_20); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_1, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_22); x_24 = l_Lean_Meta_mkSizeOfSpecLemmaInstance___closed__3; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -8376,7 +8376,7 @@ x_30 = lean_ctor_get(x_23, 0); lean_inc(x_30); lean_dec(x_23); x_31 = lean_unsigned_to_nat(0u); -x_32 = l_Lean_Expr_getAppNumArgsAux(x_1, x_31); +x_32 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_31); x_33 = l_Lean_Meta_mkSizeOfSpecLemmaInstance___closed__3; lean_inc(x_32); x_34 = lean_mk_array(x_32, x_33); @@ -8532,7 +8532,7 @@ x_88 = lean_ctor_get(x_81, 0); lean_inc(x_88); lean_dec(x_81); x_89 = lean_unsigned_to_nat(0u); -x_90 = l_Lean_Expr_getAppNumArgsAux(x_1, x_89); +x_90 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_89); x_91 = l_Lean_Meta_mkSizeOfSpecLemmaInstance___closed__3; lean_inc(x_90); x_92 = lean_mk_array(x_90, x_91); @@ -12028,7 +12028,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_SizeOf_0__Lean_Meta_SizeOfSpecNes { 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; x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_1, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_17); lean_inc(x_18); x_19 = lean_mk_array(x_18, x_2); x_20 = lean_unsigned_to_nat(1u); @@ -12531,7 +12531,7 @@ x_40 = lean_ctor_get(x_39, 0); lean_inc(x_40); lean_dec(x_39); x_41 = lean_unsigned_to_nat(0u); -x_42 = l_Lean_Expr_getAppNumArgsAux(x_29, x_41); +x_42 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_29, x_41); x_43 = l_Lean_Meta_mkSizeOfSpecLemmaInstance___closed__3; lean_inc(x_42); x_44 = lean_mk_array(x_42, x_43); @@ -12720,7 +12720,7 @@ lean_dec(x_4); lean_dec(x_2); x_71 = l_Lean_Expr_const___override(x_17, x_12); x_72 = lean_unsigned_to_nat(0u); -x_73 = l_Lean_Expr_getAppNumArgsAux(x_1, x_72); +x_73 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_72); x_74 = l_Lean_Meta_mkSizeOfSpecLemmaInstance___closed__3; lean_inc(x_73); x_75 = lean_mk_array(x_73, x_74); @@ -12819,7 +12819,7 @@ x_100 = lean_ctor_get(x_99, 0); lean_inc(x_100); lean_dec(x_99); x_101 = lean_unsigned_to_nat(0u); -x_102 = l_Lean_Expr_getAppNumArgsAux(x_89, x_101); +x_102 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_89, x_101); x_103 = l_Lean_Meta_mkSizeOfSpecLemmaInstance___closed__3; lean_inc(x_102); x_104 = lean_mk_array(x_102, x_103); @@ -13014,7 +13014,7 @@ lean_dec(x_4); lean_dec(x_2); x_131 = l_Lean_Expr_const___override(x_17, x_12); x_132 = lean_unsigned_to_nat(0u); -x_133 = l_Lean_Expr_getAppNumArgsAux(x_1, x_132); +x_133 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_132); x_134 = l_Lean_Meta_mkSizeOfSpecLemmaInstance___closed__3; lean_inc(x_133); x_135 = lean_mk_array(x_133, x_134); @@ -14631,7 +14631,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_SizeOf_0__Lean_Meta_SizeOfSpecNes { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Expr_getAppNumArgsAux(x_2, x_9); +x_10 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_9); x_11 = l_Lean_Meta_mkSizeOfSpecLemmaInstance___closed__3; lean_inc(x_10); x_12 = lean_mk_array(x_10, x_11); @@ -14683,7 +14683,7 @@ lean_inc(x_30); x_31 = lean_ctor_get(x_29, 1); lean_inc(x_31); lean_dec(x_29); -x_32 = l_Lean_Expr_getAppNumArgsAux(x_30, x_9); +x_32 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_30, x_9); lean_inc(x_32); x_33 = lean_mk_array(x_32, x_11); x_34 = lean_nat_sub(x_32, x_13); diff --git a/stage0/stdlib/Lean/Meta/SynthInstance.c b/stage0/stdlib/Lean/Meta/SynthInstance.c index 66e864cdc102..0ac3f6e9e1e4 100644 --- a/stage0/stdlib/Lean/Meta/SynthInstance.c +++ b/stage0/stdlib/Lean/Meta/SynthInstance.c @@ -19,7 +19,6 @@ LEAN_EXPORT lean_object* l_Lean_Core_withCurrHeartbeats___at_Lean_Meta_SynthInst LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_getMaxHeartbeats___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_Meta_synthInstance_x3f___spec__6(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_instInhabitedAnswer___closed__1; static lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_preprocessArgs___closed__2; @@ -40,6 +39,7 @@ static lean_object* l_Lean_Meta_SynthInstance_getMaxHeartbeats___closed__1; static lean_object* l_Lean_Meta_SynthInstance_instInhabitedAnswer___closed__2; lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_getTop(lean_object*); +lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_preprocessArgs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_MkTableKey_normLevel(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); @@ -50,6 +50,7 @@ uint8_t l_Std_PersistentHashMap_contains___at_Lean_isExprMVarAssigned___spec__1( LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_Meta_synthInstance_x3f___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_State_resumeStack___default; +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_tryAnswer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Option_toLOption___rarg(lean_object*); LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_SynthInstance_MkTableKey_normExpr___spec__2(lean_object*, lean_object*); @@ -60,7 +61,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_tryAnswer___lambda__1___boxed LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_MkTableKey_State_emap___default; static lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_mkAnswer___lambda__2___closed__3; static lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_preprocessLevels___closed__1; -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); +lean_object* l_Lean_Level_succ___override(lean_object*); static lean_object* l_Lean_Meta_SynthInstance_addAnswer___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withMCtx___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_mkAnswer___spec__1(lean_object*); extern lean_object* l_Lean_maxRecDepthErrorMessage; @@ -82,6 +83,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_getResult(lean_object*); size_t lean_usize_sub(size_t, size_t); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_SynthInstance_isNewAnswer___spec__1(lean_object*, lean_object*, size_t, size_t); uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); uint8_t l_Lean_Level_hasMVar(lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_instInhabitedGeneratorNode___closed__1; @@ -111,6 +113,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_addAnswer___lambda__1(lean_ob lean_object* l_Std_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); static lean_object* l_Lean_Meta_SynthInstance_newSubgoal___lambda__3___closed__1; lean_object* l_Lean_Meta_isClass_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_tryResolveCore___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_instInhabitedSynthM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_MkTableKey_instMonadMCtxM___lambda__1(lean_object*, lean_object*); @@ -120,6 +123,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_resume(lean_object*, lean_obj static lean_object* l_Lean_Meta_synthInstance_x3f___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_Meta_synthInstance_x3f___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_tryResolveCore___lambda__4___closed__4; +uint8_t l_ptrEqList___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_synthInstance_x3f___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_SynthInstance___hyg_6____closed__1; LEAN_EXPORT lean_object* l_StateT_get___at_Lean_Meta_SynthInstance_MkTableKey_instMonadMCtxM___spec__1(lean_object*); @@ -170,6 +174,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthI static lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_mkAnswer___closed__2; uint8_t lean_expr_has_loose_bvar(lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); +lean_object* l_Lean_simpLevelIMax_x27(lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_SynthInstance_isNewAnswer___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -231,17 +236,18 @@ static lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Meta_SynthInst LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_mapMetaM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isExprMVarAssignable___at_Lean_Meta_SynthInstance_tryResolveCore___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_SynthInstance_getInstances___spec__6(lean_object*, lean_object*, size_t, size_t, lean_object*); -lean_object* lean_level_update_max(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_instInhabitedGeneratorNode; LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Meta_SynthInstance_getInstances___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_tryResolveCore___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_isDefEqStuckExceptionId; LEAN_EXPORT lean_object* l_Lean_isLevelMVarAssignable___at_Lean_Meta_SynthInstance_tryResolveCore___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); uint8_t lean_is_out_param(lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_generate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_simpLevelMax_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_initFn____x40_Lean_Meta_SynthInstance___hyg_75____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_CoreM_0__Lean_Core_withCurrHeartbeatsImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -260,6 +266,7 @@ lean_object* l_instInhabited___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_main___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_modifyTop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Meta_SynthInstance_newSubgoal___spec__7(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_MkTableKey_instMonadMCtxM___lambda__2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_mkTableKeyFor___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_newSubgoal___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -270,6 +277,7 @@ lean_object* l_Std_HashMapImp_find_x3f___at___private_Lean_Meta_AbstractMVars_0_ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_TableEntry_answers___default; static lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_preprocessArgs___closed__1; lean_object* l_Lean_markUsedAssignment___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_synthInstance_x3f___lambda__5___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_addAnswer___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); @@ -340,7 +348,6 @@ lean_object* l_Lean_Expr_bvar___override(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_preprocessOutParam(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_instMonadMetaM; LEAN_EXPORT lean_object* l_Lean_isExprMVarAssignable___at_Lean_Meta_SynthInstance_MkTableKey_normExpr___spec__1(lean_object*, lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isForall(lean_object*); uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -364,7 +371,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_getNextToResume___boxed(lean_ LEAN_EXPORT lean_object* l_List_anyM___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_resume___closed__7; -lean_object* lean_expr_update_proj(lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_preprocessLevels___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceOptions(lean_object*); @@ -395,10 +401,10 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_State_result_x3f___default; lean_object* l_Lean_Meta_DiscrTree_getUnify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Meta_SynthInstance_getInstances___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_fvar___override(lean_object*); +size_t lean_ptr_addr(lean_object*); static lean_object* l_Lean_Meta_SynthInstance_wakeUp___closed__2; lean_object* l_Lean_Core_checkMaxHeartbeatsCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_tryResolveCore___lambda__3___closed__6; -lean_object* lean_level_update_imax(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_synthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_redLength___rarg(lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); @@ -407,8 +413,8 @@ static lean_object* l_Lean_Meta_SynthInstance_getInstances___lambda__2___closed_ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_State_tableEntries___default; static lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_trySynthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Meta_SynthInstance_tryResolve___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMCtxImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern uint8_t l_instInhabitedBool; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_SynthInstance_consume___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -425,7 +431,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthI static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_SynthInstance_getInstances___spec__5___closed__4; lean_object* l_Lean_throwError___at_Lean_Meta_abstractRange___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_resume___closed__6; -lean_object* lean_expr_update_sort(lean_object*, lean_object*); extern lean_object* l_Id_instMonadId; LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_synth___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_wakeUp___closed__1; @@ -485,12 +490,10 @@ lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_tryResolveCore___lambda__3___closed__5; lean_object* l_List_toArrayAux___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_SynthInstance_main___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_getMaxHeartbeats(lean_object*); -lean_object* lean_level_update_succ(lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_tryResolve___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_Std_PersistentHashMap_insert___at_Lean_Meta_synthInstance_x3f___spec__4(lean_object*, lean_object*, lean_object*); @@ -517,6 +520,7 @@ lean_object* lean_array_pop(lean_object*); static lean_object* l_Lean_Meta_SynthInstance_tryResolveCore___lambda__3___closed__3; lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l_Lean_Meta_synthInstance_x3f___closed__1; +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); static size_t l_Std_PersistentHashMap_findAux___at_Lean_Meta_synthInstance_x3f___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_tryResolveCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_Meta_synthInstance_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); @@ -530,6 +534,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_consume___lambda__2___boxed(l LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_MkTableKey_State_nextIdx___default; LEAN_EXPORT lean_object* l_Lean_Meta_withMCtx___at_Lean_Meta_SynthInstance_newSubgoal___spec__10(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_SynthInstance_addAnswer___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_generate___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SynthInstance_instInhabitedGeneratorNode___closed__2; LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_Meta_synthInstance_x3f___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -552,7 +557,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_getInstances___lambda__1(lean static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_SynthInstance___hyg_6____closed__7; LEAN_EXPORT uint8_t l_Std_AssocList_contains___at_Lean_Meta_SynthInstance_newSubgoal___spec__4(lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); -lean_object* lean_expr_update_app(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addTrace___at_Lean_Meta_SynthInstance_newSubgoal___spec__9___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_tryResolveCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_getInstances___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -588,7 +592,6 @@ static lean_object* l___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstan uint8_t lean_has_out_params(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_SynthInstance_mkTableKeyFor___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_SynthInstance_removeUnusedArguments_x3f___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_expr_update_const(lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__7___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_SynthInstance_consume___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_SynthInstance_main___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1505,271 +1508,457 @@ case 1: lean_object* x_5; lean_object* x_6; uint8_t x_7; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); +lean_inc(x_5); x_6 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_5, x_2); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) { -lean_object* x_8; lean_object* x_9; +lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_level_update_succ(x_1, x_8); -lean_ctor_set(x_6, 0, x_9); +x_9 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_10 = lean_ptr_addr(x_8); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_1); +x_12 = l_Lean_Level_succ___override(x_8); +lean_ctor_set(x_6, 0, x_12); return x_6; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_6, 0); -x_11 = lean_ctor_get(x_6, 1); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_6); -x_12 = lean_level_update_succ(x_1, x_10); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +lean_dec(x_8); +lean_ctor_set(x_6, 0, x_1); +return x_6; } } -case 2: +else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_14 = lean_ctor_get(x_1, 0); +lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_6, 0); +x_14 = lean_ctor_get(x_6, 1); lean_inc(x_14); -x_15 = lean_ctor_get(x_1, 1); -lean_inc(x_15); -x_16 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_14, x_2); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_15, x_18); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +lean_inc(x_13); +lean_dec(x_6); +x_15 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_16 = lean_ptr_addr(x_13); +x_17 = lean_usize_dec_eq(x_15, x_16); +if (x_17 == 0) { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_level_update_max(x_1, x_17, x_21); -lean_ctor_set(x_19, 0, x_22); +lean_object* x_18; lean_object* x_19; +lean_dec(x_1); +x_18 = l_Lean_Level_succ___override(x_13); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_14); return x_19; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_19, 0); -x_24 = lean_ctor_get(x_19, 1); +lean_object* x_20; +lean_dec(x_13); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_1); +lean_ctor_set(x_20, 1, x_14); +return x_20; +} +} +} +case 2: +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_21 = lean_ctor_get(x_1, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_1, 1); +lean_inc(x_22); +lean_inc(x_21); +x_23 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_21, x_2); +x_24 = lean_ctor_get(x_23, 0); lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_19); -x_25 = lean_level_update_max(x_1, x_17, x_23); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +lean_inc(x_22); +x_26 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_22, x_25); +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) +{ +lean_object* x_28; size_t x_29; size_t x_30; uint8_t x_31; +x_28 = lean_ctor_get(x_26, 0); +x_29 = lean_ptr_addr(x_21); +lean_dec(x_21); +x_30 = lean_ptr_addr(x_24); +x_31 = lean_usize_dec_eq(x_29, x_30); +if (x_31 == 0) +{ +lean_object* x_32; +lean_dec(x_22); +lean_dec(x_1); +x_32 = l_Lean_mkLevelMax_x27(x_24, x_28); +lean_ctor_set(x_26, 0, x_32); return x_26; } -} -case 3: +else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_27 = lean_ctor_get(x_1, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_1, 1); -lean_inc(x_28); -x_29 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_27, x_2); -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_28, x_31); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) +size_t x_33; size_t x_34; uint8_t x_35; +x_33 = lean_ptr_addr(x_22); +lean_dec(x_22); +x_34 = lean_ptr_addr(x_28); +x_35 = lean_usize_dec_eq(x_33, x_34); +if (x_35 == 0) { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_level_update_imax(x_1, x_30, x_34); -lean_ctor_set(x_32, 0, x_35); -return x_32; +lean_object* x_36; +lean_dec(x_1); +x_36 = l_Lean_mkLevelMax_x27(x_24, x_28); +lean_ctor_set(x_26, 0, x_36); +return x_26; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_32, 0); -x_37 = lean_ctor_get(x_32, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_32); -x_38 = lean_level_update_imax(x_1, x_30, x_36); -x_39 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_37); -return x_39; +lean_object* x_37; +x_37 = l_Lean_simpLevelMax_x27(x_24, x_28, x_1); +lean_dec(x_1); +lean_dec(x_28); +lean_dec(x_24); +lean_ctor_set(x_26, 0, x_37); +return x_26; } } -case 5: -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_40 = lean_ctor_get(x_1, 0); -lean_inc(x_40); -lean_inc(x_40); -x_41 = l_Lean_isLevelMVarAssignable___at_Lean_Meta_SynthInstance_MkTableKey_normLevel___spec__1(x_40, x_2); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_unbox(x_42); -lean_dec(x_42); -if (x_43 == 0) +} +else { -uint8_t x_44; -lean_dec(x_40); -x_44 = !lean_is_exclusive(x_41); -if (x_44 == 0) +lean_object* x_38; lean_object* x_39; size_t x_40; size_t x_41; uint8_t x_42; +x_38 = lean_ctor_get(x_26, 0); +x_39 = lean_ctor_get(x_26, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_26); +x_40 = lean_ptr_addr(x_21); +lean_dec(x_21); +x_41 = lean_ptr_addr(x_24); +x_42 = lean_usize_dec_eq(x_40, x_41); +if (x_42 == 0) { -lean_object* x_45; -x_45 = lean_ctor_get(x_41, 0); -lean_dec(x_45); -lean_ctor_set(x_41, 0, x_1); -return x_41; +lean_object* x_43; lean_object* x_44; +lean_dec(x_22); +lean_dec(x_1); +x_43 = l_Lean_mkLevelMax_x27(x_24, x_38); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_39); +return x_44; } else { -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_41, 1); -lean_inc(x_46); -lean_dec(x_41); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_1); -lean_ctor_set(x_47, 1, x_46); -return x_47; -} +size_t x_45; size_t x_46; uint8_t x_47; +x_45 = lean_ptr_addr(x_22); +lean_dec(x_22); +x_46 = lean_ptr_addr(x_38); +x_47 = lean_usize_dec_eq(x_45, x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; +lean_dec(x_1); +x_48 = l_Lean_mkLevelMax_x27(x_24, x_38); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_39); +return x_49; } else { -uint8_t x_48; +lean_object* x_50; lean_object* x_51; +x_50 = l_Lean_simpLevelMax_x27(x_24, x_38, x_1); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_41); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_49 = lean_ctor_get(x_41, 1); -x_50 = lean_ctor_get(x_41, 0); -lean_dec(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_inc(x_40); -lean_inc(x_51); -x_52 = l_Std_HashMapImp_find_x3f___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__1(x_51, x_40); -if (lean_obj_tag(x_52) == 0) +lean_dec(x_38); +lean_dec(x_24); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_39); +return x_51; +} +} +} +} +case 3: { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_53 = lean_ctor_get(x_49, 0); -lean_inc(x_53); -x_54 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel___closed__2; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; +x_52 = lean_ctor_get(x_1, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_1, 1); lean_inc(x_53); -x_55 = l_Lean_Name_num___override(x_54, x_53); -x_56 = l_Lean_Level_param___override(x_55); -x_57 = lean_unsigned_to_nat(1u); -x_58 = lean_nat_add(x_53, x_57); -lean_dec(x_53); +lean_inc(x_52); +x_54 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_52, x_2); +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_59 = l_Std_HashMap_insert___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__3(x_51, x_40, x_56); -x_60 = lean_ctor_get(x_49, 2); -lean_inc(x_60); -x_61 = lean_ctor_get(x_49, 3); -lean_inc(x_61); -lean_dec(x_49); -x_62 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_62, 0, x_58); -lean_ctor_set(x_62, 1, x_59); -lean_ctor_set(x_62, 2, x_60); -lean_ctor_set(x_62, 3, x_61); -lean_ctor_set(x_41, 1, x_62); -lean_ctor_set(x_41, 0, x_56); -return x_41; -} -else +lean_dec(x_54); +lean_inc(x_53); +x_57 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_53, x_56); +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) { -lean_object* x_63; -lean_dec(x_51); -lean_dec(x_40); -x_63 = lean_ctor_get(x_52, 0); -lean_inc(x_63); +lean_object* x_59; size_t x_60; size_t x_61; uint8_t x_62; +x_59 = lean_ctor_get(x_57, 0); +x_60 = lean_ptr_addr(x_52); lean_dec(x_52); -lean_ctor_set(x_41, 0, x_63); -return x_41; -} +x_61 = lean_ptr_addr(x_55); +x_62 = lean_usize_dec_eq(x_60, x_61); +if (x_62 == 0) +{ +lean_object* x_63; +lean_dec(x_53); +lean_dec(x_1); +x_63 = l_Lean_mkLevelIMax_x27(x_55, x_59); +lean_ctor_set(x_57, 0, x_63); +return x_57; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_41, 1); -lean_inc(x_64); -lean_dec(x_41); -x_65 = lean_ctor_get(x_64, 1); -lean_inc(x_65); -lean_inc(x_40); -lean_inc(x_65); -x_66 = l_Std_HashMapImp_find_x3f___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__1(x_65, x_40); -if (lean_obj_tag(x_66) == 0) +size_t x_64; size_t x_65; uint8_t x_66; +x_64 = lean_ptr_addr(x_53); +lean_dec(x_53); +x_65 = lean_ptr_addr(x_59); +x_66 = lean_usize_dec_eq(x_64, x_65); +if (x_66 == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_67 = lean_ctor_get(x_64, 0); -lean_inc(x_67); -x_68 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel___closed__2; -lean_inc(x_67); -x_69 = l_Lean_Name_num___override(x_68, x_67); -x_70 = l_Lean_Level_param___override(x_69); -x_71 = lean_unsigned_to_nat(1u); -x_72 = lean_nat_add(x_67, x_71); -lean_dec(x_67); -lean_inc(x_70); -x_73 = l_Std_HashMap_insert___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__3(x_65, x_40, x_70); -x_74 = lean_ctor_get(x_64, 2); -lean_inc(x_74); -x_75 = lean_ctor_get(x_64, 3); -lean_inc(x_75); -lean_dec(x_64); -x_76 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_76, 0, x_72); -lean_ctor_set(x_76, 1, x_73); -lean_ctor_set(x_76, 2, x_74); -lean_ctor_set(x_76, 3, x_75); -x_77 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_77, 0, x_70); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_67; +lean_dec(x_1); +x_67 = l_Lean_mkLevelIMax_x27(x_55, x_59); +lean_ctor_set(x_57, 0, x_67); +return x_57; } else { -lean_object* x_78; lean_object* x_79; -lean_dec(x_65); -lean_dec(x_40); -x_78 = lean_ctor_get(x_66, 0); -lean_inc(x_78); -lean_dec(x_66); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_78); -lean_ctor_set(x_79, 1, x_64); -return x_79; +lean_object* x_68; +x_68 = l_Lean_simpLevelIMax_x27(x_55, x_59, x_1); +lean_dec(x_1); +lean_ctor_set(x_57, 0, x_68); +return x_57; } } } +else +{ +lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; uint8_t x_73; +x_69 = lean_ctor_get(x_57, 0); +x_70 = lean_ctor_get(x_57, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_57); +x_71 = lean_ptr_addr(x_52); +lean_dec(x_52); +x_72 = lean_ptr_addr(x_55); +x_73 = lean_usize_dec_eq(x_71, x_72); +if (x_73 == 0) +{ +lean_object* x_74; lean_object* x_75; +lean_dec(x_53); +lean_dec(x_1); +x_74 = l_Lean_mkLevelIMax_x27(x_55, x_69); +x_75 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_70); +return x_75; } -default: +else +{ +size_t x_76; size_t x_77; uint8_t x_78; +x_76 = lean_ptr_addr(x_53); +lean_dec(x_53); +x_77 = lean_ptr_addr(x_69); +x_78 = lean_usize_dec_eq(x_76, x_77); +if (x_78 == 0) { -lean_object* x_80; +lean_object* x_79; lean_object* x_80; +lean_dec(x_1); +x_79 = l_Lean_mkLevelIMax_x27(x_55, x_69); x_80 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_80, 0, x_1); -lean_ctor_set(x_80, 1, x_2); +lean_ctor_set(x_80, 0, x_79); +lean_ctor_set(x_80, 1, x_70); return x_80; } +else +{ +lean_object* x_81; lean_object* x_82; +x_81 = l_Lean_simpLevelIMax_x27(x_55, x_69, x_1); +lean_dec(x_1); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_70); +return x_82; } } } } -LEAN_EXPORT lean_object* l_Lean_isExprMVarAssignable___at_Lean_Meta_SynthInstance_MkTableKey_normExpr___spec__1(lean_object* x_1, lean_object* x_2) { -_start: +case 5: { -lean_object* x_3; uint8_t x_4; +lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; +x_83 = lean_ctor_get(x_1, 0); +lean_inc(x_83); +lean_inc(x_83); +x_84 = l_Lean_isLevelMVarAssignable___at_Lean_Meta_SynthInstance_MkTableKey_normLevel___spec__1(x_83, x_2); +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) +{ +uint8_t x_87; +lean_dec(x_83); +x_87 = !lean_is_exclusive(x_84); +if (x_87 == 0) +{ +lean_object* x_88; +x_88 = lean_ctor_get(x_84, 0); +lean_dec(x_88); +lean_ctor_set(x_84, 0, x_1); +return x_84; +} +else +{ +lean_object* x_89; lean_object* x_90; +x_89 = lean_ctor_get(x_84, 1); +lean_inc(x_89); +lean_dec(x_84); +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_1); +lean_ctor_set(x_90, 1, x_89); +return x_90; +} +} +else +{ +uint8_t x_91; +lean_dec(x_1); +x_91 = !lean_is_exclusive(x_84); +if (x_91 == 0) +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_92 = lean_ctor_get(x_84, 1); +x_93 = lean_ctor_get(x_84, 0); +lean_dec(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +lean_inc(x_83); +lean_inc(x_94); +x_95 = l_Std_HashMapImp_find_x3f___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__1(x_94, x_83); +if (lean_obj_tag(x_95) == 0) +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_96 = lean_ctor_get(x_92, 0); +lean_inc(x_96); +x_97 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel___closed__2; +lean_inc(x_96); +x_98 = l_Lean_Name_num___override(x_97, x_96); +x_99 = l_Lean_Level_param___override(x_98); +x_100 = lean_unsigned_to_nat(1u); +x_101 = lean_nat_add(x_96, x_100); +lean_dec(x_96); +lean_inc(x_99); +x_102 = l_Std_HashMap_insert___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__3(x_94, x_83, x_99); +x_103 = lean_ctor_get(x_92, 2); +lean_inc(x_103); +x_104 = lean_ctor_get(x_92, 3); +lean_inc(x_104); +lean_dec(x_92); +x_105 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_105, 0, x_101); +lean_ctor_set(x_105, 1, x_102); +lean_ctor_set(x_105, 2, x_103); +lean_ctor_set(x_105, 3, x_104); +lean_ctor_set(x_84, 1, x_105); +lean_ctor_set(x_84, 0, x_99); +return x_84; +} +else +{ +lean_object* x_106; +lean_dec(x_94); +lean_dec(x_83); +x_106 = lean_ctor_get(x_95, 0); +lean_inc(x_106); +lean_dec(x_95); +lean_ctor_set(x_84, 0, x_106); +return x_84; +} +} +else +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_84, 1); +lean_inc(x_107); +lean_dec(x_84); +x_108 = lean_ctor_get(x_107, 1); +lean_inc(x_108); +lean_inc(x_83); +lean_inc(x_108); +x_109 = l_Std_HashMapImp_find_x3f___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__1(x_108, x_83); +if (lean_obj_tag(x_109) == 0) +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_110 = lean_ctor_get(x_107, 0); +lean_inc(x_110); +x_111 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel___closed__2; +lean_inc(x_110); +x_112 = l_Lean_Name_num___override(x_111, x_110); +x_113 = l_Lean_Level_param___override(x_112); +x_114 = lean_unsigned_to_nat(1u); +x_115 = lean_nat_add(x_110, x_114); +lean_dec(x_110); +lean_inc(x_113); +x_116 = l_Std_HashMap_insert___at___private_Lean_Meta_AbstractMVars_0__Lean_Meta_AbstractMVars_abstractLevelMVars___spec__3(x_108, x_83, x_113); +x_117 = lean_ctor_get(x_107, 2); +lean_inc(x_117); +x_118 = lean_ctor_get(x_107, 3); +lean_inc(x_118); +lean_dec(x_107); +x_119 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_119, 0, x_115); +lean_ctor_set(x_119, 1, x_116); +lean_ctor_set(x_119, 2, x_117); +lean_ctor_set(x_119, 3, x_118); +x_120 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_120, 0, x_113); +lean_ctor_set(x_120, 1, x_119); +return x_120; +} +else +{ +lean_object* x_121; lean_object* x_122; +lean_dec(x_108); +lean_dec(x_83); +x_121 = lean_ctor_get(x_109, 0); +lean_inc(x_121); +lean_dec(x_109); +x_122 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_122, 0, x_121); +lean_ctor_set(x_122, 1, x_107); +return x_122; +} +} +} +} +default: +{ +lean_object* x_123; +x_123 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_123, 0, x_1); +lean_ctor_set(x_123, 1, x_2); +return x_123; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_isExprMVarAssignable___at_Lean_Meta_SynthInstance_MkTableKey_normExpr___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; uint8_t x_4; x_3 = l_Lean_markUsedAssignment___at_Lean_Meta_SynthInstance_MkTableKey_normLevel___spec__2(x_2); x_4 = !lean_is_exclusive(x_3); if (x_4 == 0) @@ -2084,293 +2273,861 @@ return x_44; } case 3: { -lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_45 = lean_ctor_get(x_1, 0); -lean_inc(x_45); -x_46 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_45, x_2); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_45 = lean_ctor_get(x_1, 0); +lean_inc(x_45); +lean_inc(x_45); +x_46 = l_Lean_Meta_SynthInstance_MkTableKey_normLevel(x_45, x_2); +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) +{ +lean_object* x_48; size_t x_49; size_t x_50; uint8_t x_51; +x_48 = lean_ctor_get(x_46, 0); +x_49 = lean_ptr_addr(x_45); +lean_dec(x_45); +x_50 = lean_ptr_addr(x_48); +x_51 = lean_usize_dec_eq(x_49, x_50); +if (x_51 == 0) +{ +lean_object* x_52; +lean_dec(x_1); +x_52 = l_Lean_Expr_sort___override(x_48); +lean_ctor_set(x_46, 0, x_52); +return x_46; +} +else +{ +lean_dec(x_48); +lean_ctor_set(x_46, 0, x_1); +return x_46; +} +} +else +{ +lean_object* x_53; lean_object* x_54; size_t x_55; size_t x_56; uint8_t x_57; +x_53 = lean_ctor_get(x_46, 0); +x_54 = lean_ctor_get(x_46, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_46); +x_55 = lean_ptr_addr(x_45); +lean_dec(x_45); +x_56 = lean_ptr_addr(x_53); +x_57 = lean_usize_dec_eq(x_55, x_56); +if (x_57 == 0) +{ +lean_object* x_58; lean_object* x_59; +lean_dec(x_1); +x_58 = l_Lean_Expr_sort___override(x_53); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_54); +return x_59; +} +else +{ +lean_object* x_60; +lean_dec(x_53); +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_1); +lean_ctor_set(x_60, 1, x_54); +return x_60; +} +} +} +case 4: +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; +x_61 = lean_ctor_get(x_1, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_1, 1); +lean_inc(x_62); +lean_inc(x_62); +x_63 = l_List_mapM___at_Lean_Meta_SynthInstance_MkTableKey_normExpr___spec__2(x_62, x_2); +x_64 = !lean_is_exclusive(x_63); +if (x_64 == 0) +{ +lean_object* x_65; uint8_t x_66; +x_65 = lean_ctor_get(x_63, 0); +x_66 = l_ptrEqList___rarg(x_62, x_65); +lean_dec(x_62); +if (x_66 == 0) +{ +lean_object* x_67; +lean_dec(x_1); +x_67 = l_Lean_Expr_const___override(x_61, x_65); +lean_ctor_set(x_63, 0, x_67); +return x_63; +} +else +{ +lean_dec(x_65); +lean_dec(x_61); +lean_ctor_set(x_63, 0, x_1); +return x_63; +} +} +else +{ +lean_object* x_68; lean_object* x_69; uint8_t x_70; +x_68 = lean_ctor_get(x_63, 0); +x_69 = lean_ctor_get(x_63, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_63); +x_70 = l_ptrEqList___rarg(x_62, x_68); +lean_dec(x_62); +if (x_70 == 0) +{ +lean_object* x_71; lean_object* x_72; +lean_dec(x_1); +x_71 = l_Lean_Expr_const___override(x_61, x_68); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_69); +return x_72; +} +else +{ +lean_object* x_73; +lean_dec(x_68); +lean_dec(x_61); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_1); +lean_ctor_set(x_73, 1, x_69); +return x_73; +} +} +} +case 5: +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; +x_74 = lean_ctor_get(x_1, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_1, 1); +lean_inc(x_75); +lean_inc(x_74); +x_76 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_74, x_2); +x_77 = lean_ctor_get(x_76, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_76, 1); +lean_inc(x_78); +lean_dec(x_76); +lean_inc(x_75); +x_79 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_75, x_78); +x_80 = !lean_is_exclusive(x_79); +if (x_80 == 0) +{ +lean_object* x_81; size_t x_82; size_t x_83; uint8_t x_84; +x_81 = lean_ctor_get(x_79, 0); +x_82 = lean_ptr_addr(x_74); +lean_dec(x_74); +x_83 = lean_ptr_addr(x_77); +x_84 = lean_usize_dec_eq(x_82, x_83); +if (x_84 == 0) +{ +lean_object* x_85; +lean_dec(x_75); +lean_dec(x_1); +x_85 = l_Lean_Expr_app___override(x_77, x_81); +lean_ctor_set(x_79, 0, x_85); +return x_79; +} +else +{ +size_t x_86; size_t x_87; uint8_t x_88; +x_86 = lean_ptr_addr(x_75); +lean_dec(x_75); +x_87 = lean_ptr_addr(x_81); +x_88 = lean_usize_dec_eq(x_86, x_87); +if (x_88 == 0) +{ +lean_object* x_89; +lean_dec(x_1); +x_89 = l_Lean_Expr_app___override(x_77, x_81); +lean_ctor_set(x_79, 0, x_89); +return x_79; +} +else +{ +lean_dec(x_81); +lean_dec(x_77); +lean_ctor_set(x_79, 0, x_1); +return x_79; +} +} +} +else +{ +lean_object* x_90; lean_object* x_91; size_t x_92; size_t x_93; uint8_t x_94; +x_90 = lean_ctor_get(x_79, 0); +x_91 = lean_ctor_get(x_79, 1); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_79); +x_92 = lean_ptr_addr(x_74); +lean_dec(x_74); +x_93 = lean_ptr_addr(x_77); +x_94 = lean_usize_dec_eq(x_92, x_93); +if (x_94 == 0) +{ +lean_object* x_95; lean_object* x_96; +lean_dec(x_75); +lean_dec(x_1); +x_95 = l_Lean_Expr_app___override(x_77, x_90); +x_96 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_95); +lean_ctor_set(x_96, 1, x_91); +return x_96; +} +else +{ +size_t x_97; size_t x_98; uint8_t x_99; +x_97 = lean_ptr_addr(x_75); +lean_dec(x_75); +x_98 = lean_ptr_addr(x_90); +x_99 = lean_usize_dec_eq(x_97, x_98); +if (x_99 == 0) +{ +lean_object* x_100; lean_object* x_101; +lean_dec(x_1); +x_100 = l_Lean_Expr_app___override(x_77, x_90); +x_101 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_91); +return x_101; +} +else +{ +lean_object* x_102; +lean_dec(x_90); +lean_dec(x_77); +x_102 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_102, 0, x_1); +lean_ctor_set(x_102, 1, x_91); +return x_102; +} +} +} +} +case 6: +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; uint8_t x_111; +x_103 = lean_ctor_get(x_1, 0); +lean_inc(x_103); +x_104 = lean_ctor_get(x_1, 1); +lean_inc(x_104); +x_105 = lean_ctor_get(x_1, 2); +lean_inc(x_105); +x_106 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_104); +x_107 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_104, x_2); +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +lean_inc(x_105); +x_110 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_105, x_109); +x_111 = !lean_is_exclusive(x_110); +if (x_111 == 0) +{ +lean_object* x_112; lean_object* x_113; size_t x_114; size_t x_115; uint8_t x_116; +x_112 = lean_ctor_get(x_110, 0); +lean_inc(x_105); +lean_inc(x_104); +lean_inc(x_103); +x_113 = l_Lean_Expr_lam___override(x_103, x_104, x_105, x_106); +x_114 = lean_ptr_addr(x_104); +lean_dec(x_104); +x_115 = lean_ptr_addr(x_108); +x_116 = lean_usize_dec_eq(x_114, x_115); +if (x_116 == 0) +{ +lean_object* x_117; +lean_dec(x_113); +lean_dec(x_105); +x_117 = l_Lean_Expr_lam___override(x_103, x_108, x_112, x_106); +lean_ctor_set(x_110, 0, x_117); +return x_110; +} +else +{ +size_t x_118; size_t x_119; uint8_t x_120; +x_118 = lean_ptr_addr(x_105); +lean_dec(x_105); +x_119 = lean_ptr_addr(x_112); +x_120 = lean_usize_dec_eq(x_118, x_119); +if (x_120 == 0) +{ +lean_object* x_121; +lean_dec(x_113); +x_121 = l_Lean_Expr_lam___override(x_103, x_108, x_112, x_106); +lean_ctor_set(x_110, 0, x_121); +return x_110; +} +else +{ +uint8_t x_122; +x_122 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_106, x_106); +if (x_122 == 0) +{ +lean_object* x_123; +lean_dec(x_113); +x_123 = l_Lean_Expr_lam___override(x_103, x_108, x_112, x_106); +lean_ctor_set(x_110, 0, x_123); +return x_110; +} +else +{ +lean_dec(x_112); +lean_dec(x_108); +lean_dec(x_103); +lean_ctor_set(x_110, 0, x_113); +return x_110; +} +} +} +} +else +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; size_t x_127; size_t x_128; uint8_t x_129; +x_124 = lean_ctor_get(x_110, 0); +x_125 = lean_ctor_get(x_110, 1); +lean_inc(x_125); +lean_inc(x_124); +lean_dec(x_110); +lean_inc(x_105); +lean_inc(x_104); +lean_inc(x_103); +x_126 = l_Lean_Expr_lam___override(x_103, x_104, x_105, x_106); +x_127 = lean_ptr_addr(x_104); +lean_dec(x_104); +x_128 = lean_ptr_addr(x_108); +x_129 = lean_usize_dec_eq(x_127, x_128); +if (x_129 == 0) +{ +lean_object* x_130; lean_object* x_131; +lean_dec(x_126); +lean_dec(x_105); +x_130 = l_Lean_Expr_lam___override(x_103, x_108, x_124, x_106); +x_131 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_125); +return x_131; +} +else +{ +size_t x_132; size_t x_133; uint8_t x_134; +x_132 = lean_ptr_addr(x_105); +lean_dec(x_105); +x_133 = lean_ptr_addr(x_124); +x_134 = lean_usize_dec_eq(x_132, x_133); +if (x_134 == 0) +{ +lean_object* x_135; lean_object* x_136; +lean_dec(x_126); +x_135 = l_Lean_Expr_lam___override(x_103, x_108, x_124, x_106); +x_136 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_136, 0, x_135); +lean_ctor_set(x_136, 1, x_125); +return x_136; +} +else +{ +uint8_t x_137; +x_137 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_106, x_106); +if (x_137 == 0) +{ +lean_object* x_138; lean_object* x_139; +lean_dec(x_126); +x_138 = l_Lean_Expr_lam___override(x_103, x_108, x_124, x_106); +x_139 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_125); +return x_139; +} +else +{ +lean_object* x_140; +lean_dec(x_124); +lean_dec(x_108); +lean_dec(x_103); +x_140 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_140, 0, x_126); +lean_ctor_set(x_140, 1, x_125); +return x_140; +} +} +} +} +} +case 7: +{ +lean_object* x_141; lean_object* x_142; lean_object* x_143; uint8_t x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; uint8_t x_149; +x_141 = lean_ctor_get(x_1, 0); +lean_inc(x_141); +x_142 = lean_ctor_get(x_1, 1); +lean_inc(x_142); +x_143 = lean_ctor_get(x_1, 2); +lean_inc(x_143); +x_144 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_142); +x_145 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_142, x_2); +x_146 = lean_ctor_get(x_145, 0); +lean_inc(x_146); +x_147 = lean_ctor_get(x_145, 1); +lean_inc(x_147); +lean_dec(x_145); +lean_inc(x_143); +x_148 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_143, x_147); +x_149 = !lean_is_exclusive(x_148); +if (x_149 == 0) +{ +lean_object* x_150; lean_object* x_151; size_t x_152; size_t x_153; uint8_t x_154; +x_150 = lean_ctor_get(x_148, 0); +lean_inc(x_143); +lean_inc(x_142); +lean_inc(x_141); +x_151 = l_Lean_Expr_forallE___override(x_141, x_142, x_143, x_144); +x_152 = lean_ptr_addr(x_142); +lean_dec(x_142); +x_153 = lean_ptr_addr(x_146); +x_154 = lean_usize_dec_eq(x_152, x_153); +if (x_154 == 0) +{ +lean_object* x_155; +lean_dec(x_151); +lean_dec(x_143); +x_155 = l_Lean_Expr_forallE___override(x_141, x_146, x_150, x_144); +lean_ctor_set(x_148, 0, x_155); +return x_148; +} +else +{ +size_t x_156; size_t x_157; uint8_t x_158; +x_156 = lean_ptr_addr(x_143); +lean_dec(x_143); +x_157 = lean_ptr_addr(x_150); +x_158 = lean_usize_dec_eq(x_156, x_157); +if (x_158 == 0) +{ +lean_object* x_159; +lean_dec(x_151); +x_159 = l_Lean_Expr_forallE___override(x_141, x_146, x_150, x_144); +lean_ctor_set(x_148, 0, x_159); +return x_148; +} +else +{ +uint8_t x_160; +x_160 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_144, x_144); +if (x_160 == 0) +{ +lean_object* x_161; +lean_dec(x_151); +x_161 = l_Lean_Expr_forallE___override(x_141, x_146, x_150, x_144); +lean_ctor_set(x_148, 0, x_161); +return x_148; +} +else +{ +lean_dec(x_150); +lean_dec(x_146); +lean_dec(x_141); +lean_ctor_set(x_148, 0, x_151); +return x_148; +} +} +} +} +else +{ +lean_object* x_162; lean_object* x_163; lean_object* x_164; size_t x_165; size_t x_166; uint8_t x_167; +x_162 = lean_ctor_get(x_148, 0); +x_163 = lean_ctor_get(x_148, 1); +lean_inc(x_163); +lean_inc(x_162); +lean_dec(x_148); +lean_inc(x_143); +lean_inc(x_142); +lean_inc(x_141); +x_164 = l_Lean_Expr_forallE___override(x_141, x_142, x_143, x_144); +x_165 = lean_ptr_addr(x_142); +lean_dec(x_142); +x_166 = lean_ptr_addr(x_146); +x_167 = lean_usize_dec_eq(x_165, x_166); +if (x_167 == 0) +{ +lean_object* x_168; lean_object* x_169; +lean_dec(x_164); +lean_dec(x_143); +x_168 = l_Lean_Expr_forallE___override(x_141, x_146, x_162, x_144); +x_169 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_169, 0, x_168); +lean_ctor_set(x_169, 1, x_163); +return x_169; +} +else +{ +size_t x_170; size_t x_171; uint8_t x_172; +x_170 = lean_ptr_addr(x_143); +lean_dec(x_143); +x_171 = lean_ptr_addr(x_162); +x_172 = lean_usize_dec_eq(x_170, x_171); +if (x_172 == 0) +{ +lean_object* x_173; lean_object* x_174; +lean_dec(x_164); +x_173 = l_Lean_Expr_forallE___override(x_141, x_146, x_162, x_144); +x_174 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_174, 0, x_173); +lean_ctor_set(x_174, 1, x_163); +return x_174; +} +else +{ +uint8_t x_175; +x_175 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_144, x_144); +if (x_175 == 0) +{ +lean_object* x_176; lean_object* x_177; +lean_dec(x_164); +x_176 = l_Lean_Expr_forallE___override(x_141, x_146, x_162, x_144); +x_177 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_177, 0, x_176); +lean_ctor_set(x_177, 1, x_163); +return x_177; +} +else +{ +lean_object* x_178; +lean_dec(x_162); +lean_dec(x_146); +lean_dec(x_141); +x_178 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_178, 0, x_164); +lean_ctor_set(x_178, 1, x_163); +return x_178; +} +} +} +} +} +case 8: +{ +lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; uint8_t x_191; +x_179 = lean_ctor_get(x_1, 0); +lean_inc(x_179); +x_180 = lean_ctor_get(x_1, 1); +lean_inc(x_180); +x_181 = lean_ctor_get(x_1, 2); +lean_inc(x_181); +x_182 = lean_ctor_get(x_1, 3); +lean_inc(x_182); +x_183 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); +lean_inc(x_180); +x_184 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_180, x_2); +x_185 = lean_ctor_get(x_184, 0); +lean_inc(x_185); +x_186 = lean_ctor_get(x_184, 1); +lean_inc(x_186); +lean_dec(x_184); +lean_inc(x_181); +x_187 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_181, x_186); +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +lean_inc(x_182); +x_190 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_182, x_189); +x_191 = !lean_is_exclusive(x_190); +if (x_191 == 0) +{ +lean_object* x_192; size_t x_193; size_t x_194; uint8_t x_195; +x_192 = lean_ctor_get(x_190, 0); +x_193 = lean_ptr_addr(x_180); +lean_dec(x_180); +x_194 = lean_ptr_addr(x_185); +x_195 = lean_usize_dec_eq(x_193, x_194); +if (x_195 == 0) { -lean_object* x_48; lean_object* x_49; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_expr_update_sort(x_1, x_48); -lean_ctor_set(x_46, 0, x_49); -return x_46; +lean_object* x_196; +lean_dec(x_182); +lean_dec(x_181); +lean_dec(x_1); +x_196 = l_Lean_Expr_letE___override(x_179, x_185, x_188, x_192, x_183); +lean_ctor_set(x_190, 0, x_196); +return x_190; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_50 = lean_ctor_get(x_46, 0); -x_51 = lean_ctor_get(x_46, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_46); -x_52 = lean_expr_update_sort(x_1, x_50); -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_51); -return x_53; -} +size_t x_197; size_t x_198; uint8_t x_199; +x_197 = lean_ptr_addr(x_181); +lean_dec(x_181); +x_198 = lean_ptr_addr(x_188); +x_199 = lean_usize_dec_eq(x_197, x_198); +if (x_199 == 0) +{ +lean_object* x_200; +lean_dec(x_182); +lean_dec(x_1); +x_200 = l_Lean_Expr_letE___override(x_179, x_185, x_188, x_192, x_183); +lean_ctor_set(x_190, 0, x_200); +return x_190; } -case 4: +else { -lean_object* x_54; lean_object* x_55; uint8_t x_56; -x_54 = lean_ctor_get(x_1, 1); -lean_inc(x_54); -x_55 = l_List_mapM___at_Lean_Meta_SynthInstance_MkTableKey_normExpr___spec__2(x_54, x_2); -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) +size_t x_201; size_t x_202; uint8_t x_203; +x_201 = lean_ptr_addr(x_182); +lean_dec(x_182); +x_202 = lean_ptr_addr(x_192); +x_203 = lean_usize_dec_eq(x_201, x_202); +if (x_203 == 0) { -lean_object* x_57; lean_object* x_58; -x_57 = lean_ctor_get(x_55, 0); -x_58 = lean_expr_update_const(x_1, x_57); -lean_ctor_set(x_55, 0, x_58); -return x_55; +lean_object* x_204; +lean_dec(x_1); +x_204 = l_Lean_Expr_letE___override(x_179, x_185, x_188, x_192, x_183); +lean_ctor_set(x_190, 0, x_204); +return x_190; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_59 = lean_ctor_get(x_55, 0); -x_60 = lean_ctor_get(x_55, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_55); -x_61 = lean_expr_update_const(x_1, x_59); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_60); -return x_62; +lean_dec(x_192); +lean_dec(x_188); +lean_dec(x_185); +lean_dec(x_179); +lean_ctor_set(x_190, 0, x_1); +return x_190; } } -case 5: +} +} +else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; -x_63 = lean_ctor_get(x_1, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_1, 1); -lean_inc(x_64); -x_65 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_63, x_2); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -lean_dec(x_65); -x_68 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_64, x_67); -x_69 = !lean_is_exclusive(x_68); -if (x_69 == 0) +lean_object* x_205; lean_object* x_206; size_t x_207; size_t x_208; uint8_t x_209; +x_205 = lean_ctor_get(x_190, 0); +x_206 = lean_ctor_get(x_190, 1); +lean_inc(x_206); +lean_inc(x_205); +lean_dec(x_190); +x_207 = lean_ptr_addr(x_180); +lean_dec(x_180); +x_208 = lean_ptr_addr(x_185); +x_209 = lean_usize_dec_eq(x_207, x_208); +if (x_209 == 0) { -lean_object* x_70; lean_object* x_71; -x_70 = lean_ctor_get(x_68, 0); -x_71 = lean_expr_update_app(x_1, x_66, x_70); -lean_ctor_set(x_68, 0, x_71); -return x_68; +lean_object* x_210; lean_object* x_211; +lean_dec(x_182); +lean_dec(x_181); +lean_dec(x_1); +x_210 = l_Lean_Expr_letE___override(x_179, x_185, x_188, x_205, x_183); +x_211 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_211, 0, x_210); +lean_ctor_set(x_211, 1, x_206); +return x_211; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_72 = lean_ctor_get(x_68, 0); -x_73 = lean_ctor_get(x_68, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_68); -x_74 = lean_expr_update_app(x_1, x_66, x_72); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_74); -lean_ctor_set(x_75, 1, x_73); -return x_75; -} +size_t x_212; size_t x_213; uint8_t x_214; +x_212 = lean_ptr_addr(x_181); +lean_dec(x_181); +x_213 = lean_ptr_addr(x_188); +x_214 = lean_usize_dec_eq(x_212, x_213); +if (x_214 == 0) +{ +lean_object* x_215; lean_object* x_216; +lean_dec(x_182); +lean_dec(x_1); +x_215 = l_Lean_Expr_letE___override(x_179, x_185, x_188, x_205, x_183); +x_216 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_216, 0, x_215); +lean_ctor_set(x_216, 1, x_206); +return x_216; } -case 6: +else { -lean_object* x_76; lean_object* x_77; uint8_t x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; -x_76 = lean_ctor_get(x_1, 1); -lean_inc(x_76); -x_77 = lean_ctor_get(x_1, 2); -lean_inc(x_77); -x_78 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_79 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_76, x_2); -x_80 = lean_ctor_get(x_79, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_79, 1); -lean_inc(x_81); -lean_dec(x_79); -x_82 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_77, x_81); -x_83 = !lean_is_exclusive(x_82); -if (x_83 == 0) -{ -lean_object* x_84; lean_object* x_85; -x_84 = lean_ctor_get(x_82, 0); -x_85 = lean_expr_update_lambda(x_1, x_78, x_80, x_84); -lean_ctor_set(x_82, 0, x_85); -return x_82; +size_t x_217; size_t x_218; uint8_t x_219; +x_217 = lean_ptr_addr(x_182); +lean_dec(x_182); +x_218 = lean_ptr_addr(x_205); +x_219 = lean_usize_dec_eq(x_217, x_218); +if (x_219 == 0) +{ +lean_object* x_220; lean_object* x_221; +lean_dec(x_1); +x_220 = l_Lean_Expr_letE___override(x_179, x_185, x_188, x_205, x_183); +x_221 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_221, 0, x_220); +lean_ctor_set(x_221, 1, x_206); +return x_221; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_86 = lean_ctor_get(x_82, 0); -x_87 = lean_ctor_get(x_82, 1); -lean_inc(x_87); -lean_inc(x_86); -lean_dec(x_82); -x_88 = lean_expr_update_lambda(x_1, x_78, x_80, x_86); -x_89 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_87); -return x_89; +lean_object* x_222; +lean_dec(x_205); +lean_dec(x_188); +lean_dec(x_185); +lean_dec(x_179); +x_222 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_222, 0, x_1); +lean_ctor_set(x_222, 1, x_206); +return x_222; } } -case 7: +} +} +} +case 10: { -lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; -x_90 = lean_ctor_get(x_1, 1); -lean_inc(x_90); -x_91 = lean_ctor_get(x_1, 2); -lean_inc(x_91); -x_92 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_93 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_90, x_2); -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_93, 1); -lean_inc(x_95); -lean_dec(x_93); -x_96 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_91, x_95); -x_97 = !lean_is_exclusive(x_96); -if (x_97 == 0) +lean_object* x_223; lean_object* x_224; lean_object* x_225; uint8_t x_226; +x_223 = lean_ctor_get(x_1, 0); +lean_inc(x_223); +x_224 = lean_ctor_get(x_1, 1); +lean_inc(x_224); +lean_inc(x_224); +x_225 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_224, x_2); +x_226 = !lean_is_exclusive(x_225); +if (x_226 == 0) +{ +lean_object* x_227; size_t x_228; size_t x_229; uint8_t x_230; +x_227 = lean_ctor_get(x_225, 0); +x_228 = lean_ptr_addr(x_224); +lean_dec(x_224); +x_229 = lean_ptr_addr(x_227); +x_230 = lean_usize_dec_eq(x_228, x_229); +if (x_230 == 0) { -lean_object* x_98; lean_object* x_99; -x_98 = lean_ctor_get(x_96, 0); -x_99 = lean_expr_update_forall(x_1, x_92, x_94, x_98); -lean_ctor_set(x_96, 0, x_99); -return x_96; +lean_object* x_231; +lean_dec(x_1); +x_231 = l_Lean_Expr_mdata___override(x_223, x_227); +lean_ctor_set(x_225, 0, x_231); +return x_225; } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_100 = lean_ctor_get(x_96, 0); -x_101 = lean_ctor_get(x_96, 1); -lean_inc(x_101); -lean_inc(x_100); -lean_dec(x_96); -x_102 = lean_expr_update_forall(x_1, x_92, x_94, x_100); -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_102); -lean_ctor_set(x_103, 1, x_101); -return x_103; +lean_dec(x_227); +lean_dec(x_223); +lean_ctor_set(x_225, 0, x_1); +return x_225; } } -case 8: +else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; -x_104 = lean_ctor_get(x_1, 1); -lean_inc(x_104); -x_105 = lean_ctor_get(x_1, 2); -lean_inc(x_105); -x_106 = lean_ctor_get(x_1, 3); -lean_inc(x_106); -x_107 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_104, x_2); -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_105, x_109); -x_111 = lean_ctor_get(x_110, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_110, 1); -lean_inc(x_112); -lean_dec(x_110); -x_113 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_106, x_112); -x_114 = !lean_is_exclusive(x_113); -if (x_114 == 0) +lean_object* x_232; lean_object* x_233; size_t x_234; size_t x_235; uint8_t x_236; +x_232 = lean_ctor_get(x_225, 0); +x_233 = lean_ctor_get(x_225, 1); +lean_inc(x_233); +lean_inc(x_232); +lean_dec(x_225); +x_234 = lean_ptr_addr(x_224); +lean_dec(x_224); +x_235 = lean_ptr_addr(x_232); +x_236 = lean_usize_dec_eq(x_234, x_235); +if (x_236 == 0) { -lean_object* x_115; lean_object* x_116; -x_115 = lean_ctor_get(x_113, 0); -x_116 = lean_expr_update_let(x_1, x_108, x_111, x_115); -lean_ctor_set(x_113, 0, x_116); -return x_113; +lean_object* x_237; lean_object* x_238; +lean_dec(x_1); +x_237 = l_Lean_Expr_mdata___override(x_223, x_232); +x_238 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_238, 0, x_237); +lean_ctor_set(x_238, 1, x_233); +return x_238; } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_117 = lean_ctor_get(x_113, 0); -x_118 = lean_ctor_get(x_113, 1); -lean_inc(x_118); -lean_inc(x_117); -lean_dec(x_113); -x_119 = lean_expr_update_let(x_1, x_108, x_111, x_117); -x_120 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_120, 0, x_119); -lean_ctor_set(x_120, 1, x_118); -return x_120; +lean_object* x_239; +lean_dec(x_232); +lean_dec(x_223); +x_239 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_239, 0, x_1); +lean_ctor_set(x_239, 1, x_233); +return x_239; } } -case 10: +} +case 11: { -lean_object* x_121; lean_object* x_122; uint8_t x_123; -x_121 = lean_ctor_get(x_1, 1); -lean_inc(x_121); -x_122 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_121, x_2); -x_123 = !lean_is_exclusive(x_122); -if (x_123 == 0) +lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; uint8_t x_244; +x_240 = lean_ctor_get(x_1, 0); +lean_inc(x_240); +x_241 = lean_ctor_get(x_1, 1); +lean_inc(x_241); +x_242 = lean_ctor_get(x_1, 2); +lean_inc(x_242); +lean_inc(x_242); +x_243 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_242, x_2); +x_244 = !lean_is_exclusive(x_243); +if (x_244 == 0) +{ +lean_object* x_245; size_t x_246; size_t x_247; uint8_t x_248; +x_245 = lean_ctor_get(x_243, 0); +x_246 = lean_ptr_addr(x_242); +lean_dec(x_242); +x_247 = lean_ptr_addr(x_245); +x_248 = lean_usize_dec_eq(x_246, x_247); +if (x_248 == 0) { -lean_object* x_124; lean_object* x_125; -x_124 = lean_ctor_get(x_122, 0); -x_125 = lean_expr_update_mdata(x_1, x_124); -lean_ctor_set(x_122, 0, x_125); -return x_122; +lean_object* x_249; +lean_dec(x_1); +x_249 = l_Lean_Expr_proj___override(x_240, x_241, x_245); +lean_ctor_set(x_243, 0, x_249); +return x_243; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_126 = lean_ctor_get(x_122, 0); -x_127 = lean_ctor_get(x_122, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_122); -x_128 = lean_expr_update_mdata(x_1, x_126); -x_129 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_129, 0, x_128); -lean_ctor_set(x_129, 1, x_127); -return x_129; +lean_dec(x_245); +lean_dec(x_241); +lean_dec(x_240); +lean_ctor_set(x_243, 0, x_1); +return x_243; } } -case 11: +else { -lean_object* x_130; lean_object* x_131; uint8_t x_132; -x_130 = lean_ctor_get(x_1, 2); -lean_inc(x_130); -x_131 = l_Lean_Meta_SynthInstance_MkTableKey_normExpr(x_130, x_2); -x_132 = !lean_is_exclusive(x_131); -if (x_132 == 0) -{ -lean_object* x_133; lean_object* x_134; -x_133 = lean_ctor_get(x_131, 0); -x_134 = lean_expr_update_proj(x_1, x_133); -lean_ctor_set(x_131, 0, x_134); -return x_131; +lean_object* x_250; lean_object* x_251; size_t x_252; size_t x_253; uint8_t x_254; +x_250 = lean_ctor_get(x_243, 0); +x_251 = lean_ctor_get(x_243, 1); +lean_inc(x_251); +lean_inc(x_250); +lean_dec(x_243); +x_252 = lean_ptr_addr(x_242); +lean_dec(x_242); +x_253 = lean_ptr_addr(x_250); +x_254 = lean_usize_dec_eq(x_252, x_253); +if (x_254 == 0) +{ +lean_object* x_255; lean_object* x_256; +lean_dec(x_1); +x_255 = l_Lean_Expr_proj___override(x_240, x_241, x_250); +x_256 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_256, 0, x_255); +lean_ctor_set(x_256, 1, x_251); +return x_256; } else { -lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; -x_135 = lean_ctor_get(x_131, 0); -x_136 = lean_ctor_get(x_131, 1); -lean_inc(x_136); -lean_inc(x_135); -lean_dec(x_131); -x_137 = lean_expr_update_proj(x_1, x_135); -x_138 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_138, 0, x_137); -lean_ctor_set(x_138, 1, x_136); -return x_138; +lean_object* x_257; +lean_dec(x_250); +lean_dec(x_241); +lean_dec(x_240); +x_257 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_257, 0, x_1); +lean_ctor_set(x_257, 1, x_251); +return x_257; +} } } default: { -lean_object* x_139; -x_139 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_139, 0, x_1); -lean_ctor_set(x_139, 1, x_2); -return x_139; +lean_object* x_258; +x_258 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_258, 0, x_1); +lean_ctor_set(x_258, 1, x_2); +return x_258; } } } @@ -3009,66 +3766,107 @@ 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_inc(x_31); lean_inc(x_1); x_33 = l_Std_PersistentHashMap_contains___at_Lean_NameSSet_contains___spec__3(x_1, x_31); if (x_33 == 0) { lean_object* x_34; uint8_t x_35; +lean_inc(x_32); x_34 = l_List_mapM___at_Lean_Meta_SynthInstance_getInstances___spec__3(x_32, x_6, x_7, x_8, x_9, x_10); x_35 = !lean_is_exclusive(x_34); if (x_35 == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; +lean_object* x_36; uint8_t x_37; x_36 = lean_ctor_get(x_34, 0); -x_37 = lean_expr_update_const(x_30, x_36); -x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_34, 0, x_38); +x_37 = l_ptrEqList___rarg(x_32, x_36); +lean_dec(x_32); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; +lean_dec(x_30); +x_38 = l_Lean_Expr_const___override(x_31, x_36); +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_34, 0, x_39); x_13 = x_34; goto block_29; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_39 = lean_ctor_get(x_34, 0); -x_40 = lean_ctor_get(x_34, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_34); -x_41 = lean_expr_update_const(x_30, x_39); -x_42 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_42, 0, x_41); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_40); -x_13 = x_43; +lean_object* x_40; +lean_dec(x_36); +lean_dec(x_31); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_30); +lean_ctor_set(x_34, 0, x_40); +x_13 = x_34; goto block_29; } } else { -lean_object* x_44; lean_object* x_45; +lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_41 = lean_ctor_get(x_34, 0); +x_42 = lean_ctor_get(x_34, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_34); +x_43 = l_ptrEqList___rarg(x_32, x_41); lean_dec(x_32); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_dec(x_30); -x_44 = lean_box(0); -x_45 = lean_alloc_ctor(0, 2, 0); +x_44 = l_Lean_Expr_const___override(x_31, x_41); +x_45 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_10); -x_13 = x_45; +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_42); +x_13 = x_46; +goto block_29; +} +else +{ +lean_object* x_47; lean_object* x_48; +lean_dec(x_41); +lean_dec(x_31); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_30); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_42); +x_13 = x_48; goto block_29; } } +} else { -lean_object* x_46; lean_object* x_47; +lean_object* x_49; lean_object* x_50; +lean_dec(x_32); +lean_dec(x_31); +lean_dec(x_30); +x_49 = lean_box(0); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_10); +x_13 = x_50; +goto block_29; +} +} +else +{ +lean_object* x_51; lean_object* x_52; lean_dec(x_30); -x_46 = l_Array_foldlMUnsafe_fold___at_Lean_Meta_SynthInstance_getInstances___spec__5___closed__4; +x_51 = l_Array_foldlMUnsafe_fold___at_Lean_Meta_SynthInstance_getInstances___spec__5___closed__4; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_47 = l_panic___at___private_Lean_Meta_WHNF_0__Lean_Meta_cached_x3f___spec__4(x_46, x_6, x_7, x_8, x_9, x_10); -x_13 = x_47; +x_52 = l_panic___at___private_Lean_Meta_WHNF_0__Lean_Meta_cached_x3f___spec__4(x_51, x_6, x_7, x_8, x_9, x_10); +x_13 = x_52; goto block_29; } block_29: @@ -3140,16 +3938,16 @@ return x_28; } else { -lean_object* x_48; +lean_object* x_53; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_1); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_5); -lean_ctor_set(x_48, 1, x_10); -return x_48; +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_5); +lean_ctor_set(x_53, 1, x_10); +return x_53; } } } @@ -21136,7 +21934,7 @@ lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean lean_free_object(x_11); lean_dec(x_1); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_3, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_17); x_19 = l___private_Lean_Meta_SynthInstance_0__Lean_Meta_preprocessOutParam___lambda__1___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -21274,7 +22072,7 @@ else lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_dec(x_1); x_48 = lean_unsigned_to_nat(0u); -x_49 = l_Lean_Expr_getAppNumArgsAux(x_3, x_48); +x_49 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_48); x_50 = l___private_Lean_Meta_SynthInstance_0__Lean_Meta_preprocessOutParam___lambda__1___closed__1; lean_inc(x_49); x_51 = lean_mk_array(x_49, x_50); diff --git a/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c b/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c index e7ecc80cd4b1..1765c5d8b9ca 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c +++ b/stage0/stdlib/Lean/Meta/Tactic/AC/Main.c @@ -340,7 +340,7 @@ static lean_object* _init_l_Lean_Meta_AC_instContextInformationProdPreContextArr lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__1___closed__1; x_2 = l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_AC_instContextInformationProdPreContextArrayBool___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Apply.c b/stage0/stdlib/Lean/Meta/Tactic/Apply.c index a5767c3d2d33..623ba8425ed5 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Apply.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Apply.c @@ -690,7 +690,7 @@ static lean_object* _init_l_Nat_forM_loop___at_Lean_Meta_synthAppInstances___spe 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_Nat_forM_loop___at_Lean_Meta_synthAppInstances___spec__1___closed__1; x_2 = l_Nat_forM_loop___at_Lean_Meta_synthAppInstances___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_forM_loop___at_Lean_Meta_synthAppInstances___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Assert.c b/stage0/stdlib/Lean/Meta/Tactic/Assert.c index 3ad6b45f3c1a..f2c45366c163 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Assert.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Assert.c @@ -1271,7 +1271,7 @@ static lean_object* _init_l_Nat_foldAux___at_Lean_Meta_assertAfter___spec__7___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_Nat_foldAux___at_Lean_Meta_assertAfter___spec__7___closed__1; x_2 = l_Nat_foldAux___at_Lean_Meta_assertAfter___spec__7___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_foldAux___at_Lean_Meta_assertAfter___spec__7___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Cases.c b/stage0/stdlib/Lean/Meta/Tactic/Cases.c index 566197cc4188..b23bf0bb6886 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Cases.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Cases.c @@ -199,6 +199,7 @@ static lean_object* l_Lean_Meta_Cases_cases___lambda__2___closed__11; LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_Meta_casesRec___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_mkEqAndProof___closed__3; static lean_object* l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNewEqs_loop___rarg___closed__2; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_generalizeTargetsEq___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_byCases(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -281,7 +282,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Cases_cases(lean_object*, lean_object*, lea LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNewEqs_loop___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_substEqs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_Cases_hasIndepIndices___spec__31(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNewEqs_loop___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_observing_x3f___at_Lean_Meta_casesRec___spec__2___at_Lean_Meta_casesRec___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -610,7 +610,7 @@ x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); lean_dec(x_20); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_8, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_8, x_22); x_24 = l_Lean_Meta_getInductiveUniverseAndParams___closed__1; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -683,7 +683,7 @@ x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); lean_dec(x_38); x_40 = lean_unsigned_to_nat(0u); -x_41 = l_Lean_Expr_getAppNumArgsAux(x_8, x_40); +x_41 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_8, x_40); x_42 = l_Lean_Meta_getInductiveUniverseAndParams___closed__1; lean_inc(x_41); x_43 = lean_mk_array(x_41, x_42); @@ -1154,7 +1154,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNe lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNewEqs_loop___rarg___closed__1; x_2 = l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNewEqs_loop___rarg___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Meta_Tactic_Cases_0__Lean_Meta_withNewEqs_loop___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2796,7 +2796,7 @@ x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); lean_dec(x_19); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_20, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_20, x_22); x_24 = l_Lean_Meta_getInductiveUniverseAndParams___closed__1; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -3475,7 +3475,7 @@ x_24 = lean_ctor_get(x_22, 1); lean_inc(x_24); lean_dec(x_22); x_25 = lean_unsigned_to_nat(0u); -x_26 = l_Lean_Expr_getAppNumArgsAux(x_23, x_25); +x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_23, x_25); x_27 = l_Lean_Meta_getInductiveUniverseAndParams___closed__1; lean_inc(x_26); x_28 = lean_mk_array(x_26, x_27); @@ -3626,7 +3626,7 @@ x_57 = lean_ctor_get(x_55, 1); lean_inc(x_57); lean_dec(x_55); x_58 = lean_unsigned_to_nat(0u); -x_59 = l_Lean_Expr_getAppNumArgsAux(x_56, x_58); +x_59 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_56, x_58); x_60 = l_Lean_Meta_getInductiveUniverseAndParams___closed__1; lean_inc(x_59); x_61 = lean_mk_array(x_59, x_60); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Constructor.c b/stage0/stdlib/Lean/Meta/Tactic/Constructor.c index 3da56d292b04..ea138d038e09 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Constructor.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Constructor.c @@ -14,6 +14,7 @@ extern "C" { #endif static lean_object* l_Lean_Meta_existsIntro___lambda__2___closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_constructor___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_existsIntro___lambda__2___closed__3; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Meta_constructor___lambda__2___closed__1; @@ -24,12 +25,14 @@ lean_object* lean_environment_find(lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Meta_existsIntro___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_constructor___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; lean_object* l_Lean_Meta_checkApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_constructor___closed__2; lean_object* l_Lean_Meta_apply(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_constructor___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withMVarContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallMetaTelescopeReducingAux(lean_object*, uint8_t, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -38,6 +41,7 @@ static lean_object* l_Lean_Meta_constructor___closed__1; static lean_object* l_Lean_Meta_constructor___lambda__1___closed__1; static lean_object* l_Lean_Meta_existsIntro___lambda__2___closed__4; static lean_object* l_Lean_Meta_constructor___lambda__1___closed__2; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_constructor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_constructor___lambda__2___closed__4; static lean_object* l_Lean_Meta_constructor___lambda__1___closed__3; @@ -49,14 +53,13 @@ LEAN_EXPORT lean_object* l_Lean_Meta_constructor___lambda__1___boxed(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* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_existsIntro___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Meta_checkNotAssigned(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_existsIntro___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_constructor___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_constructor___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_existsIntro___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_existsIntro___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_existsIntro___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_constructor___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_constructor___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_ofSubarray___rarg(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); @@ -68,53 +71,52 @@ static lean_object* l_Lean_Meta_existsIntro___lambda__2___closed__6; static lean_object* l_Lean_Meta_constructor___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_existsIntro(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_constructor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_constructor___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_constructor(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_constructor___spec__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) { _start: { -if (lean_obj_tag(x_4) == 0) +if (lean_obj_tag(x_5) == 0) { -lean_object* x_11; +lean_object* x_12; +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_5); -lean_ctor_set(x_11, 1, x_10); -return x_11; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_6); +lean_ctor_set(x_12, 1, x_11); +return x_12; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; -lean_dec(x_5); -x_12 = lean_ctor_get(x_4, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_4, 1); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_6); +x_13 = lean_ctor_get(x_5, 0); lean_inc(x_13); -lean_dec(x_4); -lean_inc(x_2); -x_14 = l_Lean_Expr_const___override(x_12, x_2); -x_15 = 0; +x_14 = lean_ctor_get(x_5, 1); +lean_inc(x_14); +lean_dec(x_5); +lean_inc(x_3); +x_15 = l_Lean_Expr_const___override(x_13, x_3); +lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_1); -x_16 = l_Lean_Meta_apply(x_1, x_14, x_15, x_6, x_7, x_8, x_9, x_10); +x_16 = l_Lean_Meta_apply(x_1, x_15, x_2, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_16) == 0) { uint8_t x_17; -lean_dec(x_13); +lean_dec(x_14); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); x_17 = !lean_is_exclusive(x_16); if (x_17 == 0) @@ -156,14 +158,14 @@ lean_object* x_28; x_28 = lean_ctor_get(x_16, 1); lean_inc(x_28); lean_dec(x_16); -lean_inc(x_3); +lean_inc(x_4); { -lean_object* _tmp_3 = x_13; -lean_object* _tmp_4 = x_3; -lean_object* _tmp_9 = x_28; -x_4 = _tmp_3; +lean_object* _tmp_4 = x_14; +lean_object* _tmp_5 = x_4; +lean_object* _tmp_10 = x_28; x_5 = _tmp_4; -x_10 = _tmp_9; +x_6 = _tmp_5; +x_11 = _tmp_10; } goto _start; } @@ -247,220 +249,220 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_constructor___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Meta_constructor___lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_8; -lean_inc(x_5); -lean_inc(x_3); +lean_object* x_9; +lean_inc(x_6); +lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_8 = l_Lean_Meta_checkNotAssigned(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_8) == 0) +x_9 = l_Lean_Meta_checkNotAssigned(x_1, x_2, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_3); lean_inc(x_1); -x_10 = l_Lean_Meta_getMVarType_x27(x_1, x_3, x_4, x_5, x_6, x_9); -if (lean_obj_tag(x_10) == 0) +x_11 = l_Lean_Meta_getMVarType_x27(x_1, x_4, x_5, x_6, x_7, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Expr_getAppFn(x_11); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); lean_dec(x_11); -if (lean_obj_tag(x_13) == 4) +x_14 = l_Lean_Expr_getAppFn(x_12); +lean_dec(x_12); +if (lean_obj_tag(x_14) == 4) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_st_ref_get(x_6, x_12); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_st_ref_get(x_7, x_13); +x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 0); +x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -x_20 = lean_environment_find(x_19, x_14); -if (lean_obj_tag(x_20) == 0) +x_20 = lean_ctor_get(x_18, 0); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_environment_find(x_20, x_15); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_21; lean_object* x_22; -lean_dec(x_15); -x_21 = l_Lean_Meta_constructor___lambda__2___closed__3; -x_22 = l_Lean_Meta_throwTacticEx___rarg(x_2, x_1, x_21, x_3, x_4, x_5, x_6, x_18); -lean_dec(x_6); -lean_dec(x_4); -return x_22; +lean_object* x_22; lean_object* x_23; +lean_dec(x_16); +x_22 = l_Lean_Meta_constructor___lambda__2___closed__3; +x_23 = l_Lean_Meta_throwTacticEx___rarg(x_2, x_1, x_22, x_4, x_5, x_6, x_7, x_19); +lean_dec(x_7); +lean_dec(x_5); +return x_23; } else { -lean_object* x_23; -x_23 = lean_ctor_get(x_20, 0); -lean_inc(x_23); -lean_dec(x_20); -if (lean_obj_tag(x_23) == 5) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_24 = lean_ctor_get(x_23, 0); +lean_object* x_24; +x_24 = lean_ctor_get(x_21, 0); lean_inc(x_24); -lean_dec(x_23); -x_25 = lean_ctor_get(x_24, 4); +lean_dec(x_21); +if (lean_obj_tag(x_24) == 5) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); lean_dec(x_24); -x_26 = l_Lean_Meta_constructor___lambda__2___closed__4; +x_26 = lean_ctor_get(x_25, 4); +lean_inc(x_26); +lean_dec(x_25); +x_27 = l_Lean_Meta_constructor___lambda__2___closed__4; +lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_3); lean_inc(x_1); -x_27 = l_List_forIn_loop___at_Lean_Meta_constructor___spec__1(x_1, x_15, x_26, x_25, x_26, x_3, x_4, x_5, x_6, x_18); -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); +x_28 = l_List_forIn_loop___at_Lean_Meta_constructor___spec__1(x_1, x_3, x_16, x_27, x_26, x_27, x_4, x_5, x_6, x_7, x_19); x_29 = lean_ctor_get(x_28, 0); lean_inc(x_29); -lean_dec(x_28); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_27, 1); +x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); -lean_dec(x_27); -x_31 = lean_box(0); -x_32 = l_Lean_Meta_constructor___lambda__1(x_2, x_1, x_31, x_3, x_4, x_5, x_6, x_30); -lean_dec(x_6); -lean_dec(x_4); -return x_32; +lean_dec(x_29); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_28, 1); +lean_inc(x_31); +lean_dec(x_28); +x_32 = lean_box(0); +x_33 = l_Lean_Meta_constructor___lambda__1(x_2, x_1, x_32, x_4, x_5, x_6, x_7, x_31); +lean_dec(x_7); +lean_dec(x_5); +return x_33; } else { -uint8_t x_33; +uint8_t x_34; +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_33 = !lean_is_exclusive(x_27); -if (x_33 == 0) +x_34 = !lean_is_exclusive(x_28); +if (x_34 == 0) { -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_27, 0); -lean_dec(x_34); -x_35 = lean_ctor_get(x_29, 0); -lean_inc(x_35); -lean_dec(x_29); -lean_ctor_set(x_27, 0, x_35); -return x_27; +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_28, 0); +lean_dec(x_35); +x_36 = lean_ctor_get(x_30, 0); +lean_inc(x_36); +lean_dec(x_30); +lean_ctor_set(x_28, 0, x_36); +return x_28; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_27, 1); -lean_inc(x_36); -lean_dec(x_27); -x_37 = lean_ctor_get(x_29, 0); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_28, 1); lean_inc(x_37); -lean_dec(x_29); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_36); -return x_38; +lean_dec(x_28); +x_38 = lean_ctor_get(x_30, 0); +lean_inc(x_38); +lean_dec(x_30); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +return x_39; } } } else { -lean_object* x_39; lean_object* x_40; -lean_dec(x_23); -lean_dec(x_15); -x_39 = l_Lean_Meta_constructor___lambda__2___closed__3; -x_40 = l_Lean_Meta_throwTacticEx___rarg(x_2, x_1, x_39, x_3, x_4, x_5, x_6, x_18); -lean_dec(x_6); -lean_dec(x_4); -return x_40; +lean_object* x_40; lean_object* x_41; +lean_dec(x_24); +lean_dec(x_16); +x_40 = l_Lean_Meta_constructor___lambda__2___closed__3; +x_41 = l_Lean_Meta_throwTacticEx___rarg(x_2, x_1, x_40, x_4, x_5, x_6, x_7, x_19); +lean_dec(x_7); +lean_dec(x_5); +return x_41; } } } else { -lean_object* x_41; lean_object* x_42; -lean_dec(x_13); -x_41 = l_Lean_Meta_constructor___lambda__2___closed__3; -x_42 = l_Lean_Meta_throwTacticEx___rarg(x_2, x_1, x_41, x_3, x_4, x_5, x_6, x_12); -lean_dec(x_6); -lean_dec(x_4); -return x_42; +lean_object* x_42; lean_object* x_43; +lean_dec(x_14); +x_42 = l_Lean_Meta_constructor___lambda__2___closed__3; +x_43 = l_Lean_Meta_throwTacticEx___rarg(x_2, x_1, x_42, x_4, x_5, x_6, x_7, x_13); +lean_dec(x_7); +lean_dec(x_5); +return x_43; } } else { -uint8_t x_43; +uint8_t x_44; +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_43 = !lean_is_exclusive(x_10); -if (x_43 == 0) +x_44 = !lean_is_exclusive(x_11); +if (x_44 == 0) { -return x_10; +return x_11; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_10, 0); -x_45 = lean_ctor_get(x_10, 1); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_11, 0); +x_46 = lean_ctor_get(x_11, 1); +lean_inc(x_46); lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_10); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -return x_46; +lean_dec(x_11); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } else { -uint8_t x_47; +uint8_t x_48; +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_8); -if (x_47 == 0) +x_48 = !lean_is_exclusive(x_9); +if (x_48 == 0) { -return x_8; +return x_9; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_8, 0); -x_49 = lean_ctor_get(x_8, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_9, 0); +x_50 = lean_ctor_get(x_9, 1); +lean_inc(x_50); lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_8); -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_9); +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; } } } @@ -483,17 +485,29 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_constructor(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Meta_constructor(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = l_Lean_Meta_constructor___closed__2; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = l_Lean_Meta_constructor___closed__2; +x_9 = lean_box(x_2); lean_inc(x_1); -x_8 = lean_alloc_closure((void*)(l_Lean_Meta_constructor___lambda__2), 7, 2); -lean_closure_set(x_8, 0, x_1); -lean_closure_set(x_8, 1, x_7); -x_9 = l_Lean_Meta_withMVarContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_8, x_2, x_3, x_4, x_5, x_6); -return x_9; +x_10 = lean_alloc_closure((void*)(l_Lean_Meta_constructor___lambda__2___boxed), 8, 3); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_8); +lean_closure_set(x_10, 2, x_9); +x_11 = l_Lean_Meta_withMVarContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_10, x_3, x_4, x_5, x_6, x_7); +return x_11; +} +} +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Meta_constructor___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; lean_object* x_13; +x_12 = lean_unbox(x_2); +lean_dec(x_2); +x_13 = l_List_forIn_loop___at_Lean_Meta_constructor___spec__1(x_1, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_13; } } LEAN_EXPORT lean_object* l_Lean_Meta_constructor___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) { @@ -507,6 +521,26 @@ lean_dec(x_3); return x_9; } } +LEAN_EXPORT lean_object* l_Lean_Meta_constructor___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_3); +lean_dec(x_3); +x_10 = l_Lean_Meta_constructor___lambda__2(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_constructor___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_2); +lean_dec(x_2); +x_9 = l_Lean_Meta_constructor(x_1, x_8, x_3, x_4, x_5, x_6, x_7); +return x_9; +} +} static lean_object* _init_l_Lean_Meta_existsIntro___lambda__1___closed__1() { _start: { @@ -555,7 +589,7 @@ lean_inc(x_14); lean_dec(x_13); x_15 = l_Lean_Expr_const___override(x_14, x_2); x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_3, x_16); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_16); x_18 = l_Lean_Meta_existsIntro___lambda__1___closed__1; lean_inc(x_17); x_19 = lean_mk_array(x_17, x_18); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Contradiction.c b/stage0/stdlib/Lean/Meta/Tactic/Contradiction.c index e3a925efea93..7fb7aa136412 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Contradiction.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Contradiction.c @@ -121,6 +121,7 @@ static lean_object* l_Lean_Meta_ElimEmptyInductive_elim___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_ElimEmptyInductive_elim___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_commitWhen___at_Lean_Meta_ElimEmptyInductive_elim___spec__7___at_Lean_Meta_ElimEmptyInductive_elim___spec__8___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Contradiction_0__Lean_Meta_nestedFalseElim(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Contradiction_Config_searchFuel___default; LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at_Lean_Meta_ElimEmptyInductive_elim___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); @@ -178,7 +179,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Contradiction_0__Lean_Meta LEAN_EXPORT lean_object* l_Lean_commitWhen___at_Lean_Meta_ElimEmptyInductive_elim___spec__7___at_Lean_Meta_ElimEmptyInductive_elim___spec__8___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Cases_cases(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_contradictionCore___spec__4___lambda__3___closed__7; lean_object* l_Lean_Meta_matchConstructorApp_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_checkNotAssigned(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -6415,7 +6415,7 @@ x_44 = lean_ctor_get(x_42, 1); lean_inc(x_44); lean_dec(x_42); x_45 = lean_unsigned_to_nat(0u); -x_46 = l_Lean_Expr_getAppNumArgsAux(x_25, x_45); +x_46 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_25, x_45); x_47 = l_Array_forInUnsafe_loop___at_Lean_Meta_contradictionCore___spec__4___lambda__3___closed__8; lean_inc(x_46); x_48 = lean_mk_array(x_46, x_47); @@ -6612,7 +6612,7 @@ x_106 = lean_ctor_get(x_104, 1); lean_inc(x_106); lean_dec(x_104); x_107 = lean_unsigned_to_nat(0u); -x_108 = l_Lean_Expr_getAppNumArgsAux(x_25, x_107); +x_108 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_25, x_107); x_109 = l_Array_forInUnsafe_loop___at_Lean_Meta_contradictionCore___spec__4___lambda__3___closed__8; lean_inc(x_108); x_110 = lean_mk_array(x_108, x_109); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Delta.c b/stage0/stdlib/Lean/Meta/Tactic/Delta.c index cbe9eb57812b..a2c10a167be9 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Delta.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Delta.c @@ -26,13 +26,13 @@ lean_object* l_Lean_Meta_withMVarContext___at___private_Lean_Meta_SynthInstance_ lean_object* l_Lean_Meta_getMVarType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_deltaLocalDecl___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_name(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); uint8_t l_Lean_ConstantInfo_hasValue(lean_object*); lean_object* l_Lean_Core_instantiateValueLevelParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_delta_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_changeLocalDecl(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Meta_checkNotAssigned(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_deltaTarget___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_betaRev(lean_object*, lean_object*, uint8_t, uint8_t); @@ -158,7 +158,7 @@ if (x_31 == 0) { lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; uint8_t x_37; lean_object* x_38; x_32 = lean_ctor_get(x_30, 0); -x_33 = l_Lean_Expr_getAppNumArgsAux(x_1, x_25); +x_33 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_25); x_34 = lean_mk_empty_array_with_capacity(x_33); lean_dec(x_33); x_35 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_34); @@ -178,7 +178,7 @@ x_40 = lean_ctor_get(x_30, 1); lean_inc(x_40); lean_inc(x_39); lean_dec(x_30); -x_41 = l_Lean_Expr_getAppNumArgsAux(x_1, x_25); +x_41 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_25); x_42 = lean_mk_empty_array_with_capacity(x_41); lean_dec(x_41); x_43 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_42); @@ -275,7 +275,7 @@ if (lean_is_exclusive(x_61)) { lean_dec_ref(x_61); x_64 = lean_box(0); } -x_65 = l_Lean_Expr_getAppNumArgsAux(x_1, x_56); +x_65 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_56); x_66 = lean_mk_empty_array_with_capacity(x_65); lean_dec(x_65); x_67 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_66); @@ -418,7 +418,7 @@ if (lean_is_exclusive(x_96)) { lean_dec_ref(x_96); x_99 = lean_box(0); } -x_100 = l_Lean_Expr_getAppNumArgsAux(x_1, x_90); +x_100 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_90); x_101 = lean_mk_empty_array_with_capacity(x_100); lean_dec(x_100); x_102 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_101); diff --git a/stage0/stdlib/Lean/Meta/Tactic/ElimInfo.c b/stage0/stdlib/Lean/Meta/Tactic/ElimInfo.c index dbae063635b5..c471a056b27f 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/ElimInfo.c +++ b/stage0/stdlib/Lean/Meta/Tactic/ElimInfo.c @@ -209,6 +209,7 @@ static lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_mkCustomEliminator___s LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_mkCustomEliminator___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_getElimInfo___lambda__2___closed__2; lean_object* l_Lean_markUsedAssignment___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_getCustomEliminator_x3f___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Meta_Tactic_ElimInfo_0__Lean_Meta_reprCustomEliminator____x40_Lean_Meta_Tactic_ElimInfo___hyg_1429____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_getElimInfo___spec__7___boxed(lean_object*, lean_object*, lean_object*); @@ -322,7 +323,6 @@ LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Meta_addImplicitTargets_collect__ static lean_object* l___private_Lean_Meta_Tactic_ElimInfo_0__Lean_Meta_reprCustomEliminator____x40_Lean_Meta_Tactic_ElimInfo___hyg_1429____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_ElimInfo_0__Lean_Meta_reprElimInfo____x40_Lean_Meta_Tactic_ElimInfo___hyg_122____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_Meta_getElimInfo___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Tactic_ElimInfo___hyg_2150____lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); extern uint8_t l_instInhabitedBool; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_Meta_addCustomEliminatorEntry___spec__4(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1564,7 +1564,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Meta_getElimInfo___sp lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Meta_getElimInfo___spec__6___closed__2; x_2 = l_Std_Range_forIn_loop___at_Lean_Meta_getElimInfo___spec__6___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Meta_getElimInfo___spec__6___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2228,7 +2228,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getElimInfo___lambda__4(lean_object* x_1, l lean_object* x_10; 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_30; uint8_t x_46; x_10 = l_Lean_Expr_getAppFn(x_4); x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_4, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_11); x_13 = l_Lean_Meta_getElimInfo___lambda__4___closed__1; lean_inc(x_12); x_14 = lean_mk_array(x_12, x_13); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Generalize.c b/stage0/stdlib/Lean/Meta/Tactic/Generalize.c index 0f25d16fce9f..6f32c17e5817 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Generalize.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Generalize.c @@ -537,7 +537,7 @@ static lean_object* _init_l_Lean_Meta_generalize_go_x27___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_generalize_go_x27___closed__1; x_2 = l_Lean_Meta_generalize_go_x27___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_generalize_go_x27___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Induction.c b/stage0/stdlib/Lean/Meta/Tactic/Induction.c index 3d280b8dfc71..567c5f83a4b2 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Induction.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Induction.c @@ -103,6 +103,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Induction_0__Lean_Meta_fin uint8_t l_Lean_Expr_isHeadBetaTarget(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_induction___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); static lean_object* l_Lean_Meta_instInhabitedInductionSubgoal___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Induction_0__Lean_Meta_finalize_loop___lambda__2___boxed(lean_object**); @@ -151,7 +152,6 @@ static lean_object* l_List_forM___at_Lean_Meta_induction___spec__1___closed__2; lean_object* l_List_redLength___rarg(lean_object*); static lean_object* l_Nat_forM_loop___at_Lean_Meta_induction___spec__3___lambda__1___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Meta_induction___spec__6___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forM___at_Lean_Meta_induction___spec__1___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_induction___spec__4___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*); @@ -829,7 +829,7 @@ static lean_object* _init_l_Nat_foldAux___at___private_Lean_Meta_Tactic_Inductio 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_Nat_foldAux___at___private_Lean_Meta_Tactic_Induction_0__Lean_Meta_finalize_loop___spec__2___closed__1; x_2 = l_Nat_foldAux___at___private_Lean_Meta_Tactic_Induction_0__Lean_Meta_finalize_loop___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_foldAux___at___private_Lean_Meta_Tactic_Induction_0__Lean_Meta_finalize_loop___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4560,7 +4560,7 @@ x_37 = lean_ctor_get(x_33, 0); lean_inc(x_37); lean_dec(x_33); x_38 = lean_unsigned_to_nat(0u); -x_39 = l_Lean_Expr_getAppNumArgsAux(x_37, x_38); +x_39 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_37, x_38); x_40 = l_Lean_Expr_withAppAux___at_Lean_Meta_induction___spec__8___lambda__1___closed__1; lean_inc(x_39); x_41 = lean_mk_array(x_39, x_40); @@ -7867,7 +7867,7 @@ x_29 = lean_ctor_get(x_25, 0); lean_inc(x_29); lean_dec(x_25); x_30 = lean_unsigned_to_nat(0u); -x_31 = l_Lean_Expr_getAppNumArgsAux(x_29, x_30); +x_31 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_29, x_30); x_32 = l_Lean_Expr_withAppAux___at_Lean_Meta_induction___spec__8___lambda__1___closed__1; lean_inc(x_31); x_33 = lean_mk_array(x_31, x_32); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Injection.c b/stage0/stdlib/Lean/Meta/Tactic/Injection.c index 84e6b3a1a8f9..0aca813685e2 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Injection.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Injection.c @@ -131,7 +131,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Meta_getCtorNumPropFi lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Meta_getCtorNumPropFields___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_Meta_getCtorNumPropFields___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Meta_getCtorNumPropFields___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Intro.c b/stage0/stdlib/Lean/Meta/Tactic/Intro.c index 19a51e4e3dec..c51414b4a94f 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Intro.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Intro.c @@ -72,6 +72,7 @@ lean_object* l_Lean_addTrace___rarg(lean_object*, lean_object*, lean_object*, le lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* l_Lean_monadNameGeneratorLift___rarg(lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___rarg(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); lean_object* l_Lean_Expr_headBeta(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp_loop___rarg___lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp_loop(lean_object*); @@ -131,7 +132,6 @@ static lean_object* l___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp_lo static lean_object* l___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp_loop___rarg___lambda__2___closed__17; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp_loop___rarg___lambda__2___closed__2; -lean_object* l_Lean_Expr_consumeMDataAndTypeAnnotations(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_getIntrosSize___boxed(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Intro_0__Lean_Meta_introNImp_loop___rarg___lambda__2___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_intro1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -412,7 +412,7 @@ lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); lean_inc(x_20); lean_dec(x_18); -x_21 = l_Lean_Expr_consumeMDataAndTypeAnnotations(x_19); +x_21 = l_Lean_Expr_cleanupAnnotations(x_19); x_22 = l_Lean_Expr_isForall(x_21); if (x_22 == 0) { @@ -1993,7 +1993,7 @@ static lean_object* _init_l_Lean_Meta_intro___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_intro___closed__1; x_2 = l_Lean_Meta_intro___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_intro___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Basic.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Basic.c index 26d0a205911e..8c3ea9ccb7f1 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Basic.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Basic.c @@ -34,6 +34,7 @@ static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__17; static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__9; static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__8; static lean_object* l_Lean_Meta_Linear_isLinearTerm___closed__12; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__15; static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__22; static lean_object* l_Lean_Meta_Linear_isLinearTerm___closed__1; @@ -46,7 +47,6 @@ static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__18; static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__6; static lean_object* l_Lean_Meta_Linear_isLinearTerm___closed__7; static lean_object* l_Lean_Meta_Linear_isLinearTerm___closed__16; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__10; static lean_object* l_Lean_Meta_Linear_isLinearCnstr___closed__20; static lean_object* l_Lean_Meta_Linear_isLinearTerm___closed__11; @@ -542,7 +542,7 @@ else { lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; x_21 = lean_unsigned_to_nat(0u); -x_22 = l_Lean_Expr_getAppNumArgsAux(x_1, x_21); +x_22 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_21); x_23 = lean_unsigned_to_nat(1u); x_24 = lean_nat_dec_eq(x_22, x_23); lean_dec(x_22); diff --git a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Basic.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Basic.c index 91163a85ac15..40c1e9ceefec 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Basic.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Basic.c @@ -111,6 +111,7 @@ lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Nat_Basic_0__Lean_Meta_Linear_Nat_reprExpr____x40_Lean_Meta_Tactic_LinearArith_Nat_Basic___hyg_4_(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Nat_Basic_0__Lean_Meta_Linear_Nat_reprExprCnstr____x40_Lean_Meta_Tactic_LinearArith_Nat_Basic___hyg_267____closed__29; static lean_object* l_Lean_Meta_Linear_Nat_reflTrue___closed__6; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Nat_Basic_0__Lean_Meta_Linear_Nat_reprExpr____x40_Lean_Meta_Tactic_LinearArith_Nat_Basic___hyg_4____closed__1; lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_ToLinear_toLinearExpr_visit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -163,7 +164,6 @@ static lean_object* l_Lean_Meta_Linear_Nat_ToLinear_toLinearCnstr_x3f___closed__ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Nat_Basic_0__Lean_Meta_Linear_Nat_reprExpr____x40_Lean_Meta_Tactic_LinearArith_Nat_Basic___hyg_4____closed__10; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_LinearArith_Nat_Basic_0__Lean_Meta_Linear_Nat_reprExprCnstr____x40_Lean_Meta_Tactic_LinearArith_Nat_Basic___hyg_267____boxed(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_LinearArith_Nat_Basic_0__Lean_Meta_Linear_Nat_reprExprCnstr____x40_Lean_Meta_Tactic_LinearArith_Nat_Basic___hyg_267____closed__1; static lean_object* l_Lean_Meta_Linear_Nat_reflTrue___closed__3; uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -2079,7 +2079,7 @@ static lean_object* _init_l_Lean_Meta_Linear_Nat_LinearExpr_toArith___closed__4( lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Linear_Nat_LinearExpr_toArith___closed__1; x_2 = l_Lean_Meta_Linear_Nat_LinearExpr_toArith___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_Linear_Nat_LinearExpr_toArith___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -3133,7 +3133,7 @@ x_15 = lean_ctor_get(x_8, 0); lean_inc(x_15); lean_dec(x_8); x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_1, x_16); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_16); x_103 = l_Lean_Meta_Linear_Nat_ToLinear_toLinearExpr_visit___closed__4; x_104 = lean_name_eq(x_15, x_103); if (x_104 == 0) @@ -4342,7 +4342,7 @@ x_22 = lean_ctor_get(x_8, 0); lean_inc(x_22); lean_dec(x_8); x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Lean_Expr_getAppNumArgsAux(x_1, x_23); +x_24 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_23); x_191 = l_Lean_Meta_Linear_Nat_ToLinear_toLinearCnstr_x3f___closed__17; x_192 = lean_name_eq(x_22, x_191); if (x_192 == 0) diff --git a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c index b8f1a5597b0e..83f3f64d7a57 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c @@ -62,6 +62,7 @@ static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__2; static lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__3; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__25; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__21; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__1; lean_object* l_Nat_Linear_PolyCnstr_toExpr(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__7; @@ -81,7 +82,6 @@ static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__4 static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___closed__11; uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16; @@ -1885,7 +1885,7 @@ x_14 = lean_ctor_get(x_4, 0); x_15 = lean_box(0); x_16 = l_Lean_Expr_const___override(x_5, x_15); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_2, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_17); x_19 = lean_unsigned_to_nat(2u); x_20 = lean_nat_sub(x_18, x_19); x_21 = lean_unsigned_to_nat(1u); @@ -2112,7 +2112,7 @@ lean_dec(x_4); x_80 = lean_box(0); x_81 = l_Lean_Expr_const___override(x_5, x_80); x_82 = lean_unsigned_to_nat(0u); -x_83 = l_Lean_Expr_getAppNumArgsAux(x_2, x_82); +x_83 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_82); x_84 = lean_unsigned_to_nat(2u); x_85 = lean_nat_sub(x_83, x_84); x_86 = lean_unsigned_to_nat(1u); @@ -2545,7 +2545,7 @@ else { lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; x_25 = lean_unsigned_to_nat(0u); -x_26 = l_Lean_Expr_getAppNumArgsAux(x_11, x_25); +x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_25); x_27 = lean_unsigned_to_nat(2u); x_28 = lean_nat_sub(x_26, x_27); x_29 = lean_nat_sub(x_28, x_8); @@ -2613,7 +2613,7 @@ else { lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; x_46 = lean_unsigned_to_nat(0u); -x_47 = l_Lean_Expr_getAppNumArgsAux(x_11, x_46); +x_47 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_46); x_48 = lean_unsigned_to_nat(3u); x_49 = lean_nat_sub(x_47, x_48); x_50 = lean_nat_sub(x_49, x_8); @@ -2681,7 +2681,7 @@ else { lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; x_67 = lean_unsigned_to_nat(0u); -x_68 = l_Lean_Expr_getAppNumArgsAux(x_11, x_67); +x_68 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_67); x_69 = lean_unsigned_to_nat(2u); x_70 = lean_nat_sub(x_68, x_69); x_71 = lean_nat_sub(x_70, x_8); @@ -2793,7 +2793,7 @@ else { lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; x_96 = lean_unsigned_to_nat(0u); -x_97 = l_Lean_Expr_getAppNumArgsAux(x_11, x_96); +x_97 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_96); x_98 = lean_unsigned_to_nat(3u); x_99 = lean_nat_sub(x_97, x_98); x_100 = lean_nat_sub(x_99, x_8); diff --git a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c index 0ac8116f2058..d359a7ed058e 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Solver.c @@ -4642,7 +4642,7 @@ static lean_object* _init_l_Lean_Meta_Linear_State_getBestLowerBound_x3f___close lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Linear_State_getBestLowerBound_x3f___closed__1; x_2 = l_Lean_Meta_Linear_State_getBestLowerBound_x3f___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_Linear_State_getBestLowerBound_x3f___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Simp/Main.c b/stage0/stdlib/Lean/Meta/Tactic/Simp/Main.c index 1fadf3998691..9d6a8e20a3c5 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Simp/Main.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Simp/Main.c @@ -26,7 +26,6 @@ static lean_object* l_Lean_Meta_Simp_isOfNatNatLit___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_unfold_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_dsimpMain(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); lean_object* l_Lean_Meta_replaceTargetDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkImpCongrCtx(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); @@ -75,6 +74,7 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v lean_object* l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(lean_object*); static lean_object* l_Lean_Meta_Simp_simp_trySimpCongrTheorem_x3f___lambda__9___closed__1; lean_object* l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__9___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_simpArrow___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_trySimpCongrTheorem_x3f___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -93,7 +93,6 @@ static lean_object* l_Lean_Meta_Simp_removeUnnecessaryCasts_isDummyEqRec___close LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_Meta_Simp_simp_simpProj___spec__4___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_simpLet___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Simp_simp_tryAutoCongrTheorem_x3f___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_dischargeEqnThmHypothesis_x3f_go_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Simp_throwCongrHypothesisFailed___rarg___closed__2; @@ -386,6 +385,7 @@ uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Simp_simp_trySimpCongrTheorem_x3f___lambda__4___closed__2; uint8_t l_Lean_Exception_isMaxRecDepth(lean_object*); static lean_object* l_Lean_Meta_Simp_simp_tryAutoCongrTheorem_x3f___lambda__5___closed__4; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Simp_SimpLetCase_noConfusion___rarg___closed__1; static lean_object* l_Lean_Meta_Simp_simp_simpArrow___lambda__4___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Simp_DefaultMethods_discharge_x3f___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -502,7 +502,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_trySimpCongrTheorem_x3f(lean_obje uint8_t l_Lean_Expr_isLambda(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_withNewLemmas___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_dsimpGoal___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_fvarId(lean_object*); static lean_object* l_Lean_Meta_Simp_initFn____x40_Lean_Meta_Tactic_Simp_Main___hyg_5____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_cacheResult(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -551,6 +550,7 @@ lean_object* l_Lean_Expr_fvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_exprDependsOn___at_Lean_Meta_Simp_simp_simpProj___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_dsimpGoal___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__10___boxed(lean_object**); +size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_Meta_mkForallCongr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_tryAutoCongrTheorem_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); @@ -559,7 +559,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_simp___lambda__2(lean_object*, lean_object* LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Meta_Simp_simp_cacheResult___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_trySynthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_dsimpGoal___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_anyMUnsafe_any___at_Lean_Meta_Simp_simp_trySimpCongrTheorem_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_applySimpResultToTarget(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -690,6 +689,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Simp_simp_congr static lean_object* l_Lean_Meta_Simp_simp_simpArrow___lambda__4___closed__9; lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Simp_simp_simpForall___closed__8; +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_dsimpGoal___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_findSomeRevMAux___at_Lean_Meta_Simp_dischargeUsingAssumption_x3f___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_simpLoop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -702,6 +702,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_applySimpResultToProp(lean_object*, lean_ob static lean_object* l_Lean_Meta_Simp_simp_simpArrow___lambda__4___closed__2; static lean_object* l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___lambda__7___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_Simp_simp_processCongrHypothesis___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_DefaultMethods_discharge_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_Simp_lambdaTelescopeDSimp_go___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkExpectedTypeHint(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2021,8 +2022,8 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Si lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__1; x_2 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__2; -x_3 = lean_unsigned_to_nat(1135u); -x_4 = lean_unsigned_to_nat(23u); +x_3 = lean_unsigned_to_nat(1471u); +x_4 = lean_unsigned_to_nat(24u); x_5 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -2040,21 +2041,79 @@ x_11 = lean_ctor_get(x_2, 1); lean_inc(x_11); if (lean_obj_tag(x_1) == 7) { -uint8_t x_131; lean_object* x_132; -x_131 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_132 = lean_expr_update_forall(x_1, x_131, x_9, x_10); -x_12 = x_132; +lean_object* x_131; lean_object* x_132; lean_object* x_133; uint8_t x_134; lean_object* x_135; size_t x_136; size_t x_137; uint8_t x_138; +x_131 = lean_ctor_get(x_1, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_1, 1); +lean_inc(x_132); +x_133 = lean_ctor_get(x_1, 2); +lean_inc(x_133); +x_134 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_133); +lean_inc(x_132); +lean_inc(x_131); +x_135 = l_Lean_Expr_forallE___override(x_131, x_132, x_133, x_134); +x_136 = lean_ptr_addr(x_132); +lean_dec(x_132); +x_137 = lean_ptr_addr(x_9); +x_138 = lean_usize_dec_eq(x_136, x_137); +if (x_138 == 0) +{ +lean_object* x_139; +lean_dec(x_135); +lean_dec(x_133); +x_139 = l_Lean_Expr_forallE___override(x_131, x_9, x_10, x_134); +x_12 = x_139; +goto block_130; +} +else +{ +size_t x_140; size_t x_141; uint8_t x_142; +x_140 = lean_ptr_addr(x_133); +lean_dec(x_133); +x_141 = lean_ptr_addr(x_10); +x_142 = lean_usize_dec_eq(x_140, x_141); +if (x_142 == 0) +{ +lean_object* x_143; +lean_dec(x_135); +x_143 = l_Lean_Expr_forallE___override(x_131, x_9, x_10, x_134); +x_12 = x_143; goto block_130; } else { -lean_object* x_133; lean_object* x_134; +uint8_t x_144; +x_144 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_134, x_134); +if (x_144 == 0) +{ +lean_object* x_145; +lean_dec(x_135); +x_145 = l_Lean_Expr_forallE___override(x_131, x_9, x_10, x_134); +x_12 = x_145; +goto block_130; +} +else +{ +lean_dec(x_131); +lean_dec(x_10); +lean_dec(x_9); +x_12 = x_135; +goto block_130; +} +} +} +} +else +{ +lean_object* x_146; lean_object* x_147; lean_dec(x_10); lean_dec(x_9); lean_dec(x_1); -x_133 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; -x_134 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_133); -x_12 = x_134; +x_146 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; +x_147 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_146); +x_12 = x_147; goto block_130; } block_130: @@ -3121,7 +3180,7 @@ if (x_52 == 0) lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; x_53 = lean_ctor_get(x_43, 0); x_54 = lean_unsigned_to_nat(0u); -x_55 = l_Lean_Expr_getAppNumArgsAux(x_40, x_54); +x_55 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_40, x_54); x_56 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_55); x_57 = lean_mk_array(x_55, x_56); @@ -3140,7 +3199,7 @@ x_62 = lean_ctor_get(x_43, 0); lean_inc(x_62); lean_dec(x_43); x_63 = lean_unsigned_to_nat(0u); -x_64 = l_Lean_Expr_getAppNumArgsAux(x_40, x_63); +x_64 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_40, x_63); x_65 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_64); x_66 = lean_mk_array(x_64, x_65); @@ -3171,7 +3230,7 @@ if (lean_is_exclusive(x_43)) { x_74 = lean_box(0); } x_75 = lean_unsigned_to_nat(0u); -x_76 = l_Lean_Expr_getAppNumArgsAux(x_40, x_75); +x_76 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_40, x_75); x_77 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_76); x_78 = lean_mk_array(x_76, x_77); @@ -3683,7 +3742,7 @@ if (lean_is_exclusive(x_191)) { x_199 = lean_box(0); } x_200 = lean_unsigned_to_nat(0u); -x_201 = l_Lean_Expr_getAppNumArgsAux(x_188, x_200); +x_201 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_188, x_200); x_202 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_201); x_203 = lean_mk_array(x_201, x_202); @@ -7815,7 +7874,7 @@ case 5: { lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; x_19 = lean_unsigned_to_nat(0u); -x_20 = l_Lean_Expr_getAppNumArgsAux(x_18, x_19); +x_20 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_18, x_19); x_21 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_20); x_22 = lean_mk_array(x_20, x_21); @@ -7848,9 +7907,11 @@ return x_31; } case 10: { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_18, 1); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_18, 0); lean_inc(x_32); +x_33 = lean_ctor_get(x_18, 1); +lean_inc(x_33); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); @@ -7859,26 +7920,46 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); +lean_inc(x_33); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_33 = l_Lean_Meta_transform_visit___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__2(x_1, x_2, x_3, x_4, x_5, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_33) == 0) +x_34 = l_Lean_Meta_transform_visit___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__2(x_1, x_2, x_3, x_4, x_5, x_33, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); +lean_object* x_35; lean_object* x_36; size_t x_37; size_t x_38; uint8_t x_39; +x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = lean_ptr_addr(x_33); lean_dec(x_33); -x_36 = lean_expr_update_mdata(x_18, x_34); -x_37 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__3(x_1, x_2, x_3, x_4, x_5, x_36, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_35); -return x_37; +x_38 = lean_ptr_addr(x_35); +x_39 = lean_usize_dec_eq(x_37, x_38); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; +lean_dec(x_18); +x_40 = l_Lean_Expr_mdata___override(x_32, x_35); +x_41 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__3(x_1, x_2, x_3, x_4, x_5, x_40, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_36); +return x_41; } else { -uint8_t x_38; +lean_object* x_42; +lean_dec(x_35); +lean_dec(x_32); +x_42 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__3(x_1, x_2, x_3, x_4, x_5, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_36); +return x_42; +} +} +else +{ +uint8_t x_43; +lean_dec(x_33); +lean_dec(x_32); lean_dec(x_18); lean_dec(x_14); lean_dec(x_13); @@ -7892,31 +7973,35 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_38 = !lean_is_exclusive(x_33); -if (x_38 == 0) +x_43 = !lean_is_exclusive(x_34); +if (x_43 == 0) { -return x_33; +return x_34; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_33, 0); -x_40 = lean_ctor_get(x_33, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_33); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_34, 0); +x_45 = lean_ctor_get(x_34, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_34); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } } } case 11: { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_18, 2); -lean_inc(x_42); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_47 = lean_ctor_get(x_18, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_18, 1); +lean_inc(x_48); +x_49 = lean_ctor_get(x_18, 2); +lean_inc(x_49); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); @@ -7925,26 +8010,48 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); +lean_inc(x_49); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_43 = l_Lean_Meta_transform_visit___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__2(x_1, x_2, x_3, x_4, x_5, x_42, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_43) == 0) +x_50 = l_Lean_Meta_transform_visit___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__2(x_1, x_2, x_3, x_4, x_5, x_49, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_50) == 0) { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_43, 1); -lean_inc(x_45); -lean_dec(x_43); -x_46 = lean_expr_update_proj(x_18, x_44); -x_47 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__3(x_1, x_2, x_3, x_4, x_5, x_46, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_45); -return x_47; +lean_object* x_51; lean_object* x_52; size_t x_53; size_t x_54; uint8_t x_55; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_53 = lean_ptr_addr(x_49); +lean_dec(x_49); +x_54 = lean_ptr_addr(x_51); +x_55 = lean_usize_dec_eq(x_53, x_54); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; +lean_dec(x_18); +x_56 = l_Lean_Expr_proj___override(x_47, x_48, x_51); +x_57 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__3(x_1, x_2, x_3, x_4, x_5, x_56, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_52); +return x_57; } else { -uint8_t x_48; +lean_object* x_58; +lean_dec(x_51); +lean_dec(x_48); +lean_dec(x_47); +x_58 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__3(x_1, x_2, x_3, x_4, x_5, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_52); +return x_58; +} +} +else +{ +uint8_t x_59; +lean_dec(x_49); +lean_dec(x_48); +lean_dec(x_47); lean_dec(x_18); lean_dec(x_14); lean_dec(x_13); @@ -7958,31 +8065,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_43); -if (x_48 == 0) +x_59 = !lean_is_exclusive(x_50); +if (x_59 == 0) { -return x_43; +return x_50; } else { -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; +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_50, 0); +x_61 = lean_ctor_get(x_50, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_50); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +return x_62; } } } default: { -lean_object* x_52; -x_52 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__3(x_1, x_2, x_3, x_4, x_5, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -return x_52; +lean_object* x_63; +x_63 = l_Lean_Meta_transform_visit_visitPost___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__3(x_1, x_2, x_3, x_4, x_5, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +return x_63; } } } @@ -10239,7 +10346,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_Meta_Simp_removeUnnec lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_Meta_Simp_removeUnnecessaryCasts___spec__1___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_Meta_Simp_removeUnnecessaryCasts___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_Meta_Simp_removeUnnecessaryCasts___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10455,7 +10562,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Simp_removeUnnecessaryCasts(lean_object* x_ { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Lean_Expr_getAppNumArgsAux(x_1, x_7); +x_8 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_7); x_9 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_8); x_10 = lean_mk_array(x_8, x_9); @@ -19045,272 +19152,503 @@ lean_dec(x_114); lean_ctor_set(x_85, 0, x_115); if (lean_obj_tag(x_2) == 7) { -uint8_t x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_117 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_118 = lean_expr_update_forall(x_2, x_117, x_4, x_103); -x_119 = lean_unsigned_to_nat(0u); -x_120 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_85); -lean_ctor_set(x_120, 2, x_119); -x_27 = x_120; +lean_object* x_117; lean_object* x_118; lean_object* x_119; uint8_t x_120; lean_object* x_121; size_t x_122; size_t x_123; uint8_t x_124; +x_117 = lean_ctor_get(x_2, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_2, 1); +lean_inc(x_118); +x_119 = lean_ctor_get(x_2, 2); +lean_inc(x_119); +x_120 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_119); +lean_inc(x_118); +lean_inc(x_117); +x_121 = l_Lean_Expr_forallE___override(x_117, x_118, x_119, x_120); +x_122 = lean_ptr_addr(x_118); +lean_dec(x_118); +x_123 = lean_ptr_addr(x_4); +x_124 = lean_usize_dec_eq(x_122, x_123); +if (x_124 == 0) +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_dec(x_121); +lean_dec(x_119); +x_125 = l_Lean_Expr_forallE___override(x_117, x_4, x_103, x_120); +x_126 = lean_unsigned_to_nat(0u); +x_127 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_85); +lean_ctor_set(x_127, 2, x_126); +x_27 = x_127; x_28 = x_116; goto block_48; } else { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +size_t x_128; size_t x_129; uint8_t x_130; +x_128 = lean_ptr_addr(x_119); +lean_dec(x_119); +x_129 = lean_ptr_addr(x_103); +x_130 = lean_usize_dec_eq(x_128, x_129); +if (x_130 == 0) +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; +lean_dec(x_121); +x_131 = l_Lean_Expr_forallE___override(x_117, x_4, x_103, x_120); +x_132 = lean_unsigned_to_nat(0u); +x_133 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_133, 0, x_131); +lean_ctor_set(x_133, 1, x_85); +lean_ctor_set(x_133, 2, x_132); +x_27 = x_133; +x_28 = x_116; +goto block_48; +} +else +{ +uint8_t x_134; +x_134 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_120, x_120); +if (x_134 == 0) +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; +lean_dec(x_121); +x_135 = l_Lean_Expr_forallE___override(x_117, x_4, x_103, x_120); +x_136 = lean_unsigned_to_nat(0u); +x_137 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_137, 0, x_135); +lean_ctor_set(x_137, 1, x_85); +lean_ctor_set(x_137, 2, x_136); +x_27 = x_137; +x_28 = x_116; +goto block_48; +} +else +{ +lean_object* x_138; lean_object* x_139; +lean_dec(x_117); +lean_dec(x_103); +lean_dec(x_4); +x_138 = lean_unsigned_to_nat(0u); +x_139 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_139, 0, x_121); +lean_ctor_set(x_139, 1, x_85); +lean_ctor_set(x_139, 2, x_138); +x_27 = x_139; +x_28 = x_116; +goto block_48; +} +} +} +} +else +{ +lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_dec(x_103); lean_dec(x_4); lean_dec(x_2); -x_121 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; -x_122 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_121); -x_123 = lean_unsigned_to_nat(0u); -x_124 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_124, 0, x_122); -lean_ctor_set(x_124, 1, x_85); -lean_ctor_set(x_124, 2, x_123); -x_27 = x_124; +x_140 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; +x_141 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_140); +x_142 = lean_unsigned_to_nat(0u); +x_143 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_143, 0, x_141); +lean_ctor_set(x_143, 1, x_85); +lean_ctor_set(x_143, 2, x_142); +x_27 = x_143; x_28 = x_116; goto block_48; } } else { -lean_object* x_125; lean_object* x_126; +lean_object* x_144; lean_object* x_145; lean_dec(x_103); lean_free_object(x_85); lean_dec(x_4); lean_dec(x_2); -x_125 = lean_ctor_get(x_114, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_114, 1); -lean_inc(x_126); +x_144 = lean_ctor_get(x_114, 0); +lean_inc(x_144); +x_145 = lean_ctor_get(x_114, 1); +lean_inc(x_145); lean_dec(x_114); -x_49 = x_125; -x_50 = x_126; +x_49 = x_144; +x_50 = x_145; goto block_70; } } else { -uint8_t x_127; uint8_t x_128; uint8_t x_129; uint8_t x_130; uint8_t x_131; uint8_t x_132; uint8_t x_133; uint8_t x_134; uint8_t x_135; uint8_t x_136; uint8_t x_137; uint8_t x_138; uint8_t x_139; uint8_t x_140; lean_object* x_141; lean_object* x_142; -x_127 = lean_ctor_get_uint8(x_107, 0); -x_128 = lean_ctor_get_uint8(x_107, 1); -x_129 = lean_ctor_get_uint8(x_107, 2); -x_130 = lean_ctor_get_uint8(x_107, 3); -x_131 = lean_ctor_get_uint8(x_107, 4); -x_132 = lean_ctor_get_uint8(x_107, 6); -x_133 = lean_ctor_get_uint8(x_107, 7); -x_134 = lean_ctor_get_uint8(x_107, 8); -x_135 = lean_ctor_get_uint8(x_107, 9); -x_136 = lean_ctor_get_uint8(x_107, 10); -x_137 = lean_ctor_get_uint8(x_107, 11); -x_138 = lean_ctor_get_uint8(x_107, 12); -x_139 = lean_ctor_get_uint8(x_107, 13); +uint8_t x_146; uint8_t x_147; uint8_t x_148; uint8_t x_149; uint8_t x_150; uint8_t x_151; uint8_t x_152; uint8_t x_153; uint8_t x_154; uint8_t x_155; uint8_t x_156; uint8_t x_157; uint8_t x_158; uint8_t x_159; lean_object* x_160; lean_object* x_161; +x_146 = lean_ctor_get_uint8(x_107, 0); +x_147 = lean_ctor_get_uint8(x_107, 1); +x_148 = lean_ctor_get_uint8(x_107, 2); +x_149 = lean_ctor_get_uint8(x_107, 3); +x_150 = lean_ctor_get_uint8(x_107, 4); +x_151 = lean_ctor_get_uint8(x_107, 6); +x_152 = lean_ctor_get_uint8(x_107, 7); +x_153 = lean_ctor_get_uint8(x_107, 8); +x_154 = lean_ctor_get_uint8(x_107, 9); +x_155 = lean_ctor_get_uint8(x_107, 10); +x_156 = lean_ctor_get_uint8(x_107, 11); +x_157 = lean_ctor_get_uint8(x_107, 12); +x_158 = lean_ctor_get_uint8(x_107, 13); lean_dec(x_107); -x_140 = 1; -x_141 = lean_alloc_ctor(0, 0, 14); -lean_ctor_set_uint8(x_141, 0, x_127); -lean_ctor_set_uint8(x_141, 1, x_128); -lean_ctor_set_uint8(x_141, 2, x_129); -lean_ctor_set_uint8(x_141, 3, x_130); -lean_ctor_set_uint8(x_141, 4, x_131); -lean_ctor_set_uint8(x_141, 5, x_140); -lean_ctor_set_uint8(x_141, 6, x_132); -lean_ctor_set_uint8(x_141, 7, x_133); -lean_ctor_set_uint8(x_141, 8, x_134); -lean_ctor_set_uint8(x_141, 9, x_135); -lean_ctor_set_uint8(x_141, 10, x_136); -lean_ctor_set_uint8(x_141, 11, x_137); -lean_ctor_set_uint8(x_141, 12, x_138); -lean_ctor_set_uint8(x_141, 13, x_139); -lean_ctor_set(x_9, 0, x_141); +x_159 = 1; +x_160 = lean_alloc_ctor(0, 0, 14); +lean_ctor_set_uint8(x_160, 0, x_146); +lean_ctor_set_uint8(x_160, 1, x_147); +lean_ctor_set_uint8(x_160, 2, x_148); +lean_ctor_set_uint8(x_160, 3, x_149); +lean_ctor_set_uint8(x_160, 4, x_150); +lean_ctor_set_uint8(x_160, 5, x_159); +lean_ctor_set_uint8(x_160, 6, x_151); +lean_ctor_set_uint8(x_160, 7, x_152); +lean_ctor_set_uint8(x_160, 8, x_153); +lean_ctor_set_uint8(x_160, 9, x_154); +lean_ctor_set_uint8(x_160, 10, x_155); +lean_ctor_set_uint8(x_160, 11, x_156); +lean_ctor_set_uint8(x_160, 12, x_157); +lean_ctor_set_uint8(x_160, 13, x_158); +lean_ctor_set(x_9, 0, x_160); lean_inc(x_12); -x_142 = l_Lean_Meta_mkImpCongrCtx(x_108, x_101, x_9, x_10, x_11, x_12, x_109); -if (lean_obj_tag(x_142) == 0) +x_161 = l_Lean_Meta_mkImpCongrCtx(x_108, x_101, x_9, x_10, x_11, x_12, x_109); +if (lean_obj_tag(x_161) == 0) { -lean_object* x_143; lean_object* x_144; -x_143 = lean_ctor_get(x_142, 0); -lean_inc(x_143); -x_144 = lean_ctor_get(x_142, 1); -lean_inc(x_144); -lean_dec(x_142); -lean_ctor_set(x_85, 0, x_143); +lean_object* x_162; lean_object* x_163; +x_162 = lean_ctor_get(x_161, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_161, 1); +lean_inc(x_163); +lean_dec(x_161); +lean_ctor_set(x_85, 0, x_162); if (lean_obj_tag(x_2) == 7) { -uint8_t x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_145 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_146 = lean_expr_update_forall(x_2, x_145, x_4, x_103); -x_147 = lean_unsigned_to_nat(0u); -x_148 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_148, 0, x_146); -lean_ctor_set(x_148, 1, x_85); -lean_ctor_set(x_148, 2, x_147); -x_27 = x_148; -x_28 = x_144; +lean_object* x_164; lean_object* x_165; lean_object* x_166; uint8_t x_167; lean_object* x_168; size_t x_169; size_t x_170; uint8_t x_171; +x_164 = lean_ctor_get(x_2, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_2, 1); +lean_inc(x_165); +x_166 = lean_ctor_get(x_2, 2); +lean_inc(x_166); +x_167 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_166); +lean_inc(x_165); +lean_inc(x_164); +x_168 = l_Lean_Expr_forallE___override(x_164, x_165, x_166, x_167); +x_169 = lean_ptr_addr(x_165); +lean_dec(x_165); +x_170 = lean_ptr_addr(x_4); +x_171 = lean_usize_dec_eq(x_169, x_170); +if (x_171 == 0) +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; +lean_dec(x_168); +lean_dec(x_166); +x_172 = l_Lean_Expr_forallE___override(x_164, x_4, x_103, x_167); +x_173 = lean_unsigned_to_nat(0u); +x_174 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_174, 0, x_172); +lean_ctor_set(x_174, 1, x_85); +lean_ctor_set(x_174, 2, x_173); +x_27 = x_174; +x_28 = x_163; +goto block_48; +} +else +{ +size_t x_175; size_t x_176; uint8_t x_177; +x_175 = lean_ptr_addr(x_166); +lean_dec(x_166); +x_176 = lean_ptr_addr(x_103); +x_177 = lean_usize_dec_eq(x_175, x_176); +if (x_177 == 0) +{ +lean_object* x_178; lean_object* x_179; lean_object* x_180; +lean_dec(x_168); +x_178 = l_Lean_Expr_forallE___override(x_164, x_4, x_103, x_167); +x_179 = lean_unsigned_to_nat(0u); +x_180 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_180, 0, x_178); +lean_ctor_set(x_180, 1, x_85); +lean_ctor_set(x_180, 2, x_179); +x_27 = x_180; +x_28 = x_163; goto block_48; } else { -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; +uint8_t x_181; +x_181 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_167, x_167); +if (x_181 == 0) +{ +lean_object* x_182; lean_object* x_183; lean_object* x_184; +lean_dec(x_168); +x_182 = l_Lean_Expr_forallE___override(x_164, x_4, x_103, x_167); +x_183 = lean_unsigned_to_nat(0u); +x_184 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_184, 0, x_182); +lean_ctor_set(x_184, 1, x_85); +lean_ctor_set(x_184, 2, x_183); +x_27 = x_184; +x_28 = x_163; +goto block_48; +} +else +{ +lean_object* x_185; lean_object* x_186; +lean_dec(x_164); +lean_dec(x_103); +lean_dec(x_4); +x_185 = lean_unsigned_to_nat(0u); +x_186 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_186, 0, x_168); +lean_ctor_set(x_186, 1, x_85); +lean_ctor_set(x_186, 2, x_185); +x_27 = x_186; +x_28 = x_163; +goto block_48; +} +} +} +} +else +{ +lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_dec(x_103); lean_dec(x_4); lean_dec(x_2); -x_149 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; -x_150 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_149); -x_151 = lean_unsigned_to_nat(0u); -x_152 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_152, 0, x_150); -lean_ctor_set(x_152, 1, x_85); -lean_ctor_set(x_152, 2, x_151); -x_27 = x_152; -x_28 = x_144; +x_187 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; +x_188 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_187); +x_189 = lean_unsigned_to_nat(0u); +x_190 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_190, 0, x_188); +lean_ctor_set(x_190, 1, x_85); +lean_ctor_set(x_190, 2, x_189); +x_27 = x_190; +x_28 = x_163; goto block_48; } } else { -lean_object* x_153; lean_object* x_154; +lean_object* x_191; lean_object* x_192; lean_dec(x_103); lean_free_object(x_85); lean_dec(x_4); lean_dec(x_2); -x_153 = lean_ctor_get(x_142, 0); -lean_inc(x_153); -x_154 = lean_ctor_get(x_142, 1); -lean_inc(x_154); -lean_dec(x_142); -x_49 = x_153; -x_50 = x_154; +x_191 = lean_ctor_get(x_161, 0); +lean_inc(x_191); +x_192 = lean_ctor_get(x_161, 1); +lean_inc(x_192); +lean_dec(x_161); +x_49 = x_191; +x_50 = x_192; goto block_70; } } } else { -lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; uint8_t x_160; uint8_t x_161; uint8_t x_162; uint8_t x_163; uint8_t x_164; uint8_t x_165; uint8_t x_166; uint8_t x_167; uint8_t x_168; uint8_t x_169; uint8_t x_170; uint8_t x_171; uint8_t x_172; lean_object* x_173; uint8_t x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; -x_155 = lean_ctor_get(x_9, 1); -x_156 = lean_ctor_get(x_9, 2); -x_157 = lean_ctor_get(x_9, 3); -x_158 = lean_ctor_get(x_9, 4); -x_159 = lean_ctor_get(x_9, 5); -lean_inc(x_159); -lean_inc(x_158); -lean_inc(x_157); -lean_inc(x_156); -lean_inc(x_155); +lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; uint8_t x_198; uint8_t x_199; uint8_t x_200; uint8_t x_201; uint8_t x_202; uint8_t x_203; uint8_t x_204; uint8_t x_205; uint8_t x_206; uint8_t x_207; uint8_t x_208; uint8_t x_209; uint8_t x_210; lean_object* x_211; uint8_t x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; +x_193 = lean_ctor_get(x_9, 1); +x_194 = lean_ctor_get(x_9, 2); +x_195 = lean_ctor_get(x_9, 3); +x_196 = lean_ctor_get(x_9, 4); +x_197 = lean_ctor_get(x_9, 5); +lean_inc(x_197); +lean_inc(x_196); +lean_inc(x_195); +lean_inc(x_194); +lean_inc(x_193); lean_dec(x_9); -x_160 = lean_ctor_get_uint8(x_107, 0); -x_161 = lean_ctor_get_uint8(x_107, 1); -x_162 = lean_ctor_get_uint8(x_107, 2); -x_163 = lean_ctor_get_uint8(x_107, 3); -x_164 = lean_ctor_get_uint8(x_107, 4); -x_165 = lean_ctor_get_uint8(x_107, 6); -x_166 = lean_ctor_get_uint8(x_107, 7); -x_167 = lean_ctor_get_uint8(x_107, 8); -x_168 = lean_ctor_get_uint8(x_107, 9); -x_169 = lean_ctor_get_uint8(x_107, 10); -x_170 = lean_ctor_get_uint8(x_107, 11); -x_171 = lean_ctor_get_uint8(x_107, 12); -x_172 = lean_ctor_get_uint8(x_107, 13); +x_198 = lean_ctor_get_uint8(x_107, 0); +x_199 = lean_ctor_get_uint8(x_107, 1); +x_200 = lean_ctor_get_uint8(x_107, 2); +x_201 = lean_ctor_get_uint8(x_107, 3); +x_202 = lean_ctor_get_uint8(x_107, 4); +x_203 = lean_ctor_get_uint8(x_107, 6); +x_204 = lean_ctor_get_uint8(x_107, 7); +x_205 = lean_ctor_get_uint8(x_107, 8); +x_206 = lean_ctor_get_uint8(x_107, 9); +x_207 = lean_ctor_get_uint8(x_107, 10); +x_208 = lean_ctor_get_uint8(x_107, 11); +x_209 = lean_ctor_get_uint8(x_107, 12); +x_210 = lean_ctor_get_uint8(x_107, 13); if (lean_is_exclusive(x_107)) { - x_173 = x_107; + x_211 = x_107; } else { lean_dec_ref(x_107); - x_173 = lean_box(0); -} -x_174 = 1; -if (lean_is_scalar(x_173)) { - x_175 = lean_alloc_ctor(0, 0, 14); -} else { - x_175 = x_173; -} -lean_ctor_set_uint8(x_175, 0, x_160); -lean_ctor_set_uint8(x_175, 1, x_161); -lean_ctor_set_uint8(x_175, 2, x_162); -lean_ctor_set_uint8(x_175, 3, x_163); -lean_ctor_set_uint8(x_175, 4, x_164); -lean_ctor_set_uint8(x_175, 5, x_174); -lean_ctor_set_uint8(x_175, 6, x_165); -lean_ctor_set_uint8(x_175, 7, x_166); -lean_ctor_set_uint8(x_175, 8, x_167); -lean_ctor_set_uint8(x_175, 9, x_168); -lean_ctor_set_uint8(x_175, 10, x_169); -lean_ctor_set_uint8(x_175, 11, x_170); -lean_ctor_set_uint8(x_175, 12, x_171); -lean_ctor_set_uint8(x_175, 13, x_172); -x_176 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_176, 0, x_175); -lean_ctor_set(x_176, 1, x_155); -lean_ctor_set(x_176, 2, x_156); -lean_ctor_set(x_176, 3, x_157); -lean_ctor_set(x_176, 4, x_158); -lean_ctor_set(x_176, 5, x_159); + x_211 = lean_box(0); +} +x_212 = 1; +if (lean_is_scalar(x_211)) { + x_213 = lean_alloc_ctor(0, 0, 14); +} else { + x_213 = x_211; +} +lean_ctor_set_uint8(x_213, 0, x_198); +lean_ctor_set_uint8(x_213, 1, x_199); +lean_ctor_set_uint8(x_213, 2, x_200); +lean_ctor_set_uint8(x_213, 3, x_201); +lean_ctor_set_uint8(x_213, 4, x_202); +lean_ctor_set_uint8(x_213, 5, x_212); +lean_ctor_set_uint8(x_213, 6, x_203); +lean_ctor_set_uint8(x_213, 7, x_204); +lean_ctor_set_uint8(x_213, 8, x_205); +lean_ctor_set_uint8(x_213, 9, x_206); +lean_ctor_set_uint8(x_213, 10, x_207); +lean_ctor_set_uint8(x_213, 11, x_208); +lean_ctor_set_uint8(x_213, 12, x_209); +lean_ctor_set_uint8(x_213, 13, x_210); +x_214 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_214, 0, x_213); +lean_ctor_set(x_214, 1, x_193); +lean_ctor_set(x_214, 2, x_194); +lean_ctor_set(x_214, 3, x_195); +lean_ctor_set(x_214, 4, x_196); +lean_ctor_set(x_214, 5, x_197); lean_inc(x_12); -x_177 = l_Lean_Meta_mkImpCongrCtx(x_108, x_101, x_176, x_10, x_11, x_12, x_109); -if (lean_obj_tag(x_177) == 0) +x_215 = l_Lean_Meta_mkImpCongrCtx(x_108, x_101, x_214, x_10, x_11, x_12, x_109); +if (lean_obj_tag(x_215) == 0) { -lean_object* x_178; lean_object* x_179; -x_178 = lean_ctor_get(x_177, 0); -lean_inc(x_178); -x_179 = lean_ctor_get(x_177, 1); -lean_inc(x_179); -lean_dec(x_177); -lean_ctor_set(x_85, 0, x_178); +lean_object* x_216; lean_object* x_217; +x_216 = lean_ctor_get(x_215, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_215, 1); +lean_inc(x_217); +lean_dec(x_215); +lean_ctor_set(x_85, 0, x_216); if (lean_obj_tag(x_2) == 7) { -uint8_t x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_180 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_181 = lean_expr_update_forall(x_2, x_180, x_4, x_103); -x_182 = lean_unsigned_to_nat(0u); -x_183 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_183, 0, x_181); -lean_ctor_set(x_183, 1, x_85); -lean_ctor_set(x_183, 2, x_182); -x_27 = x_183; -x_28 = x_179; +lean_object* x_218; lean_object* x_219; lean_object* x_220; uint8_t x_221; lean_object* x_222; size_t x_223; size_t x_224; uint8_t x_225; +x_218 = lean_ctor_get(x_2, 0); +lean_inc(x_218); +x_219 = lean_ctor_get(x_2, 1); +lean_inc(x_219); +x_220 = lean_ctor_get(x_2, 2); +lean_inc(x_220); +x_221 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_220); +lean_inc(x_219); +lean_inc(x_218); +x_222 = l_Lean_Expr_forallE___override(x_218, x_219, x_220, x_221); +x_223 = lean_ptr_addr(x_219); +lean_dec(x_219); +x_224 = lean_ptr_addr(x_4); +x_225 = lean_usize_dec_eq(x_223, x_224); +if (x_225 == 0) +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; +lean_dec(x_222); +lean_dec(x_220); +x_226 = l_Lean_Expr_forallE___override(x_218, x_4, x_103, x_221); +x_227 = lean_unsigned_to_nat(0u); +x_228 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_228, 0, x_226); +lean_ctor_set(x_228, 1, x_85); +lean_ctor_set(x_228, 2, x_227); +x_27 = x_228; +x_28 = x_217; goto block_48; } else { -lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +size_t x_229; size_t x_230; uint8_t x_231; +x_229 = lean_ptr_addr(x_220); +lean_dec(x_220); +x_230 = lean_ptr_addr(x_103); +x_231 = lean_usize_dec_eq(x_229, x_230); +if (x_231 == 0) +{ +lean_object* x_232; lean_object* x_233; lean_object* x_234; +lean_dec(x_222); +x_232 = l_Lean_Expr_forallE___override(x_218, x_4, x_103, x_221); +x_233 = lean_unsigned_to_nat(0u); +x_234 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_234, 0, x_232); +lean_ctor_set(x_234, 1, x_85); +lean_ctor_set(x_234, 2, x_233); +x_27 = x_234; +x_28 = x_217; +goto block_48; +} +else +{ +uint8_t x_235; +x_235 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_221, x_221); +if (x_235 == 0) +{ +lean_object* x_236; lean_object* x_237; lean_object* x_238; +lean_dec(x_222); +x_236 = l_Lean_Expr_forallE___override(x_218, x_4, x_103, x_221); +x_237 = lean_unsigned_to_nat(0u); +x_238 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_238, 0, x_236); +lean_ctor_set(x_238, 1, x_85); +lean_ctor_set(x_238, 2, x_237); +x_27 = x_238; +x_28 = x_217; +goto block_48; +} +else +{ +lean_object* x_239; lean_object* x_240; +lean_dec(x_218); +lean_dec(x_103); +lean_dec(x_4); +x_239 = lean_unsigned_to_nat(0u); +x_240 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_240, 0, x_222); +lean_ctor_set(x_240, 1, x_85); +lean_ctor_set(x_240, 2, x_239); +x_27 = x_240; +x_28 = x_217; +goto block_48; +} +} +} +} +else +{ +lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_dec(x_103); lean_dec(x_4); lean_dec(x_2); -x_184 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; -x_185 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_184); -x_186 = lean_unsigned_to_nat(0u); -x_187 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_187, 0, x_185); -lean_ctor_set(x_187, 1, x_85); -lean_ctor_set(x_187, 2, x_186); -x_27 = x_187; -x_28 = x_179; +x_241 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; +x_242 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_241); +x_243 = lean_unsigned_to_nat(0u); +x_244 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_244, 0, x_242); +lean_ctor_set(x_244, 1, x_85); +lean_ctor_set(x_244, 2, x_243); +x_27 = x_244; +x_28 = x_217; goto block_48; } } else { -lean_object* x_188; lean_object* x_189; +lean_object* x_245; lean_object* x_246; lean_dec(x_103); lean_free_object(x_85); lean_dec(x_4); lean_dec(x_2); -x_188 = lean_ctor_get(x_177, 0); -lean_inc(x_188); -x_189 = lean_ctor_get(x_177, 1); -lean_inc(x_189); -lean_dec(x_177); -x_49 = x_188; -x_50 = x_189; +x_245 = lean_ctor_get(x_215, 0); +lean_inc(x_245); +x_246 = lean_ctor_get(x_215, 1); +lean_inc(x_246); +lean_dec(x_215); +x_49 = x_245; +x_50 = x_246; goto block_70; } } } else { -lean_object* x_190; lean_object* x_191; +lean_object* x_247; lean_object* x_248; lean_dec(x_103); lean_dec(x_101); lean_free_object(x_85); @@ -19319,300 +19657,300 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_4); lean_dec(x_2); -x_190 = lean_ctor_get(x_106, 0); -lean_inc(x_190); -x_191 = lean_ctor_get(x_106, 1); -lean_inc(x_191); +x_247 = lean_ctor_get(x_106, 0); +lean_inc(x_247); +x_248 = lean_ctor_get(x_106, 1); +lean_inc(x_248); lean_dec(x_106); -x_49 = x_190; -x_50 = x_191; +x_49 = x_247; +x_50 = x_248; goto block_70; } } else { -lean_object* x_192; +lean_object* x_249; lean_dec(x_4); lean_dec(x_2); -x_192 = l_Lean_Meta_mkForallFVars(x_96, x_103, x_97, x_98, x_99, x_9, x_10, x_11, x_12, x_102); -if (lean_obj_tag(x_192) == 0) +x_249 = l_Lean_Meta_mkForallFVars(x_96, x_103, x_97, x_98, x_99, x_9, x_10, x_11, x_12, x_102); +if (lean_obj_tag(x_249) == 0) { -lean_object* x_193; lean_object* x_194; lean_object* x_195; -x_193 = lean_ctor_get(x_192, 0); -lean_inc(x_193); -x_194 = lean_ctor_get(x_192, 1); -lean_inc(x_194); -lean_dec(x_192); +lean_object* x_250; lean_object* x_251; lean_object* x_252; +x_250 = lean_ctor_get(x_249, 0); +lean_inc(x_250); +x_251 = lean_ctor_get(x_249, 1); +lean_inc(x_251); +lean_dec(x_249); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_195 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_194); -if (lean_obj_tag(x_195) == 0) +x_252 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_251); +if (lean_obj_tag(x_252) == 0) { -lean_object* x_196; lean_object* x_197; lean_object* x_198; uint8_t x_199; -x_196 = lean_ctor_get(x_9, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_195, 0); -lean_inc(x_197); -x_198 = lean_ctor_get(x_195, 1); -lean_inc(x_198); -lean_dec(x_195); -x_199 = !lean_is_exclusive(x_9); -if (x_199 == 0) -{ -lean_object* x_200; uint8_t x_201; -x_200 = lean_ctor_get(x_9, 0); -lean_dec(x_200); -x_201 = !lean_is_exclusive(x_196); -if (x_201 == 0) -{ -uint8_t x_202; lean_object* x_203; -x_202 = 1; -lean_ctor_set_uint8(x_196, 5, x_202); +lean_object* x_253; lean_object* x_254; lean_object* x_255; uint8_t x_256; +x_253 = lean_ctor_get(x_9, 0); +lean_inc(x_253); +x_254 = lean_ctor_get(x_252, 0); +lean_inc(x_254); +x_255 = lean_ctor_get(x_252, 1); +lean_inc(x_255); +lean_dec(x_252); +x_256 = !lean_is_exclusive(x_9); +if (x_256 == 0) +{ +lean_object* x_257; uint8_t x_258; +x_257 = lean_ctor_get(x_9, 0); +lean_dec(x_257); +x_258 = !lean_is_exclusive(x_253); +if (x_258 == 0) +{ +uint8_t x_259; lean_object* x_260; +x_259 = 1; +lean_ctor_set_uint8(x_253, 5, x_259); lean_inc(x_12); -x_203 = l_Lean_Meta_mkImpDepCongrCtx(x_197, x_101, x_9, x_10, x_11, x_12, x_198); -if (lean_obj_tag(x_203) == 0) +x_260 = l_Lean_Meta_mkImpDepCongrCtx(x_254, x_101, x_9, x_10, x_11, x_12, x_255); +if (lean_obj_tag(x_260) == 0) { -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; -x_204 = lean_ctor_get(x_203, 0); -lean_inc(x_204); -x_205 = lean_ctor_get(x_203, 1); -lean_inc(x_205); -lean_dec(x_203); -lean_ctor_set(x_85, 0, x_204); -x_206 = lean_unsigned_to_nat(0u); -x_207 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_207, 0, x_193); -lean_ctor_set(x_207, 1, x_85); -lean_ctor_set(x_207, 2, x_206); -x_27 = x_207; -x_28 = x_205; +lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; +x_261 = lean_ctor_get(x_260, 0); +lean_inc(x_261); +x_262 = lean_ctor_get(x_260, 1); +lean_inc(x_262); +lean_dec(x_260); +lean_ctor_set(x_85, 0, x_261); +x_263 = lean_unsigned_to_nat(0u); +x_264 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_264, 0, x_250); +lean_ctor_set(x_264, 1, x_85); +lean_ctor_set(x_264, 2, x_263); +x_27 = x_264; +x_28 = x_262; goto block_48; } else { -lean_object* x_208; lean_object* x_209; -lean_dec(x_193); +lean_object* x_265; lean_object* x_266; +lean_dec(x_250); lean_free_object(x_85); -x_208 = lean_ctor_get(x_203, 0); -lean_inc(x_208); -x_209 = lean_ctor_get(x_203, 1); -lean_inc(x_209); -lean_dec(x_203); -x_49 = x_208; -x_50 = x_209; +x_265 = lean_ctor_get(x_260, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_260, 1); +lean_inc(x_266); +lean_dec(x_260); +x_49 = x_265; +x_50 = x_266; goto block_70; } } else { -uint8_t x_210; uint8_t x_211; uint8_t x_212; uint8_t x_213; uint8_t x_214; uint8_t x_215; uint8_t x_216; uint8_t x_217; uint8_t x_218; uint8_t x_219; uint8_t x_220; uint8_t x_221; uint8_t x_222; uint8_t x_223; lean_object* x_224; lean_object* x_225; -x_210 = lean_ctor_get_uint8(x_196, 0); -x_211 = lean_ctor_get_uint8(x_196, 1); -x_212 = lean_ctor_get_uint8(x_196, 2); -x_213 = lean_ctor_get_uint8(x_196, 3); -x_214 = lean_ctor_get_uint8(x_196, 4); -x_215 = lean_ctor_get_uint8(x_196, 6); -x_216 = lean_ctor_get_uint8(x_196, 7); -x_217 = lean_ctor_get_uint8(x_196, 8); -x_218 = lean_ctor_get_uint8(x_196, 9); -x_219 = lean_ctor_get_uint8(x_196, 10); -x_220 = lean_ctor_get_uint8(x_196, 11); -x_221 = lean_ctor_get_uint8(x_196, 12); -x_222 = lean_ctor_get_uint8(x_196, 13); -lean_dec(x_196); -x_223 = 1; -x_224 = lean_alloc_ctor(0, 0, 14); -lean_ctor_set_uint8(x_224, 0, x_210); -lean_ctor_set_uint8(x_224, 1, x_211); -lean_ctor_set_uint8(x_224, 2, x_212); -lean_ctor_set_uint8(x_224, 3, x_213); -lean_ctor_set_uint8(x_224, 4, x_214); -lean_ctor_set_uint8(x_224, 5, x_223); -lean_ctor_set_uint8(x_224, 6, x_215); -lean_ctor_set_uint8(x_224, 7, x_216); -lean_ctor_set_uint8(x_224, 8, x_217); -lean_ctor_set_uint8(x_224, 9, x_218); -lean_ctor_set_uint8(x_224, 10, x_219); -lean_ctor_set_uint8(x_224, 11, x_220); -lean_ctor_set_uint8(x_224, 12, x_221); -lean_ctor_set_uint8(x_224, 13, x_222); -lean_ctor_set(x_9, 0, x_224); +uint8_t x_267; uint8_t x_268; uint8_t x_269; uint8_t x_270; uint8_t x_271; uint8_t x_272; uint8_t x_273; uint8_t x_274; uint8_t x_275; uint8_t x_276; uint8_t x_277; uint8_t x_278; uint8_t x_279; uint8_t x_280; lean_object* x_281; lean_object* x_282; +x_267 = lean_ctor_get_uint8(x_253, 0); +x_268 = lean_ctor_get_uint8(x_253, 1); +x_269 = lean_ctor_get_uint8(x_253, 2); +x_270 = lean_ctor_get_uint8(x_253, 3); +x_271 = lean_ctor_get_uint8(x_253, 4); +x_272 = lean_ctor_get_uint8(x_253, 6); +x_273 = lean_ctor_get_uint8(x_253, 7); +x_274 = lean_ctor_get_uint8(x_253, 8); +x_275 = lean_ctor_get_uint8(x_253, 9); +x_276 = lean_ctor_get_uint8(x_253, 10); +x_277 = lean_ctor_get_uint8(x_253, 11); +x_278 = lean_ctor_get_uint8(x_253, 12); +x_279 = lean_ctor_get_uint8(x_253, 13); +lean_dec(x_253); +x_280 = 1; +x_281 = lean_alloc_ctor(0, 0, 14); +lean_ctor_set_uint8(x_281, 0, x_267); +lean_ctor_set_uint8(x_281, 1, x_268); +lean_ctor_set_uint8(x_281, 2, x_269); +lean_ctor_set_uint8(x_281, 3, x_270); +lean_ctor_set_uint8(x_281, 4, x_271); +lean_ctor_set_uint8(x_281, 5, x_280); +lean_ctor_set_uint8(x_281, 6, x_272); +lean_ctor_set_uint8(x_281, 7, x_273); +lean_ctor_set_uint8(x_281, 8, x_274); +lean_ctor_set_uint8(x_281, 9, x_275); +lean_ctor_set_uint8(x_281, 10, x_276); +lean_ctor_set_uint8(x_281, 11, x_277); +lean_ctor_set_uint8(x_281, 12, x_278); +lean_ctor_set_uint8(x_281, 13, x_279); +lean_ctor_set(x_9, 0, x_281); lean_inc(x_12); -x_225 = l_Lean_Meta_mkImpDepCongrCtx(x_197, x_101, x_9, x_10, x_11, x_12, x_198); -if (lean_obj_tag(x_225) == 0) +x_282 = l_Lean_Meta_mkImpDepCongrCtx(x_254, x_101, x_9, x_10, x_11, x_12, x_255); +if (lean_obj_tag(x_282) == 0) { -lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; -x_226 = lean_ctor_get(x_225, 0); -lean_inc(x_226); -x_227 = lean_ctor_get(x_225, 1); -lean_inc(x_227); -lean_dec(x_225); -lean_ctor_set(x_85, 0, x_226); -x_228 = lean_unsigned_to_nat(0u); -x_229 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_229, 0, x_193); -lean_ctor_set(x_229, 1, x_85); -lean_ctor_set(x_229, 2, x_228); -x_27 = x_229; -x_28 = x_227; +lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; +x_283 = lean_ctor_get(x_282, 0); +lean_inc(x_283); +x_284 = lean_ctor_get(x_282, 1); +lean_inc(x_284); +lean_dec(x_282); +lean_ctor_set(x_85, 0, x_283); +x_285 = lean_unsigned_to_nat(0u); +x_286 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_286, 0, x_250); +lean_ctor_set(x_286, 1, x_85); +lean_ctor_set(x_286, 2, x_285); +x_27 = x_286; +x_28 = x_284; goto block_48; } else { -lean_object* x_230; lean_object* x_231; -lean_dec(x_193); +lean_object* x_287; lean_object* x_288; +lean_dec(x_250); lean_free_object(x_85); -x_230 = lean_ctor_get(x_225, 0); -lean_inc(x_230); -x_231 = lean_ctor_get(x_225, 1); -lean_inc(x_231); -lean_dec(x_225); -x_49 = x_230; -x_50 = x_231; +x_287 = lean_ctor_get(x_282, 0); +lean_inc(x_287); +x_288 = lean_ctor_get(x_282, 1); +lean_inc(x_288); +lean_dec(x_282); +x_49 = x_287; +x_50 = x_288; goto block_70; } } } else { -lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; uint8_t x_237; uint8_t x_238; uint8_t x_239; uint8_t x_240; uint8_t x_241; uint8_t x_242; uint8_t x_243; uint8_t x_244; uint8_t x_245; uint8_t x_246; uint8_t x_247; uint8_t x_248; uint8_t x_249; lean_object* x_250; uint8_t x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; -x_232 = lean_ctor_get(x_9, 1); -x_233 = lean_ctor_get(x_9, 2); -x_234 = lean_ctor_get(x_9, 3); -x_235 = lean_ctor_get(x_9, 4); -x_236 = lean_ctor_get(x_9, 5); -lean_inc(x_236); -lean_inc(x_235); -lean_inc(x_234); -lean_inc(x_233); -lean_inc(x_232); -lean_dec(x_9); -x_237 = lean_ctor_get_uint8(x_196, 0); -x_238 = lean_ctor_get_uint8(x_196, 1); -x_239 = lean_ctor_get_uint8(x_196, 2); -x_240 = lean_ctor_get_uint8(x_196, 3); -x_241 = lean_ctor_get_uint8(x_196, 4); -x_242 = lean_ctor_get_uint8(x_196, 6); -x_243 = lean_ctor_get_uint8(x_196, 7); -x_244 = lean_ctor_get_uint8(x_196, 8); -x_245 = lean_ctor_get_uint8(x_196, 9); -x_246 = lean_ctor_get_uint8(x_196, 10); -x_247 = lean_ctor_get_uint8(x_196, 11); -x_248 = lean_ctor_get_uint8(x_196, 12); -x_249 = lean_ctor_get_uint8(x_196, 13); -if (lean_is_exclusive(x_196)) { - x_250 = x_196; -} else { - lean_dec_ref(x_196); - x_250 = lean_box(0); -} -x_251 = 1; -if (lean_is_scalar(x_250)) { - x_252 = lean_alloc_ctor(0, 0, 14); -} else { - x_252 = x_250; -} -lean_ctor_set_uint8(x_252, 0, x_237); -lean_ctor_set_uint8(x_252, 1, x_238); -lean_ctor_set_uint8(x_252, 2, x_239); -lean_ctor_set_uint8(x_252, 3, x_240); -lean_ctor_set_uint8(x_252, 4, x_241); -lean_ctor_set_uint8(x_252, 5, x_251); -lean_ctor_set_uint8(x_252, 6, x_242); -lean_ctor_set_uint8(x_252, 7, x_243); -lean_ctor_set_uint8(x_252, 8, x_244); -lean_ctor_set_uint8(x_252, 9, x_245); -lean_ctor_set_uint8(x_252, 10, x_246); -lean_ctor_set_uint8(x_252, 11, x_247); -lean_ctor_set_uint8(x_252, 12, x_248); -lean_ctor_set_uint8(x_252, 13, x_249); -x_253 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_253, 0, x_252); -lean_ctor_set(x_253, 1, x_232); -lean_ctor_set(x_253, 2, x_233); -lean_ctor_set(x_253, 3, x_234); -lean_ctor_set(x_253, 4, x_235); -lean_ctor_set(x_253, 5, x_236); +lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; uint8_t x_295; uint8_t x_296; uint8_t x_297; uint8_t x_298; uint8_t x_299; uint8_t x_300; uint8_t x_301; uint8_t x_302; uint8_t x_303; uint8_t x_304; uint8_t x_305; uint8_t x_306; lean_object* x_307; uint8_t x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; +x_289 = lean_ctor_get(x_9, 1); +x_290 = lean_ctor_get(x_9, 2); +x_291 = lean_ctor_get(x_9, 3); +x_292 = lean_ctor_get(x_9, 4); +x_293 = lean_ctor_get(x_9, 5); +lean_inc(x_293); +lean_inc(x_292); +lean_inc(x_291); +lean_inc(x_290); +lean_inc(x_289); +lean_dec(x_9); +x_294 = lean_ctor_get_uint8(x_253, 0); +x_295 = lean_ctor_get_uint8(x_253, 1); +x_296 = lean_ctor_get_uint8(x_253, 2); +x_297 = lean_ctor_get_uint8(x_253, 3); +x_298 = lean_ctor_get_uint8(x_253, 4); +x_299 = lean_ctor_get_uint8(x_253, 6); +x_300 = lean_ctor_get_uint8(x_253, 7); +x_301 = lean_ctor_get_uint8(x_253, 8); +x_302 = lean_ctor_get_uint8(x_253, 9); +x_303 = lean_ctor_get_uint8(x_253, 10); +x_304 = lean_ctor_get_uint8(x_253, 11); +x_305 = lean_ctor_get_uint8(x_253, 12); +x_306 = lean_ctor_get_uint8(x_253, 13); +if (lean_is_exclusive(x_253)) { + x_307 = x_253; +} else { + lean_dec_ref(x_253); + x_307 = lean_box(0); +} +x_308 = 1; +if (lean_is_scalar(x_307)) { + x_309 = lean_alloc_ctor(0, 0, 14); +} else { + x_309 = x_307; +} +lean_ctor_set_uint8(x_309, 0, x_294); +lean_ctor_set_uint8(x_309, 1, x_295); +lean_ctor_set_uint8(x_309, 2, x_296); +lean_ctor_set_uint8(x_309, 3, x_297); +lean_ctor_set_uint8(x_309, 4, x_298); +lean_ctor_set_uint8(x_309, 5, x_308); +lean_ctor_set_uint8(x_309, 6, x_299); +lean_ctor_set_uint8(x_309, 7, x_300); +lean_ctor_set_uint8(x_309, 8, x_301); +lean_ctor_set_uint8(x_309, 9, x_302); +lean_ctor_set_uint8(x_309, 10, x_303); +lean_ctor_set_uint8(x_309, 11, x_304); +lean_ctor_set_uint8(x_309, 12, x_305); +lean_ctor_set_uint8(x_309, 13, x_306); +x_310 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_310, 0, x_309); +lean_ctor_set(x_310, 1, x_289); +lean_ctor_set(x_310, 2, x_290); +lean_ctor_set(x_310, 3, x_291); +lean_ctor_set(x_310, 4, x_292); +lean_ctor_set(x_310, 5, x_293); lean_inc(x_12); -x_254 = l_Lean_Meta_mkImpDepCongrCtx(x_197, x_101, x_253, x_10, x_11, x_12, x_198); -if (lean_obj_tag(x_254) == 0) -{ -lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; -x_255 = lean_ctor_get(x_254, 0); -lean_inc(x_255); -x_256 = lean_ctor_get(x_254, 1); -lean_inc(x_256); -lean_dec(x_254); -lean_ctor_set(x_85, 0, x_255); -x_257 = lean_unsigned_to_nat(0u); -x_258 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_258, 0, x_193); -lean_ctor_set(x_258, 1, x_85); -lean_ctor_set(x_258, 2, x_257); -x_27 = x_258; -x_28 = x_256; +x_311 = l_Lean_Meta_mkImpDepCongrCtx(x_254, x_101, x_310, x_10, x_11, x_12, x_255); +if (lean_obj_tag(x_311) == 0) +{ +lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; +x_312 = lean_ctor_get(x_311, 0); +lean_inc(x_312); +x_313 = lean_ctor_get(x_311, 1); +lean_inc(x_313); +lean_dec(x_311); +lean_ctor_set(x_85, 0, x_312); +x_314 = lean_unsigned_to_nat(0u); +x_315 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_315, 0, x_250); +lean_ctor_set(x_315, 1, x_85); +lean_ctor_set(x_315, 2, x_314); +x_27 = x_315; +x_28 = x_313; goto block_48; } else { -lean_object* x_259; lean_object* x_260; -lean_dec(x_193); +lean_object* x_316; lean_object* x_317; +lean_dec(x_250); lean_free_object(x_85); -x_259 = lean_ctor_get(x_254, 0); -lean_inc(x_259); -x_260 = lean_ctor_get(x_254, 1); -lean_inc(x_260); -lean_dec(x_254); -x_49 = x_259; -x_50 = x_260; +x_316 = lean_ctor_get(x_311, 0); +lean_inc(x_316); +x_317 = lean_ctor_get(x_311, 1); +lean_inc(x_317); +lean_dec(x_311); +x_49 = x_316; +x_50 = x_317; goto block_70; } } } else { -lean_object* x_261; lean_object* x_262; -lean_dec(x_193); +lean_object* x_318; lean_object* x_319; +lean_dec(x_250); lean_dec(x_101); lean_free_object(x_85); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -x_261 = lean_ctor_get(x_195, 0); -lean_inc(x_261); -x_262 = lean_ctor_get(x_195, 1); -lean_inc(x_262); -lean_dec(x_195); -x_49 = x_261; -x_50 = x_262; +x_318 = lean_ctor_get(x_252, 0); +lean_inc(x_318); +x_319 = lean_ctor_get(x_252, 1); +lean_inc(x_319); +lean_dec(x_252); +x_49 = x_318; +x_50 = x_319; goto block_70; } } else { -lean_object* x_263; lean_object* x_264; +lean_object* x_320; lean_object* x_321; lean_dec(x_101); lean_free_object(x_85); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_3); -x_263 = lean_ctor_get(x_192, 0); -lean_inc(x_263); -x_264 = lean_ctor_get(x_192, 1); -lean_inc(x_264); -lean_dec(x_192); -x_49 = x_263; -x_50 = x_264; +x_320 = lean_ctor_get(x_249, 0); +lean_inc(x_320); +x_321 = lean_ctor_get(x_249, 1); +lean_inc(x_321); +lean_dec(x_249); +x_49 = x_320; +x_50 = x_321; goto block_70; } } } else { -lean_object* x_265; lean_object* x_266; +lean_object* x_322; lean_object* x_323; lean_dec(x_96); lean_free_object(x_85); lean_dec(x_84); @@ -19623,73 +19961,73 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_265 = lean_ctor_get(x_100, 0); -lean_inc(x_265); -x_266 = lean_ctor_get(x_100, 1); -lean_inc(x_266); +x_322 = lean_ctor_get(x_100, 0); +lean_inc(x_322); +x_323 = lean_ctor_get(x_100, 1); +lean_inc(x_323); lean_dec(x_100); -x_49 = x_265; -x_50 = x_266; +x_49 = x_322; +x_50 = x_323; goto block_70; } } else { -lean_object* x_267; lean_object* x_268; lean_object* x_269; uint8_t x_270; uint8_t x_271; uint8_t x_272; lean_object* x_273; -x_267 = lean_ctor_get(x_85, 0); -lean_inc(x_267); +lean_object* x_324; lean_object* x_325; lean_object* x_326; uint8_t x_327; uint8_t x_328; uint8_t x_329; lean_object* x_330; +x_324 = lean_ctor_get(x_85, 0); +lean_inc(x_324); lean_dec(x_85); -x_268 = l_Lean_Meta_Simp_simp_simpLet___lambda__1___closed__1; +x_325 = l_Lean_Meta_Simp_simp_simpLet___lambda__1___closed__1; lean_inc(x_5); -x_269 = lean_array_push(x_268, x_5); -x_270 = 0; -x_271 = 1; -x_272 = 1; -lean_inc(x_269); -x_273 = l_Lean_Meta_mkLambdaFVars(x_269, x_267, x_270, x_271, x_272, x_9, x_10, x_11, x_12, x_92); -if (lean_obj_tag(x_273) == 0) +x_326 = lean_array_push(x_325, x_5); +x_327 = 0; +x_328 = 1; +x_329 = 1; +lean_inc(x_326); +x_330 = l_Lean_Meta_mkLambdaFVars(x_326, x_324, x_327, x_328, x_329, x_9, x_10, x_11, x_12, x_92); +if (lean_obj_tag(x_330) == 0) { -lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; uint8_t x_278; -x_274 = lean_ctor_get(x_273, 0); -lean_inc(x_274); -x_275 = lean_ctor_get(x_273, 1); -lean_inc(x_275); -lean_dec(x_273); -x_276 = lean_ctor_get(x_84, 0); -lean_inc(x_276); +lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; uint8_t x_335; +x_331 = lean_ctor_get(x_330, 0); +lean_inc(x_331); +x_332 = lean_ctor_get(x_330, 1); +lean_inc(x_332); +lean_dec(x_330); +x_333 = lean_ctor_get(x_84, 0); +lean_inc(x_333); lean_dec(x_84); -x_277 = l_Lean_Expr_fvarId_x21(x_5); -x_278 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_277, x_276); -lean_dec(x_277); -if (x_278 == 0) +x_334 = l_Lean_Expr_fvarId_x21(x_5); +x_335 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_334, x_333); +lean_dec(x_334); +if (x_335 == 0) { -lean_object* x_279; -lean_dec(x_269); +lean_object* x_336; +lean_dec(x_326); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_279 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_275); -if (lean_obj_tag(x_279) == 0) -{ -lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; uint8_t x_289; uint8_t x_290; uint8_t x_291; uint8_t x_292; uint8_t x_293; uint8_t x_294; uint8_t x_295; uint8_t x_296; uint8_t x_297; uint8_t x_298; uint8_t x_299; uint8_t x_300; uint8_t x_301; lean_object* x_302; uint8_t x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; -x_280 = lean_ctor_get(x_9, 0); -lean_inc(x_280); -x_281 = lean_ctor_get(x_279, 0); -lean_inc(x_281); -x_282 = lean_ctor_get(x_279, 1); -lean_inc(x_282); -lean_dec(x_279); -x_283 = lean_ctor_get(x_9, 1); -lean_inc(x_283); -x_284 = lean_ctor_get(x_9, 2); -lean_inc(x_284); -x_285 = lean_ctor_get(x_9, 3); -lean_inc(x_285); -x_286 = lean_ctor_get(x_9, 4); -lean_inc(x_286); -x_287 = lean_ctor_get(x_9, 5); -lean_inc(x_287); +x_336 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_332); +if (lean_obj_tag(x_336) == 0) +{ +lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; uint8_t x_346; uint8_t x_347; uint8_t x_348; uint8_t x_349; uint8_t x_350; uint8_t x_351; uint8_t x_352; uint8_t x_353; uint8_t x_354; uint8_t x_355; uint8_t x_356; uint8_t x_357; uint8_t x_358; lean_object* x_359; uint8_t x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; +x_337 = lean_ctor_get(x_9, 0); +lean_inc(x_337); +x_338 = lean_ctor_get(x_336, 0); +lean_inc(x_338); +x_339 = lean_ctor_get(x_336, 1); +lean_inc(x_339); +lean_dec(x_336); +x_340 = lean_ctor_get(x_9, 1); +lean_inc(x_340); +x_341 = lean_ctor_get(x_9, 2); +lean_inc(x_341); +x_342 = lean_ctor_get(x_9, 3); +lean_inc(x_342); +x_343 = lean_ctor_get(x_9, 4); +lean_inc(x_343); +x_344 = lean_ctor_get(x_9, 5); +lean_inc(x_344); if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 0); lean_ctor_release(x_9, 1); @@ -19697,180 +20035,257 @@ if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 3); lean_ctor_release(x_9, 4); lean_ctor_release(x_9, 5); - x_288 = x_9; + x_345 = x_9; } else { lean_dec_ref(x_9); - x_288 = lean_box(0); -} -x_289 = lean_ctor_get_uint8(x_280, 0); -x_290 = lean_ctor_get_uint8(x_280, 1); -x_291 = lean_ctor_get_uint8(x_280, 2); -x_292 = lean_ctor_get_uint8(x_280, 3); -x_293 = lean_ctor_get_uint8(x_280, 4); -x_294 = lean_ctor_get_uint8(x_280, 6); -x_295 = lean_ctor_get_uint8(x_280, 7); -x_296 = lean_ctor_get_uint8(x_280, 8); -x_297 = lean_ctor_get_uint8(x_280, 9); -x_298 = lean_ctor_get_uint8(x_280, 10); -x_299 = lean_ctor_get_uint8(x_280, 11); -x_300 = lean_ctor_get_uint8(x_280, 12); -x_301 = lean_ctor_get_uint8(x_280, 13); -if (lean_is_exclusive(x_280)) { - x_302 = x_280; -} else { - lean_dec_ref(x_280); - x_302 = lean_box(0); -} -x_303 = 1; -if (lean_is_scalar(x_302)) { - x_304 = lean_alloc_ctor(0, 0, 14); -} else { - x_304 = x_302; -} -lean_ctor_set_uint8(x_304, 0, x_289); -lean_ctor_set_uint8(x_304, 1, x_290); -lean_ctor_set_uint8(x_304, 2, x_291); -lean_ctor_set_uint8(x_304, 3, x_292); -lean_ctor_set_uint8(x_304, 4, x_293); -lean_ctor_set_uint8(x_304, 5, x_303); -lean_ctor_set_uint8(x_304, 6, x_294); -lean_ctor_set_uint8(x_304, 7, x_295); -lean_ctor_set_uint8(x_304, 8, x_296); -lean_ctor_set_uint8(x_304, 9, x_297); -lean_ctor_set_uint8(x_304, 10, x_298); -lean_ctor_set_uint8(x_304, 11, x_299); -lean_ctor_set_uint8(x_304, 12, x_300); -lean_ctor_set_uint8(x_304, 13, x_301); -if (lean_is_scalar(x_288)) { - x_305 = lean_alloc_ctor(0, 6, 0); -} else { - x_305 = x_288; -} -lean_ctor_set(x_305, 0, x_304); -lean_ctor_set(x_305, 1, x_283); -lean_ctor_set(x_305, 2, x_284); -lean_ctor_set(x_305, 3, x_285); -lean_ctor_set(x_305, 4, x_286); -lean_ctor_set(x_305, 5, x_287); + x_345 = lean_box(0); +} +x_346 = lean_ctor_get_uint8(x_337, 0); +x_347 = lean_ctor_get_uint8(x_337, 1); +x_348 = lean_ctor_get_uint8(x_337, 2); +x_349 = lean_ctor_get_uint8(x_337, 3); +x_350 = lean_ctor_get_uint8(x_337, 4); +x_351 = lean_ctor_get_uint8(x_337, 6); +x_352 = lean_ctor_get_uint8(x_337, 7); +x_353 = lean_ctor_get_uint8(x_337, 8); +x_354 = lean_ctor_get_uint8(x_337, 9); +x_355 = lean_ctor_get_uint8(x_337, 10); +x_356 = lean_ctor_get_uint8(x_337, 11); +x_357 = lean_ctor_get_uint8(x_337, 12); +x_358 = lean_ctor_get_uint8(x_337, 13); +if (lean_is_exclusive(x_337)) { + x_359 = x_337; +} else { + lean_dec_ref(x_337); + x_359 = lean_box(0); +} +x_360 = 1; +if (lean_is_scalar(x_359)) { + x_361 = lean_alloc_ctor(0, 0, 14); +} else { + x_361 = x_359; +} +lean_ctor_set_uint8(x_361, 0, x_346); +lean_ctor_set_uint8(x_361, 1, x_347); +lean_ctor_set_uint8(x_361, 2, x_348); +lean_ctor_set_uint8(x_361, 3, x_349); +lean_ctor_set_uint8(x_361, 4, x_350); +lean_ctor_set_uint8(x_361, 5, x_360); +lean_ctor_set_uint8(x_361, 6, x_351); +lean_ctor_set_uint8(x_361, 7, x_352); +lean_ctor_set_uint8(x_361, 8, x_353); +lean_ctor_set_uint8(x_361, 9, x_354); +lean_ctor_set_uint8(x_361, 10, x_355); +lean_ctor_set_uint8(x_361, 11, x_356); +lean_ctor_set_uint8(x_361, 12, x_357); +lean_ctor_set_uint8(x_361, 13, x_358); +if (lean_is_scalar(x_345)) { + x_362 = lean_alloc_ctor(0, 6, 0); +} else { + x_362 = x_345; +} +lean_ctor_set(x_362, 0, x_361); +lean_ctor_set(x_362, 1, x_340); +lean_ctor_set(x_362, 2, x_341); +lean_ctor_set(x_362, 3, x_342); +lean_ctor_set(x_362, 4, x_343); +lean_ctor_set(x_362, 5, x_344); lean_inc(x_12); -x_306 = l_Lean_Meta_mkImpCongrCtx(x_281, x_274, x_305, x_10, x_11, x_12, x_282); -if (lean_obj_tag(x_306) == 0) -{ -lean_object* x_307; lean_object* x_308; lean_object* x_309; -x_307 = lean_ctor_get(x_306, 0); -lean_inc(x_307); -x_308 = lean_ctor_get(x_306, 1); -lean_inc(x_308); -lean_dec(x_306); -x_309 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_309, 0, x_307); +x_363 = l_Lean_Meta_mkImpCongrCtx(x_338, x_331, x_362, x_10, x_11, x_12, x_339); +if (lean_obj_tag(x_363) == 0) +{ +lean_object* x_364; lean_object* x_365; lean_object* x_366; +x_364 = lean_ctor_get(x_363, 0); +lean_inc(x_364); +x_365 = lean_ctor_get(x_363, 1); +lean_inc(x_365); +lean_dec(x_363); +x_366 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_366, 0, x_364); if (lean_obj_tag(x_2) == 7) { -uint8_t x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; -x_310 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_311 = lean_expr_update_forall(x_2, x_310, x_4, x_276); -x_312 = lean_unsigned_to_nat(0u); -x_313 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_313, 0, x_311); -lean_ctor_set(x_313, 1, x_309); -lean_ctor_set(x_313, 2, x_312); -x_27 = x_313; -x_28 = x_308; +lean_object* x_367; lean_object* x_368; lean_object* x_369; uint8_t x_370; lean_object* x_371; size_t x_372; size_t x_373; uint8_t x_374; +x_367 = lean_ctor_get(x_2, 0); +lean_inc(x_367); +x_368 = lean_ctor_get(x_2, 1); +lean_inc(x_368); +x_369 = lean_ctor_get(x_2, 2); +lean_inc(x_369); +x_370 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_369); +lean_inc(x_368); +lean_inc(x_367); +x_371 = l_Lean_Expr_forallE___override(x_367, x_368, x_369, x_370); +x_372 = lean_ptr_addr(x_368); +lean_dec(x_368); +x_373 = lean_ptr_addr(x_4); +x_374 = lean_usize_dec_eq(x_372, x_373); +if (x_374 == 0) +{ +lean_object* x_375; lean_object* x_376; lean_object* x_377; +lean_dec(x_371); +lean_dec(x_369); +x_375 = l_Lean_Expr_forallE___override(x_367, x_4, x_333, x_370); +x_376 = lean_unsigned_to_nat(0u); +x_377 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_377, 0, x_375); +lean_ctor_set(x_377, 1, x_366); +lean_ctor_set(x_377, 2, x_376); +x_27 = x_377; +x_28 = x_365; goto block_48; } else { -lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; -lean_dec(x_276); -lean_dec(x_4); -lean_dec(x_2); -x_314 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; -x_315 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_314); -x_316 = lean_unsigned_to_nat(0u); -x_317 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_317, 0, x_315); -lean_ctor_set(x_317, 1, x_309); -lean_ctor_set(x_317, 2, x_316); -x_27 = x_317; -x_28 = x_308; +size_t x_378; size_t x_379; uint8_t x_380; +x_378 = lean_ptr_addr(x_369); +lean_dec(x_369); +x_379 = lean_ptr_addr(x_333); +x_380 = lean_usize_dec_eq(x_378, x_379); +if (x_380 == 0) +{ +lean_object* x_381; lean_object* x_382; lean_object* x_383; +lean_dec(x_371); +x_381 = l_Lean_Expr_forallE___override(x_367, x_4, x_333, x_370); +x_382 = lean_unsigned_to_nat(0u); +x_383 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_383, 0, x_381); +lean_ctor_set(x_383, 1, x_366); +lean_ctor_set(x_383, 2, x_382); +x_27 = x_383; +x_28 = x_365; goto block_48; } +else +{ +uint8_t x_384; +x_384 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_370, x_370); +if (x_384 == 0) +{ +lean_object* x_385; lean_object* x_386; lean_object* x_387; +lean_dec(x_371); +x_385 = l_Lean_Expr_forallE___override(x_367, x_4, x_333, x_370); +x_386 = lean_unsigned_to_nat(0u); +x_387 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_387, 0, x_385); +lean_ctor_set(x_387, 1, x_366); +lean_ctor_set(x_387, 2, x_386); +x_27 = x_387; +x_28 = x_365; +goto block_48; } else { -lean_object* x_318; lean_object* x_319; -lean_dec(x_276); +lean_object* x_388; lean_object* x_389; +lean_dec(x_367); +lean_dec(x_333); +lean_dec(x_4); +x_388 = lean_unsigned_to_nat(0u); +x_389 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_389, 0, x_371); +lean_ctor_set(x_389, 1, x_366); +lean_ctor_set(x_389, 2, x_388); +x_27 = x_389; +x_28 = x_365; +goto block_48; +} +} +} +} +else +{ +lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; +lean_dec(x_333); lean_dec(x_4); lean_dec(x_2); -x_318 = lean_ctor_get(x_306, 0); -lean_inc(x_318); -x_319 = lean_ctor_get(x_306, 1); -lean_inc(x_319); -lean_dec(x_306); -x_49 = x_318; -x_50 = x_319; +x_390 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; +x_391 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_390); +x_392 = lean_unsigned_to_nat(0u); +x_393 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_393, 0, x_391); +lean_ctor_set(x_393, 1, x_366); +lean_ctor_set(x_393, 2, x_392); +x_27 = x_393; +x_28 = x_365; +goto block_48; +} +} +else +{ +lean_object* x_394; lean_object* x_395; +lean_dec(x_333); +lean_dec(x_4); +lean_dec(x_2); +x_394 = lean_ctor_get(x_363, 0); +lean_inc(x_394); +x_395 = lean_ctor_get(x_363, 1); +lean_inc(x_395); +lean_dec(x_363); +x_49 = x_394; +x_50 = x_395; goto block_70; } } else { -lean_object* x_320; lean_object* x_321; -lean_dec(x_276); -lean_dec(x_274); +lean_object* x_396; lean_object* x_397; +lean_dec(x_333); +lean_dec(x_331); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_4); lean_dec(x_2); -x_320 = lean_ctor_get(x_279, 0); -lean_inc(x_320); -x_321 = lean_ctor_get(x_279, 1); -lean_inc(x_321); -lean_dec(x_279); -x_49 = x_320; -x_50 = x_321; +x_396 = lean_ctor_get(x_336, 0); +lean_inc(x_396); +x_397 = lean_ctor_get(x_336, 1); +lean_inc(x_397); +lean_dec(x_336); +x_49 = x_396; +x_50 = x_397; goto block_70; } } else { -lean_object* x_322; +lean_object* x_398; lean_dec(x_4); lean_dec(x_2); -x_322 = l_Lean_Meta_mkForallFVars(x_269, x_276, x_270, x_271, x_272, x_9, x_10, x_11, x_12, x_275); -if (lean_obj_tag(x_322) == 0) +x_398 = l_Lean_Meta_mkForallFVars(x_326, x_333, x_327, x_328, x_329, x_9, x_10, x_11, x_12, x_332); +if (lean_obj_tag(x_398) == 0) { -lean_object* x_323; lean_object* x_324; lean_object* x_325; -x_323 = lean_ctor_get(x_322, 0); -lean_inc(x_323); -x_324 = lean_ctor_get(x_322, 1); -lean_inc(x_324); -lean_dec(x_322); +lean_object* x_399; lean_object* x_400; lean_object* x_401; +x_399 = lean_ctor_get(x_398, 0); +lean_inc(x_399); +x_400 = lean_ctor_get(x_398, 1); +lean_inc(x_400); +lean_dec(x_398); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_325 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_324); -if (lean_obj_tag(x_325) == 0) +x_401 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_400); +if (lean_obj_tag(x_401) == 0) { -lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; uint8_t x_335; uint8_t x_336; uint8_t x_337; uint8_t x_338; uint8_t x_339; uint8_t x_340; uint8_t x_341; uint8_t x_342; uint8_t x_343; uint8_t x_344; uint8_t x_345; uint8_t x_346; uint8_t x_347; lean_object* x_348; uint8_t x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; -x_326 = lean_ctor_get(x_9, 0); -lean_inc(x_326); -x_327 = lean_ctor_get(x_325, 0); -lean_inc(x_327); -x_328 = lean_ctor_get(x_325, 1); -lean_inc(x_328); -lean_dec(x_325); -x_329 = lean_ctor_get(x_9, 1); -lean_inc(x_329); -x_330 = lean_ctor_get(x_9, 2); -lean_inc(x_330); -x_331 = lean_ctor_get(x_9, 3); -lean_inc(x_331); -x_332 = lean_ctor_get(x_9, 4); -lean_inc(x_332); -x_333 = lean_ctor_get(x_9, 5); -lean_inc(x_333); +lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; uint8_t x_411; uint8_t x_412; uint8_t x_413; uint8_t x_414; uint8_t x_415; uint8_t x_416; uint8_t x_417; uint8_t x_418; uint8_t x_419; uint8_t x_420; uint8_t x_421; uint8_t x_422; uint8_t x_423; lean_object* x_424; uint8_t x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; +x_402 = lean_ctor_get(x_9, 0); +lean_inc(x_402); +x_403 = lean_ctor_get(x_401, 0); +lean_inc(x_403); +x_404 = lean_ctor_get(x_401, 1); +lean_inc(x_404); +lean_dec(x_401); +x_405 = lean_ctor_get(x_9, 1); +lean_inc(x_405); +x_406 = lean_ctor_get(x_9, 2); +lean_inc(x_406); +x_407 = lean_ctor_get(x_9, 3); +lean_inc(x_407); +x_408 = lean_ctor_get(x_9, 4); +lean_inc(x_408); +x_409 = lean_ctor_get(x_9, 5); +lean_inc(x_409); if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 0); lean_ctor_release(x_9, 1); @@ -19878,137 +20293,137 @@ if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 3); lean_ctor_release(x_9, 4); lean_ctor_release(x_9, 5); - x_334 = x_9; + x_410 = x_9; } else { lean_dec_ref(x_9); - x_334 = lean_box(0); -} -x_335 = lean_ctor_get_uint8(x_326, 0); -x_336 = lean_ctor_get_uint8(x_326, 1); -x_337 = lean_ctor_get_uint8(x_326, 2); -x_338 = lean_ctor_get_uint8(x_326, 3); -x_339 = lean_ctor_get_uint8(x_326, 4); -x_340 = lean_ctor_get_uint8(x_326, 6); -x_341 = lean_ctor_get_uint8(x_326, 7); -x_342 = lean_ctor_get_uint8(x_326, 8); -x_343 = lean_ctor_get_uint8(x_326, 9); -x_344 = lean_ctor_get_uint8(x_326, 10); -x_345 = lean_ctor_get_uint8(x_326, 11); -x_346 = lean_ctor_get_uint8(x_326, 12); -x_347 = lean_ctor_get_uint8(x_326, 13); -if (lean_is_exclusive(x_326)) { - x_348 = x_326; -} else { - lean_dec_ref(x_326); - x_348 = lean_box(0); -} -x_349 = 1; -if (lean_is_scalar(x_348)) { - x_350 = lean_alloc_ctor(0, 0, 14); -} else { - x_350 = x_348; -} -lean_ctor_set_uint8(x_350, 0, x_335); -lean_ctor_set_uint8(x_350, 1, x_336); -lean_ctor_set_uint8(x_350, 2, x_337); -lean_ctor_set_uint8(x_350, 3, x_338); -lean_ctor_set_uint8(x_350, 4, x_339); -lean_ctor_set_uint8(x_350, 5, x_349); -lean_ctor_set_uint8(x_350, 6, x_340); -lean_ctor_set_uint8(x_350, 7, x_341); -lean_ctor_set_uint8(x_350, 8, x_342); -lean_ctor_set_uint8(x_350, 9, x_343); -lean_ctor_set_uint8(x_350, 10, x_344); -lean_ctor_set_uint8(x_350, 11, x_345); -lean_ctor_set_uint8(x_350, 12, x_346); -lean_ctor_set_uint8(x_350, 13, x_347); -if (lean_is_scalar(x_334)) { - x_351 = lean_alloc_ctor(0, 6, 0); -} else { - x_351 = x_334; -} -lean_ctor_set(x_351, 0, x_350); -lean_ctor_set(x_351, 1, x_329); -lean_ctor_set(x_351, 2, x_330); -lean_ctor_set(x_351, 3, x_331); -lean_ctor_set(x_351, 4, x_332); -lean_ctor_set(x_351, 5, x_333); + x_410 = lean_box(0); +} +x_411 = lean_ctor_get_uint8(x_402, 0); +x_412 = lean_ctor_get_uint8(x_402, 1); +x_413 = lean_ctor_get_uint8(x_402, 2); +x_414 = lean_ctor_get_uint8(x_402, 3); +x_415 = lean_ctor_get_uint8(x_402, 4); +x_416 = lean_ctor_get_uint8(x_402, 6); +x_417 = lean_ctor_get_uint8(x_402, 7); +x_418 = lean_ctor_get_uint8(x_402, 8); +x_419 = lean_ctor_get_uint8(x_402, 9); +x_420 = lean_ctor_get_uint8(x_402, 10); +x_421 = lean_ctor_get_uint8(x_402, 11); +x_422 = lean_ctor_get_uint8(x_402, 12); +x_423 = lean_ctor_get_uint8(x_402, 13); +if (lean_is_exclusive(x_402)) { + x_424 = x_402; +} else { + lean_dec_ref(x_402); + x_424 = lean_box(0); +} +x_425 = 1; +if (lean_is_scalar(x_424)) { + x_426 = lean_alloc_ctor(0, 0, 14); +} else { + x_426 = x_424; +} +lean_ctor_set_uint8(x_426, 0, x_411); +lean_ctor_set_uint8(x_426, 1, x_412); +lean_ctor_set_uint8(x_426, 2, x_413); +lean_ctor_set_uint8(x_426, 3, x_414); +lean_ctor_set_uint8(x_426, 4, x_415); +lean_ctor_set_uint8(x_426, 5, x_425); +lean_ctor_set_uint8(x_426, 6, x_416); +lean_ctor_set_uint8(x_426, 7, x_417); +lean_ctor_set_uint8(x_426, 8, x_418); +lean_ctor_set_uint8(x_426, 9, x_419); +lean_ctor_set_uint8(x_426, 10, x_420); +lean_ctor_set_uint8(x_426, 11, x_421); +lean_ctor_set_uint8(x_426, 12, x_422); +lean_ctor_set_uint8(x_426, 13, x_423); +if (lean_is_scalar(x_410)) { + x_427 = lean_alloc_ctor(0, 6, 0); +} else { + x_427 = x_410; +} +lean_ctor_set(x_427, 0, x_426); +lean_ctor_set(x_427, 1, x_405); +lean_ctor_set(x_427, 2, x_406); +lean_ctor_set(x_427, 3, x_407); +lean_ctor_set(x_427, 4, x_408); +lean_ctor_set(x_427, 5, x_409); lean_inc(x_12); -x_352 = l_Lean_Meta_mkImpDepCongrCtx(x_327, x_274, x_351, x_10, x_11, x_12, x_328); -if (lean_obj_tag(x_352) == 0) +x_428 = l_Lean_Meta_mkImpDepCongrCtx(x_403, x_331, x_427, x_10, x_11, x_12, x_404); +if (lean_obj_tag(x_428) == 0) { -lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; -x_353 = lean_ctor_get(x_352, 0); -lean_inc(x_353); -x_354 = lean_ctor_get(x_352, 1); -lean_inc(x_354); -lean_dec(x_352); -x_355 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_355, 0, x_353); -x_356 = lean_unsigned_to_nat(0u); -x_357 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_357, 0, x_323); -lean_ctor_set(x_357, 1, x_355); -lean_ctor_set(x_357, 2, x_356); -x_27 = x_357; -x_28 = x_354; +lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; +x_429 = lean_ctor_get(x_428, 0); +lean_inc(x_429); +x_430 = lean_ctor_get(x_428, 1); +lean_inc(x_430); +lean_dec(x_428); +x_431 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_431, 0, x_429); +x_432 = lean_unsigned_to_nat(0u); +x_433 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_433, 0, x_399); +lean_ctor_set(x_433, 1, x_431); +lean_ctor_set(x_433, 2, x_432); +x_27 = x_433; +x_28 = x_430; goto block_48; } else { -lean_object* x_358; lean_object* x_359; -lean_dec(x_323); -x_358 = lean_ctor_get(x_352, 0); -lean_inc(x_358); -x_359 = lean_ctor_get(x_352, 1); -lean_inc(x_359); -lean_dec(x_352); -x_49 = x_358; -x_50 = x_359; +lean_object* x_434; lean_object* x_435; +lean_dec(x_399); +x_434 = lean_ctor_get(x_428, 0); +lean_inc(x_434); +x_435 = lean_ctor_get(x_428, 1); +lean_inc(x_435); +lean_dec(x_428); +x_49 = x_434; +x_50 = x_435; goto block_70; } } else { -lean_object* x_360; lean_object* x_361; -lean_dec(x_323); -lean_dec(x_274); +lean_object* x_436; lean_object* x_437; +lean_dec(x_399); +lean_dec(x_331); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -x_360 = lean_ctor_get(x_325, 0); -lean_inc(x_360); -x_361 = lean_ctor_get(x_325, 1); -lean_inc(x_361); -lean_dec(x_325); -x_49 = x_360; -x_50 = x_361; +x_436 = lean_ctor_get(x_401, 0); +lean_inc(x_436); +x_437 = lean_ctor_get(x_401, 1); +lean_inc(x_437); +lean_dec(x_401); +x_49 = x_436; +x_50 = x_437; goto block_70; } } else { -lean_object* x_362; lean_object* x_363; -lean_dec(x_274); +lean_object* x_438; lean_object* x_439; +lean_dec(x_331); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_3); -x_362 = lean_ctor_get(x_322, 0); -lean_inc(x_362); -x_363 = lean_ctor_get(x_322, 1); -lean_inc(x_363); -lean_dec(x_322); -x_49 = x_362; -x_50 = x_363; +x_438 = lean_ctor_get(x_398, 0); +lean_inc(x_438); +x_439 = lean_ctor_get(x_398, 1); +lean_inc(x_439); +lean_dec(x_398); +x_49 = x_438; +x_50 = x_439; goto block_70; } } } else { -lean_object* x_364; lean_object* x_365; -lean_dec(x_269); +lean_object* x_440; lean_object* x_441; +lean_dec(x_326); lean_dec(x_84); lean_dec(x_11); lean_dec(x_10); @@ -20017,13 +20432,13 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_364 = lean_ctor_get(x_273, 0); -lean_inc(x_364); -x_365 = lean_ctor_get(x_273, 1); -lean_inc(x_365); -lean_dec(x_273); -x_49 = x_364; -x_50 = x_365; +x_440 = lean_ctor_get(x_330, 0); +lean_inc(x_440); +x_441 = lean_ctor_get(x_330, 1); +lean_inc(x_441); +lean_dec(x_330); +x_49 = x_440; +x_50 = x_441; goto block_70; } } @@ -20031,7 +20446,7 @@ goto block_70; } else { -lean_object* x_366; lean_object* x_367; +lean_object* x_442; lean_object* x_443; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -20039,148 +20454,148 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_366 = lean_ctor_get(x_83, 0); -lean_inc(x_366); -x_367 = lean_ctor_get(x_83, 1); -lean_inc(x_367); +x_442 = lean_ctor_get(x_83, 0); +lean_inc(x_442); +x_443 = lean_ctor_get(x_83, 1); +lean_inc(x_443); lean_dec(x_83); -x_49 = x_366; -x_50 = x_367; +x_49 = x_442; +x_50 = x_443; goto block_70; } } else { -lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; -x_368 = lean_ctor_get(x_7, 0); -x_369 = lean_ctor_get(x_7, 2); -x_370 = lean_ctor_get(x_7, 3); -x_371 = lean_ctor_get(x_7, 4); -lean_inc(x_371); -lean_inc(x_370); -lean_inc(x_369); -lean_inc(x_368); +lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; +x_444 = lean_ctor_get(x_7, 0); +x_445 = lean_ctor_get(x_7, 2); +x_446 = lean_ctor_get(x_7, 3); +x_447 = lean_ctor_get(x_7, 4); +lean_inc(x_447); +lean_inc(x_446); +lean_inc(x_445); +lean_inc(x_444); lean_dec(x_7); -x_372 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_372, 0, x_368); -lean_ctor_set(x_372, 1, x_19); -lean_ctor_set(x_372, 2, x_369); -lean_ctor_set(x_372, 3, x_370); -lean_ctor_set(x_372, 4, x_371); +x_448 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_448, 0, x_444); +lean_ctor_set(x_448, 1, x_19); +lean_ctor_set(x_448, 2, x_445); +lean_ctor_set(x_448, 3, x_446); +lean_ctor_set(x_448, 4, x_447); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_373 = l_Lean_Meta_Simp_simp(x_1, x_6, x_372, x_8, x_9, x_10, x_11, x_12, x_80); -if (lean_obj_tag(x_373) == 0) +x_449 = l_Lean_Meta_Simp_simp(x_1, x_6, x_448, x_8, x_9, x_10, x_11, x_12, x_80); +if (lean_obj_tag(x_449) == 0) { -lean_object* x_374; lean_object* x_375; -x_374 = lean_ctor_get(x_373, 0); -lean_inc(x_374); -x_375 = lean_ctor_get(x_374, 1); -lean_inc(x_375); -if (lean_obj_tag(x_375) == 0) +lean_object* x_450; lean_object* x_451; +x_450 = lean_ctor_get(x_449, 0); +lean_inc(x_450); +x_451 = lean_ctor_get(x_450, 1); +lean_inc(x_451); +if (lean_obj_tag(x_451) == 0) { -lean_object* x_376; lean_object* x_377; +lean_object* x_452; lean_object* x_453; lean_dec(x_5); lean_dec(x_4); -x_376 = lean_ctor_get(x_373, 1); -lean_inc(x_376); -lean_dec(x_373); +x_452 = lean_ctor_get(x_449, 1); +lean_inc(x_452); +lean_dec(x_449); lean_inc(x_12); -x_377 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr(x_2, x_3, x_374, x_9, x_10, x_11, x_12, x_376); -if (lean_obj_tag(x_377) == 0) +x_453 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr(x_2, x_3, x_450, x_9, x_10, x_11, x_12, x_452); +if (lean_obj_tag(x_453) == 0) { -lean_object* x_378; lean_object* x_379; -x_378 = lean_ctor_get(x_377, 0); -lean_inc(x_378); -x_379 = lean_ctor_get(x_377, 1); -lean_inc(x_379); -lean_dec(x_377); -x_27 = x_378; -x_28 = x_379; +lean_object* x_454; lean_object* x_455; +x_454 = lean_ctor_get(x_453, 0); +lean_inc(x_454); +x_455 = lean_ctor_get(x_453, 1); +lean_inc(x_455); +lean_dec(x_453); +x_27 = x_454; +x_28 = x_455; goto block_48; } else { -lean_object* x_380; lean_object* x_381; -x_380 = lean_ctor_get(x_377, 0); -lean_inc(x_380); -x_381 = lean_ctor_get(x_377, 1); -lean_inc(x_381); -lean_dec(x_377); -x_49 = x_380; -x_50 = x_381; +lean_object* x_456; lean_object* x_457; +x_456 = lean_ctor_get(x_453, 0); +lean_inc(x_456); +x_457 = lean_ctor_get(x_453, 1); +lean_inc(x_457); +lean_dec(x_453); +x_49 = x_456; +x_50 = x_457; goto block_70; } } else { -lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; uint8_t x_387; uint8_t x_388; uint8_t x_389; lean_object* x_390; -x_382 = lean_ctor_get(x_373, 1); -lean_inc(x_382); -lean_dec(x_373); -x_383 = lean_ctor_get(x_375, 0); -lean_inc(x_383); -if (lean_is_exclusive(x_375)) { - lean_ctor_release(x_375, 0); - x_384 = x_375; +lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; uint8_t x_463; uint8_t x_464; uint8_t x_465; lean_object* x_466; +x_458 = lean_ctor_get(x_449, 1); +lean_inc(x_458); +lean_dec(x_449); +x_459 = lean_ctor_get(x_451, 0); +lean_inc(x_459); +if (lean_is_exclusive(x_451)) { + lean_ctor_release(x_451, 0); + x_460 = x_451; } else { - lean_dec_ref(x_375); - x_384 = lean_box(0); + lean_dec_ref(x_451); + x_460 = lean_box(0); } -x_385 = l_Lean_Meta_Simp_simp_simpLet___lambda__1___closed__1; +x_461 = l_Lean_Meta_Simp_simp_simpLet___lambda__1___closed__1; lean_inc(x_5); -x_386 = lean_array_push(x_385, x_5); -x_387 = 0; -x_388 = 1; -x_389 = 1; -lean_inc(x_386); -x_390 = l_Lean_Meta_mkLambdaFVars(x_386, x_383, x_387, x_388, x_389, x_9, x_10, x_11, x_12, x_382); -if (lean_obj_tag(x_390) == 0) -{ -lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; uint8_t x_395; -x_391 = lean_ctor_get(x_390, 0); -lean_inc(x_391); -x_392 = lean_ctor_get(x_390, 1); -lean_inc(x_392); -lean_dec(x_390); -x_393 = lean_ctor_get(x_374, 0); -lean_inc(x_393); -lean_dec(x_374); -x_394 = l_Lean_Expr_fvarId_x21(x_5); -x_395 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_394, x_393); -lean_dec(x_394); -if (x_395 == 0) +x_462 = lean_array_push(x_461, x_5); +x_463 = 0; +x_464 = 1; +x_465 = 1; +lean_inc(x_462); +x_466 = l_Lean_Meta_mkLambdaFVars(x_462, x_459, x_463, x_464, x_465, x_9, x_10, x_11, x_12, x_458); +if (lean_obj_tag(x_466) == 0) { -lean_object* x_396; -lean_dec(x_386); +lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; uint8_t x_471; +x_467 = lean_ctor_get(x_466, 0); +lean_inc(x_467); +x_468 = lean_ctor_get(x_466, 1); +lean_inc(x_468); +lean_dec(x_466); +x_469 = lean_ctor_get(x_450, 0); +lean_inc(x_469); +lean_dec(x_450); +x_470 = l_Lean_Expr_fvarId_x21(x_5); +x_471 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_470, x_469); +lean_dec(x_470); +if (x_471 == 0) +{ +lean_object* x_472; +lean_dec(x_462); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_396 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_392); -if (lean_obj_tag(x_396) == 0) -{ -lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; uint8_t x_406; uint8_t x_407; uint8_t x_408; uint8_t x_409; uint8_t x_410; uint8_t x_411; uint8_t x_412; uint8_t x_413; uint8_t x_414; uint8_t x_415; uint8_t x_416; uint8_t x_417; uint8_t x_418; lean_object* x_419; uint8_t x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; -x_397 = lean_ctor_get(x_9, 0); -lean_inc(x_397); -x_398 = lean_ctor_get(x_396, 0); -lean_inc(x_398); -x_399 = lean_ctor_get(x_396, 1); -lean_inc(x_399); -lean_dec(x_396); -x_400 = lean_ctor_get(x_9, 1); -lean_inc(x_400); -x_401 = lean_ctor_get(x_9, 2); -lean_inc(x_401); -x_402 = lean_ctor_get(x_9, 3); -lean_inc(x_402); -x_403 = lean_ctor_get(x_9, 4); -lean_inc(x_403); -x_404 = lean_ctor_get(x_9, 5); -lean_inc(x_404); +x_472 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_468); +if (lean_obj_tag(x_472) == 0) +{ +lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; uint8_t x_482; uint8_t x_483; uint8_t x_484; uint8_t x_485; uint8_t x_486; uint8_t x_487; uint8_t x_488; uint8_t x_489; uint8_t x_490; uint8_t x_491; uint8_t x_492; uint8_t x_493; uint8_t x_494; lean_object* x_495; uint8_t x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; +x_473 = lean_ctor_get(x_9, 0); +lean_inc(x_473); +x_474 = lean_ctor_get(x_472, 0); +lean_inc(x_474); +x_475 = lean_ctor_get(x_472, 1); +lean_inc(x_475); +lean_dec(x_472); +x_476 = lean_ctor_get(x_9, 1); +lean_inc(x_476); +x_477 = lean_ctor_get(x_9, 2); +lean_inc(x_477); +x_478 = lean_ctor_get(x_9, 3); +lean_inc(x_478); +x_479 = lean_ctor_get(x_9, 4); +lean_inc(x_479); +x_480 = lean_ctor_get(x_9, 5); +lean_inc(x_480); if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 0); lean_ctor_release(x_9, 1); @@ -20188,186 +20603,263 @@ if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 3); lean_ctor_release(x_9, 4); lean_ctor_release(x_9, 5); - x_405 = x_9; + x_481 = x_9; } else { lean_dec_ref(x_9); - x_405 = lean_box(0); -} -x_406 = lean_ctor_get_uint8(x_397, 0); -x_407 = lean_ctor_get_uint8(x_397, 1); -x_408 = lean_ctor_get_uint8(x_397, 2); -x_409 = lean_ctor_get_uint8(x_397, 3); -x_410 = lean_ctor_get_uint8(x_397, 4); -x_411 = lean_ctor_get_uint8(x_397, 6); -x_412 = lean_ctor_get_uint8(x_397, 7); -x_413 = lean_ctor_get_uint8(x_397, 8); -x_414 = lean_ctor_get_uint8(x_397, 9); -x_415 = lean_ctor_get_uint8(x_397, 10); -x_416 = lean_ctor_get_uint8(x_397, 11); -x_417 = lean_ctor_get_uint8(x_397, 12); -x_418 = lean_ctor_get_uint8(x_397, 13); -if (lean_is_exclusive(x_397)) { - x_419 = x_397; -} else { - lean_dec_ref(x_397); - x_419 = lean_box(0); -} -x_420 = 1; -if (lean_is_scalar(x_419)) { - x_421 = lean_alloc_ctor(0, 0, 14); -} else { - x_421 = x_419; -} -lean_ctor_set_uint8(x_421, 0, x_406); -lean_ctor_set_uint8(x_421, 1, x_407); -lean_ctor_set_uint8(x_421, 2, x_408); -lean_ctor_set_uint8(x_421, 3, x_409); -lean_ctor_set_uint8(x_421, 4, x_410); -lean_ctor_set_uint8(x_421, 5, x_420); -lean_ctor_set_uint8(x_421, 6, x_411); -lean_ctor_set_uint8(x_421, 7, x_412); -lean_ctor_set_uint8(x_421, 8, x_413); -lean_ctor_set_uint8(x_421, 9, x_414); -lean_ctor_set_uint8(x_421, 10, x_415); -lean_ctor_set_uint8(x_421, 11, x_416); -lean_ctor_set_uint8(x_421, 12, x_417); -lean_ctor_set_uint8(x_421, 13, x_418); -if (lean_is_scalar(x_405)) { - x_422 = lean_alloc_ctor(0, 6, 0); -} else { - x_422 = x_405; -} -lean_ctor_set(x_422, 0, x_421); -lean_ctor_set(x_422, 1, x_400); -lean_ctor_set(x_422, 2, x_401); -lean_ctor_set(x_422, 3, x_402); -lean_ctor_set(x_422, 4, x_403); -lean_ctor_set(x_422, 5, x_404); + x_481 = lean_box(0); +} +x_482 = lean_ctor_get_uint8(x_473, 0); +x_483 = lean_ctor_get_uint8(x_473, 1); +x_484 = lean_ctor_get_uint8(x_473, 2); +x_485 = lean_ctor_get_uint8(x_473, 3); +x_486 = lean_ctor_get_uint8(x_473, 4); +x_487 = lean_ctor_get_uint8(x_473, 6); +x_488 = lean_ctor_get_uint8(x_473, 7); +x_489 = lean_ctor_get_uint8(x_473, 8); +x_490 = lean_ctor_get_uint8(x_473, 9); +x_491 = lean_ctor_get_uint8(x_473, 10); +x_492 = lean_ctor_get_uint8(x_473, 11); +x_493 = lean_ctor_get_uint8(x_473, 12); +x_494 = lean_ctor_get_uint8(x_473, 13); +if (lean_is_exclusive(x_473)) { + x_495 = x_473; +} else { + lean_dec_ref(x_473); + x_495 = lean_box(0); +} +x_496 = 1; +if (lean_is_scalar(x_495)) { + x_497 = lean_alloc_ctor(0, 0, 14); +} else { + x_497 = x_495; +} +lean_ctor_set_uint8(x_497, 0, x_482); +lean_ctor_set_uint8(x_497, 1, x_483); +lean_ctor_set_uint8(x_497, 2, x_484); +lean_ctor_set_uint8(x_497, 3, x_485); +lean_ctor_set_uint8(x_497, 4, x_486); +lean_ctor_set_uint8(x_497, 5, x_496); +lean_ctor_set_uint8(x_497, 6, x_487); +lean_ctor_set_uint8(x_497, 7, x_488); +lean_ctor_set_uint8(x_497, 8, x_489); +lean_ctor_set_uint8(x_497, 9, x_490); +lean_ctor_set_uint8(x_497, 10, x_491); +lean_ctor_set_uint8(x_497, 11, x_492); +lean_ctor_set_uint8(x_497, 12, x_493); +lean_ctor_set_uint8(x_497, 13, x_494); +if (lean_is_scalar(x_481)) { + x_498 = lean_alloc_ctor(0, 6, 0); +} else { + x_498 = x_481; +} +lean_ctor_set(x_498, 0, x_497); +lean_ctor_set(x_498, 1, x_476); +lean_ctor_set(x_498, 2, x_477); +lean_ctor_set(x_498, 3, x_478); +lean_ctor_set(x_498, 4, x_479); +lean_ctor_set(x_498, 5, x_480); lean_inc(x_12); -x_423 = l_Lean_Meta_mkImpCongrCtx(x_398, x_391, x_422, x_10, x_11, x_12, x_399); -if (lean_obj_tag(x_423) == 0) -{ -lean_object* x_424; lean_object* x_425; lean_object* x_426; -x_424 = lean_ctor_get(x_423, 0); -lean_inc(x_424); -x_425 = lean_ctor_get(x_423, 1); -lean_inc(x_425); -lean_dec(x_423); -if (lean_is_scalar(x_384)) { - x_426 = lean_alloc_ctor(1, 1, 0); +x_499 = l_Lean_Meta_mkImpCongrCtx(x_474, x_467, x_498, x_10, x_11, x_12, x_475); +if (lean_obj_tag(x_499) == 0) +{ +lean_object* x_500; lean_object* x_501; lean_object* x_502; +x_500 = lean_ctor_get(x_499, 0); +lean_inc(x_500); +x_501 = lean_ctor_get(x_499, 1); +lean_inc(x_501); +lean_dec(x_499); +if (lean_is_scalar(x_460)) { + x_502 = lean_alloc_ctor(1, 1, 0); } else { - x_426 = x_384; + x_502 = x_460; } -lean_ctor_set(x_426, 0, x_424); +lean_ctor_set(x_502, 0, x_500); if (lean_obj_tag(x_2) == 7) { -uint8_t x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; -x_427 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_428 = lean_expr_update_forall(x_2, x_427, x_4, x_393); -x_429 = lean_unsigned_to_nat(0u); -x_430 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_430, 0, x_428); -lean_ctor_set(x_430, 1, x_426); -lean_ctor_set(x_430, 2, x_429); -x_27 = x_430; -x_28 = x_425; +lean_object* x_503; lean_object* x_504; lean_object* x_505; uint8_t x_506; lean_object* x_507; size_t x_508; size_t x_509; uint8_t x_510; +x_503 = lean_ctor_get(x_2, 0); +lean_inc(x_503); +x_504 = lean_ctor_get(x_2, 1); +lean_inc(x_504); +x_505 = lean_ctor_get(x_2, 2); +lean_inc(x_505); +x_506 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_505); +lean_inc(x_504); +lean_inc(x_503); +x_507 = l_Lean_Expr_forallE___override(x_503, x_504, x_505, x_506); +x_508 = lean_ptr_addr(x_504); +lean_dec(x_504); +x_509 = lean_ptr_addr(x_4); +x_510 = lean_usize_dec_eq(x_508, x_509); +if (x_510 == 0) +{ +lean_object* x_511; lean_object* x_512; lean_object* x_513; +lean_dec(x_507); +lean_dec(x_505); +x_511 = l_Lean_Expr_forallE___override(x_503, x_4, x_469, x_506); +x_512 = lean_unsigned_to_nat(0u); +x_513 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_513, 0, x_511); +lean_ctor_set(x_513, 1, x_502); +lean_ctor_set(x_513, 2, x_512); +x_27 = x_513; +x_28 = x_501; +goto block_48; +} +else +{ +size_t x_514; size_t x_515; uint8_t x_516; +x_514 = lean_ptr_addr(x_505); +lean_dec(x_505); +x_515 = lean_ptr_addr(x_469); +x_516 = lean_usize_dec_eq(x_514, x_515); +if (x_516 == 0) +{ +lean_object* x_517; lean_object* x_518; lean_object* x_519; +lean_dec(x_507); +x_517 = l_Lean_Expr_forallE___override(x_503, x_4, x_469, x_506); +x_518 = lean_unsigned_to_nat(0u); +x_519 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_519, 0, x_517); +lean_ctor_set(x_519, 1, x_502); +lean_ctor_set(x_519, 2, x_518); +x_27 = x_519; +x_28 = x_501; goto block_48; } else { -lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; -lean_dec(x_393); +uint8_t x_520; +x_520 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_506, x_506); +if (x_520 == 0) +{ +lean_object* x_521; lean_object* x_522; lean_object* x_523; +lean_dec(x_507); +x_521 = l_Lean_Expr_forallE___override(x_503, x_4, x_469, x_506); +x_522 = lean_unsigned_to_nat(0u); +x_523 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_523, 0, x_521); +lean_ctor_set(x_523, 1, x_502); +lean_ctor_set(x_523, 2, x_522); +x_27 = x_523; +x_28 = x_501; +goto block_48; +} +else +{ +lean_object* x_524; lean_object* x_525; +lean_dec(x_503); +lean_dec(x_469); +lean_dec(x_4); +x_524 = lean_unsigned_to_nat(0u); +x_525 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_525, 0, x_507); +lean_ctor_set(x_525, 1, x_502); +lean_ctor_set(x_525, 2, x_524); +x_27 = x_525; +x_28 = x_501; +goto block_48; +} +} +} +} +else +{ +lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; +lean_dec(x_469); lean_dec(x_4); lean_dec(x_2); -x_431 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; -x_432 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_431); -x_433 = lean_unsigned_to_nat(0u); -x_434 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_434, 0, x_432); -lean_ctor_set(x_434, 1, x_426); -lean_ctor_set(x_434, 2, x_433); -x_27 = x_434; -x_28 = x_425; +x_526 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; +x_527 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_526); +x_528 = lean_unsigned_to_nat(0u); +x_529 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_529, 0, x_527); +lean_ctor_set(x_529, 1, x_502); +lean_ctor_set(x_529, 2, x_528); +x_27 = x_529; +x_28 = x_501; goto block_48; } } else { -lean_object* x_435; lean_object* x_436; -lean_dec(x_393); -lean_dec(x_384); +lean_object* x_530; lean_object* x_531; +lean_dec(x_469); +lean_dec(x_460); lean_dec(x_4); lean_dec(x_2); -x_435 = lean_ctor_get(x_423, 0); -lean_inc(x_435); -x_436 = lean_ctor_get(x_423, 1); -lean_inc(x_436); -lean_dec(x_423); -x_49 = x_435; -x_50 = x_436; +x_530 = lean_ctor_get(x_499, 0); +lean_inc(x_530); +x_531 = lean_ctor_get(x_499, 1); +lean_inc(x_531); +lean_dec(x_499); +x_49 = x_530; +x_50 = x_531; goto block_70; } } else { -lean_object* x_437; lean_object* x_438; -lean_dec(x_393); -lean_dec(x_391); -lean_dec(x_384); +lean_object* x_532; lean_object* x_533; +lean_dec(x_469); +lean_dec(x_467); +lean_dec(x_460); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_4); lean_dec(x_2); -x_437 = lean_ctor_get(x_396, 0); -lean_inc(x_437); -x_438 = lean_ctor_get(x_396, 1); -lean_inc(x_438); -lean_dec(x_396); -x_49 = x_437; -x_50 = x_438; +x_532 = lean_ctor_get(x_472, 0); +lean_inc(x_532); +x_533 = lean_ctor_get(x_472, 1); +lean_inc(x_533); +lean_dec(x_472); +x_49 = x_532; +x_50 = x_533; goto block_70; } } else { -lean_object* x_439; +lean_object* x_534; lean_dec(x_4); lean_dec(x_2); -x_439 = l_Lean_Meta_mkForallFVars(x_386, x_393, x_387, x_388, x_389, x_9, x_10, x_11, x_12, x_392); -if (lean_obj_tag(x_439) == 0) +x_534 = l_Lean_Meta_mkForallFVars(x_462, x_469, x_463, x_464, x_465, x_9, x_10, x_11, x_12, x_468); +if (lean_obj_tag(x_534) == 0) { -lean_object* x_440; lean_object* x_441; lean_object* x_442; -x_440 = lean_ctor_get(x_439, 0); -lean_inc(x_440); -x_441 = lean_ctor_get(x_439, 1); -lean_inc(x_441); -lean_dec(x_439); +lean_object* x_535; lean_object* x_536; lean_object* x_537; +x_535 = lean_ctor_get(x_534, 0); +lean_inc(x_535); +x_536 = lean_ctor_get(x_534, 1); +lean_inc(x_536); +lean_dec(x_534); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_442 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_441); -if (lean_obj_tag(x_442) == 0) -{ -lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; uint8_t x_452; uint8_t x_453; uint8_t x_454; uint8_t x_455; uint8_t x_456; uint8_t x_457; uint8_t x_458; uint8_t x_459; uint8_t x_460; uint8_t x_461; uint8_t x_462; uint8_t x_463; uint8_t x_464; lean_object* x_465; uint8_t x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; -x_443 = lean_ctor_get(x_9, 0); -lean_inc(x_443); -x_444 = lean_ctor_get(x_442, 0); -lean_inc(x_444); -x_445 = lean_ctor_get(x_442, 1); -lean_inc(x_445); -lean_dec(x_442); -x_446 = lean_ctor_get(x_9, 1); -lean_inc(x_446); -x_447 = lean_ctor_get(x_9, 2); -lean_inc(x_447); -x_448 = lean_ctor_get(x_9, 3); -lean_inc(x_448); -x_449 = lean_ctor_get(x_9, 4); -lean_inc(x_449); -x_450 = lean_ctor_get(x_9, 5); -lean_inc(x_450); +x_537 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_536); +if (lean_obj_tag(x_537) == 0) +{ +lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; uint8_t x_547; uint8_t x_548; uint8_t x_549; uint8_t x_550; uint8_t x_551; uint8_t x_552; uint8_t x_553; uint8_t x_554; uint8_t x_555; uint8_t x_556; uint8_t x_557; uint8_t x_558; uint8_t x_559; lean_object* x_560; uint8_t x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; +x_538 = lean_ctor_get(x_9, 0); +lean_inc(x_538); +x_539 = lean_ctor_get(x_537, 0); +lean_inc(x_539); +x_540 = lean_ctor_get(x_537, 1); +lean_inc(x_540); +lean_dec(x_537); +x_541 = lean_ctor_get(x_9, 1); +lean_inc(x_541); +x_542 = lean_ctor_get(x_9, 2); +lean_inc(x_542); +x_543 = lean_ctor_get(x_9, 3); +lean_inc(x_543); +x_544 = lean_ctor_get(x_9, 4); +lean_inc(x_544); +x_545 = lean_ctor_get(x_9, 5); +lean_inc(x_545); if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 0); lean_ctor_release(x_9, 1); @@ -20375,146 +20867,146 @@ if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 3); lean_ctor_release(x_9, 4); lean_ctor_release(x_9, 5); - x_451 = x_9; + x_546 = x_9; } else { lean_dec_ref(x_9); - x_451 = lean_box(0); -} -x_452 = lean_ctor_get_uint8(x_443, 0); -x_453 = lean_ctor_get_uint8(x_443, 1); -x_454 = lean_ctor_get_uint8(x_443, 2); -x_455 = lean_ctor_get_uint8(x_443, 3); -x_456 = lean_ctor_get_uint8(x_443, 4); -x_457 = lean_ctor_get_uint8(x_443, 6); -x_458 = lean_ctor_get_uint8(x_443, 7); -x_459 = lean_ctor_get_uint8(x_443, 8); -x_460 = lean_ctor_get_uint8(x_443, 9); -x_461 = lean_ctor_get_uint8(x_443, 10); -x_462 = lean_ctor_get_uint8(x_443, 11); -x_463 = lean_ctor_get_uint8(x_443, 12); -x_464 = lean_ctor_get_uint8(x_443, 13); -if (lean_is_exclusive(x_443)) { - x_465 = x_443; -} else { - lean_dec_ref(x_443); - x_465 = lean_box(0); -} -x_466 = 1; -if (lean_is_scalar(x_465)) { - x_467 = lean_alloc_ctor(0, 0, 14); -} else { - x_467 = x_465; -} -lean_ctor_set_uint8(x_467, 0, x_452); -lean_ctor_set_uint8(x_467, 1, x_453); -lean_ctor_set_uint8(x_467, 2, x_454); -lean_ctor_set_uint8(x_467, 3, x_455); -lean_ctor_set_uint8(x_467, 4, x_456); -lean_ctor_set_uint8(x_467, 5, x_466); -lean_ctor_set_uint8(x_467, 6, x_457); -lean_ctor_set_uint8(x_467, 7, x_458); -lean_ctor_set_uint8(x_467, 8, x_459); -lean_ctor_set_uint8(x_467, 9, x_460); -lean_ctor_set_uint8(x_467, 10, x_461); -lean_ctor_set_uint8(x_467, 11, x_462); -lean_ctor_set_uint8(x_467, 12, x_463); -lean_ctor_set_uint8(x_467, 13, x_464); -if (lean_is_scalar(x_451)) { - x_468 = lean_alloc_ctor(0, 6, 0); -} else { - x_468 = x_451; -} -lean_ctor_set(x_468, 0, x_467); -lean_ctor_set(x_468, 1, x_446); -lean_ctor_set(x_468, 2, x_447); -lean_ctor_set(x_468, 3, x_448); -lean_ctor_set(x_468, 4, x_449); -lean_ctor_set(x_468, 5, x_450); + x_546 = lean_box(0); +} +x_547 = lean_ctor_get_uint8(x_538, 0); +x_548 = lean_ctor_get_uint8(x_538, 1); +x_549 = lean_ctor_get_uint8(x_538, 2); +x_550 = lean_ctor_get_uint8(x_538, 3); +x_551 = lean_ctor_get_uint8(x_538, 4); +x_552 = lean_ctor_get_uint8(x_538, 6); +x_553 = lean_ctor_get_uint8(x_538, 7); +x_554 = lean_ctor_get_uint8(x_538, 8); +x_555 = lean_ctor_get_uint8(x_538, 9); +x_556 = lean_ctor_get_uint8(x_538, 10); +x_557 = lean_ctor_get_uint8(x_538, 11); +x_558 = lean_ctor_get_uint8(x_538, 12); +x_559 = lean_ctor_get_uint8(x_538, 13); +if (lean_is_exclusive(x_538)) { + x_560 = x_538; +} else { + lean_dec_ref(x_538); + x_560 = lean_box(0); +} +x_561 = 1; +if (lean_is_scalar(x_560)) { + x_562 = lean_alloc_ctor(0, 0, 14); +} else { + x_562 = x_560; +} +lean_ctor_set_uint8(x_562, 0, x_547); +lean_ctor_set_uint8(x_562, 1, x_548); +lean_ctor_set_uint8(x_562, 2, x_549); +lean_ctor_set_uint8(x_562, 3, x_550); +lean_ctor_set_uint8(x_562, 4, x_551); +lean_ctor_set_uint8(x_562, 5, x_561); +lean_ctor_set_uint8(x_562, 6, x_552); +lean_ctor_set_uint8(x_562, 7, x_553); +lean_ctor_set_uint8(x_562, 8, x_554); +lean_ctor_set_uint8(x_562, 9, x_555); +lean_ctor_set_uint8(x_562, 10, x_556); +lean_ctor_set_uint8(x_562, 11, x_557); +lean_ctor_set_uint8(x_562, 12, x_558); +lean_ctor_set_uint8(x_562, 13, x_559); +if (lean_is_scalar(x_546)) { + x_563 = lean_alloc_ctor(0, 6, 0); +} else { + x_563 = x_546; +} +lean_ctor_set(x_563, 0, x_562); +lean_ctor_set(x_563, 1, x_541); +lean_ctor_set(x_563, 2, x_542); +lean_ctor_set(x_563, 3, x_543); +lean_ctor_set(x_563, 4, x_544); +lean_ctor_set(x_563, 5, x_545); lean_inc(x_12); -x_469 = l_Lean_Meta_mkImpDepCongrCtx(x_444, x_391, x_468, x_10, x_11, x_12, x_445); -if (lean_obj_tag(x_469) == 0) +x_564 = l_Lean_Meta_mkImpDepCongrCtx(x_539, x_467, x_563, x_10, x_11, x_12, x_540); +if (lean_obj_tag(x_564) == 0) { -lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; -x_470 = lean_ctor_get(x_469, 0); -lean_inc(x_470); -x_471 = lean_ctor_get(x_469, 1); -lean_inc(x_471); -lean_dec(x_469); -if (lean_is_scalar(x_384)) { - x_472 = lean_alloc_ctor(1, 1, 0); -} else { - x_472 = x_384; -} -lean_ctor_set(x_472, 0, x_470); -x_473 = lean_unsigned_to_nat(0u); -x_474 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_474, 0, x_440); -lean_ctor_set(x_474, 1, x_472); -lean_ctor_set(x_474, 2, x_473); -x_27 = x_474; -x_28 = x_471; +lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; +x_565 = lean_ctor_get(x_564, 0); +lean_inc(x_565); +x_566 = lean_ctor_get(x_564, 1); +lean_inc(x_566); +lean_dec(x_564); +if (lean_is_scalar(x_460)) { + x_567 = lean_alloc_ctor(1, 1, 0); +} else { + x_567 = x_460; +} +lean_ctor_set(x_567, 0, x_565); +x_568 = lean_unsigned_to_nat(0u); +x_569 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_569, 0, x_535); +lean_ctor_set(x_569, 1, x_567); +lean_ctor_set(x_569, 2, x_568); +x_27 = x_569; +x_28 = x_566; goto block_48; } else { -lean_object* x_475; lean_object* x_476; -lean_dec(x_440); -lean_dec(x_384); -x_475 = lean_ctor_get(x_469, 0); -lean_inc(x_475); -x_476 = lean_ctor_get(x_469, 1); -lean_inc(x_476); -lean_dec(x_469); -x_49 = x_475; -x_50 = x_476; +lean_object* x_570; lean_object* x_571; +lean_dec(x_535); +lean_dec(x_460); +x_570 = lean_ctor_get(x_564, 0); +lean_inc(x_570); +x_571 = lean_ctor_get(x_564, 1); +lean_inc(x_571); +lean_dec(x_564); +x_49 = x_570; +x_50 = x_571; goto block_70; } } else { -lean_object* x_477; lean_object* x_478; -lean_dec(x_440); -lean_dec(x_391); -lean_dec(x_384); +lean_object* x_572; lean_object* x_573; +lean_dec(x_535); +lean_dec(x_467); +lean_dec(x_460); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -x_477 = lean_ctor_get(x_442, 0); -lean_inc(x_477); -x_478 = lean_ctor_get(x_442, 1); -lean_inc(x_478); -lean_dec(x_442); -x_49 = x_477; -x_50 = x_478; +x_572 = lean_ctor_get(x_537, 0); +lean_inc(x_572); +x_573 = lean_ctor_get(x_537, 1); +lean_inc(x_573); +lean_dec(x_537); +x_49 = x_572; +x_50 = x_573; goto block_70; } } else { -lean_object* x_479; lean_object* x_480; -lean_dec(x_391); -lean_dec(x_384); +lean_object* x_574; lean_object* x_575; +lean_dec(x_467); +lean_dec(x_460); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_3); -x_479 = lean_ctor_get(x_439, 0); -lean_inc(x_479); -x_480 = lean_ctor_get(x_439, 1); -lean_inc(x_480); -lean_dec(x_439); -x_49 = x_479; -x_50 = x_480; +x_574 = lean_ctor_get(x_534, 0); +lean_inc(x_574); +x_575 = lean_ctor_get(x_534, 1); +lean_inc(x_575); +lean_dec(x_534); +x_49 = x_574; +x_50 = x_575; goto block_70; } } } else { -lean_object* x_481; lean_object* x_482; -lean_dec(x_386); -lean_dec(x_384); -lean_dec(x_374); +lean_object* x_576; lean_object* x_577; +lean_dec(x_462); +lean_dec(x_460); +lean_dec(x_450); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -20522,20 +21014,20 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_481 = lean_ctor_get(x_390, 0); -lean_inc(x_481); -x_482 = lean_ctor_get(x_390, 1); -lean_inc(x_482); -lean_dec(x_390); -x_49 = x_481; -x_50 = x_482; +x_576 = lean_ctor_get(x_466, 0); +lean_inc(x_576); +x_577 = lean_ctor_get(x_466, 1); +lean_inc(x_577); +lean_dec(x_466); +x_49 = x_576; +x_50 = x_577; goto block_70; } } } else { -lean_object* x_483; lean_object* x_484; +lean_object* x_578; lean_object* x_579; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -20543,177 +21035,177 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_483 = lean_ctor_get(x_373, 0); -lean_inc(x_483); -x_484 = lean_ctor_get(x_373, 1); -lean_inc(x_484); -lean_dec(x_373); -x_49 = x_483; -x_50 = x_484; +x_578 = lean_ctor_get(x_449, 0); +lean_inc(x_578); +x_579 = lean_ctor_get(x_449, 1); +lean_inc(x_579); +lean_dec(x_449); +x_49 = x_578; +x_50 = x_579; goto block_70; } } } else { -lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; -x_485 = lean_ctor_get(x_74, 1); -x_486 = lean_ctor_get(x_74, 2); -lean_inc(x_486); -lean_inc(x_485); +lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; lean_object* x_592; +x_580 = lean_ctor_get(x_74, 1); +x_581 = lean_ctor_get(x_74, 2); +lean_inc(x_581); +lean_inc(x_580); lean_dec(x_74); -x_487 = l_Lean_Meta_transform___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__1___closed__1; -x_488 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_488, 0, x_487); -lean_ctor_set(x_488, 1, x_485); -lean_ctor_set(x_488, 2, x_486); -x_489 = lean_st_ref_set(x_8, x_488, x_75); -x_490 = lean_ctor_get(x_489, 1); -lean_inc(x_490); -lean_dec(x_489); -x_491 = lean_ctor_get(x_7, 0); -lean_inc(x_491); -x_492 = lean_ctor_get(x_7, 2); -lean_inc(x_492); -x_493 = lean_ctor_get(x_7, 3); -lean_inc(x_493); -x_494 = lean_ctor_get(x_7, 4); -lean_inc(x_494); +x_582 = l_Lean_Meta_transform___at___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_dsimp___spec__1___closed__1; +x_583 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_583, 0, x_582); +lean_ctor_set(x_583, 1, x_580); +lean_ctor_set(x_583, 2, x_581); +x_584 = lean_st_ref_set(x_8, x_583, x_75); +x_585 = lean_ctor_get(x_584, 1); +lean_inc(x_585); +lean_dec(x_584); +x_586 = lean_ctor_get(x_7, 0); +lean_inc(x_586); +x_587 = lean_ctor_get(x_7, 2); +lean_inc(x_587); +x_588 = lean_ctor_get(x_7, 3); +lean_inc(x_588); +x_589 = lean_ctor_get(x_7, 4); +lean_inc(x_589); if (lean_is_exclusive(x_7)) { lean_ctor_release(x_7, 0); lean_ctor_release(x_7, 1); lean_ctor_release(x_7, 2); lean_ctor_release(x_7, 3); lean_ctor_release(x_7, 4); - x_495 = x_7; + x_590 = x_7; } else { lean_dec_ref(x_7); - x_495 = lean_box(0); + x_590 = lean_box(0); } -if (lean_is_scalar(x_495)) { - x_496 = lean_alloc_ctor(0, 5, 0); +if (lean_is_scalar(x_590)) { + x_591 = lean_alloc_ctor(0, 5, 0); } else { - x_496 = x_495; + x_591 = x_590; } -lean_ctor_set(x_496, 0, x_491); -lean_ctor_set(x_496, 1, x_19); -lean_ctor_set(x_496, 2, x_492); -lean_ctor_set(x_496, 3, x_493); -lean_ctor_set(x_496, 4, x_494); +lean_ctor_set(x_591, 0, x_586); +lean_ctor_set(x_591, 1, x_19); +lean_ctor_set(x_591, 2, x_587); +lean_ctor_set(x_591, 3, x_588); +lean_ctor_set(x_591, 4, x_589); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_497 = l_Lean_Meta_Simp_simp(x_1, x_6, x_496, x_8, x_9, x_10, x_11, x_12, x_490); -if (lean_obj_tag(x_497) == 0) +x_592 = l_Lean_Meta_Simp_simp(x_1, x_6, x_591, x_8, x_9, x_10, x_11, x_12, x_585); +if (lean_obj_tag(x_592) == 0) { -lean_object* x_498; lean_object* x_499; -x_498 = lean_ctor_get(x_497, 0); -lean_inc(x_498); -x_499 = lean_ctor_get(x_498, 1); -lean_inc(x_499); -if (lean_obj_tag(x_499) == 0) +lean_object* x_593; lean_object* x_594; +x_593 = lean_ctor_get(x_592, 0); +lean_inc(x_593); +x_594 = lean_ctor_get(x_593, 1); +lean_inc(x_594); +if (lean_obj_tag(x_594) == 0) { -lean_object* x_500; lean_object* x_501; +lean_object* x_595; lean_object* x_596; lean_dec(x_5); lean_dec(x_4); -x_500 = lean_ctor_get(x_497, 1); -lean_inc(x_500); -lean_dec(x_497); +x_595 = lean_ctor_get(x_592, 1); +lean_inc(x_595); +lean_dec(x_592); lean_inc(x_12); -x_501 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr(x_2, x_3, x_498, x_9, x_10, x_11, x_12, x_500); -if (lean_obj_tag(x_501) == 0) -{ -lean_object* x_502; lean_object* x_503; -x_502 = lean_ctor_get(x_501, 0); -lean_inc(x_502); -x_503 = lean_ctor_get(x_501, 1); -lean_inc(x_503); -lean_dec(x_501); -x_27 = x_502; -x_28 = x_503; +x_596 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr(x_2, x_3, x_593, x_9, x_10, x_11, x_12, x_595); +if (lean_obj_tag(x_596) == 0) +{ +lean_object* x_597; lean_object* x_598; +x_597 = lean_ctor_get(x_596, 0); +lean_inc(x_597); +x_598 = lean_ctor_get(x_596, 1); +lean_inc(x_598); +lean_dec(x_596); +x_27 = x_597; +x_28 = x_598; goto block_48; } else { -lean_object* x_504; lean_object* x_505; -x_504 = lean_ctor_get(x_501, 0); -lean_inc(x_504); -x_505 = lean_ctor_get(x_501, 1); -lean_inc(x_505); -lean_dec(x_501); -x_49 = x_504; -x_50 = x_505; +lean_object* x_599; lean_object* x_600; +x_599 = lean_ctor_get(x_596, 0); +lean_inc(x_599); +x_600 = lean_ctor_get(x_596, 1); +lean_inc(x_600); +lean_dec(x_596); +x_49 = x_599; +x_50 = x_600; goto block_70; } } else { -lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; uint8_t x_511; uint8_t x_512; uint8_t x_513; lean_object* x_514; -x_506 = lean_ctor_get(x_497, 1); -lean_inc(x_506); -lean_dec(x_497); -x_507 = lean_ctor_get(x_499, 0); -lean_inc(x_507); -if (lean_is_exclusive(x_499)) { - lean_ctor_release(x_499, 0); - x_508 = x_499; +lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; uint8_t x_606; uint8_t x_607; uint8_t x_608; lean_object* x_609; +x_601 = lean_ctor_get(x_592, 1); +lean_inc(x_601); +lean_dec(x_592); +x_602 = lean_ctor_get(x_594, 0); +lean_inc(x_602); +if (lean_is_exclusive(x_594)) { + lean_ctor_release(x_594, 0); + x_603 = x_594; } else { - lean_dec_ref(x_499); - x_508 = lean_box(0); + lean_dec_ref(x_594); + x_603 = lean_box(0); } -x_509 = l_Lean_Meta_Simp_simp_simpLet___lambda__1___closed__1; +x_604 = l_Lean_Meta_Simp_simp_simpLet___lambda__1___closed__1; lean_inc(x_5); -x_510 = lean_array_push(x_509, x_5); -x_511 = 0; -x_512 = 1; -x_513 = 1; -lean_inc(x_510); -x_514 = l_Lean_Meta_mkLambdaFVars(x_510, x_507, x_511, x_512, x_513, x_9, x_10, x_11, x_12, x_506); -if (lean_obj_tag(x_514) == 0) +x_605 = lean_array_push(x_604, x_5); +x_606 = 0; +x_607 = 1; +x_608 = 1; +lean_inc(x_605); +x_609 = l_Lean_Meta_mkLambdaFVars(x_605, x_602, x_606, x_607, x_608, x_9, x_10, x_11, x_12, x_601); +if (lean_obj_tag(x_609) == 0) { -lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; uint8_t x_519; -x_515 = lean_ctor_get(x_514, 0); -lean_inc(x_515); -x_516 = lean_ctor_get(x_514, 1); -lean_inc(x_516); -lean_dec(x_514); -x_517 = lean_ctor_get(x_498, 0); -lean_inc(x_517); -lean_dec(x_498); -x_518 = l_Lean_Expr_fvarId_x21(x_5); -x_519 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_518, x_517); -lean_dec(x_518); -if (x_519 == 0) -{ -lean_object* x_520; -lean_dec(x_510); +lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; uint8_t x_614; +x_610 = lean_ctor_get(x_609, 0); +lean_inc(x_610); +x_611 = lean_ctor_get(x_609, 1); +lean_inc(x_611); +lean_dec(x_609); +x_612 = lean_ctor_get(x_593, 0); +lean_inc(x_612); +lean_dec(x_593); +x_613 = l_Lean_Expr_fvarId_x21(x_5); +x_614 = l_Lean_Expr_hasAnyFVar_visit___at_Lean_Expr_containsFVar___spec__1(x_613, x_612); +lean_dec(x_613); +if (x_614 == 0) +{ +lean_object* x_615; +lean_dec(x_605); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_520 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_516); -if (lean_obj_tag(x_520) == 0) +x_615 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_611); +if (lean_obj_tag(x_615) == 0) { -lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; uint8_t x_530; uint8_t x_531; uint8_t x_532; uint8_t x_533; uint8_t x_534; uint8_t x_535; uint8_t x_536; uint8_t x_537; uint8_t x_538; uint8_t x_539; uint8_t x_540; uint8_t x_541; uint8_t x_542; lean_object* x_543; uint8_t x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; -x_521 = lean_ctor_get(x_9, 0); -lean_inc(x_521); -x_522 = lean_ctor_get(x_520, 0); -lean_inc(x_522); -x_523 = lean_ctor_get(x_520, 1); -lean_inc(x_523); -lean_dec(x_520); -x_524 = lean_ctor_get(x_9, 1); -lean_inc(x_524); -x_525 = lean_ctor_get(x_9, 2); -lean_inc(x_525); -x_526 = lean_ctor_get(x_9, 3); -lean_inc(x_526); -x_527 = lean_ctor_get(x_9, 4); -lean_inc(x_527); -x_528 = lean_ctor_get(x_9, 5); -lean_inc(x_528); +lean_object* x_616; lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; uint8_t x_625; uint8_t x_626; uint8_t x_627; uint8_t x_628; uint8_t x_629; uint8_t x_630; uint8_t x_631; uint8_t x_632; uint8_t x_633; uint8_t x_634; uint8_t x_635; uint8_t x_636; uint8_t x_637; lean_object* x_638; uint8_t x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; +x_616 = lean_ctor_get(x_9, 0); +lean_inc(x_616); +x_617 = lean_ctor_get(x_615, 0); +lean_inc(x_617); +x_618 = lean_ctor_get(x_615, 1); +lean_inc(x_618); +lean_dec(x_615); +x_619 = lean_ctor_get(x_9, 1); +lean_inc(x_619); +x_620 = lean_ctor_get(x_9, 2); +lean_inc(x_620); +x_621 = lean_ctor_get(x_9, 3); +lean_inc(x_621); +x_622 = lean_ctor_get(x_9, 4); +lean_inc(x_622); +x_623 = lean_ctor_get(x_9, 5); +lean_inc(x_623); if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 0); lean_ctor_release(x_9, 1); @@ -20721,186 +21213,263 @@ if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 3); lean_ctor_release(x_9, 4); lean_ctor_release(x_9, 5); - x_529 = x_9; + x_624 = x_9; } else { lean_dec_ref(x_9); - x_529 = lean_box(0); -} -x_530 = lean_ctor_get_uint8(x_521, 0); -x_531 = lean_ctor_get_uint8(x_521, 1); -x_532 = lean_ctor_get_uint8(x_521, 2); -x_533 = lean_ctor_get_uint8(x_521, 3); -x_534 = lean_ctor_get_uint8(x_521, 4); -x_535 = lean_ctor_get_uint8(x_521, 6); -x_536 = lean_ctor_get_uint8(x_521, 7); -x_537 = lean_ctor_get_uint8(x_521, 8); -x_538 = lean_ctor_get_uint8(x_521, 9); -x_539 = lean_ctor_get_uint8(x_521, 10); -x_540 = lean_ctor_get_uint8(x_521, 11); -x_541 = lean_ctor_get_uint8(x_521, 12); -x_542 = lean_ctor_get_uint8(x_521, 13); -if (lean_is_exclusive(x_521)) { - x_543 = x_521; -} else { - lean_dec_ref(x_521); - x_543 = lean_box(0); -} -x_544 = 1; -if (lean_is_scalar(x_543)) { - x_545 = lean_alloc_ctor(0, 0, 14); -} else { - x_545 = x_543; -} -lean_ctor_set_uint8(x_545, 0, x_530); -lean_ctor_set_uint8(x_545, 1, x_531); -lean_ctor_set_uint8(x_545, 2, x_532); -lean_ctor_set_uint8(x_545, 3, x_533); -lean_ctor_set_uint8(x_545, 4, x_534); -lean_ctor_set_uint8(x_545, 5, x_544); -lean_ctor_set_uint8(x_545, 6, x_535); -lean_ctor_set_uint8(x_545, 7, x_536); -lean_ctor_set_uint8(x_545, 8, x_537); -lean_ctor_set_uint8(x_545, 9, x_538); -lean_ctor_set_uint8(x_545, 10, x_539); -lean_ctor_set_uint8(x_545, 11, x_540); -lean_ctor_set_uint8(x_545, 12, x_541); -lean_ctor_set_uint8(x_545, 13, x_542); -if (lean_is_scalar(x_529)) { - x_546 = lean_alloc_ctor(0, 6, 0); -} else { - x_546 = x_529; -} -lean_ctor_set(x_546, 0, x_545); -lean_ctor_set(x_546, 1, x_524); -lean_ctor_set(x_546, 2, x_525); -lean_ctor_set(x_546, 3, x_526); -lean_ctor_set(x_546, 4, x_527); -lean_ctor_set(x_546, 5, x_528); + x_624 = lean_box(0); +} +x_625 = lean_ctor_get_uint8(x_616, 0); +x_626 = lean_ctor_get_uint8(x_616, 1); +x_627 = lean_ctor_get_uint8(x_616, 2); +x_628 = lean_ctor_get_uint8(x_616, 3); +x_629 = lean_ctor_get_uint8(x_616, 4); +x_630 = lean_ctor_get_uint8(x_616, 6); +x_631 = lean_ctor_get_uint8(x_616, 7); +x_632 = lean_ctor_get_uint8(x_616, 8); +x_633 = lean_ctor_get_uint8(x_616, 9); +x_634 = lean_ctor_get_uint8(x_616, 10); +x_635 = lean_ctor_get_uint8(x_616, 11); +x_636 = lean_ctor_get_uint8(x_616, 12); +x_637 = lean_ctor_get_uint8(x_616, 13); +if (lean_is_exclusive(x_616)) { + x_638 = x_616; +} else { + lean_dec_ref(x_616); + x_638 = lean_box(0); +} +x_639 = 1; +if (lean_is_scalar(x_638)) { + x_640 = lean_alloc_ctor(0, 0, 14); +} else { + x_640 = x_638; +} +lean_ctor_set_uint8(x_640, 0, x_625); +lean_ctor_set_uint8(x_640, 1, x_626); +lean_ctor_set_uint8(x_640, 2, x_627); +lean_ctor_set_uint8(x_640, 3, x_628); +lean_ctor_set_uint8(x_640, 4, x_629); +lean_ctor_set_uint8(x_640, 5, x_639); +lean_ctor_set_uint8(x_640, 6, x_630); +lean_ctor_set_uint8(x_640, 7, x_631); +lean_ctor_set_uint8(x_640, 8, x_632); +lean_ctor_set_uint8(x_640, 9, x_633); +lean_ctor_set_uint8(x_640, 10, x_634); +lean_ctor_set_uint8(x_640, 11, x_635); +lean_ctor_set_uint8(x_640, 12, x_636); +lean_ctor_set_uint8(x_640, 13, x_637); +if (lean_is_scalar(x_624)) { + x_641 = lean_alloc_ctor(0, 6, 0); +} else { + x_641 = x_624; +} +lean_ctor_set(x_641, 0, x_640); +lean_ctor_set(x_641, 1, x_619); +lean_ctor_set(x_641, 2, x_620); +lean_ctor_set(x_641, 3, x_621); +lean_ctor_set(x_641, 4, x_622); +lean_ctor_set(x_641, 5, x_623); lean_inc(x_12); -x_547 = l_Lean_Meta_mkImpCongrCtx(x_522, x_515, x_546, x_10, x_11, x_12, x_523); -if (lean_obj_tag(x_547) == 0) +x_642 = l_Lean_Meta_mkImpCongrCtx(x_617, x_610, x_641, x_10, x_11, x_12, x_618); +if (lean_obj_tag(x_642) == 0) { -lean_object* x_548; lean_object* x_549; lean_object* x_550; -x_548 = lean_ctor_get(x_547, 0); -lean_inc(x_548); -x_549 = lean_ctor_get(x_547, 1); -lean_inc(x_549); -lean_dec(x_547); -if (lean_is_scalar(x_508)) { - x_550 = lean_alloc_ctor(1, 1, 0); +lean_object* x_643; lean_object* x_644; lean_object* x_645; +x_643 = lean_ctor_get(x_642, 0); +lean_inc(x_643); +x_644 = lean_ctor_get(x_642, 1); +lean_inc(x_644); +lean_dec(x_642); +if (lean_is_scalar(x_603)) { + x_645 = lean_alloc_ctor(1, 1, 0); } else { - x_550 = x_508; + x_645 = x_603; } -lean_ctor_set(x_550, 0, x_548); +lean_ctor_set(x_645, 0, x_643); if (lean_obj_tag(x_2) == 7) { -uint8_t x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; -x_551 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_552 = lean_expr_update_forall(x_2, x_551, x_4, x_517); -x_553 = lean_unsigned_to_nat(0u); -x_554 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_554, 0, x_552); -lean_ctor_set(x_554, 1, x_550); -lean_ctor_set(x_554, 2, x_553); -x_27 = x_554; -x_28 = x_549; +lean_object* x_646; lean_object* x_647; lean_object* x_648; uint8_t x_649; lean_object* x_650; size_t x_651; size_t x_652; uint8_t x_653; +x_646 = lean_ctor_get(x_2, 0); +lean_inc(x_646); +x_647 = lean_ctor_get(x_2, 1); +lean_inc(x_647); +x_648 = lean_ctor_get(x_2, 2); +lean_inc(x_648); +x_649 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_648); +lean_inc(x_647); +lean_inc(x_646); +x_650 = l_Lean_Expr_forallE___override(x_646, x_647, x_648, x_649); +x_651 = lean_ptr_addr(x_647); +lean_dec(x_647); +x_652 = lean_ptr_addr(x_4); +x_653 = lean_usize_dec_eq(x_651, x_652); +if (x_653 == 0) +{ +lean_object* x_654; lean_object* x_655; lean_object* x_656; +lean_dec(x_650); +lean_dec(x_648); +x_654 = l_Lean_Expr_forallE___override(x_646, x_4, x_612, x_649); +x_655 = lean_unsigned_to_nat(0u); +x_656 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_656, 0, x_654); +lean_ctor_set(x_656, 1, x_645); +lean_ctor_set(x_656, 2, x_655); +x_27 = x_656; +x_28 = x_644; goto block_48; } else { -lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; -lean_dec(x_517); +size_t x_657; size_t x_658; uint8_t x_659; +x_657 = lean_ptr_addr(x_648); +lean_dec(x_648); +x_658 = lean_ptr_addr(x_612); +x_659 = lean_usize_dec_eq(x_657, x_658); +if (x_659 == 0) +{ +lean_object* x_660; lean_object* x_661; lean_object* x_662; +lean_dec(x_650); +x_660 = l_Lean_Expr_forallE___override(x_646, x_4, x_612, x_649); +x_661 = lean_unsigned_to_nat(0u); +x_662 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_662, 0, x_660); +lean_ctor_set(x_662, 1, x_645); +lean_ctor_set(x_662, 2, x_661); +x_27 = x_662; +x_28 = x_644; +goto block_48; +} +else +{ +uint8_t x_663; +x_663 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_649, x_649); +if (x_663 == 0) +{ +lean_object* x_664; lean_object* x_665; lean_object* x_666; +lean_dec(x_650); +x_664 = l_Lean_Expr_forallE___override(x_646, x_4, x_612, x_649); +x_665 = lean_unsigned_to_nat(0u); +x_666 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_666, 0, x_664); +lean_ctor_set(x_666, 1, x_645); +lean_ctor_set(x_666, 2, x_665); +x_27 = x_666; +x_28 = x_644; +goto block_48; +} +else +{ +lean_object* x_667; lean_object* x_668; +lean_dec(x_646); +lean_dec(x_612); +lean_dec(x_4); +x_667 = lean_unsigned_to_nat(0u); +x_668 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_668, 0, x_650); +lean_ctor_set(x_668, 1, x_645); +lean_ctor_set(x_668, 2, x_667); +x_27 = x_668; +x_28 = x_644; +goto block_48; +} +} +} +} +else +{ +lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; +lean_dec(x_612); lean_dec(x_4); lean_dec(x_2); -x_555 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; -x_556 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_555); -x_557 = lean_unsigned_to_nat(0u); -x_558 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_558, 0, x_556); -lean_ctor_set(x_558, 1, x_550); -lean_ctor_set(x_558, 2, x_557); -x_27 = x_558; -x_28 = x_549; +x_669 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__4; +x_670 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_669); +x_671 = lean_unsigned_to_nat(0u); +x_672 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_672, 0, x_670); +lean_ctor_set(x_672, 1, x_645); +lean_ctor_set(x_672, 2, x_671); +x_27 = x_672; +x_28 = x_644; goto block_48; } } else { -lean_object* x_559; lean_object* x_560; -lean_dec(x_517); -lean_dec(x_508); +lean_object* x_673; lean_object* x_674; +lean_dec(x_612); +lean_dec(x_603); lean_dec(x_4); lean_dec(x_2); -x_559 = lean_ctor_get(x_547, 0); -lean_inc(x_559); -x_560 = lean_ctor_get(x_547, 1); -lean_inc(x_560); -lean_dec(x_547); -x_49 = x_559; -x_50 = x_560; +x_673 = lean_ctor_get(x_642, 0); +lean_inc(x_673); +x_674 = lean_ctor_get(x_642, 1); +lean_inc(x_674); +lean_dec(x_642); +x_49 = x_673; +x_50 = x_674; goto block_70; } } else { -lean_object* x_561; lean_object* x_562; -lean_dec(x_517); -lean_dec(x_515); -lean_dec(x_508); +lean_object* x_675; lean_object* x_676; +lean_dec(x_612); +lean_dec(x_610); +lean_dec(x_603); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_4); lean_dec(x_2); -x_561 = lean_ctor_get(x_520, 0); -lean_inc(x_561); -x_562 = lean_ctor_get(x_520, 1); -lean_inc(x_562); -lean_dec(x_520); -x_49 = x_561; -x_50 = x_562; +x_675 = lean_ctor_get(x_615, 0); +lean_inc(x_675); +x_676 = lean_ctor_get(x_615, 1); +lean_inc(x_676); +lean_dec(x_615); +x_49 = x_675; +x_50 = x_676; goto block_70; } } else { -lean_object* x_563; +lean_object* x_677; lean_dec(x_4); lean_dec(x_2); -x_563 = l_Lean_Meta_mkForallFVars(x_510, x_517, x_511, x_512, x_513, x_9, x_10, x_11, x_12, x_516); -if (lean_obj_tag(x_563) == 0) +x_677 = l_Lean_Meta_mkForallFVars(x_605, x_612, x_606, x_607, x_608, x_9, x_10, x_11, x_12, x_611); +if (lean_obj_tag(x_677) == 0) { -lean_object* x_564; lean_object* x_565; lean_object* x_566; -x_564 = lean_ctor_get(x_563, 0); -lean_inc(x_564); -x_565 = lean_ctor_get(x_563, 1); -lean_inc(x_565); -lean_dec(x_563); +lean_object* x_678; lean_object* x_679; lean_object* x_680; +x_678 = lean_ctor_get(x_677, 0); +lean_inc(x_678); +x_679 = lean_ctor_get(x_677, 1); +lean_inc(x_679); +lean_dec(x_677); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -x_566 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_565); -if (lean_obj_tag(x_566) == 0) -{ -lean_object* x_567; lean_object* x_568; lean_object* x_569; lean_object* x_570; lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; uint8_t x_576; uint8_t x_577; uint8_t x_578; uint8_t x_579; uint8_t x_580; uint8_t x_581; uint8_t x_582; uint8_t x_583; uint8_t x_584; uint8_t x_585; uint8_t x_586; uint8_t x_587; uint8_t x_588; lean_object* x_589; uint8_t x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; -x_567 = lean_ctor_get(x_9, 0); -lean_inc(x_567); -x_568 = lean_ctor_get(x_566, 0); -lean_inc(x_568); -x_569 = lean_ctor_get(x_566, 1); -lean_inc(x_569); -lean_dec(x_566); -x_570 = lean_ctor_get(x_9, 1); -lean_inc(x_570); -x_571 = lean_ctor_get(x_9, 2); -lean_inc(x_571); -x_572 = lean_ctor_get(x_9, 3); -lean_inc(x_572); -x_573 = lean_ctor_get(x_9, 4); -lean_inc(x_573); -x_574 = lean_ctor_get(x_9, 5); -lean_inc(x_574); +x_680 = l_Lean_Meta_Simp_Result_getProof(x_3, x_9, x_10, x_11, x_12, x_679); +if (lean_obj_tag(x_680) == 0) +{ +lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; uint8_t x_690; uint8_t x_691; uint8_t x_692; uint8_t x_693; uint8_t x_694; uint8_t x_695; uint8_t x_696; uint8_t x_697; uint8_t x_698; uint8_t x_699; uint8_t x_700; uint8_t x_701; uint8_t x_702; lean_object* x_703; uint8_t x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; +x_681 = lean_ctor_get(x_9, 0); +lean_inc(x_681); +x_682 = lean_ctor_get(x_680, 0); +lean_inc(x_682); +x_683 = lean_ctor_get(x_680, 1); +lean_inc(x_683); +lean_dec(x_680); +x_684 = lean_ctor_get(x_9, 1); +lean_inc(x_684); +x_685 = lean_ctor_get(x_9, 2); +lean_inc(x_685); +x_686 = lean_ctor_get(x_9, 3); +lean_inc(x_686); +x_687 = lean_ctor_get(x_9, 4); +lean_inc(x_687); +x_688 = lean_ctor_get(x_9, 5); +lean_inc(x_688); if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 0); lean_ctor_release(x_9, 1); @@ -20908,146 +21477,146 @@ if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 3); lean_ctor_release(x_9, 4); lean_ctor_release(x_9, 5); - x_575 = x_9; + x_689 = x_9; } else { lean_dec_ref(x_9); - x_575 = lean_box(0); -} -x_576 = lean_ctor_get_uint8(x_567, 0); -x_577 = lean_ctor_get_uint8(x_567, 1); -x_578 = lean_ctor_get_uint8(x_567, 2); -x_579 = lean_ctor_get_uint8(x_567, 3); -x_580 = lean_ctor_get_uint8(x_567, 4); -x_581 = lean_ctor_get_uint8(x_567, 6); -x_582 = lean_ctor_get_uint8(x_567, 7); -x_583 = lean_ctor_get_uint8(x_567, 8); -x_584 = lean_ctor_get_uint8(x_567, 9); -x_585 = lean_ctor_get_uint8(x_567, 10); -x_586 = lean_ctor_get_uint8(x_567, 11); -x_587 = lean_ctor_get_uint8(x_567, 12); -x_588 = lean_ctor_get_uint8(x_567, 13); -if (lean_is_exclusive(x_567)) { - x_589 = x_567; -} else { - lean_dec_ref(x_567); - x_589 = lean_box(0); -} -x_590 = 1; -if (lean_is_scalar(x_589)) { - x_591 = lean_alloc_ctor(0, 0, 14); -} else { - x_591 = x_589; -} -lean_ctor_set_uint8(x_591, 0, x_576); -lean_ctor_set_uint8(x_591, 1, x_577); -lean_ctor_set_uint8(x_591, 2, x_578); -lean_ctor_set_uint8(x_591, 3, x_579); -lean_ctor_set_uint8(x_591, 4, x_580); -lean_ctor_set_uint8(x_591, 5, x_590); -lean_ctor_set_uint8(x_591, 6, x_581); -lean_ctor_set_uint8(x_591, 7, x_582); -lean_ctor_set_uint8(x_591, 8, x_583); -lean_ctor_set_uint8(x_591, 9, x_584); -lean_ctor_set_uint8(x_591, 10, x_585); -lean_ctor_set_uint8(x_591, 11, x_586); -lean_ctor_set_uint8(x_591, 12, x_587); -lean_ctor_set_uint8(x_591, 13, x_588); -if (lean_is_scalar(x_575)) { - x_592 = lean_alloc_ctor(0, 6, 0); -} else { - x_592 = x_575; -} -lean_ctor_set(x_592, 0, x_591); -lean_ctor_set(x_592, 1, x_570); -lean_ctor_set(x_592, 2, x_571); -lean_ctor_set(x_592, 3, x_572); -lean_ctor_set(x_592, 4, x_573); -lean_ctor_set(x_592, 5, x_574); + x_689 = lean_box(0); +} +x_690 = lean_ctor_get_uint8(x_681, 0); +x_691 = lean_ctor_get_uint8(x_681, 1); +x_692 = lean_ctor_get_uint8(x_681, 2); +x_693 = lean_ctor_get_uint8(x_681, 3); +x_694 = lean_ctor_get_uint8(x_681, 4); +x_695 = lean_ctor_get_uint8(x_681, 6); +x_696 = lean_ctor_get_uint8(x_681, 7); +x_697 = lean_ctor_get_uint8(x_681, 8); +x_698 = lean_ctor_get_uint8(x_681, 9); +x_699 = lean_ctor_get_uint8(x_681, 10); +x_700 = lean_ctor_get_uint8(x_681, 11); +x_701 = lean_ctor_get_uint8(x_681, 12); +x_702 = lean_ctor_get_uint8(x_681, 13); +if (lean_is_exclusive(x_681)) { + x_703 = x_681; +} else { + lean_dec_ref(x_681); + x_703 = lean_box(0); +} +x_704 = 1; +if (lean_is_scalar(x_703)) { + x_705 = lean_alloc_ctor(0, 0, 14); +} else { + x_705 = x_703; +} +lean_ctor_set_uint8(x_705, 0, x_690); +lean_ctor_set_uint8(x_705, 1, x_691); +lean_ctor_set_uint8(x_705, 2, x_692); +lean_ctor_set_uint8(x_705, 3, x_693); +lean_ctor_set_uint8(x_705, 4, x_694); +lean_ctor_set_uint8(x_705, 5, x_704); +lean_ctor_set_uint8(x_705, 6, x_695); +lean_ctor_set_uint8(x_705, 7, x_696); +lean_ctor_set_uint8(x_705, 8, x_697); +lean_ctor_set_uint8(x_705, 9, x_698); +lean_ctor_set_uint8(x_705, 10, x_699); +lean_ctor_set_uint8(x_705, 11, x_700); +lean_ctor_set_uint8(x_705, 12, x_701); +lean_ctor_set_uint8(x_705, 13, x_702); +if (lean_is_scalar(x_689)) { + x_706 = lean_alloc_ctor(0, 6, 0); +} else { + x_706 = x_689; +} +lean_ctor_set(x_706, 0, x_705); +lean_ctor_set(x_706, 1, x_684); +lean_ctor_set(x_706, 2, x_685); +lean_ctor_set(x_706, 3, x_686); +lean_ctor_set(x_706, 4, x_687); +lean_ctor_set(x_706, 5, x_688); lean_inc(x_12); -x_593 = l_Lean_Meta_mkImpDepCongrCtx(x_568, x_515, x_592, x_10, x_11, x_12, x_569); -if (lean_obj_tag(x_593) == 0) +x_707 = l_Lean_Meta_mkImpDepCongrCtx(x_682, x_610, x_706, x_10, x_11, x_12, x_683); +if (lean_obj_tag(x_707) == 0) { -lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; -x_594 = lean_ctor_get(x_593, 0); -lean_inc(x_594); -x_595 = lean_ctor_get(x_593, 1); -lean_inc(x_595); -lean_dec(x_593); -if (lean_is_scalar(x_508)) { - x_596 = lean_alloc_ctor(1, 1, 0); -} else { - x_596 = x_508; -} -lean_ctor_set(x_596, 0, x_594); -x_597 = lean_unsigned_to_nat(0u); -x_598 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_598, 0, x_564); -lean_ctor_set(x_598, 1, x_596); -lean_ctor_set(x_598, 2, x_597); -x_27 = x_598; -x_28 = x_595; +lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; +x_708 = lean_ctor_get(x_707, 0); +lean_inc(x_708); +x_709 = lean_ctor_get(x_707, 1); +lean_inc(x_709); +lean_dec(x_707); +if (lean_is_scalar(x_603)) { + x_710 = lean_alloc_ctor(1, 1, 0); +} else { + x_710 = x_603; +} +lean_ctor_set(x_710, 0, x_708); +x_711 = lean_unsigned_to_nat(0u); +x_712 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_712, 0, x_678); +lean_ctor_set(x_712, 1, x_710); +lean_ctor_set(x_712, 2, x_711); +x_27 = x_712; +x_28 = x_709; goto block_48; } else { -lean_object* x_599; lean_object* x_600; -lean_dec(x_564); -lean_dec(x_508); -x_599 = lean_ctor_get(x_593, 0); -lean_inc(x_599); -x_600 = lean_ctor_get(x_593, 1); -lean_inc(x_600); -lean_dec(x_593); -x_49 = x_599; -x_50 = x_600; +lean_object* x_713; lean_object* x_714; +lean_dec(x_678); +lean_dec(x_603); +x_713 = lean_ctor_get(x_707, 0); +lean_inc(x_713); +x_714 = lean_ctor_get(x_707, 1); +lean_inc(x_714); +lean_dec(x_707); +x_49 = x_713; +x_50 = x_714; goto block_70; } } else { -lean_object* x_601; lean_object* x_602; -lean_dec(x_564); -lean_dec(x_515); -lean_dec(x_508); +lean_object* x_715; lean_object* x_716; +lean_dec(x_678); +lean_dec(x_610); +lean_dec(x_603); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -x_601 = lean_ctor_get(x_566, 0); -lean_inc(x_601); -x_602 = lean_ctor_get(x_566, 1); -lean_inc(x_602); -lean_dec(x_566); -x_49 = x_601; -x_50 = x_602; +x_715 = lean_ctor_get(x_680, 0); +lean_inc(x_715); +x_716 = lean_ctor_get(x_680, 1); +lean_inc(x_716); +lean_dec(x_680); +x_49 = x_715; +x_50 = x_716; goto block_70; } } else { -lean_object* x_603; lean_object* x_604; -lean_dec(x_515); -lean_dec(x_508); +lean_object* x_717; lean_object* x_718; +lean_dec(x_610); +lean_dec(x_603); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_3); -x_603 = lean_ctor_get(x_563, 0); -lean_inc(x_603); -x_604 = lean_ctor_get(x_563, 1); -lean_inc(x_604); -lean_dec(x_563); -x_49 = x_603; -x_50 = x_604; +x_717 = lean_ctor_get(x_677, 0); +lean_inc(x_717); +x_718 = lean_ctor_get(x_677, 1); +lean_inc(x_718); +lean_dec(x_677); +x_49 = x_717; +x_50 = x_718; goto block_70; } } } else { -lean_object* x_605; lean_object* x_606; -lean_dec(x_510); -lean_dec(x_508); -lean_dec(x_498); +lean_object* x_719; lean_object* x_720; +lean_dec(x_605); +lean_dec(x_603); +lean_dec(x_593); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -21055,20 +21624,20 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_605 = lean_ctor_get(x_514, 0); -lean_inc(x_605); -x_606 = lean_ctor_get(x_514, 1); -lean_inc(x_606); -lean_dec(x_514); -x_49 = x_605; -x_50 = x_606; +x_719 = lean_ctor_get(x_609, 0); +lean_inc(x_719); +x_720 = lean_ctor_get(x_609, 1); +lean_inc(x_720); +lean_dec(x_609); +x_49 = x_719; +x_50 = x_720; goto block_70; } } } else { -lean_object* x_607; lean_object* x_608; +lean_object* x_721; lean_object* x_722; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -21076,13 +21645,13 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_607 = lean_ctor_get(x_497, 0); -lean_inc(x_607); -x_608 = lean_ctor_get(x_497, 1); -lean_inc(x_608); -lean_dec(x_497); -x_49 = x_607; -x_50 = x_608; +x_721 = lean_ctor_get(x_592, 0); +lean_inc(x_721); +x_722 = lean_ctor_get(x_592, 1); +lean_inc(x_722); +lean_dec(x_592); +x_49 = x_721; +x_50 = x_722; goto block_70; } } @@ -21247,7 +21816,7 @@ return x_69; } else { -uint8_t x_609; +uint8_t x_723; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -21260,23 +21829,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_609 = !lean_is_exclusive(x_18); -if (x_609 == 0) +x_723 = !lean_is_exclusive(x_18); +if (x_723 == 0) { return x_18; } else { -lean_object* x_610; lean_object* x_611; lean_object* x_612; -x_610 = lean_ctor_get(x_18, 0); -x_611 = lean_ctor_get(x_18, 1); -lean_inc(x_611); -lean_inc(x_610); +lean_object* x_724; lean_object* x_725; lean_object* x_726; +x_724 = lean_ctor_get(x_18, 0); +x_725 = lean_ctor_get(x_18, 1); +lean_inc(x_725); +lean_inc(x_724); lean_dec(x_18); -x_612 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_612, 0, x_610); -lean_ctor_set(x_612, 1, x_611); -return x_612; +x_726 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_726, 0, x_724); +lean_ctor_set(x_726, 1, x_725); +return x_726; } } } @@ -23325,7 +23894,7 @@ x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -24811,7 +25380,7 @@ if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_1, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_17); x_19 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -24895,7 +25464,7 @@ if (x_36 == 0) { lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; x_37 = lean_unsigned_to_nat(0u); -x_38 = l_Lean_Expr_getAppNumArgsAux(x_1, x_37); +x_38 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_37); x_39 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_38); x_40 = lean_mk_array(x_38, x_39); @@ -33905,7 +34474,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_tryAutoCongrTheorem_x3f___lambda_ 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; size_t x_26; size_t x_27; lean_object* x_28; lean_dec(x_4); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -34143,7 +34712,7 @@ lean_inc(x_23); x_24 = lean_array_get_size(x_23); lean_dec(x_23); x_25 = lean_unsigned_to_nat(0u); -x_26 = l_Lean_Expr_getAppNumArgsAux(x_1, x_25); +x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_25); x_27 = lean_nat_dec_eq(x_24, x_26); lean_dec(x_26); lean_dec(x_24); @@ -34187,7 +34756,7 @@ lean_inc(x_33); x_34 = lean_array_get_size(x_33); lean_dec(x_33); x_35 = lean_unsigned_to_nat(0u); -x_36 = l_Lean_Expr_getAppNumArgsAux(x_1, x_35); +x_36 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_35); x_37 = lean_nat_dec_eq(x_34, x_36); lean_dec(x_36); lean_dec(x_34); @@ -35564,8 +36133,8 @@ lean_dec(x_18); x_20 = l_Lean_Expr_appArg_x21(x_1); lean_dec(x_1); x_21 = lean_unsigned_to_nat(0u); -x_22 = l_Lean_Expr_getAppNumArgsAux(x_19, x_21); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_8, x_21); +x_22 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_19, x_21); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_8, x_21); x_24 = lean_nat_dec_lt(x_22, x_23); if (x_24 == 0) { @@ -36553,7 +37122,7 @@ lean_dec(x_13); x_16 = l_Lean_Expr_appArg_x21(x_1); lean_dec(x_1); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_16, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_16, x_17); x_19 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_reduceProjFn_x3f___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -38574,7 +39143,7 @@ static lean_object* _init_l_Lean_Meta_Simp_simp_simpProj___lambda__1___closed__1 _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateProj!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateProj!Impl", 46); return x_1; } } @@ -38592,8 +39161,8 @@ static lean_object* _init_l_Lean_Meta_Simp_simp_simpProj___lambda__1___closed__3 lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_Tactic_Simp_Main_0__Lean_Meta_Simp_mkImpCongr___closed__1; x_2 = l_Lean_Meta_Simp_simp_simpProj___lambda__1___closed__1; -x_3 = lean_unsigned_to_nat(1121u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1445u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Meta_Simp_simp_simpProj___lambda__1___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -38605,19 +39174,40 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Simp_simp_simpProj___lambda__1(lean_object* lean_object* x_11; if (lean_obj_tag(x_1) == 11) { -lean_object* x_69; +lean_object* x_69; lean_object* x_70; lean_object* x_71; size_t x_72; size_t x_73; uint8_t x_74; +x_69 = lean_ctor_get(x_1, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_1, 1); +lean_inc(x_70); +x_71 = lean_ctor_get(x_1, 2); +lean_inc(x_71); +x_72 = lean_ptr_addr(x_71); +lean_dec(x_71); +x_73 = lean_ptr_addr(x_2); +x_74 = lean_usize_dec_eq(x_72, x_73); +if (x_74 == 0) +{ +lean_object* x_75; lean_inc(x_2); +x_75 = l_Lean_Expr_proj___override(x_69, x_70, x_2); +x_11 = x_75; +goto block_68; +} +else +{ +lean_dec(x_70); +lean_dec(x_69); lean_inc(x_1); -x_69 = lean_expr_update_proj(x_1, x_2); -x_11 = x_69; +x_11 = x_1; goto block_68; } +} else { -lean_object* x_70; lean_object* x_71; -x_70 = l_Lean_Meta_Simp_simp_simpProj___lambda__1___closed__3; -x_71 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_70); -x_11 = x_71; +lean_object* x_76; lean_object* x_77; +x_76 = l_Lean_Meta_Simp_simp_simpProj___lambda__1___closed__3; +x_77 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_76); +x_11 = x_77; goto block_68; } block_68: @@ -39064,19 +39654,41 @@ lean_inc(x_46); lean_dec(x_42); if (lean_obj_tag(x_1) == 11) { -lean_object* x_96; +lean_object* x_96; lean_object* x_97; lean_object* x_98; size_t x_99; size_t x_100; uint8_t x_101; +x_96 = lean_ctor_get(x_1, 0); +lean_inc(x_96); +x_97 = lean_ctor_get(x_1, 1); +lean_inc(x_97); +x_98 = lean_ctor_get(x_1, 2); +lean_inc(x_98); +x_99 = lean_ptr_addr(x_98); +lean_dec(x_98); +x_100 = lean_ptr_addr(x_45); +x_101 = lean_usize_dec_eq(x_99, x_100); +if (x_101 == 0) +{ +lean_object* x_102; +x_102 = l_Lean_Expr_proj___override(x_96, x_97, x_45); +x_47 = x_102; +goto block_95; +} +else +{ +lean_dec(x_97); +lean_dec(x_96); +lean_dec(x_45); lean_inc(x_1); -x_96 = lean_expr_update_proj(x_1, x_45); -x_47 = x_96; +x_47 = x_1; goto block_95; } +} else { -lean_object* x_97; lean_object* x_98; +lean_object* x_103; lean_object* x_104; lean_dec(x_45); -x_97 = l_Lean_Meta_Simp_simp_simpProj___lambda__1___closed__3; -x_98 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_97); -x_47 = x_98; +x_103 = l_Lean_Meta_Simp_simp_simpProj___lambda__1___closed__3; +x_104 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_103); +x_47 = x_104; goto block_95; } block_95: @@ -39335,37 +39947,37 @@ return x_94; } else { -uint8_t x_99; +uint8_t x_105; lean_dec(x_40); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_99 = !lean_is_exclusive(x_41); -if (x_99 == 0) +x_105 = !lean_is_exclusive(x_41); +if (x_105 == 0) { return x_41; } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_100 = lean_ctor_get(x_41, 0); -x_101 = lean_ctor_get(x_41, 1); -lean_inc(x_101); -lean_inc(x_100); +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_41, 0); +x_107 = lean_ctor_get(x_41, 1); +lean_inc(x_107); +lean_inc(x_106); lean_dec(x_41); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_100); -lean_ctor_set(x_102, 1, x_101); -return x_102; +x_108 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_108, 0, x_106); +lean_ctor_set(x_108, 1, x_107); +return x_108; } } } } else { -uint8_t x_103; +uint8_t x_109; lean_dec(x_13); lean_dec(x_8); lean_dec(x_7); @@ -39375,29 +39987,29 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_103 = !lean_is_exclusive(x_20); -if (x_103 == 0) +x_109 = !lean_is_exclusive(x_20); +if (x_109 == 0) { return x_20; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_20, 0); -x_105 = lean_ctor_get(x_20, 1); -lean_inc(x_105); -lean_inc(x_104); +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_20, 0); +x_111 = lean_ctor_get(x_20, 1); +lean_inc(x_111); +lean_inc(x_110); lean_dec(x_20); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_104); -lean_ctor_set(x_106, 1, x_105); -return x_106; +x_112 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_112, 0, x_110); +lean_ctor_set(x_112, 1, x_111); +return x_112; } } } else { -uint8_t x_107; +uint8_t x_113; lean_dec(x_13); lean_dec(x_8); lean_dec(x_7); @@ -39407,29 +40019,29 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_107 = !lean_is_exclusive(x_14); -if (x_107 == 0) +x_113 = !lean_is_exclusive(x_14); +if (x_113 == 0) { return x_14; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_14, 0); -x_109 = lean_ctor_get(x_14, 1); -lean_inc(x_109); -lean_inc(x_108); +lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_114 = lean_ctor_get(x_14, 0); +x_115 = lean_ctor_get(x_14, 1); +lean_inc(x_115); +lean_inc(x_114); lean_dec(x_14); -x_110 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_110, 0, x_108); -lean_ctor_set(x_110, 1, x_109); -return x_110; +x_116 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +return x_116; } } } else { -uint8_t x_111; +uint8_t x_117; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -39438,49 +40050,49 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_111 = !lean_is_exclusive(x_10); -if (x_111 == 0) +x_117 = !lean_is_exclusive(x_10); +if (x_117 == 0) { -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_112 = lean_ctor_get(x_10, 0); -lean_dec(x_112); -x_113 = lean_ctor_get(x_11, 0); -lean_inc(x_113); +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_118 = lean_ctor_get(x_10, 0); +lean_dec(x_118); +x_119 = lean_ctor_get(x_11, 0); +lean_inc(x_119); lean_dec(x_11); -x_114 = lean_box(0); -x_115 = lean_unsigned_to_nat(0u); -x_116 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_116, 0, x_113); -lean_ctor_set(x_116, 1, x_114); -lean_ctor_set(x_116, 2, x_115); -lean_ctor_set(x_10, 0, x_116); +x_120 = lean_box(0); +x_121 = lean_unsigned_to_nat(0u); +x_122 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_122, 0, x_119); +lean_ctor_set(x_122, 1, x_120); +lean_ctor_set(x_122, 2, x_121); +lean_ctor_set(x_10, 0, x_122); return x_10; } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_117 = lean_ctor_get(x_10, 1); -lean_inc(x_117); +lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_123 = lean_ctor_get(x_10, 1); +lean_inc(x_123); lean_dec(x_10); -x_118 = lean_ctor_get(x_11, 0); -lean_inc(x_118); +x_124 = lean_ctor_get(x_11, 0); +lean_inc(x_124); lean_dec(x_11); -x_119 = lean_box(0); -x_120 = lean_unsigned_to_nat(0u); -x_121 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_121, 0, x_118); -lean_ctor_set(x_121, 1, x_119); -lean_ctor_set(x_121, 2, x_120); -x_122 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_122, 0, x_121); -lean_ctor_set(x_122, 1, x_117); -return x_122; +x_125 = lean_box(0); +x_126 = lean_unsigned_to_nat(0u); +x_127 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_127, 0, x_124); +lean_ctor_set(x_127, 1, x_125); +lean_ctor_set(x_127, 2, x_126); +x_128 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_128, 0, x_127); +lean_ctor_set(x_128, 1, x_123); +return x_128; } } } else { -uint8_t x_123; +uint8_t x_129; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -39489,23 +40101,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_123 = !lean_is_exclusive(x_10); -if (x_123 == 0) +x_129 = !lean_is_exclusive(x_10); +if (x_129 == 0) { return x_10; } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_124 = lean_ctor_get(x_10, 0); -x_125 = lean_ctor_get(x_10, 1); -lean_inc(x_125); -lean_inc(x_124); +lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_130 = lean_ctor_get(x_10, 0); +x_131 = lean_ctor_get(x_10, 1); +lean_inc(x_131); +lean_inc(x_130); lean_dec(x_10); -x_126 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_126, 0, x_124); -lean_ctor_set(x_126, 1, x_125); -return x_126; +x_132 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_132, 0, x_130); +lean_ctor_set(x_132, 1, x_131); +return x_132; } } } diff --git a/stage0/stdlib/Lean/Meta/Tactic/Simp/Rewrite.c b/stage0/stdlib/Lean/Meta/Tactic/Simp/Rewrite.c index 0c984442923f..47ac98ec84eb 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Simp/Rewrite.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Simp/Rewrite.c @@ -163,6 +163,7 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Simp_rewritePost___s static lean_object* l___private_Lean_Meta_Tactic_Simp_Rewrite_0__Lean_Meta_Simp_tryTheoremCore_go___lambda__7___closed__2; LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Meta_Simp_tryTheoremWithExtraArgs_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_Simp_synthesizeArgs___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Simp_rewriteUsingDecide_x3f___closed__3; lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Simp_synthesizeArgs_synthesizeInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -231,7 +232,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Simp_rewritePost(lean_object*, lean_object* static lean_object* l_Lean_Meta_Simp_synthesizeArgs_synthesizeInstance___closed__10; lean_object* l_Lean_Meta_trySynthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); extern uint8_t l_instInhabitedBool; lean_object* l_Lean_Meta_Linear_simp_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -9308,8 +9308,8 @@ lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint x_37 = lean_ctor_get(x_34, 1); x_38 = lean_ctor_get(x_34, 0); lean_dec(x_38); -x_39 = l_Lean_Expr_getAppNumArgsAux(x_32, x_33); -x_40 = l_Lean_Expr_getAppNumArgsAux(x_1, x_33); +x_39 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_32, x_33); +x_40 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_33); x_41 = lean_nat_dec_lt(x_39, x_40); if (x_41 == 0) { @@ -9349,8 +9349,8 @@ lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; x_44 = lean_ctor_get(x_34, 1); lean_inc(x_44); lean_dec(x_34); -x_45 = l_Lean_Expr_getAppNumArgsAux(x_32, x_33); -x_46 = l_Lean_Expr_getAppNumArgsAux(x_1, x_33); +x_45 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_32, x_33); +x_46 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_33); x_47 = lean_nat_dec_lt(x_45, x_46); if (x_47 == 0) { @@ -14581,7 +14581,7 @@ static lean_object* _init_l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Simp_si lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Simp_simpMatch_x3f___spec__1___closed__2; x_2 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Simp_simpMatch_x3f___spec__1___closed__3; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Simp_simpMatch_x3f___spec__1___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -14649,7 +14649,7 @@ if (x_22 == 0) lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; x_23 = lean_ctor_get(x_13, 0); x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_Expr_getAppNumArgsAux(x_1, x_24); +x_25 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_24); x_26 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Simp_simpMatch_x3f___spec__1___closed__1; lean_inc(x_25); x_27 = lean_mk_array(x_25, x_26); @@ -14759,7 +14759,7 @@ x_59 = lean_ctor_get(x_13, 0); lean_inc(x_59); lean_dec(x_13); x_60 = lean_unsigned_to_nat(0u); -x_61 = l_Lean_Expr_getAppNumArgsAux(x_1, x_60); +x_61 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_60); x_62 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Simp_simpMatch_x3f___spec__1___closed__1; lean_inc(x_61); x_63 = lean_mk_array(x_61, x_62); @@ -14882,7 +14882,7 @@ if (lean_is_exclusive(x_13)) { x_99 = lean_box(0); } x_100 = lean_unsigned_to_nat(0u); -x_101 = l_Lean_Expr_getAppNumArgsAux(x_1, x_100); +x_101 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_100); x_102 = l_Lean_Meta_matchMatcherApp_x3f___at_Lean_Meta_Simp_simpMatch_x3f___spec__1___closed__1; lean_inc(x_101); x_103 = lean_mk_array(x_101, x_102); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpAll.c b/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpAll.c index d1fd23e885b6..be07f61b53a2 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpAll.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpAll.c @@ -2134,7 +2134,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at___private_Lean_Meta_Tactic lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at___private_Lean_Meta_Tactic_Simp_SimpAll_0__Lean_Meta_SimpAll_loop___spec__4___closed__18; x_2 = l_Std_Range_forIn_loop___at___private_Lean_Meta_Tactic_Simp_SimpAll_0__Lean_Meta_SimpAll_loop___spec__4___closed__19; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at___private_Lean_Meta_Tactic_Simp_SimpAll_0__Lean_Meta_SimpAll_loop___spec__4___closed__20; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpCongrTheorems.c b/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpCongrTheorems.c index 5321ec7a2ab5..dd0e0c75f9a6 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpCongrTheorems.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpCongrTheorems.c @@ -175,6 +175,7 @@ static lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheorem__ LEAN_EXPORT lean_object* l_Lean_Meta_getSimpCongrTheorems___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheorem___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpCongrTheorems_0__Lean_Meta_reprSimpCongrTheorem____x40_Lean_Meta_Tactic_Simp_SimpCongrTheorems___hyg_51____closed__19; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Nat_repr(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_Meta_addSimpCongrTheoremEntry___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_SMap_find_x3f___at_Lean_Meta_SimpCongrTheorems_get___spec__1(lean_object*, lean_object*); @@ -262,7 +263,6 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheo lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_addSimpCongrTheoremEntry___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheorem___spec__5___closed__1; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); uint8_t l_Lean_Expr_isMVar(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpCongrTheorems_0__Lean_Meta_reprSimpCongrTheorem____x40_Lean_Meta_Tactic_Simp_SimpCongrTheorems___hyg_51____closed__8; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_foldlM___at___private_Lean_Meta_Tactic_Simp_SimpCongrTheorems_0__Lean_Meta_reprSimpCongrTheorems____x40_Lean_Meta_Tactic_Simp_SimpCongrTheorems___hyg_148____spec__11(lean_object*); @@ -4524,7 +4524,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheo { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; lean_object* x_20; lean_object* x_21; x_11 = lean_unsigned_to_nat(0u); -x_12 = l_Lean_Expr_getAppNumArgsAux(x_1, x_11); +x_12 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_11); x_13 = l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheorem___spec__9___lambda__2___closed__1; lean_inc(x_12); x_14 = lean_mk_array(x_12, x_13); @@ -8010,7 +8010,7 @@ else lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_10); x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Lean_Expr_getAppNumArgsAux(x_7, x_22); +x_23 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_7, x_22); x_24 = l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheorem___spec__9___lambda__2___closed__1; lean_inc(x_23); x_25 = lean_mk_array(x_23, x_24); @@ -8172,7 +8172,7 @@ x_42 = l_Lean_Expr_appArg_x21(x_41); lean_dec(x_41); x_43 = l_Lean_Expr_appArg_x21(x_27); x_44 = lean_unsigned_to_nat(0u); -x_45 = l_Lean_Expr_getAppNumArgsAux(x_42, x_44); +x_45 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_42, x_44); x_46 = l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheorem___spec__9___lambda__2___closed__1; lean_inc(x_45); x_47 = lean_mk_array(x_45, x_46); @@ -8450,7 +8450,7 @@ x_116 = l_Lean_Expr_appArg_x21(x_115); lean_dec(x_115); x_117 = l_Lean_Expr_appArg_x21(x_101); x_118 = lean_unsigned_to_nat(0u); -x_119 = l_Lean_Expr_getAppNumArgsAux(x_116, x_118); +x_119 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_116, x_118); x_120 = l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheorem___spec__9___lambda__2___closed__1; lean_inc(x_119); x_121 = lean_mk_array(x_119, x_120); @@ -8767,7 +8767,7 @@ x_198 = l_Lean_Expr_appArg_x21(x_197); lean_dec(x_197); x_199 = l_Lean_Expr_appArg_x21(x_183); x_200 = lean_unsigned_to_nat(0u); -x_201 = l_Lean_Expr_getAppNumArgsAux(x_198, x_200); +x_201 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_198, x_200); x_202 = l_Array_forInUnsafe_loop___at_Lean_Meta_mkSimpCongrTheorem___spec__9___lambda__2___closed__1; lean_inc(x_201); x_203 = lean_mk_array(x_201, x_202); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpTheorems.c b/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpTheorems.c index 8908fc7fac40..1249518d6912 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpTheorems.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Simp/SimpTheorems.c @@ -72,9 +72,11 @@ static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_ LEAN_EXPORT lean_object* l_Lean_Meta_addSimpTheoremEntry_updateLemmaNames(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkAppM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__6; +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__110; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_isRflTheorem___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_SimpTheorems_erase___rarg___closed__1; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__111; lean_object* l_Lean_registerSimpleScopedEnvExtension___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Meta_addSimpTheoremEntry___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -102,6 +104,7 @@ static lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Meta_addSimpTheorem_ LEAN_EXPORT uint8_t l_Lean_Meta_SimpTheorems_isDeclToUnfold(lean_object*, lean_object*); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__59; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__113; LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_addSimpTheoremEntry___spec__15(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_isPerm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); @@ -115,6 +118,7 @@ static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_ lean_object* l_Lean_Expr_appFn_x21(lean_object*); lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at___aux__Init__Notation______macroRules__precMax__1___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__8; +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__107; LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_add(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__21; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_Meta_addSimpTheoremEntry___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -133,6 +137,7 @@ lean_object* l_Lean_throwError___at___private_Lean_Meta_InferType_0__Lean_Meta_i lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_SimpTheoremsArray_eraseTheorem___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__17; +uint8_t l_ptrEqList___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_commandRegister__simp__attr_______closed__4; static lean_object* l_Lean_Meta_commandRegister__simp__attr_______closed__17; static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__1; @@ -154,6 +159,7 @@ lean_object* lean_string_utf8_byte_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isRflProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__82; static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_shouldPreprocess___closed__1; +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__112; LEAN_EXPORT lean_object* l_Std_AssocList_contains___at_Lean_Meta_registerSimpAttr___spec__2___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__61; static lean_object* l_Lean_Meta_instInhabitedSimpTheorems___closed__2; @@ -183,6 +189,7 @@ static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems___ static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__90; LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Meta_mkSimpAttr___spec__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getAttrParamOptPrio(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__114; static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__3___closed__12; LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorem_keys___default; uint64_t l_Lean_Name_hash___override(lean_object*); @@ -190,6 +197,7 @@ lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__26; static lean_object* l_Lean_Meta_instInhabitedSimpTheorems___closed__1; static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__19; +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__104; LEAN_EXPORT lean_object* l_Lean_Meta_isRflTheorem(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_addSimpTheoremEntry___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -201,6 +209,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_toUnfoldThms___default; static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__51; LEAN_EXPORT lean_object* l_Lean_Meta_instBEqSimpTheorem___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_commandRegister__simp__attr_______closed__12; +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__109; static lean_object* l_Lean_Meta_SimpTheorems_toUnfoldThms___default___closed__3; static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___closed__7; lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); @@ -263,6 +272,7 @@ static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addSimpTheor static lean_object* l_Lean_Meta_SimpTheorem_getName___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_commandRegister__simp__attr____; static lean_object* l_Lean_Meta_SimpTheorem_getName___closed__2; +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__105; static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_Meta_isRflTheorem___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -270,6 +280,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_mkSimpExt___lambda__1(lean_object*, lean_ob lean_object* l_Lean_Syntax_getId(lean_object*); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__56; extern lean_object* l_Lean_Expr_instHashableExpr; +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__115; static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__66; static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__11; lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); @@ -313,6 +324,7 @@ static lean_object* l_Lean_Meta_commandRegister__simp__attr_______closed__7; size_t lean_usize_mul(size_t, size_t); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__49; lean_object* l_Lean_Expr_bvar___override(lean_object*); +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__106; static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__3___closed__9; static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__24; LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheorems_eraseCore(lean_object*, lean_object*); @@ -375,6 +387,7 @@ static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__9; static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__3___closed__8; static lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_SimpTheoremsArray_eraseTheorem(lean_object*, lean_object*); +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__103; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_SimpTheoremsArray_isErased___spec__1(lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_Meta_whnfR(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Meta_addSimpTheoremEntry___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -441,6 +454,7 @@ uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__18; static lean_object* l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addSimpTheoremEntry___spec__1___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*); +static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__108; static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__15; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_isRflTheorem___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -590,7 +604,6 @@ lean_object* l_Std_PersistentHashMap_erase___at_Lean_Meta_Instances_eraseCore___ uint64_t l_Lean_Meta_DiscrTree_Key_hash(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAux___at_Lean_Meta_SimpTheorems_erase___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__57; -lean_object* lean_expr_update_const(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkSimpAttr___lambda__1___closed__14; static lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at_Lean_Meta_addSimpTheoremEntry___spec__9___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_instInhabitedSimpEntry; @@ -2903,7 +2916,7 @@ static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addSim lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addSimpTheoremEntry___spec__1___closed__1; x_2 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addSimpTheoremEntry___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_addSimpTheoremEntry___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -13922,7 +13935,7 @@ static lean_object* _init_l_Lean_Meta_SimpTheorem_getValue___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateConst!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateConst!Impl", 47); return x_1; } } @@ -13940,8 +13953,8 @@ static lean_object* _init_l_Lean_Meta_SimpTheorem_getValue___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_SimpTheorem_getValue___closed__1; x_2 = l_Lean_Meta_SimpTheorem_getValue___closed__2; -x_3 = lean_unsigned_to_nat(1090u); -x_4 = lean_unsigned_to_nat(20u); +x_3 = lean_unsigned_to_nat(1412u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Meta_SimpTheorem_getValue___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -14067,54 +14080,93 @@ uint8_t x_42; x_42 = !lean_is_exclusive(x_41); if (x_42 == 0) { -lean_object* x_43; lean_object* x_44; +lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; x_43 = lean_ctor_get(x_41, 0); -x_44 = lean_expr_update_const(x_7, x_43); -lean_ctor_set(x_41, 0, x_44); +x_44 = lean_ctor_get(x_7, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_7, 1); +lean_inc(x_45); +x_46 = l_ptrEqList___rarg(x_45, x_43); +lean_dec(x_45); +if (x_46 == 0) +{ +lean_object* x_47; +lean_dec(x_7); +x_47 = l_Lean_Expr_const___override(x_44, x_43); +lean_ctor_set(x_41, 0, x_47); return x_41; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_45 = lean_ctor_get(x_41, 0); -x_46 = lean_ctor_get(x_41, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_41); -x_47 = lean_expr_update_const(x_7, x_45); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_47); -lean_ctor_set(x_48, 1, x_46); -return x_48; +lean_dec(x_44); +lean_dec(x_43); +lean_ctor_set(x_41, 0, x_7); +return x_41; } } else { -uint8_t x_49; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; +x_48 = lean_ctor_get(x_41, 0); +x_49 = lean_ctor_get(x_41, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_41); +x_50 = lean_ctor_get(x_7, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_7, 1); +lean_inc(x_51); +x_52 = l_ptrEqList___rarg(x_51, x_48); +lean_dec(x_51); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; lean_dec(x_7); -x_49 = !lean_is_exclusive(x_41); -if (x_49 == 0) +x_53 = l_Lean_Expr_const___override(x_50, x_48); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_49); +return x_54; +} +else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_41, 0); +lean_object* x_55; lean_dec(x_50); -x_51 = l_Lean_Meta_SimpTheorem_getValue___closed__4; -x_52 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_51); -lean_ctor_set(x_41, 0, x_52); +lean_dec(x_48); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_7); +lean_ctor_set(x_55, 1, x_49); +return x_55; +} +} +} +else +{ +uint8_t x_56; +lean_dec(x_7); +x_56 = !lean_is_exclusive(x_41); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_41, 0); +lean_dec(x_57); +x_58 = l_Lean_Meta_SimpTheorem_getValue___closed__4; +x_59 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_58); +lean_ctor_set(x_41, 0, x_59); return x_41; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_53 = lean_ctor_get(x_41, 1); -lean_inc(x_53); +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_60 = lean_ctor_get(x_41, 1); +lean_inc(x_60); lean_dec(x_41); -x_54 = l_Lean_Meta_SimpTheorem_getValue___closed__4; -x_55 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_54); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_53); -return x_56; +x_61 = l_Lean_Meta_SimpTheorem_getValue___closed__4; +x_62 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_61); +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_60); +return x_63; } } } @@ -14127,102 +14179,127 @@ return x_35; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; -x_57 = lean_ctor_get(x_35, 0); -x_58 = lean_ctor_get(x_35, 1); -lean_inc(x_58); -lean_inc(x_57); +lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; +x_64 = lean_ctor_get(x_35, 0); +x_65 = lean_ctor_get(x_35, 1); +lean_inc(x_65); +lean_inc(x_64); lean_dec(x_35); -x_59 = l_Lean_ConstantInfo_levelParams(x_57); -lean_dec(x_57); -x_60 = l_List_isEmpty___rarg(x_59); -if (x_60 == 0) +x_66 = l_Lean_ConstantInfo_levelParams(x_64); +lean_dec(x_64); +x_67 = l_List_isEmpty___rarg(x_66); +if (x_67 == 0) { -lean_object* x_61; -x_61 = l_List_mapM___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkFun___spec__1(x_59, x_2, x_3, x_4, x_5, x_58); +lean_object* x_68; +x_68 = l_List_mapM___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkFun___spec__1(x_66, x_2, x_3, x_4, x_5, x_65); if (lean_obj_tag(x_7) == 4) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_64 = x_61; +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_71 = x_68; } else { - lean_dec_ref(x_61); - x_64 = lean_box(0); + lean_dec_ref(x_68); + x_71 = lean_box(0); } -x_65 = lean_expr_update_const(x_7, x_62); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(0, 2, 0); +x_72 = lean_ctor_get(x_7, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_7, 1); +lean_inc(x_73); +x_74 = l_ptrEqList___rarg(x_73, x_69); +lean_dec(x_73); +if (x_74 == 0) +{ +lean_object* x_75; lean_object* x_76; +lean_dec(x_7); +x_75 = l_Lean_Expr_const___override(x_72, x_69); +if (lean_is_scalar(x_71)) { + x_76 = lean_alloc_ctor(0, 2, 0); } else { - x_66 = x_64; + x_76 = x_71; +} +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_70); +return x_76; +} +else +{ +lean_object* x_77; +lean_dec(x_72); +lean_dec(x_69); +if (lean_is_scalar(x_71)) { + x_77 = lean_alloc_ctor(0, 2, 0); +} else { + x_77 = x_71; +} +lean_ctor_set(x_77, 0, x_7); +lean_ctor_set(x_77, 1, x_70); +return x_77; } -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_63); -return x_66; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_dec(x_7); -x_67 = lean_ctor_get(x_61, 1); -lean_inc(x_67); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_68 = x_61; +x_78 = lean_ctor_get(x_68, 1); +lean_inc(x_78); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_79 = x_68; } else { - lean_dec_ref(x_61); - x_68 = lean_box(0); + lean_dec_ref(x_68); + x_79 = lean_box(0); } -x_69 = l_Lean_Meta_SimpTheorem_getValue___closed__4; -x_70 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_69); -if (lean_is_scalar(x_68)) { - x_71 = lean_alloc_ctor(0, 2, 0); +x_80 = l_Lean_Meta_SimpTheorem_getValue___closed__4; +x_81 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_80); +if (lean_is_scalar(x_79)) { + x_82 = lean_alloc_ctor(0, 2, 0); } else { - x_71 = x_68; + x_82 = x_79; } -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_67); -return x_71; +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_78); +return x_82; } } else { -lean_object* x_72; -lean_dec(x_59); -x_72 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_72, 0, x_7); -lean_ctor_set(x_72, 1, x_58); -return x_72; +lean_object* x_83; +lean_dec(x_66); +x_83 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_83, 0, x_7); +lean_ctor_set(x_83, 1, x_65); +return x_83; } } } else { -uint8_t x_73; +uint8_t x_84; lean_dec(x_7); -x_73 = !lean_is_exclusive(x_35); -if (x_73 == 0) +x_84 = !lean_is_exclusive(x_35); +if (x_84 == 0) { return x_35; } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_35, 0); -x_75 = lean_ctor_get(x_35, 1); -lean_inc(x_75); -lean_inc(x_74); +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_35, 0); +x_86 = lean_ctor_get(x_35, 1); +lean_inc(x_86); +lean_inc(x_85); lean_dec(x_35); -x_76 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_76, 0, x_74); -lean_ctor_set(x_76, 1, x_75); -return x_76; +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +return x_87; } } } @@ -16223,6 +16300,24 @@ return x_3; static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__10() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("declModifiers", 13); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__7; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__10; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__5; @@ -16234,7 +16329,108 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__11() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(6u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__13; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__14; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__15; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__17; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__18; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__11; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__19; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__21() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("initializeKeyword", 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__7; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__21; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__23() { _start: { lean_object* x_1; @@ -16242,22 +16438,22 @@ x_1 = lean_mk_string_from_bytes("ext", 3); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__24() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__11; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__23; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__13() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__11; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__23; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__24; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16265,17 +16461,17 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__14() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__26() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__11; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__23; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__15() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__27() { _start: { lean_object* x_1; @@ -16283,17 +16479,17 @@ x_1 = lean_mk_string_from_bytes("Term", 4); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta_mkSimpAttr___lambda__1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__15; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__27; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__17() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__29() { _start: { lean_object* x_1; @@ -16301,17 +16497,17 @@ x_1 = lean_mk_string_from_bytes("typeSpec", 8); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__18() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__30() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__17; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__29; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__19() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__31() { _start: { lean_object* x_1; @@ -16319,22 +16515,22 @@ x_1 = lean_mk_string_from_bytes("SimpExtension", 13); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__20() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__32() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__19; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__31; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__21() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__19; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__31; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__20; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__32; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16342,51 +16538,51 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__22() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__34() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__19; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__31; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__23() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__35() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta_commandRegister__simp__attr_______closed__2; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__19; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__31; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__24() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__36() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__23; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__35; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__25() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__37() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__24; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__36; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__26() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__38() { _start: { lean_object* x_1; lean_object* x_2; @@ -16395,7 +16591,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__27() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__39() { _start: { lean_object* x_1; @@ -16403,7 +16599,7 @@ x_1 = lean_mk_string_from_bytes("←", 3); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__40() { _start: { lean_object* x_1; lean_object* x_2; @@ -16412,7 +16608,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__29() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__41() { _start: { lean_object* x_1; @@ -16420,17 +16616,17 @@ x_1 = lean_mk_string_from_bytes("doSeqIndent", 11); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__30() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__42() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__29; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__41; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__31() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__43() { _start: { lean_object* x_1; @@ -16438,17 +16634,17 @@ x_1 = lean_mk_string_from_bytes("doSeqItem", 9); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__32() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__44() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__31; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__43; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__33() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__45() { _start: { lean_object* x_1; @@ -16456,17 +16652,17 @@ x_1 = lean_mk_string_from_bytes("doExpr", 6); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__34() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__46() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__33; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__45; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__35() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__47() { _start: { lean_object* x_1; @@ -16474,17 +16670,17 @@ x_1 = lean_mk_string_from_bytes("app", 3); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__36() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__35; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__47; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__37() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__49() { _start: { lean_object* x_1; @@ -16492,22 +16688,22 @@ x_1 = lean_mk_string_from_bytes("registerSimpAttr", 16); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__38() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__50() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__37; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__49; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__39() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__51() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__37; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__49; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__38; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__50; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16515,51 +16711,51 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__40() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__52() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__37; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__49; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__41() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__53() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta_commandRegister__simp__attr_______closed__2; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__37; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__49; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__42() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__54() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__41; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__53; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__43() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__55() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__42; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__54; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__44() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__56() { _start: { lean_object* x_1; lean_object* x_2; @@ -16568,17 +16764,17 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__45() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__57() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__44; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__10; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__56; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__20; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__46() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__58() { _start: { lean_object* x_1; @@ -16586,17 +16782,17 @@ x_1 = lean_mk_string_from_bytes("syntax", 6); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__47() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__59() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__7; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__46; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__58; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__48() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__60() { _start: { lean_object* x_1; @@ -16604,33 +16800,33 @@ x_1 = lean_mk_string_from_bytes("attrKind", 8); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__49() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__61() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__48; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__60; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__50() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__62() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__3___closed__9; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__10; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__51() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__63() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__49; -x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__50; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__61; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__62; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16638,7 +16834,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__52() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__64() { _start: { lean_object* x_1; @@ -16646,17 +16842,17 @@ x_1 = lean_mk_string_from_bytes("namedName", 9); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__53() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__65() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__7; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__52; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__64; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__54() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__66() { _start: { lean_object* x_1; @@ -16664,7 +16860,7 @@ x_1 = lean_mk_string_from_bytes("(", 1); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__55() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__67() { _start: { lean_object* x_1; @@ -16672,7 +16868,7 @@ x_1 = lean_mk_string_from_bytes("name", 4); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__56() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__68() { _start: { lean_object* x_1; @@ -16680,7 +16876,7 @@ x_1 = lean_mk_string_from_bytes(":=", 2); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__57() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__69() { _start: { lean_object* x_1; @@ -16688,7 +16884,7 @@ x_1 = lean_mk_string_from_bytes(")", 1); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__58() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__70() { _start: { lean_object* x_1; lean_object* x_2; @@ -16697,7 +16893,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__59() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__71() { _start: { lean_object* x_1; @@ -16705,17 +16901,17 @@ x_1 = lean_mk_string_from_bytes("Syntax", 6); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__60() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__72() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta_mkSimpAttr___lambda__1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__59; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__71; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__61() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__73() { _start: { lean_object* x_1; @@ -16723,17 +16919,17 @@ x_1 = lean_mk_string_from_bytes("atom", 4); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__62() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__74() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__60; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__61; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__72; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__73; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__63() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__75() { _start: { lean_object* x_1; @@ -16741,17 +16937,17 @@ x_1 = lean_mk_string_from_bytes("stx_?", 5); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__64() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__76() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__63; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__75; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__65() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__77() { _start: { lean_object* x_1; @@ -16759,17 +16955,17 @@ x_1 = lean_mk_string_from_bytes("paren", 5); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__66() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__78() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__60; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__65; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__72; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__77; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__67() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__79() { _start: { lean_object* x_1; @@ -16777,17 +16973,17 @@ x_1 = lean_mk_string_from_bytes("stx_<|>_", 8); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__68() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__80() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__67; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__79; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__69() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__81() { _start: { lean_object* x_1; @@ -16795,17 +16991,17 @@ x_1 = lean_mk_string_from_bytes("cat", 3); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__70() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__82() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__60; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__69; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__72; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__81; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__71() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__83() { _start: { lean_object* x_1; @@ -16813,22 +17009,22 @@ x_1 = lean_mk_string_from_bytes("Parser.Tactic.simpPre", 21); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__72() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__84() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__71; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__83; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__73() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__85() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__71; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__83; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__72; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__84; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16836,7 +17032,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__74() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__86() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -16846,7 +17042,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__75() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__87() { _start: { lean_object* x_1; @@ -16854,51 +17050,51 @@ x_1 = lean_mk_string_from_bytes("simpPre", 7); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__76() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__88() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__74; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__75; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__86; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__87; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__77() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__89() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Meta_mkSimpAttr___lambda__1___closed__18; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__75; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__87; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__78() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__90() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__77; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__89; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__79() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__91() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__78; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__90; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__80() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__92() { _start: { lean_object* x_1; @@ -16906,7 +17102,7 @@ x_1 = lean_mk_string_from_bytes("<|>", 3); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__81() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__93() { _start: { lean_object* x_1; @@ -16914,22 +17110,22 @@ x_1 = lean_mk_string_from_bytes("Parser.Tactic.simpPost", 22); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__82() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__94() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__81; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__93; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__83() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__95() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__81; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__93; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__82; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__94; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -16937,17 +17133,17 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__84() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__96() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__74; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__86; x_2 = l_Lean_Meta_mkSimpAttr___lambda__1___closed__19; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__85() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__97() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -16959,19 +17155,19 @@ lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__86() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__98() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__85; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__97; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__87() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__99() { _start: { lean_object* x_1; @@ -16979,7 +17175,7 @@ x_1 = lean_mk_string_from_bytes("?", 1); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__88() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__100() { _start: { lean_object* x_1; @@ -16987,22 +17183,22 @@ x_1 = lean_mk_string_from_bytes("prio", 4); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__89() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__101() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__88; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__100; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__90() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__102() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__88; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__100; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__89; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__101; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -17010,17 +17206,17 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__91() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__103() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__88; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__100; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__92() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__104() { _start: { lean_object* x_1; @@ -17028,22 +17224,22 @@ x_1 = lean_mk_string_from_bytes("attr", 4); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__93() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__105() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__92; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__104; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__94() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__106() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__92; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__104; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__93; +x_3 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__105; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -17051,46 +17247,56 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__95() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__107() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__92; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__104; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__96() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__108() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(9u); +x_1 = lean_unsigned_to_nat(10u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__97() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__109() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__96; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__10; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__108; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__98() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__110() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__97; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__51; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__109; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__99() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__111() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__110; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__63; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__112() { _start: { lean_object* x_1; @@ -17098,17 +17304,17 @@ x_1 = lean_mk_string_from_bytes("quotedName", 10); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__100() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__113() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__16; -x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__99; +x_1 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28; +x_2 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__112; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__101() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__114() { _start: { lean_object* x_1; @@ -17116,7 +17322,7 @@ x_1 = lean_mk_string_from_bytes(".", 1); return x_1; } } -static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__102() { +static lean_object* _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__115() { _start: { lean_object* x_1; @@ -17144,7 +17350,7 @@ return x_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; x_8 = lean_unsigned_to_nat(1u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); x_10 = lean_unsigned_to_nat(2u); @@ -17182,358 +17388,364 @@ lean_inc(x_19); x_25 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_25, 0, x_19); lean_ctor_set(x_25, 1, x_24); -x_26 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__14; +x_26 = l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__3___closed__9; +x_27 = lean_array_push(x_26, x_25); +x_28 = lean_box(2); +x_29 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__22; +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_27); +x_31 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__26; lean_inc(x_22); lean_inc(x_23); -x_27 = l_Lean_addMacroScope(x_23, x_26, x_22); -x_28 = lean_box(0); -x_29 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__13; +x_32 = l_Lean_addMacroScope(x_23, x_31, x_22); +x_33 = lean_box(0); +x_34 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__25; lean_inc(x_19); -x_30 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_30, 0, x_19); -lean_ctor_set(x_30, 1, x_29); -lean_ctor_set(x_30, 2, x_27); -lean_ctor_set(x_30, 3, x_28); -x_31 = l_Lean_Meta_instToFormatSimpTheorem___closed__1; +x_35 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_35, 0, x_19); +lean_ctor_set(x_35, 1, x_34); +lean_ctor_set(x_35, 2, x_32); +lean_ctor_set(x_35, 3, x_33); +x_36 = l_Lean_Meta_instToFormatSimpTheorem___closed__1; lean_inc(x_19); -x_32 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_32, 0, x_19); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__22; +x_37 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_37, 0, x_19); +lean_ctor_set(x_37, 1, x_36); +x_38 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__34; lean_inc(x_22); lean_inc(x_23); -x_34 = l_Lean_addMacroScope(x_23, x_33, x_22); -x_35 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__21; -x_36 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__25; +x_39 = l_Lean_addMacroScope(x_23, x_38, x_22); +x_40 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__33; +x_41 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__37; lean_inc(x_19); -x_37 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_37, 0, x_19); -lean_ctor_set(x_37, 1, x_35); -lean_ctor_set(x_37, 2, x_34); -lean_ctor_set(x_37, 3, x_36); -x_38 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__26; -lean_inc(x_32); -x_39 = lean_array_push(x_38, x_32); -x_40 = lean_array_push(x_39, x_37); -x_41 = lean_box(2); -x_42 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__18; -x_43 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -lean_ctor_set(x_43, 2, x_40); -x_44 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__27; +x_42 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_42, 0, x_19); +lean_ctor_set(x_42, 1, x_40); +lean_ctor_set(x_42, 2, x_39); +lean_ctor_set(x_42, 3, x_41); +x_43 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__38; +lean_inc(x_37); +x_44 = lean_array_push(x_43, x_37); +x_45 = lean_array_push(x_44, x_42); +x_46 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__30; +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_28); +lean_ctor_set(x_47, 1, x_46); +lean_ctor_set(x_47, 2, x_45); +x_48 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__39; lean_inc(x_19); -x_45 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_45, 0, x_19); -lean_ctor_set(x_45, 1, x_44); -x_46 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__28; -x_47 = lean_array_push(x_46, x_30); -x_48 = lean_array_push(x_47, x_43); -x_49 = lean_array_push(x_48, x_45); -x_50 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__5; -x_51 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_51, 0, x_41); -lean_ctor_set(x_51, 1, x_50); -lean_ctor_set(x_51, 2, x_49); -x_52 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__40; +x_49 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_49, 0, x_19); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__40; +x_51 = lean_array_push(x_50, x_35); +x_52 = lean_array_push(x_51, x_47); +x_53 = lean_array_push(x_52, x_49); +x_54 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__5; +x_55 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_55, 0, x_28); +lean_ctor_set(x_55, 1, x_54); +lean_ctor_set(x_55, 2, x_53); +x_56 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__52; lean_inc(x_22); lean_inc(x_23); -x_53 = l_Lean_addMacroScope(x_23, x_52, x_22); -x_54 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__39; -x_55 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__43; +x_57 = l_Lean_addMacroScope(x_23, x_56, x_22); +x_58 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__51; +x_59 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__55; lean_inc(x_19); -x_56 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_56, 0, x_19); -lean_ctor_set(x_56, 1, x_54); -lean_ctor_set(x_56, 2, x_53); -lean_ctor_set(x_56, 3, x_55); +x_60 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_60, 0, x_19); +lean_ctor_set(x_60, 1, x_58); +lean_ctor_set(x_60, 2, x_57); +lean_ctor_set(x_60, 3, x_59); lean_inc(x_12); -x_57 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_28, x_12); -x_58 = lean_array_push(x_38, x_56); -x_59 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__45; -x_60 = lean_array_push(x_59, x_25); -x_61 = lean_array_push(x_60, x_51); -x_62 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__46; -lean_inc(x_19); -x_63 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_63, 0, x_19); -lean_ctor_set(x_63, 1, x_62); -x_64 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__54; -lean_inc(x_19); -x_65 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_65, 0, x_19); -lean_ctor_set(x_65, 1, x_64); -x_66 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__55; +x_61 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_33, x_12); +x_62 = lean_array_push(x_43, x_60); +x_63 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__57; +x_64 = lean_array_push(x_63, x_30); +x_65 = lean_array_push(x_64, x_55); +x_66 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__58; lean_inc(x_19); x_67 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_67, 0, x_19); lean_ctor_set(x_67, 1, x_66); -x_68 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__56; +x_68 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__66; lean_inc(x_19); x_69 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_69, 0, x_19); lean_ctor_set(x_69, 1, x_68); -x_70 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__57; +x_70 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__67; lean_inc(x_19); x_71 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_71, 0, x_19); lean_ctor_set(x_71, 1, x_70); -x_72 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__58; -lean_inc(x_65); -x_73 = lean_array_push(x_72, x_65); -x_74 = lean_array_push(x_73, x_67); -x_75 = lean_array_push(x_74, x_69); -x_76 = lean_array_push(x_75, x_17); -lean_inc(x_71); -x_77 = lean_array_push(x_76, x_71); -x_78 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__53; -x_79 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_79, 0, x_41); -lean_ctor_set(x_79, 1, x_78); -lean_ctor_set(x_79, 2, x_77); -x_80 = l___private_Lean_Meta_Tactic_Simp_SimpTheorems_0__Lean_Meta_preprocess_go___lambda__3___closed__9; -x_81 = lean_array_push(x_80, x_79); -x_82 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_82, 0, x_41); -lean_ctor_set(x_82, 1, x_50); -lean_ctor_set(x_82, 2, x_81); -x_83 = l_Lean_Syntax_mkStrLit(x_14, x_41); +x_72 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__68; +lean_inc(x_19); +x_73 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_73, 0, x_19); +lean_ctor_set(x_73, 1, x_72); +x_74 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__69; +lean_inc(x_19); +x_75 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_75, 0, x_19); +lean_ctor_set(x_75, 1, x_74); +x_76 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__70; +lean_inc(x_69); +x_77 = lean_array_push(x_76, x_69); +x_78 = lean_array_push(x_77, x_71); +x_79 = lean_array_push(x_78, x_73); +x_80 = lean_array_push(x_79, x_17); +lean_inc(x_75); +x_81 = lean_array_push(x_80, x_75); +x_82 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__65; +x_83 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_83, 0, x_28); +lean_ctor_set(x_83, 1, x_82); +lean_ctor_set(x_83, 2, x_81); +x_84 = lean_array_push(x_26, x_83); +x_85 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_85, 0, x_28); +lean_ctor_set(x_85, 1, x_54); +lean_ctor_set(x_85, 2, x_84); +x_86 = l_Lean_Syntax_mkStrLit(x_14, x_28); lean_dec(x_14); -x_84 = lean_array_push(x_80, x_83); -x_85 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__62; -x_86 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_86, 0, x_41); -lean_ctor_set(x_86, 1, x_85); -lean_ctor_set(x_86, 2, x_84); -x_87 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__76; +x_87 = lean_array_push(x_26, x_86); +x_88 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__74; +x_89 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_89, 0, x_28); +lean_ctor_set(x_89, 1, x_88); +lean_ctor_set(x_89, 2, x_87); +x_90 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__88; lean_inc(x_22); lean_inc(x_23); -x_88 = l_Lean_addMacroScope(x_23, x_87, x_22); -x_89 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__73; -x_90 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__79; +x_91 = l_Lean_addMacroScope(x_23, x_90, x_22); +x_92 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__85; +x_93 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__91; lean_inc(x_19); -x_91 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_91, 0, x_19); -lean_ctor_set(x_91, 1, x_89); -lean_ctor_set(x_91, 2, x_88); -lean_ctor_set(x_91, 3, x_90); -x_92 = lean_array_push(x_38, x_91); -x_93 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__10; -x_94 = lean_array_push(x_92, x_93); -x_95 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__70; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_41); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_94); -x_97 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__80; +x_94 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_94, 0, x_19); +lean_ctor_set(x_94, 1, x_92); +lean_ctor_set(x_94, 2, x_91); +lean_ctor_set(x_94, 3, x_93); +x_95 = lean_array_push(x_43, x_94); +x_96 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__12; +x_97 = lean_array_push(x_95, x_96); +x_98 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__82; +x_99 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_99, 0, x_28); +lean_ctor_set(x_99, 1, x_98); +lean_ctor_set(x_99, 2, x_97); +x_100 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__92; lean_inc(x_19); -x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_19); -lean_ctor_set(x_98, 1, x_97); -x_99 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__84; +x_101 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_101, 0, x_19); +lean_ctor_set(x_101, 1, x_100); +x_102 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__96; lean_inc(x_22); lean_inc(x_23); -x_100 = l_Lean_addMacroScope(x_23, x_99, x_22); -x_101 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__83; -x_102 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__86; +x_103 = l_Lean_addMacroScope(x_23, x_102, x_22); +x_104 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__95; +x_105 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__98; lean_inc(x_19); -x_103 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_103, 0, x_19); -lean_ctor_set(x_103, 1, x_101); -lean_ctor_set(x_103, 2, x_100); -lean_ctor_set(x_103, 3, x_102); -x_104 = lean_array_push(x_38, x_103); -x_105 = lean_array_push(x_104, x_93); -x_106 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_106, 0, x_41); -lean_ctor_set(x_106, 1, x_95); -lean_ctor_set(x_106, 2, x_105); -x_107 = lean_array_push(x_46, x_96); -x_108 = lean_array_push(x_107, x_98); -x_109 = lean_array_push(x_108, x_106); -x_110 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__68; -x_111 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_111, 0, x_41); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_111, 2, x_109); -x_112 = lean_array_push(x_80, x_111); -x_113 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_113, 0, x_41); -lean_ctor_set(x_113, 1, x_50); -lean_ctor_set(x_113, 2, x_112); -x_114 = lean_array_push(x_46, x_65); -lean_inc(x_114); -x_115 = lean_array_push(x_114, x_113); -lean_inc(x_71); -x_116 = lean_array_push(x_115, x_71); -x_117 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__66; -x_118 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_118, 0, x_41); -lean_ctor_set(x_118, 1, x_117); -lean_ctor_set(x_118, 2, x_116); -x_119 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__87; +x_106 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_106, 0, x_19); +lean_ctor_set(x_106, 1, x_104); +lean_ctor_set(x_106, 2, x_103); +lean_ctor_set(x_106, 3, x_105); +x_107 = lean_array_push(x_43, x_106); +x_108 = lean_array_push(x_107, x_96); +x_109 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_109, 0, x_28); +lean_ctor_set(x_109, 1, x_98); +lean_ctor_set(x_109, 2, x_108); +x_110 = lean_array_push(x_50, x_99); +x_111 = lean_array_push(x_110, x_101); +x_112 = lean_array_push(x_111, x_109); +x_113 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__80; +x_114 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_114, 0, x_28); +lean_ctor_set(x_114, 1, x_113); +lean_ctor_set(x_114, 2, x_112); +x_115 = lean_array_push(x_26, x_114); +x_116 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_116, 0, x_28); +lean_ctor_set(x_116, 1, x_54); +lean_ctor_set(x_116, 2, x_115); +x_117 = lean_array_push(x_50, x_69); +lean_inc(x_117); +x_118 = lean_array_push(x_117, x_116); +lean_inc(x_75); +x_119 = lean_array_push(x_118, x_75); +x_120 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__78; +x_121 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_121, 0, x_28); +lean_ctor_set(x_121, 1, x_120); +lean_ctor_set(x_121, 2, x_119); +x_122 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__99; lean_inc(x_19); -x_120 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_120, 0, x_19); -lean_ctor_set(x_120, 1, x_119); -x_121 = lean_array_push(x_38, x_118); -lean_inc(x_120); -x_122 = lean_array_push(x_121, x_120); -x_123 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__64; -x_124 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_124, 0, x_41); -lean_ctor_set(x_124, 1, x_123); -lean_ctor_set(x_124, 2, x_122); -x_125 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__91; +x_123 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_123, 0, x_19); +lean_ctor_set(x_123, 1, x_122); +x_124 = lean_array_push(x_43, x_121); +lean_inc(x_123); +x_125 = lean_array_push(x_124, x_123); +x_126 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__76; +x_127 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_127, 0, x_28); +lean_ctor_set(x_127, 1, x_126); +lean_ctor_set(x_127, 2, x_125); +x_128 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__103; lean_inc(x_22); lean_inc(x_23); -x_126 = l_Lean_addMacroScope(x_23, x_125, x_22); -x_127 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__90; +x_129 = l_Lean_addMacroScope(x_23, x_128, x_22); +x_130 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__102; lean_inc(x_19); -x_128 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_128, 0, x_19); -lean_ctor_set(x_128, 1, x_127); -lean_ctor_set(x_128, 2, x_126); -lean_ctor_set(x_128, 3, x_28); -x_129 = lean_array_push(x_38, x_128); -x_130 = lean_array_push(x_129, x_93); -x_131 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_131, 0, x_41); -lean_ctor_set(x_131, 1, x_95); -lean_ctor_set(x_131, 2, x_130); -x_132 = lean_array_push(x_80, x_131); -x_133 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_133, 0, x_41); -lean_ctor_set(x_133, 1, x_50); -lean_ctor_set(x_133, 2, x_132); -x_134 = lean_array_push(x_114, x_133); -x_135 = lean_array_push(x_134, x_71); +x_131 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_131, 0, x_19); +lean_ctor_set(x_131, 1, x_130); +lean_ctor_set(x_131, 2, x_129); +lean_ctor_set(x_131, 3, x_33); +x_132 = lean_array_push(x_43, x_131); +x_133 = lean_array_push(x_132, x_96); +x_134 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_134, 0, x_28); +lean_ctor_set(x_134, 1, x_98); +lean_ctor_set(x_134, 2, x_133); +x_135 = lean_array_push(x_26, x_134); x_136 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_136, 0, x_41); -lean_ctor_set(x_136, 1, x_117); +lean_ctor_set(x_136, 0, x_28); +lean_ctor_set(x_136, 1, x_54); lean_ctor_set(x_136, 2, x_135); -x_137 = lean_array_push(x_38, x_136); -x_138 = lean_array_push(x_137, x_120); +x_137 = lean_array_push(x_117, x_136); +x_138 = lean_array_push(x_137, x_75); x_139 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_139, 0, x_41); -lean_ctor_set(x_139, 1, x_123); +lean_ctor_set(x_139, 0, x_28); +lean_ctor_set(x_139, 1, x_120); lean_ctor_set(x_139, 2, x_138); -x_140 = lean_array_push(x_46, x_86); -x_141 = lean_array_push(x_140, x_124); -x_142 = lean_array_push(x_141, x_139); -x_143 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_143, 0, x_41); -lean_ctor_set(x_143, 1, x_50); -lean_ctor_set(x_143, 2, x_142); -x_144 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__95; -x_145 = l_Lean_addMacroScope(x_23, x_144, x_22); -x_146 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__94; -x_147 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_147, 0, x_19); -lean_ctor_set(x_147, 1, x_146); -lean_ctor_set(x_147, 2, x_145); -lean_ctor_set(x_147, 3, x_28); -x_148 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__98; -x_149 = lean_array_push(x_148, x_63); -x_150 = lean_array_push(x_149, x_93); -x_151 = lean_array_push(x_150, x_82); -x_152 = lean_array_push(x_151, x_93); -x_153 = lean_array_push(x_152, x_143); -x_154 = lean_array_push(x_153, x_32); -x_155 = lean_array_push(x_154, x_147); -x_156 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__47; -x_157 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_157, 0, x_41); -lean_ctor_set(x_157, 1, x_156); -lean_ctor_set(x_157, 2, x_155); -if (lean_obj_tag(x_57) == 0) -{ -lean_object* x_185; -x_185 = l_Lean_quoteNameMk(x_12); -x_158 = x_185; -goto block_184; -} -else -{ -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; +x_140 = lean_array_push(x_43, x_139); +x_141 = lean_array_push(x_140, x_123); +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_28); +lean_ctor_set(x_142, 1, x_126); +lean_ctor_set(x_142, 2, x_141); +x_143 = lean_array_push(x_50, x_89); +x_144 = lean_array_push(x_143, x_127); +x_145 = lean_array_push(x_144, x_142); +x_146 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_146, 0, x_28); +lean_ctor_set(x_146, 1, x_54); +lean_ctor_set(x_146, 2, x_145); +x_147 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__107; +x_148 = l_Lean_addMacroScope(x_23, x_147, x_22); +x_149 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__106; +x_150 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_150, 0, x_19); +lean_ctor_set(x_150, 1, x_149); +lean_ctor_set(x_150, 2, x_148); +lean_ctor_set(x_150, 3, x_33); +x_151 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__111; +x_152 = lean_array_push(x_151, x_67); +x_153 = lean_array_push(x_152, x_96); +x_154 = lean_array_push(x_153, x_85); +x_155 = lean_array_push(x_154, x_96); +x_156 = lean_array_push(x_155, x_146); +x_157 = lean_array_push(x_156, x_37); +x_158 = lean_array_push(x_157, x_150); +x_159 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__59; +x_160 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_160, 0, x_28); +lean_ctor_set(x_160, 1, x_159); +lean_ctor_set(x_160, 2, x_158); +if (lean_obj_tag(x_61) == 0) +{ +lean_object* x_188; +x_188 = l_Lean_quoteNameMk(x_12); +x_161 = x_188; +goto block_187; +} +else +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_dec(x_12); -x_186 = lean_ctor_get(x_57, 0); -lean_inc(x_186); -lean_dec(x_57); -x_187 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__101; -x_188 = l_String_intercalate(x_187, x_186); -x_189 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__102; -x_190 = lean_string_append(x_189, x_188); -lean_dec(x_188); -x_191 = l_Lean_Syntax_mkNameLit(x_190, x_41); -x_192 = lean_array_push(x_80, x_191); -x_193 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__100; -x_194 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_194, 0, x_41); -lean_ctor_set(x_194, 1, x_193); -lean_ctor_set(x_194, 2, x_192); -x_158 = x_194; -goto block_184; -} -block_184: -{ -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_159 = lean_array_push(x_38, x_158); -x_160 = lean_array_push(x_159, x_11); -x_161 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_161, 0, x_41); -lean_ctor_set(x_161, 1, x_50); -lean_ctor_set(x_161, 2, x_160); -x_162 = lean_array_push(x_58, x_161); -x_163 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__36; +x_189 = lean_ctor_get(x_61, 0); +lean_inc(x_189); +lean_dec(x_61); +x_190 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__114; +x_191 = l_String_intercalate(x_190, x_189); +x_192 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__115; +x_193 = lean_string_append(x_192, x_191); +lean_dec(x_191); +x_194 = l_Lean_Syntax_mkNameLit(x_193, x_28); +x_195 = lean_array_push(x_26, x_194); +x_196 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__113; +x_197 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_197, 0, x_28); +lean_ctor_set(x_197, 1, x_196); +lean_ctor_set(x_197, 2, x_195); +x_161 = x_197; +goto block_187; +} +block_187: +{ +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; +x_162 = lean_array_push(x_43, x_161); +x_163 = lean_array_push(x_162, x_11); x_164 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_164, 0, x_41); -lean_ctor_set(x_164, 1, x_163); -lean_ctor_set(x_164, 2, x_162); -x_165 = lean_array_push(x_80, x_164); -x_166 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__34; +lean_ctor_set(x_164, 0, x_28); +lean_ctor_set(x_164, 1, x_54); +lean_ctor_set(x_164, 2, x_163); +x_165 = lean_array_push(x_62, x_164); +x_166 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__48; x_167 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_167, 0, x_41); +lean_ctor_set(x_167, 0, x_28); lean_ctor_set(x_167, 1, x_166); lean_ctor_set(x_167, 2, x_165); -x_168 = lean_array_push(x_38, x_167); -x_169 = lean_array_push(x_168, x_93); -x_170 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__32; -x_171 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_171, 0, x_41); -lean_ctor_set(x_171, 1, x_170); -lean_ctor_set(x_171, 2, x_169); -x_172 = lean_array_push(x_80, x_171); -x_173 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_173, 0, x_41); -lean_ctor_set(x_173, 1, x_50); -lean_ctor_set(x_173, 2, x_172); -x_174 = lean_array_push(x_80, x_173); -x_175 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__30; +x_168 = lean_array_push(x_26, x_167); +x_169 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__46; +x_170 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_170, 0, x_28); +lean_ctor_set(x_170, 1, x_169); +lean_ctor_set(x_170, 2, x_168); +x_171 = lean_array_push(x_43, x_170); +x_172 = lean_array_push(x_171, x_96); +x_173 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__44; +x_174 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_174, 0, x_28); +lean_ctor_set(x_174, 1, x_173); +lean_ctor_set(x_174, 2, x_172); +x_175 = lean_array_push(x_26, x_174); x_176 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_176, 0, x_41); -lean_ctor_set(x_176, 1, x_175); -lean_ctor_set(x_176, 2, x_174); -x_177 = lean_array_push(x_61, x_176); -x_178 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__9; +lean_ctor_set(x_176, 0, x_28); +lean_ctor_set(x_176, 1, x_54); +lean_ctor_set(x_176, 2, x_175); +x_177 = lean_array_push(x_26, x_176); +x_178 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__42; x_179 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_179, 0, x_41); +lean_ctor_set(x_179, 0, x_28); lean_ctor_set(x_179, 1, x_178); lean_ctor_set(x_179, 2, x_177); -x_180 = lean_array_push(x_38, x_179); -x_181 = lean_array_push(x_180, x_157); +x_180 = lean_array_push(x_65, x_179); +x_181 = l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__9; x_182 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_182, 0, x_41); -lean_ctor_set(x_182, 1, x_50); -lean_ctor_set(x_182, 2, x_181); +lean_ctor_set(x_182, 0, x_28); +lean_ctor_set(x_182, 1, x_181); +lean_ctor_set(x_182, 2, x_180); +x_183 = lean_array_push(x_43, x_182); +x_184 = lean_array_push(x_183, x_160); +x_185 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_185, 0, x_28); +lean_ctor_set(x_185, 1, x_54); +lean_ctor_set(x_185, 2, x_184); if (lean_is_scalar(x_21)) { - x_183 = lean_alloc_ctor(0, 2, 0); + x_186 = lean_alloc_ctor(0, 2, 0); } else { - x_183 = x_21; + x_186 = x_21; } -lean_ctor_set(x_183, 0, x_182); -lean_ctor_set(x_183, 1, x_20); -return x_183; +lean_ctor_set(x_186, 0, x_185); +lean_ctor_set(x_186, 1, x_20); +return x_186; } } } @@ -18107,6 +18319,32 @@ l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean_ lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__101); l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__102 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__102(); lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__102); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__103 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__103(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__103); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__104 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__104(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__104); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__105 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__105(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__105); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__106 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__106(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__106); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__107 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__107(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__107); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__108 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__108(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__108); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__109 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__109(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__109); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__110 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__110(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__110); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__111 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__111(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__111); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__112 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__112(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__112); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__113 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__113(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__113); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__114 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__114(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__114); +l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__115 = _init_l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__115(); +lean_mark_persistent(l_Lean_Meta___aux__Lean__Meta__Tactic__Simp__SimpTheorems______macroRules__Lean__Meta__commandRegister__simp__attr______1___closed__115); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Meta/Tactic/Split.c b/stage0/stdlib/Lean/Meta/Tactic/Split.c index 784be51d2fa1..4aa282b9975c 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Split.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Split.c @@ -179,6 +179,7 @@ static lean_object* l_Lean_Meta_Split_applyMatchSplitter___lambda__3___closed__1 LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_generalizeMatchDiscrs_mkNewTarget___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); static lean_object* l_Lean_Meta_splitTarget_x3f_go___closed__3; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Split_applyMatchSplitter___lambda__3___closed__2; lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_generalizeMatchDiscrs___lambda__7___closed__1; @@ -241,7 +242,6 @@ static lean_object* l_Lean_Meta_Split_applyMatchSplitter___lambda__9___closed__1 LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Meta_Split_splitMatch___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Split_applyMatchSplitter___lambda__8(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_Lean_Meta_applySimpResultToTarget(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Split_splitMatch___closed__5; static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_generalizeMatchDiscrs_mkNewTarget___spec__1___closed__11; @@ -1966,7 +1966,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_withEqs_go___rarg___closed__3; x_2 = l___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_withEqs_go___rarg___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Meta_Tactic_Split_0__Lean_Meta_Split_withEqs_go___rarg___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4906,7 +4906,7 @@ else { lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_8, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_8, x_17); x_19 = l_Lean_Meta_Match_MatcherInfo_arity(x_4); x_20 = lean_nat_dec_eq(x_18, x_19); lean_dec(x_19); @@ -9864,7 +9864,7 @@ x_9 = lean_ctor_get(x_6, 0); lean_inc(x_9); lean_dec(x_6); x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_4, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_4, x_10); x_12 = l_Lean_Meta_Split_findSplit_x3f_isCandidate___closed__1; lean_inc(x_11); x_13 = lean_mk_array(x_11, x_12); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Subst.c b/stage0/stdlib/Lean/Meta/Tactic/Subst.c index c2e0df131693..9a75ed3654bc 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Subst.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Subst.c @@ -301,7 +301,7 @@ static lean_object* _init_l_Nat_foldM_loop___at_Lean_Meta_substCore___spec__1___ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Nat_foldM_loop___at_Lean_Meta_substCore___spec__1___closed__1; x_2 = l_Nat_foldM_loop___at_Lean_Meta_substCore___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Nat_foldM_loop___at_Lean_Meta_substCore___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Transform.c b/stage0/stdlib/Lean/Meta/Transform.c index aed371f5a291..94a954c6fcc0 100644 --- a/stage0/stdlib/Lean/Meta/Transform.c +++ b/stage0/stdlib/Lean/Meta/Transform.c @@ -15,7 +15,6 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lean_Core_withIncRecDepth___at_Lean_Core_transform_visit___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLetFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_eraseInaccessibleAnnotations___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -25,6 +24,7 @@ size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Core_transform_visit___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Core_transform_visit___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Core_betaReduce___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Core_transform(lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -33,12 +33,13 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_zetaReduce___s lean_object* l_Lean_Meta_mkForallFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_transform_visit___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_zetaReduce___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -57,6 +58,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet(lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Core_transform_visit___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Core_betaReduce___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -66,6 +68,7 @@ static lean_object* l_Lean_Core_transform_visit___rarg___lambda__6___closed__3; LEAN_EXPORT lean_object* l_Lean_Core_transform___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___at_Lean_Meta_zetaReduce___spec__5(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_Core_betaReduce___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_transform_visit___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); @@ -164,6 +167,7 @@ LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Meta_transform_visit___spec__3 LEAN_EXPORT lean_object* l_Lean_Core_transform___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withIncRecDepth___at_Lean_Meta_zetaReduce___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Core_betaReduce___closed__2; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Core_betaReduce___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_transform_visit___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_transform_visit_visitForall___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -204,7 +208,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec_ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_transform_visit___spec__2___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_transform_visit_visitLambda___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -214,7 +217,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda___at_Lean_Meta_ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_transform_visit_visitForall___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Core_transform_visit___rarg___lambda__9___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -225,10 +227,10 @@ lean_object* l_Lean_LocalDecl_value_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_transform_visit_visitLambda___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withIncRecDepth___at_Lean_Meta_transform_visit___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Core_transform_visit___rarg___lambda__9___closed__1; +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLetDecl___at_Lean_Meta_zetaReduce___spec__9(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform___rarg___lambda__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLambda___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___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*); @@ -268,7 +270,6 @@ uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Core_transform_visit___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___at_Lean_Meta_zetaReduce___spec__2___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars___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_throwMaxRecDepthAt___at_Lean_Core_transform_visit___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -286,6 +287,7 @@ LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_zetaReduce___s LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitForall(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_zetaReduce(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_eraseInaccessibleAnnotations___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -294,6 +296,7 @@ static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Core_transform_visit___s LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_transform___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Core_transform_visit___rarg___lambda__10___closed__3; LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_zetaReduce___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -776,8 +779,8 @@ static lean_object* _init_l_Lean_Core_transform_visit___rarg___lambda__2___close lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__1; x_2 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__2; -x_3 = lean_unsigned_to_nat(1149u); -x_4 = lean_unsigned_to_nat(19u); +x_3 = lean_unsigned_to_nat(1491u); +x_4 = lean_unsigned_to_nat(20u); x_5 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -788,22 +791,81 @@ LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg___lambda__2(lean_obj { if (lean_obj_tag(x_1) == 6) { -uint8_t x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_12 = lean_expr_update_lambda(x_1, x_11, x_9, x_10); -x_13 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_12, x_8); -return x_13; +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; size_t x_16; size_t x_17; uint8_t x_18; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +x_13 = lean_ctor_get(x_1, 2); +lean_inc(x_13); +x_14 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_15 = l_Lean_Expr_lam___override(x_11, x_12, x_13, x_14); +x_16 = lean_ptr_addr(x_12); +lean_dec(x_12); +x_17 = lean_ptr_addr(x_9); +x_18 = lean_usize_dec_eq(x_16, x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_15); +lean_dec(x_13); +x_19 = l_Lean_Expr_lam___override(x_11, x_9, x_10, x_14); +x_20 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_19, x_8); +return x_20; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +size_t x_21; size_t x_22; uint8_t x_23; +x_21 = lean_ptr_addr(x_13); +lean_dec(x_13); +x_22 = lean_ptr_addr(x_10); +x_23 = lean_usize_dec_eq(x_21, x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_15); +x_24 = l_Lean_Expr_lam___override(x_11, x_9, x_10, x_14); +x_25 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_24, x_8); +return x_25; +} +else +{ +uint8_t x_26; +x_26 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_14, x_14); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +lean_dec(x_15); +x_27 = l_Lean_Expr_lam___override(x_11, x_9, x_10, x_14); +x_28 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_27, x_8); +return x_28; +} +else +{ +lean_object* x_29; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_29 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_15, x_8); +return x_29; +} +} +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_dec(x_10); lean_dec(x_9); lean_dec(x_1); -x_14 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__4; -x_15 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_14); -x_16 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_15, x_8); -return x_16; +x_30 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__4; +x_31 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_30); +x_32 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_31, x_8); +return x_32; } } } @@ -855,8 +917,8 @@ static lean_object* _init_l_Lean_Core_transform_visit___rarg___lambda__4___close lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__1; x_2 = l_Lean_Core_transform_visit___rarg___lambda__4___closed__1; -x_3 = lean_unsigned_to_nat(1135u); -x_4 = lean_unsigned_to_nat(23u); +x_3 = lean_unsigned_to_nat(1471u); +x_4 = lean_unsigned_to_nat(24u); x_5 = l_Lean_Core_transform_visit___rarg___lambda__4___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -867,22 +929,81 @@ LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg___lambda__4(lean_obj { if (lean_obj_tag(x_1) == 7) { -uint8_t x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_12 = lean_expr_update_forall(x_1, x_11, x_9, x_10); -x_13 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_12, x_8); -return x_13; +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; size_t x_16; size_t x_17; uint8_t x_18; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +x_13 = lean_ctor_get(x_1, 2); +lean_inc(x_13); +x_14 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_dec(x_1); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +x_15 = l_Lean_Expr_forallE___override(x_11, x_12, x_13, x_14); +x_16 = lean_ptr_addr(x_12); +lean_dec(x_12); +x_17 = lean_ptr_addr(x_9); +x_18 = lean_usize_dec_eq(x_16, x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_15); +lean_dec(x_13); +x_19 = l_Lean_Expr_forallE___override(x_11, x_9, x_10, x_14); +x_20 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_19, x_8); +return x_20; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +size_t x_21; size_t x_22; uint8_t x_23; +x_21 = lean_ptr_addr(x_13); +lean_dec(x_13); +x_22 = lean_ptr_addr(x_10); +x_23 = lean_usize_dec_eq(x_21, x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_15); +x_24 = l_Lean_Expr_forallE___override(x_11, x_9, x_10, x_14); +x_25 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_24, x_8); +return x_25; +} +else +{ +uint8_t x_26; +x_26 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_14, x_14); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +lean_dec(x_15); +x_27 = l_Lean_Expr_forallE___override(x_11, x_9, x_10, x_14); +x_28 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_27, x_8); +return x_28; +} +else +{ +lean_object* x_29; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_29 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_15, x_8); +return x_29; +} +} +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_dec(x_10); lean_dec(x_9); lean_dec(x_1); -x_14 = l_Lean_Core_transform_visit___rarg___lambda__4___closed__3; -x_15 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_14); -x_16 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_15, x_8); -return x_16; +x_30 = l_Lean_Core_transform_visit___rarg___lambda__4___closed__3; +x_31 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_30); +x_32 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_31, x_8); +return x_32; } } } @@ -916,7 +1037,7 @@ static lean_object* _init_l_Lean_Core_transform_visit___rarg___lambda__6___close _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateLet!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateLet!Impl", 45); return x_1; } } @@ -934,8 +1055,8 @@ static lean_object* _init_l_Lean_Core_transform_visit___rarg___lambda__6___close lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__1; x_2 = l_Lean_Core_transform_visit___rarg___lambda__6___closed__1; -x_3 = lean_unsigned_to_nat(1158u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1500u); +x_4 = lean_unsigned_to_nat(22u); x_5 = l_Lean_Core_transform_visit___rarg___lambda__6___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -946,22 +1067,85 @@ LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg___lambda__6(lean_obj { if (lean_obj_tag(x_1) == 8) { -lean_object* x_12; lean_object* x_13; -x_12 = lean_expr_update_let(x_1, x_9, x_10, x_11); -x_13 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_12, x_8); -return x_13; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; size_t x_17; size_t x_18; uint8_t x_19; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +x_14 = lean_ctor_get(x_1, 2); +lean_inc(x_14); +x_15 = lean_ctor_get(x_1, 3); +lean_inc(x_15); +x_16 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); +x_17 = lean_ptr_addr(x_13); +lean_dec(x_13); +x_18 = lean_ptr_addr(x_9); +x_19 = lean_usize_dec_eq(x_17, x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_1); +x_20 = l_Lean_Expr_letE___override(x_12, x_9, x_10, x_11, x_16); +x_21 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_20, x_8); +return x_21; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +size_t x_22; size_t x_23; uint8_t x_24; +x_22 = lean_ptr_addr(x_14); +lean_dec(x_14); +x_23 = lean_ptr_addr(x_10); +x_24 = lean_usize_dec_eq(x_22, x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_15); +lean_dec(x_1); +x_25 = l_Lean_Expr_letE___override(x_12, x_9, x_10, x_11, x_16); +x_26 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_25, x_8); +return x_26; +} +else +{ +size_t x_27; size_t x_28; uint8_t x_29; +x_27 = lean_ptr_addr(x_15); +lean_dec(x_15); +x_28 = lean_ptr_addr(x_11); +x_29 = lean_usize_dec_eq(x_27, x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; +lean_dec(x_1); +x_30 = l_Lean_Expr_letE___override(x_12, x_9, x_10, x_11, x_16); +x_31 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_30, x_8); +return x_31; +} +else +{ +lean_object* x_32; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_32 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_1, x_8); +return x_32; +} +} +} +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_1); -x_14 = l_Lean_Core_transform_visit___rarg___lambda__6___closed__3; -x_15 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_14); -x_16 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_15, x_8); -return x_16; +x_33 = l_Lean_Core_transform_visit___rarg___lambda__6___closed__3; +x_34 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_33); +x_35 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_34, x_8); +return x_35; } } } @@ -1025,7 +1209,7 @@ static lean_object* _init_l_Lean_Core_transform_visit___rarg___lambda__9___close _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateMData!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateMData!Impl", 47); return x_1; } } @@ -1043,8 +1227,8 @@ static lean_object* _init_l_Lean_Core_transform_visit___rarg___lambda__9___close lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__1; x_2 = l_Lean_Core_transform_visit___rarg___lambda__9___closed__1; -x_3 = lean_unsigned_to_nat(1116u); -x_4 = lean_unsigned_to_nat(16u); +x_3 = lean_unsigned_to_nat(1434u); +x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_Core_transform_visit___rarg___lambda__9___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -1055,20 +1239,41 @@ LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg___lambda__9(lean_obj { if (lean_obj_tag(x_1) == 10) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_expr_update_mdata(x_1, x_9); -x_11 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_10, x_8); -return x_11; +lean_object* x_10; lean_object* x_11; size_t x_12; size_t x_13; uint8_t x_14; +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_ptr_addr(x_11); +lean_dec(x_11); +x_13 = lean_ptr_addr(x_9); +x_14 = lean_usize_dec_eq(x_12, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = l_Lean_Expr_mdata___override(x_10, x_9); +x_16 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_15, x_8); +return x_16; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_17; +lean_dec(x_10); +lean_dec(x_9); +x_17 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_1, x_8); +return x_17; +} +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_dec(x_9); lean_dec(x_1); -x_12 = l_Lean_Core_transform_visit___rarg___lambda__9___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_13, x_8); -return x_14; +x_18 = l_Lean_Core_transform_visit___rarg___lambda__9___closed__3; +x_19 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_18); +x_20 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_19, x_8); +return x_20; } } } @@ -1076,7 +1281,7 @@ static lean_object* _init_l_Lean_Core_transform_visit___rarg___lambda__10___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateProj!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateProj!Impl", 46); return x_1; } } @@ -1094,8 +1299,8 @@ static lean_object* _init_l_Lean_Core_transform_visit___rarg___lambda__10___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Core_transform_visit___rarg___lambda__2___closed__1; x_2 = l_Lean_Core_transform_visit___rarg___lambda__10___closed__1; -x_3 = lean_unsigned_to_nat(1121u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1445u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_Core_transform_visit___rarg___lambda__10___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -1106,20 +1311,44 @@ LEAN_EXPORT lean_object* l_Lean_Core_transform_visit___rarg___lambda__10(lean_ob { if (lean_obj_tag(x_1) == 11) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_expr_update_proj(x_1, x_9); -x_11 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_10, x_8); -return x_11; +lean_object* x_10; lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; uint8_t x_15; +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_ctor_get(x_1, 2); +lean_inc(x_12); +x_13 = lean_ptr_addr(x_12); +lean_dec(x_12); +x_14 = lean_ptr_addr(x_9); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_1); +x_16 = l_Lean_Expr_proj___override(x_10, x_11, x_9); +x_17 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_16, x_8); +return x_17; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_18; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_18 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_1, x_8); +return x_18; +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_dec(x_9); lean_dec(x_1); -x_12 = l_Lean_Core_transform_visit___rarg___lambda__10___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_13, x_8); -return x_14; +x_19 = l_Lean_Core_transform_visit___rarg___lambda__10___closed__3; +x_20 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_19); +x_21 = l_Lean_Core_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_20, x_8); +return x_21; } } } @@ -1168,7 +1397,7 @@ case 5: { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_14, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_14, x_15); x_17 = l_Lean_Core_transform_visit___rarg___lambda__11___closed__1; lean_inc(x_16); x_18 = lean_mk_array(x_16, x_17); @@ -2479,7 +2708,7 @@ case 5: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_12, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_12, x_13); x_15 = l_Lean_Core_transform_visit___rarg___lambda__11___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -2491,53 +2720,112 @@ return x_19; } case 6: { -lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_12, 1); +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; +x_20 = lean_ctor_get(x_12, 0); lean_inc(x_20); -x_21 = lean_ctor_get(x_12, 2); +x_21 = lean_ctor_get(x_12, 1); lean_inc(x_21); -x_22 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 8); +x_22 = lean_ctor_get(x_12, 2); +lean_inc(x_22); +x_23 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 8); +lean_dec(x_12); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_21); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_23 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_20, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_23) == 0) +x_24 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_21, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_dec(x_23); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_22); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_26 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_21, x_6, x_7, x_8, x_25); -if (lean_obj_tag(x_26) == 0) +x_27 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_22, x_6, x_7, x_8, x_26); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); +lean_object* x_28; lean_object* x_29; lean_object* x_30; size_t x_31; size_t x_32; uint8_t x_33; +x_28 = lean_ctor_get(x_27, 0); lean_inc(x_28); -lean_dec(x_26); -x_29 = lean_expr_update_lambda(x_12, x_22, x_24, x_27); -x_30 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_29, x_6, x_7, x_8, x_28); -return x_30; +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +lean_inc(x_22); +lean_inc(x_21); +lean_inc(x_20); +x_30 = l_Lean_Expr_lam___override(x_20, x_21, x_22, x_23); +x_31 = lean_ptr_addr(x_21); +lean_dec(x_21); +x_32 = lean_ptr_addr(x_25); +x_33 = lean_usize_dec_eq(x_31, x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_30); +lean_dec(x_22); +x_34 = l_Lean_Expr_lam___override(x_20, x_25, x_28, x_23); +x_35 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_34, x_6, x_7, x_8, x_29); +return x_35; } else { -uint8_t x_31; -lean_dec(x_24); -lean_dec(x_12); +size_t x_36; size_t x_37; uint8_t x_38; +x_36 = lean_ptr_addr(x_22); +lean_dec(x_22); +x_37 = lean_ptr_addr(x_28); +x_38 = lean_usize_dec_eq(x_36, x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +lean_dec(x_30); +x_39 = l_Lean_Expr_lam___override(x_20, x_25, x_28, x_23); +x_40 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_39, x_6, x_7, x_8, x_29); +return x_40; +} +else +{ +uint8_t x_41; +x_41 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_23, x_23); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +lean_dec(x_30); +x_42 = l_Lean_Expr_lam___override(x_20, x_25, x_28, x_23); +x_43 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_42, x_6, x_7, x_8, x_29); +return x_43; +} +else +{ +lean_object* x_44; +lean_dec(x_28); +lean_dec(x_25); +lean_dec(x_20); +x_44 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_30, x_6, x_7, x_8, x_29); +return x_44; +} +} +} +} +else +{ +uint8_t x_45; +lean_dec(x_25); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2545,31 +2833,32 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_31 = !lean_is_exclusive(x_26); -if (x_31 == 0) +x_45 = !lean_is_exclusive(x_27); +if (x_45 == 0) { -return x_26; +return x_27; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_26, 0); -x_33 = lean_ctor_get(x_26, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_26); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_27, 0); +x_47 = lean_ctor_get(x_27, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_27); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; } } } else { -uint8_t x_35; +uint8_t x_49; +lean_dec(x_22); lean_dec(x_21); -lean_dec(x_12); +lean_dec(x_20); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2577,75 +2866,134 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_35 = !lean_is_exclusive(x_23); -if (x_35 == 0) +x_49 = !lean_is_exclusive(x_24); +if (x_49 == 0) { -return x_23; +return x_24; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_23, 0); -x_37 = lean_ctor_get(x_23, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_23); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_24, 0); +x_51 = lean_ctor_get(x_24, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_24); +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; } } } case 7: { -lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; -x_39 = lean_ctor_get(x_12, 1); -lean_inc(x_39); -x_40 = lean_ctor_get(x_12, 2); -lean_inc(x_40); -x_41 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 8); +lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; +x_53 = lean_ctor_get(x_12, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_12, 1); +lean_inc(x_54); +x_55 = lean_ctor_get(x_12, 2); +lean_inc(x_55); +x_56 = lean_ctor_get_uint8(x_12, sizeof(void*)*3 + 8); +lean_dec(x_12); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_54); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_42 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_39, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_42) == 0) +x_57 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_54, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_57) == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_57, 1); +lean_inc(x_59); +lean_dec(x_57); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_55); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_45 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_40, x_6, x_7, x_8, x_44); -if (lean_obj_tag(x_45) == 0) +x_60 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_55, x_6, x_7, x_8, x_59); +if (lean_obj_tag(x_60) == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_48 = lean_expr_update_forall(x_12, x_41, x_43, x_46); -x_49 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_48, x_6, x_7, x_8, x_47); -return x_49; +lean_object* x_61; lean_object* x_62; lean_object* x_63; size_t x_64; size_t x_65; uint8_t x_66; +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_60, 1); +lean_inc(x_62); +lean_dec(x_60); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +x_63 = l_Lean_Expr_forallE___override(x_53, x_54, x_55, x_56); +x_64 = lean_ptr_addr(x_54); +lean_dec(x_54); +x_65 = lean_ptr_addr(x_58); +x_66 = lean_usize_dec_eq(x_64, x_65); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_dec(x_63); +lean_dec(x_55); +x_67 = l_Lean_Expr_forallE___override(x_53, x_58, x_61, x_56); +x_68 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_67, x_6, x_7, x_8, x_62); +return x_68; } else { -uint8_t x_50; -lean_dec(x_43); -lean_dec(x_12); +size_t x_69; size_t x_70; uint8_t x_71; +x_69 = lean_ptr_addr(x_55); +lean_dec(x_55); +x_70 = lean_ptr_addr(x_61); +x_71 = lean_usize_dec_eq(x_69, x_70); +if (x_71 == 0) +{ +lean_object* x_72; lean_object* x_73; +lean_dec(x_63); +x_72 = l_Lean_Expr_forallE___override(x_53, x_58, x_61, x_56); +x_73 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_72, x_6, x_7, x_8, x_62); +return x_73; +} +else +{ +uint8_t x_74; +x_74 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_56, x_56); +if (x_74 == 0) +{ +lean_object* x_75; lean_object* x_76; +lean_dec(x_63); +x_75 = l_Lean_Expr_forallE___override(x_53, x_58, x_61, x_56); +x_76 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_75, x_6, x_7, x_8, x_62); +return x_76; +} +else +{ +lean_object* x_77; +lean_dec(x_61); +lean_dec(x_58); +lean_dec(x_53); +x_77 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_63, x_6, x_7, x_8, x_62); +return x_77; +} +} +} +} +else +{ +uint8_t x_78; +lean_dec(x_58); +lean_dec(x_55); +lean_dec(x_54); +lean_dec(x_53); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2653,31 +3001,32 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_50 = !lean_is_exclusive(x_45); -if (x_50 == 0) +x_78 = !lean_is_exclusive(x_60); +if (x_78 == 0) { -return x_45; +return x_60; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_45, 0); -x_52 = lean_ctor_get(x_45, 1); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_45); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_51); -lean_ctor_set(x_53, 1, x_52); -return x_53; +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_60, 0); +x_80 = lean_ctor_get(x_60, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_60); +x_81 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +return x_81; } } } else { -uint8_t x_54; -lean_dec(x_40); -lean_dec(x_12); +uint8_t x_82; +lean_dec(x_55); +lean_dec(x_54); +lean_dec(x_53); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -2685,92 +3034,156 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_54 = !lean_is_exclusive(x_42); -if (x_54 == 0) +x_82 = !lean_is_exclusive(x_57); +if (x_82 == 0) { -return x_42; +return x_57; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_42, 0); -x_56 = lean_ctor_get(x_42, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_42); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -return x_57; +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_57, 0); +x_84 = lean_ctor_get(x_57, 1); +lean_inc(x_84); +lean_inc(x_83); +lean_dec(x_57); +x_85 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +return x_85; } } } case 8: { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_58 = lean_ctor_get(x_12, 1); -lean_inc(x_58); -x_59 = lean_ctor_get(x_12, 2); -lean_inc(x_59); -x_60 = lean_ctor_get(x_12, 3); -lean_inc(x_60); +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; lean_object* x_91; +x_86 = lean_ctor_get(x_12, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_12, 1); +lean_inc(x_87); +x_88 = lean_ctor_get(x_12, 2); +lean_inc(x_88); +x_89 = lean_ctor_get(x_12, 3); +lean_inc(x_89); +x_90 = lean_ctor_get_uint8(x_12, sizeof(void*)*4 + 8); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_87); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_61 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_58, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_61) == 0) +x_91 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_87, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_91) == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); +lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_91, 1); +lean_inc(x_93); +lean_dec(x_91); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_88); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_64 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_59, x_6, x_7, x_8, x_63); -if (lean_obj_tag(x_64) == 0) +x_94 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_88, x_6, x_7, x_8, x_93); +if (lean_obj_tag(x_94) == 0) { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_64, 1); -lean_inc(x_66); -lean_dec(x_64); +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +lean_dec(x_94); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_89); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_67 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_60, x_6, x_7, x_8, x_66); -if (lean_obj_tag(x_67) == 0) +x_97 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_89, x_6, x_7, x_8, x_96); +if (lean_obj_tag(x_97) == 0) +{ +lean_object* x_98; lean_object* x_99; size_t x_100; size_t x_101; uint8_t x_102; +x_98 = lean_ctor_get(x_97, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_97, 1); +lean_inc(x_99); +lean_dec(x_97); +x_100 = lean_ptr_addr(x_87); +lean_dec(x_87); +x_101 = lean_ptr_addr(x_92); +x_102 = lean_usize_dec_eq(x_100, x_101); +if (x_102 == 0) +{ +lean_object* x_103; lean_object* x_104; +lean_dec(x_89); +lean_dec(x_88); +lean_dec(x_12); +x_103 = l_Lean_Expr_letE___override(x_86, x_92, x_95, x_98, x_90); +x_104 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_103, x_6, x_7, x_8, x_99); +return x_104; +} +else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_expr_update_let(x_12, x_62, x_65, x_68); -x_71 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_70, x_6, x_7, x_8, x_69); -return x_71; +size_t x_105; size_t x_106; uint8_t x_107; +x_105 = lean_ptr_addr(x_88); +lean_dec(x_88); +x_106 = lean_ptr_addr(x_95); +x_107 = lean_usize_dec_eq(x_105, x_106); +if (x_107 == 0) +{ +lean_object* x_108; lean_object* x_109; +lean_dec(x_89); +lean_dec(x_12); +x_108 = l_Lean_Expr_letE___override(x_86, x_92, x_95, x_98, x_90); +x_109 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_108, x_6, x_7, x_8, x_99); +return x_109; +} +else +{ +size_t x_110; size_t x_111; uint8_t x_112; +x_110 = lean_ptr_addr(x_89); +lean_dec(x_89); +x_111 = lean_ptr_addr(x_98); +x_112 = lean_usize_dec_eq(x_110, x_111); +if (x_112 == 0) +{ +lean_object* x_113; lean_object* x_114; +lean_dec(x_12); +x_113 = l_Lean_Expr_letE___override(x_86, x_92, x_95, x_98, x_90); +x_114 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_113, x_6, x_7, x_8, x_99); +return x_114; +} +else +{ +lean_object* x_115; +lean_dec(x_98); +lean_dec(x_95); +lean_dec(x_92); +lean_dec(x_86); +x_115 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_12, x_6, x_7, x_8, x_99); +return x_115; +} +} +} } else { -uint8_t x_72; -lean_dec(x_65); -lean_dec(x_62); +uint8_t x_116; +lean_dec(x_95); +lean_dec(x_92); +lean_dec(x_89); +lean_dec(x_88); +lean_dec(x_87); +lean_dec(x_86); lean_dec(x_12); lean_dec(x_8); lean_dec(x_7); @@ -2779,31 +3192,34 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_72 = !lean_is_exclusive(x_67); -if (x_72 == 0) +x_116 = !lean_is_exclusive(x_97); +if (x_116 == 0) { -return x_67; +return x_97; } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_67, 0); -x_74 = lean_ctor_get(x_67, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_67); -x_75 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -return x_75; +lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_117 = lean_ctor_get(x_97, 0); +x_118 = lean_ctor_get(x_97, 1); +lean_inc(x_118); +lean_inc(x_117); +lean_dec(x_97); +x_119 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_119, 0, x_117); +lean_ctor_set(x_119, 1, x_118); +return x_119; } } } else { -uint8_t x_76; -lean_dec(x_62); -lean_dec(x_60); +uint8_t x_120; +lean_dec(x_92); +lean_dec(x_89); +lean_dec(x_88); +lean_dec(x_87); +lean_dec(x_86); lean_dec(x_12); lean_dec(x_8); lean_dec(x_7); @@ -2812,31 +3228,33 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_76 = !lean_is_exclusive(x_64); -if (x_76 == 0) +x_120 = !lean_is_exclusive(x_94); +if (x_120 == 0) { -return x_64; +return x_94; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_64, 0); -x_78 = lean_ctor_get(x_64, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_64); -x_79 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_79, 0, x_77); -lean_ctor_set(x_79, 1, x_78); -return x_79; +lean_object* x_121; lean_object* x_122; lean_object* x_123; +x_121 = lean_ctor_get(x_94, 0); +x_122 = lean_ctor_get(x_94, 1); +lean_inc(x_122); +lean_inc(x_121); +lean_dec(x_94); +x_123 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_123, 0, x_121); +lean_ctor_set(x_123, 1, x_122); +return x_123; } } } else { -uint8_t x_80; -lean_dec(x_60); -lean_dec(x_59); +uint8_t x_124; +lean_dec(x_89); +lean_dec(x_88); +lean_dec(x_87); +lean_dec(x_86); lean_dec(x_12); lean_dec(x_8); lean_dec(x_7); @@ -2845,54 +3263,76 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_80 = !lean_is_exclusive(x_61); -if (x_80 == 0) +x_124 = !lean_is_exclusive(x_91); +if (x_124 == 0) { -return x_61; +return x_91; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_61, 0); -x_82 = lean_ctor_get(x_61, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_61); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -return x_83; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_91, 0); +x_126 = lean_ctor_get(x_91, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_91); +x_127 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_126); +return x_127; } } } case 10: { -lean_object* x_84; lean_object* x_85; -x_84 = lean_ctor_get(x_12, 1); -lean_inc(x_84); +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_12, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_12, 1); +lean_inc(x_129); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_129); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_85 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_84, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_85) == 0) +x_130 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_129, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_130) == 0) +{ +lean_object* x_131; lean_object* x_132; size_t x_133; size_t x_134; uint8_t x_135; +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_130, 1); +lean_inc(x_132); +lean_dec(x_130); +x_133 = lean_ptr_addr(x_129); +lean_dec(x_129); +x_134 = lean_ptr_addr(x_131); +x_135 = lean_usize_dec_eq(x_133, x_134); +if (x_135 == 0) +{ +lean_object* x_136; lean_object* x_137; +lean_dec(x_12); +x_136 = l_Lean_Expr_mdata___override(x_128, x_131); +x_137 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_136, x_6, x_7, x_8, x_132); +return x_137; +} +else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_86 = lean_ctor_get(x_85, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_85, 1); -lean_inc(x_87); -lean_dec(x_85); -x_88 = lean_expr_update_mdata(x_12, x_86); -x_89 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_88, x_6, x_7, x_8, x_87); -return x_89; +lean_object* x_138; +lean_dec(x_131); +lean_dec(x_128); +x_138 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_12, x_6, x_7, x_8, x_132); +return x_138; +} } else { -uint8_t x_90; +uint8_t x_139; +lean_dec(x_129); +lean_dec(x_128); lean_dec(x_12); lean_dec(x_8); lean_dec(x_7); @@ -2901,54 +3341,80 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_90 = !lean_is_exclusive(x_85); -if (x_90 == 0) +x_139 = !lean_is_exclusive(x_130); +if (x_139 == 0) { -return x_85; +return x_130; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_85, 0); -x_92 = lean_ctor_get(x_85, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_85); -x_93 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_93, 0, x_91); -lean_ctor_set(x_93, 1, x_92); -return x_93; +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_130, 0); +x_141 = lean_ctor_get(x_130, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_130); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } } case 11: { -lean_object* x_94; lean_object* x_95; -x_94 = lean_ctor_get(x_12, 2); -lean_inc(x_94); +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_143 = lean_ctor_get(x_12, 0); +lean_inc(x_143); +x_144 = lean_ctor_get(x_12, 1); +lean_inc(x_144); +x_145 = lean_ctor_get(x_12, 2); +lean_inc(x_145); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); +lean_inc(x_145); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_95 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_94, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_95) == 0) +x_146 = l_Lean_Core_transform_visit___at_Lean_Core_betaReduce___spec__2(x_1, x_2, x_3, x_4, x_145, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_146) == 0) +{ +lean_object* x_147; lean_object* x_148; size_t x_149; size_t x_150; uint8_t x_151; +x_147 = lean_ctor_get(x_146, 0); +lean_inc(x_147); +x_148 = lean_ctor_get(x_146, 1); +lean_inc(x_148); +lean_dec(x_146); +x_149 = lean_ptr_addr(x_145); +lean_dec(x_145); +x_150 = lean_ptr_addr(x_147); +x_151 = lean_usize_dec_eq(x_149, x_150); +if (x_151 == 0) +{ +lean_object* x_152; lean_object* x_153; +lean_dec(x_12); +x_152 = l_Lean_Expr_proj___override(x_143, x_144, x_147); +x_153 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_152, x_6, x_7, x_8, x_148); +return x_153; +} +else { -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; -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 = lean_expr_update_proj(x_12, x_96); -x_99 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_98, x_6, x_7, x_8, x_97); -return x_99; +lean_object* x_154; +lean_dec(x_147); +lean_dec(x_144); +lean_dec(x_143); +x_154 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_12, x_6, x_7, x_8, x_148); +return x_154; +} } else { -uint8_t x_100; +uint8_t x_155; +lean_dec(x_145); +lean_dec(x_144); +lean_dec(x_143); lean_dec(x_12); lean_dec(x_8); lean_dec(x_7); @@ -2957,31 +3423,31 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_100 = !lean_is_exclusive(x_95); -if (x_100 == 0) +x_155 = !lean_is_exclusive(x_146); +if (x_155 == 0) { -return x_95; +return x_146; } else { -lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_101 = lean_ctor_get(x_95, 0); -x_102 = lean_ctor_get(x_95, 1); -lean_inc(x_102); -lean_inc(x_101); -lean_dec(x_95); -x_103 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -return x_103; +lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_156 = lean_ctor_get(x_146, 0); +x_157 = lean_ctor_get(x_146, 1); +lean_inc(x_157); +lean_inc(x_156); +lean_dec(x_146); +x_158 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_158, 0, x_156); +lean_ctor_set(x_158, 1, x_157); +return x_158; } } } default: { -lean_object* x_104; -x_104 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_12, x_6, x_7, x_8, x_9); -return x_104; +lean_object* x_159; +x_159 = l_Lean_Core_transform_visit_visitPost___at_Lean_Core_betaReduce___spec__3(x_1, x_2, x_3, x_4, x_12, x_6, x_7, x_8, x_9); +return x_159; } } } @@ -3944,20 +4410,41 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___rarg___lambda__1(lean_obj { if (lean_obj_tag(x_1) == 10) { -lean_object* x_12; lean_object* x_13; -x_12 = lean_expr_update_mdata(x_1, x_11); -x_13 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_12, x_10); -return x_13; +lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; uint8_t x_16; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +x_14 = lean_ptr_addr(x_13); +lean_dec(x_13); +x_15 = lean_ptr_addr(x_11); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_1); +x_17 = l_Lean_Expr_mdata___override(x_12, x_11); +x_18 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17, x_10); +return x_18; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_19; +lean_dec(x_12); +lean_dec(x_11); +x_19 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_1, x_10); +return x_19; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_dec(x_11); lean_dec(x_1); -x_14 = l_Lean_Core_transform_visit___rarg___lambda__9___closed__3; -x_15 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_14); -x_16 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15, x_10); -return x_16; +x_20 = l_Lean_Core_transform_visit___rarg___lambda__9___closed__3; +x_21 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_20); +x_22 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_21, x_10); +return x_22; } } } @@ -3966,20 +4453,44 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit___rarg___lambda__2(lean_obj { if (lean_obj_tag(x_1) == 11) { -lean_object* x_12; lean_object* x_13; -x_12 = lean_expr_update_proj(x_1, x_11); -x_13 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_12, x_10); -return x_13; +lean_object* x_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; uint8_t x_17; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +x_14 = lean_ctor_get(x_1, 2); +lean_inc(x_14); +x_15 = lean_ptr_addr(x_14); +lean_dec(x_14); +x_16 = lean_ptr_addr(x_11); +x_17 = lean_usize_dec_eq(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_1); +x_18 = l_Lean_Expr_proj___override(x_12, x_13, x_11); +x_19 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_18, x_10); +return x_19; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_20; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +x_20 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_1, x_10); +return x_20; +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_dec(x_11); lean_dec(x_1); -x_14 = l_Lean_Core_transform_visit___rarg___lambda__10___closed__3; -x_15 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_14); -x_16 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15, x_10); -return x_16; +x_21 = l_Lean_Core_transform_visit___rarg___lambda__10___closed__3; +x_22 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_21); +x_23 = l_Lean_Meta_transform_visit_visitPost___rarg(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_22, x_10); +return x_23; } } } @@ -4029,7 +4540,7 @@ case 5: { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_16, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_16, x_17); x_19 = l_Lean_Core_transform_visit___rarg___lambda__11___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -7007,7 +7518,7 @@ case 5: { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_15, x_16); +x_17 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_15, x_16); x_18 = l_Lean_Core_transform_visit___rarg___lambda__11___closed__1; lean_inc(x_17); x_19 = lean_mk_array(x_17, x_18); @@ -7040,34 +7551,56 @@ return x_28; } case 10: { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_15, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_15, 0); lean_inc(x_29); +x_30 = lean_ctor_get(x_15, 1); +lean_inc(x_30); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); +lean_inc(x_30); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_30 = l_Lean_Meta_transform_visit___at_Lean_Meta_zetaReduce___spec__2(x_1, x_2, x_3, x_4, x_5, x_29, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_30) == 0) +x_31 = l_Lean_Meta_transform_visit___at_Lean_Meta_zetaReduce___spec__2(x_1, x_2, x_3, x_4, x_5, x_30, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); +lean_object* x_32; lean_object* x_33; size_t x_34; size_t x_35; uint8_t x_36; +x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = lean_ptr_addr(x_30); lean_dec(x_30); -x_33 = lean_expr_update_mdata(x_15, x_31); -x_34 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___spec__3(x_1, x_2, x_3, x_4, x_5, x_33, x_7, x_8, x_9, x_10, x_11, x_32); -return x_34; +x_35 = lean_ptr_addr(x_32); +x_36 = lean_usize_dec_eq(x_34, x_35); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; +lean_dec(x_15); +x_37 = l_Lean_Expr_mdata___override(x_29, x_32); +x_38 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___spec__3(x_1, x_2, x_3, x_4, x_5, x_37, x_7, x_8, x_9, x_10, x_11, x_33); +return x_38; +} +else +{ +lean_object* x_39; +lean_dec(x_32); +lean_dec(x_29); +x_39 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___spec__3(x_1, x_2, x_3, x_4, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_33); +return x_39; +} } else { -uint8_t x_35; +uint8_t x_40; +lean_dec(x_30); +lean_dec(x_29); lean_dec(x_15); lean_dec(x_11); lean_dec(x_10); @@ -7078,56 +7611,82 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_35 = !lean_is_exclusive(x_30); -if (x_35 == 0) +x_40 = !lean_is_exclusive(x_31); +if (x_40 == 0) { -return x_30; +return x_31; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_30, 0); -x_37 = lean_ctor_get(x_30, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_30); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_31, 0); +x_42 = lean_ctor_get(x_31, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_31); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } case 11: { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_15, 2); -lean_inc(x_39); +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_15, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_15, 1); +lean_inc(x_45); +x_46 = lean_ctor_get(x_15, 2); +lean_inc(x_46); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); +lean_inc(x_46); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); lean_inc(x_1); -x_40 = l_Lean_Meta_transform_visit___at_Lean_Meta_zetaReduce___spec__2(x_1, x_2, x_3, x_4, x_5, x_39, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_40) == 0) +x_47 = l_Lean_Meta_transform_visit___at_Lean_Meta_zetaReduce___spec__2(x_1, x_2, x_3, x_4, x_5, x_46, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_47) == 0) { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); -x_43 = lean_expr_update_proj(x_15, x_41); -x_44 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___spec__3(x_1, x_2, x_3, x_4, x_5, x_43, x_7, x_8, x_9, x_10, x_11, x_42); -return x_44; +lean_object* x_48; lean_object* x_49; size_t x_50; size_t x_51; uint8_t x_52; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = lean_ptr_addr(x_46); +lean_dec(x_46); +x_51 = lean_ptr_addr(x_48); +x_52 = lean_usize_dec_eq(x_50, x_51); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; +lean_dec(x_15); +x_53 = l_Lean_Expr_proj___override(x_44, x_45, x_48); +x_54 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___spec__3(x_1, x_2, x_3, x_4, x_5, x_53, x_7, x_8, x_9, x_10, x_11, x_49); +return x_54; } else { -uint8_t x_45; +lean_object* x_55; +lean_dec(x_48); +lean_dec(x_45); +lean_dec(x_44); +x_55 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___spec__3(x_1, x_2, x_3, x_4, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_49); +return x_55; +} +} +else +{ +uint8_t x_56; +lean_dec(x_46); +lean_dec(x_45); +lean_dec(x_44); lean_dec(x_15); lean_dec(x_11); lean_dec(x_10); @@ -7138,31 +7697,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_45 = !lean_is_exclusive(x_40); -if (x_45 == 0) +x_56 = !lean_is_exclusive(x_47); +if (x_56 == 0) { -return x_40; +return x_47; } 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_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_47, 0); +x_58 = lean_ctor_get(x_47, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_47); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } default: { -lean_object* x_49; -x_49 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___spec__3(x_1, x_2, x_3, x_4, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_12); -return x_49; +lean_object* x_60; +x_60 = l_Lean_Meta_transform_visit_visitPost___at_Lean_Meta_zetaReduce___spec__3(x_1, x_2, x_3, x_4, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_12); +return x_60; } } } diff --git a/stage0/stdlib/Lean/Meta/UnificationHint.c b/stage0/stdlib/Lean/Meta/UnificationHint.c index eaa3e44fe062..b5a624d93599 100644 --- a/stage0/stdlib/Lean/Meta/UnificationHint.c +++ b/stage0/stdlib/Lean/Meta/UnificationHint.c @@ -2441,7 +2441,7 @@ static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_Unific lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_UnificationHints_add___spec__1___closed__1; x_2 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_UnificationHints_add___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Meta_DiscrTree_insertCore___at_Lean_Meta_UnificationHints_add___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/WHNF.c b/stage0/stdlib/Lean/Meta/WHNF.c index cbcd6930b936..50fac404be0b 100644 --- a/stage0/stdlib/Lean/Meta/WHNF.c +++ b/stage0/stdlib/Lean/Meta/WHNF.c @@ -53,7 +53,6 @@ lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_getDelayedMVarAssignment LEAN_EXPORT lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_whnfMatcher___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_deltaBetaDefinition___at_Lean_Meta_unfoldDefinition_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_EXPORT lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_getRecRuleFor(lean_object*, lean_object*); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at___private_Lean_Meta_WHNF_0__Lean_Meta_cached_x3f___spec__1(lean_object*, lean_object*); lean_object* l_Nat_div___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -83,6 +82,7 @@ lean_object* lean_environment_find(lean_object*, lean_object*); static lean_object* l_Lean_Meta_toCtorIfLit___closed__7; static lean_object* l_Lean_Meta_toCtorIfLit___closed__24; lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getStuckMVar_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_toCtorIfLit___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_getStructuralRecArgPos_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -132,7 +132,7 @@ size_t lean_usize_shift_right(size_t, size_t); static lean_object* l_Lean_Meta_reduceNative_x3f___closed__14; LEAN_EXPORT lean_object* l_Lean_Meta_smartUnfoldingMatch_x3f(lean_object*); lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); -uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(uint8_t, uint8_t); +uint8_t l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(uint8_t, uint8_t); static lean_object* l_Lean_Meta_toCtorIfLit___closed__16; static lean_object* l_Lean_Meta_canUnfoldAtMatcher___closed__10; uint8_t lean_usize_dec_lt(size_t, size_t); @@ -248,6 +248,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_reduceMatcher_x3f___lambda__2___boxed(lean_ lean_object* l_Lean_markUsedAssignment___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_canUnfoldAtMatcher___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_toCtorIfLit(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_matchConstAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_cached_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_cached_x3f___closed__1; @@ -328,7 +329,6 @@ uint8_t l_Lean_Expr_isLambda(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_smartUnfoldingReduce_x3f_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_reduceNat_x3f___closed__8; static lean_object* l_Lean_Meta_canUnfoldAtMatcher___closed__39; -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go___spec__3___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_reduceNat_x3f___closed__17; static lean_object* l_Lean_Meta_canUnfoldAtMatcher___closed__35; @@ -356,13 +356,13 @@ static lean_object* l_Lean_Meta_canUnfoldAtMatcher___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_reduceMatcher_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_reduceQuotRec___rarg___closed__3; static lean_object* l_Lean_Meta_canUnfoldAtMatcher___closed__17; +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_reduceNat_x3f___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_unfoldProjInst_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_reduceNat_x3f___closed__21; static lean_object* l_Lean_Meta_smartUnfoldingReduce_x3f_go___closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Std_Format_initFn____x40_Lean_Data_Format___hyg_57____spec__1(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_List_find_x3f___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_object* l_Lean_Meta_getLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1285,7 +1285,7 @@ lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean x_22 = lean_ctor_get(x_12, 0); x_23 = l_Lean_Expr_const___override(x_22, x_10); x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_Expr_getAppNumArgsAux(x_1, x_24); +x_25 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_24); x_26 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_25); x_27 = lean_mk_array(x_25, x_26); @@ -1306,7 +1306,7 @@ lean_inc(x_33); lean_dec(x_12); x_34 = l_Lean_Expr_const___override(x_33, x_10); x_35 = lean_unsigned_to_nat(0u); -x_36 = l_Lean_Expr_getAppNumArgsAux(x_1, x_35); +x_36 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_35); x_37 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_36); x_38 = lean_mk_array(x_36, x_37); @@ -1339,7 +1339,7 @@ if (lean_is_exclusive(x_12)) { } x_48 = l_Lean_Expr_const___override(x_46, x_10); x_49 = lean_unsigned_to_nat(0u); -x_50 = l_Lean_Expr_getAppNumArgsAux(x_1, x_49); +x_50 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_49); x_51 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_50); x_52 = lean_mk_array(x_50, x_51); @@ -2012,7 +2012,7 @@ else { lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; uint8_t x_192; x_179 = lean_unsigned_to_nat(0u); -x_180 = l_Lean_Expr_getAppNumArgsAux(x_16, x_179); +x_180 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_16, x_179); x_181 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_180); x_182 = lean_mk_array(x_180, x_181); @@ -2943,7 +2943,7 @@ else { lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; uint8_t x_298; x_285 = lean_unsigned_to_nat(0u); -x_286 = l_Lean_Expr_getAppNumArgsAux(x_201, x_285); +x_286 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_201, x_285); x_287 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_286); x_288 = lean_mk_array(x_286, x_287); @@ -3981,7 +3981,7 @@ x_31 = lean_ctor_get(x_29, 1); lean_inc(x_31); lean_dec(x_29); x_32 = lean_unsigned_to_nat(0u); -x_33 = l_Lean_Expr_getAppNumArgsAux(x_3, x_32); +x_33 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_32); lean_inc(x_33); x_34 = lean_mk_array(x_33, x_19); x_35 = lean_unsigned_to_nat(1u); @@ -4170,7 +4170,7 @@ x_69 = lean_ctor_get(x_67, 1); lean_inc(x_69); lean_dec(x_67); x_70 = lean_unsigned_to_nat(0u); -x_71 = l_Lean_Expr_getAppNumArgsAux(x_3, x_70); +x_71 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_70); lean_inc(x_71); x_72 = lean_mk_array(x_71, x_58); x_73 = lean_unsigned_to_nat(1u); @@ -4896,7 +4896,7 @@ x_23 = lean_ctor_get(x_20, 0); lean_inc(x_23); lean_dec(x_20); x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_Expr_getAppNumArgsAux(x_18, x_24); +x_25 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_18, x_24); x_26 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_25); x_27 = lean_mk_array(x_25, x_26); @@ -5197,7 +5197,7 @@ static lean_object* _init_l___private_Lean_Meta_WHNF_0__Lean_Meta_reduceQuotRec_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l___private_Lean_Meta_WHNF_0__Lean_Meta_reduceQuotRec___rarg___closed__1; x_2 = l___private_Lean_Meta_WHNF_0__Lean_Meta_reduceQuotRec___rarg___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Meta_WHNF_0__Lean_Meta_reduceQuotRec___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -6045,7 +6045,7 @@ x_35 = lean_ctor_get(x_33, 0); lean_inc(x_35); lean_dec(x_33); x_36 = lean_unsigned_to_nat(0u); -x_37 = l_Lean_Expr_getAppNumArgsAux(x_1, x_36); +x_37 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_36); x_38 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_37); x_39 = lean_mk_array(x_37, x_38); @@ -6066,7 +6066,7 @@ x_45 = lean_ctor_get(x_33, 0); lean_inc(x_45); lean_dec(x_33); x_46 = lean_unsigned_to_nat(0u); -x_47 = l_Lean_Expr_getAppNumArgsAux(x_1, x_46); +x_47 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_46); x_48 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_47); x_49 = lean_mk_array(x_47, x_48); @@ -6498,7 +6498,7 @@ static lean_object* _init_l_Lean_Meta_whnfEasyCases___closed__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; x_1 = l_Lean_Meta_whnfEasyCases___closed__2; x_2 = l_Lean_Meta_whnfEasyCases___closed__3; -x_3 = lean_unsigned_to_nat(290u); +x_3 = lean_unsigned_to_nat(289u); x_4 = lean_unsigned_to_nat(26u); x_5 = l_Lean_Meta_whnfEasyCases___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10112,7 +10112,7 @@ lean_inc(x_9); lean_dec(x_7); x_10 = 2; x_11 = lean_unbox(x_8); -x_12 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_11, x_10); +x_12 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_11, x_10); if (x_12 == 0) { lean_object* x_13; uint8_t x_14; lean_object* x_15; @@ -10258,7 +10258,7 @@ uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_obje lean_dec(x_7); x_32 = lean_nat_dec_lt(x_21, x_3); x_33 = lean_unsigned_to_nat(0u); -x_34 = l_Lean_Expr_getAppNumArgsAux(x_5, x_33); +x_34 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_33); lean_inc(x_34); x_35 = lean_mk_array(x_34, x_1); x_36 = lean_unsigned_to_nat(1u); @@ -10343,7 +10343,7 @@ uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_obje lean_dec(x_7); x_66 = lean_nat_dec_lt(x_56, x_3); x_67 = lean_unsigned_to_nat(0u); -x_68 = l_Lean_Expr_getAppNumArgsAux(x_5, x_67); +x_68 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_5, x_67); lean_inc(x_68); x_69 = lean_mk_array(x_68, x_1); x_70 = lean_unsigned_to_nat(1u); @@ -10657,7 +10657,7 @@ if (x_21 == 0) lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; x_22 = lean_ctor_get(x_11, 0); x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Lean_Expr_getAppNumArgsAux(x_1, x_23); +x_24 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_23); x_25 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_24); x_26 = lean_mk_array(x_24, x_25); @@ -10826,7 +10826,7 @@ x_61 = lean_ctor_get(x_11, 0); lean_inc(x_61); lean_dec(x_11); x_62 = lean_unsigned_to_nat(0u); -x_63 = l_Lean_Expr_getAppNumArgsAux(x_1, x_62); +x_63 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_62); x_64 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_63); x_65 = lean_mk_array(x_63, x_64); @@ -11007,7 +11007,7 @@ if (lean_is_exclusive(x_11)) { x_103 = lean_box(0); } x_104 = lean_unsigned_to_nat(0u); -x_105 = l_Lean_Expr_getAppNumArgsAux(x_1, x_104); +x_105 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_104); x_106 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_105); x_107 = lean_mk_array(x_105, x_106); @@ -11309,7 +11309,7 @@ x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); lean_dec(x_18); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_8, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_8, x_20); x_22 = lean_ctor_get(x_19, 3); lean_inc(x_22); lean_dec(x_19); @@ -11366,7 +11366,7 @@ x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); lean_dec(x_31); x_33 = lean_unsigned_to_nat(0u); -x_34 = l_Lean_Expr_getAppNumArgsAux(x_8, x_33); +x_34 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_8, x_33); x_35 = lean_ctor_get(x_32, 3); lean_inc(x_35); lean_dec(x_32); @@ -11452,7 +11452,7 @@ x_53 = lean_ctor_get(x_51, 0); lean_inc(x_53); lean_dec(x_51); x_54 = lean_unsigned_to_nat(0u); -x_55 = l_Lean_Expr_getAppNumArgsAux(x_8, x_54); +x_55 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_8, x_54); x_56 = lean_ctor_get(x_53, 3); lean_inc(x_56); lean_dec(x_53); @@ -11810,7 +11810,7 @@ x_26 = lean_ctor_get(x_22, 1); lean_inc(x_26); lean_dec(x_22); x_27 = lean_unsigned_to_nat(0u); -x_28 = l_Lean_Expr_getAppNumArgsAux(x_2, x_27); +x_28 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_27); x_29 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_28); x_30 = lean_mk_array(x_28, x_29); @@ -11932,7 +11932,7 @@ x_59 = lean_ctor_get(x_56, 1); lean_inc(x_59); lean_dec(x_56); x_60 = lean_unsigned_to_nat(0u); -x_61 = l_Lean_Expr_getAppNumArgsAux(x_2, x_60); +x_61 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_60); x_62 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_61); x_63 = lean_mk_array(x_61, x_62); @@ -12041,7 +12041,7 @@ x_88 = lean_ctor_get(x_84, 1); lean_inc(x_88); lean_dec(x_84); x_89 = lean_unsigned_to_nat(0u); -x_90 = l_Lean_Expr_getAppNumArgsAux(x_2, x_89); +x_90 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_89); x_91 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_90); x_92 = lean_mk_array(x_90, x_91); @@ -14775,7 +14775,7 @@ static lean_object* _init_l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go__ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_whnfEasyCases___closed__2; x_2 = l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go___spec__3___lambda__3___closed__1; -x_3 = lean_unsigned_to_nat(519u); +x_3 = lean_unsigned_to_nat(518u); x_4 = lean_unsigned_to_nat(13u); x_5 = l_Lean_Meta_whnfEasyCases___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -15002,7 +15002,7 @@ x_45 = lean_ctor_get(x_38, 1); lean_inc(x_45); lean_dec(x_38); x_46 = lean_unsigned_to_nat(0u); -x_47 = l_Lean_Expr_getAppNumArgsAux(x_19, x_46); +x_47 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_19, x_46); x_48 = lean_mk_empty_array_with_capacity(x_47); lean_dec(x_47); lean_inc(x_19); @@ -15022,7 +15022,7 @@ x_53 = lean_ctor_get(x_35, 0); lean_inc(x_53); lean_dec(x_35); x_54 = lean_unsigned_to_nat(0u); -x_55 = l_Lean_Expr_getAppNumArgsAux(x_19, x_54); +x_55 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_19, x_54); x_56 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_55); x_57 = lean_mk_array(x_55, x_56); @@ -15049,7 +15049,7 @@ x_65 = lean_ctor_get(x_35, 0); lean_inc(x_65); lean_dec(x_35); x_66 = lean_unsigned_to_nat(0u); -x_67 = l_Lean_Expr_getAppNumArgsAux(x_19, x_66); +x_67 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_19, x_66); x_68 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_67); x_69 = lean_mk_array(x_67, x_68); @@ -15224,7 +15224,7 @@ else lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; lean_object* x_107; lean_dec(x_11); x_101 = lean_unsigned_to_nat(0u); -x_102 = l_Lean_Expr_getAppNumArgsAux(x_1, x_101); +x_102 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_101); x_103 = lean_mk_empty_array_with_capacity(x_102); lean_dec(x_102); x_104 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_103); @@ -17030,277 +17030,419 @@ return x_70; } case 10: { -lean_object* x_71; lean_object* x_72; -x_71 = lean_ctor_get(x_1, 1); +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_1, 0); lean_inc(x_71); -x_72 = l_Lean_Meta_smartUnfoldingMatch_x3f(x_1); -if (lean_obj_tag(x_72) == 0) -{ -lean_object* x_73; -x_73 = l_Lean_Meta_smartUnfoldingReduce_x3f_go(x_71, x_2, x_3, x_4, x_5, x_6); +x_72 = lean_ctor_get(x_1, 1); +lean_inc(x_72); +x_73 = l_Lean_Meta_smartUnfoldingMatch_x3f(x_1); if (lean_obj_tag(x_73) == 0) { lean_object* x_74; -x_74 = lean_ctor_get(x_73, 0); -lean_inc(x_74); +lean_inc(x_72); +x_74 = l_Lean_Meta_smartUnfoldingReduce_x3f_go(x_72, x_2, x_3, x_4, x_5, x_6); if (lean_obj_tag(x_74) == 0) { -uint8_t x_75; +lean_object* x_75; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +if (lean_obj_tag(x_75) == 0) +{ +uint8_t x_76; +lean_dec(x_72); +lean_dec(x_71); lean_dec(x_1); -x_75 = !lean_is_exclusive(x_73); -if (x_75 == 0) +x_76 = !lean_is_exclusive(x_74); +if (x_76 == 0) { -lean_object* x_76; lean_object* x_77; -x_76 = lean_ctor_get(x_73, 0); -lean_dec(x_76); -x_77 = lean_box(0); -lean_ctor_set(x_73, 0, x_77); -return x_73; +lean_object* x_77; lean_object* x_78; +x_77 = lean_ctor_get(x_74, 0); +lean_dec(x_77); +x_78 = lean_box(0); +lean_ctor_set(x_74, 0, x_78); +return x_74; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_73, 1); -lean_inc(x_78); -lean_dec(x_73); -x_79 = lean_box(0); -x_80 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_74, 1); +lean_inc(x_79); +lean_dec(x_74); +x_80 = lean_box(0); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_79); +return x_81; } } else { -uint8_t x_81; -x_81 = !lean_is_exclusive(x_73); -if (x_81 == 0) +uint8_t x_82; +x_82 = !lean_is_exclusive(x_74); +if (x_82 == 0) { -lean_object* x_82; uint8_t x_83; -x_82 = lean_ctor_get(x_73, 0); -lean_dec(x_82); -x_83 = !lean_is_exclusive(x_74); -if (x_83 == 0) +lean_object* x_83; uint8_t x_84; +x_83 = lean_ctor_get(x_74, 0); +lean_dec(x_83); +x_84 = !lean_is_exclusive(x_75); +if (x_84 == 0) { -lean_object* x_84; lean_object* x_85; -x_84 = lean_ctor_get(x_74, 0); -x_85 = lean_expr_update_mdata(x_1, x_84); -lean_ctor_set(x_74, 0, x_85); -return x_73; +lean_object* x_85; size_t x_86; size_t x_87; uint8_t x_88; +x_85 = lean_ctor_get(x_75, 0); +x_86 = lean_ptr_addr(x_72); +lean_dec(x_72); +x_87 = lean_ptr_addr(x_85); +x_88 = lean_usize_dec_eq(x_86, x_87); +if (x_88 == 0) +{ +lean_object* x_89; +lean_dec(x_1); +x_89 = l_Lean_Expr_mdata___override(x_71, x_85); +lean_ctor_set(x_75, 0, x_89); +return x_74; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_74, 0); -lean_inc(x_86); -lean_dec(x_74); -x_87 = lean_expr_update_mdata(x_1, x_86); -x_88 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_88, 0, x_87); -lean_ctor_set(x_73, 0, x_88); -return x_73; +lean_dec(x_85); +lean_dec(x_71); +lean_ctor_set(x_75, 0, x_1); +return x_74; } } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_89 = lean_ctor_get(x_73, 1); -lean_inc(x_89); -lean_dec(x_73); -x_90 = lean_ctor_get(x_74, 0); +lean_object* x_90; size_t x_91; size_t x_92; uint8_t x_93; +x_90 = lean_ctor_get(x_75, 0); lean_inc(x_90); -if (lean_is_exclusive(x_74)) { - lean_ctor_release(x_74, 0); - x_91 = x_74; +lean_dec(x_75); +x_91 = lean_ptr_addr(x_72); +lean_dec(x_72); +x_92 = lean_ptr_addr(x_90); +x_93 = lean_usize_dec_eq(x_91, x_92); +if (x_93 == 0) +{ +lean_object* x_94; lean_object* x_95; +lean_dec(x_1); +x_94 = l_Lean_Expr_mdata___override(x_71, x_90); +x_95 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_95, 0, x_94); +lean_ctor_set(x_74, 0, x_95); +return x_74; +} +else +{ +lean_object* x_96; +lean_dec(x_90); +lean_dec(x_71); +x_96 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_96, 0, x_1); +lean_ctor_set(x_74, 0, x_96); +return x_74; +} +} +} +else +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; size_t x_100; size_t x_101; uint8_t x_102; +x_97 = lean_ctor_get(x_74, 1); +lean_inc(x_97); +lean_dec(x_74); +x_98 = lean_ctor_get(x_75, 0); +lean_inc(x_98); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + x_99 = x_75; } else { - lean_dec_ref(x_74); - x_91 = lean_box(0); + lean_dec_ref(x_75); + x_99 = lean_box(0); } -x_92 = lean_expr_update_mdata(x_1, x_90); -if (lean_is_scalar(x_91)) { - x_93 = lean_alloc_ctor(1, 1, 0); +x_100 = lean_ptr_addr(x_72); +lean_dec(x_72); +x_101 = lean_ptr_addr(x_98); +x_102 = lean_usize_dec_eq(x_100, x_101); +if (x_102 == 0) +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_1); +x_103 = l_Lean_Expr_mdata___override(x_71, x_98); +if (lean_is_scalar(x_99)) { + x_104 = lean_alloc_ctor(1, 1, 0); } else { - x_93 = x_91; + x_104 = x_99; +} +lean_ctor_set(x_104, 0, x_103); +x_105 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_104); +lean_ctor_set(x_105, 1, x_97); +return x_105; +} +else +{ +lean_object* x_106; lean_object* x_107; +lean_dec(x_98); +lean_dec(x_71); +if (lean_is_scalar(x_99)) { + x_106 = lean_alloc_ctor(1, 1, 0); +} else { + x_106 = x_99; +} +lean_ctor_set(x_106, 0, x_1); +x_107 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set(x_107, 1, x_97); +return x_107; } -lean_ctor_set(x_93, 0, x_92); -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_89); -return x_94; } } } else { -uint8_t x_95; +uint8_t x_108; +lean_dec(x_72); +lean_dec(x_71); lean_dec(x_1); -x_95 = !lean_is_exclusive(x_73); -if (x_95 == 0) +x_108 = !lean_is_exclusive(x_74); +if (x_108 == 0) { -return x_73; +return x_74; } else { -lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_96 = lean_ctor_get(x_73, 0); -x_97 = lean_ctor_get(x_73, 1); -lean_inc(x_97); -lean_inc(x_96); -lean_dec(x_73); -x_98 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_98, 0, x_96); -lean_ctor_set(x_98, 1, x_97); -return x_98; +lean_object* x_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 { -lean_object* x_99; lean_object* x_100; +lean_object* x_112; lean_object* x_113; +lean_dec(x_72); lean_dec(x_71); lean_dec(x_1); -x_99 = lean_ctor_get(x_72, 0); -lean_inc(x_99); -lean_dec(x_72); -x_100 = l_Lean_Meta_smartUnfoldingReduce_x3f_goMatch(x_99, x_2, x_3, x_4, x_5, x_6); -return x_100; +x_112 = lean_ctor_get(x_73, 0); +lean_inc(x_112); +lean_dec(x_73); +x_113 = l_Lean_Meta_smartUnfoldingReduce_x3f_goMatch(x_112, x_2, x_3, x_4, x_5, x_6); +return x_113; } } case 11: { -lean_object* x_101; lean_object* x_102; -x_101 = lean_ctor_get(x_1, 2); -lean_inc(x_101); -x_102 = l_Lean_Meta_smartUnfoldingReduce_x3f_go(x_101, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_102) == 0) +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_114 = lean_ctor_get(x_1, 0); +lean_inc(x_114); +x_115 = lean_ctor_get(x_1, 1); +lean_inc(x_115); +x_116 = lean_ctor_get(x_1, 2); +lean_inc(x_116); +lean_inc(x_116); +x_117 = l_Lean_Meta_smartUnfoldingReduce_x3f_go(x_116, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_117) == 0) { -lean_object* x_103; -x_103 = lean_ctor_get(x_102, 0); -lean_inc(x_103); -if (lean_obj_tag(x_103) == 0) +lean_object* x_118; +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +if (lean_obj_tag(x_118) == 0) { -uint8_t x_104; +uint8_t x_119; +lean_dec(x_116); +lean_dec(x_115); +lean_dec(x_114); lean_dec(x_1); -x_104 = !lean_is_exclusive(x_102); -if (x_104 == 0) +x_119 = !lean_is_exclusive(x_117); +if (x_119 == 0) { -lean_object* x_105; lean_object* x_106; -x_105 = lean_ctor_get(x_102, 0); -lean_dec(x_105); -x_106 = lean_box(0); -lean_ctor_set(x_102, 0, x_106); -return x_102; +lean_object* x_120; lean_object* x_121; +x_120 = lean_ctor_get(x_117, 0); +lean_dec(x_120); +x_121 = lean_box(0); +lean_ctor_set(x_117, 0, x_121); +return x_117; } else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_107 = lean_ctor_get(x_102, 1); -lean_inc(x_107); -lean_dec(x_102); -x_108 = lean_box(0); -x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_107); -return x_109; +lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_117, 1); +lean_inc(x_122); +lean_dec(x_117); +x_123 = lean_box(0); +x_124 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_124, 0, x_123); +lean_ctor_set(x_124, 1, x_122); +return x_124; } } else { -uint8_t x_110; -x_110 = !lean_is_exclusive(x_102); -if (x_110 == 0) +uint8_t x_125; +x_125 = !lean_is_exclusive(x_117); +if (x_125 == 0) { -lean_object* x_111; uint8_t x_112; -x_111 = lean_ctor_get(x_102, 0); -lean_dec(x_111); -x_112 = !lean_is_exclusive(x_103); -if (x_112 == 0) +lean_object* x_126; uint8_t x_127; +x_126 = lean_ctor_get(x_117, 0); +lean_dec(x_126); +x_127 = !lean_is_exclusive(x_118); +if (x_127 == 0) { -lean_object* x_113; lean_object* x_114; -x_113 = lean_ctor_get(x_103, 0); -x_114 = lean_expr_update_proj(x_1, x_113); -lean_ctor_set(x_103, 0, x_114); -return x_102; +lean_object* x_128; size_t x_129; size_t x_130; uint8_t x_131; +x_128 = lean_ctor_get(x_118, 0); +x_129 = lean_ptr_addr(x_116); +lean_dec(x_116); +x_130 = lean_ptr_addr(x_128); +x_131 = lean_usize_dec_eq(x_129, x_130); +if (x_131 == 0) +{ +lean_object* x_132; +lean_dec(x_1); +x_132 = l_Lean_Expr_proj___override(x_114, x_115, x_128); +lean_ctor_set(x_118, 0, x_132); +return x_117; } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_115 = lean_ctor_get(x_103, 0); -lean_inc(x_115); -lean_dec(x_103); -x_116 = lean_expr_update_proj(x_1, x_115); -x_117 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_117, 0, x_116); -lean_ctor_set(x_102, 0, x_117); -return x_102; +lean_dec(x_128); +lean_dec(x_115); +lean_dec(x_114); +lean_ctor_set(x_118, 0, x_1); +return x_117; } } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_118 = lean_ctor_get(x_102, 1); -lean_inc(x_118); -lean_dec(x_102); -x_119 = lean_ctor_get(x_103, 0); -lean_inc(x_119); -if (lean_is_exclusive(x_103)) { - lean_ctor_release(x_103, 0); - x_120 = x_103; +lean_object* x_133; size_t x_134; size_t x_135; uint8_t x_136; +x_133 = lean_ctor_get(x_118, 0); +lean_inc(x_133); +lean_dec(x_118); +x_134 = lean_ptr_addr(x_116); +lean_dec(x_116); +x_135 = lean_ptr_addr(x_133); +x_136 = lean_usize_dec_eq(x_134, x_135); +if (x_136 == 0) +{ +lean_object* x_137; lean_object* x_138; +lean_dec(x_1); +x_137 = l_Lean_Expr_proj___override(x_114, x_115, x_133); +x_138 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_138, 0, x_137); +lean_ctor_set(x_117, 0, x_138); +return x_117; +} +else +{ +lean_object* x_139; +lean_dec(x_133); +lean_dec(x_115); +lean_dec(x_114); +x_139 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_139, 0, x_1); +lean_ctor_set(x_117, 0, x_139); +return x_117; +} +} +} +else +{ +lean_object* x_140; lean_object* x_141; lean_object* x_142; size_t x_143; size_t x_144; uint8_t x_145; +x_140 = lean_ctor_get(x_117, 1); +lean_inc(x_140); +lean_dec(x_117); +x_141 = lean_ctor_get(x_118, 0); +lean_inc(x_141); +if (lean_is_exclusive(x_118)) { + lean_ctor_release(x_118, 0); + x_142 = x_118; } else { - lean_dec_ref(x_103); - x_120 = lean_box(0); + lean_dec_ref(x_118); + x_142 = lean_box(0); } -x_121 = lean_expr_update_proj(x_1, x_119); -if (lean_is_scalar(x_120)) { - x_122 = lean_alloc_ctor(1, 1, 0); +x_143 = lean_ptr_addr(x_116); +lean_dec(x_116); +x_144 = lean_ptr_addr(x_141); +x_145 = lean_usize_dec_eq(x_143, x_144); +if (x_145 == 0) +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; +lean_dec(x_1); +x_146 = l_Lean_Expr_proj___override(x_114, x_115, x_141); +if (lean_is_scalar(x_142)) { + x_147 = lean_alloc_ctor(1, 1, 0); } else { - x_122 = x_120; + x_147 = x_142; +} +lean_ctor_set(x_147, 0, x_146); +x_148 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_148, 0, x_147); +lean_ctor_set(x_148, 1, x_140); +return x_148; +} +else +{ +lean_object* x_149; lean_object* x_150; +lean_dec(x_141); +lean_dec(x_115); +lean_dec(x_114); +if (lean_is_scalar(x_142)) { + x_149 = lean_alloc_ctor(1, 1, 0); +} else { + x_149 = x_142; +} +lean_ctor_set(x_149, 0, x_1); +x_150 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_150, 0, x_149); +lean_ctor_set(x_150, 1, x_140); +return x_150; } -lean_ctor_set(x_122, 0, x_121); -x_123 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_123, 0, x_122); -lean_ctor_set(x_123, 1, x_118); -return x_123; } } } else { -uint8_t x_124; +uint8_t x_151; +lean_dec(x_116); +lean_dec(x_115); +lean_dec(x_114); lean_dec(x_1); -x_124 = !lean_is_exclusive(x_102); -if (x_124 == 0) +x_151 = !lean_is_exclusive(x_117); +if (x_151 == 0) { -return x_102; +return x_117; } else { -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_102, 0); -x_126 = lean_ctor_get(x_102, 1); -lean_inc(x_126); -lean_inc(x_125); -lean_dec(x_102); -x_127 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_127, 0, x_125); -lean_ctor_set(x_127, 1, x_126); -return x_127; +lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_152 = lean_ctor_get(x_117, 0); +x_153 = lean_ctor_get(x_117, 1); +lean_inc(x_153); +lean_inc(x_152); +lean_dec(x_117); +x_154 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_154, 0, x_152); +lean_ctor_set(x_154, 1, x_153); +return x_154; } } } default: { -lean_object* x_128; lean_object* x_129; +lean_object* x_155; lean_object* x_156; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_128 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_128, 0, x_1); -x_129 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_129, 0, x_128); -lean_ctor_set(x_129, 1, x_6); -return x_129; +x_155 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_155, 0, x_1); +x_156 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_156, 0, x_155); +lean_ctor_set(x_156, 1, x_6); +return x_156; } } } @@ -17972,7 +18114,7 @@ if (x_72 == 0) lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; x_73 = lean_ctor_get(x_63, 0); x_74 = lean_unsigned_to_nat(0u); -x_75 = l_Lean_Expr_getAppNumArgsAux(x_57, x_74); +x_75 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_57, x_74); x_76 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_75); x_77 = lean_mk_array(x_75, x_76); @@ -17992,7 +18134,7 @@ x_83 = lean_ctor_get(x_63, 0); lean_inc(x_83); lean_dec(x_63); x_84 = lean_unsigned_to_nat(0u); -x_85 = l_Lean_Expr_getAppNumArgsAux(x_57, x_84); +x_85 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_57, x_84); x_86 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_85); x_87 = lean_mk_array(x_85, x_86); @@ -18024,7 +18166,7 @@ if (lean_is_exclusive(x_63)) { x_96 = lean_box(0); } x_97 = lean_unsigned_to_nat(0u); -x_98 = l_Lean_Expr_getAppNumArgsAux(x_57, x_97); +x_98 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_57, x_97); x_99 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_98); x_100 = lean_mk_array(x_98, x_99); @@ -19250,7 +19392,7 @@ else { lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_free_object(x_81); -x_100 = l_Lean_Expr_getAppNumArgsAux(x_1, x_90); +x_100 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_90); x_101 = lean_mk_empty_array_with_capacity(x_100); lean_dec(x_100); x_102 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_101); @@ -19316,7 +19458,7 @@ else { lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; lean_free_object(x_113); -x_120 = l_Lean_Expr_getAppNumArgsAux(x_1, x_90); +x_120 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_90); x_121 = lean_mk_empty_array_with_capacity(x_120); lean_dec(x_120); x_122 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_121); @@ -19355,7 +19497,7 @@ return x_128; else { lean_object* x_129; lean_object* x_130; lean_object* x_131; uint8_t x_132; lean_object* x_133; -x_129 = l_Lean_Expr_getAppNumArgsAux(x_1, x_90); +x_129 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_90); x_130 = lean_mk_empty_array_with_capacity(x_129); lean_dec(x_129); x_131 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_130); @@ -19414,7 +19556,7 @@ if (lean_obj_tag(x_140) == 1) { lean_object* x_141; lean_object* x_142; lean_object* x_143; uint8_t x_144; lean_object* x_145; lean_dec(x_88); -x_141 = l_Lean_Expr_getAppNumArgsAux(x_1, x_90); +x_141 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_90); x_142 = lean_mk_empty_array_with_capacity(x_141); lean_inc(x_1); x_143 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_142); @@ -19458,7 +19600,7 @@ else { lean_object* x_153; lean_object* x_154; lean_object* x_155; uint8_t x_156; lean_object* x_157; lean_free_object(x_146); -x_153 = l_Lean_Expr_getAppNumArgsAux(x_1, x_90); +x_153 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_90); x_154 = lean_mk_empty_array_with_capacity(x_153); lean_dec(x_153); x_155 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_154); @@ -19497,7 +19639,7 @@ return x_161; else { lean_object* x_162; lean_object* x_163; lean_object* x_164; uint8_t x_165; lean_object* x_166; -x_162 = l_Lean_Expr_getAppNumArgsAux(x_1, x_90); +x_162 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_90); x_163 = lean_mk_empty_array_with_capacity(x_162); lean_dec(x_162); x_164 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_163); @@ -19614,7 +19756,7 @@ return x_187; else { lean_object* x_188; lean_object* x_189; lean_object* x_190; uint8_t x_191; lean_object* x_192; -x_188 = l_Lean_Expr_getAppNumArgsAux(x_1, x_176); +x_188 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_176); x_189 = lean_mk_empty_array_with_capacity(x_188); lean_dec(x_188); x_190 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_189); @@ -19688,7 +19830,7 @@ else { lean_object* x_208; lean_object* x_209; lean_object* x_210; uint8_t x_211; lean_object* x_212; lean_dec(x_204); -x_208 = l_Lean_Expr_getAppNumArgsAux(x_1, x_176); +x_208 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_176); x_209 = lean_mk_empty_array_with_capacity(x_208); lean_dec(x_208); x_210 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_209); @@ -19743,7 +19885,7 @@ if (lean_obj_tag(x_217) == 1) { lean_object* x_218; lean_object* x_219; lean_object* x_220; uint8_t x_221; lean_object* x_222; lean_dec(x_174); -x_218 = l_Lean_Expr_getAppNumArgsAux(x_1, x_176); +x_218 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_176); x_219 = lean_mk_empty_array_with_capacity(x_218); lean_inc(x_1); x_220 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_219); @@ -19796,7 +19938,7 @@ else { lean_object* x_230; lean_object* x_231; lean_object* x_232; uint8_t x_233; lean_object* x_234; lean_dec(x_226); -x_230 = l_Lean_Expr_getAppNumArgsAux(x_1, x_176); +x_230 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_176); x_231 = lean_mk_empty_array_with_capacity(x_230); lean_dec(x_230); x_232 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_231); @@ -19916,7 +20058,7 @@ x_10 = lean_ctor_get(x_7, 1); x_11 = 3; x_12 = lean_unbox(x_9); lean_dec(x_9); -x_13 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_12, x_11); +x_13 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_12, x_11); if (x_13 == 0) { lean_object* x_14; @@ -19947,7 +20089,7 @@ lean_dec(x_7); x_18 = 3; x_19 = lean_unbox(x_16); lean_dec(x_16); -x_20 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9875_(x_19, x_18); +x_20 = l___private_Init_Meta_0__Lean_Meta_beqTransparencyMode____x40_Init_Meta___hyg_9966_(x_19, x_18); if (x_20 == 0) { lean_object* x_21; lean_object* x_22; @@ -22123,7 +22265,7 @@ x_46 = lean_ctor_get(x_37, 1); lean_inc(x_46); lean_dec(x_37); x_47 = lean_unsigned_to_nat(0u); -x_48 = l_Lean_Expr_getAppNumArgsAux(x_1, x_47); +x_48 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_47); x_49 = lean_mk_empty_array_with_capacity(x_48); lean_dec(x_48); x_50 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_49); @@ -22146,7 +22288,7 @@ x_54 = lean_ctor_get(x_34, 0); lean_inc(x_54); lean_dec(x_34); x_55 = lean_unsigned_to_nat(0u); -x_56 = l_Lean_Expr_getAppNumArgsAux(x_1, x_55); +x_56 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_55); x_57 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_56); x_58 = lean_mk_array(x_56, x_57); @@ -22172,7 +22314,7 @@ x_66 = lean_ctor_get(x_34, 0); lean_inc(x_66); lean_dec(x_34); x_67 = lean_unsigned_to_nat(0u); -x_68 = l_Lean_Expr_getAppNumArgsAux(x_1, x_67); +x_68 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_67); x_69 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_68); x_70 = lean_mk_array(x_68, x_69); @@ -22373,7 +22515,7 @@ x_108 = lean_ctor_get(x_101, 1); lean_inc(x_108); lean_dec(x_101); x_109 = lean_unsigned_to_nat(0u); -x_110 = l_Lean_Expr_getAppNumArgsAux(x_1, x_109); +x_110 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_109); x_111 = lean_mk_empty_array_with_capacity(x_110); lean_dec(x_110); x_112 = l___private_Lean_Expr_0__Lean_Expr_getAppRevArgsAux(x_1, x_111); @@ -22396,7 +22538,7 @@ x_116 = lean_ctor_get(x_98, 0); lean_inc(x_116); lean_dec(x_98); x_117 = lean_unsigned_to_nat(0u); -x_118 = l_Lean_Expr_getAppNumArgsAux(x_1, x_117); +x_118 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_117); x_119 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_118); x_120 = lean_mk_array(x_118, x_119); @@ -22422,7 +22564,7 @@ x_128 = lean_ctor_get(x_98, 0); lean_inc(x_128); lean_dec(x_98); x_129 = lean_unsigned_to_nat(0u); -x_130 = l_Lean_Expr_getAppNumArgsAux(x_1, x_129); +x_130 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_129); x_131 = l___private_Lean_Meta_WHNF_0__Lean_Meta_mkNullaryCtor___closed__1; lean_inc(x_130); x_132 = lean_mk_array(x_130, x_131); @@ -28424,7 +28566,7 @@ static lean_object* _init_l___private_Lean_Meta_WHNF_0__Lean_Meta_cached_x3f___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_Lean_Meta_whnfEasyCases___closed__2; x_2 = l___private_Lean_Meta_WHNF_0__Lean_Meta_cached_x3f___closed__1; -x_3 = lean_unsigned_to_nat(810u); +x_3 = lean_unsigned_to_nat(809u); x_4 = lean_unsigned_to_nat(34u); x_5 = l_Lean_Meta_whnfEasyCases___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -29174,7 +29316,7 @@ static lean_object* _init_l___private_Lean_Meta_WHNF_0__Lean_Meta_cache___closed lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_whnfEasyCases___closed__2; x_2 = l___private_Lean_Meta_WHNF_0__Lean_Meta_cache___closed__1; -x_3 = lean_unsigned_to_nat(819u); +x_3 = lean_unsigned_to_nat(818u); x_4 = lean_unsigned_to_nat(34u); x_5 = l_Lean_Meta_whnfEasyCases___closed__4; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/MetavarContext.c b/stage0/stdlib/Lean/MetavarContext.c index 199804f603dd..840185c57966 100644 --- a/stage0/stdlib/Lean/MetavarContext.c +++ b/stage0/stdlib/Lean/MetavarContext.c @@ -27,7 +27,6 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v LEAN_EXPORT lean_object* l_Lean_instantiateMVarDeclMVars___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_MkBinding_mkBinding___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_instantiateLCtxMVars___spec__6(lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateExprMVars___spec__28___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAtAux___at_Lean_isLevelMVarAssigned___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_MetavarContext_0__Lean_reprMetavarKind____x40_Lean_MetavarContext___hyg_101____closed__16; @@ -74,6 +73,7 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_shoul LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_getLevelMVarAssignment_x3f___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_MetavarContext_LevelMVarToParam_main_visitApp___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_assignLevelMVar___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_exprDependsOn___spec__9(lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateExprMVars___spec__45___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -165,7 +165,6 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_assignLevelMVar___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_addLevelMVarDecl(lean_object*, lean_object*); static lean_object* l_Lean_instantiateExprMVars___rarg___lambda__9___closed__1; -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_instantiateExprMVars___spec__48___rarg___lambda__10(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -182,6 +181,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_instantiateMVarsCore__ static lean_object* l_Lean_instantiateExprMVars___rarg___lambda__9___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_MetavarContext_addLevelMVarDecl___spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__2___closed__2; +lean_object* l_Lean_Level_succ___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_eAssignment___default; LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateExprMVars___spec__47(lean_object*, lean_object*); @@ -270,6 +270,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_instantiateLCtxMVar LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_instantiateLCtxMVars___spec__12___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__11(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_setMVarKind(lean_object*, lean_object*, uint8_t); +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_addExprMVarDeclExp___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isLevelMVarAssigned(lean_object*); @@ -377,6 +378,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore__ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_localDeclDependsOn___spec__35(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__101(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at_Lean_localDeclDependsOn___spec__29___boxed(lean_object*, lean_object*); +uint8_t l_ptrEqList___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_exprDependsOn_x27___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_localDeclDependsOn_x27___spec__49(lean_object*, lean_object*, size_t, size_t); @@ -454,6 +456,7 @@ LEAN_EXPORT lean_object* l_Lean_assignExprMVar___at___private_Lean_MetavarContex LEAN_EXPORT lean_object* l_Lean_MetavarContext_getExprAssignmentDomain(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_instantiateMVarsCore___spec__42___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_instantiateExprMVars___spec__48___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_anyAux___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__50___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_anyM___at_Lean_hasAssignedMVar___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t); @@ -515,6 +518,7 @@ uint8_t lean_expr_has_loose_bvar(lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldRevM_loop___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_mkAuxMVarType___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_localDeclDependsOn_x27___spec__37(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_simpLevelIMax_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_localDeclDependsOnPred___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_assignLevelMVar___at_Lean_instantiateExprMVars___spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); @@ -698,13 +702,13 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_exprDependsOn_x27___sp LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__35(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__15___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_LevelMVarToParam_visitLevel(lean_object*, lean_object*, lean_object*); -lean_object* lean_level_update_max(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__14___rarg(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__41(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__39___rarg(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_getLocalDeclWithSmallestIdx___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_hasAssignableMVar___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); static lean_object* l_Lean_MetavarContext_LevelMVarToParam_instMonadCacheExprStructEqExprM___closed__1; lean_object* l_Lean_Name_toString(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_MetavarKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); @@ -717,6 +721,7 @@ uint8_t l_Lean_Expr_hasExprMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_instantiateExprMVars___spec__13___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__6(lean_object*, lean_object*); +lean_object* l_Lean_simpLevelMax_x27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_MkBinding_abstractRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateExprMVars___spec__34(lean_object*, lean_object*); @@ -763,6 +768,7 @@ LEAN_EXPORT lean_object* l_Lean_MetavarContext_MkBinding_elimMVarDeps(lean_objec LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__104(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_instantiateExprMVars___spec__48(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_MetavarContext_MkBinding_instToStringException___spec__1(lean_object*, size_t, size_t, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Expr_getRevArg_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_StateRefT_x27_get___at_Lean_MetavarContext_instMonadMCtxStateRefT_x27MetavarContextST___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__24(lean_object*); @@ -787,6 +793,7 @@ LEAN_EXPORT lean_object* l_Lean_instantiateMVarDeclMVars___rarg___lambda__1___bo LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAux___at_Lean_isExprMVarAssigned___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_LevelMVarToParam_State_cache___default; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_erase___at_Lean_MetavarContext_setMVarUserName___spec__1(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getLevelMVarAssignment_x3f(lean_object*); LEAN_EXPORT lean_object* l_StateRefT_x27_get___at_Lean_instMonadMCtxStateRefT_x27MetavarContextST___spec__1___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at_Lean_localDeclDependsOn_x27___spec__38(lean_object*, lean_object*); @@ -798,6 +805,7 @@ LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAtAux___at_Lean_isMVarD LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_instantiateLCtxMVars___spec__12(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__29___rarg(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_MetavarContext_getDecl___closed__3; +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__9(lean_object*, lean_object*, size_t, size_t); @@ -1010,7 +1018,6 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v LEAN_EXPORT lean_object* l_Lean_isMVarDelayedAssigned___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__83___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_instantiateMVarsCore___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at_Lean_localDeclDependsOn_x27___spec__47___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_instantiateExprMVars___spec__48___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1053,7 +1060,6 @@ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_v LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateExprMVars___spec__27___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__13(lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_localDeclDependsOn___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_foldlMAux___at_Lean_MetavarContext_getExprAssignmentDomain___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1142,10 +1148,10 @@ LEAN_EXPORT lean_object* l_Std_PersistentArray_foldlM___at_Lean_instantiateLCtxM LEAN_EXPORT lean_object* l_Nat_forM_loop___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__115(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_MetavarContext_addLevelMVarDecl___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__72(lean_object*, lean_object*, size_t, size_t); +size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__12___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__38___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateExprMVars___spec__19___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*); -lean_object* lean_level_update_imax(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVarDeclMVars___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_assignLevelMVar___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isExprMVarAssignable___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimMVar___spec__1___boxed(lean_object*, lean_object*, lean_object*); @@ -1157,6 +1163,7 @@ LEAN_EXPORT lean_object* l_List_mapM___at_Lean_instantiateMVarsCore___spec__12(l LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_localDeclDependsOn___spec__9(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_index(lean_object*); +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__88(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT uint8_t l_Lean_MetavarKind_isSyntheticOpaque(uint8_t); LEAN_EXPORT lean_object* l_Lean_exprDependsOn_x27___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1164,7 +1171,6 @@ LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_localDeclDependsOn___spec__ LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__69___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_instMonadMCtxStateRefT_x27MetavarContextST(lean_object*); static lean_object* l_Lean_instantiateExprMVars___rarg___lambda__18___closed__1; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_instantiateLCtxMVars___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_mkAuxMVarType_abstractRangeAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashSet___at_Lean_DependsOn_State_visited___default___spec__1(lean_object*); @@ -1220,7 +1226,6 @@ uint8_t l_Lean_Expr_isMVar(lean_object*); uint8_t lean_expr_equal(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__69(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isExprMVarAssigned___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_sort(lean_object*, lean_object*); extern lean_object* l_Id_instMonadId; static lean_object* l___private_Lean_MetavarContext_0__Lean_reprMetavarKind____x40_Lean_MetavarContext___hyg_101____closed__2; LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at_Lean_localDeclDependsOn___spec__36(lean_object*, lean_object*); @@ -1388,12 +1393,10 @@ LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__70___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_instantiateMVarsCore___spec__18___boxed(lean_object*, lean_object*); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MetavarContext_isWellFormed___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_MetavarContext_MkBinding_collectForwardDeps___spec__112(lean_object*, lean_object*, size_t, size_t); lean_object* l_panic___at_Lean_TSyntax_getNat___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimApp___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_level_update_succ(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_anyM___at_Lean_hasAssignableMVar___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at_Lean_getDelayedMVarAssignment_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Std_Data_PersistentArray_0__Std_PersistentArray_foldlFromMAux___at_Lean_instantiateLCtxMVars___spec__3___rarg___closed__1; @@ -1459,6 +1462,7 @@ lean_object* l___private_Lean_Expr_0__Lean_mkAppRangeAux(lean_object*, lean_obje LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateExprMVars___spec__22___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__21(lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_DependsOn_instMonadMCtxM___spec__2___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at_Lean_MetavarContext_findUserName_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_assignDelayedMVar___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_elimMVar___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1516,6 +1520,7 @@ LEAN_EXPORT lean_object* l_Lean_MetavarContext_lAssignment___default; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_instantiateLCtxMVars___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_exprDependsOn___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_isLevelMVarAssignable___rarg___lambda__1___closed__4; +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_instantiateExprMVars___spec__48___rarg___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_assignExprMVar___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonadReaderT___rarg(lean_object*); @@ -1635,6 +1640,7 @@ LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at_Lean_exprDependsOn___sp LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_localDeclDependsOn_x27___spec__25(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Nat_foldRevM_loop___at___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_mkAuxMVarType___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_MetavarContext_MkBinding_instMonadMCtxM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_instantiateLCtxMVars___spec__8___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_markUsedAssignment___at_Lean_instantiateMVarsCore___spec__11___boxed(lean_object*, lean_object*); @@ -1721,7 +1727,6 @@ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_exprDependsOn___spec__ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_localDeclDependsOn___spec__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_localDeclDependsOn(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_localDeclDependsOn___spec__16(lean_object*, lean_object*, size_t, size_t); -lean_object* lean_expr_update_const(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateExprMVars___spec__35___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__35(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_instantiateMVarsCore___spec__20(lean_object*); @@ -8228,7 +8233,7 @@ static lean_object* _init_l_Lean_instantiateLevelMVars___rarg___lambda__1___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateSucc!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateSucc!Impl", 48); return x_1; } } @@ -8246,8 +8251,8 @@ static lean_object* _init_l_Lean_instantiateLevelMVars___rarg___lambda__1___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__1; x_2 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(538u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(527u); +x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -8258,32 +8263,50 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__1(lean_ob { if (lean_obj_tag(x_2) == 1) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); lean_dec(x_1); x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); lean_dec(x_4); -x_6 = lean_level_update_succ(x_2, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ptr_addr(x_6); +lean_dec(x_6); +x_8 = lean_ptr_addr(x_3); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_2); +x_10 = l_Lean_Level_succ___override(x_3); +x_11 = lean_apply_2(x_5, lean_box(0), x_10); +return x_11; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_12; +lean_dec(x_3); +x_12 = lean_apply_2(x_5, lean_box(0), x_2); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_3); lean_dec(x_2); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__4; -x_11 = l_panic___at_Lean_Level_normalize___spec__1(x_10); -x_12 = lean_apply_2(x_9, lean_box(0), x_11); -return x_12; +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__4; +x_16 = l_panic___at_Lean_Level_normalize___spec__1(x_15); +x_17 = lean_apply_2(x_14, lean_box(0), x_16); +return x_17; } } } @@ -8291,7 +8314,7 @@ static lean_object* _init_l_Lean_instantiateLevelMVars___rarg___lambda__2___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateMax!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateMax!Impl", 47); return x_1; } } @@ -8309,8 +8332,8 @@ static lean_object* _init_l_Lean_instantiateLevelMVars___rarg___lambda__2___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__1; x_2 = l_Lean_instantiateLevelMVars___rarg___lambda__2___closed__1; -x_3 = lean_unsigned_to_nat(547u); -x_4 = lean_unsigned_to_nat(14u); +x_3 = lean_unsigned_to_nat(538u); +x_4 = lean_unsigned_to_nat(19u); x_5 = l_Lean_instantiateLevelMVars___rarg___lambda__2___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -8321,33 +8344,64 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__2(lean_ob { if (lean_obj_tag(x_2) == 2) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_level_update_max(x_2, x_3, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_ctor_get(x_2, 1); +x_9 = lean_ptr_addr(x_7); +x_10 = lean_ptr_addr(x_3); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = l_Lean_mkLevelMax_x27(x_3, x_4); +x_13 = lean_apply_2(x_6, lean_box(0), x_12); +return x_13; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +size_t x_14; size_t x_15; uint8_t x_16; +x_14 = lean_ptr_addr(x_8); +x_15 = lean_ptr_addr(x_4); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = l_Lean_mkLevelMax_x27(x_3, x_4); +x_18 = lean_apply_2(x_6, lean_box(0), x_17); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; +x_19 = l_Lean_simpLevelMax_x27(x_3, x_4, x_2); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); +x_20 = lean_apply_2(x_6, lean_box(0), x_19); +return x_20; +} +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_dec(x_4); +lean_dec(x_3); +x_21 = lean_ctor_get(x_1, 0); +lean_inc(x_21); lean_dec(x_1); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = l_Lean_instantiateLevelMVars___rarg___lambda__2___closed__3; -x_12 = l_panic___at_Lean_Level_normalize___spec__1(x_11); -x_13 = lean_apply_2(x_10, lean_box(0), x_12); -return x_13; +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_23 = l_Lean_instantiateLevelMVars___rarg___lambda__2___closed__3; +x_24 = l_panic___at_Lean_Level_normalize___spec__1(x_23); +x_25 = lean_apply_2(x_22, lean_box(0), x_24); +return x_25; } } } @@ -8357,7 +8411,7 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__3(lean_ob lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_inc(x_1); x_7 = l_Lean_instantiateLevelMVars___rarg(x_1, x_2, x_3); -x_8 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___rarg___lambda__2), 4, 3); +x_8 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___rarg___lambda__2___boxed), 4, 3); lean_closure_set(x_8, 0, x_1); lean_closure_set(x_8, 1, x_4); lean_closure_set(x_8, 2, x_6); @@ -8369,7 +8423,7 @@ static lean_object* _init_l_Lean_instantiateLevelMVars___rarg___lambda__4___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Level.updateIMax!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Level.0.Lean.Level.updateIMax!Impl", 48); return x_1; } } @@ -8387,8 +8441,8 @@ static lean_object* _init_l_Lean_instantiateLevelMVars___rarg___lambda__4___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__1; x_2 = l_Lean_instantiateLevelMVars___rarg___lambda__4___closed__1; -x_3 = lean_unsigned_to_nat(556u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(549u); +x_4 = lean_unsigned_to_nat(20u); x_5 = l_Lean_instantiateLevelMVars___rarg___lambda__4___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -8399,33 +8453,62 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__4(lean_ob { if (lean_obj_tag(x_2) == 3) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_level_update_imax(x_2, x_3, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_ctor_get(x_2, 1); +x_9 = lean_ptr_addr(x_7); +x_10 = lean_ptr_addr(x_3); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = l_Lean_mkLevelIMax_x27(x_3, x_4); +x_13 = lean_apply_2(x_6, lean_box(0), x_12); +return x_13; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +size_t x_14; size_t x_15; uint8_t x_16; +x_14 = lean_ptr_addr(x_8); +x_15 = lean_ptr_addr(x_4); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = l_Lean_mkLevelIMax_x27(x_3, x_4); +x_18 = lean_apply_2(x_6, lean_box(0), x_17); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; +x_19 = l_Lean_simpLevelIMax_x27(x_3, x_4, x_2); +x_20 = lean_apply_2(x_6, lean_box(0), x_19); +return x_20; +} +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); +x_21 = lean_ctor_get(x_1, 0); +lean_inc(x_21); lean_dec(x_1); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = l_Lean_instantiateLevelMVars___rarg___lambda__4___closed__3; -x_12 = l_panic___at_Lean_Level_normalize___spec__1(x_11); -x_13 = lean_apply_2(x_10, lean_box(0), x_12); -return x_13; +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_23 = l_Lean_instantiateLevelMVars___rarg___lambda__4___closed__3; +x_24 = l_panic___at_Lean_Level_normalize___spec__1(x_23); +x_25 = lean_apply_2(x_22, lean_box(0), x_24); +return x_25; } } } @@ -8435,7 +8518,7 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__5(lean_ob lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_inc(x_1); x_7 = l_Lean_instantiateLevelMVars___rarg(x_1, x_2, x_3); -x_8 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___rarg___lambda__4), 4, 3); +x_8 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___rarg___lambda__4___boxed), 4, 3); lean_closure_set(x_8, 0, x_1); lean_closure_set(x_8, 1, x_4); lean_closure_set(x_8, 2, x_6); @@ -8632,6 +8715,24 @@ x_2 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___rarg), 3, 0); return x_2; } } +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_instantiateLevelMVars___rarg___lambda__2(x_1, x_2, x_3, x_4); +lean_dec(x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_instantiateLevelMVars___rarg___lambda__4(x_1, x_2, x_3, x_4); +lean_dec(x_2); +return x_5; +} +} LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_instantiateExprMVars___spec__2(lean_object* x_1, lean_object* x_2) { _start: { @@ -9185,32 +9286,56 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprM { if (lean_obj_tag(x_1) == 1) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_level_update_succ(x_1, x_3); -x_5 = lean_ctor_get(x_2, 0); -lean_inc(x_5); +lean_object* x_4; size_t x_5; size_t x_6; uint8_t x_7; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_6 = lean_ptr_addr(x_3); +x_7 = lean_usize_dec_eq(x_5, x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_1); +x_8 = l_Lean_Level_succ___override(x_3); +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); lean_dec(x_2); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_apply_2(x_6, lean_box(0), x_4); -return x_7; +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = lean_apply_2(x_10, lean_box(0), x_8); +return x_11; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_dec(x_3); +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); +lean_dec(x_2); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_apply_2(x_13, lean_box(0), x_1); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_dec(x_3); lean_dec(x_1); -x_8 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__4; -x_9 = l_panic___at_Lean_Level_normalize___spec__1(x_8); -x_10 = lean_ctor_get(x_2, 0); -lean_inc(x_10); +x_15 = l_Lean_instantiateLevelMVars___rarg___lambda__1___closed__4; +x_16 = l_panic___at_Lean_Level_normalize___spec__1(x_15); +x_17 = lean_ctor_get(x_2, 0); +lean_inc(x_17); lean_dec(x_2); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_apply_2(x_11, lean_box(0), x_9); -return x_12; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = lean_apply_2(x_18, lean_box(0), x_16); +return x_19; } } } @@ -9219,25 +9344,16 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprM { if (lean_obj_tag(x_1) == 2) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_level_update_max(x_1, x_3, x_4); -x_6 = lean_ctor_get(x_2, 0); -lean_inc(x_6); -lean_dec(x_2); -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_apply_2(x_7, lean_box(0), x_5); -return x_8; -} -else +lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_1, 1); +x_7 = lean_ptr_addr(x_5); +x_8 = lean_ptr_addr(x_3); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_9 = l_Lean_instantiateLevelMVars___rarg___lambda__2___closed__3; -x_10 = l_panic___at_Lean_Level_normalize___spec__1(x_9); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = l_Lean_mkLevelMax_x27(x_3, x_4); x_11 = lean_ctor_get(x_2, 0); lean_inc(x_11); lean_dec(x_2); @@ -9247,6 +9363,58 @@ lean_dec(x_11); x_13 = lean_apply_2(x_12, lean_box(0), x_10); return x_13; } +else +{ +size_t x_14; size_t x_15; uint8_t x_16; +x_14 = lean_ptr_addr(x_6); +x_15 = lean_ptr_addr(x_4); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = l_Lean_mkLevelMax_x27(x_3, x_4); +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +lean_dec(x_2); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_apply_2(x_19, lean_box(0), x_17); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = l_Lean_simpLevelMax_x27(x_3, x_4, x_1); +lean_dec(x_4); +lean_dec(x_3); +x_22 = lean_ctor_get(x_2, 0); +lean_inc(x_22); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_apply_2(x_23, lean_box(0), x_21); +return x_24; +} +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_4); +lean_dec(x_3); +x_25 = l_Lean_instantiateLevelMVars___rarg___lambda__2___closed__3; +x_26 = l_panic___at_Lean_Level_normalize___spec__1(x_25); +x_27 = lean_ctor_get(x_2, 0); +lean_inc(x_27); +lean_dec(x_2); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_apply_2(x_28, lean_box(0), x_26); +return x_29; +} } } LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { @@ -9255,7 +9423,7 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprM lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_inc(x_1); x_9 = l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg(x_1, x_2, x_3, x_4, x_5); -x_10 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__2), 4, 3); +x_10 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__2___boxed), 4, 3); lean_closure_set(x_10, 0, x_6); lean_closure_set(x_10, 1, x_1); lean_closure_set(x_10, 2, x_8); @@ -9268,25 +9436,16 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprM { if (lean_obj_tag(x_1) == 3) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_level_update_imax(x_1, x_3, x_4); -x_6 = lean_ctor_get(x_2, 0); -lean_inc(x_6); -lean_dec(x_2); -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_apply_2(x_7, lean_box(0), x_5); -return x_8; -} -else +lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_1, 1); +x_7 = lean_ptr_addr(x_5); +x_8 = lean_ptr_addr(x_3); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_9 = l_Lean_instantiateLevelMVars___rarg___lambda__4___closed__3; -x_10 = l_panic___at_Lean_Level_normalize___spec__1(x_9); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = l_Lean_mkLevelIMax_x27(x_3, x_4); x_11 = lean_ctor_get(x_2, 0); lean_inc(x_11); lean_dec(x_2); @@ -9296,6 +9455,56 @@ lean_dec(x_11); x_13 = lean_apply_2(x_12, lean_box(0), x_10); return x_13; } +else +{ +size_t x_14; size_t x_15; uint8_t x_16; +x_14 = lean_ptr_addr(x_6); +x_15 = lean_ptr_addr(x_4); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = l_Lean_mkLevelIMax_x27(x_3, x_4); +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +lean_dec(x_2); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_apply_2(x_19, lean_box(0), x_17); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = l_Lean_simpLevelIMax_x27(x_3, x_4, x_1); +x_22 = lean_ctor_get(x_2, 0); +lean_inc(x_22); +lean_dec(x_2); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_apply_2(x_23, lean_box(0), x_21); +return x_24; +} +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_4); +lean_dec(x_3); +x_25 = l_Lean_instantiateLevelMVars___rarg___lambda__4___closed__3; +x_26 = l_panic___at_Lean_Level_normalize___spec__1(x_25); +x_27 = lean_ctor_get(x_2, 0); +lean_inc(x_27); +lean_dec(x_2); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_apply_2(x_28, lean_box(0), x_26); +return x_29; +} } } LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { @@ -9304,7 +9513,7 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprM lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_inc(x_1); x_9 = l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg(x_1, x_2, x_3, x_4, x_5); -x_10 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__4), 4, 3); +x_10 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__4___boxed), 4, 3); lean_closure_set(x_10, 0, x_6); lean_closure_set(x_10, 1, x_1); lean_closure_set(x_10, 2, x_8); @@ -9618,7 +9827,7 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprM lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_inc(x_1); x_9 = l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__15___rarg(x_1, x_2, x_3, x_4, x_5); -x_10 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__2), 4, 3); +x_10 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__2___boxed), 4, 3); lean_closure_set(x_10, 0, x_6); lean_closure_set(x_10, 1, x_1); lean_closure_set(x_10, 2, x_8); @@ -9632,7 +9841,7 @@ LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprM lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_inc(x_1); x_9 = l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__15___rarg(x_1, x_2, x_3, x_4, x_5); -x_10 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__4), 4, 3); +x_10 = lean_alloc_closure((void*)(l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__4___boxed), 4, 3); lean_closure_set(x_10, 0, x_6); lean_closure_set(x_10, 1, x_1); lean_closure_set(x_10, 2, x_8); @@ -13203,7 +13412,7 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__9___close _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateSort!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateSort!Impl", 46); return x_1; } } @@ -13221,8 +13430,8 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__9___close lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__1; x_2 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__2; -x_3 = lean_unsigned_to_nat(1099u); -x_4 = lean_unsigned_to_nat(16u); +x_3 = lean_unsigned_to_nat(1423u); +x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -13233,32 +13442,50 @@ LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__9(lean_obj { if (lean_obj_tag(x_2) == 3) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); lean_dec(x_1); x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); lean_dec(x_4); -x_6 = lean_expr_update_sort(x_2, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ptr_addr(x_6); +lean_dec(x_6); +x_8 = lean_ptr_addr(x_3); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_2); +x_10 = l_Lean_Expr_sort___override(x_3); +x_11 = lean_apply_2(x_5, lean_box(0), x_10); +return x_11; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_12; +lean_dec(x_3); +x_12 = lean_apply_2(x_5, lean_box(0), x_2); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_3); lean_dec(x_2); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__4; -x_11 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_10); -x_12 = lean_apply_2(x_9, lean_box(0), x_11); -return x_12; +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__4; +x_16 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_15); +x_17 = lean_apply_2(x_14, lean_box(0), x_16); +return x_17; } } } @@ -13266,7 +13493,7 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__10___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateConst!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateConst!Impl", 47); return x_1; } } @@ -13284,8 +13511,8 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__10___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__1; x_2 = l_Lean_instantiateExprMVars___rarg___lambda__10___closed__1; -x_3 = lean_unsigned_to_nat(1090u); -x_4 = lean_unsigned_to_nat(20u); +x_3 = lean_unsigned_to_nat(1412u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_instantiateExprMVars___rarg___lambda__10___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -13296,32 +13523,51 @@ LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__10(lean_ob { if (lean_obj_tag(x_2) == 4) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); lean_dec(x_1); x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); lean_dec(x_4); -x_6 = lean_expr_update_const(x_2, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +x_8 = l_ptrEqList___rarg(x_7, x_3); +lean_dec(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_9 = l_Lean_Expr_const___override(x_6, x_3); +x_10 = lean_apply_2(x_5, lean_box(0), x_9); +return x_10; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_11; +lean_dec(x_6); +lean_dec(x_3); +x_11 = lean_apply_2(x_5, lean_box(0), x_2); +return x_11; +} +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_dec(x_3); lean_dec(x_2); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = l_Lean_instantiateExprMVars___rarg___lambda__10___closed__3; -x_11 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_10); -x_12 = lean_apply_2(x_9, lean_box(0), x_11); -return x_12; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = l_Lean_instantiateExprMVars___rarg___lambda__10___closed__3; +x_15 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_14); +x_16 = lean_apply_2(x_13, lean_box(0), x_15); +return x_16; } } } @@ -13347,8 +13593,8 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__11___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__1; x_2 = l_Lean_instantiateExprMVars___rarg___lambda__11___closed__1; -x_3 = lean_unsigned_to_nat(1149u); -x_4 = lean_unsigned_to_nat(19u); +x_3 = lean_unsigned_to_nat(1491u); +x_4 = lean_unsigned_to_nat(20u); x_5 = l_Lean_instantiateExprMVars___rarg___lambda__11___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -13359,34 +13605,93 @@ LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__11(lean_ob { if (lean_obj_tag(x_2) == 6) { -lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; +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; size_t x_12; size_t x_13; uint8_t x_14; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_8 = lean_expr_update_lambda(x_2, x_7, x_3, x_4); -x_9 = lean_apply_2(x_6, lean_box(0), x_8); -return x_9; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_2, 1); +lean_inc(x_8); +x_9 = lean_ctor_get(x_2, 2); +lean_inc(x_9); +x_10 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_11 = l_Lean_Expr_lam___override(x_7, x_8, x_9, x_10); +x_12 = lean_ptr_addr(x_8); +lean_dec(x_8); +x_13 = lean_ptr_addr(x_3); +x_14 = lean_usize_dec_eq(x_12, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_11); +lean_dec(x_9); +x_15 = l_Lean_Expr_lam___override(x_7, x_3, x_4, x_10); +x_16 = lean_apply_2(x_6, lean_box(0), x_15); +return x_16; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +size_t x_17; size_t x_18; uint8_t x_19; +x_17 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_18 = lean_ptr_addr(x_4); +x_19 = lean_usize_dec_eq(x_17, x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +lean_dec(x_11); +x_20 = l_Lean_Expr_lam___override(x_7, x_3, x_4, x_10); +x_21 = lean_apply_2(x_6, lean_box(0), x_20); +return x_21; +} +else +{ +uint8_t x_22; +x_22 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_10, x_10); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_11); +x_23 = l_Lean_Expr_lam___override(x_7, x_3, x_4, x_10); +x_24 = lean_apply_2(x_6, lean_box(0), x_23); +return x_24; +} +else +{ +lean_object* x_25; +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +x_25 = lean_apply_2(x_6, lean_box(0), x_11); +return x_25; +} +} +} +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = l_Lean_instantiateExprMVars___rarg___lambda__11___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = lean_apply_2(x_11, lean_box(0), x_13); -return x_14; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = l_Lean_instantiateExprMVars___rarg___lambda__11___closed__3; +x_29 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_28); +x_30 = lean_apply_2(x_27, lean_box(0), x_29); +return x_30; } } } @@ -13426,8 +13731,8 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__13___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__1; x_2 = l_Lean_instantiateExprMVars___rarg___lambda__13___closed__1; -x_3 = lean_unsigned_to_nat(1135u); -x_4 = lean_unsigned_to_nat(23u); +x_3 = lean_unsigned_to_nat(1471u); +x_4 = lean_unsigned_to_nat(24u); x_5 = l_Lean_instantiateExprMVars___rarg___lambda__13___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -13438,34 +13743,93 @@ LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__13(lean_ob { if (lean_obj_tag(x_2) == 7) { -lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; +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; size_t x_12; size_t x_13; uint8_t x_14; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); -x_7 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -x_8 = lean_expr_update_forall(x_2, x_7, x_3, x_4); -x_9 = lean_apply_2(x_6, lean_box(0), x_8); -return x_9; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_2, 1); +lean_inc(x_8); +x_9 = lean_ctor_get(x_2, 2); +lean_inc(x_9); +x_10 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_11 = l_Lean_Expr_forallE___override(x_7, x_8, x_9, x_10); +x_12 = lean_ptr_addr(x_8); +lean_dec(x_8); +x_13 = lean_ptr_addr(x_3); +x_14 = lean_usize_dec_eq(x_12, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_11); +lean_dec(x_9); +x_15 = l_Lean_Expr_forallE___override(x_7, x_3, x_4, x_10); +x_16 = lean_apply_2(x_6, lean_box(0), x_15); +return x_16; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +size_t x_17; size_t x_18; uint8_t x_19; +x_17 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_18 = lean_ptr_addr(x_4); +x_19 = lean_usize_dec_eq(x_17, x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +lean_dec(x_11); +x_20 = l_Lean_Expr_forallE___override(x_7, x_3, x_4, x_10); +x_21 = lean_apply_2(x_6, lean_box(0), x_20); +return x_21; +} +else +{ +uint8_t x_22; +x_22 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_10, x_10); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_11); +x_23 = l_Lean_Expr_forallE___override(x_7, x_3, x_4, x_10); +x_24 = lean_apply_2(x_6, lean_box(0), x_23); +return x_24; +} +else +{ +lean_object* x_25; +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +x_25 = lean_apply_2(x_6, lean_box(0), x_11); +return x_25; +} +} +} +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = l_Lean_instantiateExprMVars___rarg___lambda__13___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = lean_apply_2(x_11, lean_box(0), x_13); -return x_14; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = l_Lean_instantiateExprMVars___rarg___lambda__13___closed__3; +x_29 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_28); +x_30 = lean_apply_2(x_27, lean_box(0), x_29); +return x_30; } } } @@ -13487,7 +13851,7 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__15___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateLet!", 20); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateLet!Impl", 45); return x_1; } } @@ -13505,8 +13869,8 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__15___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__1; x_2 = l_Lean_instantiateExprMVars___rarg___lambda__15___closed__1; -x_3 = lean_unsigned_to_nat(1158u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1500u); +x_4 = lean_unsigned_to_nat(22u); x_5 = l_Lean_instantiateExprMVars___rarg___lambda__15___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -13517,34 +13881,97 @@ LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__15(lean_ob { if (lean_obj_tag(x_2) == 8) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; size_t x_13; size_t x_14; uint8_t x_15; x_6 = lean_ctor_get(x_1, 0); lean_inc(x_6); lean_dec(x_1); x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); -x_8 = lean_expr_update_let(x_2, x_3, x_4, x_5); -x_9 = lean_apply_2(x_7, lean_box(0), x_8); -return x_9; +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_ctor_get(x_2, 2); +lean_inc(x_10); +x_11 = lean_ctor_get(x_2, 3); +lean_inc(x_11); +x_12 = lean_ctor_get_uint8(x_2, sizeof(void*)*4 + 8); +x_13 = lean_ptr_addr(x_9); +lean_dec(x_9); +x_14 = lean_ptr_addr(x_3); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_2); +x_16 = l_Lean_Expr_letE___override(x_8, x_3, x_4, x_5, x_12); +x_17 = lean_apply_2(x_7, lean_box(0), x_16); +return x_17; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +size_t x_18; size_t x_19; uint8_t x_20; +x_18 = lean_ptr_addr(x_10); +lean_dec(x_10); +x_19 = lean_ptr_addr(x_4); +x_20 = lean_usize_dec_eq(x_18, x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_11); +lean_dec(x_2); +x_21 = l_Lean_Expr_letE___override(x_8, x_3, x_4, x_5, x_12); +x_22 = lean_apply_2(x_7, lean_box(0), x_21); +return x_22; +} +else +{ +size_t x_23; size_t x_24; uint8_t x_25; +x_23 = lean_ptr_addr(x_11); +lean_dec(x_11); +x_24 = lean_ptr_addr(x_5); +x_25 = lean_usize_dec_eq(x_23, x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +lean_dec(x_2); +x_26 = l_Lean_Expr_letE___override(x_8, x_3, x_4, x_5, x_12); +x_27 = lean_apply_2(x_7, lean_box(0), x_26); +return x_27; +} +else +{ +lean_object* x_28; +lean_dec(x_8); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_28 = lean_apply_2(x_7, lean_box(0), x_2); +return x_28; +} +} +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +x_29 = lean_ctor_get(x_1, 0); +lean_inc(x_29); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = l_Lean_instantiateExprMVars___rarg___lambda__15___closed__3; -x_13 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_12); -x_14 = lean_apply_2(x_11, lean_box(0), x_13); -return x_14; +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +x_31 = l_Lean_instantiateExprMVars___rarg___lambda__15___closed__3; +x_32 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_31); +x_33 = lean_apply_2(x_30, lean_box(0), x_32); +return x_33; } } } @@ -13592,7 +14019,7 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__18___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateMData!", 22); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateMData!Impl", 47); return x_1; } } @@ -13610,8 +14037,8 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__18___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__1; x_2 = l_Lean_instantiateExprMVars___rarg___lambda__18___closed__1; -x_3 = lean_unsigned_to_nat(1116u); -x_4 = lean_unsigned_to_nat(16u); +x_3 = lean_unsigned_to_nat(1434u); +x_4 = lean_unsigned_to_nat(17u); x_5 = l_Lean_instantiateExprMVars___rarg___lambda__18___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -13622,32 +14049,53 @@ LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__18(lean_ob { if (lean_obj_tag(x_2) == 10) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; uint8_t x_10; x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); lean_dec(x_1); x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); lean_dec(x_4); -x_6 = lean_expr_update_mdata(x_2, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +x_8 = lean_ptr_addr(x_7); +lean_dec(x_7); +x_9 = lean_ptr_addr(x_3); +x_10 = lean_usize_dec_eq(x_8, x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +lean_dec(x_2); +x_11 = l_Lean_Expr_mdata___override(x_6, x_3); +x_12 = lean_apply_2(x_5, lean_box(0), x_11); +return x_12; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_13; +lean_dec(x_6); +lean_dec(x_3); +x_13 = lean_apply_2(x_5, lean_box(0), x_2); +return x_13; +} +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_dec(x_3); lean_dec(x_2); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +x_14 = lean_ctor_get(x_1, 0); +lean_inc(x_14); lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = l_Lean_instantiateExprMVars___rarg___lambda__18___closed__3; -x_11 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_10); -x_12 = lean_apply_2(x_9, lean_box(0), x_11); -return x_12; +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = l_Lean_instantiateExprMVars___rarg___lambda__18___closed__3; +x_17 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_16); +x_18 = lean_apply_2(x_15, lean_box(0), x_17); +return x_18; } } } @@ -13655,7 +14103,7 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__19___clos _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Expr.updateProj!", 21); +x_1 = lean_mk_string_from_bytes("_private.Lean.Expr.0.Lean.Expr.updateProj!Impl", 46); return x_1; } } @@ -13673,8 +14121,8 @@ static lean_object* _init_l_Lean_instantiateExprMVars___rarg___lambda__19___clos lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_instantiateExprMVars___rarg___lambda__9___closed__1; x_2 = l_Lean_instantiateExprMVars___rarg___lambda__19___closed__1; -x_3 = lean_unsigned_to_nat(1121u); -x_4 = lean_unsigned_to_nat(15u); +x_3 = lean_unsigned_to_nat(1445u); +x_4 = lean_unsigned_to_nat(18u); x_5 = l_Lean_instantiateExprMVars___rarg___lambda__19___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; @@ -13685,32 +14133,56 @@ LEAN_EXPORT lean_object* l_Lean_instantiateExprMVars___rarg___lambda__19(lean_ob { if (lean_obj_tag(x_2) == 11) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); lean_dec(x_1); x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); lean_dec(x_4); -x_6 = lean_expr_update_proj(x_2, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +x_8 = lean_ctor_get(x_2, 2); +lean_inc(x_8); +x_9 = lean_ptr_addr(x_8); +lean_dec(x_8); +x_10 = lean_ptr_addr(x_3); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_2); +x_12 = l_Lean_Expr_proj___override(x_6, x_7, x_3); +x_13 = lean_apply_2(x_5, lean_box(0), x_12); +return x_13; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_14; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +x_14 = lean_apply_2(x_5, lean_box(0), x_2); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_dec(x_3); lean_dec(x_2); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +x_15 = lean_ctor_get(x_1, 0); +lean_inc(x_15); lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = l_Lean_instantiateExprMVars___rarg___lambda__19___closed__3; -x_11 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_10); -x_12 = lean_apply_2(x_9, lean_box(0), x_11); -return x_12; +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = l_Lean_instantiateExprMVars___rarg___lambda__19___closed__3; +x_18 = l_panic___at_Lean_Expr_getRevArg_x21___spec__1(x_17); +x_19 = lean_apply_2(x_16, lean_box(0), x_18); +return x_19; } } } @@ -13817,7 +14289,7 @@ case 5: 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_dec(x_8); x_27 = lean_unsigned_to_nat(0u); -x_28 = l_Lean_Expr_getAppNumArgsAux(x_1, x_27); +x_28 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_27); x_29 = l_Lean_instantiateExprMVars___rarg___lambda__20___closed__1; lean_inc(x_28); x_30 = lean_mk_array(x_28, x_29); @@ -14212,6 +14684,24 @@ lean_dec(x_2); return x_6; } } +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__2(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__4(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} LEAN_EXPORT lean_object* l_Lean_instantiateLevelMVars___at_Lean_instantiateExprMVars___spec__12___rarg___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { @@ -16184,6 +16674,7 @@ case 1: lean_object* x_5; lean_object* x_6; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); +lean_inc(x_5); x_6 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_5, x_2, x_3, x_4); if (lean_obj_tag(x_6) == 0) { @@ -16191,232 +16682,227 @@ uint8_t x_7; x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) { -lean_object* x_8; lean_object* x_9; +lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_level_update_succ(x_1, x_8); -lean_ctor_set(x_6, 0, x_9); +x_9 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_10 = lean_ptr_addr(x_8); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_1); +x_12 = l_Lean_Level_succ___override(x_8); +lean_ctor_set(x_6, 0, x_12); return x_6; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_6, 0); -x_11 = lean_ctor_get(x_6, 1); -lean_inc(x_11); -lean_inc(x_10); +lean_dec(x_8); +lean_ctor_set(x_6, 0, x_1); +return x_6; +} +} +else +{ +lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_6, 0); +x_14 = lean_ctor_get(x_6, 1); +lean_inc(x_14); +lean_inc(x_13); lean_dec(x_6); -x_12 = lean_level_update_succ(x_1, x_10); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +x_15 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_16 = lean_ptr_addr(x_13); +x_17 = lean_usize_dec_eq(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_1); +x_18 = l_Lean_Level_succ___override(x_13); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_14); +return x_19; +} +else +{ +lean_object* x_20; +lean_dec(x_13); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_1); +lean_ctor_set(x_20, 1, x_14); +return x_20; +} } } else { -uint8_t x_14; +uint8_t x_21; +lean_dec(x_5); lean_dec(x_1); -x_14 = !lean_is_exclusive(x_6); -if (x_14 == 0) +x_21 = !lean_is_exclusive(x_6); +if (x_21 == 0) { return x_6; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_6, 0); -x_16 = lean_ctor_get(x_6, 1); -lean_inc(x_16); -lean_inc(x_15); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_6, 0); +x_23 = lean_ctor_get(x_6, 1); +lean_inc(x_23); +lean_inc(x_22); lean_dec(x_6); -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } } case 2: { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_1, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_1, 1); -lean_inc(x_19); -x_20 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_18, x_2, x_3, x_4); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_19, x_2, x_3, x_22); -if (lean_obj_tag(x_23) == 0) -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) -{ -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_level_update_max(x_1, x_21, x_25); -lean_ctor_set(x_23, 0, x_26); -return x_23; -} -else +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_1, 1); +lean_inc(x_26); +lean_inc(x_25); +x_27 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_25, x_2, x_3, x_4); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_23, 0); -x_28 = lean_ctor_get(x_23, 1); +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_27, 0); lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_23); -x_29 = lean_level_update_max(x_1, x_21, x_27); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -return x_30; -} -} -else +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +lean_inc(x_26); +x_30 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_26, x_2, x_3, x_29); +if (lean_obj_tag(x_30) == 0) { uint8_t x_31; -lean_dec(x_21); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_23); +x_31 = !lean_is_exclusive(x_30); if (x_31 == 0) { -return x_23; -} -else +lean_object* x_32; size_t x_33; size_t x_34; uint8_t x_35; +x_32 = lean_ctor_get(x_30, 0); +x_33 = lean_ptr_addr(x_25); +lean_dec(x_25); +x_34 = lean_ptr_addr(x_28); +x_35 = lean_usize_dec_eq(x_33, x_34); +if (x_35 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_23, 0); -x_33 = lean_ctor_get(x_23, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_23); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; -} -} +lean_object* x_36; +lean_dec(x_26); +lean_dec(x_1); +x_36 = l_Lean_mkLevelMax_x27(x_28, x_32); +lean_ctor_set(x_30, 0, x_36); +return x_30; } else { -uint8_t x_35; -lean_dec(x_19); -lean_dec(x_1); -x_35 = !lean_is_exclusive(x_20); -if (x_35 == 0) +size_t x_37; size_t x_38; uint8_t x_39; +x_37 = lean_ptr_addr(x_26); +lean_dec(x_26); +x_38 = lean_ptr_addr(x_32); +x_39 = lean_usize_dec_eq(x_37, x_38); +if (x_39 == 0) { -return x_20; +lean_object* x_40; +lean_dec(x_1); +x_40 = l_Lean_mkLevelMax_x27(x_28, x_32); +lean_ctor_set(x_30, 0, x_40); +return x_30; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_20, 0); -x_37 = lean_ctor_get(x_20, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_20); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_object* x_41; +x_41 = l_Lean_simpLevelMax_x27(x_28, x_32, x_1); +lean_dec(x_1); +lean_dec(x_32); +lean_dec(x_28); +lean_ctor_set(x_30, 0, x_41); +return x_30; } } } -case 3: -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_1, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_1, 1); -lean_inc(x_40); -x_41 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_39, x_2, x_3, x_4); -if (lean_obj_tag(x_41) == 0) +else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); +lean_object* x_42; lean_object* x_43; size_t x_44; size_t x_45; uint8_t x_46; +x_42 = lean_ctor_get(x_30, 0); +x_43 = lean_ctor_get(x_30, 1); lean_inc(x_43); -lean_dec(x_41); -x_44 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_40, x_2, x_3, x_43); -if (lean_obj_tag(x_44) == 0) -{ -uint8_t x_45; -x_45 = !lean_is_exclusive(x_44); -if (x_45 == 0) +lean_inc(x_42); +lean_dec(x_30); +x_44 = lean_ptr_addr(x_25); +lean_dec(x_25); +x_45 = lean_ptr_addr(x_28); +x_46 = lean_usize_dec_eq(x_44, x_45); +if (x_46 == 0) { -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_44, 0); -x_47 = lean_level_update_imax(x_1, x_42, x_46); -lean_ctor_set(x_44, 0, x_47); -return x_44; +lean_object* x_47; lean_object* x_48; +lean_dec(x_26); +lean_dec(x_1); +x_47 = l_Lean_mkLevelMax_x27(x_28, x_42); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_43); +return x_48; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = lean_ctor_get(x_44, 0); -x_49 = lean_ctor_get(x_44, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_44); -x_50 = lean_level_update_imax(x_1, x_42, x_48); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_49); -return x_51; -} -} -else +size_t x_49; size_t x_50; uint8_t x_51; +x_49 = lean_ptr_addr(x_26); +lean_dec(x_26); +x_50 = lean_ptr_addr(x_42); +x_51 = lean_usize_dec_eq(x_49, x_50); +if (x_51 == 0) { -uint8_t x_52; -lean_dec(x_42); +lean_object* x_52; lean_object* x_53; lean_dec(x_1); -x_52 = !lean_is_exclusive(x_44); -if (x_52 == 0) -{ -return x_44; +x_52 = l_Lean_mkLevelMax_x27(x_28, x_42); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_43); +return x_53; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_44, 0); -x_54 = lean_ctor_get(x_44, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_44); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); +lean_object* x_54; lean_object* x_55; +x_54 = l_Lean_simpLevelMax_x27(x_28, x_42, x_1); +lean_dec(x_1); +lean_dec(x_42); +lean_dec(x_28); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_43); return x_55; } } } +} else { uint8_t x_56; -lean_dec(x_40); +lean_dec(x_28); +lean_dec(x_26); +lean_dec(x_25); lean_dec(x_1); -x_56 = !lean_is_exclusive(x_41); +x_56 = !lean_is_exclusive(x_30); if (x_56 == 0) { -return x_41; +return x_30; } else { lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_41, 0); -x_58 = lean_ctor_get(x_41, 1); +x_57 = lean_ctor_get(x_30, 0); +x_58 = lean_ctor_get(x_30, 1); lean_inc(x_58); lean_inc(x_57); -lean_dec(x_41); +lean_dec(x_30); x_59 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_59, 0, x_57); lean_ctor_set(x_59, 1, x_58); @@ -16424,67 +16910,145 @@ return x_59; } } } -case 5: +else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_84; -x_60 = lean_ctor_get(x_1, 0); -lean_inc(x_60); -x_84 = lean_st_ref_get(x_3, x_4); -if (lean_obj_tag(x_84) == 0) +uint8_t x_60; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_1); +x_60 = !lean_is_exclusive(x_27); +if (x_60 == 0) { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_ctor_get(x_85, 5); -lean_inc(x_87); -lean_dec(x_85); -lean_inc(x_60); -x_88 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_87, x_60); -if (lean_obj_tag(x_88) == 0) +return x_27; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_27, 0); +x_62 = lean_ctor_get(x_27, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_27); +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +return x_63; +} +} +} +case 3: +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_1, 0); +lean_inc(x_64); +x_65 = lean_ctor_get(x_1, 1); +lean_inc(x_65); +lean_inc(x_64); +x_66 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_64, x_2, x_3, x_4); +if (lean_obj_tag(x_66) == 0) +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_66, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_66, 1); +lean_inc(x_68); +lean_dec(x_66); +lean_inc(x_65); +x_69 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_65, x_2, x_3, x_68); +if (lean_obj_tag(x_69) == 0) +{ +uint8_t x_70; +x_70 = !lean_is_exclusive(x_69); +if (x_70 == 0) +{ +lean_object* x_71; size_t x_72; size_t x_73; uint8_t x_74; +x_71 = lean_ctor_get(x_69, 0); +x_72 = lean_ptr_addr(x_64); +lean_dec(x_64); +x_73 = lean_ptr_addr(x_67); +x_74 = lean_usize_dec_eq(x_72, x_73); +if (x_74 == 0) { -x_61 = x_88; -x_62 = x_86; -goto block_83; +lean_object* x_75; +lean_dec(x_65); +lean_dec(x_1); +x_75 = l_Lean_mkLevelIMax_x27(x_67, x_71); +lean_ctor_set(x_69, 0, x_75); +return x_69; } else { -lean_object* x_89; -x_89 = l_Lean_markUsedAssignment___at_Lean_instantiateMVarsCore___spec__8___rarg(x_3, x_86); -if (lean_obj_tag(x_89) == 0) +size_t x_76; size_t x_77; uint8_t x_78; +x_76 = lean_ptr_addr(x_65); +lean_dec(x_65); +x_77 = lean_ptr_addr(x_71); +x_78 = lean_usize_dec_eq(x_76, x_77); +if (x_78 == 0) { -lean_object* x_90; -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); -lean_dec(x_89); -x_61 = x_88; -x_62 = x_90; -goto block_83; +lean_object* x_79; +lean_dec(x_1); +x_79 = l_Lean_mkLevelIMax_x27(x_67, x_71); +lean_ctor_set(x_69, 0, x_79); +return x_69; } else { -uint8_t x_91; -lean_dec(x_88); -lean_dec(x_60); +lean_object* x_80; +x_80 = l_Lean_simpLevelIMax_x27(x_67, x_71, x_1); lean_dec(x_1); -x_91 = !lean_is_exclusive(x_89); -if (x_91 == 0) +lean_ctor_set(x_69, 0, x_80); +return x_69; +} +} +} +else { -return x_89; +lean_object* x_81; lean_object* x_82; size_t x_83; size_t x_84; uint8_t x_85; +x_81 = lean_ctor_get(x_69, 0); +x_82 = lean_ctor_get(x_69, 1); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_69); +x_83 = lean_ptr_addr(x_64); +lean_dec(x_64); +x_84 = lean_ptr_addr(x_67); +x_85 = lean_usize_dec_eq(x_83, x_84); +if (x_85 == 0) +{ +lean_object* x_86; lean_object* x_87; +lean_dec(x_65); +lean_dec(x_1); +x_86 = l_Lean_mkLevelIMax_x27(x_67, x_81); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_82); +return x_87; } else { -lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_92 = lean_ctor_get(x_89, 0); -x_93 = lean_ctor_get(x_89, 1); -lean_inc(x_93); -lean_inc(x_92); -lean_dec(x_89); -x_94 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_94, 0, x_92); -lean_ctor_set(x_94, 1, x_93); +size_t x_88; size_t x_89; uint8_t x_90; +x_88 = lean_ptr_addr(x_65); +lean_dec(x_65); +x_89 = lean_ptr_addr(x_81); +x_90 = lean_usize_dec_eq(x_88, x_89); +if (x_90 == 0) +{ +lean_object* x_91; lean_object* x_92; +lean_dec(x_1); +x_91 = l_Lean_mkLevelIMax_x27(x_67, x_81); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_82); +return x_92; +} +else +{ +lean_object* x_93; lean_object* x_94; +x_93 = l_Lean_simpLevelIMax_x27(x_67, x_81, x_1); +lean_dec(x_1); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_82); return x_94; } } @@ -16493,138 +17057,257 @@ return x_94; else { uint8_t x_95; -lean_dec(x_60); +lean_dec(x_67); +lean_dec(x_65); +lean_dec(x_64); lean_dec(x_1); -x_95 = !lean_is_exclusive(x_84); +x_95 = !lean_is_exclusive(x_69); if (x_95 == 0) { -return x_84; +return x_69; } else { lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_96 = lean_ctor_get(x_84, 0); -x_97 = lean_ctor_get(x_84, 1); +x_96 = lean_ctor_get(x_69, 0); +x_97 = lean_ctor_get(x_69, 1); lean_inc(x_97); lean_inc(x_96); -lean_dec(x_84); +lean_dec(x_69); x_98 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_98, 0, x_96); lean_ctor_set(x_98, 1, x_97); return x_98; } } -block_83: +} +else { -if (lean_obj_tag(x_61) == 0) +uint8_t x_99; +lean_dec(x_65); +lean_dec(x_64); +lean_dec(x_1); +x_99 = !lean_is_exclusive(x_66); +if (x_99 == 0) { -lean_object* x_63; -lean_dec(x_60); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_1); -lean_ctor_set(x_63, 1, x_62); -return x_63; +return x_66; +} +else +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_66, 0); +x_101 = lean_ctor_get(x_66, 1); +lean_inc(x_101); +lean_inc(x_100); +lean_dec(x_66); +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_100); +lean_ctor_set(x_102, 1, x_101); +return x_102; +} +} +} +case 5: +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_127; +x_103 = lean_ctor_get(x_1, 0); +lean_inc(x_103); +x_127 = lean_st_ref_get(x_3, x_4); +if (lean_obj_tag(x_127) == 0) +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_128 = lean_ctor_get(x_127, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_127, 1); +lean_inc(x_129); +lean_dec(x_127); +x_130 = lean_ctor_get(x_128, 5); +lean_inc(x_130); +lean_dec(x_128); +lean_inc(x_103); +x_131 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_130, x_103); +if (lean_obj_tag(x_131) == 0) +{ +x_104 = x_131; +x_105 = x_129; +goto block_126; +} +else +{ +lean_object* x_132; +x_132 = l_Lean_markUsedAssignment___at_Lean_instantiateMVarsCore___spec__8___rarg(x_3, x_129); +if (lean_obj_tag(x_132) == 0) +{ +lean_object* x_133; +x_133 = lean_ctor_get(x_132, 1); +lean_inc(x_133); +lean_dec(x_132); +x_104 = x_131; +x_105 = x_133; +goto block_126; } else { -lean_object* x_64; uint8_t x_65; +uint8_t x_134; +lean_dec(x_131); +lean_dec(x_103); lean_dec(x_1); -x_64 = lean_ctor_get(x_61, 0); -lean_inc(x_64); -lean_dec(x_61); -x_65 = l_Lean_Level_hasMVar(x_64); -if (x_65 == 0) +x_134 = !lean_is_exclusive(x_132); +if (x_134 == 0) { -lean_object* x_66; -lean_dec(x_60); -x_66 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_62); -return x_66; +return x_132; } else { -lean_object* x_67; -x_67 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_64, x_2, x_3, x_62); -if (lean_obj_tag(x_67) == 0) +lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_135 = lean_ctor_get(x_132, 0); +x_136 = lean_ctor_get(x_132, 1); +lean_inc(x_136); +lean_inc(x_135); +lean_dec(x_132); +x_137 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_137, 0, x_135); +lean_ctor_set(x_137, 1, x_136); +return x_137; +} +} +} +} +else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -lean_inc(x_68); -x_70 = l_Lean_assignLevelMVar___at_Lean_instantiateMVarsCore___spec__7___rarg(x_60, x_68, x_2, x_3, x_69); -if (lean_obj_tag(x_70) == 0) +uint8_t x_138; +lean_dec(x_103); +lean_dec(x_1); +x_138 = !lean_is_exclusive(x_127); +if (x_138 == 0) { -uint8_t x_71; -x_71 = !lean_is_exclusive(x_70); -if (x_71 == 0) +return x_127; +} +else { -lean_object* x_72; -x_72 = lean_ctor_get(x_70, 0); -lean_dec(x_72); -lean_ctor_set(x_70, 0, x_68); -return x_70; +lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_139 = lean_ctor_get(x_127, 0); +x_140 = lean_ctor_get(x_127, 1); +lean_inc(x_140); +lean_inc(x_139); +lean_dec(x_127); +x_141 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_141, 0, x_139); +lean_ctor_set(x_141, 1, x_140); +return x_141; +} +} +block_126: +{ +if (lean_obj_tag(x_104) == 0) +{ +lean_object* x_106; +lean_dec(x_103); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_1); +lean_ctor_set(x_106, 1, x_105); +return x_106; } else { -lean_object* x_73; lean_object* x_74; -x_73 = lean_ctor_get(x_70, 1); -lean_inc(x_73); -lean_dec(x_70); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_68); -lean_ctor_set(x_74, 1, x_73); -return x_74; +lean_object* x_107; uint8_t x_108; +lean_dec(x_1); +x_107 = lean_ctor_get(x_104, 0); +lean_inc(x_107); +lean_dec(x_104); +x_108 = l_Lean_Level_hasMVar(x_107); +if (x_108 == 0) +{ +lean_object* x_109; +lean_dec(x_103); +x_109 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 1, x_105); +return x_109; } +else +{ +lean_object* x_110; +x_110 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_107, x_2, x_3, x_105); +if (lean_obj_tag(x_110) == 0) +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +lean_dec(x_110); +lean_inc(x_111); +x_113 = l_Lean_assignLevelMVar___at_Lean_instantiateMVarsCore___spec__7___rarg(x_103, x_111, x_2, x_3, x_112); +if (lean_obj_tag(x_113) == 0) +{ +uint8_t x_114; +x_114 = !lean_is_exclusive(x_113); +if (x_114 == 0) +{ +lean_object* x_115; +x_115 = lean_ctor_get(x_113, 0); +lean_dec(x_115); +lean_ctor_set(x_113, 0, x_111); +return x_113; } else { -uint8_t x_75; -lean_dec(x_68); -x_75 = !lean_is_exclusive(x_70); -if (x_75 == 0) +lean_object* x_116; lean_object* x_117; +x_116 = lean_ctor_get(x_113, 1); +lean_inc(x_116); +lean_dec(x_113); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_111); +lean_ctor_set(x_117, 1, x_116); +return x_117; +} +} +else { -return x_70; +uint8_t x_118; +lean_dec(x_111); +x_118 = !lean_is_exclusive(x_113); +if (x_118 == 0) +{ +return x_113; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_70, 0); -x_77 = lean_ctor_get(x_70, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_70); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_ctor_get(x_113, 0); +x_120 = lean_ctor_get(x_113, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_113); +x_121 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_121, 0, x_119); +lean_ctor_set(x_121, 1, x_120); +return x_121; } } } else { -uint8_t x_79; -lean_dec(x_60); -x_79 = !lean_is_exclusive(x_67); -if (x_79 == 0) +uint8_t x_122; +lean_dec(x_103); +x_122 = !lean_is_exclusive(x_110); +if (x_122 == 0) { -return x_67; +return x_110; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_80 = lean_ctor_get(x_67, 0); -x_81 = lean_ctor_get(x_67, 1); -lean_inc(x_81); -lean_inc(x_80); -lean_dec(x_67); -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -return x_82; +lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_123 = lean_ctor_get(x_110, 0); +x_124 = lean_ctor_get(x_110, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_110); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +return x_125; } } } @@ -16633,11 +17316,11 @@ return x_82; } default: { -lean_object* x_99; -x_99 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_99, 0, x_1); -lean_ctor_set(x_99, 1, x_4); -return x_99; +lean_object* x_142; +x_142 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_142, 0, x_1); +lean_ctor_set(x_142, 1, x_4); +return x_142; } } } @@ -17029,6 +17712,7 @@ case 1: lean_object* x_5; lean_object* x_6; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); +lean_inc(x_5); x_6 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_5, x_2, x_3, x_4); if (lean_obj_tag(x_6) == 0) { @@ -17036,232 +17720,227 @@ uint8_t x_7; x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) { -lean_object* x_8; lean_object* x_9; +lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_level_update_succ(x_1, x_8); -lean_ctor_set(x_6, 0, x_9); +x_9 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_10 = lean_ptr_addr(x_8); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_1); +x_12 = l_Lean_Level_succ___override(x_8); +lean_ctor_set(x_6, 0, x_12); return x_6; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_6, 0); -x_11 = lean_ctor_get(x_6, 1); -lean_inc(x_11); -lean_inc(x_10); +lean_dec(x_8); +lean_ctor_set(x_6, 0, x_1); +return x_6; +} +} +else +{ +lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_6, 0); +x_14 = lean_ctor_get(x_6, 1); +lean_inc(x_14); +lean_inc(x_13); lean_dec(x_6); -x_12 = lean_level_update_succ(x_1, x_10); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +x_15 = lean_ptr_addr(x_5); +lean_dec(x_5); +x_16 = lean_ptr_addr(x_13); +x_17 = lean_usize_dec_eq(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_1); +x_18 = l_Lean_Level_succ___override(x_13); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_14); +return x_19; +} +else +{ +lean_object* x_20; +lean_dec(x_13); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_1); +lean_ctor_set(x_20, 1, x_14); +return x_20; +} } } else { -uint8_t x_14; +uint8_t x_21; +lean_dec(x_5); lean_dec(x_1); -x_14 = !lean_is_exclusive(x_6); -if (x_14 == 0) +x_21 = !lean_is_exclusive(x_6); +if (x_21 == 0) { return x_6; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_6, 0); -x_16 = lean_ctor_get(x_6, 1); -lean_inc(x_16); -lean_inc(x_15); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_6, 0); +x_23 = lean_ctor_get(x_6, 1); +lean_inc(x_23); +lean_inc(x_22); lean_dec(x_6); -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } } case 2: { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_1, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_1, 1); -lean_inc(x_19); -x_20 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_18, x_2, x_3, x_4); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_19, x_2, x_3, x_22); -if (lean_obj_tag(x_23) == 0) -{ -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) -{ -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_level_update_max(x_1, x_21, x_25); -lean_ctor_set(x_23, 0, x_26); -return x_23; -} -else +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_1, 1); +lean_inc(x_26); +lean_inc(x_25); +x_27 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_25, x_2, x_3, x_4); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_23, 0); -x_28 = lean_ctor_get(x_23, 1); +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_27, 0); lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_23); -x_29 = lean_level_update_max(x_1, x_21, x_27); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -return x_30; -} -} -else +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +lean_inc(x_26); +x_30 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_26, x_2, x_3, x_29); +if (lean_obj_tag(x_30) == 0) { uint8_t x_31; -lean_dec(x_21); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_23); +x_31 = !lean_is_exclusive(x_30); if (x_31 == 0) { -return x_23; -} -else +lean_object* x_32; size_t x_33; size_t x_34; uint8_t x_35; +x_32 = lean_ctor_get(x_30, 0); +x_33 = lean_ptr_addr(x_25); +lean_dec(x_25); +x_34 = lean_ptr_addr(x_28); +x_35 = lean_usize_dec_eq(x_33, x_34); +if (x_35 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_23, 0); -x_33 = lean_ctor_get(x_23, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_23); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; -} -} +lean_object* x_36; +lean_dec(x_26); +lean_dec(x_1); +x_36 = l_Lean_mkLevelMax_x27(x_28, x_32); +lean_ctor_set(x_30, 0, x_36); +return x_30; } else { -uint8_t x_35; -lean_dec(x_19); -lean_dec(x_1); -x_35 = !lean_is_exclusive(x_20); -if (x_35 == 0) +size_t x_37; size_t x_38; uint8_t x_39; +x_37 = lean_ptr_addr(x_26); +lean_dec(x_26); +x_38 = lean_ptr_addr(x_32); +x_39 = lean_usize_dec_eq(x_37, x_38); +if (x_39 == 0) { -return x_20; +lean_object* x_40; +lean_dec(x_1); +x_40 = l_Lean_mkLevelMax_x27(x_28, x_32); +lean_ctor_set(x_30, 0, x_40); +return x_30; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_20, 0); -x_37 = lean_ctor_get(x_20, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_20); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_object* x_41; +x_41 = l_Lean_simpLevelMax_x27(x_28, x_32, x_1); +lean_dec(x_1); +lean_dec(x_32); +lean_dec(x_28); +lean_ctor_set(x_30, 0, x_41); +return x_30; } } } -case 3: -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_1, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_1, 1); -lean_inc(x_40); -x_41 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_39, x_2, x_3, x_4); -if (lean_obj_tag(x_41) == 0) +else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); +lean_object* x_42; lean_object* x_43; size_t x_44; size_t x_45; uint8_t x_46; +x_42 = lean_ctor_get(x_30, 0); +x_43 = lean_ctor_get(x_30, 1); lean_inc(x_43); -lean_dec(x_41); -x_44 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_40, x_2, x_3, x_43); -if (lean_obj_tag(x_44) == 0) -{ -uint8_t x_45; -x_45 = !lean_is_exclusive(x_44); -if (x_45 == 0) +lean_inc(x_42); +lean_dec(x_30); +x_44 = lean_ptr_addr(x_25); +lean_dec(x_25); +x_45 = lean_ptr_addr(x_28); +x_46 = lean_usize_dec_eq(x_44, x_45); +if (x_46 == 0) { -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_44, 0); -x_47 = lean_level_update_imax(x_1, x_42, x_46); -lean_ctor_set(x_44, 0, x_47); -return x_44; +lean_object* x_47; lean_object* x_48; +lean_dec(x_26); +lean_dec(x_1); +x_47 = l_Lean_mkLevelMax_x27(x_28, x_42); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_43); +return x_48; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = lean_ctor_get(x_44, 0); -x_49 = lean_ctor_get(x_44, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_44); -x_50 = lean_level_update_imax(x_1, x_42, x_48); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_49); -return x_51; -} -} -else +size_t x_49; size_t x_50; uint8_t x_51; +x_49 = lean_ptr_addr(x_26); +lean_dec(x_26); +x_50 = lean_ptr_addr(x_42); +x_51 = lean_usize_dec_eq(x_49, x_50); +if (x_51 == 0) { -uint8_t x_52; -lean_dec(x_42); +lean_object* x_52; lean_object* x_53; lean_dec(x_1); -x_52 = !lean_is_exclusive(x_44); -if (x_52 == 0) -{ -return x_44; +x_52 = l_Lean_mkLevelMax_x27(x_28, x_42); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_43); +return x_53; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_44, 0); -x_54 = lean_ctor_get(x_44, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_44); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); +lean_object* x_54; lean_object* x_55; +x_54 = l_Lean_simpLevelMax_x27(x_28, x_42, x_1); +lean_dec(x_1); +lean_dec(x_42); +lean_dec(x_28); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_43); return x_55; } } } +} else { uint8_t x_56; -lean_dec(x_40); +lean_dec(x_28); +lean_dec(x_26); +lean_dec(x_25); lean_dec(x_1); -x_56 = !lean_is_exclusive(x_41); +x_56 = !lean_is_exclusive(x_30); if (x_56 == 0) { -return x_41; +return x_30; } else { lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_41, 0); -x_58 = lean_ctor_get(x_41, 1); +x_57 = lean_ctor_get(x_30, 0); +x_58 = lean_ctor_get(x_30, 1); lean_inc(x_58); lean_inc(x_57); -lean_dec(x_41); +lean_dec(x_30); x_59 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_59, 0, x_57); lean_ctor_set(x_59, 1, x_58); @@ -17269,67 +17948,145 @@ return x_59; } } } -case 5: +else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_84; -x_60 = lean_ctor_get(x_1, 0); -lean_inc(x_60); -x_84 = lean_st_ref_get(x_3, x_4); -if (lean_obj_tag(x_84) == 0) +uint8_t x_60; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_1); +x_60 = !lean_is_exclusive(x_27); +if (x_60 == 0) { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_ctor_get(x_85, 5); -lean_inc(x_87); -lean_dec(x_85); -lean_inc(x_60); -x_88 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_87, x_60); -if (lean_obj_tag(x_88) == 0) +return x_27; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_27, 0); +x_62 = lean_ctor_get(x_27, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_27); +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +return x_63; +} +} +} +case 3: +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_1, 0); +lean_inc(x_64); +x_65 = lean_ctor_get(x_1, 1); +lean_inc(x_65); +lean_inc(x_64); +x_66 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_64, x_2, x_3, x_4); +if (lean_obj_tag(x_66) == 0) { -x_61 = x_88; -x_62 = x_86; -goto block_83; +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_66, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_66, 1); +lean_inc(x_68); +lean_dec(x_66); +lean_inc(x_65); +x_69 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_65, x_2, x_3, x_68); +if (lean_obj_tag(x_69) == 0) +{ +uint8_t x_70; +x_70 = !lean_is_exclusive(x_69); +if (x_70 == 0) +{ +lean_object* x_71; size_t x_72; size_t x_73; uint8_t x_74; +x_71 = lean_ctor_get(x_69, 0); +x_72 = lean_ptr_addr(x_64); +lean_dec(x_64); +x_73 = lean_ptr_addr(x_67); +x_74 = lean_usize_dec_eq(x_72, x_73); +if (x_74 == 0) +{ +lean_object* x_75; +lean_dec(x_65); +lean_dec(x_1); +x_75 = l_Lean_mkLevelIMax_x27(x_67, x_71); +lean_ctor_set(x_69, 0, x_75); +return x_69; } else { -lean_object* x_89; -x_89 = l_Lean_markUsedAssignment___at_Lean_instantiateMVarsCore___spec__11___rarg(x_3, x_86); -if (lean_obj_tag(x_89) == 0) +size_t x_76; size_t x_77; uint8_t x_78; +x_76 = lean_ptr_addr(x_65); +lean_dec(x_65); +x_77 = lean_ptr_addr(x_71); +x_78 = lean_usize_dec_eq(x_76, x_77); +if (x_78 == 0) { -lean_object* x_90; -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); -lean_dec(x_89); -x_61 = x_88; -x_62 = x_90; -goto block_83; +lean_object* x_79; +lean_dec(x_1); +x_79 = l_Lean_mkLevelIMax_x27(x_67, x_71); +lean_ctor_set(x_69, 0, x_79); +return x_69; } else { -uint8_t x_91; -lean_dec(x_88); -lean_dec(x_60); +lean_object* x_80; +x_80 = l_Lean_simpLevelIMax_x27(x_67, x_71, x_1); lean_dec(x_1); -x_91 = !lean_is_exclusive(x_89); -if (x_91 == 0) +lean_ctor_set(x_69, 0, x_80); +return x_69; +} +} +} +else { -return x_89; +lean_object* x_81; lean_object* x_82; size_t x_83; size_t x_84; uint8_t x_85; +x_81 = lean_ctor_get(x_69, 0); +x_82 = lean_ctor_get(x_69, 1); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_69); +x_83 = lean_ptr_addr(x_64); +lean_dec(x_64); +x_84 = lean_ptr_addr(x_67); +x_85 = lean_usize_dec_eq(x_83, x_84); +if (x_85 == 0) +{ +lean_object* x_86; lean_object* x_87; +lean_dec(x_65); +lean_dec(x_1); +x_86 = l_Lean_mkLevelIMax_x27(x_67, x_81); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_82); +return x_87; } else { -lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_92 = lean_ctor_get(x_89, 0); -x_93 = lean_ctor_get(x_89, 1); -lean_inc(x_93); -lean_inc(x_92); -lean_dec(x_89); -x_94 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_94, 0, x_92); -lean_ctor_set(x_94, 1, x_93); +size_t x_88; size_t x_89; uint8_t x_90; +x_88 = lean_ptr_addr(x_65); +lean_dec(x_65); +x_89 = lean_ptr_addr(x_81); +x_90 = lean_usize_dec_eq(x_88, x_89); +if (x_90 == 0) +{ +lean_object* x_91; lean_object* x_92; +lean_dec(x_1); +x_91 = l_Lean_mkLevelIMax_x27(x_67, x_81); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_82); +return x_92; +} +else +{ +lean_object* x_93; lean_object* x_94; +x_93 = l_Lean_simpLevelIMax_x27(x_67, x_81, x_1); +lean_dec(x_1); +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_82); return x_94; } } @@ -17338,138 +18095,257 @@ return x_94; else { uint8_t x_95; -lean_dec(x_60); +lean_dec(x_67); +lean_dec(x_65); +lean_dec(x_64); lean_dec(x_1); -x_95 = !lean_is_exclusive(x_84); +x_95 = !lean_is_exclusive(x_69); if (x_95 == 0) { -return x_84; +return x_69; } else { lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_96 = lean_ctor_get(x_84, 0); -x_97 = lean_ctor_get(x_84, 1); +x_96 = lean_ctor_get(x_69, 0); +x_97 = lean_ctor_get(x_69, 1); lean_inc(x_97); lean_inc(x_96); -lean_dec(x_84); +lean_dec(x_69); x_98 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_98, 0, x_96); lean_ctor_set(x_98, 1, x_97); return x_98; } } -block_83: +} +else { -if (lean_obj_tag(x_61) == 0) +uint8_t x_99; +lean_dec(x_65); +lean_dec(x_64); +lean_dec(x_1); +x_99 = !lean_is_exclusive(x_66); +if (x_99 == 0) { -lean_object* x_63; -lean_dec(x_60); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_1); -lean_ctor_set(x_63, 1, x_62); -return x_63; +return x_66; +} +else +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_66, 0); +x_101 = lean_ctor_get(x_66, 1); +lean_inc(x_101); +lean_inc(x_100); +lean_dec(x_66); +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_100); +lean_ctor_set(x_102, 1, x_101); +return x_102; +} +} +} +case 5: +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_127; +x_103 = lean_ctor_get(x_1, 0); +lean_inc(x_103); +x_127 = lean_st_ref_get(x_3, x_4); +if (lean_obj_tag(x_127) == 0) +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_128 = lean_ctor_get(x_127, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_127, 1); +lean_inc(x_129); +lean_dec(x_127); +x_130 = lean_ctor_get(x_128, 5); +lean_inc(x_130); +lean_dec(x_128); +lean_inc(x_103); +x_131 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_130, x_103); +if (lean_obj_tag(x_131) == 0) +{ +x_104 = x_131; +x_105 = x_129; +goto block_126; +} +else +{ +lean_object* x_132; +x_132 = l_Lean_markUsedAssignment___at_Lean_instantiateMVarsCore___spec__11___rarg(x_3, x_129); +if (lean_obj_tag(x_132) == 0) +{ +lean_object* x_133; +x_133 = lean_ctor_get(x_132, 1); +lean_inc(x_133); +lean_dec(x_132); +x_104 = x_131; +x_105 = x_133; +goto block_126; } else { -lean_object* x_64; uint8_t x_65; +uint8_t x_134; +lean_dec(x_131); +lean_dec(x_103); lean_dec(x_1); -x_64 = lean_ctor_get(x_61, 0); -lean_inc(x_64); -lean_dec(x_61); -x_65 = l_Lean_Level_hasMVar(x_64); -if (x_65 == 0) +x_134 = !lean_is_exclusive(x_132); +if (x_134 == 0) { -lean_object* x_66; -lean_dec(x_60); -x_66 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_62); -return x_66; +return x_132; } else { -lean_object* x_67; -x_67 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_64, x_2, x_3, x_62); -if (lean_obj_tag(x_67) == 0) +lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_135 = lean_ctor_get(x_132, 0); +x_136 = lean_ctor_get(x_132, 1); +lean_inc(x_136); +lean_inc(x_135); +lean_dec(x_132); +x_137 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_137, 0, x_135); +lean_ctor_set(x_137, 1, x_136); +return x_137; +} +} +} +} +else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -lean_inc(x_68); -x_70 = l_Lean_assignLevelMVar___at_Lean_instantiateMVarsCore___spec__10___rarg(x_60, x_68, x_2, x_3, x_69); -if (lean_obj_tag(x_70) == 0) +uint8_t x_138; +lean_dec(x_103); +lean_dec(x_1); +x_138 = !lean_is_exclusive(x_127); +if (x_138 == 0) { -uint8_t x_71; -x_71 = !lean_is_exclusive(x_70); -if (x_71 == 0) +return x_127; +} +else { -lean_object* x_72; -x_72 = lean_ctor_get(x_70, 0); -lean_dec(x_72); -lean_ctor_set(x_70, 0, x_68); -return x_70; +lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_139 = lean_ctor_get(x_127, 0); +x_140 = lean_ctor_get(x_127, 1); +lean_inc(x_140); +lean_inc(x_139); +lean_dec(x_127); +x_141 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_141, 0, x_139); +lean_ctor_set(x_141, 1, x_140); +return x_141; +} +} +block_126: +{ +if (lean_obj_tag(x_104) == 0) +{ +lean_object* x_106; +lean_dec(x_103); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_1); +lean_ctor_set(x_106, 1, x_105); +return x_106; } else { -lean_object* x_73; lean_object* x_74; -x_73 = lean_ctor_get(x_70, 1); -lean_inc(x_73); -lean_dec(x_70); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_68); -lean_ctor_set(x_74, 1, x_73); -return x_74; +lean_object* x_107; uint8_t x_108; +lean_dec(x_1); +x_107 = lean_ctor_get(x_104, 0); +lean_inc(x_107); +lean_dec(x_104); +x_108 = l_Lean_Level_hasMVar(x_107); +if (x_108 == 0) +{ +lean_object* x_109; +lean_dec(x_103); +x_109 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 1, x_105); +return x_109; +} +else +{ +lean_object* x_110; +x_110 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__9___rarg(x_107, x_2, x_3, x_105); +if (lean_obj_tag(x_110) == 0) +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +lean_dec(x_110); +lean_inc(x_111); +x_113 = l_Lean_assignLevelMVar___at_Lean_instantiateMVarsCore___spec__10___rarg(x_103, x_111, x_2, x_3, x_112); +if (lean_obj_tag(x_113) == 0) +{ +uint8_t x_114; +x_114 = !lean_is_exclusive(x_113); +if (x_114 == 0) +{ +lean_object* x_115; +x_115 = lean_ctor_get(x_113, 0); +lean_dec(x_115); +lean_ctor_set(x_113, 0, x_111); +return x_113; +} +else +{ +lean_object* x_116; lean_object* x_117; +x_116 = lean_ctor_get(x_113, 1); +lean_inc(x_116); +lean_dec(x_113); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_111); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } else { -uint8_t x_75; -lean_dec(x_68); -x_75 = !lean_is_exclusive(x_70); -if (x_75 == 0) +uint8_t x_118; +lean_dec(x_111); +x_118 = !lean_is_exclusive(x_113); +if (x_118 == 0) { -return x_70; +return x_113; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_70, 0); -x_77 = lean_ctor_get(x_70, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_70); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_ctor_get(x_113, 0); +x_120 = lean_ctor_get(x_113, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_113); +x_121 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_121, 0, x_119); +lean_ctor_set(x_121, 1, x_120); +return x_121; } } } else { -uint8_t x_79; -lean_dec(x_60); -x_79 = !lean_is_exclusive(x_67); -if (x_79 == 0) +uint8_t x_122; +lean_dec(x_103); +x_122 = !lean_is_exclusive(x_110); +if (x_122 == 0) { -return x_67; +return x_110; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_80 = lean_ctor_get(x_67, 0); -x_81 = lean_ctor_get(x_67, 1); -lean_inc(x_81); -lean_inc(x_80); -lean_dec(x_67); -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -return x_82; +lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_123 = lean_ctor_get(x_110, 0); +x_124 = lean_ctor_get(x_110, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_110); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +return x_125; } } } @@ -17478,11 +18354,11 @@ return x_82; } default: { -lean_object* x_99; -x_99 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_99, 0, x_1); -lean_ctor_set(x_99, 1, x_4); -return x_99; +lean_object* x_142; +x_142 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_142, 0, x_1); +lean_ctor_set(x_142, 1, x_4); +return x_142; } } } @@ -22507,350 +23383,365 @@ case 3: lean_object* x_82; lean_object* x_83; x_82 = lean_ctor_get(x_1, 0); lean_inc(x_82); +lean_inc(x_82); x_83 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_82, x_2, x_3, x_48); if (lean_obj_tag(x_83) == 0) { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_object* x_84; lean_object* x_85; size_t x_86; size_t x_87; uint8_t x_88; x_84 = lean_ctor_get(x_83, 0); lean_inc(x_84); x_85 = lean_ctor_get(x_83, 1); lean_inc(x_85); lean_dec(x_83); -lean_inc(x_1); -x_86 = lean_expr_update_sort(x_1, x_84); -x_87 = lean_st_ref_take(x_2, x_85); -if (lean_obj_tag(x_87) == 0) -{ -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_88 = lean_ctor_get(x_87, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_87, 1); -lean_inc(x_89); -lean_dec(x_87); -lean_inc(x_86); -x_90 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_88, x_1, x_86); -x_91 = lean_st_ref_set(x_2, x_90, x_89); -if (lean_obj_tag(x_91) == 0) -{ -uint8_t x_92; -x_92 = !lean_is_exclusive(x_91); -if (x_92 == 0) +x_86 = lean_ptr_addr(x_82); +lean_dec(x_82); +x_87 = lean_ptr_addr(x_84); +x_88 = lean_usize_dec_eq(x_86, x_87); +if (x_88 == 0) { -lean_object* x_93; -x_93 = lean_ctor_get(x_91, 0); -lean_dec(x_93); -lean_ctor_set(x_91, 0, x_86); -return x_91; +lean_object* x_89; +x_89 = l_Lean_Expr_sort___override(x_84); +x_8 = x_89; +x_9 = x_85; +goto block_27; } else { -lean_object* x_94; lean_object* x_95; -x_94 = lean_ctor_get(x_91, 1); -lean_inc(x_94); -lean_dec(x_91); -x_95 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_95, 0, x_86); -lean_ctor_set(x_95, 1, x_94); -return x_95; +lean_dec(x_84); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_85; +goto block_27; } } else { -uint8_t x_96; -lean_dec(x_86); -x_96 = !lean_is_exclusive(x_91); -if (x_96 == 0) +uint8_t x_90; +lean_dec(x_82); +lean_dec(x_1); +x_90 = !lean_is_exclusive(x_83); +if (x_90 == 0) { -return x_91; +return x_83; } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_91, 0); -x_98 = lean_ctor_get(x_91, 1); -lean_inc(x_98); -lean_inc(x_97); -lean_dec(x_91); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_83, 0); +x_92 = lean_ctor_get(x_83, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_83); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +return x_93; } } } -else +case 4: { -uint8_t x_100; -lean_dec(x_86); -lean_dec(x_1); -x_100 = !lean_is_exclusive(x_87); -if (x_100 == 0) +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_1, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_1, 1); +lean_inc(x_95); +lean_inc(x_95); +x_96 = l_List_mapM___at_Lean_instantiateMVarsCore___spec__12___rarg(x_5, x_95, x_2, x_3, x_48); +if (lean_obj_tag(x_96) == 0) { -return x_87; +lean_object* x_97; lean_object* x_98; uint8_t x_99; +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +lean_dec(x_96); +x_99 = l_ptrEqList___rarg(x_95, x_97); +lean_dec(x_95); +if (x_99 == 0) +{ +lean_object* x_100; +x_100 = l_Lean_Expr_const___override(x_94, x_97); +x_8 = x_100; +x_9 = x_98; +goto block_27; } else { -lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_101 = lean_ctor_get(x_87, 0); -x_102 = lean_ctor_get(x_87, 1); -lean_inc(x_102); -lean_inc(x_101); -lean_dec(x_87); -x_103 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -return x_103; -} +lean_dec(x_97); +lean_dec(x_94); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_98; +goto block_27; } } else { -uint8_t x_104; +uint8_t x_101; +lean_dec(x_95); +lean_dec(x_94); lean_dec(x_1); -x_104 = !lean_is_exclusive(x_83); -if (x_104 == 0) +x_101 = !lean_is_exclusive(x_96); +if (x_101 == 0) { -return x_83; +return x_96; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_83, 0); -x_106 = lean_ctor_get(x_83, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_83); -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_102; lean_object* x_103; lean_object* x_104; +x_102 = lean_ctor_get(x_96, 0); +x_103 = lean_ctor_get(x_96, 1); +lean_inc(x_103); +lean_inc(x_102); +lean_dec(x_96); +x_104 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +return x_104; } } } -case 4: -{ -lean_object* x_108; lean_object* x_109; -x_108 = lean_ctor_get(x_1, 1); -lean_inc(x_108); -x_109 = l_List_mapM___at_Lean_instantiateMVarsCore___spec__12___rarg(x_5, x_108, x_2, x_3, x_48); -if (lean_obj_tag(x_109) == 0) +case 5: { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_110 = lean_ctor_get(x_109, 0); -lean_inc(x_110); -x_111 = lean_ctor_get(x_109, 1); -lean_inc(x_111); -lean_dec(x_109); +lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_105 = lean_unsigned_to_nat(0u); +x_106 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_105); +x_107 = l_Lean_instantiateExprMVars___rarg___lambda__20___closed__1; +lean_inc(x_106); +x_108 = lean_mk_array(x_106, x_107); +x_109 = lean_unsigned_to_nat(1u); +x_110 = lean_nat_sub(x_106, x_109); +lean_dec(x_106); lean_inc(x_1); -x_112 = lean_expr_update_const(x_1, x_110); -x_113 = lean_st_ref_take(x_2, x_111); -if (lean_obj_tag(x_113) == 0) +x_111 = l_Lean_Expr_withAppAux___at_Lean_instantiateMVarsCore___spec__42___rarg(x_5, x_1, x_108, x_110, x_2, x_3, x_48); +if (lean_obj_tag(x_111) == 0) { -lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_114 = lean_ctor_get(x_113, 0); -lean_inc(x_114); -x_115 = lean_ctor_get(x_113, 1); +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_111, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_111, 1); +lean_inc(x_113); +lean_dec(x_111); +x_114 = lean_st_ref_take(x_2, x_113); +if (lean_obj_tag(x_114) == 0) +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_115 = lean_ctor_get(x_114, 0); lean_inc(x_115); -lean_dec(x_113); +x_116 = lean_ctor_get(x_114, 1); +lean_inc(x_116); +lean_dec(x_114); lean_inc(x_112); -x_116 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_114, x_1, x_112); -x_117 = lean_st_ref_set(x_2, x_116, x_115); -if (lean_obj_tag(x_117) == 0) +x_117 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_115, x_1, x_112); +x_118 = lean_st_ref_set(x_2, x_117, x_116); +if (lean_obj_tag(x_118) == 0) { -uint8_t x_118; -x_118 = !lean_is_exclusive(x_117); -if (x_118 == 0) +uint8_t x_119; +x_119 = !lean_is_exclusive(x_118); +if (x_119 == 0) { -lean_object* x_119; -x_119 = lean_ctor_get(x_117, 0); -lean_dec(x_119); -lean_ctor_set(x_117, 0, x_112); -return x_117; +lean_object* x_120; +x_120 = lean_ctor_get(x_118, 0); +lean_dec(x_120); +lean_ctor_set(x_118, 0, x_112); +return x_118; } else { -lean_object* x_120; lean_object* x_121; -x_120 = lean_ctor_get(x_117, 1); -lean_inc(x_120); -lean_dec(x_117); -x_121 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_121, 0, x_112); -lean_ctor_set(x_121, 1, x_120); -return x_121; +lean_object* x_121; lean_object* x_122; +x_121 = lean_ctor_get(x_118, 1); +lean_inc(x_121); +lean_dec(x_118); +x_122 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_122, 0, x_112); +lean_ctor_set(x_122, 1, x_121); +return x_122; } } else { -uint8_t x_122; +uint8_t x_123; lean_dec(x_112); -x_122 = !lean_is_exclusive(x_117); -if (x_122 == 0) +x_123 = !lean_is_exclusive(x_118); +if (x_123 == 0) { -return x_117; +return x_118; } else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_123 = lean_ctor_get(x_117, 0); -x_124 = lean_ctor_get(x_117, 1); +lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_124 = lean_ctor_get(x_118, 0); +x_125 = lean_ctor_get(x_118, 1); +lean_inc(x_125); lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_117); -x_125 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_124); -return x_125; +lean_dec(x_118); +x_126 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +return x_126; } } } else { -uint8_t x_126; +uint8_t x_127; lean_dec(x_112); lean_dec(x_1); -x_126 = !lean_is_exclusive(x_113); -if (x_126 == 0) +x_127 = !lean_is_exclusive(x_114); +if (x_127 == 0) { -return x_113; +return x_114; } else { -lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_127 = lean_ctor_get(x_113, 0); -x_128 = lean_ctor_get(x_113, 1); +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_114, 0); +x_129 = lean_ctor_get(x_114, 1); +lean_inc(x_129); lean_inc(x_128); -lean_inc(x_127); -lean_dec(x_113); -x_129 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_129, 0, x_127); -lean_ctor_set(x_129, 1, x_128); -return x_129; +lean_dec(x_114); +x_130 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +return x_130; } } } else { -uint8_t x_130; +uint8_t x_131; lean_dec(x_1); -x_130 = !lean_is_exclusive(x_109); -if (x_130 == 0) +x_131 = !lean_is_exclusive(x_111); +if (x_131 == 0) { -return x_109; +return x_111; } else { -lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_131 = lean_ctor_get(x_109, 0); -x_132 = lean_ctor_get(x_109, 1); +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_111, 0); +x_133 = lean_ctor_get(x_111, 1); +lean_inc(x_133); lean_inc(x_132); -lean_inc(x_131); -lean_dec(x_109); -x_133 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_133, 0, x_131); -lean_ctor_set(x_133, 1, x_132); -return x_133; +lean_dec(x_111); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; } } } -case 5: +case 6: { -lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -x_134 = lean_unsigned_to_nat(0u); -x_135 = l_Lean_Expr_getAppNumArgsAux(x_1, x_134); -x_136 = l_Lean_instantiateExprMVars___rarg___lambda__20___closed__1; +lean_object* x_135; lean_object* x_136; lean_object* x_137; uint8_t x_138; lean_object* x_139; +x_135 = lean_ctor_get(x_1, 0); lean_inc(x_135); -x_137 = lean_mk_array(x_135, x_136); -x_138 = lean_unsigned_to_nat(1u); -x_139 = lean_nat_sub(x_135, x_138); -lean_dec(x_135); -lean_inc(x_1); -x_140 = l_Lean_Expr_withAppAux___at_Lean_instantiateMVarsCore___spec__42___rarg(x_5, x_1, x_137, x_139, x_2, x_3, x_48); -if (lean_obj_tag(x_140) == 0) +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_1, 2); +lean_inc(x_137); +x_138 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_inc(x_136); +x_139 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_136, x_2, x_3, x_48); +if (lean_obj_tag(x_139) == 0) { -lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_141 = lean_ctor_get(x_140, 0); +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_139, 0); +lean_inc(x_140); +x_141 = lean_ctor_get(x_139, 1); lean_inc(x_141); -x_142 = lean_ctor_get(x_140, 1); -lean_inc(x_142); -lean_dec(x_140); -x_143 = lean_st_ref_take(x_2, x_142); -if (lean_obj_tag(x_143) == 0) +lean_dec(x_139); +lean_inc(x_137); +x_142 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_137, x_2, x_3, x_141); +if (lean_obj_tag(x_142) == 0) { -lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_144 = lean_ctor_get(x_143, 0); +lean_object* x_143; lean_object* x_144; lean_object* x_145; size_t x_146; size_t x_147; uint8_t x_148; +x_143 = lean_ctor_get(x_142, 0); +lean_inc(x_143); +x_144 = lean_ctor_get(x_142, 1); lean_inc(x_144); -x_145 = lean_ctor_get(x_143, 1); -lean_inc(x_145); -lean_dec(x_143); -lean_inc(x_141); -x_146 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_144, x_1, x_141); -x_147 = lean_st_ref_set(x_2, x_146, x_145); -if (lean_obj_tag(x_147) == 0) -{ -uint8_t x_148; -x_148 = !lean_is_exclusive(x_147); +lean_dec(x_142); +lean_inc(x_137); +lean_inc(x_136); +lean_inc(x_135); +x_145 = l_Lean_Expr_lam___override(x_135, x_136, x_137, x_138); +x_146 = lean_ptr_addr(x_136); +lean_dec(x_136); +x_147 = lean_ptr_addr(x_140); +x_148 = lean_usize_dec_eq(x_146, x_147); if (x_148 == 0) { lean_object* x_149; -x_149 = lean_ctor_get(x_147, 0); -lean_dec(x_149); -lean_ctor_set(x_147, 0, x_141); -return x_147; +lean_dec(x_145); +lean_dec(x_137); +x_149 = l_Lean_Expr_lam___override(x_135, x_140, x_143, x_138); +x_8 = x_149; +x_9 = x_144; +goto block_27; } else { -lean_object* x_150; lean_object* x_151; -x_150 = lean_ctor_get(x_147, 1); -lean_inc(x_150); -lean_dec(x_147); -x_151 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_151, 0, x_141); -lean_ctor_set(x_151, 1, x_150); -return x_151; -} +size_t x_150; size_t x_151; uint8_t x_152; +x_150 = lean_ptr_addr(x_137); +lean_dec(x_137); +x_151 = lean_ptr_addr(x_143); +x_152 = lean_usize_dec_eq(x_150, x_151); +if (x_152 == 0) +{ +lean_object* x_153; +lean_dec(x_145); +x_153 = l_Lean_Expr_lam___override(x_135, x_140, x_143, x_138); +x_8 = x_153; +x_9 = x_144; +goto block_27; } else { -uint8_t x_152; -lean_dec(x_141); -x_152 = !lean_is_exclusive(x_147); -if (x_152 == 0) +uint8_t x_154; +x_154 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_138, x_138); +if (x_154 == 0) { -return x_147; +lean_object* x_155; +lean_dec(x_145); +x_155 = l_Lean_Expr_lam___override(x_135, x_140, x_143, x_138); +x_8 = x_155; +x_9 = x_144; +goto block_27; } else { -lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_153 = lean_ctor_get(x_147, 0); -x_154 = lean_ctor_get(x_147, 1); -lean_inc(x_154); -lean_inc(x_153); -lean_dec(x_147); -x_155 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_155, 0, x_153); -lean_ctor_set(x_155, 1, x_154); -return x_155; +lean_dec(x_143); +lean_dec(x_140); +lean_dec(x_135); +x_8 = x_145; +x_9 = x_144; +goto block_27; +} } } } else { uint8_t x_156; -lean_dec(x_141); +lean_dec(x_140); +lean_dec(x_137); +lean_dec(x_136); +lean_dec(x_135); lean_dec(x_1); -x_156 = !lean_is_exclusive(x_143); +x_156 = !lean_is_exclusive(x_142); if (x_156 == 0) { -return x_143; +return x_142; } else { lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_157 = lean_ctor_get(x_143, 0); -x_158 = lean_ctor_get(x_143, 1); +x_157 = lean_ctor_get(x_142, 0); +x_158 = lean_ctor_get(x_142, 1); lean_inc(x_158); lean_inc(x_157); -lean_dec(x_143); +lean_dec(x_142); x_159 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_159, 0, x_157); lean_ctor_set(x_159, 1, x_158); @@ -22861,20 +23752,23 @@ return x_159; else { uint8_t x_160; +lean_dec(x_137); +lean_dec(x_136); +lean_dec(x_135); lean_dec(x_1); -x_160 = !lean_is_exclusive(x_140); +x_160 = !lean_is_exclusive(x_139); if (x_160 == 0) { -return x_140; +return x_139; } else { lean_object* x_161; lean_object* x_162; lean_object* x_163; -x_161 = lean_ctor_get(x_140, 0); -x_162 = lean_ctor_get(x_140, 1); +x_161 = lean_ctor_get(x_139, 0); +x_162 = lean_ctor_get(x_139, 1); lean_inc(x_162); lean_inc(x_161); -lean_dec(x_140); +lean_dec(x_139); x_163 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_163, 0, x_161); lean_ctor_set(x_163, 1, x_162); @@ -22882,1580 +23776,1652 @@ return x_163; } } } -case 6: +case 7: { -lean_object* x_164; lean_object* x_165; uint8_t x_166; lean_object* x_167; -x_164 = lean_ctor_get(x_1, 1); +lean_object* x_164; lean_object* x_165; lean_object* x_166; uint8_t x_167; lean_object* x_168; +x_164 = lean_ctor_get(x_1, 0); lean_inc(x_164); -x_165 = lean_ctor_get(x_1, 2); +x_165 = lean_ctor_get(x_1, 1); lean_inc(x_165); -x_166 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_167 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_164, x_2, x_3, x_48); -if (lean_obj_tag(x_167) == 0) +x_166 = lean_ctor_get(x_1, 2); +lean_inc(x_166); +x_167 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_inc(x_165); +x_168 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_165, x_2, x_3, x_48); +if (lean_obj_tag(x_168) == 0) { -lean_object* x_168; lean_object* x_169; lean_object* x_170; -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -x_169 = lean_ctor_get(x_167, 1); +lean_object* x_169; lean_object* x_170; lean_object* x_171; +x_169 = lean_ctor_get(x_168, 0); lean_inc(x_169); -lean_dec(x_167); -x_170 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_165, x_2, x_3, x_169); -if (lean_obj_tag(x_170) == 0) +x_170 = lean_ctor_get(x_168, 1); +lean_inc(x_170); +lean_dec(x_168); +lean_inc(x_166); +x_171 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_166, x_2, x_3, x_170); +if (lean_obj_tag(x_171) == 0) { -lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; -x_171 = lean_ctor_get(x_170, 0); -lean_inc(x_171); -x_172 = lean_ctor_get(x_170, 1); +lean_object* x_172; lean_object* x_173; lean_object* x_174; size_t x_175; size_t x_176; uint8_t x_177; +x_172 = lean_ctor_get(x_171, 0); lean_inc(x_172); -lean_dec(x_170); -lean_inc(x_1); -x_173 = lean_expr_update_lambda(x_1, x_166, x_168, x_171); -x_174 = lean_st_ref_take(x_2, x_172); -if (lean_obj_tag(x_174) == 0) -{ -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_175 = lean_ctor_get(x_174, 0); -lean_inc(x_175); -x_176 = lean_ctor_get(x_174, 1); -lean_inc(x_176); -lean_dec(x_174); +x_173 = lean_ctor_get(x_171, 1); lean_inc(x_173); -x_177 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_175, x_1, x_173); -x_178 = lean_st_ref_set(x_2, x_177, x_176); -if (lean_obj_tag(x_178) == 0) -{ -uint8_t x_179; -x_179 = !lean_is_exclusive(x_178); -if (x_179 == 0) +lean_dec(x_171); +lean_inc(x_166); +lean_inc(x_165); +lean_inc(x_164); +x_174 = l_Lean_Expr_forallE___override(x_164, x_165, x_166, x_167); +x_175 = lean_ptr_addr(x_165); +lean_dec(x_165); +x_176 = lean_ptr_addr(x_169); +x_177 = lean_usize_dec_eq(x_175, x_176); +if (x_177 == 0) { -lean_object* x_180; -x_180 = lean_ctor_get(x_178, 0); -lean_dec(x_180); -lean_ctor_set(x_178, 0, x_173); -return x_178; +lean_object* x_178; +lean_dec(x_174); +lean_dec(x_166); +x_178 = l_Lean_Expr_forallE___override(x_164, x_169, x_172, x_167); +x_8 = x_178; +x_9 = x_173; +goto block_27; } else { -lean_object* x_181; lean_object* x_182; -x_181 = lean_ctor_get(x_178, 1); -lean_inc(x_181); -lean_dec(x_178); -x_182 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_182, 0, x_173); -lean_ctor_set(x_182, 1, x_181); -return x_182; -} +size_t x_179; size_t x_180; uint8_t x_181; +x_179 = lean_ptr_addr(x_166); +lean_dec(x_166); +x_180 = lean_ptr_addr(x_172); +x_181 = lean_usize_dec_eq(x_179, x_180); +if (x_181 == 0) +{ +lean_object* x_182; +lean_dec(x_174); +x_182 = l_Lean_Expr_forallE___override(x_164, x_169, x_172, x_167); +x_8 = x_182; +x_9 = x_173; +goto block_27; } else { uint8_t x_183; -lean_dec(x_173); -x_183 = !lean_is_exclusive(x_178); +x_183 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_167, x_167); if (x_183 == 0) { -return x_178; -} -else -{ -lean_object* x_184; lean_object* x_185; lean_object* x_186; -x_184 = lean_ctor_get(x_178, 0); -x_185 = lean_ctor_get(x_178, 1); -lean_inc(x_185); -lean_inc(x_184); -lean_dec(x_178); -x_186 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_186, 0, x_184); -lean_ctor_set(x_186, 1, x_185); -return x_186; -} -} +lean_object* x_184; +lean_dec(x_174); +x_184 = l_Lean_Expr_forallE___override(x_164, x_169, x_172, x_167); +x_8 = x_184; +x_9 = x_173; +goto block_27; } else { -uint8_t x_187; -lean_dec(x_173); -lean_dec(x_1); -x_187 = !lean_is_exclusive(x_174); -if (x_187 == 0) -{ -return x_174; +lean_dec(x_172); +lean_dec(x_169); +lean_dec(x_164); +x_8 = x_174; +x_9 = x_173; +goto block_27; } -else -{ -lean_object* x_188; lean_object* x_189; lean_object* x_190; -x_188 = lean_ctor_get(x_174, 0); -x_189 = lean_ctor_get(x_174, 1); -lean_inc(x_189); -lean_inc(x_188); -lean_dec(x_174); -x_190 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_190, 0, x_188); -lean_ctor_set(x_190, 1, x_189); -return x_190; } } } else { -uint8_t x_191; -lean_dec(x_168); +uint8_t x_185; +lean_dec(x_169); +lean_dec(x_166); +lean_dec(x_165); +lean_dec(x_164); lean_dec(x_1); -x_191 = !lean_is_exclusive(x_170); -if (x_191 == 0) +x_185 = !lean_is_exclusive(x_171); +if (x_185 == 0) { -return x_170; +return x_171; } else { -lean_object* x_192; lean_object* x_193; lean_object* x_194; -x_192 = lean_ctor_get(x_170, 0); -x_193 = lean_ctor_get(x_170, 1); -lean_inc(x_193); -lean_inc(x_192); -lean_dec(x_170); -x_194 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_194, 0, x_192); -lean_ctor_set(x_194, 1, x_193); -return x_194; +lean_object* x_186; lean_object* x_187; lean_object* x_188; +x_186 = lean_ctor_get(x_171, 0); +x_187 = lean_ctor_get(x_171, 1); +lean_inc(x_187); +lean_inc(x_186); +lean_dec(x_171); +x_188 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_188, 0, x_186); +lean_ctor_set(x_188, 1, x_187); +return x_188; } } } else { -uint8_t x_195; +uint8_t x_189; +lean_dec(x_166); lean_dec(x_165); +lean_dec(x_164); lean_dec(x_1); -x_195 = !lean_is_exclusive(x_167); -if (x_195 == 0) +x_189 = !lean_is_exclusive(x_168); +if (x_189 == 0) { -return x_167; +return x_168; } else { -lean_object* x_196; lean_object* x_197; lean_object* x_198; -x_196 = lean_ctor_get(x_167, 0); -x_197 = lean_ctor_get(x_167, 1); -lean_inc(x_197); -lean_inc(x_196); -lean_dec(x_167); -x_198 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_198, 0, x_196); -lean_ctor_set(x_198, 1, x_197); -return x_198; +lean_object* x_190; lean_object* x_191; lean_object* x_192; +x_190 = lean_ctor_get(x_168, 0); +x_191 = lean_ctor_get(x_168, 1); +lean_inc(x_191); +lean_inc(x_190); +lean_dec(x_168); +x_192 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_192, 0, x_190); +lean_ctor_set(x_192, 1, x_191); +return x_192; } } } -case 7: +case 8: +{ +lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; uint8_t x_197; lean_object* x_198; +x_193 = lean_ctor_get(x_1, 0); +lean_inc(x_193); +x_194 = lean_ctor_get(x_1, 1); +lean_inc(x_194); +x_195 = lean_ctor_get(x_1, 2); +lean_inc(x_195); +x_196 = lean_ctor_get(x_1, 3); +lean_inc(x_196); +x_197 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); +lean_inc(x_194); +x_198 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_194, x_2, x_3, x_48); +if (lean_obj_tag(x_198) == 0) { -lean_object* x_199; lean_object* x_200; uint8_t x_201; lean_object* x_202; -x_199 = lean_ctor_get(x_1, 1); +lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_199 = lean_ctor_get(x_198, 0); lean_inc(x_199); -x_200 = lean_ctor_get(x_1, 2); +x_200 = lean_ctor_get(x_198, 1); lean_inc(x_200); -x_201 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_202 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_199, x_2, x_3, x_48); -if (lean_obj_tag(x_202) == 0) +lean_dec(x_198); +lean_inc(x_195); +x_201 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_195, x_2, x_3, x_200); +if (lean_obj_tag(x_201) == 0) { -lean_object* x_203; lean_object* x_204; lean_object* x_205; -x_203 = lean_ctor_get(x_202, 0); +lean_object* x_202; lean_object* x_203; lean_object* x_204; +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +x_203 = lean_ctor_get(x_201, 1); lean_inc(x_203); -x_204 = lean_ctor_get(x_202, 1); -lean_inc(x_204); -lean_dec(x_202); -x_205 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_200, x_2, x_3, x_204); -if (lean_obj_tag(x_205) == 0) +lean_dec(x_201); +lean_inc(x_196); +x_204 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_196, x_2, x_3, x_203); +if (lean_obj_tag(x_204) == 0) { -lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; -x_206 = lean_ctor_get(x_205, 0); +lean_object* x_205; lean_object* x_206; size_t x_207; size_t x_208; uint8_t x_209; +x_205 = lean_ctor_get(x_204, 0); +lean_inc(x_205); +x_206 = lean_ctor_get(x_204, 1); lean_inc(x_206); -x_207 = lean_ctor_get(x_205, 1); -lean_inc(x_207); -lean_dec(x_205); -lean_inc(x_1); -x_208 = lean_expr_update_forall(x_1, x_201, x_203, x_206); -x_209 = lean_st_ref_take(x_2, x_207); -if (lean_obj_tag(x_209) == 0) +lean_dec(x_204); +x_207 = lean_ptr_addr(x_194); +lean_dec(x_194); +x_208 = lean_ptr_addr(x_199); +x_209 = lean_usize_dec_eq(x_207, x_208); +if (x_209 == 0) { -lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; -x_210 = lean_ctor_get(x_209, 0); -lean_inc(x_210); -x_211 = lean_ctor_get(x_209, 1); -lean_inc(x_211); -lean_dec(x_209); -lean_inc(x_208); -x_212 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_210, x_1, x_208); -x_213 = lean_st_ref_set(x_2, x_212, x_211); -if (lean_obj_tag(x_213) == 0) +lean_object* x_210; +lean_dec(x_196); +lean_dec(x_195); +x_210 = l_Lean_Expr_letE___override(x_193, x_199, x_202, x_205, x_197); +x_8 = x_210; +x_9 = x_206; +goto block_27; +} +else { -uint8_t x_214; -x_214 = !lean_is_exclusive(x_213); -if (x_214 == 0) +size_t x_211; size_t x_212; uint8_t x_213; +x_211 = lean_ptr_addr(x_195); +lean_dec(x_195); +x_212 = lean_ptr_addr(x_202); +x_213 = lean_usize_dec_eq(x_211, x_212); +if (x_213 == 0) { -lean_object* x_215; -x_215 = lean_ctor_get(x_213, 0); -lean_dec(x_215); -lean_ctor_set(x_213, 0, x_208); -return x_213; +lean_object* x_214; +lean_dec(x_196); +x_214 = l_Lean_Expr_letE___override(x_193, x_199, x_202, x_205, x_197); +x_8 = x_214; +x_9 = x_206; +goto block_27; } else { -lean_object* x_216; lean_object* x_217; -x_216 = lean_ctor_get(x_213, 1); -lean_inc(x_216); -lean_dec(x_213); -x_217 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_217, 0, x_208); -lean_ctor_set(x_217, 1, x_216); -return x_217; +size_t x_215; size_t x_216; uint8_t x_217; +x_215 = lean_ptr_addr(x_196); +lean_dec(x_196); +x_216 = lean_ptr_addr(x_205); +x_217 = lean_usize_dec_eq(x_215, x_216); +if (x_217 == 0) +{ +lean_object* x_218; +x_218 = l_Lean_Expr_letE___override(x_193, x_199, x_202, x_205, x_197); +x_8 = x_218; +x_9 = x_206; +goto block_27; +} +else +{ +lean_dec(x_205); +lean_dec(x_202); +lean_dec(x_199); +lean_dec(x_193); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_206; +goto block_27; +} +} } } else { -uint8_t x_218; -lean_dec(x_208); -x_218 = !lean_is_exclusive(x_213); -if (x_218 == 0) +uint8_t x_219; +lean_dec(x_202); +lean_dec(x_199); +lean_dec(x_196); +lean_dec(x_195); +lean_dec(x_194); +lean_dec(x_193); +lean_dec(x_1); +x_219 = !lean_is_exclusive(x_204); +if (x_219 == 0) { -return x_213; +return x_204; } else { -lean_object* x_219; lean_object* x_220; lean_object* x_221; -x_219 = lean_ctor_get(x_213, 0); -x_220 = lean_ctor_get(x_213, 1); +lean_object* x_220; lean_object* x_221; lean_object* x_222; +x_220 = lean_ctor_get(x_204, 0); +x_221 = lean_ctor_get(x_204, 1); +lean_inc(x_221); lean_inc(x_220); -lean_inc(x_219); -lean_dec(x_213); -x_221 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_221, 0, x_219); -lean_ctor_set(x_221, 1, x_220); -return x_221; +lean_dec(x_204); +x_222 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_222, 0, x_220); +lean_ctor_set(x_222, 1, x_221); +return x_222; } } } else { -uint8_t x_222; -lean_dec(x_208); +uint8_t x_223; +lean_dec(x_199); +lean_dec(x_196); +lean_dec(x_195); +lean_dec(x_194); +lean_dec(x_193); lean_dec(x_1); -x_222 = !lean_is_exclusive(x_209); -if (x_222 == 0) +x_223 = !lean_is_exclusive(x_201); +if (x_223 == 0) { -return x_209; +return x_201; } else { -lean_object* x_223; lean_object* x_224; lean_object* x_225; -x_223 = lean_ctor_get(x_209, 0); -x_224 = lean_ctor_get(x_209, 1); +lean_object* x_224; lean_object* x_225; lean_object* x_226; +x_224 = lean_ctor_get(x_201, 0); +x_225 = lean_ctor_get(x_201, 1); +lean_inc(x_225); lean_inc(x_224); -lean_inc(x_223); -lean_dec(x_209); -x_225 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_225, 0, x_223); -lean_ctor_set(x_225, 1, x_224); -return x_225; +lean_dec(x_201); +x_226 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_226, 0, x_224); +lean_ctor_set(x_226, 1, x_225); +return x_226; } } } else { -uint8_t x_226; -lean_dec(x_203); +uint8_t x_227; +lean_dec(x_196); +lean_dec(x_195); +lean_dec(x_194); +lean_dec(x_193); lean_dec(x_1); -x_226 = !lean_is_exclusive(x_205); -if (x_226 == 0) +x_227 = !lean_is_exclusive(x_198); +if (x_227 == 0) { -return x_205; +return x_198; } else { -lean_object* x_227; lean_object* x_228; lean_object* x_229; -x_227 = lean_ctor_get(x_205, 0); -x_228 = lean_ctor_get(x_205, 1); +lean_object* x_228; lean_object* x_229; lean_object* x_230; +x_228 = lean_ctor_get(x_198, 0); +x_229 = lean_ctor_get(x_198, 1); +lean_inc(x_229); lean_inc(x_228); -lean_inc(x_227); -lean_dec(x_205); -x_229 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_229, 0, x_227); -lean_ctor_set(x_229, 1, x_228); -return x_229; +lean_dec(x_198); +x_230 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_230, 0, x_228); +lean_ctor_set(x_230, 1, x_229); +return x_230; } } } -else +case 10: { -uint8_t x_230; -lean_dec(x_200); -lean_dec(x_1); -x_230 = !lean_is_exclusive(x_202); -if (x_230 == 0) +lean_object* x_231; lean_object* x_232; lean_object* x_233; +x_231 = lean_ctor_get(x_1, 0); +lean_inc(x_231); +x_232 = lean_ctor_get(x_1, 1); +lean_inc(x_232); +lean_inc(x_232); +x_233 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_232, x_2, x_3, x_48); +if (lean_obj_tag(x_233) == 0) { -return x_202; +lean_object* x_234; lean_object* x_235; size_t x_236; size_t x_237; uint8_t x_238; +x_234 = lean_ctor_get(x_233, 0); +lean_inc(x_234); +x_235 = lean_ctor_get(x_233, 1); +lean_inc(x_235); +lean_dec(x_233); +x_236 = lean_ptr_addr(x_232); +lean_dec(x_232); +x_237 = lean_ptr_addr(x_234); +x_238 = lean_usize_dec_eq(x_236, x_237); +if (x_238 == 0) +{ +lean_object* x_239; +x_239 = l_Lean_Expr_mdata___override(x_231, x_234); +x_8 = x_239; +x_9 = x_235; +goto block_27; } else { -lean_object* x_231; lean_object* x_232; lean_object* x_233; -x_231 = lean_ctor_get(x_202, 0); -x_232 = lean_ctor_get(x_202, 1); -lean_inc(x_232); -lean_inc(x_231); -lean_dec(x_202); -x_233 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_233, 0, x_231); -lean_ctor_set(x_233, 1, x_232); -return x_233; -} +lean_dec(x_234); +lean_dec(x_231); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_235; +goto block_27; } } -case 8: +else { -lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; -x_234 = lean_ctor_get(x_1, 1); -lean_inc(x_234); -x_235 = lean_ctor_get(x_1, 2); -lean_inc(x_235); -x_236 = lean_ctor_get(x_1, 3); -lean_inc(x_236); -x_237 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_234, x_2, x_3, x_48); -if (lean_obj_tag(x_237) == 0) -{ -lean_object* x_238; lean_object* x_239; lean_object* x_240; -x_238 = lean_ctor_get(x_237, 0); -lean_inc(x_238); -x_239 = lean_ctor_get(x_237, 1); -lean_inc(x_239); -lean_dec(x_237); -x_240 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_235, x_2, x_3, x_239); -if (lean_obj_tag(x_240) == 0) +uint8_t x_240; +lean_dec(x_232); +lean_dec(x_231); +lean_dec(x_1); +x_240 = !lean_is_exclusive(x_233); +if (x_240 == 0) +{ +return x_233; +} +else { lean_object* x_241; lean_object* x_242; lean_object* x_243; -x_241 = lean_ctor_get(x_240, 0); -lean_inc(x_241); -x_242 = lean_ctor_get(x_240, 1); +x_241 = lean_ctor_get(x_233, 0); +x_242 = lean_ctor_get(x_233, 1); lean_inc(x_242); -lean_dec(x_240); -x_243 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_236, x_2, x_3, x_242); -if (lean_obj_tag(x_243) == 0) +lean_inc(x_241); +lean_dec(x_233); +x_243 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_243, 0, x_241); +lean_ctor_set(x_243, 1, x_242); +return x_243; +} +} +} +case 11: { lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; -x_244 = lean_ctor_get(x_243, 0); +x_244 = lean_ctor_get(x_1, 0); lean_inc(x_244); -x_245 = lean_ctor_get(x_243, 1); +x_245 = lean_ctor_get(x_1, 1); lean_inc(x_245); -lean_dec(x_243); -lean_inc(x_1); -x_246 = lean_expr_update_let(x_1, x_238, x_241, x_244); -x_247 = lean_st_ref_take(x_2, x_245); +x_246 = lean_ctor_get(x_1, 2); +lean_inc(x_246); +lean_inc(x_246); +x_247 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_246, x_2, x_3, x_48); if (lean_obj_tag(x_247) == 0) { -lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; +lean_object* x_248; lean_object* x_249; size_t x_250; size_t x_251; uint8_t x_252; x_248 = lean_ctor_get(x_247, 0); lean_inc(x_248); x_249 = lean_ctor_get(x_247, 1); lean_inc(x_249); lean_dec(x_247); -lean_inc(x_246); -x_250 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_248, x_1, x_246); -x_251 = lean_st_ref_set(x_2, x_250, x_249); -if (lean_obj_tag(x_251) == 0) -{ -uint8_t x_252; -x_252 = !lean_is_exclusive(x_251); +x_250 = lean_ptr_addr(x_246); +lean_dec(x_246); +x_251 = lean_ptr_addr(x_248); +x_252 = lean_usize_dec_eq(x_250, x_251); if (x_252 == 0) { lean_object* x_253; -x_253 = lean_ctor_get(x_251, 0); -lean_dec(x_253); -lean_ctor_set(x_251, 0, x_246); -return x_251; -} -else -{ -lean_object* x_254; lean_object* x_255; -x_254 = lean_ctor_get(x_251, 1); -lean_inc(x_254); -lean_dec(x_251); -x_255 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_255, 0, x_246); -lean_ctor_set(x_255, 1, x_254); -return x_255; -} -} -else -{ -uint8_t x_256; -lean_dec(x_246); -x_256 = !lean_is_exclusive(x_251); -if (x_256 == 0) -{ -return x_251; +x_253 = l_Lean_Expr_proj___override(x_244, x_245, x_248); +x_8 = x_253; +x_9 = x_249; +goto block_27; } else { -lean_object* x_257; lean_object* x_258; lean_object* x_259; -x_257 = lean_ctor_get(x_251, 0); -x_258 = lean_ctor_get(x_251, 1); -lean_inc(x_258); -lean_inc(x_257); -lean_dec(x_251); -x_259 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_259, 0, x_257); -lean_ctor_set(x_259, 1, x_258); -return x_259; -} +lean_dec(x_248); +lean_dec(x_245); +lean_dec(x_244); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_249; +goto block_27; } } else { -uint8_t x_260; +uint8_t x_254; lean_dec(x_246); +lean_dec(x_245); +lean_dec(x_244); lean_dec(x_1); -x_260 = !lean_is_exclusive(x_247); -if (x_260 == 0) +x_254 = !lean_is_exclusive(x_247); +if (x_254 == 0) { return x_247; } else { -lean_object* x_261; lean_object* x_262; lean_object* x_263; -x_261 = lean_ctor_get(x_247, 0); -x_262 = lean_ctor_get(x_247, 1); -lean_inc(x_262); -lean_inc(x_261); +lean_object* x_255; lean_object* x_256; lean_object* x_257; +x_255 = lean_ctor_get(x_247, 0); +x_256 = lean_ctor_get(x_247, 1); +lean_inc(x_256); +lean_inc(x_255); lean_dec(x_247); -x_263 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_263, 0, x_261); -lean_ctor_set(x_263, 1, x_262); -return x_263; +x_257 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_257, 0, x_255); +lean_ctor_set(x_257, 1, x_256); +return x_257; } } } -else +default: { -uint8_t x_264; -lean_dec(x_241); -lean_dec(x_238); -lean_dec(x_1); -x_264 = !lean_is_exclusive(x_243); -if (x_264 == 0) +lean_object* x_258; +x_258 = lean_st_ref_take(x_2, x_48); +if (lean_obj_tag(x_258) == 0) { -return x_243; +lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; +x_259 = lean_ctor_get(x_258, 0); +lean_inc(x_259); +x_260 = lean_ctor_get(x_258, 1); +lean_inc(x_260); +lean_dec(x_258); +lean_inc_n(x_1, 2); +x_261 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_259, x_1, x_1); +x_262 = lean_st_ref_set(x_2, x_261, x_260); +if (lean_obj_tag(x_262) == 0) +{ +uint8_t x_263; +x_263 = !lean_is_exclusive(x_262); +if (x_263 == 0) +{ +lean_object* x_264; +x_264 = lean_ctor_get(x_262, 0); +lean_dec(x_264); +lean_ctor_set(x_262, 0, x_1); +return x_262; } else { -lean_object* x_265; lean_object* x_266; lean_object* x_267; -x_265 = lean_ctor_get(x_243, 0); -x_266 = lean_ctor_get(x_243, 1); -lean_inc(x_266); +lean_object* x_265; lean_object* x_266; +x_265 = lean_ctor_get(x_262, 1); lean_inc(x_265); -lean_dec(x_243); -x_267 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_267, 0, x_265); -lean_ctor_set(x_267, 1, x_266); -return x_267; -} +lean_dec(x_262); +x_266 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_266, 0, x_1); +lean_ctor_set(x_266, 1, x_265); +return x_266; } } else { -uint8_t x_268; -lean_dec(x_238); -lean_dec(x_236); +uint8_t x_267; lean_dec(x_1); -x_268 = !lean_is_exclusive(x_240); -if (x_268 == 0) +x_267 = !lean_is_exclusive(x_262); +if (x_267 == 0) { -return x_240; +return x_262; } else { -lean_object* x_269; lean_object* x_270; lean_object* x_271; -x_269 = lean_ctor_get(x_240, 0); -x_270 = lean_ctor_get(x_240, 1); -lean_inc(x_270); +lean_object* x_268; lean_object* x_269; lean_object* x_270; +x_268 = lean_ctor_get(x_262, 0); +x_269 = lean_ctor_get(x_262, 1); lean_inc(x_269); -lean_dec(x_240); -x_271 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_271, 0, x_269); -lean_ctor_set(x_271, 1, x_270); -return x_271; +lean_inc(x_268); +lean_dec(x_262); +x_270 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_270, 0, x_268); +lean_ctor_set(x_270, 1, x_269); +return x_270; } } } else { -uint8_t x_272; -lean_dec(x_236); -lean_dec(x_235); +uint8_t x_271; lean_dec(x_1); -x_272 = !lean_is_exclusive(x_237); -if (x_272 == 0) +x_271 = !lean_is_exclusive(x_258); +if (x_271 == 0) { -return x_237; +return x_258; } else { -lean_object* x_273; lean_object* x_274; lean_object* x_275; -x_273 = lean_ctor_get(x_237, 0); -x_274 = lean_ctor_get(x_237, 1); -lean_inc(x_274); +lean_object* x_272; lean_object* x_273; lean_object* x_274; +x_272 = lean_ctor_get(x_258, 0); +x_273 = lean_ctor_get(x_258, 1); lean_inc(x_273); -lean_dec(x_237); -x_275 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_275, 0, x_273); -lean_ctor_set(x_275, 1, x_274); -return x_275; +lean_inc(x_272); +lean_dec(x_258); +x_274 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_274, 0, x_272); +lean_ctor_set(x_274, 1, x_273); +return x_274; } } } -case 10: +} +} +else { -lean_object* x_276; lean_object* x_277; -x_276 = lean_ctor_get(x_1, 1); +lean_object* x_275; +lean_dec(x_1); +x_275 = lean_ctor_get(x_49, 0); +lean_inc(x_275); +lean_dec(x_49); +lean_ctor_set(x_45, 0, x_275); +return x_45; +} +} +else +{ +lean_object* x_276; lean_object* x_277; lean_object* x_278; +x_276 = lean_ctor_get(x_45, 0); +x_277 = lean_ctor_get(x_45, 1); +lean_inc(x_277); lean_inc(x_276); -x_277 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_276, x_2, x_3, x_48); -if (lean_obj_tag(x_277) == 0) +lean_dec(x_45); +lean_inc(x_1); +x_278 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_276, x_1); +if (lean_obj_tag(x_278) == 0) { -lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; -x_278 = lean_ctor_get(x_277, 0); -lean_inc(x_278); -x_279 = lean_ctor_get(x_277, 1); +switch (lean_obj_tag(x_1)) { +case 2: +{ +lean_object* x_279; lean_object* x_280; +x_279 = lean_ctor_get(x_1, 0); lean_inc(x_279); -lean_dec(x_277); -lean_inc(x_1); -x_280 = lean_expr_update_mdata(x_1, x_278); -x_281 = lean_st_ref_take(x_2, x_279); -if (lean_obj_tag(x_281) == 0) +x_280 = lean_st_ref_get(x_2, x_277); +if (lean_obj_tag(x_280) == 0) { -lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; -x_282 = lean_ctor_get(x_281, 0); +lean_object* x_281; lean_object* x_282; lean_object* x_283; +x_281 = lean_ctor_get(x_280, 0); +lean_inc(x_281); +x_282 = lean_ctor_get(x_280, 1); lean_inc(x_282); -x_283 = lean_ctor_get(x_281, 1); -lean_inc(x_283); -lean_dec(x_281); -lean_inc(x_280); -x_284 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_282, x_1, x_280); -x_285 = lean_st_ref_set(x_2, x_284, x_283); -if (lean_obj_tag(x_285) == 0) +lean_dec(x_280); +lean_inc(x_1); +x_283 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_281, x_1); +if (lean_obj_tag(x_283) == 0) { -uint8_t x_286; -x_286 = !lean_is_exclusive(x_285); -if (x_286 == 0) +lean_object* x_284; +lean_inc(x_279); +x_284 = l_Lean_getExprMVarAssignment_x3f___at_Lean_instantiateMVarsCore___spec__3___rarg(x_279, x_2, x_3, x_282); +if (lean_obj_tag(x_284) == 0) { -lean_object* x_287; -x_287 = lean_ctor_get(x_285, 0); -lean_dec(x_287); -lean_ctor_set(x_285, 0, x_280); -return x_285; +lean_object* x_285; +x_285 = lean_ctor_get(x_284, 0); +lean_inc(x_285); +if (lean_obj_tag(x_285) == 0) +{ +lean_object* x_286; +lean_dec(x_279); +x_286 = lean_ctor_get(x_284, 1); +lean_inc(x_286); +lean_dec(x_284); +lean_inc(x_1); +x_28 = x_1; +x_29 = x_286; +goto block_44; } else { -lean_object* x_288; lean_object* x_289; -x_288 = lean_ctor_get(x_285, 1); +lean_object* x_287; lean_object* x_288; lean_object* x_289; +x_287 = lean_ctor_get(x_284, 1); +lean_inc(x_287); +lean_dec(x_284); +x_288 = lean_ctor_get(x_285, 0); lean_inc(x_288); lean_dec(x_285); -x_289 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_289, 0, x_280); -lean_ctor_set(x_289, 1, x_288); -return x_289; -} -} -else +x_289 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_288, x_2, x_3, x_287); +if (lean_obj_tag(x_289) == 0) { -uint8_t x_290; -lean_dec(x_280); -x_290 = !lean_is_exclusive(x_285); -if (x_290 == 0) +lean_object* x_290; lean_object* x_291; lean_object* x_292; +x_290 = lean_ctor_get(x_289, 0); +lean_inc(x_290); +x_291 = lean_ctor_get(x_289, 1); +lean_inc(x_291); +lean_dec(x_289); +lean_inc(x_290); +x_292 = l_Lean_assignExprMVar___at_Lean_instantiateMVarsCore___spec__5___rarg(x_279, x_290, x_2, x_3, x_291); +if (lean_obj_tag(x_292) == 0) { -return x_285; +lean_object* x_293; +x_293 = lean_ctor_get(x_292, 1); +lean_inc(x_293); +lean_dec(x_292); +x_28 = x_290; +x_29 = x_293; +goto block_44; } else { -lean_object* x_291; lean_object* x_292; lean_object* x_293; -x_291 = lean_ctor_get(x_285, 0); -x_292 = lean_ctor_get(x_285, 1); -lean_inc(x_292); -lean_inc(x_291); -lean_dec(x_285); -x_293 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_293, 0, x_291); -lean_ctor_set(x_293, 1, x_292); -return x_293; +lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; +lean_dec(x_290); +lean_dec(x_1); +x_294 = lean_ctor_get(x_292, 0); +lean_inc(x_294); +x_295 = lean_ctor_get(x_292, 1); +lean_inc(x_295); +if (lean_is_exclusive(x_292)) { + lean_ctor_release(x_292, 0); + lean_ctor_release(x_292, 1); + x_296 = x_292; +} else { + lean_dec_ref(x_292); + x_296 = lean_box(0); } +if (lean_is_scalar(x_296)) { + x_297 = lean_alloc_ctor(1, 2, 0); +} else { + x_297 = x_296; +} +lean_ctor_set(x_297, 0, x_294); +lean_ctor_set(x_297, 1, x_295); +return x_297; } } else { -uint8_t x_294; -lean_dec(x_280); +lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; +lean_dec(x_279); lean_dec(x_1); -x_294 = !lean_is_exclusive(x_281); -if (x_294 == 0) -{ -return x_281; +x_298 = lean_ctor_get(x_289, 0); +lean_inc(x_298); +x_299 = lean_ctor_get(x_289, 1); +lean_inc(x_299); +if (lean_is_exclusive(x_289)) { + lean_ctor_release(x_289, 0); + lean_ctor_release(x_289, 1); + x_300 = x_289; +} else { + lean_dec_ref(x_289); + x_300 = lean_box(0); } -else -{ -lean_object* x_295; lean_object* x_296; lean_object* x_297; -x_295 = lean_ctor_get(x_281, 0); -x_296 = lean_ctor_get(x_281, 1); -lean_inc(x_296); -lean_inc(x_295); -lean_dec(x_281); -x_297 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_297, 0, x_295); -lean_ctor_set(x_297, 1, x_296); -return x_297; +if (lean_is_scalar(x_300)) { + x_301 = lean_alloc_ctor(1, 2, 0); +} else { + x_301 = x_300; } +lean_ctor_set(x_301, 0, x_298); +lean_ctor_set(x_301, 1, x_299); +return x_301; } } -else -{ -uint8_t x_298; -lean_dec(x_1); -x_298 = !lean_is_exclusive(x_277); -if (x_298 == 0) -{ -return x_277; } else { -lean_object* x_299; lean_object* x_300; lean_object* x_301; -x_299 = lean_ctor_get(x_277, 0); -x_300 = lean_ctor_get(x_277, 1); -lean_inc(x_300); -lean_inc(x_299); -lean_dec(x_277); -x_301 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_301, 0, x_299); -lean_ctor_set(x_301, 1, x_300); -return x_301; +lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; +lean_dec(x_279); +lean_dec(x_1); +x_302 = lean_ctor_get(x_284, 0); +lean_inc(x_302); +x_303 = lean_ctor_get(x_284, 1); +lean_inc(x_303); +if (lean_is_exclusive(x_284)) { + lean_ctor_release(x_284, 0); + lean_ctor_release(x_284, 1); + x_304 = x_284; +} else { + lean_dec_ref(x_284); + x_304 = lean_box(0); } +if (lean_is_scalar(x_304)) { + x_305 = lean_alloc_ctor(1, 2, 0); +} else { + x_305 = x_304; } +lean_ctor_set(x_305, 0, x_302); +lean_ctor_set(x_305, 1, x_303); +return x_305; } -case 11: -{ -lean_object* x_302; lean_object* x_303; -x_302 = lean_ctor_get(x_1, 2); -lean_inc(x_302); -x_303 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_302, x_2, x_3, x_48); -if (lean_obj_tag(x_303) == 0) -{ -lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; -x_304 = lean_ctor_get(x_303, 0); -lean_inc(x_304); -x_305 = lean_ctor_get(x_303, 1); -lean_inc(x_305); -lean_dec(x_303); -lean_inc(x_1); -x_306 = lean_expr_update_proj(x_1, x_304); -x_307 = lean_st_ref_take(x_2, x_305); -if (lean_obj_tag(x_307) == 0) -{ -lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; -x_308 = lean_ctor_get(x_307, 0); -lean_inc(x_308); -x_309 = lean_ctor_get(x_307, 1); -lean_inc(x_309); -lean_dec(x_307); -lean_inc(x_306); -x_310 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_308, x_1, x_306); -x_311 = lean_st_ref_set(x_2, x_310, x_309); -if (lean_obj_tag(x_311) == 0) -{ -uint8_t x_312; -x_312 = !lean_is_exclusive(x_311); -if (x_312 == 0) -{ -lean_object* x_313; -x_313 = lean_ctor_get(x_311, 0); -lean_dec(x_313); -lean_ctor_set(x_311, 0, x_306); -return x_311; } else { -lean_object* x_314; lean_object* x_315; -x_314 = lean_ctor_get(x_311, 1); -lean_inc(x_314); -lean_dec(x_311); -x_315 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_315, 0, x_306); -lean_ctor_set(x_315, 1, x_314); -return x_315; +lean_object* x_306; +lean_dec(x_279); +x_306 = lean_ctor_get(x_283, 0); +lean_inc(x_306); +lean_dec(x_283); +x_8 = x_306; +x_9 = x_282; +goto block_27; } } else { -uint8_t x_316; -lean_dec(x_306); -x_316 = !lean_is_exclusive(x_311); -if (x_316 == 0) -{ -return x_311; +lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; +lean_dec(x_279); +lean_dec(x_1); +x_307 = lean_ctor_get(x_280, 0); +lean_inc(x_307); +x_308 = lean_ctor_get(x_280, 1); +lean_inc(x_308); +if (lean_is_exclusive(x_280)) { + lean_ctor_release(x_280, 0); + lean_ctor_release(x_280, 1); + x_309 = x_280; +} else { + lean_dec_ref(x_280); + x_309 = lean_box(0); } -else -{ -lean_object* x_317; lean_object* x_318; lean_object* x_319; -x_317 = lean_ctor_get(x_311, 0); -x_318 = lean_ctor_get(x_311, 1); -lean_inc(x_318); -lean_inc(x_317); -lean_dec(x_311); -x_319 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_319, 0, x_317); -lean_ctor_set(x_319, 1, x_318); -return x_319; +if (lean_is_scalar(x_309)) { + x_310 = lean_alloc_ctor(1, 2, 0); +} else { + x_310 = x_309; } +lean_ctor_set(x_310, 0, x_307); +lean_ctor_set(x_310, 1, x_308); +return x_310; } } -else -{ -uint8_t x_320; -lean_dec(x_306); -lean_dec(x_1); -x_320 = !lean_is_exclusive(x_307); -if (x_320 == 0) +case 3: { -return x_307; +lean_object* x_311; lean_object* x_312; +x_311 = lean_ctor_get(x_1, 0); +lean_inc(x_311); +lean_inc(x_311); +x_312 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_311, x_2, x_3, x_277); +if (lean_obj_tag(x_312) == 0) +{ +lean_object* x_313; lean_object* x_314; size_t x_315; size_t x_316; uint8_t x_317; +x_313 = lean_ctor_get(x_312, 0); +lean_inc(x_313); +x_314 = lean_ctor_get(x_312, 1); +lean_inc(x_314); +lean_dec(x_312); +x_315 = lean_ptr_addr(x_311); +lean_dec(x_311); +x_316 = lean_ptr_addr(x_313); +x_317 = lean_usize_dec_eq(x_315, x_316); +if (x_317 == 0) +{ +lean_object* x_318; +x_318 = l_Lean_Expr_sort___override(x_313); +x_8 = x_318; +x_9 = x_314; +goto block_27; } else { -lean_object* x_321; lean_object* x_322; lean_object* x_323; -x_321 = lean_ctor_get(x_307, 0); -x_322 = lean_ctor_get(x_307, 1); -lean_inc(x_322); -lean_inc(x_321); -lean_dec(x_307); -x_323 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_323, 0, x_321); -lean_ctor_set(x_323, 1, x_322); -return x_323; -} +lean_dec(x_313); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_314; +goto block_27; } } else { -uint8_t x_324; +lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; +lean_dec(x_311); lean_dec(x_1); -x_324 = !lean_is_exclusive(x_303); -if (x_324 == 0) -{ -return x_303; +x_319 = lean_ctor_get(x_312, 0); +lean_inc(x_319); +x_320 = lean_ctor_get(x_312, 1); +lean_inc(x_320); +if (lean_is_exclusive(x_312)) { + lean_ctor_release(x_312, 0); + lean_ctor_release(x_312, 1); + x_321 = x_312; +} else { + lean_dec_ref(x_312); + x_321 = lean_box(0); } -else -{ -lean_object* x_325; lean_object* x_326; lean_object* x_327; -x_325 = lean_ctor_get(x_303, 0); -x_326 = lean_ctor_get(x_303, 1); -lean_inc(x_326); -lean_inc(x_325); -lean_dec(x_303); -x_327 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_327, 0, x_325); -lean_ctor_set(x_327, 1, x_326); -return x_327; +if (lean_is_scalar(x_321)) { + x_322 = lean_alloc_ctor(1, 2, 0); +} else { + x_322 = x_321; } +lean_ctor_set(x_322, 0, x_319); +lean_ctor_set(x_322, 1, x_320); +return x_322; } } -default: -{ -lean_object* x_328; -x_328 = lean_st_ref_take(x_2, x_48); -if (lean_obj_tag(x_328) == 0) +case 4: { -lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; -x_329 = lean_ctor_get(x_328, 0); -lean_inc(x_329); -x_330 = lean_ctor_get(x_328, 1); -lean_inc(x_330); -lean_dec(x_328); -lean_inc_n(x_1, 2); -x_331 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_329, x_1, x_1); -x_332 = lean_st_ref_set(x_2, x_331, x_330); -if (lean_obj_tag(x_332) == 0) +lean_object* x_323; lean_object* x_324; lean_object* x_325; +x_323 = lean_ctor_get(x_1, 0); +lean_inc(x_323); +x_324 = lean_ctor_get(x_1, 1); +lean_inc(x_324); +lean_inc(x_324); +x_325 = l_List_mapM___at_Lean_instantiateMVarsCore___spec__12___rarg(x_5, x_324, x_2, x_3, x_277); +if (lean_obj_tag(x_325) == 0) { -uint8_t x_333; -x_333 = !lean_is_exclusive(x_332); -if (x_333 == 0) +lean_object* x_326; lean_object* x_327; uint8_t x_328; +x_326 = lean_ctor_get(x_325, 0); +lean_inc(x_326); +x_327 = lean_ctor_get(x_325, 1); +lean_inc(x_327); +lean_dec(x_325); +x_328 = l_ptrEqList___rarg(x_324, x_326); +lean_dec(x_324); +if (x_328 == 0) { -lean_object* x_334; -x_334 = lean_ctor_get(x_332, 0); -lean_dec(x_334); -lean_ctor_set(x_332, 0, x_1); -return x_332; +lean_object* x_329; +x_329 = l_Lean_Expr_const___override(x_323, x_326); +x_8 = x_329; +x_9 = x_327; +goto block_27; } else { -lean_object* x_335; lean_object* x_336; -x_335 = lean_ctor_get(x_332, 1); -lean_inc(x_335); -lean_dec(x_332); -x_336 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_336, 0, x_1); -lean_ctor_set(x_336, 1, x_335); -return x_336; +lean_dec(x_326); +lean_dec(x_323); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_327; +goto block_27; } } else { -uint8_t x_337; +lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; +lean_dec(x_324); +lean_dec(x_323); lean_dec(x_1); -x_337 = !lean_is_exclusive(x_332); -if (x_337 == 0) -{ -return x_332; +x_330 = lean_ctor_get(x_325, 0); +lean_inc(x_330); +x_331 = lean_ctor_get(x_325, 1); +lean_inc(x_331); +if (lean_is_exclusive(x_325)) { + lean_ctor_release(x_325, 0); + lean_ctor_release(x_325, 1); + x_332 = x_325; +} else { + lean_dec_ref(x_325); + x_332 = lean_box(0); } -else -{ -lean_object* x_338; lean_object* x_339; lean_object* x_340; -x_338 = lean_ctor_get(x_332, 0); -x_339 = lean_ctor_get(x_332, 1); -lean_inc(x_339); -lean_inc(x_338); -lean_dec(x_332); -x_340 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_340, 0, x_338); -lean_ctor_set(x_340, 1, x_339); -return x_340; +if (lean_is_scalar(x_332)) { + x_333 = lean_alloc_ctor(1, 2, 0); +} else { + x_333 = x_332; } +lean_ctor_set(x_333, 0, x_330); +lean_ctor_set(x_333, 1, x_331); +return x_333; } } -else -{ -uint8_t x_341; -lean_dec(x_1); -x_341 = !lean_is_exclusive(x_328); -if (x_341 == 0) +case 5: { -return x_328; -} -else +lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; +x_334 = lean_unsigned_to_nat(0u); +x_335 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_334); +x_336 = l_Lean_instantiateExprMVars___rarg___lambda__20___closed__1; +lean_inc(x_335); +x_337 = lean_mk_array(x_335, x_336); +x_338 = lean_unsigned_to_nat(1u); +x_339 = lean_nat_sub(x_335, x_338); +lean_dec(x_335); +lean_inc(x_1); +x_340 = l_Lean_Expr_withAppAux___at_Lean_instantiateMVarsCore___spec__42___rarg(x_5, x_1, x_337, x_339, x_2, x_3, x_277); +if (lean_obj_tag(x_340) == 0) { -lean_object* x_342; lean_object* x_343; lean_object* x_344; -x_342 = lean_ctor_get(x_328, 0); -x_343 = lean_ctor_get(x_328, 1); -lean_inc(x_343); +lean_object* x_341; lean_object* x_342; lean_object* x_343; +x_341 = lean_ctor_get(x_340, 0); +lean_inc(x_341); +x_342 = lean_ctor_get(x_340, 1); lean_inc(x_342); -lean_dec(x_328); -x_344 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_344, 0, x_342); -lean_ctor_set(x_344, 1, x_343); -return x_344; -} -} -} -} -} -else -{ -lean_object* x_345; -lean_dec(x_1); -x_345 = lean_ctor_get(x_49, 0); +lean_dec(x_340); +x_343 = lean_st_ref_take(x_2, x_342); +if (lean_obj_tag(x_343) == 0) +{ +lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; +x_344 = lean_ctor_get(x_343, 0); +lean_inc(x_344); +x_345 = lean_ctor_get(x_343, 1); lean_inc(x_345); -lean_dec(x_49); -lean_ctor_set(x_45, 0, x_345); -return x_45; +lean_dec(x_343); +lean_inc(x_341); +x_346 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_344, x_1, x_341); +x_347 = lean_st_ref_set(x_2, x_346, x_345); +if (lean_obj_tag(x_347) == 0) +{ +lean_object* x_348; lean_object* x_349; lean_object* x_350; +x_348 = lean_ctor_get(x_347, 1); +lean_inc(x_348); +if (lean_is_exclusive(x_347)) { + lean_ctor_release(x_347, 0); + lean_ctor_release(x_347, 1); + x_349 = x_347; +} else { + lean_dec_ref(x_347); + x_349 = lean_box(0); +} +if (lean_is_scalar(x_349)) { + x_350 = lean_alloc_ctor(0, 2, 0); +} else { + x_350 = x_349; } +lean_ctor_set(x_350, 0, x_341); +lean_ctor_set(x_350, 1, x_348); +return x_350; } else { -lean_object* x_346; lean_object* x_347; lean_object* x_348; -x_346 = lean_ctor_get(x_45, 0); -x_347 = lean_ctor_get(x_45, 1); -lean_inc(x_347); -lean_inc(x_346); -lean_dec(x_45); -lean_inc(x_1); -x_348 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_346, x_1); -if (lean_obj_tag(x_348) == 0) -{ -switch (lean_obj_tag(x_1)) { -case 2: -{ -lean_object* x_349; lean_object* x_350; -x_349 = lean_ctor_get(x_1, 0); -lean_inc(x_349); -x_350 = lean_st_ref_get(x_2, x_347); -if (lean_obj_tag(x_350) == 0) -{ -lean_object* x_351; lean_object* x_352; lean_object* x_353; -x_351 = lean_ctor_get(x_350, 0); +lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; +lean_dec(x_341); +x_351 = lean_ctor_get(x_347, 0); lean_inc(x_351); -x_352 = lean_ctor_get(x_350, 1); +x_352 = lean_ctor_get(x_347, 1); lean_inc(x_352); -lean_dec(x_350); -lean_inc(x_1); -x_353 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_351, x_1); -if (lean_obj_tag(x_353) == 0) -{ -lean_object* x_354; -lean_inc(x_349); -x_354 = l_Lean_getExprMVarAssignment_x3f___at_Lean_instantiateMVarsCore___spec__3___rarg(x_349, x_2, x_3, x_352); -if (lean_obj_tag(x_354) == 0) -{ -lean_object* x_355; -x_355 = lean_ctor_get(x_354, 0); -lean_inc(x_355); -if (lean_obj_tag(x_355) == 0) -{ -lean_object* x_356; -lean_dec(x_349); -x_356 = lean_ctor_get(x_354, 1); -lean_inc(x_356); -lean_dec(x_354); -lean_inc(x_1); -x_28 = x_1; -x_29 = x_356; -goto block_44; -} -else -{ -lean_object* x_357; lean_object* x_358; lean_object* x_359; -x_357 = lean_ctor_get(x_354, 1); -lean_inc(x_357); -lean_dec(x_354); -x_358 = lean_ctor_get(x_355, 0); -lean_inc(x_358); -lean_dec(x_355); -x_359 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_358, x_2, x_3, x_357); -if (lean_obj_tag(x_359) == 0) -{ -lean_object* x_360; lean_object* x_361; lean_object* x_362; -x_360 = lean_ctor_get(x_359, 0); -lean_inc(x_360); -x_361 = lean_ctor_get(x_359, 1); -lean_inc(x_361); -lean_dec(x_359); -lean_inc(x_360); -x_362 = l_Lean_assignExprMVar___at_Lean_instantiateMVarsCore___spec__5___rarg(x_349, x_360, x_2, x_3, x_361); -if (lean_obj_tag(x_362) == 0) -{ -lean_object* x_363; -x_363 = lean_ctor_get(x_362, 1); -lean_inc(x_363); -lean_dec(x_362); -x_28 = x_360; -x_29 = x_363; -goto block_44; -} -else -{ -lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; -lean_dec(x_360); -lean_dec(x_1); -x_364 = lean_ctor_get(x_362, 0); -lean_inc(x_364); -x_365 = lean_ctor_get(x_362, 1); -lean_inc(x_365); -if (lean_is_exclusive(x_362)) { - lean_ctor_release(x_362, 0); - lean_ctor_release(x_362, 1); - x_366 = x_362; +if (lean_is_exclusive(x_347)) { + lean_ctor_release(x_347, 0); + lean_ctor_release(x_347, 1); + x_353 = x_347; } else { - lean_dec_ref(x_362); - x_366 = lean_box(0); + lean_dec_ref(x_347); + x_353 = lean_box(0); } -if (lean_is_scalar(x_366)) { - x_367 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_353)) { + x_354 = lean_alloc_ctor(1, 2, 0); } else { - x_367 = x_366; + x_354 = x_353; } -lean_ctor_set(x_367, 0, x_364); -lean_ctor_set(x_367, 1, x_365); -return x_367; +lean_ctor_set(x_354, 0, x_351); +lean_ctor_set(x_354, 1, x_352); +return x_354; } } else { -lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; -lean_dec(x_349); +lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; +lean_dec(x_341); lean_dec(x_1); -x_368 = lean_ctor_get(x_359, 0); -lean_inc(x_368); -x_369 = lean_ctor_get(x_359, 1); -lean_inc(x_369); -if (lean_is_exclusive(x_359)) { - lean_ctor_release(x_359, 0); - lean_ctor_release(x_359, 1); - x_370 = x_359; +x_355 = lean_ctor_get(x_343, 0); +lean_inc(x_355); +x_356 = lean_ctor_get(x_343, 1); +lean_inc(x_356); +if (lean_is_exclusive(x_343)) { + lean_ctor_release(x_343, 0); + lean_ctor_release(x_343, 1); + x_357 = x_343; } else { - lean_dec_ref(x_359); - x_370 = lean_box(0); + lean_dec_ref(x_343); + x_357 = lean_box(0); } -if (lean_is_scalar(x_370)) { - x_371 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_357)) { + x_358 = lean_alloc_ctor(1, 2, 0); } else { - x_371 = x_370; -} -lean_ctor_set(x_371, 0, x_368); -lean_ctor_set(x_371, 1, x_369); -return x_371; + x_358 = x_357; } +lean_ctor_set(x_358, 0, x_355); +lean_ctor_set(x_358, 1, x_356); +return x_358; } } else { -lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; -lean_dec(x_349); +lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_dec(x_1); -x_372 = lean_ctor_get(x_354, 0); -lean_inc(x_372); -x_373 = lean_ctor_get(x_354, 1); -lean_inc(x_373); -if (lean_is_exclusive(x_354)) { - lean_ctor_release(x_354, 0); - lean_ctor_release(x_354, 1); - x_374 = x_354; +x_359 = lean_ctor_get(x_340, 0); +lean_inc(x_359); +x_360 = lean_ctor_get(x_340, 1); +lean_inc(x_360); +if (lean_is_exclusive(x_340)) { + lean_ctor_release(x_340, 0); + lean_ctor_release(x_340, 1); + x_361 = x_340; } else { - lean_dec_ref(x_354); - x_374 = lean_box(0); + lean_dec_ref(x_340); + x_361 = lean_box(0); } -if (lean_is_scalar(x_374)) { - x_375 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_361)) { + x_362 = lean_alloc_ctor(1, 2, 0); } else { - x_375 = x_374; + x_362 = x_361; } -lean_ctor_set(x_375, 0, x_372); -lean_ctor_set(x_375, 1, x_373); -return x_375; +lean_ctor_set(x_362, 0, x_359); +lean_ctor_set(x_362, 1, x_360); +return x_362; } } -else +case 6: +{ +lean_object* x_363; lean_object* x_364; lean_object* x_365; uint8_t x_366; lean_object* x_367; +x_363 = lean_ctor_get(x_1, 0); +lean_inc(x_363); +x_364 = lean_ctor_get(x_1, 1); +lean_inc(x_364); +x_365 = lean_ctor_get(x_1, 2); +lean_inc(x_365); +x_366 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_inc(x_364); +x_367 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_364, x_2, x_3, x_277); +if (lean_obj_tag(x_367) == 0) +{ +lean_object* x_368; lean_object* x_369; lean_object* x_370; +x_368 = lean_ctor_get(x_367, 0); +lean_inc(x_368); +x_369 = lean_ctor_get(x_367, 1); +lean_inc(x_369); +lean_dec(x_367); +lean_inc(x_365); +x_370 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_365, x_2, x_3, x_369); +if (lean_obj_tag(x_370) == 0) { -lean_object* x_376; -lean_dec(x_349); -x_376 = lean_ctor_get(x_353, 0); -lean_inc(x_376); -lean_dec(x_353); -x_8 = x_376; -x_9 = x_352; +lean_object* x_371; lean_object* x_372; lean_object* x_373; size_t x_374; size_t x_375; uint8_t x_376; +x_371 = lean_ctor_get(x_370, 0); +lean_inc(x_371); +x_372 = lean_ctor_get(x_370, 1); +lean_inc(x_372); +lean_dec(x_370); +lean_inc(x_365); +lean_inc(x_364); +lean_inc(x_363); +x_373 = l_Lean_Expr_lam___override(x_363, x_364, x_365, x_366); +x_374 = lean_ptr_addr(x_364); +lean_dec(x_364); +x_375 = lean_ptr_addr(x_368); +x_376 = lean_usize_dec_eq(x_374, x_375); +if (x_376 == 0) +{ +lean_object* x_377; +lean_dec(x_373); +lean_dec(x_365); +x_377 = l_Lean_Expr_lam___override(x_363, x_368, x_371, x_366); +x_8 = x_377; +x_9 = x_372; goto block_27; } -} else { -lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; -lean_dec(x_349); -lean_dec(x_1); -x_377 = lean_ctor_get(x_350, 0); -lean_inc(x_377); -x_378 = lean_ctor_get(x_350, 1); -lean_inc(x_378); -if (lean_is_exclusive(x_350)) { - lean_ctor_release(x_350, 0); - lean_ctor_release(x_350, 1); - x_379 = x_350; -} else { - lean_dec_ref(x_350); - x_379 = lean_box(0); -} -if (lean_is_scalar(x_379)) { - x_380 = lean_alloc_ctor(1, 2, 0); -} else { - x_380 = x_379; -} -lean_ctor_set(x_380, 0, x_377); -lean_ctor_set(x_380, 1, x_378); -return x_380; -} +size_t x_378; size_t x_379; uint8_t x_380; +x_378 = lean_ptr_addr(x_365); +lean_dec(x_365); +x_379 = lean_ptr_addr(x_371); +x_380 = lean_usize_dec_eq(x_378, x_379); +if (x_380 == 0) +{ +lean_object* x_381; +lean_dec(x_373); +x_381 = l_Lean_Expr_lam___override(x_363, x_368, x_371, x_366); +x_8 = x_381; +x_9 = x_372; +goto block_27; } -case 3: -{ -lean_object* x_381; lean_object* x_382; -x_381 = lean_ctor_get(x_1, 0); -lean_inc(x_381); -x_382 = l_Lean_instantiateLevelMVars___at_Lean_instantiateMVarsCore___spec__6___rarg(x_381, x_2, x_3, x_347); -if (lean_obj_tag(x_382) == 0) +else { -lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; -x_383 = lean_ctor_get(x_382, 0); -lean_inc(x_383); -x_384 = lean_ctor_get(x_382, 1); -lean_inc(x_384); -lean_dec(x_382); -lean_inc(x_1); -x_385 = lean_expr_update_sort(x_1, x_383); -x_386 = lean_st_ref_take(x_2, x_384); -if (lean_obj_tag(x_386) == 0) +uint8_t x_382; +x_382 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_366, x_366); +if (x_382 == 0) { -lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; -x_387 = lean_ctor_get(x_386, 0); -lean_inc(x_387); -x_388 = lean_ctor_get(x_386, 1); -lean_inc(x_388); -lean_dec(x_386); -lean_inc(x_385); -x_389 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_387, x_1, x_385); -x_390 = lean_st_ref_set(x_2, x_389, x_388); -if (lean_obj_tag(x_390) == 0) -{ -lean_object* x_391; lean_object* x_392; lean_object* x_393; -x_391 = lean_ctor_get(x_390, 1); -lean_inc(x_391); -if (lean_is_exclusive(x_390)) { - lean_ctor_release(x_390, 0); - lean_ctor_release(x_390, 1); - x_392 = x_390; -} else { - lean_dec_ref(x_390); - x_392 = lean_box(0); -} -if (lean_is_scalar(x_392)) { - x_393 = lean_alloc_ctor(0, 2, 0); -} else { - x_393 = x_392; -} -lean_ctor_set(x_393, 0, x_385); -lean_ctor_set(x_393, 1, x_391); -return x_393; +lean_object* x_383; +lean_dec(x_373); +x_383 = l_Lean_Expr_lam___override(x_363, x_368, x_371, x_366); +x_8 = x_383; +x_9 = x_372; +goto block_27; } else { -lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; -lean_dec(x_385); -x_394 = lean_ctor_get(x_390, 0); -lean_inc(x_394); -x_395 = lean_ctor_get(x_390, 1); -lean_inc(x_395); -if (lean_is_exclusive(x_390)) { - lean_ctor_release(x_390, 0); - lean_ctor_release(x_390, 1); - x_396 = x_390; -} else { - lean_dec_ref(x_390); - x_396 = lean_box(0); +lean_dec(x_371); +lean_dec(x_368); +lean_dec(x_363); +x_8 = x_373; +x_9 = x_372; +goto block_27; } -if (lean_is_scalar(x_396)) { - x_397 = lean_alloc_ctor(1, 2, 0); -} else { - x_397 = x_396; } -lean_ctor_set(x_397, 0, x_394); -lean_ctor_set(x_397, 1, x_395); -return x_397; } } else { -lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; -lean_dec(x_385); +lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; +lean_dec(x_368); +lean_dec(x_365); +lean_dec(x_364); +lean_dec(x_363); lean_dec(x_1); -x_398 = lean_ctor_get(x_386, 0); -lean_inc(x_398); -x_399 = lean_ctor_get(x_386, 1); -lean_inc(x_399); -if (lean_is_exclusive(x_386)) { - lean_ctor_release(x_386, 0); - lean_ctor_release(x_386, 1); - x_400 = x_386; +x_384 = lean_ctor_get(x_370, 0); +lean_inc(x_384); +x_385 = lean_ctor_get(x_370, 1); +lean_inc(x_385); +if (lean_is_exclusive(x_370)) { + lean_ctor_release(x_370, 0); + lean_ctor_release(x_370, 1); + x_386 = x_370; } else { - lean_dec_ref(x_386); - x_400 = lean_box(0); + lean_dec_ref(x_370); + x_386 = lean_box(0); } -if (lean_is_scalar(x_400)) { - x_401 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_386)) { + x_387 = lean_alloc_ctor(1, 2, 0); } else { - x_401 = x_400; + x_387 = x_386; } -lean_ctor_set(x_401, 0, x_398); -lean_ctor_set(x_401, 1, x_399); -return x_401; +lean_ctor_set(x_387, 0, x_384); +lean_ctor_set(x_387, 1, x_385); +return x_387; } } else { -lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; +lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; +lean_dec(x_365); +lean_dec(x_364); +lean_dec(x_363); lean_dec(x_1); -x_402 = lean_ctor_get(x_382, 0); -lean_inc(x_402); -x_403 = lean_ctor_get(x_382, 1); -lean_inc(x_403); -if (lean_is_exclusive(x_382)) { - lean_ctor_release(x_382, 0); - lean_ctor_release(x_382, 1); - x_404 = x_382; +x_388 = lean_ctor_get(x_367, 0); +lean_inc(x_388); +x_389 = lean_ctor_get(x_367, 1); +lean_inc(x_389); +if (lean_is_exclusive(x_367)) { + lean_ctor_release(x_367, 0); + lean_ctor_release(x_367, 1); + x_390 = x_367; } else { - lean_dec_ref(x_382); - x_404 = lean_box(0); + lean_dec_ref(x_367); + x_390 = lean_box(0); } -if (lean_is_scalar(x_404)) { - x_405 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_390)) { + x_391 = lean_alloc_ctor(1, 2, 0); } else { - x_405 = x_404; + x_391 = x_390; } -lean_ctor_set(x_405, 0, x_402); -lean_ctor_set(x_405, 1, x_403); -return x_405; +lean_ctor_set(x_391, 0, x_388); +lean_ctor_set(x_391, 1, x_389); +return x_391; } } -case 4: +case 7: { -lean_object* x_406; lean_object* x_407; -x_406 = lean_ctor_get(x_1, 1); -lean_inc(x_406); -x_407 = l_List_mapM___at_Lean_instantiateMVarsCore___spec__12___rarg(x_5, x_406, x_2, x_3, x_347); -if (lean_obj_tag(x_407) == 0) -{ -lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; -x_408 = lean_ctor_get(x_407, 0); -lean_inc(x_408); -x_409 = lean_ctor_get(x_407, 1); -lean_inc(x_409); -lean_dec(x_407); -lean_inc(x_1); -x_410 = lean_expr_update_const(x_1, x_408); -x_411 = lean_st_ref_take(x_2, x_409); -if (lean_obj_tag(x_411) == 0) -{ -lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; -x_412 = lean_ctor_get(x_411, 0); -lean_inc(x_412); -x_413 = lean_ctor_get(x_411, 1); -lean_inc(x_413); -lean_dec(x_411); -lean_inc(x_410); -x_414 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_412, x_1, x_410); -x_415 = lean_st_ref_set(x_2, x_414, x_413); -if (lean_obj_tag(x_415) == 0) -{ -lean_object* x_416; lean_object* x_417; lean_object* x_418; -x_416 = lean_ctor_get(x_415, 1); -lean_inc(x_416); -if (lean_is_exclusive(x_415)) { - lean_ctor_release(x_415, 0); - lean_ctor_release(x_415, 1); - x_417 = x_415; -} else { - lean_dec_ref(x_415); - x_417 = lean_box(0); +lean_object* x_392; lean_object* x_393; lean_object* x_394; uint8_t x_395; lean_object* x_396; +x_392 = lean_ctor_get(x_1, 0); +lean_inc(x_392); +x_393 = lean_ctor_get(x_1, 1); +lean_inc(x_393); +x_394 = lean_ctor_get(x_1, 2); +lean_inc(x_394); +x_395 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_inc(x_393); +x_396 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_393, x_2, x_3, x_277); +if (lean_obj_tag(x_396) == 0) +{ +lean_object* x_397; lean_object* x_398; lean_object* x_399; +x_397 = lean_ctor_get(x_396, 0); +lean_inc(x_397); +x_398 = lean_ctor_get(x_396, 1); +lean_inc(x_398); +lean_dec(x_396); +lean_inc(x_394); +x_399 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_394, x_2, x_3, x_398); +if (lean_obj_tag(x_399) == 0) +{ +lean_object* x_400; lean_object* x_401; lean_object* x_402; size_t x_403; size_t x_404; uint8_t x_405; +x_400 = lean_ctor_get(x_399, 0); +lean_inc(x_400); +x_401 = lean_ctor_get(x_399, 1); +lean_inc(x_401); +lean_dec(x_399); +lean_inc(x_394); +lean_inc(x_393); +lean_inc(x_392); +x_402 = l_Lean_Expr_forallE___override(x_392, x_393, x_394, x_395); +x_403 = lean_ptr_addr(x_393); +lean_dec(x_393); +x_404 = lean_ptr_addr(x_397); +x_405 = lean_usize_dec_eq(x_403, x_404); +if (x_405 == 0) +{ +lean_object* x_406; +lean_dec(x_402); +lean_dec(x_394); +x_406 = l_Lean_Expr_forallE___override(x_392, x_397, x_400, x_395); +x_8 = x_406; +x_9 = x_401; +goto block_27; } -if (lean_is_scalar(x_417)) { - x_418 = lean_alloc_ctor(0, 2, 0); -} else { - x_418 = x_417; +else +{ +size_t x_407; size_t x_408; uint8_t x_409; +x_407 = lean_ptr_addr(x_394); +lean_dec(x_394); +x_408 = lean_ptr_addr(x_400); +x_409 = lean_usize_dec_eq(x_407, x_408); +if (x_409 == 0) +{ +lean_object* x_410; +lean_dec(x_402); +x_410 = l_Lean_Expr_forallE___override(x_392, x_397, x_400, x_395); +x_8 = x_410; +x_9 = x_401; +goto block_27; } -lean_ctor_set(x_418, 0, x_410); -lean_ctor_set(x_418, 1, x_416); -return x_418; +else +{ +uint8_t x_411; +x_411 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_395, x_395); +if (x_411 == 0) +{ +lean_object* x_412; +lean_dec(x_402); +x_412 = l_Lean_Expr_forallE___override(x_392, x_397, x_400, x_395); +x_8 = x_412; +x_9 = x_401; +goto block_27; } else { -lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; -lean_dec(x_410); -x_419 = lean_ctor_get(x_415, 0); -lean_inc(x_419); -x_420 = lean_ctor_get(x_415, 1); -lean_inc(x_420); -if (lean_is_exclusive(x_415)) { - lean_ctor_release(x_415, 0); - lean_ctor_release(x_415, 1); - x_421 = x_415; -} else { - lean_dec_ref(x_415); - x_421 = lean_box(0); +lean_dec(x_400); +lean_dec(x_397); +lean_dec(x_392); +x_8 = x_402; +x_9 = x_401; +goto block_27; } -if (lean_is_scalar(x_421)) { - x_422 = lean_alloc_ctor(1, 2, 0); -} else { - x_422 = x_421; } -lean_ctor_set(x_422, 0, x_419); -lean_ctor_set(x_422, 1, x_420); -return x_422; } } else { -lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; -lean_dec(x_410); +lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; +lean_dec(x_397); +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); lean_dec(x_1); -x_423 = lean_ctor_get(x_411, 0); -lean_inc(x_423); -x_424 = lean_ctor_get(x_411, 1); -lean_inc(x_424); -if (lean_is_exclusive(x_411)) { - lean_ctor_release(x_411, 0); - lean_ctor_release(x_411, 1); - x_425 = x_411; +x_413 = lean_ctor_get(x_399, 0); +lean_inc(x_413); +x_414 = lean_ctor_get(x_399, 1); +lean_inc(x_414); +if (lean_is_exclusive(x_399)) { + lean_ctor_release(x_399, 0); + lean_ctor_release(x_399, 1); + x_415 = x_399; } else { - lean_dec_ref(x_411); - x_425 = lean_box(0); + lean_dec_ref(x_399); + x_415 = lean_box(0); } -if (lean_is_scalar(x_425)) { - x_426 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_415)) { + x_416 = lean_alloc_ctor(1, 2, 0); } else { - x_426 = x_425; + x_416 = x_415; } -lean_ctor_set(x_426, 0, x_423); -lean_ctor_set(x_426, 1, x_424); -return x_426; +lean_ctor_set(x_416, 0, x_413); +lean_ctor_set(x_416, 1, x_414); +return x_416; } } else { -lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; +lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; +lean_dec(x_394); +lean_dec(x_393); +lean_dec(x_392); lean_dec(x_1); -x_427 = lean_ctor_get(x_407, 0); -lean_inc(x_427); -x_428 = lean_ctor_get(x_407, 1); -lean_inc(x_428); -if (lean_is_exclusive(x_407)) { - lean_ctor_release(x_407, 0); - lean_ctor_release(x_407, 1); - x_429 = x_407; +x_417 = lean_ctor_get(x_396, 0); +lean_inc(x_417); +x_418 = lean_ctor_get(x_396, 1); +lean_inc(x_418); +if (lean_is_exclusive(x_396)) { + lean_ctor_release(x_396, 0); + lean_ctor_release(x_396, 1); + x_419 = x_396; } else { - lean_dec_ref(x_407); - x_429 = lean_box(0); + lean_dec_ref(x_396); + x_419 = lean_box(0); } -if (lean_is_scalar(x_429)) { - x_430 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_419)) { + x_420 = lean_alloc_ctor(1, 2, 0); } else { - x_430 = x_429; + x_420 = x_419; } -lean_ctor_set(x_430, 0, x_427); -lean_ctor_set(x_430, 1, x_428); -return x_430; +lean_ctor_set(x_420, 0, x_417); +lean_ctor_set(x_420, 1, x_418); +return x_420; } } -case 5: +case 8: { -lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; -x_431 = lean_unsigned_to_nat(0u); -x_432 = l_Lean_Expr_getAppNumArgsAux(x_1, x_431); -x_433 = l_Lean_instantiateExprMVars___rarg___lambda__20___closed__1; -lean_inc(x_432); -x_434 = lean_mk_array(x_432, x_433); -x_435 = lean_unsigned_to_nat(1u); -x_436 = lean_nat_sub(x_432, x_435); +lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; uint8_t x_425; lean_object* x_426; +x_421 = lean_ctor_get(x_1, 0); +lean_inc(x_421); +x_422 = lean_ctor_get(x_1, 1); +lean_inc(x_422); +x_423 = lean_ctor_get(x_1, 2); +lean_inc(x_423); +x_424 = lean_ctor_get(x_1, 3); +lean_inc(x_424); +x_425 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); +lean_inc(x_422); +x_426 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_422, x_2, x_3, x_277); +if (lean_obj_tag(x_426) == 0) +{ +lean_object* x_427; lean_object* x_428; lean_object* x_429; +x_427 = lean_ctor_get(x_426, 0); +lean_inc(x_427); +x_428 = lean_ctor_get(x_426, 1); +lean_inc(x_428); +lean_dec(x_426); +lean_inc(x_423); +x_429 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_423, x_2, x_3, x_428); +if (lean_obj_tag(x_429) == 0) +{ +lean_object* x_430; lean_object* x_431; lean_object* x_432; +x_430 = lean_ctor_get(x_429, 0); +lean_inc(x_430); +x_431 = lean_ctor_get(x_429, 1); +lean_inc(x_431); +lean_dec(x_429); +lean_inc(x_424); +x_432 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_424, x_2, x_3, x_431); +if (lean_obj_tag(x_432) == 0) +{ +lean_object* x_433; lean_object* x_434; size_t x_435; size_t x_436; uint8_t x_437; +x_433 = lean_ctor_get(x_432, 0); +lean_inc(x_433); +x_434 = lean_ctor_get(x_432, 1); +lean_inc(x_434); lean_dec(x_432); -lean_inc(x_1); -x_437 = l_Lean_Expr_withAppAux___at_Lean_instantiateMVarsCore___spec__42___rarg(x_5, x_1, x_434, x_436, x_2, x_3, x_347); -if (lean_obj_tag(x_437) == 0) +x_435 = lean_ptr_addr(x_422); +lean_dec(x_422); +x_436 = lean_ptr_addr(x_427); +x_437 = lean_usize_dec_eq(x_435, x_436); +if (x_437 == 0) +{ +lean_object* x_438; +lean_dec(x_424); +lean_dec(x_423); +x_438 = l_Lean_Expr_letE___override(x_421, x_427, x_430, x_433, x_425); +x_8 = x_438; +x_9 = x_434; +goto block_27; +} +else { -lean_object* x_438; lean_object* x_439; lean_object* x_440; -x_438 = lean_ctor_get(x_437, 0); -lean_inc(x_438); -x_439 = lean_ctor_get(x_437, 1); -lean_inc(x_439); -lean_dec(x_437); -x_440 = lean_st_ref_take(x_2, x_439); -if (lean_obj_tag(x_440) == 0) -{ -lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; -x_441 = lean_ctor_get(x_440, 0); -lean_inc(x_441); -x_442 = lean_ctor_get(x_440, 1); -lean_inc(x_442); -lean_dec(x_440); -lean_inc(x_438); -x_443 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_441, x_1, x_438); -x_444 = lean_st_ref_set(x_2, x_443, x_442); -if (lean_obj_tag(x_444) == 0) +size_t x_439; size_t x_440; uint8_t x_441; +x_439 = lean_ptr_addr(x_423); +lean_dec(x_423); +x_440 = lean_ptr_addr(x_430); +x_441 = lean_usize_dec_eq(x_439, x_440); +if (x_441 == 0) { -lean_object* x_445; lean_object* x_446; lean_object* x_447; -x_445 = lean_ctor_get(x_444, 1); -lean_inc(x_445); -if (lean_is_exclusive(x_444)) { - lean_ctor_release(x_444, 0); - lean_ctor_release(x_444, 1); - x_446 = x_444; -} else { - lean_dec_ref(x_444); - x_446 = lean_box(0); +lean_object* x_442; +lean_dec(x_424); +x_442 = l_Lean_Expr_letE___override(x_421, x_427, x_430, x_433, x_425); +x_8 = x_442; +x_9 = x_434; +goto block_27; +} +else +{ +size_t x_443; size_t x_444; uint8_t x_445; +x_443 = lean_ptr_addr(x_424); +lean_dec(x_424); +x_444 = lean_ptr_addr(x_433); +x_445 = lean_usize_dec_eq(x_443, x_444); +if (x_445 == 0) +{ +lean_object* x_446; +x_446 = l_Lean_Expr_letE___override(x_421, x_427, x_430, x_433, x_425); +x_8 = x_446; +x_9 = x_434; +goto block_27; +} +else +{ +lean_dec(x_433); +lean_dec(x_430); +lean_dec(x_427); +lean_dec(x_421); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_434; +goto block_27; +} } -if (lean_is_scalar(x_446)) { - x_447 = lean_alloc_ctor(0, 2, 0); -} else { - x_447 = x_446; } -lean_ctor_set(x_447, 0, x_438); -lean_ctor_set(x_447, 1, x_445); -return x_447; } else { -lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; -lean_dec(x_438); -x_448 = lean_ctor_get(x_444, 0); +lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; +lean_dec(x_430); +lean_dec(x_427); +lean_dec(x_424); +lean_dec(x_423); +lean_dec(x_422); +lean_dec(x_421); +lean_dec(x_1); +x_447 = lean_ctor_get(x_432, 0); +lean_inc(x_447); +x_448 = lean_ctor_get(x_432, 1); lean_inc(x_448); -x_449 = lean_ctor_get(x_444, 1); -lean_inc(x_449); -if (lean_is_exclusive(x_444)) { - lean_ctor_release(x_444, 0); - lean_ctor_release(x_444, 1); - x_450 = x_444; +if (lean_is_exclusive(x_432)) { + lean_ctor_release(x_432, 0); + lean_ctor_release(x_432, 1); + x_449 = x_432; } else { - lean_dec_ref(x_444); - x_450 = lean_box(0); + lean_dec_ref(x_432); + x_449 = lean_box(0); } -if (lean_is_scalar(x_450)) { - x_451 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_449)) { + x_450 = lean_alloc_ctor(1, 2, 0); } else { - x_451 = x_450; + x_450 = x_449; } -lean_ctor_set(x_451, 0, x_448); -lean_ctor_set(x_451, 1, x_449); -return x_451; +lean_ctor_set(x_450, 0, x_447); +lean_ctor_set(x_450, 1, x_448); +return x_450; } } else { -lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; -lean_dec(x_438); +lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; +lean_dec(x_427); +lean_dec(x_424); +lean_dec(x_423); +lean_dec(x_422); +lean_dec(x_421); lean_dec(x_1); -x_452 = lean_ctor_get(x_440, 0); +x_451 = lean_ctor_get(x_429, 0); +lean_inc(x_451); +x_452 = lean_ctor_get(x_429, 1); lean_inc(x_452); -x_453 = lean_ctor_get(x_440, 1); -lean_inc(x_453); -if (lean_is_exclusive(x_440)) { - lean_ctor_release(x_440, 0); - lean_ctor_release(x_440, 1); - x_454 = x_440; +if (lean_is_exclusive(x_429)) { + lean_ctor_release(x_429, 0); + lean_ctor_release(x_429, 1); + x_453 = x_429; } else { - lean_dec_ref(x_440); - x_454 = lean_box(0); + lean_dec_ref(x_429); + x_453 = lean_box(0); } -if (lean_is_scalar(x_454)) { - x_455 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_453)) { + x_454 = lean_alloc_ctor(1, 2, 0); } else { - x_455 = x_454; + x_454 = x_453; } -lean_ctor_set(x_455, 0, x_452); -lean_ctor_set(x_455, 1, x_453); -return x_455; +lean_ctor_set(x_454, 0, x_451); +lean_ctor_set(x_454, 1, x_452); +return x_454; } } else { -lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; +lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; +lean_dec(x_424); +lean_dec(x_423); +lean_dec(x_422); +lean_dec(x_421); lean_dec(x_1); -x_456 = lean_ctor_get(x_437, 0); +x_455 = lean_ctor_get(x_426, 0); +lean_inc(x_455); +x_456 = lean_ctor_get(x_426, 1); lean_inc(x_456); -x_457 = lean_ctor_get(x_437, 1); -lean_inc(x_457); -if (lean_is_exclusive(x_437)) { - lean_ctor_release(x_437, 0); - lean_ctor_release(x_437, 1); - x_458 = x_437; +if (lean_is_exclusive(x_426)) { + lean_ctor_release(x_426, 0); + lean_ctor_release(x_426, 1); + x_457 = x_426; } else { - lean_dec_ref(x_437); - x_458 = lean_box(0); + lean_dec_ref(x_426); + x_457 = lean_box(0); } -if (lean_is_scalar(x_458)) { - x_459 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_457)) { + x_458 = lean_alloc_ctor(1, 2, 0); } else { - x_459 = x_458; + x_458 = x_457; } -lean_ctor_set(x_459, 0, x_456); -lean_ctor_set(x_459, 1, x_457); -return x_459; +lean_ctor_set(x_458, 0, x_455); +lean_ctor_set(x_458, 1, x_456); +return x_458; } } -case 6: +case 10: { -lean_object* x_460; lean_object* x_461; uint8_t x_462; lean_object* x_463; +lean_object* x_459; lean_object* x_460; lean_object* x_461; +x_459 = lean_ctor_get(x_1, 0); +lean_inc(x_459); x_460 = lean_ctor_get(x_1, 1); lean_inc(x_460); -x_461 = lean_ctor_get(x_1, 2); -lean_inc(x_461); -x_462 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_463 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_460, x_2, x_3, x_347); -if (lean_obj_tag(x_463) == 0) +lean_inc(x_460); +x_461 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_460, x_2, x_3, x_277); +if (lean_obj_tag(x_461) == 0) +{ +lean_object* x_462; lean_object* x_463; size_t x_464; size_t x_465; uint8_t x_466; +x_462 = lean_ctor_get(x_461, 0); +lean_inc(x_462); +x_463 = lean_ctor_get(x_461, 1); +lean_inc(x_463); +lean_dec(x_461); +x_464 = lean_ptr_addr(x_460); +lean_dec(x_460); +x_465 = lean_ptr_addr(x_462); +x_466 = lean_usize_dec_eq(x_464, x_465); +if (x_466 == 0) +{ +lean_object* x_467; +x_467 = l_Lean_Expr_mdata___override(x_459, x_462); +x_8 = x_467; +x_9 = x_463; +goto block_27; +} +else { -lean_object* x_464; lean_object* x_465; lean_object* x_466; -x_464 = lean_ctor_get(x_463, 0); -lean_inc(x_464); -x_465 = lean_ctor_get(x_463, 1); -lean_inc(x_465); -lean_dec(x_463); -x_466 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_461, x_2, x_3, x_465); -if (lean_obj_tag(x_466) == 0) +lean_dec(x_462); +lean_dec(x_459); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_463; +goto block_27; +} +} +else { -lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; -x_467 = lean_ctor_get(x_466, 0); -lean_inc(x_467); -x_468 = lean_ctor_get(x_466, 1); +lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; +lean_dec(x_460); +lean_dec(x_459); +lean_dec(x_1); +x_468 = lean_ctor_get(x_461, 0); lean_inc(x_468); -lean_dec(x_466); -lean_inc(x_1); -x_469 = lean_expr_update_lambda(x_1, x_462, x_464, x_467); -x_470 = lean_st_ref_take(x_2, x_468); -if (lean_obj_tag(x_470) == 0) -{ -lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; -x_471 = lean_ctor_get(x_470, 0); -lean_inc(x_471); -x_472 = lean_ctor_get(x_470, 1); -lean_inc(x_472); -lean_dec(x_470); +x_469 = lean_ctor_get(x_461, 1); lean_inc(x_469); -x_473 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_471, x_1, x_469); -x_474 = lean_st_ref_set(x_2, x_473, x_472); -if (lean_obj_tag(x_474) == 0) -{ -lean_object* x_475; lean_object* x_476; lean_object* x_477; -x_475 = lean_ctor_get(x_474, 1); -lean_inc(x_475); -if (lean_is_exclusive(x_474)) { - lean_ctor_release(x_474, 0); - lean_ctor_release(x_474, 1); - x_476 = x_474; +if (lean_is_exclusive(x_461)) { + lean_ctor_release(x_461, 0); + lean_ctor_release(x_461, 1); + x_470 = x_461; } else { - lean_dec_ref(x_474); - x_476 = lean_box(0); + lean_dec_ref(x_461); + x_470 = lean_box(0); } -if (lean_is_scalar(x_476)) { - x_477 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_470)) { + x_471 = lean_alloc_ctor(1, 2, 0); } else { - x_477 = x_476; + x_471 = x_470; } -lean_ctor_set(x_477, 0, x_469); -lean_ctor_set(x_477, 1, x_475); -return x_477; +lean_ctor_set(x_471, 0, x_468); +lean_ctor_set(x_471, 1, x_469); +return x_471; } -else -{ -lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; -lean_dec(x_469); -x_478 = lean_ctor_get(x_474, 0); -lean_inc(x_478); -x_479 = lean_ctor_get(x_474, 1); -lean_inc(x_479); -if (lean_is_exclusive(x_474)) { - lean_ctor_release(x_474, 0); - lean_ctor_release(x_474, 1); - x_480 = x_474; -} else { - lean_dec_ref(x_474); - x_480 = lean_box(0); } -if (lean_is_scalar(x_480)) { - x_481 = lean_alloc_ctor(1, 2, 0); -} else { - x_481 = x_480; +case 11: +{ +lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; +x_472 = lean_ctor_get(x_1, 0); +lean_inc(x_472); +x_473 = lean_ctor_get(x_1, 1); +lean_inc(x_473); +x_474 = lean_ctor_get(x_1, 2); +lean_inc(x_474); +lean_inc(x_474); +x_475 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_474, x_2, x_3, x_277); +if (lean_obj_tag(x_475) == 0) +{ +lean_object* x_476; lean_object* x_477; size_t x_478; size_t x_479; uint8_t x_480; +x_476 = lean_ctor_get(x_475, 0); +lean_inc(x_476); +x_477 = lean_ctor_get(x_475, 1); +lean_inc(x_477); +lean_dec(x_475); +x_478 = lean_ptr_addr(x_474); +lean_dec(x_474); +x_479 = lean_ptr_addr(x_476); +x_480 = lean_usize_dec_eq(x_478, x_479); +if (x_480 == 0) +{ +lean_object* x_481; +x_481 = l_Lean_Expr_proj___override(x_472, x_473, x_476); +x_8 = x_481; +x_9 = x_477; +goto block_27; } -lean_ctor_set(x_481, 0, x_478); -lean_ctor_set(x_481, 1, x_479); -return x_481; +else +{ +lean_dec(x_476); +lean_dec(x_473); +lean_dec(x_472); +lean_inc(x_1); +x_8 = x_1; +x_9 = x_477; +goto block_27; } } else { lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; -lean_dec(x_469); +lean_dec(x_474); +lean_dec(x_473); +lean_dec(x_472); lean_dec(x_1); -x_482 = lean_ctor_get(x_470, 0); +x_482 = lean_ctor_get(x_475, 0); lean_inc(x_482); -x_483 = lean_ctor_get(x_470, 1); +x_483 = lean_ctor_get(x_475, 1); lean_inc(x_483); -if (lean_is_exclusive(x_470)) { - lean_ctor_release(x_470, 0); - lean_ctor_release(x_470, 1); - x_484 = x_470; +if (lean_is_exclusive(x_475)) { + lean_ctor_release(x_475, 0); + lean_ctor_release(x_475, 1); + x_484 = x_475; } else { - lean_dec_ref(x_470); + lean_dec_ref(x_475); x_484 = lean_box(0); } if (lean_is_scalar(x_484)) { @@ -24468,861 +25434,171 @@ lean_ctor_set(x_485, 1, x_483); return x_485; } } -else +default: { -lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; -lean_dec(x_464); -lean_dec(x_1); -x_486 = lean_ctor_get(x_466, 0); -lean_inc(x_486); -x_487 = lean_ctor_get(x_466, 1); +lean_object* x_486; +x_486 = lean_st_ref_take(x_2, x_277); +if (lean_obj_tag(x_486) == 0) +{ +lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; +x_487 = lean_ctor_get(x_486, 0); lean_inc(x_487); -if (lean_is_exclusive(x_466)) { - lean_ctor_release(x_466, 0); - lean_ctor_release(x_466, 1); - x_488 = x_466; -} else { - lean_dec_ref(x_466); - x_488 = lean_box(0); -} -if (lean_is_scalar(x_488)) { - x_489 = lean_alloc_ctor(1, 2, 0); -} else { - x_489 = x_488; -} -lean_ctor_set(x_489, 0, x_486); -lean_ctor_set(x_489, 1, x_487); -return x_489; -} -} -else +x_488 = lean_ctor_get(x_486, 1); +lean_inc(x_488); +lean_dec(x_486); +lean_inc_n(x_1, 2); +x_489 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_487, x_1, x_1); +x_490 = lean_st_ref_set(x_2, x_489, x_488); +if (lean_obj_tag(x_490) == 0) { -lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; -lean_dec(x_461); -lean_dec(x_1); -x_490 = lean_ctor_get(x_463, 0); -lean_inc(x_490); -x_491 = lean_ctor_get(x_463, 1); +lean_object* x_491; lean_object* x_492; lean_object* x_493; +x_491 = lean_ctor_get(x_490, 1); lean_inc(x_491); -if (lean_is_exclusive(x_463)) { - lean_ctor_release(x_463, 0); - lean_ctor_release(x_463, 1); - x_492 = x_463; +if (lean_is_exclusive(x_490)) { + lean_ctor_release(x_490, 0); + lean_ctor_release(x_490, 1); + x_492 = x_490; } else { - lean_dec_ref(x_463); + lean_dec_ref(x_490); x_492 = lean_box(0); } if (lean_is_scalar(x_492)) { - x_493 = lean_alloc_ctor(1, 2, 0); + x_493 = lean_alloc_ctor(0, 2, 0); } else { x_493 = x_492; } -lean_ctor_set(x_493, 0, x_490); +lean_ctor_set(x_493, 0, x_1); lean_ctor_set(x_493, 1, x_491); return x_493; } -} -case 7: +else { -lean_object* x_494; lean_object* x_495; uint8_t x_496; lean_object* x_497; -x_494 = lean_ctor_get(x_1, 1); +lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; +lean_dec(x_1); +x_494 = lean_ctor_get(x_490, 0); lean_inc(x_494); -x_495 = lean_ctor_get(x_1, 2); +x_495 = lean_ctor_get(x_490, 1); lean_inc(x_495); -x_496 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -x_497 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_494, x_2, x_3, x_347); -if (lean_obj_tag(x_497) == 0) -{ -lean_object* x_498; lean_object* x_499; lean_object* x_500; -x_498 = lean_ctor_get(x_497, 0); -lean_inc(x_498); -x_499 = lean_ctor_get(x_497, 1); -lean_inc(x_499); -lean_dec(x_497); -x_500 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_495, x_2, x_3, x_499); -if (lean_obj_tag(x_500) == 0) -{ -lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; -x_501 = lean_ctor_get(x_500, 0); -lean_inc(x_501); -x_502 = lean_ctor_get(x_500, 1); -lean_inc(x_502); -lean_dec(x_500); -lean_inc(x_1); -x_503 = lean_expr_update_forall(x_1, x_496, x_498, x_501); -x_504 = lean_st_ref_take(x_2, x_502); -if (lean_obj_tag(x_504) == 0) -{ -lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; -x_505 = lean_ctor_get(x_504, 0); -lean_inc(x_505); -x_506 = lean_ctor_get(x_504, 1); -lean_inc(x_506); -lean_dec(x_504); -lean_inc(x_503); -x_507 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_505, x_1, x_503); -x_508 = lean_st_ref_set(x_2, x_507, x_506); -if (lean_obj_tag(x_508) == 0) -{ -lean_object* x_509; lean_object* x_510; lean_object* x_511; -x_509 = lean_ctor_get(x_508, 1); -lean_inc(x_509); -if (lean_is_exclusive(x_508)) { - lean_ctor_release(x_508, 0); - lean_ctor_release(x_508, 1); - x_510 = x_508; -} else { - lean_dec_ref(x_508); - x_510 = lean_box(0); -} -if (lean_is_scalar(x_510)) { - x_511 = lean_alloc_ctor(0, 2, 0); -} else { - x_511 = x_510; -} -lean_ctor_set(x_511, 0, x_503); -lean_ctor_set(x_511, 1, x_509); -return x_511; -} -else -{ -lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; -lean_dec(x_503); -x_512 = lean_ctor_get(x_508, 0); -lean_inc(x_512); -x_513 = lean_ctor_get(x_508, 1); -lean_inc(x_513); -if (lean_is_exclusive(x_508)) { - lean_ctor_release(x_508, 0); - lean_ctor_release(x_508, 1); - x_514 = x_508; +if (lean_is_exclusive(x_490)) { + lean_ctor_release(x_490, 0); + lean_ctor_release(x_490, 1); + x_496 = x_490; } else { - lean_dec_ref(x_508); - x_514 = lean_box(0); + lean_dec_ref(x_490); + x_496 = lean_box(0); } -if (lean_is_scalar(x_514)) { - x_515 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_496)) { + x_497 = lean_alloc_ctor(1, 2, 0); } else { - x_515 = x_514; + x_497 = x_496; } -lean_ctor_set(x_515, 0, x_512); -lean_ctor_set(x_515, 1, x_513); -return x_515; +lean_ctor_set(x_497, 0, x_494); +lean_ctor_set(x_497, 1, x_495); +return x_497; } } else { -lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; -lean_dec(x_503); +lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_dec(x_1); -x_516 = lean_ctor_get(x_504, 0); -lean_inc(x_516); -x_517 = lean_ctor_get(x_504, 1); -lean_inc(x_517); -if (lean_is_exclusive(x_504)) { - lean_ctor_release(x_504, 0); - lean_ctor_release(x_504, 1); - x_518 = x_504; +x_498 = lean_ctor_get(x_486, 0); +lean_inc(x_498); +x_499 = lean_ctor_get(x_486, 1); +lean_inc(x_499); +if (lean_is_exclusive(x_486)) { + lean_ctor_release(x_486, 0); + lean_ctor_release(x_486, 1); + x_500 = x_486; } else { - lean_dec_ref(x_504); - x_518 = lean_box(0); + lean_dec_ref(x_486); + x_500 = lean_box(0); } -if (lean_is_scalar(x_518)) { - x_519 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_500)) { + x_501 = lean_alloc_ctor(1, 2, 0); } else { - x_519 = x_518; + x_501 = x_500; +} +lean_ctor_set(x_501, 0, x_498); +lean_ctor_set(x_501, 1, x_499); +return x_501; +} } -lean_ctor_set(x_519, 0, x_516); -lean_ctor_set(x_519, 1, x_517); -return x_519; } } else { -lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; -lean_dec(x_498); +lean_object* x_502; lean_object* x_503; lean_dec(x_1); -x_520 = lean_ctor_get(x_500, 0); -lean_inc(x_520); -x_521 = lean_ctor_get(x_500, 1); -lean_inc(x_521); -if (lean_is_exclusive(x_500)) { - lean_ctor_release(x_500, 0); - lean_ctor_release(x_500, 1); - x_522 = x_500; -} else { - lean_dec_ref(x_500); - x_522 = lean_box(0); -} -if (lean_is_scalar(x_522)) { - x_523 = lean_alloc_ctor(1, 2, 0); -} else { - x_523 = x_522; +x_502 = lean_ctor_get(x_278, 0); +lean_inc(x_502); +lean_dec(x_278); +x_503 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_503, 0, x_502); +lean_ctor_set(x_503, 1, x_277); +return x_503; } -lean_ctor_set(x_523, 0, x_520); -lean_ctor_set(x_523, 1, x_521); -return x_523; } } else { -lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; -lean_dec(x_495); +uint8_t x_504; lean_dec(x_1); -x_524 = lean_ctor_get(x_497, 0); -lean_inc(x_524); -x_525 = lean_ctor_get(x_497, 1); -lean_inc(x_525); -if (lean_is_exclusive(x_497)) { - lean_ctor_release(x_497, 0); - lean_ctor_release(x_497, 1); - x_526 = x_497; -} else { - lean_dec_ref(x_497); - x_526 = lean_box(0); -} -if (lean_is_scalar(x_526)) { - x_527 = lean_alloc_ctor(1, 2, 0); -} else { - x_527 = x_526; +x_504 = !lean_is_exclusive(x_45); +if (x_504 == 0) +{ +return x_45; } -lean_ctor_set(x_527, 0, x_524); -lean_ctor_set(x_527, 1, x_525); -return x_527; +else +{ +lean_object* x_505; lean_object* x_506; lean_object* x_507; +x_505 = lean_ctor_get(x_45, 0); +x_506 = lean_ctor_get(x_45, 1); +lean_inc(x_506); +lean_inc(x_505); +lean_dec(x_45); +x_507 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_507, 0, x_505); +lean_ctor_set(x_507, 1, x_506); +return x_507; } } -case 8: +block_27: { -lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; -x_528 = lean_ctor_get(x_1, 1); -lean_inc(x_528); -x_529 = lean_ctor_get(x_1, 2); -lean_inc(x_529); -x_530 = lean_ctor_get(x_1, 3); -lean_inc(x_530); -x_531 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_528, x_2, x_3, x_347); -if (lean_obj_tag(x_531) == 0) -{ -lean_object* x_532; lean_object* x_533; lean_object* x_534; -x_532 = lean_ctor_get(x_531, 0); -lean_inc(x_532); -x_533 = lean_ctor_get(x_531, 1); -lean_inc(x_533); -lean_dec(x_531); -x_534 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_529, x_2, x_3, x_533); -if (lean_obj_tag(x_534) == 0) +lean_object* x_10; +x_10 = lean_st_ref_take(x_2, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_535; lean_object* x_536; lean_object* x_537; -x_535 = lean_ctor_get(x_534, 0); -lean_inc(x_535); -x_536 = lean_ctor_get(x_534, 1); -lean_inc(x_536); -lean_dec(x_534); -x_537 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_530, x_2, x_3, x_536); -if (lean_obj_tag(x_537) == 0) -{ -lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; -x_538 = lean_ctor_get(x_537, 0); -lean_inc(x_538); -x_539 = lean_ctor_get(x_537, 1); -lean_inc(x_539); -lean_dec(x_537); -lean_inc(x_1); -x_540 = lean_expr_update_let(x_1, x_532, x_535, x_538); -x_541 = lean_st_ref_take(x_2, x_539); -if (lean_obj_tag(x_541) == 0) -{ -lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; -x_542 = lean_ctor_get(x_541, 0); -lean_inc(x_542); -x_543 = lean_ctor_get(x_541, 1); -lean_inc(x_543); -lean_dec(x_541); -lean_inc(x_540); -x_544 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_542, x_1, x_540); -x_545 = lean_st_ref_set(x_2, x_544, x_543); -if (lean_obj_tag(x_545) == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +lean_inc(x_8); +x_13 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_11, x_1, x_8); +x_14 = lean_st_ref_set(x_2, x_13, x_12); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_546; lean_object* x_547; lean_object* x_548; -x_546 = lean_ctor_get(x_545, 1); -lean_inc(x_546); -if (lean_is_exclusive(x_545)) { - lean_ctor_release(x_545, 0); - lean_ctor_release(x_545, 1); - x_547 = x_545; -} else { - lean_dec_ref(x_545); - x_547 = lean_box(0); -} -if (lean_is_scalar(x_547)) { - x_548 = lean_alloc_ctor(0, 2, 0); -} else { - x_548 = x_547; -} -lean_ctor_set(x_548, 0, x_540); -lean_ctor_set(x_548, 1, x_546); -return x_548; +uint8_t x_15; +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_14, 0); +lean_dec(x_16); +lean_ctor_set(x_14, 0, x_8); +return x_14; } else { -lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; -lean_dec(x_540); -x_549 = lean_ctor_get(x_545, 0); -lean_inc(x_549); -x_550 = lean_ctor_get(x_545, 1); -lean_inc(x_550); -if (lean_is_exclusive(x_545)) { - lean_ctor_release(x_545, 0); - lean_ctor_release(x_545, 1); - x_551 = x_545; -} else { - lean_dec_ref(x_545); - x_551 = lean_box(0); -} -if (lean_is_scalar(x_551)) { - x_552 = lean_alloc_ctor(1, 2, 0); -} else { - x_552 = x_551; -} -lean_ctor_set(x_552, 0, x_549); -lean_ctor_set(x_552, 1, x_550); -return x_552; -} -} -else -{ -lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; -lean_dec(x_540); -lean_dec(x_1); -x_553 = lean_ctor_get(x_541, 0); -lean_inc(x_553); -x_554 = lean_ctor_get(x_541, 1); -lean_inc(x_554); -if (lean_is_exclusive(x_541)) { - lean_ctor_release(x_541, 0); - lean_ctor_release(x_541, 1); - x_555 = x_541; -} else { - lean_dec_ref(x_541); - x_555 = lean_box(0); -} -if (lean_is_scalar(x_555)) { - x_556 = lean_alloc_ctor(1, 2, 0); -} else { - x_556 = x_555; -} -lean_ctor_set(x_556, 0, x_553); -lean_ctor_set(x_556, 1, x_554); -return x_556; -} -} -else -{ -lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; -lean_dec(x_535); -lean_dec(x_532); -lean_dec(x_1); -x_557 = lean_ctor_get(x_537, 0); -lean_inc(x_557); -x_558 = lean_ctor_get(x_537, 1); -lean_inc(x_558); -if (lean_is_exclusive(x_537)) { - lean_ctor_release(x_537, 0); - lean_ctor_release(x_537, 1); - x_559 = x_537; -} else { - lean_dec_ref(x_537); - x_559 = lean_box(0); -} -if (lean_is_scalar(x_559)) { - x_560 = lean_alloc_ctor(1, 2, 0); -} else { - x_560 = x_559; -} -lean_ctor_set(x_560, 0, x_557); -lean_ctor_set(x_560, 1, x_558); -return x_560; -} -} -else -{ -lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; -lean_dec(x_532); -lean_dec(x_530); -lean_dec(x_1); -x_561 = lean_ctor_get(x_534, 0); -lean_inc(x_561); -x_562 = lean_ctor_get(x_534, 1); -lean_inc(x_562); -if (lean_is_exclusive(x_534)) { - lean_ctor_release(x_534, 0); - lean_ctor_release(x_534, 1); - x_563 = x_534; -} else { - lean_dec_ref(x_534); - x_563 = lean_box(0); -} -if (lean_is_scalar(x_563)) { - x_564 = lean_alloc_ctor(1, 2, 0); -} else { - x_564 = x_563; -} -lean_ctor_set(x_564, 0, x_561); -lean_ctor_set(x_564, 1, x_562); -return x_564; -} -} -else -{ -lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; -lean_dec(x_530); -lean_dec(x_529); -lean_dec(x_1); -x_565 = lean_ctor_get(x_531, 0); -lean_inc(x_565); -x_566 = lean_ctor_get(x_531, 1); -lean_inc(x_566); -if (lean_is_exclusive(x_531)) { - lean_ctor_release(x_531, 0); - lean_ctor_release(x_531, 1); - x_567 = x_531; -} else { - lean_dec_ref(x_531); - x_567 = lean_box(0); -} -if (lean_is_scalar(x_567)) { - x_568 = lean_alloc_ctor(1, 2, 0); -} else { - x_568 = x_567; -} -lean_ctor_set(x_568, 0, x_565); -lean_ctor_set(x_568, 1, x_566); -return x_568; -} -} -case 10: -{ -lean_object* x_569; lean_object* x_570; -x_569 = lean_ctor_get(x_1, 1); -lean_inc(x_569); -x_570 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_569, x_2, x_3, x_347); -if (lean_obj_tag(x_570) == 0) -{ -lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; -x_571 = lean_ctor_get(x_570, 0); -lean_inc(x_571); -x_572 = lean_ctor_get(x_570, 1); -lean_inc(x_572); -lean_dec(x_570); -lean_inc(x_1); -x_573 = lean_expr_update_mdata(x_1, x_571); -x_574 = lean_st_ref_take(x_2, x_572); -if (lean_obj_tag(x_574) == 0) -{ -lean_object* x_575; lean_object* x_576; lean_object* x_577; lean_object* x_578; -x_575 = lean_ctor_get(x_574, 0); -lean_inc(x_575); -x_576 = lean_ctor_get(x_574, 1); -lean_inc(x_576); -lean_dec(x_574); -lean_inc(x_573); -x_577 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_575, x_1, x_573); -x_578 = lean_st_ref_set(x_2, x_577, x_576); -if (lean_obj_tag(x_578) == 0) -{ -lean_object* x_579; lean_object* x_580; lean_object* x_581; -x_579 = lean_ctor_get(x_578, 1); -lean_inc(x_579); -if (lean_is_exclusive(x_578)) { - lean_ctor_release(x_578, 0); - lean_ctor_release(x_578, 1); - x_580 = x_578; -} else { - lean_dec_ref(x_578); - x_580 = lean_box(0); -} -if (lean_is_scalar(x_580)) { - x_581 = lean_alloc_ctor(0, 2, 0); -} else { - x_581 = x_580; -} -lean_ctor_set(x_581, 0, x_573); -lean_ctor_set(x_581, 1, x_579); -return x_581; -} -else -{ -lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; -lean_dec(x_573); -x_582 = lean_ctor_get(x_578, 0); -lean_inc(x_582); -x_583 = lean_ctor_get(x_578, 1); -lean_inc(x_583); -if (lean_is_exclusive(x_578)) { - lean_ctor_release(x_578, 0); - lean_ctor_release(x_578, 1); - x_584 = x_578; -} else { - lean_dec_ref(x_578); - x_584 = lean_box(0); -} -if (lean_is_scalar(x_584)) { - x_585 = lean_alloc_ctor(1, 2, 0); -} else { - x_585 = x_584; -} -lean_ctor_set(x_585, 0, x_582); -lean_ctor_set(x_585, 1, x_583); -return x_585; -} -} -else -{ -lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; -lean_dec(x_573); -lean_dec(x_1); -x_586 = lean_ctor_get(x_574, 0); -lean_inc(x_586); -x_587 = lean_ctor_get(x_574, 1); -lean_inc(x_587); -if (lean_is_exclusive(x_574)) { - lean_ctor_release(x_574, 0); - lean_ctor_release(x_574, 1); - x_588 = x_574; -} else { - lean_dec_ref(x_574); - x_588 = lean_box(0); -} -if (lean_is_scalar(x_588)) { - x_589 = lean_alloc_ctor(1, 2, 0); -} else { - x_589 = x_588; -} -lean_ctor_set(x_589, 0, x_586); -lean_ctor_set(x_589, 1, x_587); -return x_589; -} -} -else -{ -lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; -lean_dec(x_1); -x_590 = lean_ctor_get(x_570, 0); -lean_inc(x_590); -x_591 = lean_ctor_get(x_570, 1); -lean_inc(x_591); -if (lean_is_exclusive(x_570)) { - lean_ctor_release(x_570, 0); - lean_ctor_release(x_570, 1); - x_592 = x_570; -} else { - lean_dec_ref(x_570); - x_592 = lean_box(0); -} -if (lean_is_scalar(x_592)) { - x_593 = lean_alloc_ctor(1, 2, 0); -} else { - x_593 = x_592; -} -lean_ctor_set(x_593, 0, x_590); -lean_ctor_set(x_593, 1, x_591); -return x_593; -} -} -case 11: -{ -lean_object* x_594; lean_object* x_595; -x_594 = lean_ctor_get(x_1, 2); -lean_inc(x_594); -x_595 = l_Lean_instantiateExprMVars___at_Lean_instantiateMVarsCore___spec__2___rarg(x_594, x_2, x_3, x_347); -if (lean_obj_tag(x_595) == 0) -{ -lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; -x_596 = lean_ctor_get(x_595, 0); -lean_inc(x_596); -x_597 = lean_ctor_get(x_595, 1); -lean_inc(x_597); -lean_dec(x_595); -lean_inc(x_1); -x_598 = lean_expr_update_proj(x_1, x_596); -x_599 = lean_st_ref_take(x_2, x_597); -if (lean_obj_tag(x_599) == 0) -{ -lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; -x_600 = lean_ctor_get(x_599, 0); -lean_inc(x_600); -x_601 = lean_ctor_get(x_599, 1); -lean_inc(x_601); -lean_dec(x_599); -lean_inc(x_598); -x_602 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_600, x_1, x_598); -x_603 = lean_st_ref_set(x_2, x_602, x_601); -if (lean_obj_tag(x_603) == 0) -{ -lean_object* x_604; lean_object* x_605; lean_object* x_606; -x_604 = lean_ctor_get(x_603, 1); -lean_inc(x_604); -if (lean_is_exclusive(x_603)) { - lean_ctor_release(x_603, 0); - lean_ctor_release(x_603, 1); - x_605 = x_603; -} else { - lean_dec_ref(x_603); - x_605 = lean_box(0); -} -if (lean_is_scalar(x_605)) { - x_606 = lean_alloc_ctor(0, 2, 0); -} else { - x_606 = x_605; -} -lean_ctor_set(x_606, 0, x_598); -lean_ctor_set(x_606, 1, x_604); -return x_606; -} -else -{ -lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; -lean_dec(x_598); -x_607 = lean_ctor_get(x_603, 0); -lean_inc(x_607); -x_608 = lean_ctor_get(x_603, 1); -lean_inc(x_608); -if (lean_is_exclusive(x_603)) { - lean_ctor_release(x_603, 0); - lean_ctor_release(x_603, 1); - x_609 = x_603; -} else { - lean_dec_ref(x_603); - x_609 = lean_box(0); -} -if (lean_is_scalar(x_609)) { - x_610 = lean_alloc_ctor(1, 2, 0); -} else { - x_610 = x_609; -} -lean_ctor_set(x_610, 0, x_607); -lean_ctor_set(x_610, 1, x_608); -return x_610; -} -} -else -{ -lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; -lean_dec(x_598); -lean_dec(x_1); -x_611 = lean_ctor_get(x_599, 0); -lean_inc(x_611); -x_612 = lean_ctor_get(x_599, 1); -lean_inc(x_612); -if (lean_is_exclusive(x_599)) { - lean_ctor_release(x_599, 0); - lean_ctor_release(x_599, 1); - x_613 = x_599; -} else { - lean_dec_ref(x_599); - x_613 = lean_box(0); -} -if (lean_is_scalar(x_613)) { - x_614 = lean_alloc_ctor(1, 2, 0); -} else { - x_614 = x_613; -} -lean_ctor_set(x_614, 0, x_611); -lean_ctor_set(x_614, 1, x_612); -return x_614; -} -} -else -{ -lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; -lean_dec(x_1); -x_615 = lean_ctor_get(x_595, 0); -lean_inc(x_615); -x_616 = lean_ctor_get(x_595, 1); -lean_inc(x_616); -if (lean_is_exclusive(x_595)) { - lean_ctor_release(x_595, 0); - lean_ctor_release(x_595, 1); - x_617 = x_595; -} else { - lean_dec_ref(x_595); - x_617 = lean_box(0); -} -if (lean_is_scalar(x_617)) { - x_618 = lean_alloc_ctor(1, 2, 0); -} else { - x_618 = x_617; -} -lean_ctor_set(x_618, 0, x_615); -lean_ctor_set(x_618, 1, x_616); -return x_618; -} -} -default: -{ -lean_object* x_619; -x_619 = lean_st_ref_take(x_2, x_347); -if (lean_obj_tag(x_619) == 0) -{ -lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; -x_620 = lean_ctor_get(x_619, 0); -lean_inc(x_620); -x_621 = lean_ctor_get(x_619, 1); -lean_inc(x_621); -lean_dec(x_619); -lean_inc_n(x_1, 2); -x_622 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_620, x_1, x_1); -x_623 = lean_st_ref_set(x_2, x_622, x_621); -if (lean_obj_tag(x_623) == 0) -{ -lean_object* x_624; lean_object* x_625; lean_object* x_626; -x_624 = lean_ctor_get(x_623, 1); -lean_inc(x_624); -if (lean_is_exclusive(x_623)) { - lean_ctor_release(x_623, 0); - lean_ctor_release(x_623, 1); - x_625 = x_623; -} else { - lean_dec_ref(x_623); - x_625 = lean_box(0); -} -if (lean_is_scalar(x_625)) { - x_626 = lean_alloc_ctor(0, 2, 0); -} else { - x_626 = x_625; -} -lean_ctor_set(x_626, 0, x_1); -lean_ctor_set(x_626, 1, x_624); -return x_626; -} -else -{ -lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; -lean_dec(x_1); -x_627 = lean_ctor_get(x_623, 0); -lean_inc(x_627); -x_628 = lean_ctor_get(x_623, 1); -lean_inc(x_628); -if (lean_is_exclusive(x_623)) { - lean_ctor_release(x_623, 0); - lean_ctor_release(x_623, 1); - x_629 = x_623; -} else { - lean_dec_ref(x_623); - x_629 = lean_box(0); -} -if (lean_is_scalar(x_629)) { - x_630 = lean_alloc_ctor(1, 2, 0); -} else { - x_630 = x_629; -} -lean_ctor_set(x_630, 0, x_627); -lean_ctor_set(x_630, 1, x_628); -return x_630; -} -} -else -{ -lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; -lean_dec(x_1); -x_631 = lean_ctor_get(x_619, 0); -lean_inc(x_631); -x_632 = lean_ctor_get(x_619, 1); -lean_inc(x_632); -if (lean_is_exclusive(x_619)) { - lean_ctor_release(x_619, 0); - lean_ctor_release(x_619, 1); - x_633 = x_619; -} else { - lean_dec_ref(x_619); - x_633 = lean_box(0); -} -if (lean_is_scalar(x_633)) { - x_634 = lean_alloc_ctor(1, 2, 0); -} else { - x_634 = x_633; -} -lean_ctor_set(x_634, 0, x_631); -lean_ctor_set(x_634, 1, x_632); -return x_634; -} -} -} -} -else -{ -lean_object* x_635; lean_object* x_636; -lean_dec(x_1); -x_635 = lean_ctor_get(x_348, 0); -lean_inc(x_635); -lean_dec(x_348); -x_636 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_636, 0, x_635); -lean_ctor_set(x_636, 1, x_347); -return x_636; -} -} -} -else -{ -uint8_t x_637; -lean_dec(x_1); -x_637 = !lean_is_exclusive(x_45); -if (x_637 == 0) -{ -return x_45; -} -else -{ -lean_object* x_638; lean_object* x_639; lean_object* x_640; -x_638 = lean_ctor_get(x_45, 0); -x_639 = lean_ctor_get(x_45, 1); -lean_inc(x_639); -lean_inc(x_638); -lean_dec(x_45); -x_640 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_640, 0, x_638); -lean_ctor_set(x_640, 1, x_639); -return x_640; -} -} -block_27: -{ -lean_object* x_10; -x_10 = lean_st_ref_take(x_2, x_9); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -lean_inc(x_8); -x_13 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_11, x_1, x_8); -x_14 = lean_st_ref_set(x_2, x_13, x_12); -if (lean_obj_tag(x_14) == 0) -{ -uint8_t x_15; -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; -x_16 = lean_ctor_get(x_14, 0); -lean_dec(x_16); -lean_ctor_set(x_14, 0, x_8); -return x_14; -} -else -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_dec(x_14); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_8); -lean_ctor_set(x_18, 1, x_17); -return x_18; +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_8); +lean_ctor_set(x_18, 1, x_17); +return x_18; } } else @@ -53277,7 +53553,7 @@ static lean_object* _init_l_Lean_MetavarContext_getLevelDepth___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_isLevelMVarAssignable___rarg___lambda__1___closed__1; x_2 = l_Lean_MetavarContext_getLevelDepth___closed__1; -x_3 = lean_unsigned_to_nat(785u); +x_3 = lean_unsigned_to_nat(791u); x_4 = lean_unsigned_to_nat(14u); x_5 = l_Lean_MetavarContext_getDecl___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -54388,7 +54664,7 @@ static lean_object* _init_l___private_Lean_MetavarContext_0__Lean_MetavarContext 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_MetavarContext_0__Lean_MetavarContext_MkBinding_getLocalDeclWithSmallestIdx___closed__1; x_2 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_getLocalDeclWithSmallestIdx___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_getLocalDeclWithSmallestIdx___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -71563,7 +71839,7 @@ case 5: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Lean_Expr_getAppNumArgsAux(x_2, x_7); +x_8 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_7); x_9 = l_Lean_instantiateExprMVars___rarg___lambda__20___closed__1; lean_inc(x_8); x_10 = lean_mk_array(x_8, x_9); @@ -71575,225 +71851,235 @@ return x_13; } case 6: { -lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_2, 1); +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_14 = lean_ctor_get(x_2, 0); lean_inc(x_14); -x_15 = lean_ctor_get(x_2, 2); +x_15 = lean_ctor_get(x_2, 1); lean_inc(x_15); -x_16 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +x_16 = lean_ctor_get(x_2, 2); +lean_inc(x_16); +x_17 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); lean_inc(x_3); +lean_inc(x_15); lean_inc(x_1); -x_17 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_14, x_3, x_4); -if (lean_obj_tag(x_17) == 0) +x_18 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_15, x_3, x_4); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_17); -x_20 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_15, x_3, x_19); -if (lean_obj_tag(x_20) == 0) +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_16); +x_21 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_16, x_3, x_20); +if (lean_obj_tag(x_21) == 0) { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_expr_update_lambda(x_2, x_16, x_18, x_22); -lean_ctor_set(x_20, 0, x_23); -return x_20; +lean_object* x_23; lean_object* x_24; size_t x_25; size_t x_26; uint8_t x_27; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +x_24 = l_Lean_Expr_lam___override(x_14, x_15, x_16, x_17); +x_25 = lean_ptr_addr(x_15); +lean_dec(x_15); +x_26 = lean_ptr_addr(x_19); +x_27 = lean_usize_dec_eq(x_25, x_26); +if (x_27 == 0) +{ +lean_object* x_28; +lean_dec(x_24); +lean_dec(x_16); +x_28 = l_Lean_Expr_lam___override(x_14, x_19, x_23, x_17); +lean_ctor_set(x_21, 0, x_28); +return x_21; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_20, 0); -x_25 = lean_ctor_get(x_20, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_20); -x_26 = lean_expr_update_lambda(x_2, x_16, x_18, x_24); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_25); -return x_27; -} +size_t x_29; size_t x_30; uint8_t x_31; +x_29 = lean_ptr_addr(x_16); +lean_dec(x_16); +x_30 = lean_ptr_addr(x_23); +x_31 = lean_usize_dec_eq(x_29, x_30); +if (x_31 == 0) +{ +lean_object* x_32; +lean_dec(x_24); +x_32 = l_Lean_Expr_lam___override(x_14, x_19, x_23, x_17); +lean_ctor_set(x_21, 0, x_32); +return x_21; } else { -uint8_t x_28; -lean_dec(x_18); -lean_dec(x_2); -x_28 = !lean_is_exclusive(x_20); -if (x_28 == 0) +uint8_t x_33; +x_33 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_17, x_17); +if (x_33 == 0) { -return x_20; +lean_object* x_34; +lean_dec(x_24); +x_34 = l_Lean_Expr_lam___override(x_14, x_19, x_23, x_17); +lean_ctor_set(x_21, 0, x_34); +return x_21; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_20, 0); -x_30 = lean_ctor_get(x_20, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_20); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_dec(x_23); +lean_dec(x_19); +lean_dec(x_14); +lean_ctor_set(x_21, 0, x_24); +return x_21; +} } } } else { -uint8_t x_32; +lean_object* x_35; lean_object* x_36; lean_object* x_37; size_t x_38; size_t x_39; uint8_t x_40; +x_35 = lean_ctor_get(x_21, 0); +x_36 = lean_ctor_get(x_21, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_21); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +x_37 = l_Lean_Expr_lam___override(x_14, x_15, x_16, x_17); +x_38 = lean_ptr_addr(x_15); lean_dec(x_15); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_32 = !lean_is_exclusive(x_17); -if (x_32 == 0) +x_39 = lean_ptr_addr(x_19); +x_40 = lean_usize_dec_eq(x_38, x_39); +if (x_40 == 0) { -return x_17; +lean_object* x_41; lean_object* x_42; +lean_dec(x_37); +lean_dec(x_16); +x_41 = l_Lean_Expr_lam___override(x_14, x_19, x_35, x_17); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_36); +return x_42; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_17, 0); -x_34 = lean_ctor_get(x_17, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_17); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; -} -} -} -case 7: -{ -lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_2, 1); -lean_inc(x_36); -x_37 = lean_ctor_get(x_2, 2); -lean_inc(x_37); -x_38 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); -lean_inc(x_3); -lean_inc(x_1); -x_39 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_36, x_3, x_4); -if (lean_obj_tag(x_39) == 0) +size_t x_43; size_t x_44; uint8_t x_45; +x_43 = lean_ptr_addr(x_16); +lean_dec(x_16); +x_44 = lean_ptr_addr(x_35); +x_45 = lean_usize_dec_eq(x_43, x_44); +if (x_45 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); -lean_inc(x_41); -lean_dec(x_39); -x_42 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_37, x_3, x_41); -if (lean_obj_tag(x_42) == 0) +lean_object* x_46; lean_object* x_47; +lean_dec(x_37); +x_46 = l_Lean_Expr_lam___override(x_14, x_19, x_35, x_17); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_36); +return x_47; +} +else { -uint8_t x_43; -x_43 = !lean_is_exclusive(x_42); -if (x_43 == 0) +uint8_t x_48; +x_48 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_17, x_17); +if (x_48 == 0) { -lean_object* x_44; lean_object* x_45; -x_44 = lean_ctor_get(x_42, 0); -x_45 = lean_expr_update_forall(x_2, x_38, x_40, x_44); -lean_ctor_set(x_42, 0, x_45); -return x_42; +lean_object* x_49; lean_object* x_50; +lean_dec(x_37); +x_49 = l_Lean_Expr_lam___override(x_14, x_19, x_35, x_17); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_36); +return x_50; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_46 = lean_ctor_get(x_42, 0); -x_47 = lean_ctor_get(x_42, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_42); -x_48 = lean_expr_update_forall(x_2, x_38, x_40, x_46); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_47); -return x_49; +lean_object* x_51; +lean_dec(x_35); +lean_dec(x_19); +lean_dec(x_14); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_37); +lean_ctor_set(x_51, 1, x_36); +return x_51; +} +} +} } } else { -uint8_t x_50; -lean_dec(x_40); -lean_dec(x_2); -x_50 = !lean_is_exclusive(x_42); -if (x_50 == 0) +uint8_t x_52; +lean_dec(x_19); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +x_52 = !lean_is_exclusive(x_21); +if (x_52 == 0) { -return x_42; +return x_21; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_42, 0); -x_52 = lean_ctor_get(x_42, 1); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_42); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_51); -lean_ctor_set(x_53, 1, x_52); -return x_53; +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_21, 0); +x_54 = lean_ctor_get(x_21, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_21); +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_54; -lean_dec(x_37); +uint8_t x_56; +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_54 = !lean_is_exclusive(x_39); -if (x_54 == 0) +x_56 = !lean_is_exclusive(x_18); +if (x_56 == 0) { -return x_39; +return x_18; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_39, 0); -x_56 = lean_ctor_get(x_39, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_39); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -return x_57; +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_18, 0); +x_58 = lean_ctor_get(x_18, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_18); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } -case 8: +case 7: { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_58 = lean_ctor_get(x_2, 1); -lean_inc(x_58); -x_59 = lean_ctor_get(x_2, 2); -lean_inc(x_59); -x_60 = lean_ctor_get(x_2, 3); +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; lean_object* x_64; +x_60 = lean_ctor_get(x_2, 0); lean_inc(x_60); -lean_inc(x_3); -lean_inc(x_1); -x_61 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_58, x_3, x_4); -if (lean_obj_tag(x_61) == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_61, 0); +x_61 = lean_ctor_get(x_2, 1); +lean_inc(x_61); +x_62 = lean_ctor_get(x_2, 2); lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); +x_63 = lean_ctor_get_uint8(x_2, sizeof(void*)*3 + 8); +lean_dec(x_2); lean_inc(x_3); +lean_inc(x_61); lean_inc(x_1); -x_64 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_59, x_3, x_63); +x_64 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_61, x_3, x_4); if (lean_obj_tag(x_64) == 0) { lean_object* x_65; lean_object* x_66; lean_object* x_67; @@ -71802,239 +72088,676 @@ lean_inc(x_65); x_66 = lean_ctor_get(x_64, 1); lean_inc(x_66); lean_dec(x_64); -x_67 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_60, x_3, x_66); +lean_inc(x_62); +x_67 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_62, x_3, x_66); if (lean_obj_tag(x_67) == 0) { uint8_t x_68; x_68 = !lean_is_exclusive(x_67); if (x_68 == 0) { -lean_object* x_69; lean_object* x_70; +lean_object* x_69; lean_object* x_70; size_t x_71; size_t x_72; uint8_t x_73; x_69 = lean_ctor_get(x_67, 0); -x_70 = lean_expr_update_let(x_2, x_62, x_65, x_69); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +x_70 = l_Lean_Expr_forallE___override(x_60, x_61, x_62, x_63); +x_71 = lean_ptr_addr(x_61); +lean_dec(x_61); +x_72 = lean_ptr_addr(x_65); +x_73 = lean_usize_dec_eq(x_71, x_72); +if (x_73 == 0) +{ +lean_object* x_74; +lean_dec(x_70); +lean_dec(x_62); +x_74 = l_Lean_Expr_forallE___override(x_60, x_65, x_69, x_63); +lean_ctor_set(x_67, 0, x_74); +return x_67; +} +else +{ +size_t x_75; size_t x_76; uint8_t x_77; +x_75 = lean_ptr_addr(x_62); +lean_dec(x_62); +x_76 = lean_ptr_addr(x_69); +x_77 = lean_usize_dec_eq(x_75, x_76); +if (x_77 == 0) +{ +lean_object* x_78; +lean_dec(x_70); +x_78 = l_Lean_Expr_forallE___override(x_60, x_65, x_69, x_63); +lean_ctor_set(x_67, 0, x_78); +return x_67; +} +else +{ +uint8_t x_79; +x_79 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_63, x_63); +if (x_79 == 0) +{ +lean_object* x_80; +lean_dec(x_70); +x_80 = l_Lean_Expr_forallE___override(x_60, x_65, x_69, x_63); +lean_ctor_set(x_67, 0, x_80); +return x_67; +} +else +{ +lean_dec(x_69); +lean_dec(x_65); +lean_dec(x_60); lean_ctor_set(x_67, 0, x_70); return x_67; } +} +} +} else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_71 = lean_ctor_get(x_67, 0); -x_72 = lean_ctor_get(x_67, 1); -lean_inc(x_72); -lean_inc(x_71); +lean_object* x_81; lean_object* x_82; lean_object* x_83; size_t x_84; size_t x_85; uint8_t x_86; +x_81 = lean_ctor_get(x_67, 0); +x_82 = lean_ctor_get(x_67, 1); +lean_inc(x_82); +lean_inc(x_81); lean_dec(x_67); -x_73 = lean_expr_update_let(x_2, x_62, x_65, x_71); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_72); -return x_74; +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +x_83 = l_Lean_Expr_forallE___override(x_60, x_61, x_62, x_63); +x_84 = lean_ptr_addr(x_61); +lean_dec(x_61); +x_85 = lean_ptr_addr(x_65); +x_86 = lean_usize_dec_eq(x_84, x_85); +if (x_86 == 0) +{ +lean_object* x_87; lean_object* x_88; +lean_dec(x_83); +lean_dec(x_62); +x_87 = l_Lean_Expr_forallE___override(x_60, x_65, x_81, x_63); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_87); +lean_ctor_set(x_88, 1, x_82); +return x_88; } +else +{ +size_t x_89; size_t x_90; uint8_t x_91; +x_89 = lean_ptr_addr(x_62); +lean_dec(x_62); +x_90 = lean_ptr_addr(x_81); +x_91 = lean_usize_dec_eq(x_89, x_90); +if (x_91 == 0) +{ +lean_object* x_92; lean_object* x_93; +lean_dec(x_83); +x_92 = l_Lean_Expr_forallE___override(x_60, x_65, x_81, x_63); +x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_82); +return x_93; } else { -uint8_t x_75; +uint8_t x_94; +x_94 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_63, x_63); +if (x_94 == 0) +{ +lean_object* x_95; lean_object* x_96; +lean_dec(x_83); +x_95 = l_Lean_Expr_forallE___override(x_60, x_65, x_81, x_63); +x_96 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_95); +lean_ctor_set(x_96, 1, x_82); +return x_96; +} +else +{ +lean_object* x_97; +lean_dec(x_81); +lean_dec(x_65); +lean_dec(x_60); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_83); +lean_ctor_set(x_97, 1, x_82); +return x_97; +} +} +} +} +} +else +{ +uint8_t x_98; lean_dec(x_65); lean_dec(x_62); -lean_dec(x_2); -x_75 = !lean_is_exclusive(x_67); -if (x_75 == 0) +lean_dec(x_61); +lean_dec(x_60); +x_98 = !lean_is_exclusive(x_67); +if (x_98 == 0) { return x_67; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_67, 0); -x_77 = lean_ctor_get(x_67, 1); -lean_inc(x_77); -lean_inc(x_76); +lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_99 = lean_ctor_get(x_67, 0); +x_100 = lean_ctor_get(x_67, 1); +lean_inc(x_100); +lean_inc(x_99); lean_dec(x_67); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +x_101 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_101, 0, x_99); +lean_ctor_set(x_101, 1, x_100); +return x_101; } } } else { -uint8_t x_79; +uint8_t x_102; lean_dec(x_62); +lean_dec(x_61); lean_dec(x_60); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_79 = !lean_is_exclusive(x_64); -if (x_79 == 0) +x_102 = !lean_is_exclusive(x_64); +if (x_102 == 0) { return x_64; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_80 = lean_ctor_get(x_64, 0); -x_81 = lean_ctor_get(x_64, 1); -lean_inc(x_81); -lean_inc(x_80); +lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_103 = lean_ctor_get(x_64, 0); +x_104 = lean_ctor_get(x_64, 1); +lean_inc(x_104); +lean_inc(x_103); lean_dec(x_64); -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -return x_82; +x_105 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_105, 0, x_103); +lean_ctor_set(x_105, 1, x_104); +return x_105; +} +} +} +case 8: +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; lean_object* x_111; +x_106 = lean_ctor_get(x_2, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_2, 1); +lean_inc(x_107); +x_108 = lean_ctor_get(x_2, 2); +lean_inc(x_108); +x_109 = lean_ctor_get(x_2, 3); +lean_inc(x_109); +x_110 = lean_ctor_get_uint8(x_2, sizeof(void*)*4 + 8); +lean_inc(x_3); +lean_inc(x_107); +lean_inc(x_1); +x_111 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_107, x_3, x_4); +if (lean_obj_tag(x_111) == 0) +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_111, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_111, 1); +lean_inc(x_113); +lean_dec(x_111); +lean_inc(x_3); +lean_inc(x_108); +lean_inc(x_1); +x_114 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_108, x_3, x_113); +if (lean_obj_tag(x_114) == 0) +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_114, 0); +lean_inc(x_115); +x_116 = lean_ctor_get(x_114, 1); +lean_inc(x_116); +lean_dec(x_114); +lean_inc(x_109); +x_117 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_109, x_3, x_116); +if (lean_obj_tag(x_117) == 0) +{ +uint8_t x_118; +x_118 = !lean_is_exclusive(x_117); +if (x_118 == 0) +{ +lean_object* x_119; size_t x_120; size_t x_121; uint8_t x_122; +x_119 = lean_ctor_get(x_117, 0); +x_120 = lean_ptr_addr(x_107); +lean_dec(x_107); +x_121 = lean_ptr_addr(x_112); +x_122 = lean_usize_dec_eq(x_120, x_121); +if (x_122 == 0) +{ +lean_object* x_123; +lean_dec(x_109); +lean_dec(x_108); +lean_dec(x_2); +x_123 = l_Lean_Expr_letE___override(x_106, x_112, x_115, x_119, x_110); +lean_ctor_set(x_117, 0, x_123); +return x_117; +} +else +{ +size_t x_124; size_t x_125; uint8_t x_126; +x_124 = lean_ptr_addr(x_108); +lean_dec(x_108); +x_125 = lean_ptr_addr(x_115); +x_126 = lean_usize_dec_eq(x_124, x_125); +if (x_126 == 0) +{ +lean_object* x_127; +lean_dec(x_109); +lean_dec(x_2); +x_127 = l_Lean_Expr_letE___override(x_106, x_112, x_115, x_119, x_110); +lean_ctor_set(x_117, 0, x_127); +return x_117; +} +else +{ +size_t x_128; size_t x_129; uint8_t x_130; +x_128 = lean_ptr_addr(x_109); +lean_dec(x_109); +x_129 = lean_ptr_addr(x_119); +x_130 = lean_usize_dec_eq(x_128, x_129); +if (x_130 == 0) +{ +lean_object* x_131; +lean_dec(x_2); +x_131 = l_Lean_Expr_letE___override(x_106, x_112, x_115, x_119, x_110); +lean_ctor_set(x_117, 0, x_131); +return x_117; +} +else +{ +lean_dec(x_119); +lean_dec(x_115); +lean_dec(x_112); +lean_dec(x_106); +lean_ctor_set(x_117, 0, x_2); +return x_117; +} } } } else { -uint8_t x_83; -lean_dec(x_60); -lean_dec(x_59); +lean_object* x_132; lean_object* x_133; size_t x_134; size_t x_135; uint8_t x_136; +x_132 = lean_ctor_get(x_117, 0); +x_133 = lean_ctor_get(x_117, 1); +lean_inc(x_133); +lean_inc(x_132); +lean_dec(x_117); +x_134 = lean_ptr_addr(x_107); +lean_dec(x_107); +x_135 = lean_ptr_addr(x_112); +x_136 = lean_usize_dec_eq(x_134, x_135); +if (x_136 == 0) +{ +lean_object* x_137; lean_object* x_138; +lean_dec(x_109); +lean_dec(x_108); +lean_dec(x_2); +x_137 = l_Lean_Expr_letE___override(x_106, x_112, x_115, x_132, x_110); +x_138 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_138, 0, x_137); +lean_ctor_set(x_138, 1, x_133); +return x_138; +} +else +{ +size_t x_139; size_t x_140; uint8_t x_141; +x_139 = lean_ptr_addr(x_108); +lean_dec(x_108); +x_140 = lean_ptr_addr(x_115); +x_141 = lean_usize_dec_eq(x_139, x_140); +if (x_141 == 0) +{ +lean_object* x_142; lean_object* x_143; +lean_dec(x_109); +lean_dec(x_2); +x_142 = l_Lean_Expr_letE___override(x_106, x_112, x_115, x_132, x_110); +x_143 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_143, 0, x_142); +lean_ctor_set(x_143, 1, x_133); +return x_143; +} +else +{ +size_t x_144; size_t x_145; uint8_t x_146; +x_144 = lean_ptr_addr(x_109); +lean_dec(x_109); +x_145 = lean_ptr_addr(x_132); +x_146 = lean_usize_dec_eq(x_144, x_145); +if (x_146 == 0) +{ +lean_object* x_147; lean_object* x_148; +lean_dec(x_2); +x_147 = l_Lean_Expr_letE___override(x_106, x_112, x_115, x_132, x_110); +x_148 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_148, 0, x_147); +lean_ctor_set(x_148, 1, x_133); +return x_148; +} +else +{ +lean_object* x_149; +lean_dec(x_132); +lean_dec(x_115); +lean_dec(x_112); +lean_dec(x_106); +x_149 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_149, 0, x_2); +lean_ctor_set(x_149, 1, x_133); +return x_149; +} +} +} +} +} +else +{ +uint8_t x_150; +lean_dec(x_115); +lean_dec(x_112); +lean_dec(x_109); +lean_dec(x_108); +lean_dec(x_107); +lean_dec(x_106); +lean_dec(x_2); +x_150 = !lean_is_exclusive(x_117); +if (x_150 == 0) +{ +return x_117; +} +else +{ +lean_object* x_151; lean_object* x_152; lean_object* x_153; +x_151 = lean_ctor_get(x_117, 0); +x_152 = lean_ctor_get(x_117, 1); +lean_inc(x_152); +lean_inc(x_151); +lean_dec(x_117); +x_153 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_153, 0, x_151); +lean_ctor_set(x_153, 1, x_152); +return x_153; +} +} +} +else +{ +uint8_t x_154; +lean_dec(x_112); +lean_dec(x_109); +lean_dec(x_108); +lean_dec(x_107); +lean_dec(x_106); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_83 = !lean_is_exclusive(x_61); -if (x_83 == 0) +x_154 = !lean_is_exclusive(x_114); +if (x_154 == 0) { -return x_61; +return x_114; } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_84 = lean_ctor_get(x_61, 0); -x_85 = lean_ctor_get(x_61, 1); -lean_inc(x_85); -lean_inc(x_84); -lean_dec(x_61); -x_86 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_86, 0, x_84); -lean_ctor_set(x_86, 1, x_85); -return x_86; +lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_155 = lean_ctor_get(x_114, 0); +x_156 = lean_ctor_get(x_114, 1); +lean_inc(x_156); +lean_inc(x_155); +lean_dec(x_114); +x_157 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_157, 0, x_155); +lean_ctor_set(x_157, 1, x_156); +return x_157; +} +} +} +else +{ +uint8_t x_158; +lean_dec(x_109); +lean_dec(x_108); +lean_dec(x_107); +lean_dec(x_106); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_158 = !lean_is_exclusive(x_111); +if (x_158 == 0) +{ +return x_111; +} +else +{ +lean_object* x_159; lean_object* x_160; lean_object* x_161; +x_159 = lean_ctor_get(x_111, 0); +x_160 = lean_ctor_get(x_111, 1); +lean_inc(x_160); +lean_inc(x_159); +lean_dec(x_111); +x_161 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_161, 0, x_159); +lean_ctor_set(x_161, 1, x_160); +return x_161; } } } case 10: { -lean_object* x_87; lean_object* x_88; -x_87 = lean_ctor_get(x_2, 1); -lean_inc(x_87); -x_88 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_87, x_3, x_4); -if (lean_obj_tag(x_88) == 0) +lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_162 = lean_ctor_get(x_2, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_2, 1); +lean_inc(x_163); +lean_inc(x_163); +x_164 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_163, x_3, x_4); +if (lean_obj_tag(x_164) == 0) { -uint8_t x_89; -x_89 = !lean_is_exclusive(x_88); -if (x_89 == 0) +uint8_t x_165; +x_165 = !lean_is_exclusive(x_164); +if (x_165 == 0) { -lean_object* x_90; lean_object* x_91; -x_90 = lean_ctor_get(x_88, 0); -x_91 = lean_expr_update_mdata(x_2, x_90); -lean_ctor_set(x_88, 0, x_91); -return x_88; +lean_object* x_166; size_t x_167; size_t x_168; uint8_t x_169; +x_166 = lean_ctor_get(x_164, 0); +x_167 = lean_ptr_addr(x_163); +lean_dec(x_163); +x_168 = lean_ptr_addr(x_166); +x_169 = lean_usize_dec_eq(x_167, x_168); +if (x_169 == 0) +{ +lean_object* x_170; +lean_dec(x_2); +x_170 = l_Lean_Expr_mdata___override(x_162, x_166); +lean_ctor_set(x_164, 0, x_170); +return x_164; } else { -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_92 = lean_ctor_get(x_88, 0); -x_93 = lean_ctor_get(x_88, 1); -lean_inc(x_93); -lean_inc(x_92); -lean_dec(x_88); -x_94 = lean_expr_update_mdata(x_2, x_92); -x_95 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_93); -return x_95; +lean_dec(x_166); +lean_dec(x_162); +lean_ctor_set(x_164, 0, x_2); +return x_164; } } else { -uint8_t x_96; +lean_object* x_171; lean_object* x_172; size_t x_173; size_t x_174; uint8_t x_175; +x_171 = lean_ctor_get(x_164, 0); +x_172 = lean_ctor_get(x_164, 1); +lean_inc(x_172); +lean_inc(x_171); +lean_dec(x_164); +x_173 = lean_ptr_addr(x_163); +lean_dec(x_163); +x_174 = lean_ptr_addr(x_171); +x_175 = lean_usize_dec_eq(x_173, x_174); +if (x_175 == 0) +{ +lean_object* x_176; lean_object* x_177; lean_dec(x_2); -x_96 = !lean_is_exclusive(x_88); -if (x_96 == 0) +x_176 = l_Lean_Expr_mdata___override(x_162, x_171); +x_177 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_177, 0, x_176); +lean_ctor_set(x_177, 1, x_172); +return x_177; +} +else { -return x_88; +lean_object* x_178; +lean_dec(x_171); +lean_dec(x_162); +x_178 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_178, 0, x_2); +lean_ctor_set(x_178, 1, x_172); +return x_178; +} +} } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_88, 0); -x_98 = lean_ctor_get(x_88, 1); -lean_inc(x_98); -lean_inc(x_97); -lean_dec(x_88); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -return x_99; +uint8_t x_179; +lean_dec(x_163); +lean_dec(x_162); +lean_dec(x_2); +x_179 = !lean_is_exclusive(x_164); +if (x_179 == 0) +{ +return x_164; +} +else +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_180 = lean_ctor_get(x_164, 0); +x_181 = lean_ctor_get(x_164, 1); +lean_inc(x_181); +lean_inc(x_180); +lean_dec(x_164); +x_182 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_182, 0, x_180); +lean_ctor_set(x_182, 1, x_181); +return x_182; } } } case 11: { -lean_object* x_100; lean_object* x_101; -x_100 = lean_ctor_get(x_2, 2); -lean_inc(x_100); -x_101 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_100, x_3, x_4); -if (lean_obj_tag(x_101) == 0) +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; +x_183 = lean_ctor_get(x_2, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_2, 1); +lean_inc(x_184); +x_185 = lean_ctor_get(x_2, 2); +lean_inc(x_185); +lean_inc(x_185); +x_186 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_visit(x_1, x_185, x_3, x_4); +if (lean_obj_tag(x_186) == 0) { -uint8_t x_102; -x_102 = !lean_is_exclusive(x_101); -if (x_102 == 0) +uint8_t x_187; +x_187 = !lean_is_exclusive(x_186); +if (x_187 == 0) { -lean_object* x_103; lean_object* x_104; -x_103 = lean_ctor_get(x_101, 0); -x_104 = lean_expr_update_proj(x_2, x_103); -lean_ctor_set(x_101, 0, x_104); -return x_101; +lean_object* x_188; size_t x_189; size_t x_190; uint8_t x_191; +x_188 = lean_ctor_get(x_186, 0); +x_189 = lean_ptr_addr(x_185); +lean_dec(x_185); +x_190 = lean_ptr_addr(x_188); +x_191 = lean_usize_dec_eq(x_189, x_190); +if (x_191 == 0) +{ +lean_object* x_192; +lean_dec(x_2); +x_192 = l_Lean_Expr_proj___override(x_183, x_184, x_188); +lean_ctor_set(x_186, 0, x_192); +return x_186; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_105 = lean_ctor_get(x_101, 0); -x_106 = lean_ctor_get(x_101, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_101); -x_107 = lean_expr_update_proj(x_2, x_105); -x_108 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_108, 0, x_107); -lean_ctor_set(x_108, 1, x_106); -return x_108; +lean_dec(x_188); +lean_dec(x_184); +lean_dec(x_183); +lean_ctor_set(x_186, 0, x_2); +return x_186; } } else { -uint8_t x_109; +lean_object* x_193; lean_object* x_194; size_t x_195; size_t x_196; uint8_t x_197; +x_193 = lean_ctor_get(x_186, 0); +x_194 = lean_ctor_get(x_186, 1); +lean_inc(x_194); +lean_inc(x_193); +lean_dec(x_186); +x_195 = lean_ptr_addr(x_185); +lean_dec(x_185); +x_196 = lean_ptr_addr(x_193); +x_197 = lean_usize_dec_eq(x_195, x_196); +if (x_197 == 0) +{ +lean_object* x_198; lean_object* x_199; lean_dec(x_2); -x_109 = !lean_is_exclusive(x_101); -if (x_109 == 0) +x_198 = l_Lean_Expr_proj___override(x_183, x_184, x_193); +x_199 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_199, 0, x_198); +lean_ctor_set(x_199, 1, x_194); +return x_199; +} +else { -return x_101; +lean_object* x_200; +lean_dec(x_193); +lean_dec(x_184); +lean_dec(x_183); +x_200 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_200, 0, x_2); +lean_ctor_set(x_200, 1, x_194); +return x_200; +} +} } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = lean_ctor_get(x_101, 0); -x_111 = lean_ctor_get(x_101, 1); -lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_101); -x_112 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_112, 0, x_110); -lean_ctor_set(x_112, 1, x_111); -return x_112; +uint8_t x_201; +lean_dec(x_185); +lean_dec(x_184); +lean_dec(x_183); +lean_dec(x_2); +x_201 = !lean_is_exclusive(x_186); +if (x_201 == 0) +{ +return x_186; +} +else +{ +lean_object* x_202; lean_object* x_203; lean_object* x_204; +x_202 = lean_ctor_get(x_186, 0); +x_203 = lean_ctor_get(x_186, 1); +lean_inc(x_203); +lean_inc(x_202); +lean_dec(x_186); +x_204 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_204, 0, x_202); +lean_ctor_set(x_204, 1, x_203); +return x_204; } } } default: { -lean_object* x_113; +lean_object* x_205; lean_dec(x_3); lean_dec(x_1); -x_113 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_113, 0, x_2); -lean_ctor_set(x_113, 1, x_4); -return x_113; +x_205 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_205, 0, x_2); +lean_ctor_set(x_205, 1, x_4); +return x_205; } } } @@ -75308,7 +76031,7 @@ x_43 = l_Lean_Expr_mvar___override(x_42); x_44 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_mkMVarApp(x_8, x_43, x_20, x_16); x_45 = lean_ctor_get(x_7, 5); lean_inc(x_45); -x_46 = l_Lean_Expr_getAppNumArgsAux(x_44, x_11); +x_46 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_44, x_11); x_47 = lean_nat_add(x_45, x_46); lean_dec(x_46); lean_dec(x_45); @@ -75409,7 +76132,7 @@ x_74 = l_Lean_Expr_mvar___override(x_73); x_75 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_mkMVarApp(x_8, x_74, x_20, x_16); x_76 = lean_ctor_get(x_7, 5); lean_inc(x_76); -x_77 = l_Lean_Expr_getAppNumArgsAux(x_75, x_11); +x_77 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_75, x_11); x_78 = lean_nat_add(x_76, x_77); lean_dec(x_77); lean_dec(x_76); @@ -75526,7 +76249,7 @@ x_109 = l_Lean_Expr_mvar___override(x_108); x_110 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_mkMVarApp(x_8, x_109, x_20, x_16); x_111 = lean_ctor_get(x_7, 5); lean_inc(x_111); -x_112 = l_Lean_Expr_getAppNumArgsAux(x_110, x_11); +x_112 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_110, x_11); x_113 = lean_nat_add(x_111, x_112); lean_dec(x_112); lean_dec(x_111); @@ -75757,7 +76480,7 @@ x_169 = l_Lean_Expr_mvar___override(x_168); x_170 = l___private_Lean_MetavarContext_0__Lean_MetavarContext_MkBinding_mkMVarApp(x_8, x_169, x_20, x_16); x_171 = lean_ctor_get(x_7, 5); lean_inc(x_171); -x_172 = l_Lean_Expr_getAppNumArgsAux(x_170, x_11); +x_172 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_170, x_11); x_173 = lean_nat_add(x_171, x_172); lean_dec(x_172); lean_dec(x_171); @@ -80010,202 +80733,388 @@ case 1: lean_object* x_4; lean_object* x_5; uint8_t x_6; x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); +lean_inc(x_4); x_5 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_4, x_2, x_3); x_6 = !lean_is_exclusive(x_5); if (x_6 == 0) { -lean_object* x_7; lean_object* x_8; +lean_object* x_7; size_t x_8; size_t x_9; uint8_t x_10; x_7 = lean_ctor_get(x_5, 0); -x_8 = lean_level_update_succ(x_1, x_7); -lean_ctor_set(x_5, 0, x_8); +x_8 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_9 = lean_ptr_addr(x_7); +x_10 = lean_usize_dec_eq(x_8, x_9); +if (x_10 == 0) +{ +lean_object* x_11; +lean_dec(x_1); +x_11 = l_Lean_Level_succ___override(x_7); +lean_ctor_set(x_5, 0, x_11); return x_5; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_5, 0); -x_10 = lean_ctor_get(x_5, 1); -lean_inc(x_10); -lean_inc(x_9); -lean_dec(x_5); -x_11 = lean_level_update_succ(x_1, x_9); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -return x_12; +lean_dec(x_7); +lean_ctor_set(x_5, 0, x_1); +return x_5; } } -case 2: +else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_13 = lean_ctor_get(x_1, 0); +lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; uint8_t x_16; +x_12 = lean_ctor_get(x_5, 0); +x_13 = lean_ctor_get(x_5, 1); lean_inc(x_13); -x_14 = lean_ctor_get(x_1, 1); -lean_inc(x_14); -lean_inc(x_2); -x_15 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_13, x_2, x_3); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_14, x_2, x_17); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_inc(x_12); +lean_dec(x_5); +x_14 = lean_ptr_addr(x_4); +lean_dec(x_4); +x_15 = lean_ptr_addr(x_12); +x_16 = lean_usize_dec_eq(x_14, x_15); +if (x_16 == 0) { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_18, 0); -x_21 = lean_level_update_max(x_1, x_16, x_20); -lean_ctor_set(x_18, 0, x_21); +lean_object* x_17; lean_object* x_18; +lean_dec(x_1); +x_17 = l_Lean_Level_succ___override(x_12); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_13); return x_18; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_18, 0); -x_23 = lean_ctor_get(x_18, 1); +lean_object* x_19; +lean_dec(x_12); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 1, x_13); +return x_19; +} +} +} +case 2: +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_2); +lean_inc(x_20); +x_22 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_20, x_2, x_3); +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_18); -x_24 = lean_level_update_max(x_1, x_16, x_22); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +lean_inc(x_21); +x_25 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_21, x_2, x_24); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) +{ +lean_object* x_27; size_t x_28; size_t x_29; uint8_t x_30; +x_27 = lean_ctor_get(x_25, 0); +x_28 = lean_ptr_addr(x_20); +lean_dec(x_20); +x_29 = lean_ptr_addr(x_23); +x_30 = lean_usize_dec_eq(x_28, x_29); +if (x_30 == 0) +{ +lean_object* x_31; +lean_dec(x_21); +lean_dec(x_1); +x_31 = l_Lean_mkLevelMax_x27(x_23, x_27); +lean_ctor_set(x_25, 0, x_31); return x_25; } +else +{ +size_t x_32; size_t x_33; uint8_t x_34; +x_32 = lean_ptr_addr(x_21); +lean_dec(x_21); +x_33 = lean_ptr_addr(x_27); +x_34 = lean_usize_dec_eq(x_32, x_33); +if (x_34 == 0) +{ +lean_object* x_35; +lean_dec(x_1); +x_35 = l_Lean_mkLevelMax_x27(x_23, x_27); +lean_ctor_set(x_25, 0, x_35); +return x_25; +} +else +{ +lean_object* x_36; +x_36 = l_Lean_simpLevelMax_x27(x_23, x_27, x_1); +lean_dec(x_1); +lean_dec(x_27); +lean_dec(x_23); +lean_ctor_set(x_25, 0, x_36); +return x_25; +} +} +} +else +{ +lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; uint8_t x_41; +x_37 = lean_ctor_get(x_25, 0); +x_38 = lean_ctor_get(x_25, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_25); +x_39 = lean_ptr_addr(x_20); +lean_dec(x_20); +x_40 = lean_ptr_addr(x_23); +x_41 = lean_usize_dec_eq(x_39, x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +lean_dec(x_21); +lean_dec(x_1); +x_42 = l_Lean_mkLevelMax_x27(x_23, x_37); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_38); +return x_43; +} +else +{ +size_t x_44; size_t x_45; uint8_t x_46; +x_44 = lean_ptr_addr(x_21); +lean_dec(x_21); +x_45 = lean_ptr_addr(x_37); +x_46 = lean_usize_dec_eq(x_44, x_45); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; +lean_dec(x_1); +x_47 = l_Lean_mkLevelMax_x27(x_23, x_37); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_38); +return x_48; +} +else +{ +lean_object* x_49; lean_object* x_50; +x_49 = l_Lean_simpLevelMax_x27(x_23, x_37, x_1); +lean_dec(x_1); +lean_dec(x_37); +lean_dec(x_23); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_38); +return x_50; +} +} +} } case 3: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_26 = lean_ctor_get(x_1, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_1, 1); -lean_inc(x_27); +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; +x_51 = lean_ctor_get(x_1, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_1, 1); +lean_inc(x_52); lean_inc(x_2); -x_28 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_26, x_2, x_3); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_27, x_2, x_30); -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) +lean_inc(x_51); +x_53 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_51, x_2, x_3); +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +lean_dec(x_53); +lean_inc(x_52); +x_56 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_52, x_2, x_55); +x_57 = !lean_is_exclusive(x_56); +if (x_57 == 0) { -lean_object* x_33; lean_object* x_34; -x_33 = lean_ctor_get(x_31, 0); -x_34 = lean_level_update_imax(x_1, x_29, x_33); -lean_ctor_set(x_31, 0, x_34); -return x_31; +lean_object* x_58; size_t x_59; size_t x_60; uint8_t x_61; +x_58 = lean_ctor_get(x_56, 0); +x_59 = lean_ptr_addr(x_51); +lean_dec(x_51); +x_60 = lean_ptr_addr(x_54); +x_61 = lean_usize_dec_eq(x_59, x_60); +if (x_61 == 0) +{ +lean_object* x_62; +lean_dec(x_52); +lean_dec(x_1); +x_62 = l_Lean_mkLevelIMax_x27(x_54, x_58); +lean_ctor_set(x_56, 0, x_62); +return x_56; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_35 = lean_ctor_get(x_31, 0); -x_36 = lean_ctor_get(x_31, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_31); -x_37 = lean_level_update_imax(x_1, x_29, x_35); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_36); -return x_38; +size_t x_63; size_t x_64; uint8_t x_65; +x_63 = lean_ptr_addr(x_52); +lean_dec(x_52); +x_64 = lean_ptr_addr(x_58); +x_65 = lean_usize_dec_eq(x_63, x_64); +if (x_65 == 0) +{ +lean_object* x_66; +lean_dec(x_1); +x_66 = l_Lean_mkLevelIMax_x27(x_54, x_58); +lean_ctor_set(x_56, 0, x_66); +return x_56; +} +else +{ +lean_object* x_67; +x_67 = l_Lean_simpLevelIMax_x27(x_54, x_58, x_1); +lean_dec(x_1); +lean_ctor_set(x_56, 0, x_67); +return x_56; +} +} +} +else +{ +lean_object* x_68; lean_object* x_69; size_t x_70; size_t x_71; uint8_t x_72; +x_68 = lean_ctor_get(x_56, 0); +x_69 = lean_ctor_get(x_56, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_56); +x_70 = lean_ptr_addr(x_51); +lean_dec(x_51); +x_71 = lean_ptr_addr(x_54); +x_72 = lean_usize_dec_eq(x_70, x_71); +if (x_72 == 0) +{ +lean_object* x_73; lean_object* x_74; +lean_dec(x_52); +lean_dec(x_1); +x_73 = l_Lean_mkLevelIMax_x27(x_54, x_68); +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_69); +return x_74; +} +else +{ +size_t x_75; size_t x_76; uint8_t x_77; +x_75 = lean_ptr_addr(x_52); +lean_dec(x_52); +x_76 = lean_ptr_addr(x_68); +x_77 = lean_usize_dec_eq(x_75, x_76); +if (x_77 == 0) +{ +lean_object* x_78; lean_object* x_79; +lean_dec(x_1); +x_78 = l_Lean_mkLevelIMax_x27(x_54, x_68); +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_69); +return x_79; +} +else +{ +lean_object* x_80; lean_object* x_81; +x_80 = l_Lean_simpLevelIMax_x27(x_54, x_68, x_1); +lean_dec(x_1); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_69); +return x_81; +} +} } } case 5: { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_39 = lean_ctor_get(x_1, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_3, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 5); -lean_inc(x_41); -lean_dec(x_40); -lean_inc(x_39); -x_42 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_41, x_39); -if (lean_obj_tag(x_42) == 0) +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_82 = lean_ctor_get(x_1, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_3, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_83, 5); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_82); +x_85 = l_Std_PersistentHashMap_find_x3f___at_Lean_getLevelMVarAssignment_x3f___spec__1(x_84, x_82); +if (lean_obj_tag(x_85) == 0) { -lean_object* x_43; lean_object* x_44; uint8_t x_45; -x_43 = lean_ctor_get(x_2, 2); -lean_inc(x_43); -lean_inc(x_39); -x_44 = lean_apply_1(x_43, x_39); -x_45 = lean_unbox(x_44); -lean_dec(x_44); -if (x_45 == 0) +lean_object* x_86; lean_object* x_87; uint8_t x_88; +x_86 = lean_ctor_get(x_2, 2); +lean_inc(x_86); +lean_inc(x_82); +x_87 = lean_apply_1(x_86, x_82); +x_88 = lean_unbox(x_87); +lean_dec(x_87); +if (x_88 == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; lean_dec(x_1); lean_inc(x_2); -x_46 = l_Lean_MetavarContext_LevelMVarToParam_mkParamName(x_2, x_3); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = l_Lean_Level_param___override(x_47); -lean_inc(x_49); -x_50 = l_Lean_assignLevelMVar___at_Lean_MetavarContext_LevelMVarToParam_visitLevel___spec__1(x_39, x_49, x_2, x_48); +x_89 = l_Lean_MetavarContext_LevelMVarToParam_mkParamName(x_2, x_3); +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = l_Lean_Level_param___override(x_90); +lean_inc(x_92); +x_93 = l_Lean_assignLevelMVar___at_Lean_MetavarContext_LevelMVarToParam_visitLevel___spec__1(x_82, x_92, x_2, x_91); lean_dec(x_2); -x_51 = !lean_is_exclusive(x_50); -if (x_51 == 0) +x_94 = !lean_is_exclusive(x_93); +if (x_94 == 0) { -lean_object* x_52; -x_52 = lean_ctor_get(x_50, 0); -lean_dec(x_52); -lean_ctor_set(x_50, 0, x_49); -return x_50; +lean_object* x_95; +x_95 = lean_ctor_get(x_93, 0); +lean_dec(x_95); +lean_ctor_set(x_93, 0, x_92); +return x_93; } else { -lean_object* x_53; lean_object* x_54; -x_53 = lean_ctor_get(x_50, 1); -lean_inc(x_53); -lean_dec(x_50); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_49); -lean_ctor_set(x_54, 1, x_53); -return x_54; +lean_object* x_96; lean_object* x_97; +x_96 = lean_ctor_get(x_93, 1); +lean_inc(x_96); +lean_dec(x_93); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_92); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } else { -lean_object* x_55; -lean_dec(x_39); +lean_object* x_98; +lean_dec(x_82); lean_dec(x_2); -x_55 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_55, 0, x_1); -lean_ctor_set(x_55, 1, x_3); -return x_55; +x_98 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_98, 0, x_1); +lean_ctor_set(x_98, 1, x_3); +return x_98; } } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_39); +lean_object* x_99; lean_object* x_100; lean_object* x_101; +lean_dec(x_82); lean_dec(x_1); -x_56 = lean_ctor_get(x_42, 0); -lean_inc(x_56); -lean_dec(x_42); -x_57 = l_Lean_markUsedAssignment___at_Lean_MetavarContext_LevelMVarToParam_visitLevel___spec__2___rarg(x_3); -x_58 = lean_ctor_get(x_57, 1); -lean_inc(x_58); -lean_dec(x_57); -x_1 = x_56; -x_3 = x_58; +x_99 = lean_ctor_get(x_85, 0); +lean_inc(x_99); +lean_dec(x_85); +x_100 = l_Lean_markUsedAssignment___at_Lean_MetavarContext_LevelMVarToParam_visitLevel___spec__2___rarg(x_3); +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +lean_dec(x_100); +x_1 = x_99; +x_3 = x_101; goto _start; } } default: { -lean_object* x_60; +lean_object* x_103; lean_dec(x_2); -x_60 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_60, 0, x_1); -lean_ctor_set(x_60, 1, x_3); -return x_60; +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_1); +lean_ctor_set(x_103, 1, x_3); +return x_103; } } } @@ -80584,691 +81493,636 @@ return x_5; } else { -lean_object* x_6; lean_object* x_7; -x_6 = lean_ctor_get(x_3, 3); -lean_inc(x_6); +lean_object* x_6; lean_object* x_7; lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_3, 3); +lean_inc(x_20); lean_inc(x_1); -lean_inc(x_6); -x_7 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_6, x_1); -if (lean_obj_tag(x_7) == 0) +lean_inc(x_20); +x_21 = l_Std_HashMapImp_find_x3f___at_Lean_instantiateExprMVars___spec__1(x_20, x_1); +if (lean_obj_tag(x_21) == 0) { switch (lean_obj_tag(x_1)) { case 2: { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -lean_dec(x_6); -x_8 = l_Lean_instInhabitedMetavarDecl___closed__4; +lean_object* x_22; lean_object* x_23; uint8_t x_24; +lean_dec(x_20); +x_22 = l_Lean_instInhabitedMetavarDecl___closed__4; lean_inc(x_1); -x_9 = l_Lean_MetavarContext_LevelMVarToParam_main_visitApp(x_1, x_8, x_2, x_3); -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) +x_23 = l_Lean_MetavarContext_LevelMVarToParam_main_visitApp(x_1, x_22, x_2, x_3); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 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; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_9, 1); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -x_15 = lean_ctor_get(x_12, 2); -lean_inc(x_15); -x_16 = lean_ctor_get(x_12, 3); -lean_inc(x_16); -lean_dec(x_12); -lean_inc(x_11); -x_17 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_16, x_1, x_11); -x_18 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_18, 0, x_13); -lean_ctor_set(x_18, 1, x_14); -lean_ctor_set(x_18, 2, x_15); -lean_ctor_set(x_18, 3, x_17); -lean_ctor_set(x_9, 1, x_18); -return x_9; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_25 = lean_ctor_get(x_23, 0); +x_26 = lean_ctor_get(x_23, 1); +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_26, 2); +lean_inc(x_29); +x_30 = lean_ctor_get(x_26, 3); +lean_inc(x_30); +lean_dec(x_26); +lean_inc(x_25); +x_31 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_30, x_1, x_25); +x_32 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_32, 0, x_27); +lean_ctor_set(x_32, 1, x_28); +lean_ctor_set(x_32, 2, x_29); +lean_ctor_set(x_32, 3, x_31); +lean_ctor_set(x_23, 1, x_32); +return x_23; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_19 = lean_ctor_get(x_9, 0); -x_20 = lean_ctor_get(x_9, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_9); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -x_23 = lean_ctor_get(x_20, 2); -lean_inc(x_23); -x_24 = lean_ctor_get(x_20, 3); -lean_inc(x_24); -lean_dec(x_20); -lean_inc(x_19); -x_25 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_24, x_1, x_19); -x_26 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_26, 0, x_21); -lean_ctor_set(x_26, 1, x_22); -lean_ctor_set(x_26, 2, x_23); -lean_ctor_set(x_26, 3, x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_19); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} -} -case 3: -{ -lean_object* x_28; lean_object* x_29; uint8_t x_30; -lean_dec(x_6); -x_28 = lean_ctor_get(x_1, 0); -lean_inc(x_28); -x_29 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_28, x_2, x_3); -x_30 = !lean_is_exclusive(x_29); -if (x_30 == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_31 = lean_ctor_get(x_29, 0); -x_32 = lean_ctor_get(x_29, 1); -lean_inc(x_1); -x_33 = lean_expr_update_sort(x_1, x_31); -x_34 = lean_ctor_get(x_32, 0); +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_33 = lean_ctor_get(x_23, 0); +x_34 = lean_ctor_get(x_23, 1); lean_inc(x_34); -x_35 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_23); +x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); -x_36 = lean_ctor_get(x_32, 2); +x_36 = lean_ctor_get(x_34, 1); lean_inc(x_36); -x_37 = lean_ctor_get(x_32, 3); +x_37 = lean_ctor_get(x_34, 2); lean_inc(x_37); -lean_dec(x_32); +x_38 = lean_ctor_get(x_34, 3); +lean_inc(x_38); +lean_dec(x_34); lean_inc(x_33); -x_38 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_37, x_1, x_33); -x_39 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_39, 0, x_34); -lean_ctor_set(x_39, 1, x_35); -lean_ctor_set(x_39, 2, x_36); -lean_ctor_set(x_39, 3, x_38); -lean_ctor_set(x_29, 1, x_39); -lean_ctor_set(x_29, 0, x_33); -return x_29; +x_39 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_38, x_1, x_33); +x_40 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_40, 0, x_35); +lean_ctor_set(x_40, 1, x_36); +lean_ctor_set(x_40, 2, x_37); +lean_ctor_set(x_40, 3, x_39); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_33); +lean_ctor_set(x_41, 1, x_40); +return x_41; } -else +} +case 3: { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_29, 0); -x_41 = lean_ctor_get(x_29, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_29); -lean_inc(x_1); -x_42 = lean_expr_update_sort(x_1, x_40); -x_43 = lean_ctor_get(x_41, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_41, 1); +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; size_t x_46; size_t x_47; uint8_t x_48; +lean_dec(x_20); +x_42 = lean_ctor_get(x_1, 0); +lean_inc(x_42); +lean_inc(x_42); +x_43 = l_Lean_MetavarContext_LevelMVarToParam_visitLevel(x_42, x_2, x_3); +x_44 = lean_ctor_get(x_43, 0); lean_inc(x_44); -x_45 = lean_ctor_get(x_41, 2); +x_45 = lean_ctor_get(x_43, 1); lean_inc(x_45); -x_46 = lean_ctor_get(x_41, 3); -lean_inc(x_46); -lean_dec(x_41); -lean_inc(x_42); -x_47 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_46, x_1, x_42); -x_48 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_48, 0, x_43); -lean_ctor_set(x_48, 1, x_44); -lean_ctor_set(x_48, 2, x_45); -lean_ctor_set(x_48, 3, x_47); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_42); -lean_ctor_set(x_49, 1, x_48); -return x_49; +lean_dec(x_43); +x_46 = lean_ptr_addr(x_42); +lean_dec(x_42); +x_47 = lean_ptr_addr(x_44); +x_48 = lean_usize_dec_eq(x_46, x_47); +if (x_48 == 0) +{ +lean_object* x_49; +x_49 = l_Lean_Expr_sort___override(x_44); +x_6 = x_49; +x_7 = x_45; +goto block_19; +} +else +{ +lean_dec(x_44); +lean_inc(x_1); +x_6 = x_1; +x_7 = x_45; +goto block_19; } } case 4: { -lean_object* x_50; lean_object* x_51; uint8_t x_52; -lean_dec(x_6); -x_50 = lean_ctor_get(x_1, 1); +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +lean_dec(x_20); +x_50 = lean_ctor_get(x_1, 0); lean_inc(x_50); -x_51 = l_List_mapM___at_Lean_MetavarContext_LevelMVarToParam_main___spec__1(x_50, x_2, x_3); -x_52 = !lean_is_exclusive(x_51); -if (x_52 == 0) +x_51 = lean_ctor_get(x_1, 1); +lean_inc(x_51); +lean_inc(x_51); +x_52 = l_List_mapM___at_Lean_MetavarContext_LevelMVarToParam_main___spec__1(x_51, x_2, x_3); +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_ptrEqList___rarg(x_51, x_53); +lean_dec(x_51); +if (x_55 == 0) { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_53 = lean_ctor_get(x_51, 0); -x_54 = lean_ctor_get(x_51, 1); -lean_inc(x_1); -x_55 = lean_expr_update_const(x_1, x_53); -x_56 = lean_ctor_get(x_54, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_54, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_54, 2); -lean_inc(x_58); -x_59 = lean_ctor_get(x_54, 3); -lean_inc(x_59); -lean_dec(x_54); -lean_inc(x_55); -x_60 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_59, x_1, x_55); -x_61 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_61, 0, x_56); -lean_ctor_set(x_61, 1, x_57); -lean_ctor_set(x_61, 2, x_58); -lean_ctor_set(x_61, 3, x_60); -lean_ctor_set(x_51, 1, x_61); -lean_ctor_set(x_51, 0, x_55); -return x_51; +lean_object* x_56; +x_56 = l_Lean_Expr_const___override(x_50, x_53); +x_6 = x_56; +x_7 = x_54; +goto block_19; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_62 = lean_ctor_get(x_51, 0); -x_63 = lean_ctor_get(x_51, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_51); +lean_dec(x_53); +lean_dec(x_50); +lean_inc(x_1); +x_6 = x_1; +x_7 = x_54; +goto block_19; +} +} +case 5: +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; +lean_dec(x_20); +x_57 = lean_unsigned_to_nat(0u); +x_58 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_57); +x_59 = l_Lean_instantiateExprMVars___rarg___lambda__20___closed__1; +lean_inc(x_58); +x_60 = lean_mk_array(x_58, x_59); +x_61 = lean_unsigned_to_nat(1u); +x_62 = lean_nat_sub(x_58, x_61); +lean_dec(x_58); lean_inc(x_1); -x_64 = lean_expr_update_const(x_1, x_62); +x_63 = l_Lean_Expr_withAppAux___at_Lean_MetavarContext_LevelMVarToParam_main___spec__2(x_1, x_60, x_62, x_2, x_3); +x_64 = !lean_is_exclusive(x_63); +if (x_64 == 0) +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_65 = lean_ctor_get(x_63, 0); -lean_inc(x_65); x_66 = lean_ctor_get(x_63, 1); -lean_inc(x_66); -x_67 = lean_ctor_get(x_63, 2); +x_67 = lean_ctor_get(x_66, 0); lean_inc(x_67); -x_68 = lean_ctor_get(x_63, 3); +x_68 = lean_ctor_get(x_66, 1); lean_inc(x_68); -lean_dec(x_63); -lean_inc(x_64); -x_69 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_68, x_1, x_64); -x_70 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_70, 0, x_65); -lean_ctor_set(x_70, 1, x_66); -lean_ctor_set(x_70, 2, x_67); -lean_ctor_set(x_70, 3, x_69); -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_64); -lean_ctor_set(x_71, 1, x_70); -return x_71; -} +x_69 = lean_ctor_get(x_66, 2); +lean_inc(x_69); +x_70 = lean_ctor_get(x_66, 3); +lean_inc(x_70); +lean_dec(x_66); +lean_inc(x_65); +x_71 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_70, x_1, x_65); +x_72 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_72, 0, x_67); +lean_ctor_set(x_72, 1, x_68); +lean_ctor_set(x_72, 2, x_69); +lean_ctor_set(x_72, 3, x_71); +lean_ctor_set(x_63, 1, x_72); +return x_63; } -case 5: +else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; -lean_dec(x_6); -x_72 = lean_unsigned_to_nat(0u); -x_73 = l_Lean_Expr_getAppNumArgsAux(x_1, x_72); -x_74 = l_Lean_instantiateExprMVars___rarg___lambda__20___closed__1; +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_73 = lean_ctor_get(x_63, 0); +x_74 = lean_ctor_get(x_63, 1); +lean_inc(x_74); lean_inc(x_73); -x_75 = lean_mk_array(x_73, x_74); -x_76 = lean_unsigned_to_nat(1u); -x_77 = lean_nat_sub(x_73, x_76); -lean_dec(x_73); -lean_inc(x_1); -x_78 = l_Lean_Expr_withAppAux___at_Lean_MetavarContext_LevelMVarToParam_main___spec__2(x_1, x_75, x_77, x_2, x_3); -x_79 = !lean_is_exclusive(x_78); -if (x_79 == 0) +lean_dec(x_63); +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +x_77 = lean_ctor_get(x_74, 2); +lean_inc(x_77); +x_78 = lean_ctor_get(x_74, 3); +lean_inc(x_78); +lean_dec(x_74); +lean_inc(x_73); +x_79 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_78, x_1, x_73); +x_80 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_80, 0, x_75); +lean_ctor_set(x_80, 1, x_76); +lean_ctor_set(x_80, 2, x_77); +lean_ctor_set(x_80, 3, x_79); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_73); +lean_ctor_set(x_81, 1, x_80); +return x_81; +} +} +case 6: { -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_80 = lean_ctor_get(x_78, 0); -x_81 = lean_ctor_get(x_78, 1); -x_82 = lean_ctor_get(x_81, 0); +lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; size_t x_93; size_t x_94; uint8_t x_95; +lean_dec(x_20); +x_82 = lean_ctor_get(x_1, 0); lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); +x_83 = lean_ctor_get(x_1, 1); lean_inc(x_83); -x_84 = lean_ctor_get(x_81, 2); +x_84 = lean_ctor_get(x_1, 2); lean_inc(x_84); -x_85 = lean_ctor_get(x_81, 3); -lean_inc(x_85); -lean_dec(x_81); -lean_inc(x_80); -x_86 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_85, x_1, x_80); -x_87 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_87, 0, x_82); -lean_ctor_set(x_87, 1, x_83); -lean_ctor_set(x_87, 2, x_84); -lean_ctor_set(x_87, 3, x_86); -lean_ctor_set(x_78, 1, x_87); -return x_78; -} -else -{ -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_88 = lean_ctor_get(x_78, 0); -x_89 = lean_ctor_get(x_78, 1); -lean_inc(x_89); +x_85 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_inc(x_2); +lean_inc(x_83); +x_86 = l_Lean_MetavarContext_LevelMVarToParam_main(x_83, x_2, x_3); +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); lean_inc(x_88); -lean_dec(x_78); +lean_dec(x_86); +lean_inc(x_84); +x_89 = l_Lean_MetavarContext_LevelMVarToParam_main(x_84, x_2, x_88); x_90 = lean_ctor_get(x_89, 0); lean_inc(x_90); x_91 = lean_ctor_get(x_89, 1); lean_inc(x_91); -x_92 = lean_ctor_get(x_89, 2); -lean_inc(x_92); -x_93 = lean_ctor_get(x_89, 3); -lean_inc(x_93); lean_dec(x_89); -lean_inc(x_88); -x_94 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_93, x_1, x_88); -x_95 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_95, 0, x_90); -lean_ctor_set(x_95, 1, x_91); -lean_ctor_set(x_95, 2, x_92); -lean_ctor_set(x_95, 3, x_94); -x_96 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_96, 0, x_88); -lean_ctor_set(x_96, 1, x_95); -return x_96; +lean_inc(x_84); +lean_inc(x_83); +lean_inc(x_82); +x_92 = l_Lean_Expr_lam___override(x_82, x_83, x_84, x_85); +x_93 = lean_ptr_addr(x_83); +lean_dec(x_83); +x_94 = lean_ptr_addr(x_87); +x_95 = lean_usize_dec_eq(x_93, x_94); +if (x_95 == 0) +{ +lean_object* x_96; +lean_dec(x_92); +lean_dec(x_84); +x_96 = l_Lean_Expr_lam___override(x_82, x_87, x_90, x_85); +x_6 = x_96; +x_7 = x_91; +goto block_19; } +else +{ +size_t x_97; size_t x_98; uint8_t x_99; +x_97 = lean_ptr_addr(x_84); +lean_dec(x_84); +x_98 = lean_ptr_addr(x_90); +x_99 = lean_usize_dec_eq(x_97, x_98); +if (x_99 == 0) +{ +lean_object* x_100; +lean_dec(x_92); +x_100 = l_Lean_Expr_lam___override(x_82, x_87, x_90, x_85); +x_6 = x_100; +x_7 = x_91; +goto block_19; } -case 6: +else { -lean_object* x_97; lean_object* x_98; uint8_t 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_6); -x_97 = lean_ctor_get(x_1, 1); -lean_inc(x_97); -x_98 = lean_ctor_get(x_1, 2); -lean_inc(x_98); -x_99 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); -lean_inc(x_2); -x_100 = l_Lean_MetavarContext_LevelMVarToParam_main(x_97, x_2, x_3); -x_101 = lean_ctor_get(x_100, 0); -lean_inc(x_101); -x_102 = lean_ctor_get(x_100, 1); -lean_inc(x_102); -lean_dec(x_100); -x_103 = l_Lean_MetavarContext_LevelMVarToParam_main(x_98, x_2, x_102); -x_104 = !lean_is_exclusive(x_103); -if (x_104 == 0) +uint8_t x_101; +x_101 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_85, x_85); +if (x_101 == 0) { -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; -x_105 = lean_ctor_get(x_103, 0); -x_106 = lean_ctor_get(x_103, 1); -lean_inc(x_1); -x_107 = lean_expr_update_lambda(x_1, x_99, x_101, x_105); -x_108 = lean_ctor_get(x_106, 0); +lean_object* x_102; +lean_dec(x_92); +x_102 = l_Lean_Expr_lam___override(x_82, x_87, x_90, x_85); +x_6 = x_102; +x_7 = x_91; +goto block_19; +} +else +{ +lean_dec(x_90); +lean_dec(x_87); +lean_dec(x_82); +x_6 = x_92; +x_7 = x_91; +goto block_19; +} +} +} +} +case 7: +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; size_t x_114; size_t x_115; uint8_t x_116; +lean_dec(x_20); +x_103 = lean_ctor_get(x_1, 0); +lean_inc(x_103); +x_104 = lean_ctor_get(x_1, 1); +lean_inc(x_104); +x_105 = lean_ctor_get(x_1, 2); +lean_inc(x_105); +x_106 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +lean_inc(x_2); +lean_inc(x_104); +x_107 = l_Lean_MetavarContext_LevelMVarToParam_main(x_104, x_2, x_3); +x_108 = lean_ctor_get(x_107, 0); lean_inc(x_108); -x_109 = lean_ctor_get(x_106, 1); +x_109 = lean_ctor_get(x_107, 1); lean_inc(x_109); -x_110 = lean_ctor_get(x_106, 2); -lean_inc(x_110); -x_111 = lean_ctor_get(x_106, 3); +lean_dec(x_107); +lean_inc(x_105); +x_110 = l_Lean_MetavarContext_LevelMVarToParam_main(x_105, x_2, x_109); +x_111 = lean_ctor_get(x_110, 0); lean_inc(x_111); -lean_dec(x_106); -lean_inc(x_107); -x_112 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_111, x_1, x_107); -x_113 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_113, 0, x_108); -lean_ctor_set(x_113, 1, x_109); -lean_ctor_set(x_113, 2, x_110); -lean_ctor_set(x_113, 3, x_112); -lean_ctor_set(x_103, 1, x_113); -lean_ctor_set(x_103, 0, x_107); -return x_103; +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +lean_dec(x_110); +lean_inc(x_105); +lean_inc(x_104); +lean_inc(x_103); +x_113 = l_Lean_Expr_forallE___override(x_103, x_104, x_105, x_106); +x_114 = lean_ptr_addr(x_104); +lean_dec(x_104); +x_115 = lean_ptr_addr(x_108); +x_116 = lean_usize_dec_eq(x_114, x_115); +if (x_116 == 0) +{ +lean_object* x_117; +lean_dec(x_113); +lean_dec(x_105); +x_117 = l_Lean_Expr_forallE___override(x_103, x_108, x_111, x_106); +x_6 = x_117; +x_7 = x_112; +goto block_19; } else { -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; -x_114 = lean_ctor_get(x_103, 0); -x_115 = lean_ctor_get(x_103, 1); -lean_inc(x_115); -lean_inc(x_114); +size_t x_118; size_t x_119; uint8_t x_120; +x_118 = lean_ptr_addr(x_105); +lean_dec(x_105); +x_119 = lean_ptr_addr(x_111); +x_120 = lean_usize_dec_eq(x_118, x_119); +if (x_120 == 0) +{ +lean_object* x_121; +lean_dec(x_113); +x_121 = l_Lean_Expr_forallE___override(x_103, x_108, x_111, x_106); +x_6 = x_121; +x_7 = x_112; +goto block_19; +} +else +{ +uint8_t x_122; +x_122 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_106, x_106); +if (x_122 == 0) +{ +lean_object* x_123; +lean_dec(x_113); +x_123 = l_Lean_Expr_forallE___override(x_103, x_108, x_111, x_106); +x_6 = x_123; +x_7 = x_112; +goto block_19; +} +else +{ +lean_dec(x_111); +lean_dec(x_108); lean_dec(x_103); -lean_inc(x_1); -x_116 = lean_expr_update_lambda(x_1, x_99, x_101, x_114); -x_117 = lean_ctor_get(x_115, 0); -lean_inc(x_117); -x_118 = lean_ctor_get(x_115, 1); -lean_inc(x_118); -x_119 = lean_ctor_get(x_115, 2); -lean_inc(x_119); -x_120 = lean_ctor_get(x_115, 3); -lean_inc(x_120); -lean_dec(x_115); -lean_inc(x_116); -x_121 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_120, x_1, x_116); -x_122 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_122, 0, x_117); -lean_ctor_set(x_122, 1, x_118); -lean_ctor_set(x_122, 2, x_119); -lean_ctor_set(x_122, 3, x_121); -x_123 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_123, 0, x_116); -lean_ctor_set(x_123, 1, x_122); -return x_123; +x_6 = x_113; +x_7 = x_112; +goto block_19; } } -case 7: +} +} +case 8: { -lean_object* x_124; lean_object* x_125; uint8_t x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; uint8_t x_131; -lean_dec(x_6); -x_124 = lean_ctor_get(x_1, 1); +lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; size_t x_138; size_t x_139; uint8_t x_140; +lean_dec(x_20); +x_124 = lean_ctor_get(x_1, 0); lean_inc(x_124); -x_125 = lean_ctor_get(x_1, 2); +x_125 = lean_ctor_get(x_1, 1); lean_inc(x_125); -x_126 = lean_ctor_get_uint8(x_1, sizeof(void*)*3 + 8); +x_126 = lean_ctor_get(x_1, 2); +lean_inc(x_126); +x_127 = lean_ctor_get(x_1, 3); +lean_inc(x_127); +x_128 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 8); lean_inc(x_2); -x_127 = l_Lean_MetavarContext_LevelMVarToParam_main(x_124, x_2, x_3); -x_128 = lean_ctor_get(x_127, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_127, 1); -lean_inc(x_129); -lean_dec(x_127); -x_130 = l_Lean_MetavarContext_LevelMVarToParam_main(x_125, x_2, x_129); -x_131 = !lean_is_exclusive(x_130); -if (x_131 == 0) -{ -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; -x_132 = lean_ctor_get(x_130, 0); -x_133 = lean_ctor_get(x_130, 1); -lean_inc(x_1); -x_134 = lean_expr_update_forall(x_1, x_126, x_128, x_132); -x_135 = lean_ctor_get(x_133, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_133, 1); +lean_inc(x_125); +x_129 = l_Lean_MetavarContext_LevelMVarToParam_main(x_125, x_2, x_3); +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_2); +lean_inc(x_126); +x_132 = l_Lean_MetavarContext_LevelMVarToParam_main(x_126, x_2, x_131); +x_133 = lean_ctor_get(x_132, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_132, 1); +lean_inc(x_134); +lean_dec(x_132); +lean_inc(x_127); +x_135 = l_Lean_MetavarContext_LevelMVarToParam_main(x_127, x_2, x_134); +x_136 = lean_ctor_get(x_135, 0); lean_inc(x_136); -x_137 = lean_ctor_get(x_133, 2); +x_137 = lean_ctor_get(x_135, 1); lean_inc(x_137); -x_138 = lean_ctor_get(x_133, 3); -lean_inc(x_138); -lean_dec(x_133); -lean_inc(x_134); -x_139 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_138, x_1, x_134); -x_140 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_140, 0, x_135); -lean_ctor_set(x_140, 1, x_136); -lean_ctor_set(x_140, 2, x_137); -lean_ctor_set(x_140, 3, x_139); -lean_ctor_set(x_130, 1, x_140); -lean_ctor_set(x_130, 0, x_134); -return x_130; +lean_dec(x_135); +x_138 = lean_ptr_addr(x_125); +lean_dec(x_125); +x_139 = lean_ptr_addr(x_130); +x_140 = lean_usize_dec_eq(x_138, x_139); +if (x_140 == 0) +{ +lean_object* x_141; +lean_dec(x_127); +lean_dec(x_126); +x_141 = l_Lean_Expr_letE___override(x_124, x_130, x_133, x_136, x_128); +x_6 = x_141; +x_7 = x_137; +goto block_19; } else { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; -x_141 = lean_ctor_get(x_130, 0); -x_142 = lean_ctor_get(x_130, 1); -lean_inc(x_142); -lean_inc(x_141); -lean_dec(x_130); -lean_inc(x_1); -x_143 = lean_expr_update_forall(x_1, x_126, x_128, x_141); -x_144 = lean_ctor_get(x_142, 0); -lean_inc(x_144); -x_145 = lean_ctor_get(x_142, 1); -lean_inc(x_145); -x_146 = lean_ctor_get(x_142, 2); -lean_inc(x_146); -x_147 = lean_ctor_get(x_142, 3); -lean_inc(x_147); -lean_dec(x_142); -lean_inc(x_143); -x_148 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_147, x_1, x_143); -x_149 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_149, 0, x_144); -lean_ctor_set(x_149, 1, x_145); -lean_ctor_set(x_149, 2, x_146); -lean_ctor_set(x_149, 3, x_148); -x_150 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_150, 0, x_143); -lean_ctor_set(x_150, 1, x_149); -return x_150; -} +size_t x_142; size_t x_143; uint8_t x_144; +x_142 = lean_ptr_addr(x_126); +lean_dec(x_126); +x_143 = lean_ptr_addr(x_133); +x_144 = lean_usize_dec_eq(x_142, x_143); +if (x_144 == 0) +{ +lean_object* x_145; +lean_dec(x_127); +x_145 = l_Lean_Expr_letE___override(x_124, x_130, x_133, x_136, x_128); +x_6 = x_145; +x_7 = x_137; +goto block_19; } -case 8: +else { -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; uint8_t x_161; -lean_dec(x_6); -x_151 = lean_ctor_get(x_1, 1); -lean_inc(x_151); -x_152 = lean_ctor_get(x_1, 2); -lean_inc(x_152); -x_153 = lean_ctor_get(x_1, 3); -lean_inc(x_153); -lean_inc(x_2); -x_154 = l_Lean_MetavarContext_LevelMVarToParam_main(x_151, x_2, x_3); -x_155 = lean_ctor_get(x_154, 0); -lean_inc(x_155); -x_156 = lean_ctor_get(x_154, 1); -lean_inc(x_156); -lean_dec(x_154); -lean_inc(x_2); -x_157 = l_Lean_MetavarContext_LevelMVarToParam_main(x_152, x_2, x_156); -x_158 = lean_ctor_get(x_157, 0); -lean_inc(x_158); -x_159 = lean_ctor_get(x_157, 1); -lean_inc(x_159); -lean_dec(x_157); -x_160 = l_Lean_MetavarContext_LevelMVarToParam_main(x_153, x_2, x_159); -x_161 = !lean_is_exclusive(x_160); -if (x_161 == 0) +size_t x_146; size_t x_147; uint8_t x_148; +x_146 = lean_ptr_addr(x_127); +lean_dec(x_127); +x_147 = lean_ptr_addr(x_136); +x_148 = lean_usize_dec_eq(x_146, x_147); +if (x_148 == 0) { -lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; -x_162 = lean_ctor_get(x_160, 0); -x_163 = lean_ctor_get(x_160, 1); -lean_inc(x_1); -x_164 = lean_expr_update_let(x_1, x_155, x_158, x_162); -x_165 = lean_ctor_get(x_163, 0); -lean_inc(x_165); -x_166 = lean_ctor_get(x_163, 1); -lean_inc(x_166); -x_167 = lean_ctor_get(x_163, 2); -lean_inc(x_167); -x_168 = lean_ctor_get(x_163, 3); -lean_inc(x_168); -lean_dec(x_163); -lean_inc(x_164); -x_169 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_168, x_1, x_164); -x_170 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_170, 0, x_165); -lean_ctor_set(x_170, 1, x_166); -lean_ctor_set(x_170, 2, x_167); -lean_ctor_set(x_170, 3, x_169); -lean_ctor_set(x_160, 1, x_170); -lean_ctor_set(x_160, 0, x_164); -return x_160; +lean_object* x_149; +x_149 = l_Lean_Expr_letE___override(x_124, x_130, x_133, x_136, x_128); +x_6 = x_149; +x_7 = x_137; +goto block_19; } else { -lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; -x_171 = lean_ctor_get(x_160, 0); -x_172 = lean_ctor_get(x_160, 1); -lean_inc(x_172); -lean_inc(x_171); -lean_dec(x_160); +lean_dec(x_136); +lean_dec(x_133); +lean_dec(x_130); +lean_dec(x_124); lean_inc(x_1); -x_173 = lean_expr_update_let(x_1, x_155, x_158, x_171); -x_174 = lean_ctor_get(x_172, 0); -lean_inc(x_174); -x_175 = lean_ctor_get(x_172, 1); -lean_inc(x_175); -x_176 = lean_ctor_get(x_172, 2); -lean_inc(x_176); -x_177 = lean_ctor_get(x_172, 3); -lean_inc(x_177); -lean_dec(x_172); -lean_inc(x_173); -x_178 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_177, x_1, x_173); -x_179 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_179, 0, x_174); -lean_ctor_set(x_179, 1, x_175); -lean_ctor_set(x_179, 2, x_176); -lean_ctor_set(x_179, 3, x_178); -x_180 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_180, 0, x_173); -lean_ctor_set(x_180, 1, x_179); -return x_180; +x_6 = x_1; +x_7 = x_137; +goto block_19; +} +} } } case 10: { -lean_object* x_181; lean_object* x_182; uint8_t x_183; -lean_dec(x_6); -x_181 = lean_ctor_get(x_1, 1); -lean_inc(x_181); -x_182 = l_Lean_MetavarContext_LevelMVarToParam_main(x_181, x_2, x_3); -x_183 = !lean_is_exclusive(x_182); -if (x_183 == 0) +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; size_t x_155; size_t x_156; uint8_t x_157; +lean_dec(x_20); +x_150 = lean_ctor_get(x_1, 0); +lean_inc(x_150); +x_151 = lean_ctor_get(x_1, 1); +lean_inc(x_151); +lean_inc(x_151); +x_152 = l_Lean_MetavarContext_LevelMVarToParam_main(x_151, x_2, x_3); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +x_154 = lean_ctor_get(x_152, 1); +lean_inc(x_154); +lean_dec(x_152); +x_155 = lean_ptr_addr(x_151); +lean_dec(x_151); +x_156 = lean_ptr_addr(x_153); +x_157 = lean_usize_dec_eq(x_155, x_156); +if (x_157 == 0) { -lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_184 = lean_ctor_get(x_182, 0); -x_185 = lean_ctor_get(x_182, 1); -lean_inc(x_1); -x_186 = lean_expr_update_mdata(x_1, x_184); -x_187 = lean_ctor_get(x_185, 0); -lean_inc(x_187); -x_188 = lean_ctor_get(x_185, 1); -lean_inc(x_188); -x_189 = lean_ctor_get(x_185, 2); -lean_inc(x_189); -x_190 = lean_ctor_get(x_185, 3); -lean_inc(x_190); -lean_dec(x_185); -lean_inc(x_186); -x_191 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_190, x_1, x_186); -x_192 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_192, 0, x_187); -lean_ctor_set(x_192, 1, x_188); -lean_ctor_set(x_192, 2, x_189); -lean_ctor_set(x_192, 3, x_191); -lean_ctor_set(x_182, 1, x_192); -lean_ctor_set(x_182, 0, x_186); -return x_182; +lean_object* x_158; +x_158 = l_Lean_Expr_mdata___override(x_150, x_153); +x_6 = x_158; +x_7 = x_154; +goto block_19; } else { -lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; -x_193 = lean_ctor_get(x_182, 0); -x_194 = lean_ctor_get(x_182, 1); -lean_inc(x_194); -lean_inc(x_193); -lean_dec(x_182); +lean_dec(x_153); +lean_dec(x_150); lean_inc(x_1); -x_195 = lean_expr_update_mdata(x_1, x_193); -x_196 = lean_ctor_get(x_194, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_194, 1); -lean_inc(x_197); -x_198 = lean_ctor_get(x_194, 2); -lean_inc(x_198); -x_199 = lean_ctor_get(x_194, 3); -lean_inc(x_199); -lean_dec(x_194); -lean_inc(x_195); -x_200 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_199, x_1, x_195); -x_201 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_201, 0, x_196); -lean_ctor_set(x_201, 1, x_197); -lean_ctor_set(x_201, 2, x_198); -lean_ctor_set(x_201, 3, x_200); -x_202 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_202, 0, x_195); -lean_ctor_set(x_202, 1, x_201); -return x_202; +x_6 = x_1; +x_7 = x_154; +goto block_19; } } case 11: { -lean_object* x_203; lean_object* x_204; uint8_t x_205; -lean_dec(x_6); -x_203 = lean_ctor_get(x_1, 2); -lean_inc(x_203); -x_204 = l_Lean_MetavarContext_LevelMVarToParam_main(x_203, x_2, x_3); -x_205 = !lean_is_exclusive(x_204); -if (x_205 == 0) +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; size_t x_165; size_t x_166; uint8_t x_167; +lean_dec(x_20); +x_159 = lean_ctor_get(x_1, 0); +lean_inc(x_159); +x_160 = lean_ctor_get(x_1, 1); +lean_inc(x_160); +x_161 = lean_ctor_get(x_1, 2); +lean_inc(x_161); +lean_inc(x_161); +x_162 = l_Lean_MetavarContext_LevelMVarToParam_main(x_161, x_2, x_3); +x_163 = lean_ctor_get(x_162, 0); +lean_inc(x_163); +x_164 = lean_ctor_get(x_162, 1); +lean_inc(x_164); +lean_dec(x_162); +x_165 = lean_ptr_addr(x_161); +lean_dec(x_161); +x_166 = lean_ptr_addr(x_163); +x_167 = lean_usize_dec_eq(x_165, x_166); +if (x_167 == 0) { -lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; -x_206 = lean_ctor_get(x_204, 0); -x_207 = lean_ctor_get(x_204, 1); -lean_inc(x_1); -x_208 = lean_expr_update_proj(x_1, x_206); -x_209 = lean_ctor_get(x_207, 0); -lean_inc(x_209); -x_210 = lean_ctor_get(x_207, 1); -lean_inc(x_210); -x_211 = lean_ctor_get(x_207, 2); -lean_inc(x_211); -x_212 = lean_ctor_get(x_207, 3); -lean_inc(x_212); -lean_dec(x_207); -lean_inc(x_208); -x_213 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_212, x_1, x_208); -x_214 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_214, 0, x_209); -lean_ctor_set(x_214, 1, x_210); -lean_ctor_set(x_214, 2, x_211); -lean_ctor_set(x_214, 3, x_213); -lean_ctor_set(x_204, 1, x_214); -lean_ctor_set(x_204, 0, x_208); -return x_204; +lean_object* x_168; +x_168 = l_Lean_Expr_proj___override(x_159, x_160, x_163); +x_6 = x_168; +x_7 = x_164; +goto block_19; } else { -lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; -x_215 = lean_ctor_get(x_204, 0); -x_216 = lean_ctor_get(x_204, 1); -lean_inc(x_216); -lean_inc(x_215); -lean_dec(x_204); +lean_dec(x_163); +lean_dec(x_160); +lean_dec(x_159); lean_inc(x_1); -x_217 = lean_expr_update_proj(x_1, x_215); -x_218 = lean_ctor_get(x_216, 0); -lean_inc(x_218); -x_219 = lean_ctor_get(x_216, 1); -lean_inc(x_219); -x_220 = lean_ctor_get(x_216, 2); -lean_inc(x_220); -x_221 = lean_ctor_get(x_216, 3); -lean_inc(x_221); -lean_dec(x_216); -lean_inc(x_217); -x_222 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_221, x_1, x_217); -x_223 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_223, 0, x_218); -lean_ctor_set(x_223, 1, x_219); -lean_ctor_set(x_223, 2, x_220); -lean_ctor_set(x_223, 3, x_222); -x_224 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_224, 0, x_217); -lean_ctor_set(x_224, 1, x_223); -return x_224; +x_6 = x_1; +x_7 = x_164; +goto block_19; } } default: { -lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; +lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_dec(x_2); -x_225 = lean_ctor_get(x_3, 0); -lean_inc(x_225); -x_226 = lean_ctor_get(x_3, 1); -lean_inc(x_226); -x_227 = lean_ctor_get(x_3, 2); -lean_inc(x_227); +x_169 = lean_ctor_get(x_3, 0); +lean_inc(x_169); +x_170 = lean_ctor_get(x_3, 1); +lean_inc(x_170); +x_171 = lean_ctor_get(x_3, 2); +lean_inc(x_171); lean_dec(x_3); lean_inc_n(x_1, 2); -x_228 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_6, x_1, x_1); -x_229 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_229, 0, x_225); -lean_ctor_set(x_229, 1, x_226); -lean_ctor_set(x_229, 2, x_227); -lean_ctor_set(x_229, 3, x_228); -x_230 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_230, 0, x_1); -lean_ctor_set(x_230, 1, x_229); -return x_230; +x_172 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_20, x_1, x_1); +x_173 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_173, 0, x_169); +lean_ctor_set(x_173, 1, x_170); +lean_ctor_set(x_173, 2, x_171); +lean_ctor_set(x_173, 3, x_172); +x_174 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_174, 0, x_1); +lean_ctor_set(x_174, 1, x_173); +return x_174; } } } else { -lean_object* x_231; lean_object* x_232; -lean_dec(x_6); +lean_object* x_175; lean_object* x_176; +lean_dec(x_20); lean_dec(x_2); lean_dec(x_1); -x_231 = lean_ctor_get(x_7, 0); -lean_inc(x_231); +x_175 = lean_ctor_get(x_21, 0); +lean_inc(x_175); +lean_dec(x_21); +x_176 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_176, 0, x_175); +lean_ctor_set(x_176, 1, x_3); +return x_176; +} +block_19: +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_7, 3); +lean_inc(x_6); +x_10 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_9, x_1, x_6); +lean_ctor_set(x_7, 3, x_10); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_6); +lean_ctor_set(x_11, 1, x_7); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_12 = lean_ctor_get(x_7, 0); +x_13 = lean_ctor_get(x_7, 1); +x_14 = lean_ctor_get(x_7, 2); +x_15 = lean_ctor_get(x_7, 3); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); lean_dec(x_7); -x_232 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_232, 0, x_231); -lean_ctor_set(x_232, 1, x_3); -return x_232; +lean_inc(x_6); +x_16 = l_Std_HashMap_insert___at_Lean_instantiateExprMVars___spec__3(x_15, x_1, x_6); +x_17 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_17, 0, x_12); +lean_ctor_set(x_17, 1, x_13); +lean_ctor_set(x_17, 2, x_14); +lean_ctor_set(x_17, 3, x_16); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_6); +lean_ctor_set(x_18, 1, x_17); +return x_18; +} } } } diff --git a/stage0/stdlib/Lean/MonadEnv.c b/stage0/stdlib/Lean/MonadEnv.c index 530ce9899e14..6cb43d01e3e7 100644 --- a/stage0/stdlib/Lean/MonadEnv.c +++ b/stage0/stdlib/Lean/MonadEnv.c @@ -3858,7 +3858,7 @@ static lean_object* _init_l_Lean_findModuleOf_x3f___rarg___lambda__1___closed__4 lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_findModuleOf_x3f___rarg___lambda__1___closed__1; x_2 = l_Lean_findModuleOf_x3f___rarg___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_findModuleOf_x3f___rarg___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Parser/Attr.c b/stage0/stdlib/Lean/Parser/Attr.c index 22c5495801e7..66efa64480bf 100644 --- a/stage0/stdlib/Lean/Parser/Attr.c +++ b/stage0/stdlib/Lean/Parser/Attr.c @@ -16,6 +16,7 @@ extern "C" { LEAN_EXPORT lean_object* l_Lean_Parser_Attr_extern_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Attr_extern; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_declRange(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_formatter(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_class_declRange(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_instance_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Attr_class_declRange___closed__6; @@ -46,7 +47,9 @@ lean_object* l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(lean_ static lean_object* l_Lean_Parser_Attr_macro___closed__8; static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__2; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Attr___hyg_36____closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_instance_formatter(lean_object*); lean_object* l_Lean_Parser_many(lean_object*); static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio___closed__8; @@ -62,6 +65,7 @@ static lean_object* l_Lean_Parser_Attr_class_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Priority_numPrio_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_attrParser_formatter(lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_simple_formatter(lean_object*); static lean_object* l_Lean_Parser_Attr_simple_formatter___closed__7; static lean_object* l_Lean_Parser_Attr_simple___closed__1; static lean_object* l_Lean_Parser_Attr_simple_parenthesizer___closed__3; @@ -79,6 +83,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_declRange___closed_ static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__11; static lean_object* l_Lean_Parser_Attr_macro___elambda__1___lambda__1___closed__1; static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_externEntry_formatter(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Attr_class___elambda__1(lean_object*, lean_object*); extern lean_object* l_Lean_Parser_ident; @@ -90,24 +95,27 @@ static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__11; static lean_object* l_Lean_Parser_Attr_externEntry___closed__1; static lean_object* l_Lean_Parser_Attr_extern_formatter___closed__5; lean_object* l_Lean_Parser_ParserState_mkNode(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio___closed__2; static lean_object* l_Lean_Parser_Attr_export_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_priorityParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Attr_extern_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Attr_macro_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_recursor; static lean_object* l_Lean_Parser_Attr_externEntry_parenthesizer___closed__2; lean_object* l_Lean_Parser_orelseFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_simple_parenthesizer___closed__1; lean_object* l_Lean_Parser_registerBuiltinDynamicParserAttribute(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Attr_simple_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_externEntry_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__1; lean_object* l_Lean_Parser_addBuiltinParser(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_optional_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Parser_Attr_macro_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_export_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_declRange___closed__2; static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__3; static lean_object* l_Lean_Parser_Attr_recursor___closed__4; @@ -115,6 +123,7 @@ lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__6; static lean_object* l_Lean_Parser_Attr_simple_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Attr_export_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Attr_extern_declRange___closed__6; static lean_object* l_Lean_Parser_Attr_export___elambda__1___closed__12; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Attr___hyg_4____closed__2; @@ -122,6 +131,8 @@ static lean_object* l_Lean_Parser_Attr_extern_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Attr_macro_declRange___closed__3; static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__4; static lean_object* l_Lean_Parser_Attr_macro___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Attr_instance_declRange___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_macro___elambda__1(lean_object*, lean_object*); @@ -129,6 +140,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Attr_class_parenthesizer(lean_object*, le static lean_object* l_Lean_Parser_Attr_externEntry_formatter___closed__8; lean_object* l_Lean_Parser_checkPrecFn___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_extern___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_simple___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Attr_macro_declRange___closed__5; @@ -145,12 +157,15 @@ static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__5; static lean_object* l_Lean_Parser_Attr_defaultInstance_formatter___closed__3; static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__8; static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__10; +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_externEntry_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__18; lean_object* l_Lean_Parser_many_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_extern_parenthesizer___closed__4; lean_object* l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Attr_recursor___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Attr_macro___closed__5; static lean_object* l_Lean_Parser_Attr_class_formatter___closed__1; lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -159,6 +174,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_instance(lean_object*); static lean_object* l_Lean_Parser_Attr_extern_formatter___closed__3; lean_object* l_Lean_Parser_checkPrecFn(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Attr_macro_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__1; static lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__7; static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__7; static lean_object* l_Lean_Parser_Attr_recursor_parenthesizer___closed__2; @@ -167,14 +183,19 @@ static lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__2; static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__17; static lean_object* l_Lean_Parser_Attr_class___elambda__1___closed__10; static lean_object* l_Lean_Parser_Attr_externEntry_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_macro_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_externEntry___closed__4; lean_object* l_Lean_Parser_strLit___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Attr_extern_declRange___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__2; static lean_object* l_Lean_Parser_Attr_recursor___closed__2; static lean_object* l_Lean_Parser_Attr_macro___closed__6; static lean_object* l_Lean_Parser_Attr_macro___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_declRange___closed__4; uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Priority_numPrio___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio___closed__7; @@ -191,11 +212,13 @@ static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_declRange___ static lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_declRange___closed__5; static lean_object* l_Lean_Parser_Attr_defaultInstance___closed__8; lean_object* l_Lean_Parser_nonReservedSymbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__2; static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__5; static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__5; static lean_object* l_Lean_Parser_Attr_simple_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_attrParser(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Attr_simple; +static lean_object* l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__2; lean_object* l_Lean_Parser_nodeInfo(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Attr_externEntry_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__4; @@ -213,8 +236,10 @@ static lean_object* l___regBuiltin_Lean_Parser_Attr_export_declRange___closed__5 lean_object* l_Lean_Parser_nonReservedSymbolInfo(lean_object*, uint8_t); static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__10; lean_object* l_Lean_Parser_strLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_checkPrec_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Attr_instance_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Attr_extern___closed__7; static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__13; @@ -223,6 +248,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Attr_extern_declRange___closed__3 static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__3; static lean_object* l_Lean_Parser_Attr_export___closed__2; static lean_object* l_Lean_Parser_Attr_instance___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_class_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Attr_instance_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_extern_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Attr_class___elambda__1___closed__6; @@ -255,14 +281,15 @@ static lean_object* l___regBuiltin_Lean_Parser_Attr_instance_declRange___closed_ static lean_object* l_Lean_Parser_Attr_macro_formatter___closed__1; static lean_object* l_Lean_Parser_Attr_export_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Attr_simple___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Attr_recursor___elambda__1___closed__4; -static lean_object* l_Lean_Parser_Attr_extern_formatter___closed__8; static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Attr_extern_declRange___closed__7; lean_object* l_Lean_Parser_orelseInfo(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_export_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_export___elambda__1___closed__10; static lean_object* l_Lean_Parser_Attr_externEntry_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_class_formatter(lean_object*); static lean_object* l_Lean_Parser_Attr_instance_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Attr_externEntry_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Priority_numPrio_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -287,21 +314,29 @@ static lean_object* l_Lean_Parser_Attr_macro___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_recursor___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_recursor_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Attr_instance_declRange___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter(lean_object*); +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; uint32_t lean_string_utf8_get(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_macro___elambda__1___closed__3; static lean_object* l_Lean_Parser_Attr_export_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Attr_extern_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__2; lean_object* l_Lean_Parser_registerBuiltinParserAttribute(lean_object*, lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Parser_Attr_extern___closed__1; static lean_object* l_Lean_Parser_Attr_externEntry_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_instance___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Attr_instance_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Attr_export_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_recursor___elambda__1___closed__2; static lean_object* l_Lean_Parser_Attr_extern_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_export___elambda__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_recursor(lean_object*); static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__7; @@ -329,6 +364,7 @@ static lean_object* l_Lean_Parser_Attr_recursor___elambda__1___closed__8; static lean_object* l_Lean_Parser_Attr_macro_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_macro___elambda__1___closed__5; static lean_object* l_Lean_Parser_Attr_externEntry_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__1; static lean_object* l_Lean_Parser_Attr_macro_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_instance; @@ -342,6 +378,7 @@ static lean_object* l_Lean_Parser_Attr_defaultInstance_formatter___closed__4; static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_export; static lean_object* l_Lean_Parser_Attr_extern___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; lean_object* l_Lean_Parser_ident___elambda__1(lean_object*, lean_object*); uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__14; @@ -358,6 +395,7 @@ static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__14; static lean_object* l_Lean_Parser_Attr_export_formatter___closed__1; static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__1; static lean_object* l_Lean_Parser_Attr_defaultInstance_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Attr_class___elambda__1___closed__5; static lean_object* l_Lean_Parser_Attr_instance___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio(lean_object*); @@ -368,25 +406,33 @@ static lean_object* l___regBuiltin_Lean_Parser_Attr_class_declRange___closed__1; static lean_object* l_Lean_Parser_Attr_class___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_macro(lean_object*); static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__15; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Attr_defaultInstance___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_priorityParser_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Attr_macro_declRange___closed__6; lean_object* l_Lean_Parser_categoryParser(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__1; static lean_object* l_Lean_Parser_Attr_export_formatter___closed__3; static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__6; static lean_object* l_Lean_Parser_Priority_numPrio_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Priority_numPrio; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__2; static lean_object* l_Lean_Parser_Attr_export___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__2; static lean_object* l_Lean_Parser_Attr_recursor___closed__6; static lean_object* l_Lean_Parser_Attr_class___elambda__1___closed__3; static lean_object* l_Lean_Parser_Attr_macro_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio___closed__5; lean_object* l_Lean_Parser_symbolInfo(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__1; lean_object* l_Lean_Parser_orelseFnCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); extern lean_object* l_Lean_Parser_epsilonInfo; static lean_object* l_Lean_Parser_Attr_externEntry_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_extern_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Attr_externEntry___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio___closed__3; lean_object* l_Lean_Parser_categoryParser___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -402,11 +448,13 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Attr_externEntry; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_externEntry_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_priorityParser_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_class(lean_object*); static lean_object* l_Lean_Parser_Attr_class___elambda__1___closed__1; static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Attr_class_declRange___closed__7; lean_object* l_Lean_Parser_ident_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__1; static lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__9; static lean_object* l_Lean_Parser_Attr_externEntry_formatter___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_declRange___closed__5; @@ -420,6 +468,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio_declRange___clos static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_class_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Attr_extern___closed__4; static lean_object* l_Lean_Parser_Attr_externEntry___elambda__1___closed__6; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Attr___hyg_4____closed__3; @@ -448,8 +497,10 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_extern_declRange(lean_o static lean_object* l___regBuiltin_Lean_Parser_Attr_export_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_recursor___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_export_formatter(lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Attr___hyg_4____closed__6; static lean_object* l_Lean_Parser_Attr_extern___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_recursor_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Attr___hyg_36____closed__3; static lean_object* l_Lean_Parser_Attr_externEntry___closed__2; @@ -468,8 +519,10 @@ static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__2; static lean_object* l_Lean_Parser_Attr_export___elambda__1___closed__1; static lean_object* l_Lean_Parser_Attr_simple_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_export___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Attr_macro___elambda__1___closed__7; static lean_object* l_Lean_Parser_Attr_externEntry___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Attr_simple_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_defaultInstance_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_simple___closed__3; @@ -482,6 +535,7 @@ lean_object* l_Lean_Parser_numLit_formatter(lean_object*, lean_object*, lean_obj static lean_object* l___regBuiltin_Lean_Parser_Priority_numPrio_declRange___closed__4; lean_object* l_Lean_Parser_symbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_simple___elambda__1___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__1; static lean_object* l_Lean_Parser_Attr_export___elambda__1___closed__4; static lean_object* l_Lean_Parser_Attr_export___closed__4; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Attr___hyg_36____closed__5; @@ -492,9 +546,11 @@ static lean_object* l_Lean_Parser_Attr_class_parenthesizer___closed__1; lean_object* l_Lean_Parser_symbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_class_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_instance_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__2; static lean_object* l_Lean_Parser_Attr_instance___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__1; static lean_object* l_Lean_Parser_Attr_instance___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Attr_recursor_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -506,14 +562,17 @@ static lean_object* l_Lean_Parser_Attr_simple___closed__7; static lean_object* l_Lean_Parser_Attr_recursor___closed__7; static lean_object* l_Lean_Parser_Attr_instance___closed__4; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Attr___hyg_4____closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__1; static lean_object* l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__4; extern lean_object* l_Lean_Parser_strLit; static lean_object* l___regBuiltin_Lean_Parser_Attr_instance_declRange___closed__5; lean_object* l_Lean_PrettyPrinter_Formatter_andthen_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Attr_externEntry_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Attr_simple_parenthesizer___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_priorityParser(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Attr_simple___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Attr_instance___closed__1; static lean_object* l_Lean_Parser_Attr_externEntry___closed__7; @@ -1703,6 +1762,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_simple___elambda__1___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_simple_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_simple_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_simple___elambda__1___closed__4; +x_4 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_simple_parenthesizer___closed__1() { _start: { @@ -1797,6 +1902,52 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_simple___elambda__1___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_simple_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_simple___elambda__1___closed__4; +x_4 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_macro___elambda__1___lambda__1___closed__1() { _start: { @@ -2375,6 +2526,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_macro___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_macro_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_macro_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_macro___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_macro_parenthesizer___closed__1() { _start: { @@ -2439,6 +2620,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_macro___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_macro_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_macro___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_export___elambda__1___closed__1() { _start: { @@ -3010,6 +3221,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_export___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_export_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_export_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_export___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_export_parenthesizer___closed__1() { _start: { @@ -3074,6 +3315,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_export___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_export_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_export_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_export___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Attr_recursor___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -3647,6 +3918,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_recursor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_recursor_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_recursor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_recursor_parenthesizer___closed__1() { _start: { @@ -3714,6 +4015,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_recursor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_recursor_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_recursor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_class___elambda__1___closed__1() { _start: { @@ -4177,6 +4508,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_class___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_class_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_class_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_class___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_class_parenthesizer___closed__1() { _start: { @@ -4229,6 +4590,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_class___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_class_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_class_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_class___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_instance___elambda__1___closed__1() { _start: { @@ -4820,6 +5211,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_instance___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_instance_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_instance_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_instance___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_instance_parenthesizer___closed__1() { _start: { @@ -4894,6 +5315,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_instance___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_instance_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_instance___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__1() { _start: { @@ -5478,6 +5929,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_defaultInstance_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1() { _start: { @@ -5545,6 +6026,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_defaultInstance_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_externEntry___elambda__1___closed__1() { _start: { @@ -6622,6 +7133,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_externEntry___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_externEntry_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_externEntry_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_externEntry___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__1() { _start: { @@ -6666,52 +7207,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_externEntry_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Attr_extern_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Attr_extern_formatter___closed__3; -x_2 = l_Lean_Parser_Attr_extern_formatter___closed__5; +x_2 = l_Lean_Parser_Attr_extern_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Attr_extern_formatter___closed__2; -x_2 = l_Lean_Parser_Attr_extern_formatter___closed__6; +x_2 = l_Lean_Parser_Attr_extern_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Attr_extern_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Attr_extern___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Attr_extern_formatter___closed__7; +x_3 = l_Lean_Parser_Attr_extern_formatter___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -6724,11 +7257,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Attr_extern_formatter(lean_object* x_1, l { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Attr_extern_formatter___closed__1; -x_7 = l_Lean_Parser_Attr_extern_formatter___closed__8; +x_7 = l_Lean_Parser_Attr_extern_formatter___closed__7; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_extern___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_extern_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_extern_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3; +x_3 = l_Lean_Parser_Attr_extern___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_externEntry_parenthesizer___closed__1() { _start: { @@ -6836,6 +7399,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_externEntry___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_externEntry_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_externEntry___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__1() { _start: { @@ -6880,52 +7473,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_externEntry_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Attr_extern_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Attr_extern_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Attr_extern_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Attr_extern_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Attr_extern_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Attr_extern_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Attr_extern_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Attr_extern___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Attr_extern_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Attr_extern_parenthesizer___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -6938,11 +7523,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Attr_extern_parenthesizer(lean_object* x_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Attr_extern_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Attr_extern_parenthesizer___closed__8; +x_7 = l_Lean_Parser_Attr_extern_parenthesizer___closed__7; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Attr_extern___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Attr_extern_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Attr_extern___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Extra(uint8_t builtin, lean_object*); @@ -7128,6 +7743,17 @@ l_Lean_Parser_Attr_simple_formatter___closed__6 = _init_l_Lean_Parser_Attr_simpl lean_mark_persistent(l_Lean_Parser_Attr_simple_formatter___closed__6); l_Lean_Parser_Attr_simple_formatter___closed__7 = _init_l_Lean_Parser_Attr_simple_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Attr_simple_formatter___closed__7); +l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__2); +l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__3); +l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_simple_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Attr_simple_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_simple_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_simple_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_simple_parenthesizer___closed__1); l_Lean_Parser_Attr_simple_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_simple_parenthesizer___closed__2(); @@ -7142,6 +7768,17 @@ l_Lean_Parser_Attr_simple_parenthesizer___closed__6 = _init_l_Lean_Parser_Attr_s lean_mark_persistent(l_Lean_Parser_Attr_simple_parenthesizer___closed__6); l_Lean_Parser_Attr_simple_parenthesizer___closed__7 = _init_l_Lean_Parser_Attr_simple_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Attr_simple_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_Attr_simple_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_macro___elambda__1___lambda__1___closed__1 = _init_l_Lean_Parser_Attr_macro___elambda__1___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_macro___elambda__1___lambda__1___closed__1); l_Lean_Parser_Attr_macro___elambda__1___closed__1 = _init_l_Lean_Parser_Attr_macro___elambda__1___closed__1(); @@ -7204,6 +7841,13 @@ l_Lean_Parser_Attr_macro_formatter___closed__3 = _init_l_Lean_Parser_Attr_macro_ lean_mark_persistent(l_Lean_Parser_Attr_macro_formatter___closed__3); l_Lean_Parser_Attr_macro_formatter___closed__4 = _init_l_Lean_Parser_Attr_macro_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Attr_macro_formatter___closed__4); +l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_macro_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_macro_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_macro_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_macro_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_macro_parenthesizer___closed__1); l_Lean_Parser_Attr_macro_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_macro_parenthesizer___closed__2(); @@ -7212,6 +7856,13 @@ l_Lean_Parser_Attr_macro_parenthesizer___closed__3 = _init_l_Lean_Parser_Attr_ma lean_mark_persistent(l_Lean_Parser_Attr_macro_parenthesizer___closed__3); l_Lean_Parser_Attr_macro_parenthesizer___closed__4 = _init_l_Lean_Parser_Attr_macro_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Attr_macro_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_macro_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_export___elambda__1___closed__1 = _init_l_Lean_Parser_Attr_export___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_export___elambda__1___closed__1); l_Lean_Parser_Attr_export___elambda__1___closed__2 = _init_l_Lean_Parser_Attr_export___elambda__1___closed__2(); @@ -7282,6 +7933,13 @@ l_Lean_Parser_Attr_export_formatter___closed__3 = _init_l_Lean_Parser_Attr_expor lean_mark_persistent(l_Lean_Parser_Attr_export_formatter___closed__3); l_Lean_Parser_Attr_export_formatter___closed__4 = _init_l_Lean_Parser_Attr_export_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Attr_export_formatter___closed__4); +l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_export_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_export_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_export_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_export_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_export_parenthesizer___closed__1); l_Lean_Parser_Attr_export_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_export_parenthesizer___closed__2(); @@ -7290,6 +7948,13 @@ l_Lean_Parser_Attr_export_parenthesizer___closed__3 = _init_l_Lean_Parser_Attr_e lean_mark_persistent(l_Lean_Parser_Attr_export_parenthesizer___closed__3); l_Lean_Parser_Attr_export_parenthesizer___closed__4 = _init_l_Lean_Parser_Attr_export_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Attr_export_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_export_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_export_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_recursor___elambda__1___closed__1 = _init_l_Lean_Parser_Attr_recursor___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_recursor___elambda__1___closed__1); l_Lean_Parser_Attr_recursor___elambda__1___closed__2 = _init_l_Lean_Parser_Attr_recursor___elambda__1___closed__2(); @@ -7352,6 +8017,13 @@ l_Lean_Parser_Attr_recursor_formatter___closed__3 = _init_l_Lean_Parser_Attr_rec lean_mark_persistent(l_Lean_Parser_Attr_recursor_formatter___closed__3); l_Lean_Parser_Attr_recursor_formatter___closed__4 = _init_l_Lean_Parser_Attr_recursor_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Attr_recursor_formatter___closed__4); +l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_recursor_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_recursor_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_recursor_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_recursor_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_recursor_parenthesizer___closed__1); l_Lean_Parser_Attr_recursor_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_recursor_parenthesizer___closed__2(); @@ -7360,6 +8032,13 @@ l_Lean_Parser_Attr_recursor_parenthesizer___closed__3 = _init_l_Lean_Parser_Attr lean_mark_persistent(l_Lean_Parser_Attr_recursor_parenthesizer___closed__3); l_Lean_Parser_Attr_recursor_parenthesizer___closed__4 = _init_l_Lean_Parser_Attr_recursor_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Attr_recursor_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_recursor_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_class___elambda__1___closed__1 = _init_l_Lean_Parser_Attr_class___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_class___elambda__1___closed__1); l_Lean_Parser_Attr_class___elambda__1___closed__2 = _init_l_Lean_Parser_Attr_class___elambda__1___closed__2(); @@ -7422,12 +8101,26 @@ l_Lean_Parser_Attr_class_formatter___closed__2 = _init_l_Lean_Parser_Attr_class_ lean_mark_persistent(l_Lean_Parser_Attr_class_formatter___closed__2); l_Lean_Parser_Attr_class_formatter___closed__3 = _init_l_Lean_Parser_Attr_class_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Attr_class_formatter___closed__3); +l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_class_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_class_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_class_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_class_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_class_parenthesizer___closed__1); l_Lean_Parser_Attr_class_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_class_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Attr_class_parenthesizer___closed__2); l_Lean_Parser_Attr_class_parenthesizer___closed__3 = _init_l_Lean_Parser_Attr_class_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Attr_class_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_class_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_class_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_instance___elambda__1___closed__1 = _init_l_Lean_Parser_Attr_instance___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_instance___elambda__1___closed__1); l_Lean_Parser_Attr_instance___elambda__1___closed__2 = _init_l_Lean_Parser_Attr_instance___elambda__1___closed__2(); @@ -7500,6 +8193,13 @@ l_Lean_Parser_Attr_instance_formatter___closed__4 = _init_l_Lean_Parser_Attr_ins lean_mark_persistent(l_Lean_Parser_Attr_instance_formatter___closed__4); l_Lean_Parser_Attr_instance_formatter___closed__5 = _init_l_Lean_Parser_Attr_instance_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Attr_instance_formatter___closed__5); +l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_instance_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_instance_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_instance_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_instance_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_instance_parenthesizer___closed__1); l_Lean_Parser_Attr_instance_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_instance_parenthesizer___closed__2(); @@ -7510,6 +8210,13 @@ l_Lean_Parser_Attr_instance_parenthesizer___closed__4 = _init_l_Lean_Parser_Attr lean_mark_persistent(l_Lean_Parser_Attr_instance_parenthesizer___closed__4); l_Lean_Parser_Attr_instance_parenthesizer___closed__5 = _init_l_Lean_Parser_Attr_instance_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Attr_instance_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_instance_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__1 = _init_l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__1); l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__2 = _init_l_Lean_Parser_Attr_defaultInstance___elambda__1___closed__2(); @@ -7580,6 +8287,13 @@ l_Lean_Parser_Attr_defaultInstance_formatter___closed__3 = _init_l_Lean_Parser_A lean_mark_persistent(l_Lean_Parser_Attr_defaultInstance_formatter___closed__3); l_Lean_Parser_Attr_defaultInstance_formatter___closed__4 = _init_l_Lean_Parser_Attr_defaultInstance_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Attr_defaultInstance_formatter___closed__4); +l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_defaultInstance_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1); l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2(); @@ -7588,6 +8302,13 @@ l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__3 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__3); l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__4 = _init_l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_defaultInstance_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_externEntry___elambda__1___closed__1 = _init_l_Lean_Parser_Attr_externEntry___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_externEntry___elambda__1___closed__1); l_Lean_Parser_Attr_externEntry___elambda__1___closed__2 = _init_l_Lean_Parser_Attr_externEntry___elambda__1___closed__2(); @@ -7724,6 +8445,13 @@ l_Lean_Parser_Attr_externEntry_formatter___closed__7 = _init_l_Lean_Parser_Attr_ lean_mark_persistent(l_Lean_Parser_Attr_externEntry_formatter___closed__7); l_Lean_Parser_Attr_externEntry_formatter___closed__8 = _init_l_Lean_Parser_Attr_externEntry_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Attr_externEntry_formatter___closed__8); +l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_externEntry_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_externEntry_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_extern_formatter___closed__1 = _init_l_Lean_Parser_Attr_extern_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_extern_formatter___closed__1); l_Lean_Parser_Attr_extern_formatter___closed__2 = _init_l_Lean_Parser_Attr_extern_formatter___closed__2(); @@ -7738,8 +8466,13 @@ l_Lean_Parser_Attr_extern_formatter___closed__6 = _init_l_Lean_Parser_Attr_exter lean_mark_persistent(l_Lean_Parser_Attr_extern_formatter___closed__6); l_Lean_Parser_Attr_extern_formatter___closed__7 = _init_l_Lean_Parser_Attr_extern_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Attr_extern_formatter___closed__7); -l_Lean_Parser_Attr_extern_formatter___closed__8 = _init_l_Lean_Parser_Attr_extern_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Attr_extern_formatter___closed__8); +l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__1); +l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_extern_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_extern_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_externEntry_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_externEntry_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_externEntry_parenthesizer___closed__1); l_Lean_Parser_Attr_externEntry_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_externEntry_parenthesizer___closed__2(); @@ -7756,6 +8489,13 @@ l_Lean_Parser_Attr_externEntry_parenthesizer___closed__7 = _init_l_Lean_Parser_A lean_mark_persistent(l_Lean_Parser_Attr_externEntry_parenthesizer___closed__7); l_Lean_Parser_Attr_externEntry_parenthesizer___closed__8 = _init_l_Lean_Parser_Attr_externEntry_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Attr_externEntry_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_externEntry_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Attr_extern_parenthesizer___closed__1 = _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Attr_extern_parenthesizer___closed__1); l_Lean_Parser_Attr_extern_parenthesizer___closed__2 = _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__2(); @@ -7770,8 +8510,13 @@ l_Lean_Parser_Attr_extern_parenthesizer___closed__6 = _init_l_Lean_Parser_Attr_e lean_mark_persistent(l_Lean_Parser_Attr_extern_parenthesizer___closed__6); l_Lean_Parser_Attr_extern_parenthesizer___closed__7 = _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Attr_extern_parenthesizer___closed__7); -l_Lean_Parser_Attr_extern_parenthesizer___closed__8 = _init_l_Lean_Parser_Attr_extern_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Attr_extern_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Attr_extern_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Parser/Command.c b/stage0/stdlib/Lean/Parser/Command.c index 47299fd2de3d..06ba583f4771 100644 --- a/stage0/stdlib/Lean/Parser/Command.c +++ b/stage0/stdlib/Lean/Parser/Command.c @@ -16,8 +16,8 @@ extern "C" { static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_noncomputableSection_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_deriving_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__6; -static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_check_declRange___closed__6; static lean_object* l_Lean_Parser_Tactic_set__option_parenthesizer___closed__3; @@ -25,31 +25,34 @@ static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_check__failure___closed__5; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__11; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__38; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_opaque___closed__10; -static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__23; LEAN_EXPORT lean_object* l_Lean_Parser_Command_eraseAttr; +static lean_object* l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_computedField_formatter___closed__3; -static lean_object* l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__22; static lean_object* l_Lean_Parser_Command_check_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange___closed__4; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__18; static lean_object* l_Lean_Parser_Command_init__quot___closed__3; static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_classInductive_formatter___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__21; static lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_quot_docString___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__20; static lean_object* l_Lean_Parser_Command_classTk___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__10; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_print___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__1; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_export_formatter___closed__6; lean_object* l_Lean_Parser_many1Indent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -57,6 +60,7 @@ static lean_object* l_Lean_Parser_Command_noncomputableSection_formatter___close static lean_object* l_Lean_Parser_Command_print_parenthesizer___closed__3; lean_object* l_Lean_Parser_nonReservedSymbol_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_def___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2; @@ -71,8 +75,8 @@ static lean_object* l_Lean_Parser_Command_openRenaming_formatter___closed__4; static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_section___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structure_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_openDecl_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange___closed__4; static lean_object* l_Lean_Parser_Command_open___closed__3; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__7; @@ -97,23 +101,28 @@ static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_declRange___closed__1; -static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__21; LEAN_EXPORT lean_object* l_Lean_Parser_Command_check___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namespace_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__11; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__9; static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structureTk___closed__2; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Tactic_set__option___closed__9; static lean_object* l_Lean_Parser_Command_instance___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange___closed__2; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__7; static lean_object* l_Lean_Parser_Command_openHiding_formatter___closed__3; static lean_object* l_Lean_Parser_Command_variable_formatter___closed__5; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__2; static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Command_optionValue_formatter___closed__5; static lean_object* l_Lean_Parser_Command_openScoped_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_quot___closed__11; @@ -135,6 +144,7 @@ static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_optDefDeriving_formatter___closed__5; static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__2; lean_object* l_Lean_Parser_tokenAntiquotFn(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_synth_declRange___closed__3; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__3; @@ -142,12 +152,14 @@ static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_nonrec_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_quot___closed__8; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structure_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_axiom_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_axiom___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__1; static lean_object* l_Lean_Parser_Command_section___closed__3; static lean_object* l_Lean_Parser_Command_declVal___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__6; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__14; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_mutual___closed__4; @@ -158,9 +170,10 @@ static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_check_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structCtor_formatter___closed__1; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__15; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_formatter(lean_object*); static lean_object* l_Lean_Parser_Tactic_set__option___closed__1; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__13; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_exit___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__9; @@ -171,8 +184,10 @@ static lean_object* l_Lean_Parser_Command_extends___closed__2; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__11; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__13; static lean_object* l_Lean_Parser_Command_open___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__50; static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_deriving_parenthesizer___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openDecl; static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__3; static lean_object* l_Lean_Parser_Command_nonrec___elambda__1___closed__8; @@ -186,7 +201,6 @@ static lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer___closed lean_object* l_Lean_Parser_ParserState_mkError(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_instance___closed__4; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__4; -static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__28; static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_declRange___closed__3; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__12; @@ -194,21 +208,28 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange___cl static lean_object* l_Lean_Parser_Command_openScoped_formatter___closed__2; static lean_object* l_Lean_Parser_Term_open___closed__6; static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_open_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_visibility; +static lean_object* l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declId_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__28; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__1; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__10; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_section(lean_object*); static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Command_inductive___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_def_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_exit_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__2; static lean_object* l_Lean_Parser_Command_optDeriving___closed__1; static lean_object* l_Lean_Parser_Term_set__option___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_reduce_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -218,7 +239,6 @@ static lean_object* l_Lean_Parser_Command_computedFields___closed__8; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__3; static lean_object* l_Lean_Parser_Command_declSig_parenthesizer___closed__1; lean_object* l_Lean_Parser_Term_attributes_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__23; static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRange___closed__4; static lean_object* l_Lean_Parser_Command_terminationBy_parenthesizer___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namespace_declRange(lean_object*); @@ -229,6 +249,7 @@ static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___cl static lean_object* l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__5; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_variable___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationBy; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__2; static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__7; @@ -243,6 +264,7 @@ lean_object* l_Lean_Parser_Term_leftArrow_formatter(lean_object*, lean_object*, static lean_object* l_Lean_Parser_Command_synth_parenthesizer___closed__3; lean_object* l_Lean_Parser_ppSpace_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_synth___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_print_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_declRange___closed__2; static lean_object* l_Lean_Parser_Tactic_open___closed__5; static lean_object* l_Lean_Parser_Command_optDeriving_parenthesizer___closed__6; @@ -254,8 +276,11 @@ static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___cl static lean_object* l_Lean_Parser_Command_example___closed__3; lean_object* l_Lean_Parser_ppGroup_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Term_attrKind_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_ctor___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__2; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__48; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_structCtor___closed__9; static lean_object* l_Lean_Parser_Command_structureTk___closed__4; @@ -266,7 +291,10 @@ static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__13 static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__34; static lean_object* l_Lean_Parser_Command_theorem___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__2; static lean_object* l_Lean_Parser_Command_universe___elambda__1___closed__10; lean_object* l_Lean_Parser_Term_letDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__5; @@ -274,6 +302,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_classInductive; static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange___closed__1; static lean_object* l_Lean_Parser_Command_check___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenaming_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_instance___closed__1; static lean_object* l_Lean_Parser_Command_whereStructField___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_export___closed__3; @@ -281,7 +310,9 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___c static lean_object* l_Lean_Parser_Command_open_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Tactic_set__option___closed__2; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Term_quot___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_attribute___closed__7; static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_attribute_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -291,7 +322,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_noncomputable; static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__8; lean_object* l_Lean_Parser_Term_matchAlts(lean_object*); -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_open_formatter___closed__2; static lean_object* l_Lean_Parser_Command_deriving_parenthesizer___closed__5; extern lean_object* l_Lean_Parser_leadPrec; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__6; @@ -303,28 +334,32 @@ static lean_object* l_Lean_Parser_Command_terminationByCore_parenthesizer___clos static lean_object* l_Lean_Parser_Command_structCtor___closed__4; static lean_object* l_Lean_Parser_Command_opaque___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__7; -static lean_object* l_Lean_Parser_Command_visibility_formatter___closed__1; static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_terminationByCore_formatter___closed__5; lean_object* l_Lean_Parser_many(lean_object*); static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__3; static lean_object* l_Lean_Parser_Command_extends_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_declRange___closed__4; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__3; lean_object* l_Lean_Parser_Term_bracketedBinder(uint8_t); static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__22; static lean_object* l_Lean_Parser_Command_computedFields___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_print_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_print_declRange___closed__4; lean_object* l_Lean_Parser_Term_attributes___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers___boxed(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__1; static lean_object* l_Lean_Parser_Command_extends_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_nonrec___closed__5; static lean_object* l_Lean_Parser_Command_noncomputableSection_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_end_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDefDeriving_formatter___closed__3; @@ -339,6 +374,7 @@ static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__22; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2; lean_object* l_Lean_Parser_setLhsPrecFn(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__11; static lean_object* l_Lean_Parser_Term_quot___closed__4; lean_object* l_Lean_PrettyPrinter_Parenthesizer_lookahead_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -346,14 +382,15 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_reduce; static lean_object* l_Lean_Parser_Command_variable_formatter___closed__3; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_resolve__name_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_def_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenaming; static lean_object* l_Lean_Parser_Command_openScoped_formatter___closed__1; static lean_object* l_Lean_Parser_Command_partial___elambda__1___closed__3; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__33; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange___closed__7; static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__26; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_declRange___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classInductive___elambda__1(lean_object*, lean_object*); @@ -364,6 +401,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRang static lean_object* l_Lean_Parser_Command_terminationByCore___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_declModifiers___closed__8; static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__2; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_optDeclSig___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__5; @@ -376,10 +416,9 @@ static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_attribute_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__7; static lean_object* l_Lean_Parser_Command_mutual___closed__8; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_section_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_set__option_formatter___closed__5; -static lean_object* l_Lean_Parser_Command_visibility_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange___closed__4; @@ -396,23 +435,29 @@ static lean_object* l_Lean_Parser_Command_example_formatter___closed__3; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__5; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__14; -static lean_object* l_Lean_Parser_Command_openDecl_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__2; static lean_object* l_Lean_Parser_Command_optionValue___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__19; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_eval_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structCtor_formatter___closed__2; lean_object* l_Lean_Parser_symbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eval(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_opaque___closed__3; static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_universe_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__39; +static lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__1; static lean_object* l_Lean_Parser_Command_universe___closed__7; static lean_object* l_Lean_Parser_Command_printAxioms_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__23; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__13; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__13; static lean_object* l_Lean_Parser_Command_openScoped___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -422,6 +467,8 @@ static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__19; static lean_object* l_Lean_Parser_Command_openScoped___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openOnly; static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_declRange___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_print_parenthesizer(lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__24; @@ -434,10 +481,13 @@ static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__8; static lean_object* l_Lean_Parser_Command_in___closed__3; static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__24; +static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_opaque___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_export_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Term_doSeq___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__6; @@ -450,9 +500,11 @@ static lean_object* l_Lean_Parser_Command_computedField___closed__10; static lean_object* l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__3; lean_object* l_Lean_PrettyPrinter_Formatter_atomic_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__41; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__14; LEAN_EXPORT lean_object* l_Lean_Parser_Command_synth___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__1; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__7; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__2; @@ -464,19 +516,25 @@ static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__8; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_declaration___closed__7; -static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__16; +static lean_object* l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__2; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__8; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__9; static lean_object* l_Lean_Parser_Command_section___closed__5; static lean_object* l_Lean_Parser_Command_openSimple___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange___closed__4; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__18; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Command_in_declRange___closed__7; lean_object* l_Lean_Parser_group_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_declaration_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__19; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_end_formatter___closed__3; static lean_object* l_Lean_Parser_Command_def_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__6; @@ -485,16 +543,22 @@ static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_declRange___closed__3; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__1; static lean_object* l_Lean_Parser_Command_nonrec_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_set__option___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_section_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_terminationHint1_formatter___closed__1; static lean_object* l_Lean_Parser_Command_classTk___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_classTk___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_opaque___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_exit___closed__1; @@ -506,10 +570,12 @@ static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__18; static lean_object* l_Lean_Parser_Tactic_set__option_formatter___closed__3; static lean_object* l_Lean_Parser_Tactic_set__option_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_partial_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_declRange___closed__2; extern lean_object* l_Lean_Parser_pushNone; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__2; static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declVal___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__4; @@ -524,6 +590,7 @@ static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_structureTk___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__13; static lean_object* l_Lean_Parser_Command_opaque___closed__5; static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__11; @@ -542,13 +609,14 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHintMany_formatter(lea static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationBy_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__2; static lean_object* l_Lean_Parser_Command_deriving___closed__7; static lean_object* l_Lean_Parser_Command_eval_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__4; static lean_object* l_Lean_Parser_Command_terminationByElement___closed__10; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_synth___closed__2; -static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_check___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openHiding_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -563,6 +631,7 @@ static lean_object* l_Lean_Parser_Command_openHiding_formatter___closed__7; static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_openScoped___closed__5; static lean_object* l_Lean_Parser_Command_universe_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_abbrev___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_declaration___closed__3; @@ -572,20 +641,24 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_abbrev; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__14; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__27; lean_object* l_Lean_Parser_Term_binderTactic___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__9; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__4; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__16; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mutual_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__13; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_in___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_open_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__1; extern lean_object* l_Lean_Parser_ident; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_section_declRange___closed__7; @@ -600,6 +673,7 @@ static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange___closed__3; static lean_object* l_Lean_Parser_Command_declModifiers___closed__2; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__22; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_unsafe___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_open; @@ -609,21 +683,27 @@ static lean_object* l_Lean_Parser_Command_universe_formatter___closed__4; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__6; static lean_object* l_Lean_Parser_Tactic_open___closed__6; static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_section___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_axiom___closed__6; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declValEqns___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__14; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__20; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_quot_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_theorem___closed__5; static lean_object* l_Lean_Parser_Command_declVal___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_in_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__7; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange___closed__5; -static lean_object* l_Lean_Parser_Command_openDecl_formatter___closed__8; lean_object* l_id___rarg___boxed(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__1; lean_object* l_Lean_Parser_Term_bracketedBinder_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_end_formatter___closed__1; static lean_object* l_Lean_Parser_Command_abbrev___closed__5; static lean_object* l_Lean_Parser_Command_section___closed__1; static lean_object* l_Lean_Parser_Command_example___closed__6; @@ -638,6 +718,7 @@ static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__1 static lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_terminationHint1___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_private_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structInstBinder_formatter___closed__8; static lean_object* l_Lean_Parser_Command_optNamedPrio___closed__2; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__3; @@ -651,11 +732,14 @@ static lean_object* l_Lean_Parser_Tactic_open___closed__3; static lean_object* l_Lean_Parser_Command_visibility___closed__1; static lean_object* l_Lean_Parser_Term_precheckedQuot_formatter___closed__1; static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__28; static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_reduce___elambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declValSimple___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Command_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_namedPrio___closed__3; @@ -672,6 +756,9 @@ static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__5; static lean_object* l_Lean_Parser_Command_inductive___closed__5; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Command_quot_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_instance_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structure_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_section___closed__4; static lean_object* l_Lean_Parser_Command_quot___closed__7; static lean_object* l_Lean_Parser_Command_check___elambda__1___closed__3; @@ -681,6 +768,7 @@ static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__6; static lean_object* l_Lean_Parser_Command_namespace___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_def; static lean_object* l_Lean_Parser_Command_end___elambda__1___closed__10; +static lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_declSig___closed__2; static lean_object* l_Lean_Parser_Term_quot_formatter___closed__7; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__5; @@ -688,13 +776,12 @@ static lean_object* l_Lean_Parser_Command_structure___closed__2; lean_object* l_Lean_Parser_priorityParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_structFields___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__43; static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__4; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__14; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_export(lean_object*); -static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__28; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mutual; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__2; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_set__option___closed__6; static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__17; @@ -715,8 +802,6 @@ lean_object* l_Lean_Parser_Term_attributes_formatter(lean_object*, lean_object*, static lean_object* l_Lean_Parser_Command_resolve__name_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_reduce___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_namedPrio___closed__5; -static lean_object* l_Lean_Parser_Command_visibility_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__17; lean_object* l_Lean_Parser_pushNone___elambda__1___boxed(lean_object*); static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_computedFields___closed__4; @@ -731,9 +816,9 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_example; static lean_object* l_Lean_Parser_Command_classTk___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__21; static lean_object* l_Lean_Parser_Command_theorem___closed__3; -static lean_object* l_Lean_Parser_Command_openRenaming_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_declRange___closed__6; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__24; static lean_object* l_Lean_Parser_Command_opaque___closed__6; lean_object* l_Lean_Parser_orelseFn(lean_object*, lean_object*, lean_object*, lean_object*); @@ -744,6 +829,7 @@ static lean_object* l_Lean_Parser_Command_classTk_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_printAxioms_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declId___closed__4; static lean_object* l_Lean_Parser_Command_openDecl_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_end; static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__4; static lean_object* l_Lean_Parser_Command_initialize___closed__1; @@ -752,24 +838,26 @@ static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__2; -static lean_object* l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_end_formatter___closed__2; static lean_object* l_Lean_Parser_Command_attribute_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_openHiding___closed__7; static lean_object* l_Lean_Parser_Command_unsafe_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_noncomputable___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__13; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__16; static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange___closed__5; static lean_object* l_Lean_Parser_Command_openSimple___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__1; static lean_object* l_Lean_Parser_Command_instance___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_instance_formatter___closed__3; static lean_object* l_Lean_Parser_Command_whereStructField_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__2; lean_object* l_Lean_Parser_ParserState_mkTrailingNode(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_derivingClasses_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_openScoped_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_declRange___closed__5; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__15; @@ -777,25 +865,25 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___cl static lean_object* l_Lean_Parser_Term_precheckedQuot_formatter___closed__2; static lean_object* l_Lean_Parser_Command_init__quot_formatter___closed__1; static lean_object* l_Lean_Parser_Command_openRenaming_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_abbrev___elambda__1___closed__4; lean_object* l_Lean_Parser_Command_docComment_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__1; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__8; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__32; static lean_object* l_Lean_Parser_Command_openRenaming___closed__4; static lean_object* l_Lean_Parser_Command_print_formatter___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__32; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_declRange___closed__4; static lean_object* l_Lean_Parser_Command_openRenaming___closed__9; static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__10; -static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__12; static lean_object* l_Lean_Parser_Term_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Command_openDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__7; @@ -805,10 +893,11 @@ static lean_object* l_Lean_Parser_Command_terminationByCore___closed__6; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__11; lean_object* l_Lean_Parser_addBuiltinParser(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__10; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_classInductive_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_declVal___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__13; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__44; static lean_object* l_Lean_Parser_Command_openSimple___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_export___closed__12; static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__8; @@ -817,20 +906,22 @@ static lean_object* l_Lean_Parser_Command_check__failure___elambda__1___closed__ static lean_object* l_Lean_Parser_Command_whereStructField___closed__6; lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Parser_Command_declId_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structFields; -static lean_object* l_Lean_Parser_Command_openDecl_formatter___closed__4; static lean_object* l_Lean_Parser_Command_abbrev___closed__3; static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__6; lean_object* l_Lean_Parser_ppIndent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_check_formatter___closed__3; static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__8; -static lean_object* l_Lean_Parser_Command_terminationSuffix_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structInstBinder_formatter___closed__6; static lean_object* l_Lean_Parser_Command_in___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_openDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_axiom___elambda__1___closed__10; @@ -842,6 +933,7 @@ static lean_object* l_Lean_Parser_Command_declValEqns___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_optDeriving___closed__6; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__20; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__2; static lean_object* l_Lean_Parser_Command_printAxioms___closed__5; static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_abbrev___closed__7; @@ -853,9 +945,12 @@ static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structFields_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc___closed__4; static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_variable_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_quot___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__6; @@ -872,7 +967,6 @@ static lean_object* l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_reduce___elambda__1___closed__11; lean_object* l_Lean_Parser_Term_attrInstance_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_exit___closed__6; -static lean_object* l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_terminationHintMany_formatter___closed__2; static lean_object* l_Lean_Parser_Command_eval_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__12; @@ -882,10 +976,11 @@ static lean_object* l_Lean_Parser_Command_optionValue_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationBy___elambda__1(lean_object*, lean_object*); lean_object* l_Lean_Parser_unicodeSymbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__8; -static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__26; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__17; static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_universe_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -904,6 +999,7 @@ static lean_object* l_Lean_Parser_Command_eval___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_attribute___closed__12; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__1; lean_object* l_Lean_Parser_Tactic_tacticSeq___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_synth_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_whereStructField___closed__4; static lean_object* l_Lean_Parser_Command_synth___closed__7; @@ -911,6 +1007,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_extends; static lean_object* l_Lean_Parser_Command_deriving___closed__5; static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_declRange___closed__7; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_unsafe_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -926,9 +1023,12 @@ static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_in(lean_object*); static lean_object* l_Lean_Parser_Command_structInstBinder___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_exit_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openSimple; +static lean_object* l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_quot_formatter___closed__8; static lean_object* l_Lean_Parser_Command_classTk_parenthesizer___closed__1; @@ -940,11 +1040,11 @@ static lean_object* l_Lean_Parser_Command_end_formatter___closed__4; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_declRange___closed__4; static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange___closed__6; lean_object* l_Lean_Parser_checkPrecFn___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_instance; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__17; lean_object* l_Lean_Parser_sepBy1_formatter(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__5; @@ -959,16 +1059,19 @@ static lean_object* l_Lean_Parser_Command_initialize___closed__7; static lean_object* l_Lean_Parser_Command_print_formatter___closed__4; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_terminationHint1___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_instance___closed__8; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__8; static lean_object* l_Lean_Parser_Command_terminationSuffix___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openOnly___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_reduce___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_decreasingBy_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__10; -static lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__7; static lean_object* l_Lean_Parser_Command_openSimple___elambda__1___closed__8; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__17; +static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_Command_initializeKeyword_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structFields___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__9; @@ -992,47 +1095,49 @@ static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed_ static lean_object* l_Lean_Parser_Command_unsafe_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_instance___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__2; static lean_object* l_Lean_Parser_Term_precheckedQuot_formatter___closed__4; static lean_object* l_Lean_Parser_Command_classInductive_formatter___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_set__option_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_reduce___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_resolve__name___elambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__8; static lean_object* l_Lean_Parser_Term_set__option_formatter___closed__6; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__14; lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_mkAntiquot_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_open___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__20; lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__29; static lean_object* l_Lean_Parser_Command_openSimple___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange___closed__3; -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__3; static lean_object* l_Lean_Parser_Command_set__option___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange___closed__4; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_derivingClasses_formatter___closed__5; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declId; +static lean_object* l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_openOnly___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_extends_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_declRange___closed__4; static lean_object* l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_export___closed__11; -static lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__3; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_quot; static lean_object* l_Lean_Parser_Command_namespace___closed__5; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structure_formatter___closed__10; static lean_object* l_Lean_Parser_Command_optDeriving___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Command_noncomputable_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHint1(lean_object*); @@ -1053,6 +1158,8 @@ static lean_object* l_Lean_Parser_Command_declId_formatter___closed__2; lean_object* l_Lean_Parser_checkColGeFn___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_whereStructField___elambda__1___closed__1; +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_print_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__9; static lean_object* l_Lean_Parser_Command_classTk___closed__5; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__5; @@ -1084,9 +1191,7 @@ static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__ static lean_object* l_Lean_Parser_Command_private___closed__7; static lean_object* l_Lean_Parser_Command_declSig___closed__1; static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__11; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__26; static lean_object* l_Lean_Parser_Command_mutual___closed__1; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__20; static lean_object* l_Lean_Parser_Command_declId_formatter___closed__9; static lean_object* l_Lean_Parser_Command_declId___closed__3; static lean_object* l_Lean_Parser_Command_namespace___closed__3; @@ -1103,6 +1208,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving(lean_object static lean_object* l_Lean_Parser_Command_declSig_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedPrio_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_deriving_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__20; static lean_object* l_Lean_Parser_Command_quot_formatter___closed__6; static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__5; @@ -1113,6 +1219,8 @@ static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange___closed__3; static lean_object* l_Lean_Parser_Command_partial_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__4; @@ -1121,29 +1229,33 @@ static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__20; static lean_object* l_Lean_Parser_Command_private_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__10; lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__45; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__30; static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__1; static lean_object* l_Lean_Parser_Command_openScoped___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_in_declRange___closed__5; static lean_object* l_Lean_Parser_Tactic_open___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__10; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__40; static lean_object* l_Lean_Parser_Command_namespace___elambda__1___closed__12; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__2; -static lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__4; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__3; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1; lean_object* l_Lean_Parser_Term_binderTactic_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__4; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__9; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__21; -static lean_object* l_Lean_Parser_Command_openDecl_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_open___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_variable___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_extends___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_def_formatter___closed__2; static lean_object* l_Lean_Parser_Command_deriving___closed__6; static lean_object* l_Lean_Parser_Command_mutual___closed__6; static lean_object* l_Lean_Parser_Command_private___closed__5; @@ -1168,6 +1280,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declId___elambda__1(lean_object*, static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange___closed__6; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__13; static lean_object* l_Lean_Parser_Command_declId_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__2; static lean_object* l_Lean_Parser_Command_print_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_declaration___closed__12; @@ -1178,13 +1291,18 @@ static lean_object* l_Lean_Parser_Tactic_open_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_synth_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_quot_declRange___closed__5; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_def_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_classTk___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_nonrec; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_namespace___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_declRange(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_set__option___elambda__1___closed__2; lean_object* l_Lean_Parser_many1Fn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_whereStructInst___closed__8; @@ -1192,11 +1310,15 @@ static lean_object* l_Lean_Parser_Command_openDecl_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_print_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__6; static lean_object* l_Lean_Parser_Command_initialize___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__30; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenaming___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declaration___closed__16; +static lean_object* l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__1; static lean_object* l_Lean_Parser_Command_theorem___closed__6; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optionValue___elambda__1(lean_object*, lean_object*); @@ -1204,6 +1326,9 @@ static lean_object* l_Lean_Parser_Command_openHiding___closed__4; static lean_object* l_Lean_Parser_Command_inductive___closed__7; static lean_object* l_Lean_Parser_Command_axiom_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_unsafe; +static lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__15; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__35; static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_structure___closed__6; @@ -1217,6 +1342,7 @@ static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___cl static lean_object* l_Lean_Parser_Command_synth___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__2; lean_object* l_Lean_Parser_optional(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_inductive_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__24; @@ -1224,9 +1350,11 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration(lean_obj static lean_object* l_Lean_Parser_Command_check___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__13; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_declRange___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__37; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__13; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__18; +static lean_object* l___regBuiltin_Lean_Parser_Command_open_formatter___closed__1; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__19; static lean_object* l_Lean_Parser_Command_initialize___closed__8; static lean_object* l_Lean_Parser_Command_namedPrio___closed__1; @@ -1265,11 +1393,14 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_structure; static lean_object* l_Lean_Parser_Command_declModifiers___closed__6; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc___closed__6; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2; static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__18; lean_object* l_Lean_Parser_registerAliasCore___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__36; @@ -1277,13 +1408,14 @@ static lean_object* l_Lean_Parser_Command_namespace_formatter___closed__3; static lean_object* l_Lean_Parser_Command_openSimple_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenamingItem_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_def_formatter___closed__1; static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__20; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__11; lean_object* l_Lean_Parser_strLit___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__20; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__7; static lean_object* l_Lean_Parser_Command_private_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_print_formatter___closed__1; @@ -1302,11 +1434,12 @@ static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__7; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_protected_formatter___closed__2; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_classInductive_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__15; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__1; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__19; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_end_formatter___closed__2; static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_printAxioms___closed__3; @@ -1319,11 +1452,12 @@ static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_section_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_axiom_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Command_eval_declRange___closed__6; static lean_object* l_Lean_Parser_Command_decreasingBy___closed__5; -static lean_object* l_Lean_Parser_Command_structure_formatter___closed__21; static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Tactic_set__option___elambda__1___closed__1; @@ -1332,32 +1466,37 @@ static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___c lean_object* l_Lean_PrettyPrinter_Formatter_checkColGe_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_private___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__3; static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_in_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__4; static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_init__quot_formatter___closed__2; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__20; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_declRange___closed__3; -static lean_object* l_Lean_Parser_Command_terminationBy_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_computedFields_formatter___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openHiding_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_abbrev___elambda__1___closed__5; lean_object* l_Lean_ppIndent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__16; -static lean_object* l_Lean_Parser_Command_openDecl_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange___closed__4; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__23; +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; +static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_noncomputable___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__5; static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__3; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange(lean_object*); +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_unsafe_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__1; static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_nonrec_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_open_declRange___closed__1; @@ -1366,6 +1505,7 @@ static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__4; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__27; static lean_object* l_Lean_Parser_Command_eval___elambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_in_formatter___closed__3; @@ -1375,26 +1515,34 @@ static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__10; lean_object* l_Lean_ppHardLineUnlessUngrouped_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_synth; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_abbrev___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_synth_formatter(lean_object*); extern lean_object* l_Lean_Parser_Term_binderDefault; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_example_parenthesizer(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__42; +static lean_object* l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__3; static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_visibility_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_in_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationByCore_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_openSimple_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_decreasingBy_formatter___closed__2; -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474_(lean_object*); static lean_object* l_Lean_Parser_Command_reduce___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_initialize___closed__4; static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optNamedPrio_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_whereStructField___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_declVal___closed__4; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__17; +static lean_object* l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_resolve__name; static lean_object* l_Lean_Parser_Command_declValSimple___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declValEqns___elambda__1(lean_object*, lean_object*); @@ -1402,8 +1550,10 @@ static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__ static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__9; static lean_object* l_Lean_Parser_Command_example_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_check__failure_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__37; static lean_object* l_Lean_Parser_Command_attribute___closed__6; static lean_object* l_Lean_Parser_Command_optionValue_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_in; static lean_object* l_Lean_Parser_Command_opaque___elambda__1___closed__10; @@ -1411,19 +1561,17 @@ static lean_object* l_Lean_Parser_Command_openHiding___closed__8; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__16; static lean_object* l_Lean_Parser_Command_attribute_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__23; static lean_object* l_Lean_Parser_Command_declSig_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_terminationBy_formatter___closed__7; -static lean_object* l_Lean_Parser_Command_visibility_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structure_formatter___closed__6; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__8; -static lean_object* l_Lean_Parser_Command_builtin__initialize_formatter___closed__3; static lean_object* l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declaration___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange___closed__7; static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__11; static lean_object* l_Lean_Parser_Command_terminationBy___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__3; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__9; @@ -1436,23 +1584,26 @@ static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_open___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_terminationBy_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange___closed__5; static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_open_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_classTk_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__9; -LEAN_EXPORT lean_object* l_Lean_Parser_Command_builtin__initialize_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_set__option_formatter___closed__5; static lean_object* l_Lean_Parser_Command_attribute___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange___closed__5; static lean_object* l_Lean_Parser_Command_classInductive___closed__7; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__19; static lean_object* l_Lean_Parser_Command_optionValue___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_ctor_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_openSimple___closed__1; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__3; @@ -1463,6 +1614,7 @@ static lean_object* l_Lean_Parser_Command_quot_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_check_formatter___closed__2; static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__6; @@ -1476,7 +1628,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declValEqns_formatter(lean_object static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange___closed__2; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__3; -static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationByCore___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classInductive_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_check_declRange___closed__5; @@ -1485,6 +1637,7 @@ static lean_object* l_Lean_Parser_Command_opaque_formatter___closed__2; static lean_object* l_Lean_Parser_Command_whereStructField___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_in_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_attribute; +static lean_object* l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__20; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openScoped_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1497,6 +1650,7 @@ lean_object* l_Lean_Parser_nonReservedSymbolFnAux(lean_object*, lean_object*, le static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_quot_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_declRange___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_declRange___closed__5; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__24; static lean_object* l_Lean_Parser_Command_partial___elambda__1___closed__6; @@ -1508,9 +1662,13 @@ static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__6; static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__9; static lean_object* l_Lean_Parser_Tactic_set__option_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_in___elambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__3; static lean_object* l_Lean_Parser_Command_set__option___closed__10; static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__10; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__18; static lean_object* l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_whereStructField_formatter___closed__2; @@ -1522,28 +1680,34 @@ static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_decreasingBy_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__21; extern lean_object* l_Lean_Parser_Term_optType; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__1; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__10; static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__12; -static lean_object* l_Lean_Parser_Command_openDecl_formatter___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_section_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_declId___closed__2; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_declVal___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_computedField___closed__5; static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_terminationByElement___closed__11; static lean_object* l_Lean_Parser_Command_reduce_formatter___closed__3; static lean_object* l_Lean_Parser_Command_openHiding___closed__9; static lean_object* l_Lean_Parser_Command_exit_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_example_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__23; static lean_object* l_Lean_Parser_Command_classInductive___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_print_declRange(lean_object*); static lean_object* l_Lean_Parser_Tactic_set__option_parenthesizer___closed__2; -static lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__5; static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_open___closed__2; static lean_object* l_Lean_Parser_Command_terminationHint1___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__6; @@ -1560,6 +1724,7 @@ lean_object* l_Lean_Parser_checkLhsPrecFn(lean_object*, lean_object*, lean_objec LEAN_EXPORT lean_object* l_Lean_Parser_Command_eval_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_attribute___closed__3; static lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namedPrio_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__16; static lean_object* l_Lean_Parser_Tactic_set__option___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_openOnly___elambda__1___closed__7; @@ -1575,7 +1740,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_quot___elambda__1(lean_object*, l static lean_object* l___regBuiltin_Lean_Parser_Command_quot_declRange___closed__7; static lean_object* l_Lean_Parser_Command_declModifiers___closed__5; static lean_object* l_Lean_Parser_Command_structureTk___closed__1; -static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__13; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__1; static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__4; @@ -1595,14 +1759,15 @@ static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__ static lean_object* l_Lean_Parser_Command_openRenaming_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mutual___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_computedField_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__4; lean_object* l_Lean_Parser_Term_bracketedBinder_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_instance_formatter___closed__2; -static lean_object* l_Lean_Parser_Command_builtin__initialize_formatter___closed__5; static lean_object* l_Lean_Parser_Command_terminationByCore_formatter___closed__2; static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_opaque_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_openDecl___closed__6; static lean_object* l_Lean_Parser_Command_protected_formatter___closed__1; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__9; @@ -1615,6 +1780,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_openScoped; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__21; static lean_object* l___regBuiltin_Lean_Parser_Command_check_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_printAxioms_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__2; static lean_object* l_Lean_Parser_Command_instance___elambda__1___closed__14; extern lean_object* l_Lean_Parser_Term_letDecl; static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__4; @@ -1625,11 +1791,13 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1(lean_obj static lean_object* l_Lean_Parser_Command_decreasingBy_formatter___closed__1; static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_init__quot_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_synth_declRange___closed__7; static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__4; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__28; lean_object* l_Lean_Parser_Command_commentBody_parenthesizer___boxed(lean_object*); -static lean_object* l_Lean_Parser_Command_openRenaming_parenthesizer___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__2; static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__6; lean_object* l_Lean_Parser_nonReservedSymbolInfo(lean_object*, uint8_t); @@ -1647,9 +1815,10 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDefDeriving; LEAN_EXPORT lean_object* l_Lean_Parser_Command_export___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_declId_formatter___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__14; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_classTk_formatter___closed__1; -static lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__3; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__5; lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_addQuotDepthFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__10; static lean_object* l_Lean_Parser_Command_openHiding_formatter___closed__6; @@ -1661,19 +1830,23 @@ static lean_object* l_Lean_Parser_Command_optionValue_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange___closed__3; static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__7; -static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__26; static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__11; static lean_object* l_Lean_Parser_Command_openSimple_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_declRange___closed__1; static lean_object* l_Lean_Parser_Command_initialize___closed__3; static lean_object* l_Lean_Parser_Command_mutual___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHintMany(lean_object*); static lean_object* l_Lean_Parser_Command_classTk___closed__1; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_eval___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_terminationByCore___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_reduce___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__10; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namespace(lean_object*); @@ -1692,6 +1865,7 @@ static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__2; lean_object* l_Lean_Parser_notSymbol_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_universe___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_variable___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_private_formatter___closed__2; lean_object* l_Lean_Parser_Term_whereDecls_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__19; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__5; @@ -1709,10 +1883,13 @@ static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_protected___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms(lean_object*); static lean_object* l_Lean_Parser_Command_check__failure___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_private_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_end_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_set__option_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_set__option___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_theorem_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_nonrec___elambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHintMany___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structureTk___elambda__1___closed__3; @@ -1723,12 +1900,14 @@ static lean_object* l_Lean_Parser_Command_end_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_partial___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_open_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__7; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_print___closed__3; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__18; +static lean_object* l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openSimple_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__16; static lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__7; @@ -1740,13 +1919,17 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___c static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_opaque___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_optNamedPrio_formatter___closed__1; static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__17; LEAN_EXPORT lean_object* l_Lean_Parser_Command_axiom_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_openDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__22; static lean_object* l_Lean_Parser_Command_axiom___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_eval___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__2; @@ -1789,8 +1972,8 @@ static lean_object* l_Lean_Parser_Command_universe_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_example_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classTk___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_variable___closed__1; -static lean_object* l_Lean_Parser_Command_optNamedPrio_formatter___closed__2; -static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_check_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_check_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__18; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namespace___elambda__1(lean_object*, lean_object*); @@ -1802,15 +1985,21 @@ static lean_object* l_Lean_Parser_Command_reduce___elambda__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_declRange___closed__7; static lean_object* l_Lean_Parser_Command_section___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_private_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__1; static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structSimpleBinder_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classInductive_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_section_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__1; static lean_object* l_Lean_Parser_Command_deriving___closed__3; static lean_object* l_Lean_Parser_Command_moduleDoc___closed__5; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_declId_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_openSimple___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classInductive_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_abbrev_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1822,7 +2011,9 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___cl lean_object* l_Lean_Parser_Term_structInst___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_computedField___closed__7; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_open_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_unsafe___closed__5; static lean_object* l_Lean_Parser_Command_mutual___closed__9; static lean_object* l_Lean_Parser_Command_computedField_formatter___closed__8; @@ -1830,6 +2021,7 @@ static lean_object* l_Lean_Parser_Command_openScoped___closed__2; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Command_classInductive___closed__3; static lean_object* l_Lean_Parser_Command_resolve__name___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__47; LEAN_EXPORT lean_object* l_Lean_Parser_Command_computedField_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_declRange___closed__4; static lean_object* l_Lean_Parser_Command_namedPrio___closed__13; @@ -1841,10 +2033,12 @@ static lean_object* l_Lean_Parser_Command_structure_formatter___closed__2; static lean_object* l_Lean_Parser_Command_def___closed__3; static lean_object* l_Lean_Parser_Command_structInstBinder_formatter___closed__1; static lean_object* l_Lean_Parser_Term_set__option_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_extends___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__1; static lean_object* l_Lean_Parser_Command_instance___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_namespace___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_section___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__3; @@ -1854,8 +2048,8 @@ static lean_object* l_Lean_Parser_Command_nonrec___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_variable_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__6; static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__11; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__22; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__2; static lean_object* l_Lean_Parser_Command_classInductive_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_axiom_parenthesizer___closed__4; @@ -1897,30 +2091,34 @@ static lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer___closed static lean_object* l_Lean_Parser_Command_openScoped_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_decreasingBy; static lean_object* l_Lean_Parser_Command_optDeclSig___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__2; static lean_object* l_Lean_Parser_Command_protected___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__26; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_declValEqns___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_abbrev___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_end_declRange___closed__3; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__22; static lean_object* l_Lean_Parser_Command_instance___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___closed__3; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_end___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_whereStructField; LEAN_EXPORT lean_object* l_Lean_Parser_Command_end_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_opaque_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDefDeriving_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_exit___closed__7; -static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__17; static lean_object* l_Lean_Parser_Command_classInductive___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_exit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_openSimple___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_open___elambda__1___closed__11; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__14; extern lean_object* l_Lean_Parser_Term_whereDecls; static lean_object* l_Lean_Parser_Command_structureTk___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_export___closed__1; @@ -1928,25 +2126,28 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_set__option___elambda__1(lean_obj static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__5; static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__10; static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_formatter(lean_object*); static lean_object* l_Lean_Parser_Tactic_open___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange___closed__6; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_exit_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__15; +static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__31; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_section___closed__2; static lean_object* l_Lean_Parser_Command_openScoped_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__10; static lean_object* l_Lean_Parser_Command_def_formatter___closed__10; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__14; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_open___closed__4; static lean_object* l_Lean_Parser_Command_optionValue___closed__4; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_theorem; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_def_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_structure_formatter___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_set__option; static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__6; @@ -1959,7 +2160,9 @@ static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__5; static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_in___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHintMany_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_variable___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_quot_formatter___closed__3; static lean_object* l_Lean_Parser_Tactic_set__option_parenthesizer___closed__6; @@ -1976,27 +2179,36 @@ static lean_object* l_Lean_Parser_Command_openOnly_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_terminationSuffix_formatter___closed__1; static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__8; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_export_formatter___closed__1; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__7; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeclSig_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_in_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__5; static lean_object* l_Lean_Parser_Command_abbrev___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_whereStructField_formatter___closed__3; static lean_object* l_Lean_Parser_Command_export___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_classTk___closed__4; static lean_object* l_Lean_Parser_Command_declValEqns___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__2; static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_namespace___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_declRange___closed__7; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__26; static lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__19; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__25; static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_variable___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_check__failure_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__24; static lean_object* l_Lean_Parser_Command_instance_formatter___closed__5; static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__1; @@ -2005,15 +2217,14 @@ static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_computedFields_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__7; static lean_object* l_Lean_Parser_Command_openRenaming___closed__5; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Command_noncomputable_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_check_declRange___closed__7; extern lean_object* l_Lean_Parser_Term_attributes; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_protected_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__4; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__6; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__18; static lean_object* l_Lean_Parser_Command_classInductive_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_universe_formatter___closed__2; @@ -2029,7 +2240,6 @@ static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange___closed__2; static lean_object* l_Lean_Parser_Command_partial___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_declRange___closed__2; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__18; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__2; static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__1; @@ -2038,16 +2248,17 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_eval; static lean_object* l_Lean_Parser_Command_end_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_visibility___closed__3; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__22; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_theorem___closed__10; -static lean_object* l_Lean_Parser_Command_computedFields_formatter___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_print_declRange___closed__7; static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__1; static lean_object* l_Lean_Parser_Command_unsafe___closed__1; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__26; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_namespace___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_partial___closed__5; static lean_object* l_Lean_Parser_Command_check__failure___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_set__option_declRange(lean_object*); @@ -2074,6 +2285,7 @@ static lean_object* l_Lean_Parser_Command_classInductive_formatter___closed__7; extern lean_object* l_Lean_Parser_rawIdent; static lean_object* l_Lean_Parser_Command_openScoped___closed__8; static lean_object* l_Lean_Parser_Command_set__option___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_initialize___closed__5; static lean_object* l_Lean_Parser_Command_open___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_universe___elambda__1___closed__6; @@ -2090,6 +2302,7 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___c static lean_object* l_Lean_Parser_Command_declVal___closed__2; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__2; static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_exit_declRange___closed__3; static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__12; @@ -2098,11 +2311,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_partial_parenthesizer(lean_object static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__3; static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__3; static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__3; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__52; lean_object* l_Lean_Parser_many1Indent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_reduce___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_quot_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__2; static lean_object* l_Lean_Parser_Command_eval___elambda__1___closed__11; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__22; static lean_object* l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_terminationBy_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structCtor_parenthesizer___closed__2; @@ -2110,6 +2324,7 @@ static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_open_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_open___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__29; static lean_object* l_Lean_Parser_Command_structCtor___closed__1; static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__7; static lean_object* l_Lean_Parser_Command_open_formatter___closed__5; @@ -2130,16 +2345,16 @@ static lean_object* l_Lean_Parser_Command_attribute_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_namedPrio___closed__6; static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__16; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_export_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_section; -static lean_object* l_Lean_Parser_Command_structure_formatter___closed__19; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_openOnly_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_check__failure___elambda__1___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_set__option_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_openScoped___closed__1; static lean_object* l_Lean_Parser_Command_attribute_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_quot_declRange___closed__2; @@ -2153,10 +2368,12 @@ static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_optDeclSig___closed__4; static lean_object* l_Lean_Parser_Command_classInductive___closed__2; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__1; static lean_object* l_Lean_Parser_Command_def___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_declRange___closed__7; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__9; +static lean_object* l_Lean_Parser_Command_initializeKeyword_formatter___closed__3; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange___closed__1; static lean_object* l_Lean_Parser_Command_exit_formatter___closed__3; @@ -2168,17 +2385,20 @@ static lean_object* l_Lean_Parser_Command_unsafe___closed__4; static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_structFields___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange(lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__46; static lean_object* l_Lean_Parser_Command_computedFields_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structCtor_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_inductive; +static lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optNamedPrio; static lean_object* l___regBuiltin_Lean_Parser_Command_quot_docString___closed__1; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__20; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange___closed__6; +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; +static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declVal___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_def_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_quot_declRange___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange___closed__7; static lean_object* l_Lean_Parser_Command_end___elambda__1___closed__6; uint32_t lean_string_utf8_get(lean_object*, lean_object*); @@ -2187,29 +2407,30 @@ static lean_object* l_Lean_Parser_Command_declaration___closed__4; static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_set__option_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_theorem___closed__7; static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__10; -static lean_object* l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__2; static lean_object* l_Lean_Parser_Command_structureTk_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_section_declRange___closed__3; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_instance___elambda__1___closed__1; -static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__9; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_resolve__name_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__5; static lean_object* l_Lean_Parser_Command_declValEqns___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__19; static lean_object* l_Lean_Parser_Command_axiom___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_optDeriving_formatter___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_variable___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__24; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__12; static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__5; @@ -2222,13 +2443,15 @@ static lean_object* l_Lean_Parser_Command_check__failure___elambda__1___closed__ static lean_object* l_Lean_Parser_Command_declSig_formatter___closed__2; static lean_object* l_Lean_Parser_Command_instance___elambda__1___closed__9; lean_object* l_Lean_PrettyPrinter_Formatter_lookahead_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__2; static lean_object* l_Lean_Parser_Command_derivingClasses_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__34; static lean_object* l_Lean_Parser_Command_partial___closed__1; static lean_object* l_Lean_Parser_Command_variable_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_abbrev___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Command_terminationSuffix_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange___closed__7; static lean_object* l_Lean_Parser_Command_def_formatter___closed__6; @@ -2236,7 +2459,6 @@ static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__2; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__6; -static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__17; static lean_object* l_Lean_Parser_Command_classInductive___closed__4; static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_universe___closed__2; @@ -2245,25 +2467,31 @@ static lean_object* l_Lean_Parser_Command_inductive___closed__6; static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__6; lean_object* l_Lean_Parser_Command_commentBody___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__1; static lean_object* l_Lean_Parser_Command_open___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__13; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__19; static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_deriving___closed__1; static lean_object* l_Lean_Parser_Tactic_open___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_parenthesizer(lean_object*); lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__7; -static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__13; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_export_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers___elambda__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers(uint8_t); static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__42; +static lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__2; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__4; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_reduce_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_structFields___closed__3; static lean_object* l_Lean_Parser_Term_quot___closed__5; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__9; @@ -2273,6 +2501,8 @@ static lean_object* l_Lean_Parser_Command_in___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_instance_formatter___closed__8; static lean_object* l_Lean_Parser_Command_private___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_eval_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_many1Unbox_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openRenamingItem_formatter___closed__3; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__9; @@ -2290,6 +2520,7 @@ lean_object* l_Lean_PrettyPrinter_Parenthesizer_withOpenDecl_parenthesizer(lean_ static lean_object* l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_example___closed__9; static lean_object* l_Lean_Parser_Command_axiom___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__1; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_moduleDoc_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declaration___closed__9; @@ -2308,31 +2539,38 @@ static lean_object* l_Lean_Parser_Command_deriving___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_print(lean_object*); static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_eval___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_variable_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_nonrec_formatter___closed__2; static lean_object* l_Lean_Parser_Command_partial___elambda__1___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_reduce_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_set__option___closed__10; static lean_object* l_Lean_Parser_Command_moduleDoc___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Command_noncomputable___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_open___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_theorem___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_protected_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_terminationByCore___closed__5; static lean_object* l_Lean_Parser_Command_reduce_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_computedFields_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_open_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__1; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_terminationSuffix___closed__1; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_end___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_variable; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__30; static lean_object* l_Lean_Parser_Command_in___closed__2; static lean_object* l_Lean_Parser_Command_optionValue_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__10; @@ -2344,7 +2582,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange(lea LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationSuffix; static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__2; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__5; static lean_object* l_Lean_Parser_Command_classTk___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_variable_declRange(lean_object*); @@ -2352,35 +2589,42 @@ static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__1; lean_object* l_Lean_Parser_Term_ident_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_open_formatter___closed__3; static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__18; static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_declRange___closed__2; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_partial_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__5; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__25; LEAN_EXPORT lean_object* l_Lean_Parser_Command_eraseAttr_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__1; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__3; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange___closed__7; static lean_object* l_Lean_Parser_Command_abbrev___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structureTk_parenthesizer___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_set__option(lean_object*); static lean_object* l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_quot___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_quot_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_terminationSuffix_formatter___closed__2; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_noncomputable_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declSig___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__22; static lean_object* l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__8; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__8; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_unsafe_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__1; static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Command_ctor___elambda__1(lean_object*, lean_object*); @@ -2401,14 +2645,18 @@ static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__3; static lean_object* l_Lean_Parser_Command_exit_formatter___closed__1; static lean_object* l_Lean_Parser_Term_open___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_exit_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_openScoped_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classTk___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classInductive___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_variable_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_eval___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__2; lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_variable___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__12; -static lean_object* l_Lean_Parser_Command_declVal_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeclSig___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_variable___closed__6; static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__4; @@ -2431,28 +2679,33 @@ static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__10; static lean_object* l_Lean_Parser_Command_declSig_formatter___closed__1; static lean_object* l_Lean_Parser_Command_protected___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_set__option___closed__10; static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_declRange___closed__3; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structCtor; static lean_object* l_Lean_Parser_Command_reduce___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_private_formatter___closed__3; static lean_object* l_Lean_Parser_Command_terminationBy_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_synth_declRange___closed__1; static lean_object* l_Lean_Parser_Command_structure_formatter___closed__7; static lean_object* l_Lean_Parser_Command_structFields___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__2; lean_object* l_Lean_Parser_registerAlias(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationByElement___closed__2; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__26; static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_declRange___closed__5; static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_inductive___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiersF_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__23; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationBy_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_openRenaming___closed__7; static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_terminationByCore___elambda__1___closed__1; @@ -2467,6 +2720,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declSig_parenthesizer(lean_object static lean_object* l_Lean_Parser_Term_open___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_open___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__2; static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_openDecl___closed__3; @@ -2476,7 +2731,7 @@ static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__ static lean_object* l_Lean_Parser_Command_printAxioms___closed__8; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_precheckedQuot_formatter___closed__3; -static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__22; +static lean_object* l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_export; LEAN_EXPORT lean_object* l_Lean_Parser_Command_instance_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openRenaming___closed__3; @@ -2486,6 +2741,7 @@ lean_object* l_Lean_Parser_Term_binderIdent_formatter(lean_object*, lean_object* static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__3; static lean_object* l_Lean_Parser_Command_extends___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange___closed__6; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__17; LEAN_EXPORT lean_object* l_Lean_Parser_Command_synth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2501,9 +2757,10 @@ static lean_object* l_Lean_Parser_Command_abbrev___closed__2; static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_extends_formatter___closed__5; static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__8; -static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__23; +static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__19; static lean_object* l_Lean_Parser_Command_openOnly___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declValEqns___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__7; @@ -2512,23 +2769,23 @@ static lean_object* l_Lean_Parser_Command_optionValue_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__21; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__1; -static lean_object* l_Lean_Parser_Command_declVal_formatter___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_eval___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_decreasingBy___closed__6; -static lean_object* l_Lean_Parser_Term_precheckedQuot_formatter___closed__5; static lean_object* l_Lean_Parser_Command_structureTk___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_namespace___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_optionValue___closed__1; static lean_object* l_Lean_Parser_Command_init__quot___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__10; lean_object* l_Lean_PrettyPrinter_Formatter_withPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHint(lean_object*); lean_object* l_Lean_Parser_withResultOfFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_declRange___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__28; static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Tactic_open_formatter___closed__5; static lean_object* l_Lean_Parser_Command_synth___elambda__1___closed__9; @@ -2538,11 +2795,12 @@ static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__5; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__19; lean_object* l_Lean_Parser_many1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__19; static lean_object* l_Lean_Parser_Command_eraseAttr_formatter___closed__4; static lean_object* l_Lean_Parser_Command_declValEqns___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_eraseAttr___closed__2; -static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__21; +static lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_namedPrio___closed__12; static lean_object* l_Lean_Parser_Command_noncomputable___closed__3; static lean_object* l_Lean_Parser_Command_unsafe___closed__6; @@ -2553,13 +2811,13 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot_docString(lean_obj static lean_object* l_Lean_Parser_Tactic_open___closed__2; static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__4; -static lean_object* l_Lean_Parser_Command_terminationSuffix_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_declRange___closed__7; static lean_object* l_Lean_Parser_Command_resolve__name___closed__3; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__6; static lean_object* l_Lean_Parser_Command_instance_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_def___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_abbrev___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_export_formatter___closed__8; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__2; @@ -2567,21 +2825,23 @@ static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__19; static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__2; static lean_object* l_Lean_Parser_Command_terminationBy_formatter___closed__4; static lean_object* l_Lean_Parser_Command_optionValue___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_check___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__4; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__33; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__1; -static lean_object* l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_terminationByCore___elambda__1___closed__8; +static lean_object* l_Lean_Parser_Command_initializeKeyword_formatter___closed__4; static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__9; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__13; static lean_object* l_Lean_Parser_Command_mutual___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__1; static lean_object* l_Lean_Parser_Command_openSimple_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_eval_declRange___closed__5; static lean_object* l_Lean_Parser_Command_decreasingBy_formatter___closed__4; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__25; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_set__option_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_noncomputable___closed__5; @@ -2597,6 +2857,7 @@ static lean_object* l_Lean_Parser_Command_classInductive___closed__8; static lean_object* l_Lean_Parser_Command_structCtor___closed__7; static lean_object* l_Lean_Parser_Command_openOnly___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_quot_formatter___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_computedField_formatter___closed__5; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__3; static lean_object* l_Lean_Parser_Command_check_parenthesizer___closed__2; @@ -2612,7 +2873,6 @@ static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__13; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_quot___elambda__1___lambda__1___boxed(lean_object*); static lean_object* l_Lean_Parser_Command_noncomputable___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Command_declVal_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__2; @@ -2626,18 +2886,15 @@ static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_example_formatter___closed__1; static lean_object* l_Lean_Parser_Term_set__option_parenthesizer___closed__5; lean_object* l_Lean_PrettyPrinter_Formatter_skip_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_builtin__initialize_formatter___closed__1; static lean_object* l_Lean_Parser_Command_eval___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_resolve__name___closed__1; static lean_object* l_Lean_Parser_Command_axiom___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_inductive___closed__4; -static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__10; static lean_object* l_Lean_Parser_Command_export_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structCtor_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_printAxioms_formatter___closed__4; static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_terminationByElement___closed__1; -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_private; @@ -2646,7 +2903,6 @@ static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed LEAN_EXPORT lean_object* l_Lean_Parser_Command_openDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_declVal_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__27; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structSimpleBinder; lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_extends___closed__4; @@ -2661,16 +2917,16 @@ static lean_object* l_Lean_Parser_Command_unsafe_formatter___closed__3; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_synth_declRange___closed__6; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__7; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__15; +static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openScoped___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_quot___elambda__1___lambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_print_declRange___closed__5; static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__5; lean_object* l_Lean_Parser_ppLine_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_eraseAttr_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_unsafe___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__3; static lean_object* l_Lean_Parser_Command_universe___closed__8; static lean_object* l_Lean_Parser_Command_set__option___closed__9; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__12; @@ -2680,14 +2936,17 @@ static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__2; static lean_object* l_Lean_Parser_Command_nonrec___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structureTk_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__7; lean_object* l_Lean_Parser_sepBy1Indent_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__18; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__13; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eval_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_def_formatter___closed__3; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__5; @@ -2701,13 +2960,14 @@ static lean_object* l_Lean_Parser_Command_declValEqns___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_nonrec___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_quot___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_extends_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_printAxioms___closed__6; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_declRange(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end(lean_object*); static lean_object* l_Lean_Parser_Command_computedField___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__12; @@ -2717,13 +2977,13 @@ static lean_object* l_Lean_Parser_Command_universe___closed__4; static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__1; static lean_object* l_Lean_Parser_Command_openRenaming_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_section_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___closed__10; static lean_object* l_Lean_Parser_Command_resolve__name___closed__2; static lean_object* l_Lean_Parser_Command_deriving_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_optDeriving_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declValEqns_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_declRange___closed__2; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__5; @@ -2732,12 +2992,12 @@ static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__ LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHintMany___lambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__1; lean_object* l_Lean_Parser_commandParser_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__22; LEAN_EXPORT lean_object* l_Lean_Parser_Command_partial___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_synth___closed__1; static lean_object* l_Lean_Parser_Term_open___elambda__1___closed__1; -static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_end_declRange___closed__6; @@ -2745,13 +3005,15 @@ static lean_object* l_Lean_Parser_Command_openOnly___elambda__1___closed__4; lean_object* l_Lean_Parser_ident___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_quot___closed__9; extern lean_object* l_Lean_Parser_Term_binderIdent; +static lean_object* l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__18; -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__17; lean_object* l_Lean_Parser_Term_doSeq_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__6; static lean_object* l_Lean_Parser_Command_terminationHintMany_formatter___closed__3; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__49; static lean_object* l_Lean_Parser_Tactic_open___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_set__option___closed__4; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__9; @@ -2762,14 +3024,15 @@ static lean_object* l_Lean_Parser_Command_declVal___closed__1; static lean_object* l_Lean_Parser_Command_openRenaming___closed__1; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHint_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__11; uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l_Lean_Parser_Command_reduce_formatter___closed__1; static lean_object* l_Lean_Parser_Command_terminationByElement___closed__5; -static lean_object* l_Lean_Parser_Command_builtin__initialize_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__1; static lean_object* l_Lean_Parser_Tactic_set__option_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__16; -static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__20; static lean_object* l_Lean_Parser_Term_open_formatter___closed__1; static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_check; @@ -2785,6 +3048,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_whereStructField___elambda__1(lea static lean_object* l_Lean_Parser_Tactic_set__option_formatter___closed__1; extern lean_object* l_Lean_Parser_numLit; static lean_object* l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__4; extern lean_object* l_Lean_Parser_Term_leftArrow; static lean_object* l_Lean_Parser_Command_terminationBy___closed__9; @@ -2801,7 +3065,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange___clos static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__1; static lean_object* l_Lean_Parser_Command_decreasingBy___closed__8; -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_instance_formatter___closed__1; static lean_object* l_Lean_Parser_Command_init__quot___closed__2; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__15; @@ -2811,6 +3075,7 @@ static lean_object* l_Lean_Parser_Command_openSimple___closed__4; static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__7; lean_object* l_Lean_Parser_Term_ident___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__17; +static lean_object* l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__1; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__6; @@ -2820,11 +3085,15 @@ static lean_object* l_Lean_Parser_Command_example_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_in___closed__4; static lean_object* l_Lean_Parser_Command_def___closed__12; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__17; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declSig_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_deriving_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_printAxioms___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__32; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenaming_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__1; static lean_object* l_Lean_Parser_Command_check_formatter___closed__4; static lean_object* l_Lean_Parser_Command_attribute___closed__1; static lean_object* l_Lean_Parser_Command_structureTk___closed__7; @@ -2836,6 +3105,7 @@ static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__12; static lean_object* l_Lean_Parser_Command_openOnly_parenthesizer___closed__5; lean_object* l_Lean_Parser_Term_optType_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__11; lean_object* l_Lean_Parser_numLit___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_abbrev___closed__1; @@ -2853,14 +3123,20 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_quot_declRange___closed__7; static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_open_formatter___closed__6; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__24; +static lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_extends_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__2; lean_object* l_Lean_Syntax_getNumArgs(lean_object*); static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__21; @@ -2871,22 +3147,25 @@ static lean_object* l_Lean_Parser_Command_reduce_formatter___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange___closed__4; static lean_object* l_Lean_Parser_Command_example_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__18; static lean_object* l_Lean_Parser_Command_partial___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_set__option___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_namedPrio___closed__11; extern lean_object* l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; extern lean_object* l_Lean_Parser_Term_attrKind; static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__25; static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_declRange___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_declRange___closed__1; static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_terminationBy___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_axiom___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_private___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_declRange(lean_object*); @@ -2899,30 +3178,36 @@ static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__13; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__20; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__1; lean_object* l_Lean_Parser_Term_binderDefault___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__16; lean_object* l_Lean_Parser_Term_ident_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__1; static lean_object* l_Lean_Parser_Command_attribute_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Command_resolve__name_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_declRange___closed__6; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__2; static lean_object* l_Lean_Parser_Command_classInductive___closed__6; static lean_object* l_Lean_Parser_Command_namespace_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_partial_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__20; static lean_object* l_Lean_Parser_Command_eraseAttr_formatter___closed__2; static lean_object* l_Lean_Parser_Command_end___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_optDeriving_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_namespace_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_noncomputable___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__38; static lean_object* l_Lean_Parser_Command_structFields___closed__2; -static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__21; static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__19; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__16; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__8; static lean_object* l_Lean_Parser_Command_computedField___closed__6; static lean_object* l_Lean_Parser_Tactic_set__option_formatter___closed__2; @@ -2936,14 +3221,17 @@ static lean_object* l_Lean_Parser_Command_synth___closed__4; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_in_formatter___closed__1; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__6; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_whereStructInst_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_open_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_open_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_resolve__name___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_init__quot_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declId_parenthesizer(lean_object*); lean_object* l_Lean_Parser_Term_attrKind_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mutual_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_whereStructInst___closed__7; static lean_object* l_Lean_Parser_Command_declVal___closed__3; @@ -2960,9 +3248,11 @@ static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__4; static lean_object* l_Lean_Parser_Command_structCtor___closed__5; static lean_object* l_Lean_Parser_Command_decreasingBy___closed__4; static lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_whereStructField___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_openDecl___elambda__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_declRange___closed__4; @@ -2975,8 +3265,9 @@ static lean_object* l_Lean_Parser_Command_quot___closed__4; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__9; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__5; lean_object* l_Lean_Parser_Term_letDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_builtin__initialize_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_example_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_example_formatter___closed__2; static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__4; @@ -2992,7 +3283,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange___c static lean_object* l_Lean_Parser_Command_check__failure___closed__6; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__9; -static lean_object* l_Lean_Parser_Command_structure_formatter___closed__22; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_open_formatter___closed__2; static lean_object* l_Lean_Parser_Command_namespace___closed__7; @@ -3000,6 +3290,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_namespace_formatter(lean_object*, lean_object* l_Lean_Parser_categoryParser(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_check__failure___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__1; lean_object* l_Lean_Parser_ppGroup_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__25; @@ -3007,27 +3298,32 @@ static lean_object* l_Lean_Parser_Command_ctor___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_quot; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__10; lean_object* l_Lean_Parser_commandParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_example_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationSuffix_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_structCtor___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_synth_formatter___closed__1; static lean_object* l_Lean_Parser_Command_nonrec___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_computedFields_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_moduleDoc_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_axiom_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mutual_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_synth_formatter___closed__2; static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_noncomputable___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_openSimple___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__2; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_optDeclSig___elambda__1___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_set__option_declRange(lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__29; static lean_object* l_Lean_Parser_Command_structure___closed__8; static lean_object* l_Lean_Parser_Command_end___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__10; @@ -3036,10 +3332,14 @@ static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_end___closed__6; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__6; static lean_object* l_Lean_Parser_Command_noncomputable_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_section_formatter___closed__1; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__2; static lean_object* l_Lean_Parser_Command_decreasingBy___closed__2; static lean_object* l_Lean_Parser_Command_instance___closed__6; static lean_object* l_Lean_Parser_Command_namespace___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openSimple___elambda__1(lean_object*, lean_object*); @@ -3047,8 +3347,10 @@ static lean_object* l_Lean_Parser_Tactic_set__option___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_structureTk___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_namedPrio___closed__2; static lean_object* l_Lean_Parser_Command_openOnly_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_extends_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declVal_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__2; @@ -3065,8 +3367,8 @@ static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__7; static lean_object* l_Lean_Parser_Command_opaque___closed__4; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__2; static lean_object* l_Lean_Parser_Command_in_formatter___closed__2; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_optDeclSig___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__1; static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_open_formatter___closed__4; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__12; @@ -3087,16 +3389,18 @@ static lean_object* l_Lean_Parser_Command_opaque___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_eval___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_print_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_openRenaming_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_terminationByElement___closed__6; static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__16; -static lean_object* l_Lean_Parser_Command_attribute_parenthesizer___closed__12; -static lean_object* l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers___elambda__1___rarg(lean_object*); static lean_object* l_Lean_Parser_Command_computedFields_formatter___closed__5; static lean_object* l_Lean_Parser_Command_terminationBy___closed__4; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__6; static lean_object* l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_declRange___closed__3; static lean_object* l_Lean_Parser_Command_declId___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_section_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_openOnly___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_computedField_formatter___closed__6; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__8; @@ -3107,13 +3411,14 @@ static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declId_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__16; -static lean_object* l_Lean_Parser_Command_openDecl_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_synth___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_declaration___closed__1; static lean_object* l_Lean_Parser_Command_openOnly___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__6; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_inductive___closed__1; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__16; +static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_declRange___closed__5; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_declValSimple___closed__4; @@ -3123,19 +3428,20 @@ static lean_object* l_Lean_Parser_Command_ctor___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHint1_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers___elambda__1___rarg___boxed(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__2; static lean_object* l_Lean_Parser_Command_nonrec___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_def_parenthesizer___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_set__option___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__21; static lean_object* l_Lean_Parser_Command_theorem___closed__1; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_theorem___closed__4; -static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__21; static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_set__option_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_init__quot___elambda__1___closed__10; lean_object* l_Lean_Parser_Term_binderDefault_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__10; @@ -3144,7 +3450,9 @@ static lean_object* l_Lean_Parser_Command_openSimple___closed__2; lean_object* l_Lean_Parser_symbolInfo(lean_object*); static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__1; static lean_object* l_Lean_Parser_Term_open___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__17; +static lean_object* l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classTk; static lean_object* l_Lean_Parser_Command_end___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__7; @@ -3165,6 +3473,7 @@ static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__9; static lean_object* l_Lean_Parser_Command_classInductive_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer(lean_object*); extern lean_object* l_Lean_Parser_Command_docComment; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__5; @@ -3173,6 +3482,7 @@ lean_object* l_Lean_Parser_orelseFnCore(lean_object*, lean_object*, uint8_t, lea LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers___elambda__1___boxed(lean_object*); static lean_object* l_Lean_Parser_Command_structInstBinder_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_open_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__7; extern lean_object* l_Lean_Parser_epsilonInfo; lean_object* l_Lean_Parser_notSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -3181,8 +3491,10 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name(lean_o static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_def___closed__1; static lean_object* l_Lean_Parser_Command_axiom___elambda__1___closed__13; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_section_declRange___closed__4; static lean_object* l_Lean_Parser_Command_optionValue___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_opaque_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__4; @@ -3190,16 +3502,21 @@ static lean_object* l_Lean_Parser_Command_terminationByElement___closed__3; static lean_object* l_Lean_Parser_Command_terminationBy___closed__8; static lean_object* l_Lean_Parser_Command_declValSimple___closed__9; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_synth(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__2; static lean_object* l_Lean_Parser_Command_terminationByElement_formatter___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_openRenaming_formatter___closed__7; static lean_object* l_Lean_Parser_Command_structure___closed__4; static lean_object* l_Lean_Parser_Command_printAxioms___closed__2; static lean_object* l_Lean_Parser_Command_in___closed__8; static lean_object* l_Lean_Parser_Tactic_open___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openScoped_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_namespace_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__21; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__21; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_section_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_print___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__4; static lean_object* l_Lean_Parser_Command_structure_formatter___closed__13; @@ -3218,13 +3535,13 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_structureTk___elambda__1(lean_obj LEAN_EXPORT lean_object* l_Lean_Parser_Command_open___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_mutual_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_decreasingBy___closed__1; -static lean_object* l_Lean_Parser_Command_declVal_formatter___closed__4; lean_object* l_Lean_Parser_categoryParser___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__7; static lean_object* l_Lean_Parser_Tactic_open___closed__8; static lean_object* l_Lean_Parser_Term_open___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_ctor___closed__9; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__24; static lean_object* l_Lean_Parser_Command_inductive___closed__13; static lean_object* l_Lean_Parser_Command_variable___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__21; @@ -3234,7 +3551,6 @@ static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_print_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__11; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__11; -static lean_object* l_Lean_Parser_Command_structure_formatter___closed__23; static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Command_instance___elambda__1___closed__7; lean_object* l_Lean_PrettyPrinter_Formatter_withOpen_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -3245,6 +3561,7 @@ static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed static lean_object* l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_check__failure___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_openOnly___closed__6; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_declRange___closed__6; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__9; @@ -3262,14 +3579,16 @@ static lean_object* l_Lean_Parser_Command_structure___closed__9; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__16; LEAN_EXPORT lean_object* l_Lean_Parser_Command_set__option_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_computedFields___closed__3; static lean_object* l_Lean_Parser_Command_declaration___closed__2; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__9; -static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_open_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_nonrec___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_instance_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_end___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_terminationByElement___closed__8; static lean_object* l_Lean_Parser_Command_example_formatter___closed__2; @@ -3281,6 +3600,7 @@ static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__ LEAN_EXPORT lean_object* l_Lean_Parser_Command_attribute___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_computedField; static lean_object* l_Lean_Parser_Command_structureTk___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_in_parenthesizer___closed__1; @@ -3296,6 +3616,7 @@ static lean_object* l_Lean_Parser_Command_check___closed__3; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__9; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_synth___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__1; static lean_object* l_Lean_Parser_Term_quot___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namespace_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_axiom___closed__8; @@ -3306,6 +3627,7 @@ static lean_object* l_Lean_Parser_Command_classInductive___closed__12; static lean_object* l_Lean_Parser_Command_noncomputable_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiersT_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__1; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__3; static lean_object* l_Lean_Parser_Command_openOnly___closed__2; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__23; @@ -3319,25 +3641,28 @@ static lean_object* l_Lean_Parser_Command_structureTk___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_export_formatter___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_ctor_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHint_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_openDecl_parenthesizer___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_declRange___closed__3; -static lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__2; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__6; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__1; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_declValSimple___closed__1; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__2; lean_object* l_Lean_Parser_ident_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__11; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__11; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__35; static lean_object* l_Lean_Parser_Command_openHiding___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_declRange___closed__5; static lean_object* l_Lean_Parser_Command_optDeclSig_formatter___closed__10; @@ -3353,10 +3678,12 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_declRange___c LEAN_EXPORT lean_object* l_Lean_Parser_Command_openDecl___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___lambda__1___closed__1; static lean_object* l_Lean_Parser_Command_opaque___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__9; static lean_object* l_Lean_Parser_Command_terminationByCore___closed__4; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_universe_formatter___closed__3; +static lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_noncomputableSection_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenamingItem___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -3368,10 +3695,11 @@ static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__ static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_declRange___closed__3; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_resolve__name_formatter___closed__1; -static lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__1; static lean_object* l_Lean_Parser_Command_openHiding___closed__1; static lean_object* l_Lean_Parser_Command_check__failure___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__2; @@ -3379,6 +3707,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_print_declRange___closed_ static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_opaque_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_ctor_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_structure_formatter___closed__12; static lean_object* l_Lean_Parser_Command_ctor_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__2; @@ -3393,17 +3722,22 @@ static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__ static lean_object* l_Lean_Parser_Command_structureTk___closed__3; static lean_object* l_Lean_Parser_Command_variable_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_terminationBy_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declVal_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__1; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedField_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_nonrec___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__1; static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__24; static lean_object* l_Lean_Parser_Command_export_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_in_parenthesizer___closed__2; lean_object* l_Lean_Parser_numLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_opaque_formatter___closed__5; static lean_object* l_Lean_Parser_Command_deriving_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2; @@ -3418,18 +3752,20 @@ static lean_object* l_Lean_Parser_Command_quot___closed__3; static lean_object* l_Lean_Parser_Command_instance___elambda__1___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange___closed__1; static lean_object* l_Lean_Parser_Command_def_formatter___closed__9; -static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__19; +static lean_object* l_Lean_Parser_Command_initializeKeyword___closed__2; static lean_object* l_Lean_Parser_Command_classInductive___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_openRenaming___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__1; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange___closed__5; static lean_object* l_Lean_Parser_Command_protected_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_quot(lean_object*); static lean_object* l_Lean_Parser_Command_namedPrio___closed__7; static lean_object* l_Lean_Parser_Command_print___closed__8; static lean_object* l_Lean_Parser_Command_check___elambda__1___closed__10; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__38; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__21; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openOnly_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ppSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -3449,18 +3785,20 @@ static lean_object* l_Lean_Parser_Command_eraseAttr___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_quot_declRange___closed__2; static lean_object* l_Lean_Parser_Command_optDeclSig___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_openSimple_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_quot_declRange___closed__1; static lean_object* l_Lean_Parser_Tactic_set__option___closed__3; static lean_object* l_Lean_Parser_Command_computedField_parenthesizer___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange___closed__6; static lean_object* l_Lean_Parser_Command_extends_formatter___closed__1; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1; lean_object* l_String_trim(lean_object*); lean_object* l_Lean_Parser_Term_doSeq_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_def___elambda__1___closed__16; static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_declRange___closed__5; +static lean_object* l_Lean_Parser_Command_initializeKeyword_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structure___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_def_formatter___closed__1; static lean_object* l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__2; @@ -3468,6 +3806,7 @@ static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__1; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_terminationByElement___closed__4; static lean_object* l_Lean_Parser_Command_def___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_declRange___closed__7; static lean_object* l_Lean_Parser_Command_whereStructField___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_open___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); @@ -3477,12 +3816,15 @@ static lean_object* l_Lean_Parser_Command_computedFields___closed__5; static lean_object* l_Lean_Parser_Command_exit___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_section_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_nodeFn(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_open_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declValSimple; static lean_object* l_Lean_Parser_Command_eval_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_abbrev___elambda__1___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange___closed__4; static lean_object* l_Lean_Parser_Command_resolve__name___closed__5; static lean_object* l_Lean_Parser_Command_check__failure_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_moduleDoc; static lean_object* l_Lean_Parser_Command_openOnly___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__11; @@ -3494,22 +3836,23 @@ static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_axiom___closed__1; static lean_object* l_Lean_Parser_Command_partial_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__2; static lean_object* l_Lean_Parser_Command_exit___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_unsafe___elambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_Command_builtin__initialize; static lean_object* l_Lean_Parser_Command_nonrec___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_structImplicitBinder___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_variable___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_in_declRange___closed__1; -static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__29; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_noncomputable___elambda__1___closed__6; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__35; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__17; -LEAN_EXPORT lean_object* l_Lean_Parser_Command_builtin__initialize_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declaration___closed__17; static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__8; -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_variable_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__5; lean_object* l_Lean_Parser_unicodeSymbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declVal_formatter___closed__1; @@ -3519,16 +3862,13 @@ static lean_object* l_Lean_Parser_Command_open___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_declSig___closed__5; static lean_object* l_Lean_Parser_Command_structureTk___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__23; -static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__14; lean_object* l_Lean_Parser_Term_structInst_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_def_formatter___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__34; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_structFields_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Command_structureTk___closed__5; -static lean_object* l_Lean_Parser_Command_initialize___closed__10; lean_object* l_Lean_Parser_rawIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_print___closed__1; @@ -3545,10 +3885,12 @@ static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange___closed__2; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_open_formatter___closed__1; static lean_object* l_Lean_Parser_Command_eraseAttr_formatter___closed__5; static lean_object* l_Lean_Parser_Command_whereStructField___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__41; static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_computedFields_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; @@ -3557,12 +3899,11 @@ static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Command_open_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__19; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__1; static lean_object* l_Lean_Parser_Command_classTk___closed__3; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_structFields___closed__5; static lean_object* l_Lean_Parser_Command_variable___closed__2; -static lean_object* l_Lean_Parser_Command_declVal_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_deriving___closed__9; static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__6; @@ -3571,7 +3912,6 @@ static lean_object* l_Lean_Parser_Command_instance___closed__11; static lean_object* l_Lean_Parser_Command_synth___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple_formatter___closed__8; -static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__29; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__20; static lean_object* l_Lean_Parser_Command_optionValue___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__13; @@ -3580,17 +3920,19 @@ static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__3; static lean_object* l_Lean_Parser_Tactic_open___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_unsafe___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_whereStructField___closed__3; lean_object* l_Lean_ppLine_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot; static lean_object* l_Lean_Parser_Command_abbrev___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_set__option___closed__2; static lean_object* l_Lean_Parser_Command_init__quot___elambda__1___closed__6; -static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__15; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_check__failure_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_universe___elambda__1___closed__11; @@ -3600,12 +3942,13 @@ static lean_object* l_Lean_Parser_Command_terminationSuffix___elambda__1___close static lean_object* l_Lean_Parser_Command_openSimple___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_openOnly___closed__1; static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__1; -static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__9; lean_object* l_Lean_Parser_ppHardLineUnlessUngrouped_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__1; static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeclSig_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationByCore___elambda__1___closed__13; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_attribute_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_universe___closed__6; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_optDeclSig___closed__7; @@ -3616,7 +3959,6 @@ static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__13; static lean_object* l_Lean_Parser_Command_opaque_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__12; -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_open(lean_object*); static lean_object* l_Lean_Parser_Command_instance_formatter___closed__9; static lean_object* l_Lean_Parser_Command_deriving_formatter___closed__2; @@ -3635,12 +3977,13 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_unsafe_formatter(lean_object*, le static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structureTk; static lean_object* l___regBuiltin_Lean_Parser_Term_open_declRange___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__19; static lean_object* l_Lean_Parser_Command_eval_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_open; -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__4; static lean_object* l_Lean_Parser_Command_extends_formatter___closed__2; static lean_object* l_Lean_Parser_Command_end___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__51; static lean_object* l_Lean_Parser_Command_variable___closed__5; static lean_object* l_Lean_Parser_Command_optNamedPrio___closed__4; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__14; @@ -3649,7 +3992,6 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_attribute(lean_objec static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__7; static lean_object* l_Lean_Parser_Command_open_formatter___closed__4; static lean_object* l_Lean_Parser_Command_def___closed__2; -static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__20; static lean_object* l___regBuiltin_Lean_Parser_Command_variable_declRange___closed__6; static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_terminationSuffix___elambda__1___closed__1; @@ -3657,7 +3999,6 @@ lean_object* l_Lean_Parser_mkAntiquot(lean_object*, lean_object*, uint8_t, uint8 static lean_object* l_Lean_Parser_Command_print_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_init__quot___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__10; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__1; static lean_object* l_Lean_Parser_Command_ctor___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_optDeclSig___elambda__1___closed__1; lean_object* l_Lean_Parser_Term_typeSpec_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -3666,6 +4007,7 @@ static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_check__failure_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__6; static lean_object* l_Lean_Parser_Command_export___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_declSig___closed__3; static lean_object* l_Lean_Parser_Command_optionValue_formatter___closed__4; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__4; @@ -3678,6 +4020,7 @@ static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__27; static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_openRenamingItem___closed__8; static lean_object* l_Lean_Parser_Command_mutual_parenthesizer___closed__3; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_decreasingBy___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__12; lean_object* l_Lean_Parser_Tactic_tacticSeq_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -3688,6 +4031,7 @@ static lean_object* l_Lean_Parser_Command_print_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedPrio___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual___closed__3; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withOpen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer(lean_object*); lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_declValSimple___closed__5; @@ -3700,19 +4044,20 @@ static lean_object* l_Lean_Parser_Command_derivingClasses___closed__5; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_quot___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structCtor___elambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_partial; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_initialize___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_declModifiers___closed__11; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__13; -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__2; static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__2; static lean_object* l_Lean_Parser_Command_end___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_variable___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_declaration___closed__6; static lean_object* l_Lean_Parser_Command_private___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_nonrec___elambda__1___closed__2; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__39; static lean_object* l_Lean_Parser_Command_set__option_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__4; static lean_object* l_Lean_Parser_Command_check___closed__7; @@ -3732,12 +4077,13 @@ static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structExplicitBinder___elambda__1(lean_object*, lean_object*); lean_object* l_Lean_Parser_many_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_print_formatter___closed__3; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__13; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_exit_declRange___closed__5; static lean_object* l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_optNamedPrio___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__14; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__3; @@ -3764,17 +4110,19 @@ static lean_object* l_Lean_Parser_Command_declaration_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_synth_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_partial___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__2; static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_set__option(lean_object*); static lean_object* l_Lean_Parser_Command_reduce___closed__1; static lean_object* l_Lean_Parser_Command_declValSimple___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namespace; static lean_object* l_Lean_Parser_Command_print___closed__2; static lean_object* l_Lean_Parser_Command_structCtor_formatter___closed__5; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__11; static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__27; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__23; static lean_object* l_Lean_Parser_Command_openDecl___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_terminationByCore___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_declSig_formatter___closed__4; @@ -3784,6 +4132,7 @@ static lean_object* l_Lean_Parser_Command_derivingClasses___closed__15; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__25; lean_object* l_Lean_Parser_Command_commentBody_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_resolve__name_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__6; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__3; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__27; @@ -3796,24 +4145,28 @@ static lean_object* l_Lean_Parser_Command_derivingClasses___closed__14; static lean_object* l_Lean_Parser_Command_instance_formatter___closed__10; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_check__failure_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_set__option_formatter___closed__5; static lean_object* l_Lean_Parser_Command_check___elambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_namespace_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_set__option_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2; static lean_object* l_Lean_Parser_Command_openHiding_formatter___closed__1; -static lean_object* l_Lean_Parser_Command_structure_formatter___closed__20; static lean_object* l_Lean_Parser_Command_declaration___closed__15; static lean_object* l_Lean_Parser_Command_private_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declValSimple___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_quot___elambda__1___lambda__1(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_axiom___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_def_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_openHiding___closed__6; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__7; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__22; +static lean_object* l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_section_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__2; @@ -3824,6 +4177,8 @@ static lean_object* l_Lean_Parser_Command_structureTk___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange___closed__2; lean_object* l_Lean_Parser_Term_binderDefault_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eval_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_partial___elambda__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_declRange___closed__5; static lean_object* l_Lean_Parser_Term_set__option_parenthesizer___closed__4; @@ -3840,32 +4195,36 @@ static lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_attribute___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_extends_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_inductive_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_classInductive_formatter___closed__4; static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__6; extern lean_object* l_Lean_Parser_Term_matchAltsWhereDecls; +static lean_object* l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_section_declRange___closed__6; static lean_object* l_Lean_Parser_Command_moduleDoc_formatter___closed__6; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_optionValue___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_terminationByCore___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_namespace_formatter___closed__2; static lean_object* l_Lean_Parser_Command_synth_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_check_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__2; static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__10; static lean_object* l_Lean_Parser_Command_export___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_Command_opaque; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__25; static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange___closed__2; -static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__22; static lean_object* l_Lean_Parser_Command_eraseAttr___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_print_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__1; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColGe_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_open_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_printAxioms_parenthesizer___closed__5; -static lean_object* l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_set__option___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_openHiding_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Tactic_open___closed__7; @@ -3877,7 +4236,6 @@ static lean_object* l_Lean_Parser_Command_def___closed__4; static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_structImplicitBinder_formatter___closed__6; static lean_object* l_Lean_Parser_Command_declaration___closed__5; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__9; lean_object* l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__15; @@ -3885,6 +4243,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1(lean static lean_object* l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_extends___closed__6; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__18; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__20; @@ -3898,6 +4257,7 @@ static lean_object* l_Lean_Parser_Command_computedField___closed__8; static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Command_inductive_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__1; static lean_object* l_Lean_Parser_Command_axiom___elambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiersF; static lean_object* l_Lean_Parser_Command_deriving___closed__10; @@ -3905,9 +4265,9 @@ static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_derivingClasses_formatter___closed__6; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Tactic_open_declRange___closed__3; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__31; static lean_object* l___regBuiltin_Lean_Parser_Command_initialize_declRange___closed__1; static lean_object* l_Lean_Parser_Command_protected___closed__7; -static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__27; LEAN_EXPORT lean_object* l_Lean_Parser_Command_axiom; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__1; static lean_object* l_Lean_Parser_Command_exit___closed__2; @@ -3916,22 +4276,28 @@ static lean_object* l_Lean_Parser_Command_quot___closed__6; static lean_object* l_Lean_Parser_Term_open___closed__2; static lean_object* l_Lean_Parser_Command_classInductive_formatter___closed__9; static lean_object* l_Lean_Parser_Command_computedFields_parenthesizer___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__1; +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword; static lean_object* l_Lean_Parser_Command_openOnly___closed__4; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__1; static lean_object* l_Lean_Parser_Term_open_formatter___closed__5; static lean_object* l_Lean_Parser_Command_def_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_structureTk_formatter___closed__2; static lean_object* l_Lean_Parser_Command_noncomputable___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_axiom_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_derivingClasses___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_derivingClasses_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_quot_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_namespace_declRange___closed__4; static lean_object* l_Lean_Parser_Command_check__failure_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__10; static lean_object* l_Lean_Parser_Tactic_open_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declValSimple_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_synth_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_synth_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_def_formatter___closed__5; static lean_object* l_Lean_Parser_Term_quot_formatter___closed__6; @@ -3942,7 +4308,9 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_check__failure; static lean_object* l_Lean_Parser_Command_printAxioms___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_open___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder_formatter___closed__12; +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_optionValue_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_openRenaming_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__33; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__14; @@ -3953,27 +4321,26 @@ static lean_object* l_Lean_Parser_Command_structFields_formatter___closed__8; lean_object* l_Lean_Parser_Term_matchAlts_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_print___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_optDeriving___closed__4; -LEAN_EXPORT lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_open___closed__8; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__5; static lean_object* l_Lean_Parser_Tactic_open___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_extends_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_set__option_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__4; static lean_object* l_Lean_Parser_Command_unsafe___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_opaque___closed__7; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__4; static lean_object* l_Lean_Parser_Command_synth___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_openRenamingItem_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structCtor_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_extends___elambda__1___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_export_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_optDeriving___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__30; static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__3; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_synth___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__3; static lean_object* l_Lean_Parser_Command_protected___elambda__1___closed__11; @@ -3992,22 +4359,23 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenamingItem_parenthesizer(le LEAN_EXPORT lean_object* l_Lean_Parser_Command_declVal_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structureTk_formatter___closed__1; static lean_object* l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__40; static lean_object* l_Lean_Parser_Command_terminationByCore_formatter___closed__3; static lean_object* l_Lean_Parser_Command_openHiding_formatter___closed__8; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColGt_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__27; +static lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__4; static lean_object* l_Lean_Parser_Command_optDeclSig___closed__2; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_whereStructInst_formatter___closed__3; static lean_object* l_Lean_Parser_Command_decreasingBy_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__1; static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__4; extern lean_object* l_Lean_Parser_Term_structInst; static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__10; lean_object* l_Lean_Parser_symbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_synth_declRange___closed__4; static lean_object* l_Lean_Parser_Command_terminationHintMany_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__2; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_structSimpleBinder_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationHintMany___lambda__1___boxed(lean_object*, lean_object*); @@ -4016,12 +4384,16 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_opaque_formatter(lean_object*, le static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_declaration_formatter___closed__12; static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__12; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__43; LEAN_EXPORT lean_object* l_Lean_Parser_Term_set__option; lean_object* l_Lean_Parser_Term_binderIdent___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__18; static lean_object* l_Lean_Parser_Tactic_open___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declValEqns___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mutual_formatter___closed__12; static lean_object* l_Lean_Parser_Command_end___closed__1; static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__6; @@ -4032,12 +4404,14 @@ static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___c static lean_object* l_Lean_Parser_Command_example___closed__4; static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_openOnly___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__18; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_open___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_instance___closed__3; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structSimpleBinder___closed__2; static lean_object* l_Lean_Parser_Command_private_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_declRange___closed__2; @@ -4046,7 +4420,7 @@ static lean_object* l_Lean_Parser_Command_instance___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_whereStructInst___elambda__1___closed__18; static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__6; -static lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; static lean_object* l_Lean_Parser_Command_opaque___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_partial___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_resolve__name___elambda__1___closed__10; @@ -4057,6 +4431,7 @@ static lean_object* l_Lean_Parser_Command_structFields___elambda__1___closed__14 static lean_object* l_Lean_Parser_Command_inductive___closed__10; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_eval_declRange___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Tactic_open___closed__2; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_exit___elambda__1___closed__6; @@ -4065,21 +4440,25 @@ static lean_object* l_Lean_Parser_Command_structure_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_end_declRange___closed__1; lean_object* l_Lean_Parser_withOpenFn(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__1; static lean_object* l_Lean_Parser_Command_instance_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_synth___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__2; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__8; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__31; static lean_object* l_Lean_Parser_Command_structCtor_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_structureTk_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationByCore_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_check__failure___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_whereStructField_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_private_formatter___closed__1; static lean_object* l_Lean_Parser_Term_open___closed__5; static lean_object* l_Lean_Parser_Command_declValSimple___closed__7; static lean_object* l_Lean_Parser_Command_abbrev_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_check__failure_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__1; static lean_object* l_Lean_Parser_Command_mutual___elambda__1___closed__22; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_declRange___closed__5; static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__19; static lean_object* l_Lean_Parser_Command_reduce_parenthesizer___closed__3; @@ -4093,13 +4472,15 @@ static lean_object* l_Lean_Parser_Command_init__quot___closed__4; static lean_object* l_Lean_Parser_Command_terminationByCore___closed__7; static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__7; static lean_object* l_Lean_Parser_Command_optionValue_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_structure___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_open_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__2; lean_object* l_Lean_Parser_ident_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeriving_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__9; @@ -4108,6 +4489,7 @@ static lean_object* l_Lean_Parser_Command_abbrev___closed__6; static lean_object* l_Lean_Parser_Command_terminationBy___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_example___closed__2; static lean_object* l_Lean_Parser_Command_opaque_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declValEqns_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mutual___closed__5; static lean_object* l_Lean_Parser_Tactic_set__option___closed__8; @@ -4115,7 +4497,6 @@ static lean_object* l_Lean_Parser_Command_derivingClasses_parenthesizer___closed static lean_object* l_Lean_Parser_Command_declSig_formatter___closed__3; static lean_object* l_Lean_Parser_Command_declVal_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__12; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__44; static lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_declRange___closed__6; static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option(lean_object*); @@ -4131,6 +4512,7 @@ static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_namedPrio_formatter___closed__3; static lean_object* l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__7; lean_object* l_Lean_Parser_symbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__1; static lean_object* l_Lean_Parser_Command_namespace___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_quot___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_terminationByCore___closed__2; @@ -4153,6 +4535,7 @@ static lean_object* l_Lean_Parser_Command_openRenaming___elambda__1___closed__13 static lean_object* l_Lean_Parser_Command_set__option___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_declId___closed__6; static lean_object* l_Lean_Parser_Command_terminationHintMany___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_in_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -4161,12 +4544,14 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_instance_formatter(lean_object*, static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__19; static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__7; static lean_object* l_Lean_Parser_Command_in___closed__7; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__36; static lean_object* l_Lean_Parser_Command_declSig___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_print; static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__1; static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_example___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_computedField___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_namedPrio_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_optDeriving_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__9; @@ -4182,7 +4567,6 @@ static lean_object* l_Lean_Parser_Term_precheckedQuot___closed__2; static lean_object* l_Lean_Parser_Command_openDecl___closed__4; lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lean_Parser_Command_eval___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_declRange___closed__6; static lean_object* l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_resolve__name___closed__4; @@ -4192,16 +4576,18 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange___cl LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationByElement_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_ctor_formatter___closed__5; static lean_object* l_Lean_Parser_Command_structInstBinder___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_openRenamingItem_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structInstBinder_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_Command_initializeKeyword_formatter___closed__2; static lean_object* l_Lean_Parser_Command_terminationByElement___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_private_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_abbrev_formatter___closed__4; static lean_object* l_Lean_Parser_Command_universe___closed__5; static lean_object* l_Lean_Parser_Command_openHiding___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_check___closed__4; static lean_object* l_Lean_Parser_Command_optDefDeriving___closed__2; static lean_object* l_Lean_Parser_Command_classTk___elambda__1___closed__2; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__45; static lean_object* l_Lean_Parser_Command_computedField___elambda__1___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_declRange___closed__4; static lean_object* l_Lean_Parser_Command_open___closed__4; @@ -4213,7 +4599,6 @@ static lean_object* l_Lean_Parser_Command_optionValue___elambda__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_export_declRange___closed__2; static lean_object* l_Lean_Parser_Command_declId_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Command_inductive_formatter___closed__16; LEAN_EXPORT lean_object* l_Lean_Parser_Command_classInductive_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_export___closed__10; static lean_object* l_Lean_Parser_Term_open___elambda__1___closed__3; @@ -4230,18 +4615,21 @@ static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_inductive_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_computedFields___elambda__1___closed__15; lean_object* l_Lean_Parser_Term_attrKind___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__2; static lean_object* l_Lean_Parser_Command_eraseAttr___elambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_private___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_section___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__17; +static lean_object* l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__5; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__8; static lean_object* l_Lean_Parser_Command_partial_formatter___closed__1; -static lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_openHiding_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_deriving_declRange___closed__2; static lean_object* l_Lean_Parser_Command_instance_formatter___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_computedField___closed__9; +static lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1; lean_object* l_Lean_Parser_checkColGtFn___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiers_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_rawIdent___elambda__1(lean_object*, lean_object*); @@ -4250,9 +4638,12 @@ static lean_object* l_Lean_Parser_Command_deriving___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_structInstBinder_formatter___closed__4; static lean_object* l_Lean_Parser_Command_attribute_formatter___closed__3; static lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_set__option___elambda__1___closed__6; +static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__26; static lean_object* l_Lean_Parser_Command_declModifiers___elambda__2___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classTk_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_export___closed__5; static lean_object* l_Lean_Parser_Command_eval___closed__7; static lean_object* l_Lean_Parser_Command_openOnly_formatter___closed__3; @@ -4267,7 +4658,9 @@ static lean_object* l_Lean_Parser_Command_declId_formatter___closed__11; lean_object* l_Lean_Parser_many1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_structCtor_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Tactic_open___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structure_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_exit___closed__4; static lean_object* l_Lean_Parser_Command_theorem___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_quot_parenthesizer___closed__1; @@ -4283,6 +4676,7 @@ static lean_object* l_Lean_Parser_Command_structCtor___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_theorem_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_check_declRange___closed__4; static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_declSig___elambda__1___closed__12; @@ -4293,12 +4687,13 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_check_declRange___closed_ static lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Term_open_declRange___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_quot___closed__2; static lean_object* l_Lean_Parser_Command_inductive___elambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Command_structInstBinder___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structExplicitBinder___closed__10; static lean_object* l_Lean_Parser_Command_optionValue___closed__7; -static lean_object* l_Lean_Parser_Command_declVal_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__1; static lean_object* l_Lean_Parser_Tactic_set__option___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_terminationByCore___closed__1; static lean_object* l_Lean_Parser_Command_declValEqns___closed__5; @@ -4313,6 +4708,7 @@ static lean_object* l_Lean_Parser_Command_declModifiers___closed__9; static lean_object* l_Lean_Parser_Command_declModifiers_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_open_declRange___closed__1; static lean_object* l_Lean_Parser_Term_open_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_open(lean_object*); static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_structure_formatter___closed__18; @@ -4343,13 +4739,12 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_variable(lean_object static lean_object* l_Lean_Parser_Command_initialize_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_moduleDoc___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_declValEqns_formatter___closed__1; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__17; static lean_object* l_Lean_Parser_Command_structure_formatter___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Command_export_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_def_formatter___closed__4; static lean_object* l_Lean_Parser_Command_openScoped___elambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_end___closed__2; -static lean_object* l_Lean_Parser_Command_initialize_formatter___closed__12; static lean_object* l_Lean_Parser_Command_genInjectiveTheorems___closed__3; static lean_object* l_Lean_Parser_Term_quot___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_declId_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -4359,8 +4754,11 @@ static lean_object* l_Lean_Parser_Command_terminationByElement___elambda__1___cl static lean_object* l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__4; lean_object* l_Lean_Parser_termParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_classInductive___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_theorem_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eval_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__2; lean_object* l_Lean_Parser_Term_whereDecls_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_init__quot___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_set__option___closed__3; @@ -4382,9 +4780,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_quot_declRange___closed__4; static lean_object* l_Lean_Parser_Command_section___closed__6; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_structure___elambda__1___closed__21; -static lean_object* l_Lean_Parser_Command_builtin__initialize___closed__8; static lean_object* l_Lean_Parser_Command_noncomputableSection___closed__3; -static lean_object* l_Lean_Parser_Command_openDecl_formatter___closed__5; static lean_object* l_Lean_Parser_Command_opaque___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_declModifiers___closed__4; static lean_object* l_Lean_Parser_Command_structure_formatter___closed__3; @@ -4399,15 +4795,16 @@ static lean_object* l_Lean_Parser_Command_computedField_formatter___closed__7; static lean_object* l_Lean_Parser_Command_check_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_declRange___closed__1; static lean_object* l_Lean_Parser_Command_declaration___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_declId___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_partial_formatter___closed__2; static lean_object* l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__7; lean_object* l_Lean_Parser_andthenFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_declModifiers_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_nonrec___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__1; static lean_object* l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_quot___elambda__1___closed__17; -static lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__36; static lean_object* _init_l_Lean_Parser_Term_quot___elambda__1___lambda__1___closed__1() { _start: { @@ -5048,7 +5445,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_docString___close _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Syntax quotation for terms and (lists of) commands. We prefer terms, so ambiguous quotations like\n `` `($x $y) `` will be parsed as an application, not two commands. Use `` `($x:command $y:command) `` instead.\n Multiple command will be put in a `` `null `` node, but a single command will not (so that you can directly\n match against a quotation in a command kind's elaborator). ", 382); +x_1 = lean_mk_string_from_bytes("Syntax quotation for terms and (lists of) commands. We prefer terms, so ambiguous quotations like\n`` `($x $y) `` will be parsed as an application, not two commands. Use `` `($x:command $y:command) `` instead.\nMultiple command will be put in a `` `null `` node, but a single command will not (so that you can directly\nmatch against a quotation in a command kind's elaborator). ", 376); return x_1; } } @@ -5268,6 +5665,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_quot___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Term_quot___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_quot_parenthesizer___closed__1() { _start: { @@ -5374,6 +5817,52 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_quot___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_quot___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__1() { _start: { @@ -5912,30 +6401,22 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quot_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_precheckedQuot_formatter___closed__2; -x_2 = l_Lean_Parser_Term_precheckedQuot_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_precheckedQuot_formatter___closed__4; +x_3 = l_Lean_Parser_Term_precheckedQuot_formatter___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -5948,11 +6429,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot_formatter(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_precheckedQuot_formatter___closed__1; -x_7 = l_Lean_Parser_Term_precheckedQuot_formatter___closed__5; +x_7 = l_Lean_Parser_Term_precheckedQuot_formatter___closed__4; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_precheckedQuot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1() { _start: { @@ -5984,30 +6495,22 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quot_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__4; +x_3 = l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -6020,11 +6523,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_precheckedQuot_parenthesizer(lean_ob { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__5; +x_7 = l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__4; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_precheckedQuot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Command_quot___elambda__1___lambda__1(lean_object* x_1) { _start: { @@ -6580,7 +7113,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Command_quot_docString___cl _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Syntax quotation for (sequences of) commands. The identical syntax for term quotations takes priority, so ambiguous quotations like\n `` `($x $y) `` will be parsed as an application, not two commands. Use `` `($x:command $y:command) `` instead.\n Multiple commands will be put in a `` `null `` node, but a single command will not (so that you can directly\n match against a quotation in a command kind's elaborator). ", 417); +x_1 = lean_mk_string_from_bytes("Syntax quotation for (sequences of) commands. The identical syntax for term quotations takes priority, so ambiguous quotations like\n`` `($x $y) `` will be parsed as an application, not two commands. Use `` `($x:command $y:command) `` instead.\nMultiple commands will be put in a `` `null `` node, but a single command will not (so that you can directly\nmatch against a quotation in a command kind's elaborator). ", 411); return x_1; } } @@ -6790,6 +7323,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_quot___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_quot___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_quot_parenthesizer___closed__1() { _start: { @@ -6886,6 +7449,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_quot___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_quot___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__1() { _start: { @@ -10111,6 +10704,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_moduleDoc___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_moduleDoc_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_moduleDoc___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1() { _start: { @@ -10213,6 +10836,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_moduleDoc___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_moduleDoc_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_moduleDoc___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedPrio___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -27742,6 +28395,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_private_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_private___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_private_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_private_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_private_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_private___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_private_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_private_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_protected_formatter___closed__1() { _start: { @@ -27794,15 +28477,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_visibility_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_private_formatter), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_protected___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_visibility_formatter___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__2() { _start: { lean_object* x_1; @@ -27810,12 +28495,24 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_protected_formatter), 5, return x_1; } } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_protected_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_protected___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Command_visibility_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_visibility_formatter___closed__1; -x_7 = l_Lean_Parser_Command_visibility_formatter___closed__2; +x_6 = l___regBuiltin_Lean_Parser_Command_private_formatter___closed__2; +x_7 = l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__2; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -27872,6 +28569,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_noncomputable___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_noncomputable_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_noncomputable___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_unsafe_formatter___closed__1() { _start: { @@ -27924,6 +28651,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_unsafe___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_unsafe_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_unsafe___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_partial_formatter___closed__1() { _start: { @@ -27976,6 +28733,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_partial___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_partial_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_partial_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_partial___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_nonrec_formatter___closed__1() { _start: { @@ -28028,6 +28815,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_nonrec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_nonrec_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_nonrec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__1() { _start: { @@ -28085,114 +28902,82 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__6() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_noncomputable_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__7() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_unsafe_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__8; +x_1 = l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_partial_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_nonrec_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__10; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__11; +x_1 = l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__12; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__8; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__9; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__13; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__7; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__7; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__14; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__6; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__16() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__5; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__15; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__13() { _start: { lean_object* x_1; lean_object* x_2; @@ -28202,7 +28987,7 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__18() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__14() { _start: { lean_object* x_1; @@ -28210,59 +28995,59 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attributes_formatter), 5, 0) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__19() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__18; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__17; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__14; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__13; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__20() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__19; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__15; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__21() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__20; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__16; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__16; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__22() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__3; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__21; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__17; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__23() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_declModifiers_formatter___closed__22; +x_3 = l_Lean_Parser_Command_declModifiers_formatter___closed__18; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -28270,7 +29055,7 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__24() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__20() { _start: { lean_object* x_1; @@ -28278,59 +29063,59 @@ x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_skip_formatter__ return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__25() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__18; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__24; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__14; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__20; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__26() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__25; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__21; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__27() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__26; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__16; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__22; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__28() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__3; -x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__27; +x_2 = l_Lean_Parser_Command_declModifiers_formatter___closed__23; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__29() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_formatter___closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_declModifiers_formatter___closed__28; +x_3 = l_Lean_Parser_Command_declModifiers_formatter___closed__24; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -28345,7 +29130,7 @@ if (x_1 == 0) { lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = l_Lean_Parser_Command_declModifiers_formatter___closed__1; -x_8 = l_Lean_Parser_Command_declModifiers_formatter___closed__23; +x_8 = l_Lean_Parser_Command_declModifiers_formatter___closed__19; x_9 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_7, x_8, x_2, x_3, x_4, x_5, x_6); return x_9; } @@ -28353,7 +29138,7 @@ else { lean_object* x_10; lean_object* x_11; lean_object* x_12; x_10 = l_Lean_Parser_Command_declModifiers_formatter___closed__1; -x_11 = l_Lean_Parser_Command_declModifiers_formatter___closed__29; +x_11 = l_Lean_Parser_Command_declModifiers_formatter___closed__25; x_12 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_10, x_11, x_2, x_3, x_4, x_5, x_6); return x_12; } @@ -28512,6 +29297,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declId___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declId_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declId_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_declId___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_optDeclSig_formatter___closed__1() { _start: { @@ -28635,6 +29450,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_optDeclSig___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_optDeclSig_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_optDeclSig___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declValSimple_formatter___closed__1() { _start: { @@ -28749,6 +29594,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declValSimple___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declValSimple_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_declValSimple___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declValEqns_formatter___closed__1() { _start: { @@ -28799,6 +29674,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declValEqns___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declValEqns_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_declValEqns___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_whereStructField_formatter___closed__1() { _start: { @@ -28849,6 +29754,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_whereStructField___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_whereStructField_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_whereStructField___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__1() { _start: { @@ -28880,22 +29815,14 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_whereStructField_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_whereStructInst_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -28905,13 +29832,13 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_whereStructInst_formatter___closed__4; +x_1 = l_Lean_Parser_Command_whereStructInst_formatter___closed__3; x_2 = l_Lean_Parser_Command_whereStructInst___elambda__1___closed__7; -x_3 = l_Lean_Parser_Command_whereStructInst_formatter___closed__5; +x_3 = l_Lean_Parser_Command_whereStructInst_formatter___closed__4; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_sepBy1Indent_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -28919,11 +29846,11 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_whereStructInst_formatter___closed__6; +x_1 = l_Lean_Parser_Command_whereStructInst_formatter___closed__5; x_2 = l_Lean_Parser_Command_declValSimple_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28931,25 +29858,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_whereStructInst_formatter___closed__2; -x_2 = l_Lean_Parser_Command_whereStructInst_formatter___closed__7; +x_2 = l_Lean_Parser_Command_whereStructInst_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_whereStructInst___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_whereStructInst_formatter___closed__8; +x_3 = l_Lean_Parser_Command_whereStructInst_formatter___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -28962,11 +29889,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_whereStructInst_formatter(lean_ob { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_whereStructInst_formatter___closed__1; -x_7 = l_Lean_Parser_Command_whereStructInst_formatter___closed__9; +x_7 = l_Lean_Parser_Command_whereStructInst_formatter___closed__8; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_whereStructInst___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_whereStructInst_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_whereStructInst___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declVal_formatter___closed__1() { _start: { @@ -28987,45 +29944,21 @@ return x_6; static lean_object* _init_l_Lean_Parser_Command_declVal_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declValEqns_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declVal_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_whereStructInst_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declVal_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declVal_formatter___closed__2; -x_2 = l_Lean_Parser_Command_declVal_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declVal_formatter___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declValSimple_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declVal_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_declVal_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declVal_formatter___closed__5; -x_2 = l_Lean_Parser_Command_declVal_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declVal_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -29037,7 +29970,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declVal_formatter(lean_object* x_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_declVal_formatter___closed__1; -x_7 = l_Lean_Parser_Command_declVal_formatter___closed__6; +x_7 = l_Lean_Parser_Command_declVal_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -29073,22 +30006,14 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_optDeclSig_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_ppIndent_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__4() { _start: { lean_object* x_1; @@ -29096,57 +30021,49 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declVal_formatter), 5, 0) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__4; -x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__5; +x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__3; +x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declId_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; -x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; +x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__2; -x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__8; +x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_abbrev___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_abbrev_formatter___closed__9; +x_3 = l_Lean_Parser_Command_abbrev_formatter___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -29159,11 +30076,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_abbrev_formatter(lean_object* x_1 { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_abbrev_formatter___closed__1; -x_7 = l_Lean_Parser_Command_abbrev_formatter___closed__10; +x_7 = l_Lean_Parser_Command_abbrev_formatter___closed__8; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_abbrev___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_abbrev_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_abbrev___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_optDefDeriving_formatter___closed__1() { _start: { @@ -29391,6 +30338,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_terminationByElement___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationByElement_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_terminationByElement___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__1() { _start: { @@ -29422,52 +30399,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationByElement_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_terminationBy_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1Indent_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_terminationBy_formatter___closed__2; -x_2 = l_Lean_Parser_Command_terminationBy_formatter___closed__4; +x_2 = l_Lean_Parser_Command_terminationBy_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_moduleDoc_formatter___closed__4; -x_2 = l_Lean_Parser_Command_terminationBy_formatter___closed__5; +x_2 = l_Lean_Parser_Command_terminationBy_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_terminationBy_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_terminationBy___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_terminationBy_formatter___closed__6; +x_3 = l_Lean_Parser_Command_terminationBy_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -29480,11 +30449,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationBy_formatter(lean_obje { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_terminationBy_formatter___closed__1; -x_7 = l_Lean_Parser_Command_terminationBy_formatter___closed__7; +x_7 = l_Lean_Parser_Command_terminationBy_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_terminationBy___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationBy_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationBy_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_terminationBy___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_terminationHintMany_formatter___closed__1() { _start: { @@ -29694,6 +30693,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_terminationByCore___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationByCore_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_terminationByCore___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_decreasingBy_formatter___closed__1() { _start: { @@ -29776,57 +30805,63 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationBy_formatter), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_decreasingBy___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationByCore_formatter), 5, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_decreasingBy_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_decreasingBy___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__1; -x_2 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__3; +x_1 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__1; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_decreasingBy_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -29836,8 +30871,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationSuffix_formatter(lean_ _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__4; -x_7 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__6; +x_6 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__2; +x_7 = l_Lean_Parser_Command_terminationSuffix_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_andthen_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -29902,7 +30937,7 @@ static lean_object* _init_l_Lean_Parser_Command_def_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__5; +x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__4; x_2 = l_Lean_Parser_Command_def_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -29914,7 +30949,7 @@ static lean_object* _init_l_Lean_Parser_Command_def_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__4; +x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__3; x_2 = l_Lean_Parser_Command_def_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -29926,7 +30961,7 @@ static lean_object* _init_l_Lean_Parser_Command_def_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; x_2 = l_Lean_Parser_Command_def_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -29970,6 +31005,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_def_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_def___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_def_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_def_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_def_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_def___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_def_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_def_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declSig_formatter___closed__1() { _start: { @@ -30032,6 +31097,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declSig___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declSig_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declSig_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_declSig___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_theorem_formatter___closed__1() { _start: { @@ -30063,27 +31158,31 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_theorem_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declSig_formatter), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2; +x_2 = lean_alloc_closure((void*)(l_Lean_ppIndent_formatter), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; } } static lean_object* _init_l_Lean_Parser_Command_theorem_formatter___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_theorem_formatter___closed__3; -x_2 = lean_alloc_closure((void*)(l_Lean_ppIndent_formatter), 6, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__4; +x_2 = l_Lean_Parser_Command_def_formatter___closed__4; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; } } static lean_object* _init_l_Lean_Parser_Command_theorem_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__5; -x_2 = l_Lean_Parser_Command_def_formatter___closed__4; +x_1 = l_Lean_Parser_Command_theorem_formatter___closed__3; +x_2 = l_Lean_Parser_Command_theorem_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -30094,7 +31193,7 @@ static lean_object* _init_l_Lean_Parser_Command_theorem_formatter___closed__6() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; x_2 = l_Lean_Parser_Command_theorem_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -30106,7 +31205,7 @@ static lean_object* _init_l_Lean_Parser_Command_theorem_formatter___closed__7() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; +x_1 = l_Lean_Parser_Command_theorem_formatter___closed__2; x_2 = l_Lean_Parser_Command_theorem_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -30117,22 +31216,10 @@ return x_3; static lean_object* _init_l_Lean_Parser_Command_theorem_formatter___closed__8() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_formatter___closed__2; -x_2 = l_Lean_Parser_Command_theorem_formatter___closed__7; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_theorem_formatter___closed__9() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_theorem___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_theorem_formatter___closed__8; +x_3 = l_Lean_Parser_Command_theorem_formatter___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -30145,11 +31232,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_theorem_formatter(lean_object* x_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_theorem_formatter___closed__1; -x_7 = l_Lean_Parser_Command_theorem_formatter___closed__9; +x_7 = l_Lean_Parser_Command_theorem_formatter___closed__8; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_theorem___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_theorem_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_theorem_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_theorem___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_opaque_formatter___closed__1() { _start: { @@ -30182,7 +31299,7 @@ static lean_object* _init_l_Lean_Parser_Command_opaque_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declVal_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -30192,7 +31309,7 @@ static lean_object* _init_l_Lean_Parser_Command_opaque_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_formatter___closed__4; +x_1 = l_Lean_Parser_Command_theorem_formatter___closed__3; x_2 = l_Lean_Parser_Command_opaque_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -30204,7 +31321,7 @@ static lean_object* _init_l_Lean_Parser_Command_opaque_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; x_2 = l_Lean_Parser_Command_opaque_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -30248,6 +31365,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_opaque___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_opaque_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_opaque_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_opaque___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_namedPrio_formatter___closed__1() { _start: { @@ -30389,7 +31536,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_optNamedPrio_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_namedPrio___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__2() { _start: { lean_object* x_1; @@ -30397,12 +31554,24 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_namedPrio_formatter), 5, return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_optNamedPrio_formatter___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namedPrio_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_namedPrio___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_optNamedPrio_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_optDeclSig_formatter___closed__5; -x_2 = l_Lean_Parser_Command_optNamedPrio_formatter___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -30413,7 +31582,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_optNamedPrio_formatter(lean_objec _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Command_optNamedPrio_formatter___closed__2; +x_6 = l_Lean_Parser_Command_optNamedPrio_formatter___closed__1; x_7 = l_Lean_Parser_optional_formatter(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -30451,7 +31620,7 @@ static lean_object* _init_l_Lean_Parser_Command_instance_formatter___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_optDeclSig_formatter___closed__5; -x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__7; +x_2 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -30473,7 +31642,7 @@ static lean_object* _init_l_Lean_Parser_Command_instance_formatter___closed__5() { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_instance_formatter___closed__4; -x_2 = l_Lean_Parser_Command_theorem_formatter___closed__6; +x_2 = l_Lean_Parser_Command_theorem_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -30556,6 +31725,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_instance___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_instance_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_instance_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_instance___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_axiom_formatter___closed__1() { _start: { @@ -30588,8 +31787,8 @@ static lean_object* _init_l_Lean_Parser_Command_axiom_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; -x_2 = l_Lean_Parser_Command_theorem_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; +x_2 = l_Lean_Parser_Command_theorem_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -30632,6 +31831,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_axiom___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_axiom_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_axiom_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_axiom___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_example_formatter___closed__1() { _start: { @@ -30664,8 +31893,8 @@ static lean_object* _init_l_Lean_Parser_Command_example_formatter___closed__3() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_formatter___closed__4; -x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__5; +x_1 = l_Lean_Parser_Command_theorem_formatter___closed__3; +x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -30708,6 +31937,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_example_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_example___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_example_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_example_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_example_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_example___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_example_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_example_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_ctor_formatter___closed__1() { _start: { @@ -30752,7 +32011,7 @@ static lean_object* _init_l_Lean_Parser_Command_ctor_formatter___closed__4() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declId_formatter___closed__4; -x_2 = l_Lean_Parser_Command_abbrev_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -30817,6 +32076,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_ctor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_ctor_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_ctor_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_ctor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_computedField_formatter___closed__1() { _start: { @@ -30927,6 +32216,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_computedField___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_computedField_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedField_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_computedField___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__1() { _start: { @@ -30958,62 +32277,54 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_computedField_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_computedFields_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_moduleDoc_formatter___closed__4; -x_2 = l_Lean_Parser_Command_computedFields_formatter___closed__4; +x_2 = l_Lean_Parser_Command_computedFields_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_computedFields_formatter___closed__5; +x_1 = l_Lean_Parser_Command_computedFields_formatter___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_manyIndent_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_computedFields_formatter___closed__2; -x_2 = l_Lean_Parser_Command_computedFields_formatter___closed__6; +x_2 = l_Lean_Parser_Command_computedFields_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_computedFields_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_computedFields___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_computedFields_formatter___closed__7; +x_3 = l_Lean_Parser_Command_computedFields_formatter___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -31026,11 +32337,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_computedFields_formatter(lean_obj { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_computedFields_formatter___closed__1; -x_7 = l_Lean_Parser_Command_computedFields_formatter___closed__8; +x_7 = l_Lean_Parser_Command_computedFields_formatter___closed__7; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_computedFields___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_computedFields_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_computedFields___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_derivingClasses_formatter___closed__1() { _start: { @@ -31189,6 +32530,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_optDeriving___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_optDeriving_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_optDeriving___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__1() { _start: { @@ -31242,138 +32613,114 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_ctor_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_inductive_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_computedFields_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__17; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__7; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__13; +x_2 = l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_inductive_formatter___closed__8; +x_1 = l_Lean_Parser_Command_inductive_formatter___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_optDeriving_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_inductive_formatter___closed__9; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__10; +x_1 = l_Lean_Parser_Command_inductive_formatter___closed__7; +x_2 = l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_inductive_formatter___closed__6; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__11; +x_1 = l_Lean_Parser_Command_inductive_formatter___closed__5; +x_2 = l_Lean_Parser_Command_inductive_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_inductive_formatter___closed__4; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__12; +x_2 = l_Lean_Parser_Command_inductive_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__3; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__13; +x_1 = l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2; +x_2 = l_Lean_Parser_Command_inductive_formatter___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__14; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; +x_2 = l_Lean_Parser_Command_inductive_formatter___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__16() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_inductive_formatter___closed__2; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__15; +x_2 = l_Lean_Parser_Command_inductive_formatter___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_inductive_formatter___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_inductive___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_inductive_formatter___closed__16; +x_3 = l_Lean_Parser_Command_inductive_formatter___closed__13; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -31386,11 +32733,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_inductive_formatter(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_inductive_formatter___closed__1; -x_7 = l_Lean_Parser_Command_inductive_formatter___closed__17; +x_7 = l_Lean_Parser_Command_inductive_formatter___closed__14; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_inductive___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_inductive_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_inductive_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_inductive___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_classInductive_formatter___closed__1() { _start: { @@ -31455,8 +32832,8 @@ static lean_object* _init_l_Lean_Parser_Command_classInductive_formatter___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_inductive_formatter___closed__6; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__10; +x_1 = l_Lean_Parser_Command_inductive_formatter___closed__5; +x_2 = l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -31479,7 +32856,7 @@ static lean_object* _init_l_Lean_Parser_Command_classInductive_formatter___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__4; +x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__3; x_2 = l_Lean_Parser_Command_classInductive_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -31491,7 +32868,7 @@ static lean_object* _init_l_Lean_Parser_Command_classInductive_formatter___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; x_2 = l_Lean_Parser_Command_classInductive_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -31535,6 +32912,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_classInductive___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_classInductive_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_classInductive___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structureTk_formatter___closed__1() { _start: { @@ -31587,6 +32994,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structureTk___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structureTk_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_structureTk___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_classTk_formatter___closed__1() { _start: { @@ -31629,6 +33066,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_classTk___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_classTk_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classTk_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_classTk___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_extends_formatter___closed__1() { _start: { @@ -31710,6 +33177,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_extends___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_extends_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_extends_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_extends___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structCtor_formatter___closed__1() { _start: { @@ -31796,6 +33293,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structCtor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structCtor_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_structCtor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structExplicitBinder_formatter___closed__1() { _start: { @@ -31900,7 +33427,7 @@ static lean_object* _init_l_Lean_Parser_Command_structExplicitBinder_formatter__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__4; +x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__3; x_2 = l_Lean_Parser_Command_structExplicitBinder_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -31956,6 +33483,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structExplicitBinder_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structImplicitBinder_formatter___closed__1() { _start: { @@ -32010,7 +33567,7 @@ static lean_object* _init_l_Lean_Parser_Command_structImplicitBinder_formatter__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2; x_2 = l_Lean_Parser_Command_declId_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -32066,6 +33623,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structImplicitBinder_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structInstBinder_formatter___closed__1() { _start: { @@ -32130,7 +33717,7 @@ static lean_object* _init_l_Lean_Parser_Command_structInstBinder_formatter___clo _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2; x_2 = l_Lean_Parser_Command_structInstBinder_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -32186,6 +33773,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structInstBinder___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structInstBinder_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_structInstBinder___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structSimpleBinder_formatter___closed__1() { _start: { @@ -32230,7 +33847,7 @@ static lean_object* _init_l_Lean_Parser_Command_structSimpleBinder_formatter___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2; x_2 = l_Lean_Parser_Command_structExplicitBinder_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -32274,6 +33891,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structSimpleBinder_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__1() { _start: { @@ -32295,82 +33942,50 @@ return x_7; static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structInstBinder_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structSimpleBinder_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structFields_formatter___closed__2; -x_2 = l_Lean_Parser_Command_structFields_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structImplicitBinder_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structFields_formatter___closed__5; -x_2 = l_Lean_Parser_Command_structFields_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__2; +x_2 = l_Lean_Parser_Command_structFields_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structExplicitBinder_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structFields_formatter___closed__7; -x_2 = l_Lean_Parser_Command_structFields_formatter___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__2; +x_2 = l_Lean_Parser_Command_structFields_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structFields_formatter___closed__8; +x_1 = l_Lean_Parser_Command_structFields_formatter___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__6() { _start: { lean_object* x_1; @@ -32378,47 +33993,47 @@ x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_checkColGe_forma return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structFields_formatter___closed__10; -x_2 = l_Lean_Parser_Command_structFields_formatter___closed__9; +x_1 = l_Lean_Parser_Command_structFields_formatter___closed__6; +x_2 = l_Lean_Parser_Command_structFields_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_moduleDoc_formatter___closed__4; -x_2 = l_Lean_Parser_Command_structFields_formatter___closed__11; +x_2 = l_Lean_Parser_Command_structFields_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structFields_formatter___closed__12; +x_1 = l_Lean_Parser_Command_structFields_formatter___closed__8; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_manyIndent_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_structFields_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_structFields___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_structFields_formatter___closed__13; +x_3 = l_Lean_Parser_Command_structFields_formatter___closed__9; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -32431,11 +34046,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_structFields_formatter(lean_objec { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_structFields_formatter___closed__1; -x_7 = l_Lean_Parser_Command_structFields_formatter___closed__14; +x_7 = l_Lean_Parser_Command_structFields_formatter___closed__10; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structFields___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structFields_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structFields_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_structFields___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__1() { _start: { @@ -32457,32 +34102,16 @@ return x_7; static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structureTk_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_classTk_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__2; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -32494,35 +34123,27 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__5; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_extends_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -32532,157 +34153,141 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_namedPrio_formatter___closed__6; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__9; +x_2 = l_Lean_Parser_Command_structure_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structCtor_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__11; +x_1 = l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__13() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structFields_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__12; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__13; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__10; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__14; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__7; +x_2 = l_Lean_Parser_Command_structure_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__16() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__15; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__10; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__16; -x_2 = l_Lean_Parser_Command_inductive_formatter___closed__10; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__11; +x_2 = l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__18() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_optDeclSig_formatter___closed__8; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__17; +x_2 = l_Lean_Parser_Command_structure_formatter___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__19() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__8; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__18; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__5; +x_2 = l_Lean_Parser_Command_structure_formatter___closed__13; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__20() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__6; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__19; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__4; +x_2 = l_Lean_Parser_Command_structure_formatter___closed__14; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__21() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__20; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; +x_2 = l_Lean_Parser_Command_structure_formatter___closed__15; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__22() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__4; -x_2 = l_Lean_Parser_Command_structure_formatter___closed__21; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__2; +x_2 = l_Lean_Parser_Command_structure_formatter___closed__16; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__23() { +static lean_object* _init_l_Lean_Parser_Command_structure_formatter___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_structure___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_structure_formatter___closed__22; +x_3 = l_Lean_Parser_Command_structure_formatter___closed__17; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -32695,11 +34300,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_structure_formatter(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_structure_formatter___closed__1; -x_7 = l_Lean_Parser_Command_structure_formatter___closed__23; +x_7 = l_Lean_Parser_Command_structure_formatter___closed__18; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structure___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structure_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structure_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_structure___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__1() { _start: { @@ -32732,210 +34367,130 @@ return x_3; static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_classInductive_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structure_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__3; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_inductive_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__6; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_example_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__8; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_example_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_axiom_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__10; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__9; +x_1 = l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__12() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_instance_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__12; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__11; +x_1 = l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__14() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_opaque_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__14; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__13; +x_1 = l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__16() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_theorem_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__16; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__15; +x_1 = l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__18() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_def_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__19() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__18; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__17; +x_1 = l___regBuiltin_Lean_Parser_Command_def_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__20() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_abbrev_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__21() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_formatter___closed__20; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__19; +x_1 = l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__2; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__22() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declaration_formatter___closed__2; -x_2 = l_Lean_Parser_Command_declaration_formatter___closed__21; +x_2 = l_Lean_Parser_Command_declaration_formatter___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__23() { +static lean_object* _init_l_Lean_Parser_Command_declaration_formatter___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_declaration___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_declaration_formatter___closed__22; +x_3 = l_Lean_Parser_Command_declaration_formatter___closed__12; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -32948,11 +34503,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declaration_formatter(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_declaration_formatter___closed__1; -x_7 = l_Lean_Parser_Command_declaration_formatter___closed__23; +x_7 = l_Lean_Parser_Command_declaration_formatter___closed__13; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declaration___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declaration_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_declaration___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_private_parenthesizer___closed__1() { _start: { @@ -33005,6 +34590,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_private___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_private_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_private_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_private___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_protected_parenthesizer___closed__1() { _start: { @@ -33057,15 +34672,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_visibility_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_private_parenthesizer), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_protected___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_visibility_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -33073,12 +34690,24 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_protected_parenthesizer), return x_1; } } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_protected_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_protected___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Command_visibility_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_visibility_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_visibility_parenthesizer___closed__2; +x_6 = l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__2; +x_7 = l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__2; x_8 = l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -33135,6 +34764,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_noncomputable___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_noncomputable_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_noncomputable___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_unsafe_parenthesizer___closed__1() { _start: { @@ -33187,6 +34846,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_unsafe___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_unsafe_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_unsafe___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_partial_parenthesizer___closed__1() { _start: { @@ -33239,6 +34928,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_partial___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_partial_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_partial_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_partial___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_nonrec_parenthesizer___closed__1() { _start: { @@ -33291,6 +35010,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_nonrec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_nonrec_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_nonrec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__1() { _start: { @@ -33348,114 +35097,82 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__6() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_noncomputable_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__7() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_unsafe_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__8; +x_1 = l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_partial_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_nonrec_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__10; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__11; +x_1 = l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__12; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__8; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__9; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__13; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__7; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__14; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__16() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__15; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__13() { _start: { lean_object* x_1; lean_object* x_2; @@ -33465,7 +35182,7 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__18() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__14() { _start: { lean_object* x_1; @@ -33473,59 +35190,59 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attributes_parenthesizer), 5 return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__19() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__18; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__17; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__14; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__13; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__20() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__19; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__15; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__21() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__20; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__16; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__16; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__22() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__21; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__17; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__23() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__22; +x_3 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__18; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -33533,7 +35250,7 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__24() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__20() { _start: { lean_object* x_1; @@ -33541,59 +35258,59 @@ x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_skip_parenth return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__25() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__18; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__24; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__14; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__20; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__26() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__25; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__21; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__27() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__26; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__16; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__22; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__28() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__27; +x_2 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__23; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__29() { +static lean_object* _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__28; +x_3 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__24; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -33608,7 +35325,7 @@ if (x_1 == 0) { lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__1; -x_8 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__23; +x_8 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__19; x_9 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_7, x_8, x_2, x_3, x_4, x_5, x_6); return x_9; } @@ -33616,7 +35333,7 @@ else { lean_object* x_10; lean_object* x_11; lean_object* x_12; x_10 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__1; -x_11 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__29; +x_11 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__25; x_12 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_10, x_11, x_2, x_3, x_4, x_5, x_6); return x_12; } @@ -33775,6 +35492,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declId___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declId_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declId_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_declId___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1() { _start: { @@ -33898,6 +35645,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_optDeclSig___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_optDeclSig_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_optDeclSig___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declValSimple_parenthesizer___closed__1() { _start: { @@ -34012,6 +35789,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declValSimple___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declValSimple_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_declValSimple___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declValEqns_parenthesizer___closed__1() { _start: { @@ -34062,6 +35869,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declValEqns___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declValEqns_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_declValEqns___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_whereStructField_parenthesizer___closed__1() { _start: { @@ -34112,6 +35949,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_whereStructField___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_whereStructField_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_whereStructField___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1() { _start: { @@ -34143,22 +36010,14 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_whereStructField_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -34168,13 +36027,13 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__3; x_2 = l_Lean_Parser_Command_whereStructInst___elambda__1___closed__7; -x_3 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__5; +x_3 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__4; x_4 = 1; x_5 = lean_box(x_4); x_6 = lean_alloc_closure((void*)(l_Lean_Parser_sepBy1Indent_parenthesizer___boxed), 9, 4); @@ -34185,11 +36044,11 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__5; x_2 = l_Lean_Parser_Command_declValSimple_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -34197,25 +36056,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__7; +x_2 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_whereStructInst___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__8; +x_3 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -34228,11 +36087,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_whereStructInst_parenthesizer(lea { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__9; +x_7 = l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__8; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_whereStructInst___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_whereStructInst_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_whereStructInst___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__1() { _start: { @@ -34253,45 +36142,21 @@ return x_6; static lean_object* _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declValEqns_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_whereStructInst_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declVal_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_declVal_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declValSimple_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declVal_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_declVal_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declVal_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -34303,7 +36168,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declVal_parenthesizer(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_declVal_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_declVal_parenthesizer___closed__6; +x_7 = l_Lean_Parser_Command_declVal_parenthesizer___closed__3; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -34339,22 +36204,14 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_optDeclSig_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppIndent_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__4() { _start: { lean_object* x_1; @@ -34362,57 +36219,49 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declVal_parenthesizer), 5 return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; +x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declId_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__8; +x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_abbrev___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__9; +x_3 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -34425,11 +36274,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_abbrev_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__10; +x_7 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__8; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_abbrev___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_abbrev_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_abbrev___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__1() { _start: { @@ -34657,6 +36536,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_terminationByElement___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationByElement_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_terminationByElement___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__1() { _start: { @@ -34688,52 +36597,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationByElement_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1Indent_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_terminationBy___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__6; +x_3 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -34746,11 +36647,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationBy_parenthesizer(lean_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__7; +x_7 = l_Lean_Parser_Command_terminationBy_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_terminationBy___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationBy_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_terminationBy___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__1() { _start: { @@ -34960,6 +36891,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_terminationByCore___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationByCore_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_terminationByCore___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1() { _start: { @@ -35042,57 +37003,63 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationBy_parenthesizer), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_decreasingBy___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_terminationByCore_parenthesizer), 5, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_decreasingBy_parenthesizer), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_decreasingBy___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__1; -x_2 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__1; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_decreasingBy_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -35102,8 +37069,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_terminationSuffix_parenthesizer(l _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__4; -x_7 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__6; +x_6 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__2; +x_7 = l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__3; x_8 = l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -35168,7 +37135,7 @@ static lean_object* _init_l_Lean_Parser_Command_def_parenthesizer___closed__6() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__4; x_2 = l_Lean_Parser_Command_def_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -35180,7 +37147,7 @@ static lean_object* _init_l_Lean_Parser_Command_def_parenthesizer___closed__7() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; x_2 = l_Lean_Parser_Command_def_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -35192,7 +37159,7 @@ static lean_object* _init_l_Lean_Parser_Command_def_parenthesizer___closed__8() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_def_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -35236,6 +37203,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_def___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_def_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_def_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_def___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declSig_parenthesizer___closed__1() { _start: { @@ -35298,6 +37295,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declSig___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declSig_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_declSig___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__1() { _start: { @@ -35329,26 +37356,18 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declSig_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppIndent_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__4; x_2 = l_Lean_Parser_Command_def_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -35356,49 +37375,49 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__3; +x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__7; +x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_theorem___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_theorem_parenthesizer___closed__8; +x_3 = l_Lean_Parser_Command_theorem_parenthesizer___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -35411,11 +37430,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_theorem_parenthesizer(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_theorem_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_theorem_parenthesizer___closed__9; +x_7 = l_Lean_Parser_Command_theorem_parenthesizer___closed__8; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_theorem___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_theorem_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_theorem___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_opaque_parenthesizer___closed__1() { _start: { @@ -35448,7 +37497,7 @@ static lean_object* _init_l_Lean_Parser_Command_opaque_parenthesizer___closed__3 _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_declVal_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -35458,7 +37507,7 @@ static lean_object* _init_l_Lean_Parser_Command_opaque_parenthesizer___closed__4 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__3; x_2 = l_Lean_Parser_Command_opaque_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -35470,7 +37519,7 @@ static lean_object* _init_l_Lean_Parser_Command_opaque_parenthesizer___closed__5 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_opaque_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -35514,6 +37563,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_opaque___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_opaque_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_opaque___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_namedPrio_parenthesizer___closed__1() { _start: { @@ -35657,7 +37736,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_namedPrio___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -35665,12 +37754,24 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_namedPrio_parenthesizer), return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_namedPrio___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -35681,7 +37782,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_optNamedPrio_parenthesizer(lean_o _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__2; +x_6 = l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__1; x_7 = l_Lean_Parser_optional_parenthesizer(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -35719,7 +37820,7 @@ static lean_object* _init_l_Lean_Parser_Command_instance_parenthesizer___closed_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; +x_2 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -35741,7 +37842,7 @@ static lean_object* _init_l_Lean_Parser_Command_instance_parenthesizer___closed_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_instance_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -35824,6 +37925,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_instance___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_instance_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_instance_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_instance___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_axiom_parenthesizer___closed__1() { _start: { @@ -35856,8 +37987,8 @@ static lean_object* _init_l_Lean_Parser_Command_axiom_parenthesizer___closed__3( _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_theorem_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -35900,6 +38031,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_axiom___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_axiom_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_axiom___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_example_parenthesizer___closed__1() { _start: { @@ -35932,8 +38093,8 @@ static lean_object* _init_l_Lean_Parser_Command_example_parenthesizer___closed__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__3; +x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -35976,6 +38137,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_example___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_example_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_example_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_example___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_ctor_parenthesizer___closed__1() { _start: { @@ -36020,7 +38211,7 @@ static lean_object* _init_l_Lean_Parser_Command_ctor_parenthesizer___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declId_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -36085,6 +38276,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_ctor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_ctor_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_ctor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_computedField_parenthesizer___closed__1() { _start: { @@ -36195,6 +38416,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_computedField___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_computedField_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_computedField___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__1() { _start: { @@ -36226,62 +38477,54 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_computedField_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_manyIndent_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_computedFields___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -36294,11 +38537,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_computedFields_parenthesizer(lean { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__8; +x_7 = l_Lean_Parser_Command_computedFields_parenthesizer___closed__7; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_computedFields___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_computedFields_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_computedFields___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__1() { _start: { @@ -36457,6 +38730,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_optDeriving___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_optDeriving_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_optDeriving___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__1() { _start: { @@ -36510,138 +38813,114 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_ctor_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_computedFields_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__17; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__7; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__13; +x_2 = l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__8; +x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_optDeriving_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__9; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__10; +x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__7; +x_2 = l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__11; +x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__12; +x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__13; +x_1 = l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__14; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__16() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__15; +x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_inductive___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_inductive_parenthesizer___closed__16; +x_3 = l_Lean_Parser_Command_inductive_parenthesizer___closed__13; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -36654,11 +38933,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_inductive_parenthesizer(lean_obje { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_inductive_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_inductive_parenthesizer___closed__17; +x_7 = l_Lean_Parser_Command_inductive_parenthesizer___closed__14; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_inductive___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_inductive_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_inductive___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_classInductive_parenthesizer___closed__1() { _start: { @@ -36723,8 +39032,8 @@ static lean_object* _init_l_Lean_Parser_Command_classInductive_parenthesizer___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__10; +x_1 = l_Lean_Parser_Command_inductive_parenthesizer___closed__5; +x_2 = l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -36747,7 +39056,7 @@ static lean_object* _init_l_Lean_Parser_Command_classInductive_parenthesizer___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; x_2 = l_Lean_Parser_Command_classInductive_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -36759,7 +39068,7 @@ static lean_object* _init_l_Lean_Parser_Command_classInductive_parenthesizer___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_classInductive_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -36803,6 +39112,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_classInductive___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_classInductive_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_classInductive___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structureTk_parenthesizer___closed__1() { _start: { @@ -36855,6 +39194,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structureTk___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structureTk_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_structureTk___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_classTk_parenthesizer___closed__1() { _start: { @@ -36897,6 +39266,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_classTk___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_classTk_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_classTk___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_extends_parenthesizer___closed__1() { _start: { @@ -36978,6 +39377,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_extends___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_extends_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_extends_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_extends___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structCtor_parenthesizer___closed__1() { _start: { @@ -37064,6 +39493,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structCtor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structCtor_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_structCtor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1() { _start: { @@ -37168,7 +39627,7 @@ static lean_object* _init_l_Lean_Parser_Command_structExplicitBinder_parenthesiz _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; x_2 = l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -37224,6 +39683,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structExplicitBinder_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_structExplicitBinder___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1() { _start: { @@ -37278,7 +39767,7 @@ static lean_object* _init_l_Lean_Parser_Command_structImplicitBinder_parenthesiz _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_declId_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -37334,6 +39823,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structImplicitBinder_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_structImplicitBinder___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1() { _start: { @@ -37398,7 +39917,7 @@ static lean_object* _init_l_Lean_Parser_Command_structInstBinder_parenthesizer__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -37454,6 +39973,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structInstBinder___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structInstBinder_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_structInstBinder___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1() { _start: { @@ -37498,7 +40047,7 @@ static lean_object* _init_l_Lean_Parser_Command_structSimpleBinder_parenthesizer _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -37542,6 +40091,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structSimpleBinder_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_structSimpleBinder___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__1() { _start: { @@ -37563,82 +40142,50 @@ return x_7; static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structInstBinder_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structSimpleBinder_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structImplicitBinder_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structExplicitBinder_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__8; +x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__6() { _start: { lean_object* x_1; @@ -37646,47 +40193,47 @@ x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_checkColGe_p return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__10; -x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__9; +x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__11; +x_2 = l_Lean_Parser_Command_structFields_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__12; +x_1 = l_Lean_Parser_Command_structFields_parenthesizer___closed__8; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_manyIndent_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_structFields___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_structFields_parenthesizer___closed__13; +x_3 = l_Lean_Parser_Command_structFields_parenthesizer___closed__9; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -37699,11 +40246,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_structFields_parenthesizer(lean_o { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_structFields_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_structFields_parenthesizer___closed__14; +x_7 = l_Lean_Parser_Command_structFields_parenthesizer___closed__10; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structFields___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structFields_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_structFields___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__1() { _start: { @@ -37725,32 +40302,16 @@ return x_7; static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structureTk_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_classTk_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -37762,35 +40323,27 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_extends_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -37800,157 +40353,141 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_namedPrio_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structCtor_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__11; +x_1 = l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__13() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structFields_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__12; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__13; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__10; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__14; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__7; +x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__16() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__15; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__10; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__16; -x_2 = l_Lean_Parser_Command_inductive_parenthesizer___closed__10; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__11; +x_2 = l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__18() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__8; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__17; +x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__19() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__8; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__18; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__13; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__20() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__19; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__14; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__21() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__20; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__15; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__22() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__21; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_structure_parenthesizer___closed__16; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__23() { +static lean_object* _init_l_Lean_Parser_Command_structure_parenthesizer___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_structure___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_structure_parenthesizer___closed__22; +x_3 = l_Lean_Parser_Command_structure_parenthesizer___closed__17; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -37963,11 +40500,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_structure_parenthesizer(lean_obje { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_structure_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_structure_parenthesizer___closed__23; +x_7 = l_Lean_Parser_Command_structure_parenthesizer___closed__18; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_structure___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structure_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_structure_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_structure___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__1() { _start: { @@ -38000,210 +40567,130 @@ return x_3; static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_classInductive_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_structure_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_inductive_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_example_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__8; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_axiom_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__10; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__9; +x_1 = l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__12() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_instance_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__12; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__11; +x_1 = l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__14() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_opaque_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__14; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__13; +x_1 = l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__16() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_theorem_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__16; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__15; +x_1 = l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__18() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_def_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__19() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__18; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__17; +x_1 = l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__20() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_abbrev_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__21() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__20; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__19; +x_1 = l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__22() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__21; +x_2 = l_Lean_Parser_Command_declaration_parenthesizer___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__23() { +static lean_object* _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_declaration___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_declaration_parenthesizer___closed__22; +x_3 = l_Lean_Parser_Command_declaration_parenthesizer___closed__12; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -38216,11 +40703,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_declaration_parenthesizer(lean_ob { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_declaration_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_declaration_parenthesizer___closed__23; +x_7 = l_Lean_Parser_Command_declaration_parenthesizer___closed__13; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declaration___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declaration_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_declaration___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_deriving___elambda__1___closed__1() { _start: { @@ -39072,6 +41589,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_deriving___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_deriving_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_deriving___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_deriving_parenthesizer___closed__1() { _start: { @@ -39182,6 +41729,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_deriving___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_deriving_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_deriving___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__1() { _start: { @@ -39812,6 +42389,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_noncomputableSection_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1() { _start: { @@ -39898,6 +42505,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_noncomputableSection_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_section___elambda__1___closed__1() { _start: { @@ -40374,6 +43011,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_section_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_section___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_section_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_section_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_section_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_section___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_section_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_section_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_section_parenthesizer___closed__1() { _start: { @@ -40416,6 +43083,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_section___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_section_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_section_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_section___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_namespace___elambda__1___closed__1() { _start: { @@ -40987,6 +43684,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_namespace___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_namespace_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namespace_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_namespace___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_namespace_parenthesizer___closed__1() { _start: { @@ -41051,6 +43778,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_namespace___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_namespace_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_namespace___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_end___elambda__1___closed__1() { _start: { @@ -41631,6 +44388,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_end_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_end___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_end_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_end_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_end___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_end_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_end_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_end_parenthesizer___closed__1() { _start: { @@ -41695,6 +44482,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_end___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_end_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_end_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_end___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_variable___elambda__1___closed__1() { _start: { @@ -42244,7 +45061,7 @@ static lean_object* _init_l_Lean_Parser_Command_variable_formatter___closed__3() _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_formatter___closed__5; +x_1 = l_Lean_Parser_Command_structure_formatter___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -42286,6 +45103,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_variable___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_variable_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_variable_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_variable___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_variable_parenthesizer___closed__1() { _start: { @@ -42318,7 +45165,7 @@ static lean_object* _init_l_Lean_Parser_Command_variable_parenthesizer___closed_ _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_structure_parenthesizer___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -42360,6 +45207,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_variable___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_variable_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_variable_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_variable___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_universe___elambda__1___closed__1() { _start: { @@ -42940,6 +45817,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_universe___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_universe_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_universe___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_universe_parenthesizer___closed__1() { _start: { @@ -43004,6 +45911,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_universe___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_universe_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_universe_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_universe___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_check___elambda__1___closed__1() { _start: { @@ -43579,6 +46516,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_check_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_check___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_check_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_check_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_check___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_check_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_check_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_check_parenthesizer___closed__1() { _start: { @@ -43643,6 +46610,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_check___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_check_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_check___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_check__failure___elambda__1___closed__1() { _start: { @@ -44218,6 +47215,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_check__failure___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_check__failure_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_check__failure___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_check__failure_parenthesizer___closed__1() { _start: { @@ -44282,6 +47309,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_check__failure___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_check__failure_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_check__failure___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_reduce___elambda__1___closed__1() { _start: { @@ -44857,6 +47914,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_reduce___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_reduce_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_reduce_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_reduce___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_reduce_parenthesizer___closed__1() { _start: { @@ -44921,6 +48008,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_reduce___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_reduce_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_reduce___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_eval___elambda__1___closed__1() { _start: { @@ -45496,6 +48613,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_eval___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_eval_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eval_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_eval___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_eval_parenthesizer___closed__1() { _start: { @@ -45560,6 +48707,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_eval___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_eval_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eval_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_eval___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_synth___elambda__1___closed__1() { _start: { @@ -46135,6 +49312,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_synth___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_synth_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_synth_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_synth___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_synth_parenthesizer___closed__1() { _start: { @@ -46199,6 +49406,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_synth___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_synth_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_synth_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_synth___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_exit___elambda__1___closed__1() { _start: { @@ -46670,6 +49907,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_exit___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_exit_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_exit_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_exit___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_exit_parenthesizer___closed__1() { _start: { @@ -46722,6 +49989,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_exit___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_exit_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_exit_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_exit___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_print___elambda__1___closed__1() { _start: { @@ -47351,6 +50648,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_print_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_print___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_print_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_print_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_print_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_print___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_print_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_print_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_print_parenthesizer___closed__1() { _start: { @@ -47435,6 +50762,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_print___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_print_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_print_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_print___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_printAxioms___elambda__1___closed__1() { _start: { @@ -48040,6 +51397,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_printAxioms___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_printAxioms_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_printAxioms___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_printAxioms_parenthesizer___closed__1() { _start: { @@ -48119,6 +51506,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_printAxioms___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_printAxioms_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_printAxioms___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_resolve__name___elambda__1___closed__1() { _start: { @@ -48690,6 +52107,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_resolve__name___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_resolve__name_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_resolve__name___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_resolve__name_parenthesizer___closed__1() { _start: { @@ -48754,6 +52201,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_resolve__name___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_resolve__name_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_resolve__name___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_init__quot___elambda__1___closed__1() { _start: { @@ -49217,6 +52694,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_init__quot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_init__quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_init__quot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_init__quot_parenthesizer___closed__1() { _start: { @@ -49269,6 +52776,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_init__quot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_init__quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_init__quot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_optionValue___elambda__1___closed__1() { _start: { @@ -50154,6 +53691,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_set__option___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_set__option_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_set__option_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_set__option___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_optionValue_parenthesizer___closed__1() { _start: { @@ -50318,6 +53885,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_set__option___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_set__option_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_set__option___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_eraseAttr___elambda__1___closed__1() { _start: { @@ -51589,6 +55186,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_eraseAttr___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_eraseAttr_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_eraseAttr___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__1() { _start: { @@ -51621,35 +55248,27 @@ static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__3( _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_eraseAttr_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__4() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attrInstance_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_attribute_formatter___closed__3; -x_2 = l_Lean_Parser_Command_attribute_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__2; +x_2 = l_Lean_Parser_Command_attribute_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Command_attribute_formatter___closed__5; +x_1 = l_Lean_Parser_Command_attribute_formatter___closed__4; x_2 = l_Lean_Parser_Command_declId___elambda__1___closed__8; x_3 = l_Lean_Parser_Command_declId_formatter___closed__3; x_4 = 0; @@ -51662,7 +55281,7 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -51672,11 +55291,11 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_attribute_formatter___closed__7; +x_1 = l_Lean_Parser_Command_attribute_formatter___closed__6; x_2 = l_Lean_Parser_Command_structExplicitBinder_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -51684,49 +55303,49 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_attribute_formatter___closed__6; -x_2 = l_Lean_Parser_Command_attribute_formatter___closed__8; +x_1 = l_Lean_Parser_Command_attribute_formatter___closed__5; +x_2 = l_Lean_Parser_Command_attribute_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_structInstBinder_formatter___closed__2; -x_2 = l_Lean_Parser_Command_attribute_formatter___closed__9; +x_2 = l_Lean_Parser_Command_attribute_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_attribute_formatter___closed__2; -x_2 = l_Lean_Parser_Command_attribute_formatter___closed__10; +x_2 = l_Lean_Parser_Command_attribute_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_attribute_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_attribute___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_attribute_formatter___closed__11; +x_3 = l_Lean_Parser_Command_attribute_formatter___closed__10; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -51739,11 +55358,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_attribute_formatter(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_attribute_formatter___closed__1; -x_7 = l_Lean_Parser_Command_attribute_formatter___closed__12; +x_7 = l_Lean_Parser_Command_attribute_formatter___closed__11; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_attribute___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_attribute_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_attribute_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_attribute___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1() { _start: { @@ -51816,6 +55465,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_eraseAttr___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_eraseAttr_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_eraseAttr___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__1() { _start: { @@ -51848,35 +55527,27 @@ static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_eraseAttr_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attrInstance_parenthesizer), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_attribute_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_attribute_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_attribute_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Command_attribute_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_attribute_parenthesizer___closed__4; x_2 = l_Lean_Parser_Command_declId___elambda__1___closed__8; x_3 = l_Lean_Parser_Command_declId_parenthesizer___closed__3; x_4 = 0; @@ -51889,7 +55560,7 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -51899,11 +55570,11 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_attribute_parenthesizer___closed__7; +x_1 = l_Lean_Parser_Command_attribute_parenthesizer___closed__6; x_2 = l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -51911,49 +55582,49 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_attribute_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Command_attribute_parenthesizer___closed__8; +x_1 = l_Lean_Parser_Command_attribute_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Command_attribute_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_attribute_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Command_attribute_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_attribute_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_attribute_parenthesizer___closed__10; +x_2 = l_Lean_Parser_Command_attribute_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_attribute___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_attribute_parenthesizer___closed__11; +x_3 = l_Lean_Parser_Command_attribute_parenthesizer___closed__10; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -51966,11 +55637,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_attribute_parenthesizer(lean_obje { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_attribute_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_attribute_parenthesizer___closed__12; +x_7 = l_Lean_Parser_Command_attribute_parenthesizer___closed__11; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_attribute___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_attribute_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_attribute___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_export___elambda__1___closed__1() { _start: { @@ -52838,6 +56539,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_export_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_export___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_export_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_export_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_export_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_export___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_export_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_export_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_export_parenthesizer___closed__1() { _start: { @@ -52948,6 +56679,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_export___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_export_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_export_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_export___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openHiding___elambda__1___closed__1() { _start: { @@ -56172,6 +59933,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openHiding___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openHiding_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_openHiding___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openRenamingItem_formatter___closed__1() { _start: { @@ -56250,6 +60041,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openRenamingItem_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openRenaming_formatter___closed__1() { _start: { @@ -56303,16 +60124,8 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_openRenaming_formatter___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openRenamingItem_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_openRenaming_formatter___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Command_openRenaming_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__2; x_2 = l_Lean_Parser_Command_declId___elambda__1___closed__8; x_3 = l_Lean_Parser_Command_declId_formatter___closed__3; x_4 = 0; @@ -56325,25 +60138,25 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Command_openRenaming_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_openRenaming_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_openRenaming_formatter___closed__4; -x_2 = l_Lean_Parser_Command_openRenaming_formatter___closed__6; +x_2 = l_Lean_Parser_Command_openRenaming_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openRenaming_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_openRenaming_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_openRenaming___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_openRenaming_formatter___closed__7; +x_3 = l_Lean_Parser_Command_openRenaming_formatter___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -56356,11 +60169,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenaming_formatter(lean_objec { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_openRenaming_formatter___closed__1; -x_7 = l_Lean_Parser_Command_openRenaming_formatter___closed__8; +x_7 = l_Lean_Parser_Command_openRenaming_formatter___closed__7; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openRenaming___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openRenaming_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenaming_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_openRenaming___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openOnly_formatter___closed__1() { _start: { @@ -56437,6 +60280,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openOnly___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openOnly_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_openOnly___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openSimple_formatter___closed__1() { _start: { @@ -56479,6 +60352,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openSimple___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openSimple_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_openSimple___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openScoped_formatter___closed__1() { _start: { @@ -56543,15 +60446,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openSimple_formatter), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openScoped___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__2() { _start: { lean_object* x_1; @@ -56559,72 +60464,60 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openScoped_formatter), 5, return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openScoped_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_openScoped___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_openDecl_formatter___closed__1; -x_2 = l_Lean_Parser_Command_openDecl_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openOnly_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_openDecl_formatter___closed__4; -x_2 = l_Lean_Parser_Command_openDecl_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__2; +x_2 = l_Lean_Parser_Command_openDecl_formatter___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openRenaming_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_openDecl_formatter___closed__6; -x_2 = l_Lean_Parser_Command_openDecl_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__2; +x_2 = l_Lean_Parser_Command_openDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_formatter___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openHiding_formatter), 5, 0); -return x_1; -} -} LEAN_EXPORT lean_object* l_Lean_Parser_Command_openDecl_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_openDecl_formatter___closed__8; -x_7 = l_Lean_Parser_Command_openDecl_formatter___closed__7; +x_6 = l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__2; +x_7 = l_Lean_Parser_Command_openDecl_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -56711,6 +60604,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_open_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_open___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_open_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_open_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_open_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_open___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_open_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_open_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openHiding_parenthesizer___closed__1() { _start: { @@ -56827,6 +60750,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openHiding___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openHiding_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_openHiding___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1() { _start: { @@ -56905,6 +60858,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openRenamingItem_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_openRenamingItem___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__1() { _start: { @@ -56958,16 +60941,8 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openRenamingItem_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_declId___elambda__1___closed__8; x_3 = l_Lean_Parser_Command_declId_parenthesizer___closed__3; x_4 = 0; @@ -56980,25 +60955,25 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_openRenaming___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -57011,11 +60986,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_openRenaming_parenthesizer(lean_o { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__8; +x_7 = l_Lean_Parser_Command_openRenaming_parenthesizer___closed__7; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openRenaming___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openRenaming_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_openRenaming___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openOnly_parenthesizer___closed__1() { _start: { @@ -57092,6 +61097,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openOnly___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openOnly_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_openOnly___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openSimple_parenthesizer___closed__1() { _start: { @@ -57134,6 +61169,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openSimple___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openSimple_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_openSimple___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_openScoped_parenthesizer___closed__1() { _start: { @@ -57198,15 +61263,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openSimple_parenthesizer), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_openScoped___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -57214,72 +61281,60 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openScoped_parenthesizer) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_openScoped___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__1; -x_2 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openOnly_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openRenaming_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_openHiding_parenthesizer), 5, 0); -return x_1; -} -} LEAN_EXPORT lean_object* l_Lean_Parser_Command_openDecl_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__8; -x_7 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__7; +x_6 = l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__2; +x_7 = l_Lean_Parser_Command_openDecl_parenthesizer___closed__3; x_8 = l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -57366,6 +61421,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_open___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_open_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_open_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_open___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_mutual___elambda__1___closed__1() { _start: { @@ -58252,6 +62337,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_mutual___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_mutual_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mutual_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_mutual___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_mutual_parenthesizer___closed__1() { _start: { @@ -58416,37 +62531,67 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_mutual___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("initialize", 10); +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_mutual_parenthesizer), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_mutual___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("initializeKeyword", 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_quot___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__1; +x_2 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__1; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1; +x_2 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; x_3 = 1; x_4 = 0; x_5 = l_Lean_Parser_mkAntiquot(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__4() { _start: { lean_object* x_1; @@ -58454,179 +62599,81 @@ x_1 = lean_mk_string_from_bytes("initialize ", 11); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__4; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__4; x_2 = l_String_trim(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__5; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__5; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quot___elambda__1___lambda__1___boxed), 3, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Parser_Term_typeSpec; -x_2 = lean_ctor_get(x_1, 0); -lean_inc(x_2); -x_3 = l_Lean_Parser_Term_leftArrow; -x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); -x_5 = l_Lean_Parser_andthenInfo(x_2, x_4); -return x_5; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__7() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_leftArrow___elambda__1), 2, 0); +x_1 = lean_mk_string_from_bytes("builtin_initialize ", 19); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declSig___elambda__1___closed__12; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__8; -x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_ident; -x_2 = lean_ctor_get(x_1, 0); -lean_inc(x_2); -x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__7; -x_4 = l_Lean_Parser_andthenInfo(x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_terminationHintMany___closed__6; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__9; -x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__11; -x_2 = lean_alloc_closure((void*)(l_Lean_Parser_atomicFn), 3, 1); -lean_closure_set(x_2, 0, x_1); +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__7; +x_2 = l_String_trim(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__10; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__12; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__13; -x_2 = l_Lean_Parser_optional(x_1); +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__8; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quot___elambda__1___lambda__1___boxed), 3, 1); +lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__15() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeq___elambda__1), 2, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__16() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__14; -x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__15; -x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); -lean_closure_set(x_4, 0, x_2); -lean_closure_set(x_4, 1, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__6; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__16; -x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__6; +x_2 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__9; +x_3 = lean_alloc_closure((void*)(l_Lean_Parser_orelseFn), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__18() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__11; -x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__17; -x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); -lean_closure_set(x_4, 0, x_2); -lean_closure_set(x_4, 1, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__19() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__18; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_2 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_nodeFn), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__20() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__19; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__11; x_2 = l_Lean_Parser_Term_quot___elambda__1___closed__20; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); @@ -58634,243 +62681,576 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__21() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_quot___elambda__1___closed__19; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__20; +x_2 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__22() { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword___elambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint32_t x_8; uint32_t x_9; uint8_t x_10; +x_3 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__3; +x_4 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_ctor_get(x_2, 2); +lean_inc(x_7); +x_8 = lean_string_utf8_get(x_6, x_7); +lean_dec(x_7); +lean_dec(x_6); +x_9 = 36; +x_10 = lean_uint32_dec_eq(x_8, x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_dec(x_4); +x_11 = lean_unsigned_to_nat(1024u); +x_12 = l_Lean_Parser_checkPrecFn(x_11, x_1, x_2); +x_13 = lean_ctor_get(x_12, 4); +lean_inc(x_13); +x_14 = lean_box(0); +x_15 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_13, x_14); +lean_dec(x_13); +if (x_15 == 0) +{ +lean_dec(x_1); +return x_12; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_16 = lean_ctor_get(x_12, 0); +lean_inc(x_16); +x_17 = lean_array_get_size(x_16); +lean_dec(x_16); +x_18 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__6; +x_19 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__9; +x_20 = 1; +lean_inc(x_1); +x_21 = l_Lean_Parser_orelseFnCore(x_18, x_19, x_20, x_1, x_12); +x_22 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_23 = l_Lean_Parser_ParserState_mkNode(x_21, x_22, x_17); +x_24 = lean_ctor_get(x_23, 4); +lean_inc(x_24); +x_25 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_24, x_14); +lean_dec(x_24); +if (x_25 == 0) +{ +lean_dec(x_1); +return x_23; +} +else +{ +lean_object* x_26; +x_26 = l_Lean_Parser_setLhsPrecFn(x_11, x_1, x_23); +lean_dec(x_1); +return x_26; +} +} +} +else +{ +lean_object* x_27; uint8_t x_28; lean_object* x_29; +x_27 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__13; +x_28 = 0; +x_29 = l_Lean_Parser_orelseFnCore(x_4, x_27, x_28, x_1, x_2); +return x_29; +} +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__5; +x_2 = l_Lean_Parser_symbolInfo(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__8; +x_2 = l_Lean_Parser_symbolInfo(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_quot___elambda__1___lambda__1___closed__1; +x_1 = l_Lean_Parser_Command_initializeKeyword___closed__1; +x_2 = l_Lean_Parser_Command_initializeKeyword___closed__2; +x_3 = l_Lean_Parser_orelseInfo(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_2 = l_Lean_Parser_Command_initializeKeyword___closed__3; +x_3 = l_Lean_Parser_nodeInfo(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_initializeKeyword___closed__4; +x_2 = l_Lean_Parser_epsilonInfo; +x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_epsilonInfo; +x_2 = l_Lean_Parser_Command_initializeKeyword___closed__5; +x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__3; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = l_Lean_Parser_Command_initializeKeyword___closed__6; +x_4 = l_Lean_Parser_orelseInfo(x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_initializeKeyword___elambda__1), 2, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_initializeKeyword___closed__7; +x_2 = l_Lean_Parser_Command_initializeKeyword___closed__8; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Parser_Command_initializeKeyword___closed__9; +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("initialize", 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_quot___elambda__1___closed__2; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__1; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = l_Lean_Parser_mkAntiquot(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Parser_Term_typeSpec; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = l_Lean_Parser_Term_leftArrow; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +x_5 = l_Lean_Parser_andthenInfo(x_2, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_leftArrow___elambda__1), 2, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declSig___elambda__1___closed__12; x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__5; -x_3 = lean_string_append(x_1, x_2); +x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_ident; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__4; +x_4 = l_Lean_Parser_andthenInfo(x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_terminationHintMany___closed__6; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__6; +x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__23() { +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__8; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_atomicFn), 3, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__22; -x_2 = l_Lean_Parser_Term_quot___elambda__1___lambda__1___closed__1; -x_3 = lean_string_append(x_1, x_2); +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__7; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__9; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__10; +x_2 = l_Lean_Parser_optional(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeq___elambda__1), 2, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__11; +x_2 = lean_ctor_get(x_1, 1); +lean_inc(x_2); +x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__12; +x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +lean_closure_set(x_4, 0, x_2); +lean_closure_set(x_4, 1, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_initializeKeyword___closed__8; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__13; +x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declModifiers___closed__10; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__14; +x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__15; +x_3 = lean_alloc_closure((void*)(l_Lean_Parser_nodeFn), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__16; +x_2 = l_Lean_Parser_Term_quot___elambda__1___closed__20; +x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initialize___elambda__1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_quot___elambda__1___closed__19; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__17; +x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); return x_3; } } LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize___elambda__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint32_t x_12; uint32_t x_13; uint8_t x_14; -x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__14; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint32_t x_10; uint32_t x_11; uint8_t x_12; +x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__11; x_4 = lean_ctor_get(x_3, 1); lean_inc(x_4); -x_5 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__11; +x_5 = l_Lean_Parser_Command_initialize___elambda__1___closed__3; x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); -x_7 = l_Lean_Parser_Command_initialize___elambda__1___closed__3; -x_8 = lean_ctor_get(x_7, 1); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); -x_9 = lean_ctor_get(x_1, 0); +lean_dec(x_7); +x_9 = lean_ctor_get(x_2, 2); lean_inc(x_9); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); +x_10 = lean_string_utf8_get(x_8, x_9); lean_dec(x_9); -x_11 = lean_ctor_get(x_2, 2); -lean_inc(x_11); -x_12 = lean_string_utf8_get(x_10, x_11); -lean_dec(x_11); -x_13 = 36; -x_14 = lean_uint32_dec_eq(x_12, x_13); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_dec(x_8); -x_15 = lean_unsigned_to_nat(1024u); -x_16 = l_Lean_Parser_checkPrecFn(x_15, x_1, x_2); -x_17 = lean_ctor_get(x_16, 4); -lean_inc(x_17); -x_18 = lean_box(0); -x_19 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_17, x_18); -lean_dec(x_17); -if (x_19 == 0) +x_11 = 36; +x_12 = lean_uint32_dec_eq(x_10, x_11); +if (x_12 == 0) { -lean_dec(x_10); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_dec(x_6); +x_13 = lean_unsigned_to_nat(1024u); +x_14 = l_Lean_Parser_checkPrecFn(x_13, x_1, x_2); +x_15 = lean_ctor_get(x_14, 4); +lean_inc(x_15); +x_16 = lean_box(0); +x_17 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_15, x_16); +lean_dec(x_15); +if (x_17 == 0) +{ lean_dec(x_4); lean_dec(x_1); -return x_16; +return x_14; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_16, 0); -lean_inc(x_20); -x_21 = lean_array_get_size(x_20); -lean_dec(x_20); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_18 = lean_ctor_get(x_14, 0); +lean_inc(x_18); +x_19 = lean_array_get_size(x_18); +lean_dec(x_18); lean_inc(x_1); -x_22 = lean_apply_2(x_6, x_1, x_16); -x_23 = lean_ctor_get(x_22, 4); -lean_inc(x_23); -x_24 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_23, x_18); -lean_dec(x_23); -if (x_24 == 0) +x_20 = l_Lean_Parser_Command_declModifiers___elambda__2(x_1, x_14); +x_21 = lean_ctor_get(x_20, 4); +lean_inc(x_21); +x_22 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_21, x_16); +lean_dec(x_21); +if (x_22 == 0) { -lean_dec(x_10); +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_dec(x_4); -x_25 = x_22; -goto block_31; +x_23 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_24 = l_Lean_Parser_ParserState_mkNode(x_20, x_23, x_19); +x_25 = lean_ctor_get(x_24, 4); +lean_inc(x_25); +x_26 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_25, x_16); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_dec(x_1); +return x_24; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint32_t x_36; uint32_t x_37; uint8_t x_38; -x_32 = l_Lean_Parser_Command_initialize___elambda__1___closed__5; -x_33 = l_Lean_Parser_Command_initialize___elambda__1___closed__23; -lean_inc(x_1); -x_34 = l_Lean_Parser_symbolFnAux(x_32, x_33, x_1, x_22); -x_35 = lean_ctor_get(x_34, 2); -lean_inc(x_35); -x_36 = lean_string_utf8_get(x_10, x_35); -lean_dec(x_35); -lean_dec(x_10); -x_37 = 37; -x_38 = lean_uint32_dec_eq(x_36, x_37); -if (x_38 == 0) -{ -lean_object* x_39; uint8_t x_40; -x_39 = lean_ctor_get(x_34, 4); -lean_inc(x_39); -x_40 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_39, x_18); -lean_dec(x_39); -if (x_40 == 0) -{ -lean_dec(x_4); -x_25 = x_34; -goto block_31; +lean_object* x_27; +x_27 = l_Lean_Parser_setLhsPrecFn(x_13, x_1, x_24); +lean_dec(x_1); +return x_27; +} } else { -lean_object* x_41; lean_object* x_42; uint8_t x_43; +lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_inc(x_1); -x_41 = lean_apply_2(x_4, x_1, x_34); -x_42 = lean_ctor_get(x_41, 4); -lean_inc(x_42); -x_43 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_42, x_18); -lean_dec(x_42); -if (x_43 == 0) +x_28 = l_Lean_Parser_Command_initializeKeyword___elambda__1(x_1, x_20); +x_29 = lean_ctor_get(x_28, 4); +lean_inc(x_29); +x_30 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_29, x_16); +lean_dec(x_29); +if (x_30 == 0) { -x_25 = x_41; -goto block_31; +lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +lean_dec(x_4); +x_31 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_32 = l_Lean_Parser_ParserState_mkNode(x_28, x_31, x_19); +x_33 = lean_ctor_get(x_32, 4); +lean_inc(x_33); +x_34 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_33, x_16); +lean_dec(x_33); +if (x_34 == 0) +{ +lean_dec(x_1); +return x_32; } else { -lean_object* x_44; -lean_inc(x_1); -x_44 = l_Lean_Parser_Term_doSeq___elambda__1(x_1, x_41); -x_25 = x_44; -goto block_31; -} +lean_object* x_35; +x_35 = l_Lean_Parser_setLhsPrecFn(x_13, x_1, x_32); +lean_dec(x_1); +return x_35; } } else { -lean_object* x_45; lean_object* x_46; uint8_t x_47; +lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_inc(x_1); -x_45 = l_Lean_Parser_tokenAntiquotFn(x_1, x_34); -x_46 = lean_ctor_get(x_45, 4); -lean_inc(x_46); -x_47 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_46, x_18); -lean_dec(x_46); -if (x_47 == 0) -{ -lean_dec(x_4); -x_25 = x_45; -goto block_31; -} -else +x_36 = lean_apply_2(x_4, x_1, x_28); +x_37 = lean_ctor_get(x_36, 4); +lean_inc(x_37); +x_38 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_37, x_16); +lean_dec(x_37); +if (x_38 == 0) { -lean_object* x_48; lean_object* x_49; uint8_t x_50; -lean_inc(x_1); -x_48 = lean_apply_2(x_4, x_1, x_45); -x_49 = lean_ctor_get(x_48, 4); -lean_inc(x_49); -x_50 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_49, x_18); -lean_dec(x_49); -if (x_50 == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_39 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_40 = l_Lean_Parser_ParserState_mkNode(x_36, x_39, x_19); +x_41 = lean_ctor_get(x_40, 4); +lean_inc(x_41); +x_42 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_41, x_16); +lean_dec(x_41); +if (x_42 == 0) { -x_25 = x_48; -goto block_31; +lean_dec(x_1); +return x_40; } else { -lean_object* x_51; -lean_inc(x_1); -x_51 = l_Lean_Parser_Term_doSeq___elambda__1(x_1, x_48); -x_25 = x_51; -goto block_31; -} -} +lean_object* x_43; +x_43 = l_Lean_Parser_setLhsPrecFn(x_13, x_1, x_40); +lean_dec(x_1); +return x_43; } } -block_31: +else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_26 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; -x_27 = l_Lean_Parser_ParserState_mkNode(x_25, x_26, x_21); -x_28 = lean_ctor_get(x_27, 4); -lean_inc(x_28); -x_29 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_28, x_18); -lean_dec(x_28); -if (x_29 == 0) +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; +lean_inc(x_1); +x_44 = l_Lean_Parser_Term_doSeq___elambda__1(x_1, x_36); +x_45 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_46 = l_Lean_Parser_ParserState_mkNode(x_44, x_45, x_19); +x_47 = lean_ctor_get(x_46, 4); +lean_inc(x_47); +x_48 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_47, x_16); +lean_dec(x_47); +if (x_48 == 0) { lean_dec(x_1); -return x_27; +return x_46; } else { -lean_object* x_30; -x_30 = l_Lean_Parser_setLhsPrecFn(x_15, x_1, x_27); +lean_object* x_49; +x_49 = l_Lean_Parser_setLhsPrecFn(x_13, x_1, x_46); lean_dec(x_1); -return x_30; -} +return x_49; } } } -else -{ -lean_object* x_52; uint8_t x_53; lean_object* x_54; -lean_dec(x_10); -lean_dec(x_6); -lean_dec(x_4); -x_52 = l_Lean_Parser_Command_initialize___elambda__1___closed__21; -x_53 = 0; -x_54 = l_Lean_Parser_orelseFnCore(x_8, x_52, x_53, x_1, x_2); -return x_54; } } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__1() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__5; -x_2 = l_Lean_Parser_symbolInfo(x_1); -return x_2; +lean_object* x_50; uint8_t x_51; lean_object* x_52; +lean_dec(x_4); +x_50 = l_Lean_Parser_Command_initialize___elambda__1___closed__18; +x_51 = 0; +x_52 = l_Lean_Parser_orelseFnCore(x_6, x_50, x_51, x_1, x_2); +return x_52; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__2() { +} +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__14; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__11; x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); x_3 = l_Lean_Parser_Term_doSeq; @@ -58880,71 +63260,73 @@ x_5 = l_Lean_Parser_andthenInfo(x_2, x_4); return x_5; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize___closed__1; -x_2 = l_Lean_Parser_Command_initialize___closed__2; -x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_initializeKeyword; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = l_Lean_Parser_Command_initialize___closed__1; +x_4 = l_Lean_Parser_andthenInfo(x_2, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__11; +x_1 = l_Lean_Parser_Command_declaration___closed__1; x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_initialize___closed__3; +x_3 = l_Lean_Parser_Command_initialize___closed__2; x_4 = l_Lean_Parser_andthenInfo(x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_initialize___closed__4; +x_2 = l_Lean_Parser_Command_initialize___closed__3; x_3 = l_Lean_Parser_nodeInfo(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize___closed__5; +x_1 = l_Lean_Parser_Command_initialize___closed__4; x_2 = l_Lean_Parser_epsilonInfo; x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_epsilonInfo; -x_2 = l_Lean_Parser_Command_initialize___closed__6; +x_2 = l_Lean_Parser_Command_initialize___closed__5; x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__3; x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_initialize___closed__7; +x_3 = l_Lean_Parser_Command_initialize___closed__6; x_4 = l_Lean_Parser_orelseInfo(x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__8() { _start: { lean_object* x_1; @@ -58952,12 +63334,12 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_initialize___elambda__1), return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initialize___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_initialize___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize___closed__8; -x_2 = l_Lean_Parser_Command_initialize___closed__9; +x_1 = l_Lean_Parser_Command_initialize___closed__7; +x_2 = l_Lean_Parser_Command_initialize___closed__8; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -58968,7 +63350,7 @@ static lean_object* _init_l_Lean_Parser_Command_initialize() { _start: { lean_object* x_1; -x_1 = l_Lean_Parser_Command_initialize___closed__10; +x_1 = l_Lean_Parser_Command_initialize___closed__9; return x_1; } } @@ -58989,7 +63371,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initialize_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(135u); +x_1 = lean_unsigned_to_nat(136u); x_2 = lean_unsigned_to_nat(24u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -59001,8 +63383,8 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initialize_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(135u); -x_2 = lean_unsigned_to_nat(173u); +x_1 = lean_unsigned_to_nat(136u); +x_2 = lean_unsigned_to_nat(177u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -59016,7 +63398,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___regBuiltin_Lean_Parser_Command_initialize_declRange___closed__1; x_2 = lean_unsigned_to_nat(24u); x_3 = l___regBuiltin_Lean_Parser_Command_initialize_declRange___closed__2; -x_4 = lean_unsigned_to_nat(173u); +x_4 = lean_unsigned_to_nat(177u); x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -59029,7 +63411,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initialize_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(135u); +x_1 = lean_unsigned_to_nat(136u); x_2 = lean_unsigned_to_nat(28u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -59041,7 +63423,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initialize_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(135u); +x_1 = lean_unsigned_to_nat(136u); x_2 = lean_unsigned_to_nat(40u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -59087,12 +63469,12 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__1() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__1; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1; +x_2 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; x_3 = 1; x_4 = 0; x_5 = lean_box(x_3); @@ -59105,119 +63487,45 @@ lean_closure_set(x_7, 3, x_6); return x_7; } } -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__2() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__4; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_leftArrow_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declSig_formatter___closed__2; -x_2 = l_Lean_Parser_Command_initialize_formatter___closed__3; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declId_formatter___closed__4; -x_2 = l_Lean_Parser_Command_initialize_formatter___closed__4; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize_formatter___closed__5; -x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_atomic_formatter), 6, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize_formatter___closed__6; -x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__7; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeq_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize_formatter___closed__7; -x_2 = l_Lean_Parser_Command_initialize_formatter___closed__8; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize_formatter___closed__2; -x_2 = l_Lean_Parser_Command_initialize_formatter___closed__9; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__5; -x_2 = l_Lean_Parser_Command_initialize_formatter___closed__10; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +x_1 = l_Lean_Parser_Command_initializeKeyword_formatter___closed__2; +x_2 = l_Lean_Parser_Command_initializeKeyword_formatter___closed__3; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_initialize_formatter___closed__11; +x_3 = l_Lean_Parser_Command_initializeKeyword_formatter___closed__4; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -59225,721 +63533,329 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_initialize_formatter___closed__1; -x_7 = l_Lean_Parser_Command_initialize_formatter___closed__12; +x_6 = l_Lean_Parser_Command_initializeKeyword_formatter___closed__1; +x_7 = l_Lean_Parser_Command_initializeKeyword_formatter___closed__5; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__1; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; -x_3 = 1; -x_4 = 0; -x_5 = lean_box(x_3); -x_6 = lean_box(x_4); -x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_parenthesizer___boxed), 9, 4); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, x_2); -lean_closure_set(x_7, 2, x_5); -lean_closure_set(x_7, 3, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__4; -x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_parenthesizer), 6, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_leftArrow_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declSig_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__3; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declId_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__4; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize_parenthesizer___closed__5; -x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_atomic_parenthesizer), 6, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initialize_parenthesizer___closed__6; -x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeq_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__8; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initialize_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__9; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__11() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__10; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; -x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_initialize_parenthesizer___closed__11; -x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_2); -lean_closure_set(x_4, 2, x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_initialize_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_initialize_parenthesizer___closed__12; -x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); -return x_8; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("builtin_initialize", 18); +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_initializeKeyword_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_quot___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1; -x_2 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__1; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; x_3 = 1; x_4 = 0; -x_5 = l_Lean_Parser_mkAntiquot(x_1, x_2, x_3, x_4); -return x_5; +x_5 = lean_box(x_3); +x_6 = lean_box(x_4); +x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_formatter___boxed), 9, 4); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +lean_closure_set(x_7, 2, x_5); +lean_closure_set(x_7, 3, x_6); +return x_7; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("builtin_initialize ", 19); +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_leftArrow_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__4; -x_2 = l_String_trim(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5; -x_2 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quot___elambda__1___lambda__1___boxed), 3, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__6; -x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__16; -x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__11; -x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -x_3 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__7; -x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); -lean_closure_set(x_4, 0, x_2); -lean_closure_set(x_4, 1, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__8; -x_3 = lean_alloc_closure((void*)(l_Lean_Parser_nodeFn), 4, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__9; -x_2 = l_Lean_Parser_Term_quot___elambda__1___closed__20; -x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_quot___elambda__1___closed__19; -x_2 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__10; -x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_quot___elambda__1___lambda__1___closed__1; -x_2 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5; -x_3 = lean_string_append(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__12; -x_2 = l_Lean_Parser_Term_quot___elambda__1___lambda__1___closed__1; -x_3 = lean_string_append(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Parser_Command_builtin__initialize___elambda__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint32_t x_12; uint32_t x_13; uint8_t x_14; -x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__14; -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -x_5 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__11; -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -x_7 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__3; -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_ctor_get(x_2, 2); -lean_inc(x_11); -x_12 = lean_string_utf8_get(x_10, x_11); -lean_dec(x_11); -x_13 = 36; -x_14 = lean_uint32_dec_eq(x_12, x_13); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_dec(x_8); -x_15 = lean_unsigned_to_nat(1024u); -x_16 = l_Lean_Parser_checkPrecFn(x_15, x_1, x_2); -x_17 = lean_ctor_get(x_16, 4); -lean_inc(x_17); -x_18 = lean_box(0); -x_19 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_17, x_18); -lean_dec(x_17); -if (x_19 == 0) -{ -lean_dec(x_10); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_1); -return x_16; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_16, 0); -lean_inc(x_20); -x_21 = lean_array_get_size(x_20); -lean_dec(x_20); -lean_inc(x_1); -x_22 = lean_apply_2(x_6, x_1, x_16); -x_23 = lean_ctor_get(x_22, 4); -lean_inc(x_23); -x_24 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_23, x_18); -lean_dec(x_23); -if (x_24 == 0) -{ -lean_dec(x_10); -lean_dec(x_4); -x_25 = x_22; -goto block_31; -} -else -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint32_t x_36; uint32_t x_37; uint8_t x_38; -x_32 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5; -x_33 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__13; -lean_inc(x_1); -x_34 = l_Lean_Parser_symbolFnAux(x_32, x_33, x_1, x_22); -x_35 = lean_ctor_get(x_34, 2); -lean_inc(x_35); -x_36 = lean_string_utf8_get(x_10, x_35); -lean_dec(x_35); -lean_dec(x_10); -x_37 = 37; -x_38 = lean_uint32_dec_eq(x_36, x_37); -if (x_38 == 0) -{ -lean_object* x_39; uint8_t x_40; -x_39 = lean_ctor_get(x_34, 4); -lean_inc(x_39); -x_40 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_39, x_18); -lean_dec(x_39); -if (x_40 == 0) -{ -lean_dec(x_4); -x_25 = x_34; -goto block_31; -} -else -{ -lean_object* x_41; lean_object* x_42; uint8_t x_43; -lean_inc(x_1); -x_41 = lean_apply_2(x_4, x_1, x_34); -x_42 = lean_ctor_get(x_41, 4); -lean_inc(x_42); -x_43 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_42, x_18); -lean_dec(x_42); -if (x_43 == 0) -{ -x_25 = x_41; -goto block_31; -} -else -{ -lean_object* x_44; -lean_inc(x_1); -x_44 = l_Lean_Parser_Term_doSeq___elambda__1(x_1, x_41); -x_25 = x_44; -goto block_31; -} -} -} -else -{ -lean_object* x_45; lean_object* x_46; uint8_t x_47; -lean_inc(x_1); -x_45 = l_Lean_Parser_tokenAntiquotFn(x_1, x_34); -x_46 = lean_ctor_get(x_45, 4); -lean_inc(x_46); -x_47 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_46, x_18); -lean_dec(x_46); -if (x_47 == 0) -{ -lean_dec(x_4); -x_25 = x_45; -goto block_31; -} -else -{ -lean_object* x_48; lean_object* x_49; uint8_t x_50; -lean_inc(x_1); -x_48 = lean_apply_2(x_4, x_1, x_45); -x_49 = lean_ctor_get(x_48, 4); -lean_inc(x_49); -x_50 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_49, x_18); -lean_dec(x_49); -if (x_50 == 0) -{ -x_25 = x_48; -goto block_31; -} -else -{ -lean_object* x_51; -lean_inc(x_1); -x_51 = l_Lean_Parser_Term_doSeq___elambda__1(x_1, x_48); -x_25 = x_51; -goto block_31; -} -} -} -} -block_31: -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_26 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; -x_27 = l_Lean_Parser_ParserState_mkNode(x_25, x_26, x_21); -x_28 = lean_ctor_get(x_27, 4); -lean_inc(x_28); -x_29 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_28, x_18); -lean_dec(x_28); -if (x_29 == 0) -{ -lean_dec(x_1); -return x_27; -} -else -{ -lean_object* x_30; -x_30 = l_Lean_Parser_setLhsPrecFn(x_15, x_1, x_27); -lean_dec(x_1); -return x_30; -} -} +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declSig_formatter___closed__2; +x_2 = l_Lean_Parser_Command_initialize_formatter___closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; } } -else +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__4() { +_start: { -lean_object* x_52; uint8_t x_53; lean_object* x_54; -lean_dec(x_10); -lean_dec(x_6); -lean_dec(x_4); -x_52 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__11; -x_53 = 0; -x_54 = l_Lean_Parser_orelseFnCore(x_8, x_52, x_53, x_1, x_2); -return x_54; -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_declId_formatter___closed__4; +x_2 = l_Lean_Parser_Command_initialize_formatter___closed__3; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__1() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5; -x_2 = l_Lean_Parser_symbolInfo(x_1); +x_1 = l_Lean_Parser_Command_initialize_formatter___closed__4; +x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_atomic_formatter), 6, 1); +lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__2() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__6() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize___closed__1; -x_2 = l_Lean_Parser_Command_initialize___closed__2; -x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initialize_formatter___closed__5; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__7() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_declModifiers___elambda__2___closed__11; -x_2 = lean_ctor_get(x_1, 0); -lean_inc(x_2); -x_3 = l_Lean_Parser_Command_builtin__initialize___closed__2; -x_4 = l_Lean_Parser_andthenInfo(x_2, x_3); -return x_4; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeq_formatter), 5, 0); +return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_builtin__initialize___closed__3; -x_3 = l_Lean_Parser_nodeInfo(x_1, x_2); +x_1 = l_Lean_Parser_Command_initialize_formatter___closed__6; +x_2 = l_Lean_Parser_Command_initialize_formatter___closed__7; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize___closed__4; -x_2 = l_Lean_Parser_epsilonInfo; -x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); +x_1 = l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__2; +x_2 = l_Lean_Parser_Command_initialize_formatter___closed__8; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_epsilonInfo; -x_2 = l_Lean_Parser_Command_builtin__initialize___closed__5; -x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); +x_1 = l_Lean_Parser_Command_declaration_formatter___closed__2; +x_2 = l_Lean_Parser_Command_initialize_formatter___closed__9; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_initialize_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__3; -x_2 = lean_ctor_get(x_1, 0); -lean_inc(x_2); -x_3 = l_Lean_Parser_Command_builtin__initialize___closed__6; -x_4 = l_Lean_Parser_orelseInfo(x_2, x_3); +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Lean_Parser_Command_initialize_formatter___closed__10; +x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); +lean_closure_set(x_4, 0, x_1); +lean_closure_set(x_4, 1, x_2); +lean_closure_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__8() { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_builtin__initialize___elambda__1), 2, 0); -return x_1; +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = l_Lean_Parser_Command_initialize_formatter___closed__1; +x_7 = l_Lean_Parser_Command_initialize_formatter___closed__11; +x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); +return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize___closed__9() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize___closed__7; -x_2 = l_Lean_Parser_Command_builtin__initialize___closed__8; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__2() { _start: { lean_object* x_1; -x_1 = l_Lean_Parser_Command_builtin__initialize___closed__9; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_initialize_formatter), 5, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize_formatter(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_2 = l_Lean_Parser_Command_quot___elambda__1___closed__7; -x_3 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; -x_4 = 1; -x_5 = l_Lean_Parser_Command_builtin__initialize; -x_6 = lean_unsigned_to_nat(1000u); -x_7 = l_Lean_Parser_addBuiltinParser(x_2, x_3, x_4, x_5, x_6, x_1); -return x_7; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } -static lean_object* _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__1() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(136u); -x_2 = lean_unsigned_to_nat(24u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1; +x_2 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = lean_box(x_3); +x_6 = lean_box(x_4); +x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_parenthesizer___boxed), 9, 4); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +lean_closure_set(x_7, 2, x_5); +lean_closure_set(x_7, 3, x_6); +return x_7; } } -static lean_object* _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__2() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(136u); -x_2 = lean_unsigned_to_nat(189u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__4; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_parenthesizer), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__1; -x_2 = lean_unsigned_to_nat(24u); -x_3 = l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__2; -x_4 = lean_unsigned_to_nat(189u); -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__7; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_parenthesizer), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(136u); -x_2 = lean_unsigned_to_nat(28u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); +x_1 = l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__3; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(136u); -x_2 = lean_unsigned_to_nat(48u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_2 = lean_unsigned_to_nat(1024u); +x_3 = l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__4; +x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); +lean_closure_set(x_4, 0, x_1); +lean_closure_set(x_4, 1, x_2); +lean_closure_set(x_4, 2, x_3); +return x_4; } } -static lean_object* _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__6() { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initializeKeyword_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__4; -x_2 = lean_unsigned_to_nat(28u); -x_3 = l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__5; -x_4 = lean_unsigned_to_nat(48u); -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1; +x_7 = l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__5; +x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); +return x_8; } } -static lean_object* _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__7() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__3; -x_2 = l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__6; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); +x_1 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange(lean_object* x_1) { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2() { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; -x_3 = l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__7; -x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); -return x_4; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_initializeKeyword_parenthesizer), 5, 0); +return x_1; +} } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__1() { +} +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__1() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1; -x_2 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__1; +x_2 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; x_3 = 1; x_4 = 0; x_5 = lean_box(x_3); x_6 = lean_box(x_4); -x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_formatter___boxed), 9, 4); +x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_parenthesizer___boxed), 9, 4); lean_closure_set(x_7, 0, x_1); lean_closure_set(x_7, 1, x_2); lean_closure_set(x_7, 2, x_5); @@ -59947,123 +63863,109 @@ lean_closure_set(x_7, 3, x_6); return x_7; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__2() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__4; -x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_formatter), 6, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_leftArrow_parenthesizer), 5, 0); +return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize_formatter___closed__2; -x_2 = l_Lean_Parser_Command_initialize_formatter___closed__9; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +x_1 = l_Lean_Parser_Command_declSig_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__5; -x_2 = l_Lean_Parser_Command_builtin__initialize_formatter___closed__3; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +x_1 = l_Lean_Parser_Command_declId_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__3; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; -x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_builtin__initialize_formatter___closed__4; -x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_2); -lean_closure_set(x_4, 2, x_3); -return x_4; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initialize_parenthesizer___closed__4; +x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_atomic_parenthesizer), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_builtin__initialize_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__6() { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_builtin__initialize_formatter___closed__1; -x_7 = l_Lean_Parser_Command_builtin__initialize_formatter___closed__5; -x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); -return x_8; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initialize_parenthesizer___closed__5; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__1() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__7() { _start: { -lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1; -x_2 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; -x_3 = 1; -x_4 = 0; -x_5 = lean_box(x_3); -x_6 = lean_box(x_4); -x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_parenthesizer___boxed), 9, 4); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, x_2); -lean_closure_set(x_7, 2, x_5); -lean_closure_set(x_7, 3, x_6); -return x_7; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeq_parenthesizer), 5, 0); +return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__2() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__8() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__4; -x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_parenthesizer), 6, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_initialize_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__7; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__9; +x_1 = l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Command_declaration_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_initialize_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__4; +x_3 = l_Lean_Parser_Command_initialize_parenthesizer___closed__10; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -60071,16 +63973,46 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_builtin__initialize_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initialize_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__5; +x_6 = l_Lean_Parser_Command_initialize_parenthesizer___closed__1; +x_7 = l_Lean_Parser_Command_initialize_parenthesizer___closed__11; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_initialize_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_initialize___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_in___elambda__1___closed__1() { _start: { @@ -60449,6 +64381,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_in_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_in___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_in_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_in_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_in_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_in___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_in_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_in_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_in_parenthesizer___closed__1() { _start: { @@ -60493,6 +64455,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_in___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_in_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_in_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_in___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__1() { _start: { @@ -61064,6 +65056,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_genInjectiveTheorems_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1() { _start: { @@ -61128,6 +65150,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Command_declModifiersF_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -61180,7 +65232,7 @@ x_1 = l_Lean_Parser_Command_ctor___closed__2; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__1() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -61190,7 +65242,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__2() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__2() { _start: { lean_object* x_1; lean_object* x_2; @@ -61200,7 +65252,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__3() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -61210,7 +65262,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__4() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -61220,11 +65272,11 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__5() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__5() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__4; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__4; x_2 = 1; x_3 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -61232,7 +65284,7 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__6() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__6() { _start: { lean_object* x_1; @@ -61240,17 +65292,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersF_formatter) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__7() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__6; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__6; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__8() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__8() { _start: { lean_object* x_1; @@ -61258,7 +65310,7 @@ x_1 = l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__9() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__9() { _start: { lean_object* x_1; @@ -61266,17 +65318,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersF_parenthesi return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__10() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__10() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__9; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__9; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__11() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__11() { _start: { lean_object* x_1; @@ -61284,7 +65336,7 @@ x_1 = l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__12() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__12() { _start: { lean_object* x_1; @@ -61292,17 +65344,17 @@ x_1 = lean_mk_string_from_bytes("nestedDeclModifiers", 19); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__13() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__12; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__14() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__14() { _start: { lean_object* x_1; lean_object* x_2; @@ -61312,7 +65364,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__15() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__15() { _start: { lean_object* x_1; @@ -61320,17 +65372,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersT_formatter) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__16() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__15; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__15; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__17() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__17() { _start: { lean_object* x_1; @@ -61338,17 +65390,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_declModifiersT_parenthesi return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__18() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__18() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__17; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__17; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__19() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -61358,7 +65410,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__20() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__20() { _start: { lean_object* x_1; lean_object* x_2; @@ -61368,7 +65420,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__21() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__21() { _start: { lean_object* x_1; lean_object* x_2; @@ -61378,27 +65430,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__22() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__22() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__23() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__23() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__24() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -61408,7 +65460,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__25() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__25() { _start: { lean_object* x_1; lean_object* x_2; @@ -61418,7 +65470,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__26() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__26() { _start: { lean_object* x_1; lean_object* x_2; @@ -61428,27 +65480,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__27() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__27() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_theorem_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__28() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__28() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_theorem_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__29() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__29() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -61458,7 +65510,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__30() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__30() { _start: { lean_object* x_1; lean_object* x_2; @@ -61468,7 +65520,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__31() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__31() { _start: { lean_object* x_1; lean_object* x_2; @@ -61478,27 +65530,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__32() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__32() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__5; +x_1 = l_Lean_Parser_Command_abbrev_formatter___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_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__33() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__33() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___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_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__34() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__34() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -61508,7 +65560,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__35() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__35() { _start: { lean_object* x_1; lean_object* x_2; @@ -61518,7 +65570,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__36() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__36() { _start: { lean_object* x_1; lean_object* x_2; @@ -61528,27 +65580,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__37() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__37() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_abbrev_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__38() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__38() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_abbrev_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__39() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__39() { _start: { lean_object* x_1; @@ -61556,17 +65608,17 @@ x_1 = lean_mk_string_from_bytes("openDecl", 8); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__40() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__40() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__39; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__39; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__41() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__41() { _start: { lean_object* x_1; lean_object* x_2; @@ -61576,27 +65628,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__42() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__42() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_quot___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__39; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__39; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__43() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__43() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__42; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__42; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__44() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__44() { _start: { lean_object* x_1; lean_object* x_2; @@ -61606,7 +65658,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__45() { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__45() { _start: { lean_object* x_1; lean_object* x_2; @@ -61616,14 +65668,82 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493_(lean_object* x_1) { +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__46() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("docComment", 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__47() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__46; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__48() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_docComment; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__49() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_quot___elambda__1___closed__2; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__46; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__50() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__49; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__51() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_declModifiers_formatter___closed__2; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__52() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_declModifiers_parenthesizer___closed__2; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__1; -x_3 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__2; -x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__3; -x_5 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__5; +x_2 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__1; +x_3 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__2; +x_4 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__3; +x_5 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__5; x_6 = l_Lean_Parser_registerAlias(x_2, x_3, x_4, x_5, x_1); if (lean_obj_tag(x_6) == 0) { @@ -61631,8 +65751,8 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); -x_8 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__8; -x_9 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__7; +x_8 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__8; +x_9 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__7; x_10 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_2, x_9, x_7); if (lean_obj_tag(x_10) == 0) { @@ -61640,8 +65760,8 @@ lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_10, 1); lean_inc(x_11); lean_dec(x_10); -x_12 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__11; -x_13 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__10; +x_12 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__11; +x_13 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__10; x_14 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_2, x_13, x_11); if (lean_obj_tag(x_14) == 0) { @@ -61649,8 +65769,8 @@ lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; x_15 = lean_ctor_get(x_14, 1); lean_inc(x_15); lean_dec(x_14); -x_16 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__13; -x_17 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__14; +x_16 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__13; +x_17 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__14; x_18 = l_Lean_Parser_registerAlias(x_16, x_17, x_4, x_5, x_15); if (lean_obj_tag(x_18) == 0) { @@ -61658,7 +65778,7 @@ lean_object* x_19; lean_object* x_20; lean_object* x_21; x_19 = lean_ctor_get(x_18, 1); lean_inc(x_19); lean_dec(x_18); -x_20 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__16; +x_20 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__16; x_21 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_16, x_20, x_19); if (lean_obj_tag(x_21) == 0) { @@ -61666,7 +65786,7 @@ lean_object* x_22; lean_object* x_23; lean_object* x_24; x_22 = lean_ctor_get(x_21, 1); lean_inc(x_22); lean_dec(x_21); -x_23 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__18; +x_23 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__18; x_24 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_16, x_23, x_22); if (lean_obj_tag(x_24) == 0) { @@ -61674,9 +65794,9 @@ lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); lean_dec(x_24); -x_26 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__19; -x_27 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__20; -x_28 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__21; +x_26 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__19; +x_27 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__20; +x_28 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__21; x_29 = l_Lean_Parser_registerAlias(x_26, x_27, x_28, x_5, x_25); if (lean_obj_tag(x_29) == 0) { @@ -61684,7 +65804,7 @@ lean_object* x_30; lean_object* x_31; lean_object* x_32; x_30 = lean_ctor_get(x_29, 1); lean_inc(x_30); lean_dec(x_29); -x_31 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__22; +x_31 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__22; x_32 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_26, x_31, x_30); if (lean_obj_tag(x_32) == 0) { @@ -61692,7 +65812,7 @@ lean_object* x_33; lean_object* x_34; lean_object* x_35; x_33 = lean_ctor_get(x_32, 1); lean_inc(x_33); lean_dec(x_32); -x_34 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__23; +x_34 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__23; x_35 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_26, x_34, x_33); if (lean_obj_tag(x_35) == 0) { @@ -61700,9 +65820,9 @@ lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean x_36 = lean_ctor_get(x_35, 1); lean_inc(x_36); lean_dec(x_35); -x_37 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__24; -x_38 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__25; -x_39 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__26; +x_37 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__24; +x_38 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__25; +x_39 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__26; x_40 = l_Lean_Parser_registerAlias(x_37, x_38, x_39, x_5, x_36); if (lean_obj_tag(x_40) == 0) { @@ -61710,7 +65830,7 @@ lean_object* x_41; lean_object* x_42; lean_object* x_43; x_41 = lean_ctor_get(x_40, 1); lean_inc(x_41); lean_dec(x_40); -x_42 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__27; +x_42 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__27; x_43 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_37, x_42, x_41); if (lean_obj_tag(x_43) == 0) { @@ -61718,7 +65838,7 @@ lean_object* x_44; lean_object* x_45; lean_object* x_46; x_44 = lean_ctor_get(x_43, 1); lean_inc(x_44); lean_dec(x_43); -x_45 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__28; +x_45 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__28; x_46 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_37, x_45, x_44); if (lean_obj_tag(x_46) == 0) { @@ -61726,9 +65846,9 @@ lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean x_47 = lean_ctor_get(x_46, 1); lean_inc(x_47); lean_dec(x_46); -x_48 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__29; -x_49 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__30; -x_50 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__31; +x_48 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__29; +x_49 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__30; +x_50 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__31; x_51 = l_Lean_Parser_registerAlias(x_48, x_49, x_50, x_5, x_47); if (lean_obj_tag(x_51) == 0) { @@ -61736,7 +65856,7 @@ lean_object* x_52; lean_object* x_53; lean_object* x_54; x_52 = lean_ctor_get(x_51, 1); lean_inc(x_52); lean_dec(x_51); -x_53 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__32; +x_53 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__32; x_54 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_48, x_53, x_52); if (lean_obj_tag(x_54) == 0) { @@ -61744,7 +65864,7 @@ 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 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__33; +x_56 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__33; x_57 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_48, x_56, x_55); if (lean_obj_tag(x_57) == 0) { @@ -61752,9 +65872,9 @@ lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean x_58 = lean_ctor_get(x_57, 1); lean_inc(x_58); lean_dec(x_57); -x_59 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__34; -x_60 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__35; -x_61 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__36; +x_59 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__34; +x_60 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__35; +x_61 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__36; x_62 = l_Lean_Parser_registerAlias(x_59, x_60, x_61, x_5, x_58); if (lean_obj_tag(x_62) == 0) { @@ -61762,7 +65882,7 @@ lean_object* x_63; lean_object* x_64; lean_object* x_65; x_63 = lean_ctor_get(x_62, 1); lean_inc(x_63); lean_dec(x_62); -x_64 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__37; +x_64 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__37; x_65 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_59, x_64, x_63); if (lean_obj_tag(x_65) == 0) { @@ -61770,7 +65890,7 @@ lean_object* x_66; lean_object* x_67; lean_object* x_68; x_66 = lean_ctor_get(x_65, 1); lean_inc(x_66); lean_dec(x_65); -x_67 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__38; +x_67 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__38; x_68 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_59, x_67, x_66); if (lean_obj_tag(x_68) == 0) { @@ -61778,9 +65898,9 @@ lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean x_69 = lean_ctor_get(x_68, 1); lean_inc(x_69); lean_dec(x_68); -x_70 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__40; -x_71 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__41; -x_72 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__43; +x_70 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__40; +x_71 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__41; +x_72 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__43; x_73 = l_Lean_Parser_registerAlias(x_70, x_71, x_72, x_5, x_69); if (lean_obj_tag(x_73) == 0) { @@ -61788,7 +65908,7 @@ lean_object* x_74; lean_object* x_75; lean_object* x_76; x_74 = lean_ctor_get(x_73, 1); lean_inc(x_74); lean_dec(x_73); -x_75 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__44; +x_75 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__44; x_76 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_70, x_75, x_74); if (lean_obj_tag(x_76) == 0) { @@ -61796,467 +65916,562 @@ lean_object* x_77; lean_object* x_78; lean_object* x_79; x_77 = lean_ctor_get(x_76, 1); lean_inc(x_77); lean_dec(x_76); -x_78 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__45; +x_78 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__45; x_79 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_70, x_78, x_77); +if (lean_obj_tag(x_79) == 0) +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_80 = lean_ctor_get(x_79, 1); +lean_inc(x_80); +lean_dec(x_79); +x_81 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__47; +x_82 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__48; +x_83 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__50; +x_84 = l_Lean_Parser_registerAlias(x_81, x_82, x_83, x_5, x_80); +if (lean_obj_tag(x_84) == 0) +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_84, 1); +lean_inc(x_85); +lean_dec(x_84); +x_86 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__51; +x_87 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_81, x_86, x_85); +if (lean_obj_tag(x_87) == 0) +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); +x_89 = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__52; +x_90 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_81, x_89, x_88); +return x_90; +} +else +{ +uint8_t x_91; +x_91 = !lean_is_exclusive(x_87); +if (x_91 == 0) +{ +return x_87; +} +else +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_92 = lean_ctor_get(x_87, 0); +x_93 = lean_ctor_get(x_87, 1); +lean_inc(x_93); +lean_inc(x_92); +lean_dec(x_87); +x_94 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_93); +return x_94; +} +} +} +else +{ +uint8_t x_95; +x_95 = !lean_is_exclusive(x_84); +if (x_95 == 0) +{ +return x_84; +} +else +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_84, 0); +x_97 = lean_ctor_get(x_84, 1); +lean_inc(x_97); +lean_inc(x_96); +lean_dec(x_84); +x_98 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_97); +return x_98; +} +} +} +else +{ +uint8_t x_99; +x_99 = !lean_is_exclusive(x_79); +if (x_99 == 0) +{ return x_79; } else { -uint8_t x_80; -x_80 = !lean_is_exclusive(x_76); -if (x_80 == 0) +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_79, 0); +x_101 = lean_ctor_get(x_79, 1); +lean_inc(x_101); +lean_inc(x_100); +lean_dec(x_79); +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_100); +lean_ctor_set(x_102, 1, x_101); +return x_102; +} +} +} +else +{ +uint8_t x_103; +x_103 = !lean_is_exclusive(x_76); +if (x_103 == 0) { return x_76; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_76, 0); -x_82 = lean_ctor_get(x_76, 1); -lean_inc(x_82); -lean_inc(x_81); +lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_104 = lean_ctor_get(x_76, 0); +x_105 = lean_ctor_get(x_76, 1); +lean_inc(x_105); +lean_inc(x_104); lean_dec(x_76); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -return x_83; +x_106 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_106, 0, x_104); +lean_ctor_set(x_106, 1, x_105); +return x_106; } } } else { -uint8_t x_84; -x_84 = !lean_is_exclusive(x_73); -if (x_84 == 0) +uint8_t x_107; +x_107 = !lean_is_exclusive(x_73); +if (x_107 == 0) { return x_73; } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_85 = lean_ctor_get(x_73, 0); -x_86 = lean_ctor_get(x_73, 1); -lean_inc(x_86); -lean_inc(x_85); +lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_73, 0); +x_109 = lean_ctor_get(x_73, 1); +lean_inc(x_109); +lean_inc(x_108); lean_dec(x_73); -x_87 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_87, 0, x_85); -lean_ctor_set(x_87, 1, x_86); -return x_87; +x_110 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_110, 0, x_108); +lean_ctor_set(x_110, 1, x_109); +return x_110; } } } else { -uint8_t x_88; -x_88 = !lean_is_exclusive(x_68); -if (x_88 == 0) +uint8_t x_111; +x_111 = !lean_is_exclusive(x_68); +if (x_111 == 0) { return x_68; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_68, 0); -x_90 = lean_ctor_get(x_68, 1); -lean_inc(x_90); -lean_inc(x_89); +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_68, 0); +x_113 = lean_ctor_get(x_68, 1); +lean_inc(x_113); +lean_inc(x_112); lean_dec(x_68); -x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_90); -return x_91; +x_114 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +return x_114; } } } else { -uint8_t x_92; -x_92 = !lean_is_exclusive(x_65); -if (x_92 == 0) +uint8_t x_115; +x_115 = !lean_is_exclusive(x_65); +if (x_115 == 0) { return x_65; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_65, 0); -x_94 = lean_ctor_get(x_65, 1); -lean_inc(x_94); -lean_inc(x_93); +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_65, 0); +x_117 = lean_ctor_get(x_65, 1); +lean_inc(x_117); +lean_inc(x_116); lean_dec(x_65); -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -return x_95; +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; } } } else { -uint8_t x_96; -x_96 = !lean_is_exclusive(x_62); -if (x_96 == 0) +uint8_t x_119; +x_119 = !lean_is_exclusive(x_62); +if (x_119 == 0) { return x_62; } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_62, 0); -x_98 = lean_ctor_get(x_62, 1); -lean_inc(x_98); -lean_inc(x_97); +lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_120 = lean_ctor_get(x_62, 0); +x_121 = lean_ctor_get(x_62, 1); +lean_inc(x_121); +lean_inc(x_120); lean_dec(x_62); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -return x_99; +x_122 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_122, 0, x_120); +lean_ctor_set(x_122, 1, x_121); +return x_122; } } } else { -uint8_t x_100; -x_100 = !lean_is_exclusive(x_57); -if (x_100 == 0) +uint8_t x_123; +x_123 = !lean_is_exclusive(x_57); +if (x_123 == 0) { return x_57; } else { -lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_101 = lean_ctor_get(x_57, 0); -x_102 = lean_ctor_get(x_57, 1); -lean_inc(x_102); -lean_inc(x_101); +lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_124 = lean_ctor_get(x_57, 0); +x_125 = lean_ctor_get(x_57, 1); +lean_inc(x_125); +lean_inc(x_124); lean_dec(x_57); -x_103 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -return x_103; +x_126 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +return x_126; } } } else { -uint8_t x_104; -x_104 = !lean_is_exclusive(x_54); -if (x_104 == 0) +uint8_t x_127; +x_127 = !lean_is_exclusive(x_54); +if (x_127 == 0) { return x_54; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_54, 0); -x_106 = lean_ctor_get(x_54, 1); -lean_inc(x_106); -lean_inc(x_105); +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_54, 0); +x_129 = lean_ctor_get(x_54, 1); +lean_inc(x_129); +lean_inc(x_128); lean_dec(x_54); -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; +x_130 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +return x_130; } } } else { -uint8_t x_108; -x_108 = !lean_is_exclusive(x_51); -if (x_108 == 0) +uint8_t x_131; +x_131 = !lean_is_exclusive(x_51); +if (x_131 == 0) { return x_51; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_51, 0); -x_110 = lean_ctor_get(x_51, 1); -lean_inc(x_110); -lean_inc(x_109); +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_51, 0); +x_133 = lean_ctor_get(x_51, 1); +lean_inc(x_133); +lean_inc(x_132); lean_dec(x_51); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -return x_111; +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; } } } else { -uint8_t x_112; -x_112 = !lean_is_exclusive(x_46); -if (x_112 == 0) +uint8_t x_135; +x_135 = !lean_is_exclusive(x_46); +if (x_135 == 0) { return x_46; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_46, 0); -x_114 = lean_ctor_get(x_46, 1); -lean_inc(x_114); -lean_inc(x_113); +lean_object* x_136; lean_object* x_137; lean_object* x_138; +x_136 = lean_ctor_get(x_46, 0); +x_137 = lean_ctor_get(x_46, 1); +lean_inc(x_137); +lean_inc(x_136); lean_dec(x_46); -x_115 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -return x_115; +x_138 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_138, 0, x_136); +lean_ctor_set(x_138, 1, x_137); +return x_138; } } } else { -uint8_t x_116; -x_116 = !lean_is_exclusive(x_43); -if (x_116 == 0) +uint8_t x_139; +x_139 = !lean_is_exclusive(x_43); +if (x_139 == 0) { return x_43; } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_117 = lean_ctor_get(x_43, 0); -x_118 = lean_ctor_get(x_43, 1); -lean_inc(x_118); -lean_inc(x_117); +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_43, 0); +x_141 = lean_ctor_get(x_43, 1); +lean_inc(x_141); +lean_inc(x_140); lean_dec(x_43); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_117); -lean_ctor_set(x_119, 1, x_118); -return x_119; +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } } else { -uint8_t x_120; -x_120 = !lean_is_exclusive(x_40); -if (x_120 == 0) +uint8_t x_143; +x_143 = !lean_is_exclusive(x_40); +if (x_143 == 0) { return x_40; } else { -lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_121 = lean_ctor_get(x_40, 0); -x_122 = lean_ctor_get(x_40, 1); -lean_inc(x_122); -lean_inc(x_121); +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_40, 0); +x_145 = lean_ctor_get(x_40, 1); +lean_inc(x_145); +lean_inc(x_144); lean_dec(x_40); -x_123 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_123, 0, x_121); -lean_ctor_set(x_123, 1, x_122); -return x_123; +x_146 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +return x_146; } } } else { -uint8_t x_124; -x_124 = !lean_is_exclusive(x_35); -if (x_124 == 0) +uint8_t x_147; +x_147 = !lean_is_exclusive(x_35); +if (x_147 == 0) { return x_35; } else { -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_35, 0); -x_126 = lean_ctor_get(x_35, 1); -lean_inc(x_126); -lean_inc(x_125); +lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_148 = lean_ctor_get(x_35, 0); +x_149 = lean_ctor_get(x_35, 1); +lean_inc(x_149); +lean_inc(x_148); lean_dec(x_35); -x_127 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_127, 0, x_125); -lean_ctor_set(x_127, 1, x_126); -return x_127; +x_150 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_150, 0, x_148); +lean_ctor_set(x_150, 1, x_149); +return x_150; } } } else { -uint8_t x_128; -x_128 = !lean_is_exclusive(x_32); -if (x_128 == 0) +uint8_t x_151; +x_151 = !lean_is_exclusive(x_32); +if (x_151 == 0) { return x_32; } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; -x_129 = lean_ctor_get(x_32, 0); -x_130 = lean_ctor_get(x_32, 1); -lean_inc(x_130); -lean_inc(x_129); +lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_152 = lean_ctor_get(x_32, 0); +x_153 = lean_ctor_get(x_32, 1); +lean_inc(x_153); +lean_inc(x_152); lean_dec(x_32); -x_131 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_131, 0, x_129); -lean_ctor_set(x_131, 1, x_130); -return x_131; +x_154 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_154, 0, x_152); +lean_ctor_set(x_154, 1, x_153); +return x_154; } } } else { -uint8_t x_132; -x_132 = !lean_is_exclusive(x_29); -if (x_132 == 0) +uint8_t x_155; +x_155 = !lean_is_exclusive(x_29); +if (x_155 == 0) { return x_29; } else { -lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_133 = lean_ctor_get(x_29, 0); -x_134 = lean_ctor_get(x_29, 1); -lean_inc(x_134); -lean_inc(x_133); +lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_156 = lean_ctor_get(x_29, 0); +x_157 = lean_ctor_get(x_29, 1); +lean_inc(x_157); +lean_inc(x_156); lean_dec(x_29); -x_135 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_135, 0, x_133); -lean_ctor_set(x_135, 1, x_134); -return x_135; +x_158 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_158, 0, x_156); +lean_ctor_set(x_158, 1, x_157); +return x_158; } } } else { -uint8_t x_136; -x_136 = !lean_is_exclusive(x_24); -if (x_136 == 0) +uint8_t x_159; +x_159 = !lean_is_exclusive(x_24); +if (x_159 == 0) { return x_24; } else { -lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_137 = lean_ctor_get(x_24, 0); -x_138 = lean_ctor_get(x_24, 1); -lean_inc(x_138); -lean_inc(x_137); +lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_160 = lean_ctor_get(x_24, 0); +x_161 = lean_ctor_get(x_24, 1); +lean_inc(x_161); +lean_inc(x_160); lean_dec(x_24); -x_139 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); -return x_139; +x_162 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_162, 0, x_160); +lean_ctor_set(x_162, 1, x_161); +return x_162; } } } else { -uint8_t x_140; -x_140 = !lean_is_exclusive(x_21); -if (x_140 == 0) +uint8_t x_163; +x_163 = !lean_is_exclusive(x_21); +if (x_163 == 0) { return x_21; } else { -lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_141 = lean_ctor_get(x_21, 0); -x_142 = lean_ctor_get(x_21, 1); -lean_inc(x_142); -lean_inc(x_141); +lean_object* x_164; lean_object* x_165; lean_object* x_166; +x_164 = lean_ctor_get(x_21, 0); +x_165 = lean_ctor_get(x_21, 1); +lean_inc(x_165); +lean_inc(x_164); lean_dec(x_21); -x_143 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_143, 0, x_141); -lean_ctor_set(x_143, 1, x_142); -return x_143; +x_166 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_166, 0, x_164); +lean_ctor_set(x_166, 1, x_165); +return x_166; } } } else { -uint8_t x_144; -x_144 = !lean_is_exclusive(x_18); -if (x_144 == 0) +uint8_t x_167; +x_167 = !lean_is_exclusive(x_18); +if (x_167 == 0) { return x_18; } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_145 = lean_ctor_get(x_18, 0); -x_146 = lean_ctor_get(x_18, 1); -lean_inc(x_146); -lean_inc(x_145); +lean_object* x_168; lean_object* x_169; lean_object* x_170; +x_168 = lean_ctor_get(x_18, 0); +x_169 = lean_ctor_get(x_18, 1); +lean_inc(x_169); +lean_inc(x_168); lean_dec(x_18); -x_147 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_147, 0, x_145); -lean_ctor_set(x_147, 1, x_146); -return x_147; +x_170 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_170, 0, x_168); +lean_ctor_set(x_170, 1, x_169); +return x_170; } } } else { -uint8_t x_148; -x_148 = !lean_is_exclusive(x_14); -if (x_148 == 0) +uint8_t x_171; +x_171 = !lean_is_exclusive(x_14); +if (x_171 == 0) { return x_14; } else { -lean_object* x_149; lean_object* x_150; lean_object* x_151; -x_149 = lean_ctor_get(x_14, 0); -x_150 = lean_ctor_get(x_14, 1); -lean_inc(x_150); -lean_inc(x_149); +lean_object* x_172; lean_object* x_173; lean_object* x_174; +x_172 = lean_ctor_get(x_14, 0); +x_173 = lean_ctor_get(x_14, 1); +lean_inc(x_173); +lean_inc(x_172); lean_dec(x_14); -x_151 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_151, 0, x_149); -lean_ctor_set(x_151, 1, x_150); -return x_151; +x_174 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_174, 0, x_172); +lean_ctor_set(x_174, 1, x_173); +return x_174; } } } else { -uint8_t x_152; -x_152 = !lean_is_exclusive(x_10); -if (x_152 == 0) +uint8_t x_175; +x_175 = !lean_is_exclusive(x_10); +if (x_175 == 0) { return x_10; } else { -lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_153 = lean_ctor_get(x_10, 0); -x_154 = lean_ctor_get(x_10, 1); -lean_inc(x_154); -lean_inc(x_153); +lean_object* x_176; lean_object* x_177; lean_object* x_178; +x_176 = lean_ctor_get(x_10, 0); +x_177 = lean_ctor_get(x_10, 1); +lean_inc(x_177); +lean_inc(x_176); lean_dec(x_10); -x_155 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_155, 0, x_153); -lean_ctor_set(x_155, 1, x_154); -return x_155; +x_178 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_178, 0, x_176); +lean_ctor_set(x_178, 1, x_177); +return x_178; } } } else { -uint8_t x_156; -x_156 = !lean_is_exclusive(x_6); -if (x_156 == 0) +uint8_t x_179; +x_179 = !lean_is_exclusive(x_6); +if (x_179 == 0) { return x_6; } else { -lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_157 = lean_ctor_get(x_6, 0); -x_158 = lean_ctor_get(x_6, 1); -lean_inc(x_158); -lean_inc(x_157); +lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_180 = lean_ctor_get(x_6, 0); +x_181 = lean_ctor_get(x_6, 1); +lean_inc(x_181); +lean_inc(x_180); lean_dec(x_6); -x_159 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_159, 0, x_157); -lean_ctor_set(x_159, 1, x_158); -return x_159; +x_182 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_182, 0, x_180); +lean_ctor_set(x_182, 1, x_181); +return x_182; } } } @@ -62682,7 +66897,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_open_declRange___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(160u); +x_1 = lean_unsigned_to_nat(161u); x_2 = lean_unsigned_to_nat(21u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -62694,7 +66909,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_open_declRange___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(160u); +x_1 = lean_unsigned_to_nat(161u); x_2 = lean_unsigned_to_nat(125u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -62722,7 +66937,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_open_declRange___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(160u); +x_1 = lean_unsigned_to_nat(161u); x_2 = lean_unsigned_to_nat(25u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -62734,7 +66949,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_open_declRange___close _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(160u); +x_1 = lean_unsigned_to_nat(161u); x_2 = lean_unsigned_to_nat(31u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -62868,6 +67083,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_open_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_open___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_open_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_open_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_open_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Term_open___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_open_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_open_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_open_parenthesizer___closed__1() { _start: { @@ -62956,6 +67201,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_open___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_open_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_open_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_open___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_set__option___elambda__1___closed__1() { _start: { @@ -63429,7 +67704,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_set__option_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(161u); +x_1 = lean_unsigned_to_nat(162u); x_2 = lean_unsigned_to_nat(21u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -63441,7 +67716,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_set__option_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(161u); +x_1 = lean_unsigned_to_nat(162u); x_2 = lean_unsigned_to_nat(145u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -63469,7 +67744,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_set__option_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(161u); +x_1 = lean_unsigned_to_nat(162u); x_2 = lean_unsigned_to_nat(25u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -63481,7 +67756,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Term_set__option_declRange_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(161u); +x_1 = lean_unsigned_to_nat(162u); x_2 = lean_unsigned_to_nat(37u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -63625,6 +67900,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_set__option___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_set__option_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_set__option_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Term_set__option___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_set__option_parenthesizer___closed__1() { _start: { @@ -63723,6 +68028,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_set__option___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_set__option_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_set__option___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_open___elambda__1___closed__1() { _start: { @@ -64158,7 +68493,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_open_declRange___clo _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(165u); +x_1 = lean_unsigned_to_nat(166u); x_2 = lean_unsigned_to_nat(23u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -64170,7 +68505,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_open_declRange___clo _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(165u); +x_1 = lean_unsigned_to_nat(166u); x_2 = lean_unsigned_to_nat(126u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -64198,7 +68533,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_open_declRange___clo _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(165u); +x_1 = lean_unsigned_to_nat(166u); x_2 = lean_unsigned_to_nat(27u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -64210,7 +68545,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_open_declRange___clo _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(165u); +x_1 = lean_unsigned_to_nat(166u); x_2 = lean_unsigned_to_nat(33u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -64344,6 +68679,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_open___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_open_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_open_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_open___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_open_parenthesizer___closed__1() { _start: { @@ -64432,6 +68797,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_open___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_open_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_open___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_set__option___elambda__1___closed__1() { _start: { @@ -64873,7 +69268,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_set__option_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(166u); +x_1 = lean_unsigned_to_nat(167u); x_2 = lean_unsigned_to_nat(23u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -64885,7 +69280,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_set__option_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(166u); +x_1 = lean_unsigned_to_nat(167u); x_2 = lean_unsigned_to_nat(146u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -64913,7 +69308,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_set__option_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(166u); +x_1 = lean_unsigned_to_nat(167u); x_2 = lean_unsigned_to_nat(27u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -64925,7 +69320,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_set__option_declRang _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(166u); +x_1 = lean_unsigned_to_nat(167u); x_2 = lean_unsigned_to_nat(39u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -65061,6 +69456,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_set__option___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_set__option_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_set__option___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_set__option_parenthesizer___closed__1() { _start: { @@ -65151,6 +69576,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_set__option___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_set__option_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_set__option___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Term(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Do(uint8_t builtin, lean_object*); @@ -65283,6 +69738,17 @@ l_Lean_Parser_Term_quot_formatter___closed__7 = _init_l_Lean_Parser_Term_quot_fo lean_mark_persistent(l_Lean_Parser_Term_quot_formatter___closed__7); l_Lean_Parser_Term_quot_formatter___closed__8 = _init_l_Lean_Parser_Term_quot_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_quot_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quot_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Term_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_quot_parenthesizer___closed__1); l_Lean_Parser_Term_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_quot_parenthesizer___closed__2(); @@ -65299,6 +69765,17 @@ l_Lean_Parser_Term_quot_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_quo lean_mark_persistent(l_Lean_Parser_Term_quot_parenthesizer___closed__7); l_Lean_Parser_Term_quot_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_quot_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_quot_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quot_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_Term_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__1); l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_precheckedQuot___elambda__1___closed__2(); @@ -65369,8 +69846,13 @@ l_Lean_Parser_Term_precheckedQuot_formatter___closed__3 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_precheckedQuot_formatter___closed__3); l_Lean_Parser_Term_precheckedQuot_formatter___closed__4 = _init_l_Lean_Parser_Term_precheckedQuot_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_precheckedQuot_formatter___closed__4); -l_Lean_Parser_Term_precheckedQuot_formatter___closed__5 = _init_l_Lean_Parser_Term_precheckedQuot_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_precheckedQuot_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_precheckedQuot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1); l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2(); @@ -65379,8 +69861,13 @@ l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__3 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__3); l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__4); -l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_precheckedQuot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Command_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_quot___elambda__1___closed__1); l_Lean_Parser_Command_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Command_quot___elambda__1___closed__2(); @@ -65478,6 +69965,13 @@ l_Lean_Parser_Command_quot_formatter___closed__6 = _init_l_Lean_Parser_Command_q lean_mark_persistent(l_Lean_Parser_Command_quot_formatter___closed__6); l_Lean_Parser_Command_quot_formatter___closed__7 = _init_l_Lean_Parser_Command_quot_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_quot_formatter___closed__7); +l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_quot_parenthesizer___closed__1); l_Lean_Parser_Command_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_quot_parenthesizer___closed__2(); @@ -65492,6 +69986,13 @@ l_Lean_Parser_Command_quot_parenthesizer___closed__6 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_quot_parenthesizer___closed__6); l_Lean_Parser_Command_quot_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_quot_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_quot_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__1 = _init_l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__1); l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__2 = _init_l_Lean_Parser_Command_terminationHintMany___elambda__1___closed__2(); @@ -65860,6 +70361,13 @@ l_Lean_Parser_Command_moduleDoc_formatter___closed__7 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_moduleDoc_formatter___closed__7); l_Lean_Parser_Command_moduleDoc_formatter___closed__8 = _init_l_Lean_Parser_Command_moduleDoc_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_moduleDoc_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_moduleDoc_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1); l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__2(); @@ -65876,6 +70384,13 @@ l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__7 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__7); l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_moduleDoc_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_moduleDoc_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_namedPrio___elambda__1___closed__1 = _init_l_Lean_Parser_Command_namedPrio___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_namedPrio___elambda__1___closed__1); l_Lean_Parser_Command_namedPrio___elambda__1___closed__2 = _init_l_Lean_Parser_Command_namedPrio___elambda__1___closed__2(); @@ -68026,40 +72541,78 @@ l_Lean_Parser_Command_private_formatter___closed__2 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_private_formatter___closed__2); l_Lean_Parser_Command_private_formatter___closed__3 = _init_l_Lean_Parser_Command_private_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_private_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_private_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_private_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_private_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_private_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_private_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_private_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_private_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_protected_formatter___closed__1 = _init_l_Lean_Parser_Command_protected_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_protected_formatter___closed__1); l_Lean_Parser_Command_protected_formatter___closed__2 = _init_l_Lean_Parser_Command_protected_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_protected_formatter___closed__2); l_Lean_Parser_Command_protected_formatter___closed__3 = _init_l_Lean_Parser_Command_protected_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_protected_formatter___closed__3); -l_Lean_Parser_Command_visibility_formatter___closed__1 = _init_l_Lean_Parser_Command_visibility_formatter___closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_visibility_formatter___closed__1); -l_Lean_Parser_Command_visibility_formatter___closed__2 = _init_l_Lean_Parser_Command_visibility_formatter___closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_visibility_formatter___closed__2); +l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_protected_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_protected_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_noncomputable_formatter___closed__1 = _init_l_Lean_Parser_Command_noncomputable_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_noncomputable_formatter___closed__1); l_Lean_Parser_Command_noncomputable_formatter___closed__2 = _init_l_Lean_Parser_Command_noncomputable_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_noncomputable_formatter___closed__2); l_Lean_Parser_Command_noncomputable_formatter___closed__3 = _init_l_Lean_Parser_Command_noncomputable_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_noncomputable_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_noncomputable_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_noncomputable_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_unsafe_formatter___closed__1 = _init_l_Lean_Parser_Command_unsafe_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_unsafe_formatter___closed__1); l_Lean_Parser_Command_unsafe_formatter___closed__2 = _init_l_Lean_Parser_Command_unsafe_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_unsafe_formatter___closed__2); l_Lean_Parser_Command_unsafe_formatter___closed__3 = _init_l_Lean_Parser_Command_unsafe_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_unsafe_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_unsafe_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_unsafe_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_partial_formatter___closed__1 = _init_l_Lean_Parser_Command_partial_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_partial_formatter___closed__1); l_Lean_Parser_Command_partial_formatter___closed__2 = _init_l_Lean_Parser_Command_partial_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_partial_formatter___closed__2); l_Lean_Parser_Command_partial_formatter___closed__3 = _init_l_Lean_Parser_Command_partial_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_partial_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_partial_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_partial_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_nonrec_formatter___closed__1 = _init_l_Lean_Parser_Command_nonrec_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_nonrec_formatter___closed__1); l_Lean_Parser_Command_nonrec_formatter___closed__2 = _init_l_Lean_Parser_Command_nonrec_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_nonrec_formatter___closed__2); l_Lean_Parser_Command_nonrec_formatter___closed__3 = _init_l_Lean_Parser_Command_nonrec_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_nonrec_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_nonrec_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_nonrec_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declModifiers_formatter___closed__1 = _init_l_Lean_Parser_Command_declModifiers_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declModifiers_formatter___closed__1); l_Lean_Parser_Command_declModifiers_formatter___closed__2 = _init_l_Lean_Parser_Command_declModifiers_formatter___closed__2(); @@ -68110,14 +72663,6 @@ l_Lean_Parser_Command_declModifiers_formatter___closed__24 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_declModifiers_formatter___closed__24); l_Lean_Parser_Command_declModifiers_formatter___closed__25 = _init_l_Lean_Parser_Command_declModifiers_formatter___closed__25(); lean_mark_persistent(l_Lean_Parser_Command_declModifiers_formatter___closed__25); -l_Lean_Parser_Command_declModifiers_formatter___closed__26 = _init_l_Lean_Parser_Command_declModifiers_formatter___closed__26(); -lean_mark_persistent(l_Lean_Parser_Command_declModifiers_formatter___closed__26); -l_Lean_Parser_Command_declModifiers_formatter___closed__27 = _init_l_Lean_Parser_Command_declModifiers_formatter___closed__27(); -lean_mark_persistent(l_Lean_Parser_Command_declModifiers_formatter___closed__27); -l_Lean_Parser_Command_declModifiers_formatter___closed__28 = _init_l_Lean_Parser_Command_declModifiers_formatter___closed__28(); -lean_mark_persistent(l_Lean_Parser_Command_declModifiers_formatter___closed__28); -l_Lean_Parser_Command_declModifiers_formatter___closed__29 = _init_l_Lean_Parser_Command_declModifiers_formatter___closed__29(); -lean_mark_persistent(l_Lean_Parser_Command_declModifiers_formatter___closed__29); l_Lean_Parser_Command_declId_formatter___closed__1 = _init_l_Lean_Parser_Command_declId_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declId_formatter___closed__1); l_Lean_Parser_Command_declId_formatter___closed__2 = _init_l_Lean_Parser_Command_declId_formatter___closed__2(); @@ -68140,6 +72685,13 @@ l_Lean_Parser_Command_declId_formatter___closed__10 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_declId_formatter___closed__10); l_Lean_Parser_Command_declId_formatter___closed__11 = _init_l_Lean_Parser_Command_declId_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_declId_formatter___closed__11); +l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declId_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declId_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_optDeclSig_formatter___closed__1 = _init_l_Lean_Parser_Command_optDeclSig_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_optDeclSig_formatter___closed__1); l_Lean_Parser_Command_optDeclSig_formatter___closed__2 = _init_l_Lean_Parser_Command_optDeclSig_formatter___closed__2(); @@ -68160,6 +72712,13 @@ l_Lean_Parser_Command_optDeclSig_formatter___closed__9 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_optDeclSig_formatter___closed__9); l_Lean_Parser_Command_optDeclSig_formatter___closed__10 = _init_l_Lean_Parser_Command_optDeclSig_formatter___closed__10(); lean_mark_persistent(l_Lean_Parser_Command_optDeclSig_formatter___closed__10); +l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_optDeclSig_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declValSimple_formatter___closed__1 = _init_l_Lean_Parser_Command_declValSimple_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declValSimple_formatter___closed__1); l_Lean_Parser_Command_declValSimple_formatter___closed__2 = _init_l_Lean_Parser_Command_declValSimple_formatter___closed__2(); @@ -68178,18 +72737,39 @@ l_Lean_Parser_Command_declValSimple_formatter___closed__8 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_declValSimple_formatter___closed__8); l_Lean_Parser_Command_declValSimple_formatter___closed__9 = _init_l_Lean_Parser_Command_declValSimple_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_declValSimple_formatter___closed__9); +l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declValSimple_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declValSimple_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declValEqns_formatter___closed__1 = _init_l_Lean_Parser_Command_declValEqns_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declValEqns_formatter___closed__1); l_Lean_Parser_Command_declValEqns_formatter___closed__2 = _init_l_Lean_Parser_Command_declValEqns_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_declValEqns_formatter___closed__2); l_Lean_Parser_Command_declValEqns_formatter___closed__3 = _init_l_Lean_Parser_Command_declValEqns_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_declValEqns_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declValEqns_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declValEqns_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_whereStructField_formatter___closed__1 = _init_l_Lean_Parser_Command_whereStructField_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_whereStructField_formatter___closed__1); l_Lean_Parser_Command_whereStructField_formatter___closed__2 = _init_l_Lean_Parser_Command_whereStructField_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_whereStructField_formatter___closed__2); l_Lean_Parser_Command_whereStructField_formatter___closed__3 = _init_l_Lean_Parser_Command_whereStructField_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_whereStructField_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_whereStructField_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_whereStructField_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_whereStructInst_formatter___closed__1 = _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_whereStructInst_formatter___closed__1); l_Lean_Parser_Command_whereStructInst_formatter___closed__2 = _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__2(); @@ -68206,20 +72786,19 @@ l_Lean_Parser_Command_whereStructInst_formatter___closed__7 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Command_whereStructInst_formatter___closed__7); l_Lean_Parser_Command_whereStructInst_formatter___closed__8 = _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_whereStructInst_formatter___closed__8); -l_Lean_Parser_Command_whereStructInst_formatter___closed__9 = _init_l_Lean_Parser_Command_whereStructInst_formatter___closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_whereStructInst_formatter___closed__9); +l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_whereStructInst_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declVal_formatter___closed__1 = _init_l_Lean_Parser_Command_declVal_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declVal_formatter___closed__1); l_Lean_Parser_Command_declVal_formatter___closed__2 = _init_l_Lean_Parser_Command_declVal_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_declVal_formatter___closed__2); l_Lean_Parser_Command_declVal_formatter___closed__3 = _init_l_Lean_Parser_Command_declVal_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_declVal_formatter___closed__3); -l_Lean_Parser_Command_declVal_formatter___closed__4 = _init_l_Lean_Parser_Command_declVal_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_declVal_formatter___closed__4); -l_Lean_Parser_Command_declVal_formatter___closed__5 = _init_l_Lean_Parser_Command_declVal_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_declVal_formatter___closed__5); -l_Lean_Parser_Command_declVal_formatter___closed__6 = _init_l_Lean_Parser_Command_declVal_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_declVal_formatter___closed__6); l_Lean_Parser_Command_abbrev_formatter___closed__1 = _init_l_Lean_Parser_Command_abbrev_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_abbrev_formatter___closed__1); l_Lean_Parser_Command_abbrev_formatter___closed__2 = _init_l_Lean_Parser_Command_abbrev_formatter___closed__2(); @@ -68236,10 +72815,13 @@ l_Lean_Parser_Command_abbrev_formatter___closed__7 = _init_l_Lean_Parser_Command lean_mark_persistent(l_Lean_Parser_Command_abbrev_formatter___closed__7); l_Lean_Parser_Command_abbrev_formatter___closed__8 = _init_l_Lean_Parser_Command_abbrev_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_abbrev_formatter___closed__8); -l_Lean_Parser_Command_abbrev_formatter___closed__9 = _init_l_Lean_Parser_Command_abbrev_formatter___closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_abbrev_formatter___closed__9); -l_Lean_Parser_Command_abbrev_formatter___closed__10 = _init_l_Lean_Parser_Command_abbrev_formatter___closed__10(); -lean_mark_persistent(l_Lean_Parser_Command_abbrev_formatter___closed__10); +l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_abbrev_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_abbrev_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_optDefDeriving_formatter___closed__1 = _init_l_Lean_Parser_Command_optDefDeriving_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_optDefDeriving_formatter___closed__1); l_Lean_Parser_Command_optDefDeriving_formatter___closed__2 = _init_l_Lean_Parser_Command_optDefDeriving_formatter___closed__2(); @@ -68276,6 +72858,13 @@ l_Lean_Parser_Command_terminationByElement_formatter___closed__12 = _init_l_Lean lean_mark_persistent(l_Lean_Parser_Command_terminationByElement_formatter___closed__12); l_Lean_Parser_Command_terminationByElement_formatter___closed__13 = _init_l_Lean_Parser_Command_terminationByElement_formatter___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_terminationByElement_formatter___closed__13); +l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_terminationByElement_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_terminationBy_formatter___closed__1 = _init_l_Lean_Parser_Command_terminationBy_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_terminationBy_formatter___closed__1); l_Lean_Parser_Command_terminationBy_formatter___closed__2 = _init_l_Lean_Parser_Command_terminationBy_formatter___closed__2(); @@ -68288,8 +72877,13 @@ l_Lean_Parser_Command_terminationBy_formatter___closed__5 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_terminationBy_formatter___closed__5); l_Lean_Parser_Command_terminationBy_formatter___closed__6 = _init_l_Lean_Parser_Command_terminationBy_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_terminationBy_formatter___closed__6); -l_Lean_Parser_Command_terminationBy_formatter___closed__7 = _init_l_Lean_Parser_Command_terminationBy_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_terminationBy_formatter___closed__7); +l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationBy_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_terminationBy_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_terminationHintMany_formatter___closed__1 = _init_l_Lean_Parser_Command_terminationHintMany_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_terminationHintMany_formatter___closed__1); l_Lean_Parser_Command_terminationHintMany_formatter___closed__2 = _init_l_Lean_Parser_Command_terminationHintMany_formatter___closed__2(); @@ -68310,6 +72904,13 @@ l_Lean_Parser_Command_terminationByCore_formatter___closed__4 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Command_terminationByCore_formatter___closed__4); l_Lean_Parser_Command_terminationByCore_formatter___closed__5 = _init_l_Lean_Parser_Command_terminationByCore_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_terminationByCore_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_terminationByCore_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_decreasingBy_formatter___closed__1 = _init_l_Lean_Parser_Command_decreasingBy_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_decreasingBy_formatter___closed__1); l_Lean_Parser_Command_decreasingBy_formatter___closed__2 = _init_l_Lean_Parser_Command_decreasingBy_formatter___closed__2(); @@ -68322,18 +72923,19 @@ l_Lean_Parser_Command_decreasingBy_formatter___closed__5 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_decreasingBy_formatter___closed__5); l_Lean_Parser_Command_decreasingBy_formatter___closed__6 = _init_l_Lean_Parser_Command_decreasingBy_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_decreasingBy_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_decreasingBy_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_terminationSuffix_formatter___closed__1 = _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_formatter___closed__1); l_Lean_Parser_Command_terminationSuffix_formatter___closed__2 = _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_formatter___closed__2); l_Lean_Parser_Command_terminationSuffix_formatter___closed__3 = _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_formatter___closed__3); -l_Lean_Parser_Command_terminationSuffix_formatter___closed__4 = _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_formatter___closed__4); -l_Lean_Parser_Command_terminationSuffix_formatter___closed__5 = _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_formatter___closed__5); -l_Lean_Parser_Command_terminationSuffix_formatter___closed__6 = _init_l_Lean_Parser_Command_terminationSuffix_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_formatter___closed__6); l_Lean_Parser_Command_def_formatter___closed__1 = _init_l_Lean_Parser_Command_def_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_def_formatter___closed__1); l_Lean_Parser_Command_def_formatter___closed__2 = _init_l_Lean_Parser_Command_def_formatter___closed__2(); @@ -68354,6 +72956,13 @@ l_Lean_Parser_Command_def_formatter___closed__9 = _init_l_Lean_Parser_Command_de lean_mark_persistent(l_Lean_Parser_Command_def_formatter___closed__9); l_Lean_Parser_Command_def_formatter___closed__10 = _init_l_Lean_Parser_Command_def_formatter___closed__10(); lean_mark_persistent(l_Lean_Parser_Command_def_formatter___closed__10); +l___regBuiltin_Lean_Parser_Command_def_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_def_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_def_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_def_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_def_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_def_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_def_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declSig_formatter___closed__1 = _init_l_Lean_Parser_Command_declSig_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declSig_formatter___closed__1); l_Lean_Parser_Command_declSig_formatter___closed__2 = _init_l_Lean_Parser_Command_declSig_formatter___closed__2(); @@ -68362,6 +72971,13 @@ l_Lean_Parser_Command_declSig_formatter___closed__3 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_declSig_formatter___closed__3); l_Lean_Parser_Command_declSig_formatter___closed__4 = _init_l_Lean_Parser_Command_declSig_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_declSig_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declSig_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declSig_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_theorem_formatter___closed__1 = _init_l_Lean_Parser_Command_theorem_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_theorem_formatter___closed__1); l_Lean_Parser_Command_theorem_formatter___closed__2 = _init_l_Lean_Parser_Command_theorem_formatter___closed__2(); @@ -68378,8 +72994,13 @@ l_Lean_Parser_Command_theorem_formatter___closed__7 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_theorem_formatter___closed__7); l_Lean_Parser_Command_theorem_formatter___closed__8 = _init_l_Lean_Parser_Command_theorem_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_theorem_formatter___closed__8); -l_Lean_Parser_Command_theorem_formatter___closed__9 = _init_l_Lean_Parser_Command_theorem_formatter___closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_theorem_formatter___closed__9); +l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_theorem_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_theorem_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_opaque_formatter___closed__1 = _init_l_Lean_Parser_Command_opaque_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_opaque_formatter___closed__1); l_Lean_Parser_Command_opaque_formatter___closed__2 = _init_l_Lean_Parser_Command_opaque_formatter___closed__2(); @@ -68394,6 +73015,13 @@ l_Lean_Parser_Command_opaque_formatter___closed__6 = _init_l_Lean_Parser_Command lean_mark_persistent(l_Lean_Parser_Command_opaque_formatter___closed__6); l_Lean_Parser_Command_opaque_formatter___closed__7 = _init_l_Lean_Parser_Command_opaque_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_opaque_formatter___closed__7); +l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_opaque_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_opaque_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_namedPrio_formatter___closed__1 = _init_l_Lean_Parser_Command_namedPrio_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_namedPrio_formatter___closed__1); l_Lean_Parser_Command_namedPrio_formatter___closed__2 = _init_l_Lean_Parser_Command_namedPrio_formatter___closed__2(); @@ -68416,10 +73044,15 @@ l_Lean_Parser_Command_namedPrio_formatter___closed__10 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_namedPrio_formatter___closed__10); l_Lean_Parser_Command_namedPrio_formatter___closed__11 = _init_l_Lean_Parser_Command_namedPrio_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_namedPrio_formatter___closed__11); +l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namedPrio_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_namedPrio_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_optNamedPrio_formatter___closed__1 = _init_l_Lean_Parser_Command_optNamedPrio_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_optNamedPrio_formatter___closed__1); -l_Lean_Parser_Command_optNamedPrio_formatter___closed__2 = _init_l_Lean_Parser_Command_optNamedPrio_formatter___closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_optNamedPrio_formatter___closed__2); l_Lean_Parser_Command_instance_formatter___closed__1 = _init_l_Lean_Parser_Command_instance_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_instance_formatter___closed__1); l_Lean_Parser_Command_instance_formatter___closed__2 = _init_l_Lean_Parser_Command_instance_formatter___closed__2(); @@ -68442,6 +73075,13 @@ l_Lean_Parser_Command_instance_formatter___closed__10 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_instance_formatter___closed__10); l_Lean_Parser_Command_instance_formatter___closed__11 = _init_l_Lean_Parser_Command_instance_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_instance_formatter___closed__11); +l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_instance_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_instance_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_axiom_formatter___closed__1 = _init_l_Lean_Parser_Command_axiom_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_axiom_formatter___closed__1); l_Lean_Parser_Command_axiom_formatter___closed__2 = _init_l_Lean_Parser_Command_axiom_formatter___closed__2(); @@ -68452,6 +73092,13 @@ l_Lean_Parser_Command_axiom_formatter___closed__4 = _init_l_Lean_Parser_Command_ lean_mark_persistent(l_Lean_Parser_Command_axiom_formatter___closed__4); l_Lean_Parser_Command_axiom_formatter___closed__5 = _init_l_Lean_Parser_Command_axiom_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_axiom_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_axiom_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_axiom_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_example_formatter___closed__1 = _init_l_Lean_Parser_Command_example_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_example_formatter___closed__1); l_Lean_Parser_Command_example_formatter___closed__2 = _init_l_Lean_Parser_Command_example_formatter___closed__2(); @@ -68462,6 +73109,13 @@ l_Lean_Parser_Command_example_formatter___closed__4 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_example_formatter___closed__4); l_Lean_Parser_Command_example_formatter___closed__5 = _init_l_Lean_Parser_Command_example_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_example_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_example_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_example_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_example_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_example_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_example_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_example_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_example_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_ctor_formatter___closed__1 = _init_l_Lean_Parser_Command_ctor_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_ctor_formatter___closed__1); l_Lean_Parser_Command_ctor_formatter___closed__2 = _init_l_Lean_Parser_Command_ctor_formatter___closed__2(); @@ -68478,6 +73132,13 @@ l_Lean_Parser_Command_ctor_formatter___closed__7 = _init_l_Lean_Parser_Command_c lean_mark_persistent(l_Lean_Parser_Command_ctor_formatter___closed__7); l_Lean_Parser_Command_ctor_formatter___closed__8 = _init_l_Lean_Parser_Command_ctor_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_ctor_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_ctor_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_ctor_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_computedField_formatter___closed__1 = _init_l_Lean_Parser_Command_computedField_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_computedField_formatter___closed__1); l_Lean_Parser_Command_computedField_formatter___closed__2 = _init_l_Lean_Parser_Command_computedField_formatter___closed__2(); @@ -68494,6 +73155,13 @@ l_Lean_Parser_Command_computedField_formatter___closed__7 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_computedField_formatter___closed__7); l_Lean_Parser_Command_computedField_formatter___closed__8 = _init_l_Lean_Parser_Command_computedField_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_computedField_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_computedField_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_computedField_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_computedFields_formatter___closed__1 = _init_l_Lean_Parser_Command_computedFields_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_computedFields_formatter___closed__1); l_Lean_Parser_Command_computedFields_formatter___closed__2 = _init_l_Lean_Parser_Command_computedFields_formatter___closed__2(); @@ -68508,8 +73176,13 @@ l_Lean_Parser_Command_computedFields_formatter___closed__6 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_computedFields_formatter___closed__6); l_Lean_Parser_Command_computedFields_formatter___closed__7 = _init_l_Lean_Parser_Command_computedFields_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_computedFields_formatter___closed__7); -l_Lean_Parser_Command_computedFields_formatter___closed__8 = _init_l_Lean_Parser_Command_computedFields_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_computedFields_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_computedFields_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_computedFields_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_derivingClasses_formatter___closed__1 = _init_l_Lean_Parser_Command_derivingClasses_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_derivingClasses_formatter___closed__1); l_Lean_Parser_Command_derivingClasses_formatter___closed__2 = _init_l_Lean_Parser_Command_derivingClasses_formatter___closed__2(); @@ -68534,6 +73207,13 @@ l_Lean_Parser_Command_optDeriving_formatter___closed__5 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_optDeriving_formatter___closed__5); l_Lean_Parser_Command_optDeriving_formatter___closed__6 = _init_l_Lean_Parser_Command_optDeriving_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_optDeriving_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_optDeriving_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_optDeriving_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_inductive_formatter___closed__1 = _init_l_Lean_Parser_Command_inductive_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_inductive_formatter___closed__1); l_Lean_Parser_Command_inductive_formatter___closed__2 = _init_l_Lean_Parser_Command_inductive_formatter___closed__2(); @@ -68562,12 +73242,13 @@ l_Lean_Parser_Command_inductive_formatter___closed__13 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_inductive_formatter___closed__13); l_Lean_Parser_Command_inductive_formatter___closed__14 = _init_l_Lean_Parser_Command_inductive_formatter___closed__14(); lean_mark_persistent(l_Lean_Parser_Command_inductive_formatter___closed__14); -l_Lean_Parser_Command_inductive_formatter___closed__15 = _init_l_Lean_Parser_Command_inductive_formatter___closed__15(); -lean_mark_persistent(l_Lean_Parser_Command_inductive_formatter___closed__15); -l_Lean_Parser_Command_inductive_formatter___closed__16 = _init_l_Lean_Parser_Command_inductive_formatter___closed__16(); -lean_mark_persistent(l_Lean_Parser_Command_inductive_formatter___closed__16); -l_Lean_Parser_Command_inductive_formatter___closed__17 = _init_l_Lean_Parser_Command_inductive_formatter___closed__17(); -lean_mark_persistent(l_Lean_Parser_Command_inductive_formatter___closed__17); +l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_inductive_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_inductive_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_classInductive_formatter___closed__1 = _init_l_Lean_Parser_Command_classInductive_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_classInductive_formatter___closed__1); l_Lean_Parser_Command_classInductive_formatter___closed__2 = _init_l_Lean_Parser_Command_classInductive_formatter___closed__2(); @@ -68590,16 +73271,37 @@ l_Lean_Parser_Command_classInductive_formatter___closed__10 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Command_classInductive_formatter___closed__10); l_Lean_Parser_Command_classInductive_formatter___closed__11 = _init_l_Lean_Parser_Command_classInductive_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_classInductive_formatter___closed__11); +l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_classInductive_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_classInductive_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structureTk_formatter___closed__1 = _init_l_Lean_Parser_Command_structureTk_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structureTk_formatter___closed__1); l_Lean_Parser_Command_structureTk_formatter___closed__2 = _init_l_Lean_Parser_Command_structureTk_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_structureTk_formatter___closed__2); l_Lean_Parser_Command_structureTk_formatter___closed__3 = _init_l_Lean_Parser_Command_structureTk_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_structureTk_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structureTk_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structureTk_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_classTk_formatter___closed__1 = _init_l_Lean_Parser_Command_classTk_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_classTk_formatter___closed__1); l_Lean_Parser_Command_classTk_formatter___closed__2 = _init_l_Lean_Parser_Command_classTk_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_classTk_formatter___closed__2); +l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_classTk_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_classTk_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_extends_formatter___closed__1 = _init_l_Lean_Parser_Command_extends_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_extends_formatter___closed__1); l_Lean_Parser_Command_extends_formatter___closed__2 = _init_l_Lean_Parser_Command_extends_formatter___closed__2(); @@ -68610,6 +73312,13 @@ l_Lean_Parser_Command_extends_formatter___closed__4 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_extends_formatter___closed__4); l_Lean_Parser_Command_extends_formatter___closed__5 = _init_l_Lean_Parser_Command_extends_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_extends_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_extends_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_extends_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structCtor_formatter___closed__1 = _init_l_Lean_Parser_Command_structCtor_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structCtor_formatter___closed__1); l_Lean_Parser_Command_structCtor_formatter___closed__2 = _init_l_Lean_Parser_Command_structCtor_formatter___closed__2(); @@ -68622,6 +73331,13 @@ l_Lean_Parser_Command_structCtor_formatter___closed__5 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_structCtor_formatter___closed__5); l_Lean_Parser_Command_structCtor_formatter___closed__6 = _init_l_Lean_Parser_Command_structCtor_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_structCtor_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structCtor_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structCtor_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structExplicitBinder_formatter___closed__1 = _init_l_Lean_Parser_Command_structExplicitBinder_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structExplicitBinder_formatter___closed__1); l_Lean_Parser_Command_structExplicitBinder_formatter___closed__2 = _init_l_Lean_Parser_Command_structExplicitBinder_formatter___closed__2(); @@ -68648,6 +73364,13 @@ l_Lean_Parser_Command_structExplicitBinder_formatter___closed__12 = _init_l_Lean lean_mark_persistent(l_Lean_Parser_Command_structExplicitBinder_formatter___closed__12); l_Lean_Parser_Command_structExplicitBinder_formatter___closed__13 = _init_l_Lean_Parser_Command_structExplicitBinder_formatter___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_structExplicitBinder_formatter___closed__13); +l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structExplicitBinder_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structImplicitBinder_formatter___closed__1 = _init_l_Lean_Parser_Command_structImplicitBinder_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structImplicitBinder_formatter___closed__1); l_Lean_Parser_Command_structImplicitBinder_formatter___closed__2 = _init_l_Lean_Parser_Command_structImplicitBinder_formatter___closed__2(); @@ -68664,6 +73387,13 @@ l_Lean_Parser_Command_structImplicitBinder_formatter___closed__7 = _init_l_Lean_ lean_mark_persistent(l_Lean_Parser_Command_structImplicitBinder_formatter___closed__7); l_Lean_Parser_Command_structImplicitBinder_formatter___closed__8 = _init_l_Lean_Parser_Command_structImplicitBinder_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_structImplicitBinder_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structImplicitBinder_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structInstBinder_formatter___closed__1 = _init_l_Lean_Parser_Command_structInstBinder_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structInstBinder_formatter___closed__1); l_Lean_Parser_Command_structInstBinder_formatter___closed__2 = _init_l_Lean_Parser_Command_structInstBinder_formatter___closed__2(); @@ -68682,6 +73412,13 @@ l_Lean_Parser_Command_structInstBinder_formatter___closed__8 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Command_structInstBinder_formatter___closed__8); l_Lean_Parser_Command_structInstBinder_formatter___closed__9 = _init_l_Lean_Parser_Command_structInstBinder_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_structInstBinder_formatter___closed__9); +l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structInstBinder_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structSimpleBinder_formatter___closed__1 = _init_l_Lean_Parser_Command_structSimpleBinder_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structSimpleBinder_formatter___closed__1); l_Lean_Parser_Command_structSimpleBinder_formatter___closed__2 = _init_l_Lean_Parser_Command_structSimpleBinder_formatter___closed__2(); @@ -68694,6 +73431,13 @@ l_Lean_Parser_Command_structSimpleBinder_formatter___closed__5 = _init_l_Lean_Pa lean_mark_persistent(l_Lean_Parser_Command_structSimpleBinder_formatter___closed__5); l_Lean_Parser_Command_structSimpleBinder_formatter___closed__6 = _init_l_Lean_Parser_Command_structSimpleBinder_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_structSimpleBinder_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structSimpleBinder_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structFields_formatter___closed__1 = _init_l_Lean_Parser_Command_structFields_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structFields_formatter___closed__1); l_Lean_Parser_Command_structFields_formatter___closed__2 = _init_l_Lean_Parser_Command_structFields_formatter___closed__2(); @@ -68714,14 +73458,13 @@ l_Lean_Parser_Command_structFields_formatter___closed__9 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_structFields_formatter___closed__9); l_Lean_Parser_Command_structFields_formatter___closed__10 = _init_l_Lean_Parser_Command_structFields_formatter___closed__10(); lean_mark_persistent(l_Lean_Parser_Command_structFields_formatter___closed__10); -l_Lean_Parser_Command_structFields_formatter___closed__11 = _init_l_Lean_Parser_Command_structFields_formatter___closed__11(); -lean_mark_persistent(l_Lean_Parser_Command_structFields_formatter___closed__11); -l_Lean_Parser_Command_structFields_formatter___closed__12 = _init_l_Lean_Parser_Command_structFields_formatter___closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_structFields_formatter___closed__12); -l_Lean_Parser_Command_structFields_formatter___closed__13 = _init_l_Lean_Parser_Command_structFields_formatter___closed__13(); -lean_mark_persistent(l_Lean_Parser_Command_structFields_formatter___closed__13); -l_Lean_Parser_Command_structFields_formatter___closed__14 = _init_l_Lean_Parser_Command_structFields_formatter___closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_structFields_formatter___closed__14); +l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structFields_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structFields_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structure_formatter___closed__1 = _init_l_Lean_Parser_Command_structure_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structure_formatter___closed__1); l_Lean_Parser_Command_structure_formatter___closed__2 = _init_l_Lean_Parser_Command_structure_formatter___closed__2(); @@ -68758,16 +73501,13 @@ l_Lean_Parser_Command_structure_formatter___closed__17 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_structure_formatter___closed__17); l_Lean_Parser_Command_structure_formatter___closed__18 = _init_l_Lean_Parser_Command_structure_formatter___closed__18(); lean_mark_persistent(l_Lean_Parser_Command_structure_formatter___closed__18); -l_Lean_Parser_Command_structure_formatter___closed__19 = _init_l_Lean_Parser_Command_structure_formatter___closed__19(); -lean_mark_persistent(l_Lean_Parser_Command_structure_formatter___closed__19); -l_Lean_Parser_Command_structure_formatter___closed__20 = _init_l_Lean_Parser_Command_structure_formatter___closed__20(); -lean_mark_persistent(l_Lean_Parser_Command_structure_formatter___closed__20); -l_Lean_Parser_Command_structure_formatter___closed__21 = _init_l_Lean_Parser_Command_structure_formatter___closed__21(); -lean_mark_persistent(l_Lean_Parser_Command_structure_formatter___closed__21); -l_Lean_Parser_Command_structure_formatter___closed__22 = _init_l_Lean_Parser_Command_structure_formatter___closed__22(); -lean_mark_persistent(l_Lean_Parser_Command_structure_formatter___closed__22); -l_Lean_Parser_Command_structure_formatter___closed__23 = _init_l_Lean_Parser_Command_structure_formatter___closed__23(); -lean_mark_persistent(l_Lean_Parser_Command_structure_formatter___closed__23); +l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structure_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structure_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declaration_formatter___closed__1 = _init_l_Lean_Parser_Command_declaration_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__1); l_Lean_Parser_Command_declaration_formatter___closed__2 = _init_l_Lean_Parser_Command_declaration_formatter___closed__2(); @@ -68794,66 +73534,91 @@ l_Lean_Parser_Command_declaration_formatter___closed__12 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__12); l_Lean_Parser_Command_declaration_formatter___closed__13 = _init_l_Lean_Parser_Command_declaration_formatter___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__13); -l_Lean_Parser_Command_declaration_formatter___closed__14 = _init_l_Lean_Parser_Command_declaration_formatter___closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__14); -l_Lean_Parser_Command_declaration_formatter___closed__15 = _init_l_Lean_Parser_Command_declaration_formatter___closed__15(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__15); -l_Lean_Parser_Command_declaration_formatter___closed__16 = _init_l_Lean_Parser_Command_declaration_formatter___closed__16(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__16); -l_Lean_Parser_Command_declaration_formatter___closed__17 = _init_l_Lean_Parser_Command_declaration_formatter___closed__17(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__17); -l_Lean_Parser_Command_declaration_formatter___closed__18 = _init_l_Lean_Parser_Command_declaration_formatter___closed__18(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__18); -l_Lean_Parser_Command_declaration_formatter___closed__19 = _init_l_Lean_Parser_Command_declaration_formatter___closed__19(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__19); -l_Lean_Parser_Command_declaration_formatter___closed__20 = _init_l_Lean_Parser_Command_declaration_formatter___closed__20(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__20); -l_Lean_Parser_Command_declaration_formatter___closed__21 = _init_l_Lean_Parser_Command_declaration_formatter___closed__21(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__21); -l_Lean_Parser_Command_declaration_formatter___closed__22 = _init_l_Lean_Parser_Command_declaration_formatter___closed__22(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__22); -l_Lean_Parser_Command_declaration_formatter___closed__23 = _init_l_Lean_Parser_Command_declaration_formatter___closed__23(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_formatter___closed__23); +l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declaration_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declaration_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_private_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_private_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_private_parenthesizer___closed__1); l_Lean_Parser_Command_private_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_private_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_private_parenthesizer___closed__2); l_Lean_Parser_Command_private_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_private_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_private_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_private_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_private_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_protected_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_protected_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_protected_parenthesizer___closed__1); l_Lean_Parser_Command_protected_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_protected_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_protected_parenthesizer___closed__2); l_Lean_Parser_Command_protected_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_protected_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_protected_parenthesizer___closed__3); -l_Lean_Parser_Command_visibility_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_visibility_parenthesizer___closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_visibility_parenthesizer___closed__1); -l_Lean_Parser_Command_visibility_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_visibility_parenthesizer___closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_visibility_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_protected_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_protected_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_noncomputable_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_noncomputable_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_noncomputable_parenthesizer___closed__1); l_Lean_Parser_Command_noncomputable_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_noncomputable_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_noncomputable_parenthesizer___closed__2); l_Lean_Parser_Command_noncomputable_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_noncomputable_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_noncomputable_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_noncomputable_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_unsafe_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_unsafe_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_unsafe_parenthesizer___closed__1); l_Lean_Parser_Command_unsafe_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_unsafe_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_unsafe_parenthesizer___closed__2); l_Lean_Parser_Command_unsafe_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_unsafe_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_unsafe_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_unsafe_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_partial_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_partial_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_partial_parenthesizer___closed__1); l_Lean_Parser_Command_partial_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_partial_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_partial_parenthesizer___closed__2); l_Lean_Parser_Command_partial_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_partial_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_partial_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_partial_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_partial_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_nonrec_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_nonrec_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_nonrec_parenthesizer___closed__1); l_Lean_Parser_Command_nonrec_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_nonrec_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_nonrec_parenthesizer___closed__2); l_Lean_Parser_Command_nonrec_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_nonrec_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_nonrec_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_nonrec_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declModifiers_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declModifiers_parenthesizer___closed__1); l_Lean_Parser_Command_declModifiers_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__2(); @@ -68904,14 +73669,6 @@ l_Lean_Parser_Command_declModifiers_parenthesizer___closed__24 = _init_l_Lean_Pa lean_mark_persistent(l_Lean_Parser_Command_declModifiers_parenthesizer___closed__24); l_Lean_Parser_Command_declModifiers_parenthesizer___closed__25 = _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__25(); lean_mark_persistent(l_Lean_Parser_Command_declModifiers_parenthesizer___closed__25); -l_Lean_Parser_Command_declModifiers_parenthesizer___closed__26 = _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__26(); -lean_mark_persistent(l_Lean_Parser_Command_declModifiers_parenthesizer___closed__26); -l_Lean_Parser_Command_declModifiers_parenthesizer___closed__27 = _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__27(); -lean_mark_persistent(l_Lean_Parser_Command_declModifiers_parenthesizer___closed__27); -l_Lean_Parser_Command_declModifiers_parenthesizer___closed__28 = _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__28(); -lean_mark_persistent(l_Lean_Parser_Command_declModifiers_parenthesizer___closed__28); -l_Lean_Parser_Command_declModifiers_parenthesizer___closed__29 = _init_l_Lean_Parser_Command_declModifiers_parenthesizer___closed__29(); -lean_mark_persistent(l_Lean_Parser_Command_declModifiers_parenthesizer___closed__29); l_Lean_Parser_Command_declId_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_declId_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declId_parenthesizer___closed__1); l_Lean_Parser_Command_declId_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_declId_parenthesizer___closed__2(); @@ -68934,6 +73691,13 @@ l_Lean_Parser_Command_declId_parenthesizer___closed__10 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_declId_parenthesizer___closed__10); l_Lean_Parser_Command_declId_parenthesizer___closed__11 = _init_l_Lean_Parser_Command_declId_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_declId_parenthesizer___closed__11); +l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declId_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declId_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1); l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2(); @@ -68954,6 +73718,13 @@ l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__9 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__9); l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__10 = _init_l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__10(); lean_mark_persistent(l_Lean_Parser_Command_optDeclSig_parenthesizer___closed__10); +l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_optDeclSig_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declValSimple_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_declValSimple_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declValSimple_parenthesizer___closed__1); l_Lean_Parser_Command_declValSimple_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_declValSimple_parenthesizer___closed__2(); @@ -68972,18 +73743,39 @@ l_Lean_Parser_Command_declValSimple_parenthesizer___closed__8 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Command_declValSimple_parenthesizer___closed__8); l_Lean_Parser_Command_declValSimple_parenthesizer___closed__9 = _init_l_Lean_Parser_Command_declValSimple_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_declValSimple_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declValSimple_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declValEqns_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_declValEqns_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declValEqns_parenthesizer___closed__1); l_Lean_Parser_Command_declValEqns_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_declValEqns_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_declValEqns_parenthesizer___closed__2); l_Lean_Parser_Command_declValEqns_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_declValEqns_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_declValEqns_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declValEqns_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_whereStructField_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_whereStructField_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_whereStructField_parenthesizer___closed__1); l_Lean_Parser_Command_whereStructField_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_whereStructField_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_whereStructField_parenthesizer___closed__2); l_Lean_Parser_Command_whereStructField_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_whereStructField_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_whereStructField_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_whereStructField_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1); l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2(); @@ -69000,20 +73792,19 @@ l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__7 = _init_l_Lean_P lean_mark_persistent(l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__7); l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__8); -l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__9 = _init_l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_whereStructInst_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_whereStructInst_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declVal_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declVal_parenthesizer___closed__1); l_Lean_Parser_Command_declVal_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_declVal_parenthesizer___closed__2); l_Lean_Parser_Command_declVal_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_declVal_parenthesizer___closed__3); -l_Lean_Parser_Command_declVal_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_declVal_parenthesizer___closed__4); -l_Lean_Parser_Command_declVal_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_declVal_parenthesizer___closed__5); -l_Lean_Parser_Command_declVal_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_declVal_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_declVal_parenthesizer___closed__6); l_Lean_Parser_Command_abbrev_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_abbrev_parenthesizer___closed__1); l_Lean_Parser_Command_abbrev_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__2(); @@ -69030,10 +73821,13 @@ l_Lean_Parser_Command_abbrev_parenthesizer___closed__7 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_abbrev_parenthesizer___closed__7); l_Lean_Parser_Command_abbrev_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_abbrev_parenthesizer___closed__8); -l_Lean_Parser_Command_abbrev_parenthesizer___closed__9 = _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_abbrev_parenthesizer___closed__9); -l_Lean_Parser_Command_abbrev_parenthesizer___closed__10 = _init_l_Lean_Parser_Command_abbrev_parenthesizer___closed__10(); -lean_mark_persistent(l_Lean_Parser_Command_abbrev_parenthesizer___closed__10); +l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_abbrev_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__1); l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_optDefDeriving_parenthesizer___closed__2(); @@ -69070,6 +73864,13 @@ l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__12 = _init_l_ lean_mark_persistent(l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__12); l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__13 = _init_l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_terminationByElement_parenthesizer___closed__13); +l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_terminationByElement_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_terminationBy_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_terminationBy_parenthesizer___closed__1); l_Lean_Parser_Command_terminationBy_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__2(); @@ -69082,8 +73883,13 @@ l_Lean_Parser_Command_terminationBy_parenthesizer___closed__5 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Command_terminationBy_parenthesizer___closed__5); l_Lean_Parser_Command_terminationBy_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_terminationBy_parenthesizer___closed__6); -l_Lean_Parser_Command_terminationBy_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_terminationBy_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_terminationBy_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_terminationBy_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__1); l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_terminationHintMany_parenthesizer___closed__2(); @@ -69104,6 +73910,13 @@ l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__4 = _init_l_Lean lean_mark_persistent(l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__4); l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_terminationByCore_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_terminationByCore_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1); l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2(); @@ -69116,18 +73929,19 @@ l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__5 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__5); l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_decreasingBy_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_decreasingBy_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__1); l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__2); l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__3); -l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__4); -l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__5); -l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_terminationSuffix_parenthesizer___closed__6); l_Lean_Parser_Command_def_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_def_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_def_parenthesizer___closed__1); l_Lean_Parser_Command_def_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_def_parenthesizer___closed__2(); @@ -69148,6 +73962,13 @@ l_Lean_Parser_Command_def_parenthesizer___closed__9 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_def_parenthesizer___closed__9); l_Lean_Parser_Command_def_parenthesizer___closed__10 = _init_l_Lean_Parser_Command_def_parenthesizer___closed__10(); lean_mark_persistent(l_Lean_Parser_Command_def_parenthesizer___closed__10); +l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_def_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_def_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declSig_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_declSig_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declSig_parenthesizer___closed__1); l_Lean_Parser_Command_declSig_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_declSig_parenthesizer___closed__2(); @@ -69156,6 +73977,13 @@ l_Lean_Parser_Command_declSig_parenthesizer___closed__3 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_declSig_parenthesizer___closed__3); l_Lean_Parser_Command_declSig_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_declSig_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_declSig_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declSig_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_theorem_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_theorem_parenthesizer___closed__1); l_Lean_Parser_Command_theorem_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__2(); @@ -69172,8 +74000,13 @@ l_Lean_Parser_Command_theorem_parenthesizer___closed__7 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_theorem_parenthesizer___closed__7); l_Lean_Parser_Command_theorem_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_theorem_parenthesizer___closed__8); -l_Lean_Parser_Command_theorem_parenthesizer___closed__9 = _init_l_Lean_Parser_Command_theorem_parenthesizer___closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_theorem_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_theorem_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_opaque_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_opaque_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_opaque_parenthesizer___closed__1); l_Lean_Parser_Command_opaque_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_opaque_parenthesizer___closed__2(); @@ -69188,6 +74021,13 @@ l_Lean_Parser_Command_opaque_parenthesizer___closed__6 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_opaque_parenthesizer___closed__6); l_Lean_Parser_Command_opaque_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_opaque_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_opaque_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_opaque_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_namedPrio_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_namedPrio_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_namedPrio_parenthesizer___closed__1); l_Lean_Parser_Command_namedPrio_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_namedPrio_parenthesizer___closed__2(); @@ -69210,10 +74050,15 @@ l_Lean_Parser_Command_namedPrio_parenthesizer___closed__10 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_namedPrio_parenthesizer___closed__10); l_Lean_Parser_Command_namedPrio_parenthesizer___closed__11 = _init_l_Lean_Parser_Command_namedPrio_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_namedPrio_parenthesizer___closed__11); +l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_namedPrio_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__1); -l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_optNamedPrio_parenthesizer___closed__2); l_Lean_Parser_Command_instance_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_instance_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_instance_parenthesizer___closed__1); l_Lean_Parser_Command_instance_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_instance_parenthesizer___closed__2(); @@ -69236,6 +74081,13 @@ l_Lean_Parser_Command_instance_parenthesizer___closed__10 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_instance_parenthesizer___closed__10); l_Lean_Parser_Command_instance_parenthesizer___closed__11 = _init_l_Lean_Parser_Command_instance_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_instance_parenthesizer___closed__11); +l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_instance_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_instance_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_axiom_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_axiom_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_axiom_parenthesizer___closed__1); l_Lean_Parser_Command_axiom_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_axiom_parenthesizer___closed__2(); @@ -69246,6 +74098,13 @@ l_Lean_Parser_Command_axiom_parenthesizer___closed__4 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_axiom_parenthesizer___closed__4); l_Lean_Parser_Command_axiom_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_axiom_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_axiom_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_axiom_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_example_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_example_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_example_parenthesizer___closed__1); l_Lean_Parser_Command_example_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_example_parenthesizer___closed__2(); @@ -69256,6 +74115,13 @@ l_Lean_Parser_Command_example_parenthesizer___closed__4 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_example_parenthesizer___closed__4); l_Lean_Parser_Command_example_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_example_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_example_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_example_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_example_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_ctor_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_ctor_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_ctor_parenthesizer___closed__1); l_Lean_Parser_Command_ctor_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_ctor_parenthesizer___closed__2(); @@ -69272,6 +74138,13 @@ l_Lean_Parser_Command_ctor_parenthesizer___closed__7 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_ctor_parenthesizer___closed__7); l_Lean_Parser_Command_ctor_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_ctor_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_ctor_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_ctor_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_computedField_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_computedField_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_computedField_parenthesizer___closed__1); l_Lean_Parser_Command_computedField_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_computedField_parenthesizer___closed__2(); @@ -69288,6 +74161,13 @@ l_Lean_Parser_Command_computedField_parenthesizer___closed__7 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Command_computedField_parenthesizer___closed__7); l_Lean_Parser_Command_computedField_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_computedField_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_computedField_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_computedField_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_computedFields_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_computedFields_parenthesizer___closed__1); l_Lean_Parser_Command_computedFields_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__2(); @@ -69302,8 +74182,13 @@ l_Lean_Parser_Command_computedFields_parenthesizer___closed__6 = _init_l_Lean_Pa lean_mark_persistent(l_Lean_Parser_Command_computedFields_parenthesizer___closed__6); l_Lean_Parser_Command_computedFields_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_computedFields_parenthesizer___closed__7); -l_Lean_Parser_Command_computedFields_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_computedFields_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_computedFields_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_computedFields_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__1); l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_derivingClasses_parenthesizer___closed__2(); @@ -69328,6 +74213,13 @@ l_Lean_Parser_Command_optDeriving_parenthesizer___closed__5 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Command_optDeriving_parenthesizer___closed__5); l_Lean_Parser_Command_optDeriving_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_optDeriving_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_optDeriving_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_optDeriving_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_inductive_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_inductive_parenthesizer___closed__1); l_Lean_Parser_Command_inductive_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__2(); @@ -69356,12 +74248,13 @@ l_Lean_Parser_Command_inductive_parenthesizer___closed__13 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_inductive_parenthesizer___closed__13); l_Lean_Parser_Command_inductive_parenthesizer___closed__14 = _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__14(); lean_mark_persistent(l_Lean_Parser_Command_inductive_parenthesizer___closed__14); -l_Lean_Parser_Command_inductive_parenthesizer___closed__15 = _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__15(); -lean_mark_persistent(l_Lean_Parser_Command_inductive_parenthesizer___closed__15); -l_Lean_Parser_Command_inductive_parenthesizer___closed__16 = _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__16(); -lean_mark_persistent(l_Lean_Parser_Command_inductive_parenthesizer___closed__16); -l_Lean_Parser_Command_inductive_parenthesizer___closed__17 = _init_l_Lean_Parser_Command_inductive_parenthesizer___closed__17(); -lean_mark_persistent(l_Lean_Parser_Command_inductive_parenthesizer___closed__17); +l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_inductive_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_classInductive_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_classInductive_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_classInductive_parenthesizer___closed__1); l_Lean_Parser_Command_classInductive_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_classInductive_parenthesizer___closed__2(); @@ -69384,16 +74277,37 @@ l_Lean_Parser_Command_classInductive_parenthesizer___closed__10 = _init_l_Lean_P lean_mark_persistent(l_Lean_Parser_Command_classInductive_parenthesizer___closed__10); l_Lean_Parser_Command_classInductive_parenthesizer___closed__11 = _init_l_Lean_Parser_Command_classInductive_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_classInductive_parenthesizer___closed__11); +l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_classInductive_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structureTk_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_structureTk_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structureTk_parenthesizer___closed__1); l_Lean_Parser_Command_structureTk_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_structureTk_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_structureTk_parenthesizer___closed__2); l_Lean_Parser_Command_structureTk_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_structureTk_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_structureTk_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structureTk_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_classTk_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_classTk_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_classTk_parenthesizer___closed__1); l_Lean_Parser_Command_classTk_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_classTk_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_classTk_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_classTk_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_extends_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_extends_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_extends_parenthesizer___closed__1); l_Lean_Parser_Command_extends_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_extends_parenthesizer___closed__2(); @@ -69404,6 +74318,13 @@ l_Lean_Parser_Command_extends_parenthesizer___closed__4 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_extends_parenthesizer___closed__4); l_Lean_Parser_Command_extends_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_extends_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_extends_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_extends_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_extends_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structCtor_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_structCtor_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structCtor_parenthesizer___closed__1); l_Lean_Parser_Command_structCtor_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_structCtor_parenthesizer___closed__2(); @@ -69416,6 +74337,13 @@ l_Lean_Parser_Command_structCtor_parenthesizer___closed__5 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_structCtor_parenthesizer___closed__5); l_Lean_Parser_Command_structCtor_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_structCtor_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_structCtor_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structCtor_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1); l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2(); @@ -69442,6 +74370,13 @@ l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__12 = _init_l_ lean_mark_persistent(l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__12); l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__13 = _init_l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__13); +l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structExplicitBinder_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1); l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2(); @@ -69458,6 +74393,13 @@ l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__7 = _init_l_L lean_mark_persistent(l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__7); l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structImplicitBinder_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1); l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2(); @@ -69476,6 +74418,13 @@ l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__8 = _init_l_Lean_ lean_mark_persistent(l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__8); l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__9 = _init_l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_structInstBinder_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structInstBinder_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1); l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2(); @@ -69488,6 +74437,13 @@ l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__5 = _init_l_Lea lean_mark_persistent(l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__5); l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structSimpleBinder_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structFields_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structFields_parenthesizer___closed__1); l_Lean_Parser_Command_structFields_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__2(); @@ -69508,14 +74464,13 @@ l_Lean_Parser_Command_structFields_parenthesizer___closed__9 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Command_structFields_parenthesizer___closed__9); l_Lean_Parser_Command_structFields_parenthesizer___closed__10 = _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__10(); lean_mark_persistent(l_Lean_Parser_Command_structFields_parenthesizer___closed__10); -l_Lean_Parser_Command_structFields_parenthesizer___closed__11 = _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__11(); -lean_mark_persistent(l_Lean_Parser_Command_structFields_parenthesizer___closed__11); -l_Lean_Parser_Command_structFields_parenthesizer___closed__12 = _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_structFields_parenthesizer___closed__12); -l_Lean_Parser_Command_structFields_parenthesizer___closed__13 = _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__13(); -lean_mark_persistent(l_Lean_Parser_Command_structFields_parenthesizer___closed__13); -l_Lean_Parser_Command_structFields_parenthesizer___closed__14 = _init_l_Lean_Parser_Command_structFields_parenthesizer___closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_structFields_parenthesizer___closed__14); +l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structFields_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_structure_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_structure_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_structure_parenthesizer___closed__1); l_Lean_Parser_Command_structure_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_structure_parenthesizer___closed__2(); @@ -69552,16 +74507,13 @@ l_Lean_Parser_Command_structure_parenthesizer___closed__17 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_structure_parenthesizer___closed__17); l_Lean_Parser_Command_structure_parenthesizer___closed__18 = _init_l_Lean_Parser_Command_structure_parenthesizer___closed__18(); lean_mark_persistent(l_Lean_Parser_Command_structure_parenthesizer___closed__18); -l_Lean_Parser_Command_structure_parenthesizer___closed__19 = _init_l_Lean_Parser_Command_structure_parenthesizer___closed__19(); -lean_mark_persistent(l_Lean_Parser_Command_structure_parenthesizer___closed__19); -l_Lean_Parser_Command_structure_parenthesizer___closed__20 = _init_l_Lean_Parser_Command_structure_parenthesizer___closed__20(); -lean_mark_persistent(l_Lean_Parser_Command_structure_parenthesizer___closed__20); -l_Lean_Parser_Command_structure_parenthesizer___closed__21 = _init_l_Lean_Parser_Command_structure_parenthesizer___closed__21(); -lean_mark_persistent(l_Lean_Parser_Command_structure_parenthesizer___closed__21); -l_Lean_Parser_Command_structure_parenthesizer___closed__22 = _init_l_Lean_Parser_Command_structure_parenthesizer___closed__22(); -lean_mark_persistent(l_Lean_Parser_Command_structure_parenthesizer___closed__22); -l_Lean_Parser_Command_structure_parenthesizer___closed__23 = _init_l_Lean_Parser_Command_structure_parenthesizer___closed__23(); -lean_mark_persistent(l_Lean_Parser_Command_structure_parenthesizer___closed__23); +l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_structure_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_structure_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declaration_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__1); l_Lean_Parser_Command_declaration_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__2(); @@ -69588,26 +74540,13 @@ l_Lean_Parser_Command_declaration_parenthesizer___closed__12 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__12); l_Lean_Parser_Command_declaration_parenthesizer___closed__13 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__13); -l_Lean_Parser_Command_declaration_parenthesizer___closed__14 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__14); -l_Lean_Parser_Command_declaration_parenthesizer___closed__15 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__15(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__15); -l_Lean_Parser_Command_declaration_parenthesizer___closed__16 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__16(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__16); -l_Lean_Parser_Command_declaration_parenthesizer___closed__17 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__17(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__17); -l_Lean_Parser_Command_declaration_parenthesizer___closed__18 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__18(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__18); -l_Lean_Parser_Command_declaration_parenthesizer___closed__19 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__19(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__19); -l_Lean_Parser_Command_declaration_parenthesizer___closed__20 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__20(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__20); -l_Lean_Parser_Command_declaration_parenthesizer___closed__21 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__21(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__21); -l_Lean_Parser_Command_declaration_parenthesizer___closed__22 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__22(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__22); -l_Lean_Parser_Command_declaration_parenthesizer___closed__23 = _init_l_Lean_Parser_Command_declaration_parenthesizer___closed__23(); -lean_mark_persistent(l_Lean_Parser_Command_declaration_parenthesizer___closed__23); +l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_declaration_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_deriving___elambda__1___closed__1 = _init_l_Lean_Parser_Command_deriving___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_deriving___elambda__1___closed__1); l_Lean_Parser_Command_deriving___elambda__1___closed__2 = _init_l_Lean_Parser_Command_deriving___elambda__1___closed__2(); @@ -69714,6 +74653,13 @@ l_Lean_Parser_Command_deriving_formatter___closed__7 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_deriving_formatter___closed__7); l_Lean_Parser_Command_deriving_formatter___closed__8 = _init_l_Lean_Parser_Command_deriving_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_deriving_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_deriving_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_deriving_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_deriving_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_deriving_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_deriving_parenthesizer___closed__1); l_Lean_Parser_Command_deriving_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_deriving_parenthesizer___closed__2(); @@ -69730,6 +74676,13 @@ l_Lean_Parser_Command_deriving_parenthesizer___closed__7 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_deriving_parenthesizer___closed__7); l_Lean_Parser_Command_deriving_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_deriving_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_deriving_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_deriving_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__1 = _init_l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__1); l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__2 = _init_l_Lean_Parser_Command_noncomputableSection___elambda__1___closed__2(); @@ -69810,6 +74763,13 @@ l_Lean_Parser_Command_noncomputableSection_formatter___closed__5 = _init_l_Lean_ lean_mark_persistent(l_Lean_Parser_Command_noncomputableSection_formatter___closed__5); l_Lean_Parser_Command_noncomputableSection_formatter___closed__6 = _init_l_Lean_Parser_Command_noncomputableSection_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_noncomputableSection_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_noncomputableSection_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1); l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__2(); @@ -69822,6 +74782,13 @@ l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__5 = _init_l_L lean_mark_persistent(l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__5); l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_noncomputableSection_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_section___elambda__1___closed__1 = _init_l_Lean_Parser_Command_section___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_section___elambda__1___closed__1); l_Lean_Parser_Command_section___elambda__1___closed__2 = _init_l_Lean_Parser_Command_section___elambda__1___closed__2(); @@ -69872,10 +74839,24 @@ l_Lean_Parser_Command_section_formatter___closed__1 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_section_formatter___closed__1); l_Lean_Parser_Command_section_formatter___closed__2 = _init_l_Lean_Parser_Command_section_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_section_formatter___closed__2); +l___regBuiltin_Lean_Parser_Command_section_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_section_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_section_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_section_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_section_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_section_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_section_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_section_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_section_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_section_parenthesizer___closed__1); l_Lean_Parser_Command_section_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_section_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_section_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_section_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_section_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_namespace___elambda__1___closed__1 = _init_l_Lean_Parser_Command_namespace___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_namespace___elambda__1___closed__1); l_Lean_Parser_Command_namespace___elambda__1___closed__2 = _init_l_Lean_Parser_Command_namespace___elambda__1___closed__2(); @@ -69946,6 +74927,13 @@ l_Lean_Parser_Command_namespace_formatter___closed__3 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_namespace_formatter___closed__3); l_Lean_Parser_Command_namespace_formatter___closed__4 = _init_l_Lean_Parser_Command_namespace_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_namespace_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namespace_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_namespace_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_namespace_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_namespace_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_namespace_parenthesizer___closed__1); l_Lean_Parser_Command_namespace_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_namespace_parenthesizer___closed__2(); @@ -69954,6 +74942,13 @@ l_Lean_Parser_Command_namespace_parenthesizer___closed__3 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_namespace_parenthesizer___closed__3); l_Lean_Parser_Command_namespace_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_namespace_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_namespace_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_namespace_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_end___elambda__1___closed__1 = _init_l_Lean_Parser_Command_end___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_end___elambda__1___closed__1); l_Lean_Parser_Command_end___elambda__1___closed__2 = _init_l_Lean_Parser_Command_end___elambda__1___closed__2(); @@ -70024,6 +75019,13 @@ l_Lean_Parser_Command_end_formatter___closed__3 = _init_l_Lean_Parser_Command_en lean_mark_persistent(l_Lean_Parser_Command_end_formatter___closed__3); l_Lean_Parser_Command_end_formatter___closed__4 = _init_l_Lean_Parser_Command_end_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_end_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_end_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_end_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_end_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_end_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_end_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_end_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_end_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_end_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_end_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_end_parenthesizer___closed__1); l_Lean_Parser_Command_end_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_end_parenthesizer___closed__2(); @@ -70032,6 +75034,13 @@ l_Lean_Parser_Command_end_parenthesizer___closed__3 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_end_parenthesizer___closed__3); l_Lean_Parser_Command_end_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_end_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_end_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_end_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_end_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_variable___elambda__1___closed__1 = _init_l_Lean_Parser_Command_variable___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_variable___elambda__1___closed__1); l_Lean_Parser_Command_variable___elambda__1___closed__2 = _init_l_Lean_Parser_Command_variable___elambda__1___closed__2(); @@ -70104,6 +75113,13 @@ l_Lean_Parser_Command_variable_formatter___closed__4 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_variable_formatter___closed__4); l_Lean_Parser_Command_variable_formatter___closed__5 = _init_l_Lean_Parser_Command_variable_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_variable_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_variable_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_variable_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_variable_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_variable_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_variable_parenthesizer___closed__1); l_Lean_Parser_Command_variable_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_variable_parenthesizer___closed__2(); @@ -70114,6 +75130,13 @@ l_Lean_Parser_Command_variable_parenthesizer___closed__4 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_variable_parenthesizer___closed__4); l_Lean_Parser_Command_variable_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_variable_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_variable_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_variable_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_variable_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_universe___elambda__1___closed__1 = _init_l_Lean_Parser_Command_universe___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_universe___elambda__1___closed__1); l_Lean_Parser_Command_universe___elambda__1___closed__2 = _init_l_Lean_Parser_Command_universe___elambda__1___closed__2(); @@ -70184,6 +75207,13 @@ l_Lean_Parser_Command_universe_formatter___closed__3 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_universe_formatter___closed__3); l_Lean_Parser_Command_universe_formatter___closed__4 = _init_l_Lean_Parser_Command_universe_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_universe_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_universe_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_universe_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_universe_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_universe_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_universe_parenthesizer___closed__1); l_Lean_Parser_Command_universe_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_universe_parenthesizer___closed__2(); @@ -70192,6 +75222,13 @@ l_Lean_Parser_Command_universe_parenthesizer___closed__3 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_universe_parenthesizer___closed__3); l_Lean_Parser_Command_universe_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_universe_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_universe_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_universe_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_universe_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_check___elambda__1___closed__1 = _init_l_Lean_Parser_Command_check___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_check___elambda__1___closed__1); l_Lean_Parser_Command_check___elambda__1___closed__2 = _init_l_Lean_Parser_Command_check___elambda__1___closed__2(); @@ -70262,6 +75299,13 @@ l_Lean_Parser_Command_check_formatter___closed__3 = _init_l_Lean_Parser_Command_ lean_mark_persistent(l_Lean_Parser_Command_check_formatter___closed__3); l_Lean_Parser_Command_check_formatter___closed__4 = _init_l_Lean_Parser_Command_check_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_check_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_check_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_check_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_check_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_check_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_check_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_check_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_check_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_check_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_check_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_check_parenthesizer___closed__1); l_Lean_Parser_Command_check_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_check_parenthesizer___closed__2(); @@ -70270,6 +75314,13 @@ l_Lean_Parser_Command_check_parenthesizer___closed__3 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_check_parenthesizer___closed__3); l_Lean_Parser_Command_check_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_check_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_check_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_check_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_check_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_check__failure___elambda__1___closed__1 = _init_l_Lean_Parser_Command_check__failure___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_check__failure___elambda__1___closed__1); l_Lean_Parser_Command_check__failure___elambda__1___closed__2 = _init_l_Lean_Parser_Command_check__failure___elambda__1___closed__2(); @@ -70340,6 +75391,13 @@ l_Lean_Parser_Command_check__failure_formatter___closed__3 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_check__failure_formatter___closed__3); l_Lean_Parser_Command_check__failure_formatter___closed__4 = _init_l_Lean_Parser_Command_check__failure_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_check__failure_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_check__failure_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_check__failure_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_check__failure_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_check__failure_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_check__failure_parenthesizer___closed__1); l_Lean_Parser_Command_check__failure_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_check__failure_parenthesizer___closed__2(); @@ -70348,6 +75406,13 @@ l_Lean_Parser_Command_check__failure_parenthesizer___closed__3 = _init_l_Lean_Pa lean_mark_persistent(l_Lean_Parser_Command_check__failure_parenthesizer___closed__3); l_Lean_Parser_Command_check__failure_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_check__failure_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_check__failure_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_check__failure_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_reduce___elambda__1___closed__1 = _init_l_Lean_Parser_Command_reduce___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_reduce___elambda__1___closed__1); l_Lean_Parser_Command_reduce___elambda__1___closed__2 = _init_l_Lean_Parser_Command_reduce___elambda__1___closed__2(); @@ -70418,6 +75483,13 @@ l_Lean_Parser_Command_reduce_formatter___closed__3 = _init_l_Lean_Parser_Command lean_mark_persistent(l_Lean_Parser_Command_reduce_formatter___closed__3); l_Lean_Parser_Command_reduce_formatter___closed__4 = _init_l_Lean_Parser_Command_reduce_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_reduce_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_reduce_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_reduce_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_reduce_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_reduce_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_reduce_parenthesizer___closed__1); l_Lean_Parser_Command_reduce_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_reduce_parenthesizer___closed__2(); @@ -70426,6 +75498,13 @@ l_Lean_Parser_Command_reduce_parenthesizer___closed__3 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_reduce_parenthesizer___closed__3); l_Lean_Parser_Command_reduce_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_reduce_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_reduce_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_reduce_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_eval___elambda__1___closed__1 = _init_l_Lean_Parser_Command_eval___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_eval___elambda__1___closed__1); l_Lean_Parser_Command_eval___elambda__1___closed__2 = _init_l_Lean_Parser_Command_eval___elambda__1___closed__2(); @@ -70496,6 +75575,13 @@ l_Lean_Parser_Command_eval_formatter___closed__3 = _init_l_Lean_Parser_Command_e lean_mark_persistent(l_Lean_Parser_Command_eval_formatter___closed__3); l_Lean_Parser_Command_eval_formatter___closed__4 = _init_l_Lean_Parser_Command_eval_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_eval_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_eval_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_eval_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_eval_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_eval_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_eval_parenthesizer___closed__1); l_Lean_Parser_Command_eval_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_eval_parenthesizer___closed__2(); @@ -70504,6 +75590,13 @@ l_Lean_Parser_Command_eval_parenthesizer___closed__3 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_eval_parenthesizer___closed__3); l_Lean_Parser_Command_eval_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_eval_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_eval_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_eval_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_eval_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_synth___elambda__1___closed__1 = _init_l_Lean_Parser_Command_synth___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_synth___elambda__1___closed__1); l_Lean_Parser_Command_synth___elambda__1___closed__2 = _init_l_Lean_Parser_Command_synth___elambda__1___closed__2(); @@ -70574,6 +75667,13 @@ l_Lean_Parser_Command_synth_formatter___closed__3 = _init_l_Lean_Parser_Command_ lean_mark_persistent(l_Lean_Parser_Command_synth_formatter___closed__3); l_Lean_Parser_Command_synth_formatter___closed__4 = _init_l_Lean_Parser_Command_synth_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_synth_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_synth_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_synth_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_synth_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_synth_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_synth_parenthesizer___closed__1); l_Lean_Parser_Command_synth_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_synth_parenthesizer___closed__2(); @@ -70582,6 +75682,13 @@ l_Lean_Parser_Command_synth_parenthesizer___closed__3 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_synth_parenthesizer___closed__3); l_Lean_Parser_Command_synth_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_synth_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_synth_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_synth_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_synth_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_exit___elambda__1___closed__1 = _init_l_Lean_Parser_Command_exit___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_exit___elambda__1___closed__1); l_Lean_Parser_Command_exit___elambda__1___closed__2 = _init_l_Lean_Parser_Command_exit___elambda__1___closed__2(); @@ -70646,12 +75753,26 @@ l_Lean_Parser_Command_exit_formatter___closed__2 = _init_l_Lean_Parser_Command_e lean_mark_persistent(l_Lean_Parser_Command_exit_formatter___closed__2); l_Lean_Parser_Command_exit_formatter___closed__3 = _init_l_Lean_Parser_Command_exit_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_exit_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_exit_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_exit_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_exit_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_exit_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_exit_parenthesizer___closed__1); l_Lean_Parser_Command_exit_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_exit_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_exit_parenthesizer___closed__2); l_Lean_Parser_Command_exit_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_exit_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_exit_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_exit_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_exit_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_print___elambda__1___closed__1 = _init_l_Lean_Parser_Command_print___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_print___elambda__1___closed__1); l_Lean_Parser_Command_print___elambda__1___closed__2 = _init_l_Lean_Parser_Command_print___elambda__1___closed__2(); @@ -70732,6 +75853,13 @@ l_Lean_Parser_Command_print_formatter___closed__5 = _init_l_Lean_Parser_Command_ lean_mark_persistent(l_Lean_Parser_Command_print_formatter___closed__5); l_Lean_Parser_Command_print_formatter___closed__6 = _init_l_Lean_Parser_Command_print_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_print_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_print_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_print_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_print_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_print_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_print_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_print_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_print_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_print_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_print_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_print_parenthesizer___closed__1); l_Lean_Parser_Command_print_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_print_parenthesizer___closed__2(); @@ -70744,6 +75872,13 @@ l_Lean_Parser_Command_print_parenthesizer___closed__5 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_print_parenthesizer___closed__5); l_Lean_Parser_Command_print_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_print_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_print_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_print_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_print_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_printAxioms___elambda__1___closed__1 = _init_l_Lean_Parser_Command_printAxioms___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_printAxioms___elambda__1___closed__1); l_Lean_Parser_Command_printAxioms___elambda__1___closed__2 = _init_l_Lean_Parser_Command_printAxioms___elambda__1___closed__2(); @@ -70820,6 +75955,13 @@ l_Lean_Parser_Command_printAxioms_formatter___closed__4 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_printAxioms_formatter___closed__4); l_Lean_Parser_Command_printAxioms_formatter___closed__5 = _init_l_Lean_Parser_Command_printAxioms_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_printAxioms_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_printAxioms_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_printAxioms_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_printAxioms_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_printAxioms_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_printAxioms_parenthesizer___closed__1); l_Lean_Parser_Command_printAxioms_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_printAxioms_parenthesizer___closed__2(); @@ -70830,6 +75972,13 @@ l_Lean_Parser_Command_printAxioms_parenthesizer___closed__4 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Command_printAxioms_parenthesizer___closed__4); l_Lean_Parser_Command_printAxioms_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_printAxioms_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_printAxioms_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_printAxioms_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_resolve__name___elambda__1___closed__1 = _init_l_Lean_Parser_Command_resolve__name___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_resolve__name___elambda__1___closed__1); l_Lean_Parser_Command_resolve__name___elambda__1___closed__2 = _init_l_Lean_Parser_Command_resolve__name___elambda__1___closed__2(); @@ -70900,6 +76049,13 @@ l_Lean_Parser_Command_resolve__name_formatter___closed__3 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_resolve__name_formatter___closed__3); l_Lean_Parser_Command_resolve__name_formatter___closed__4 = _init_l_Lean_Parser_Command_resolve__name_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_resolve__name_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_resolve__name_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_resolve__name_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_resolve__name_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_resolve__name_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_resolve__name_parenthesizer___closed__1); l_Lean_Parser_Command_resolve__name_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_resolve__name_parenthesizer___closed__2(); @@ -70908,6 +76064,13 @@ l_Lean_Parser_Command_resolve__name_parenthesizer___closed__3 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Command_resolve__name_parenthesizer___closed__3); l_Lean_Parser_Command_resolve__name_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_resolve__name_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_resolve__name_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_resolve__name_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_init__quot___elambda__1___closed__1 = _init_l_Lean_Parser_Command_init__quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_init__quot___elambda__1___closed__1); l_Lean_Parser_Command_init__quot___elambda__1___closed__2 = _init_l_Lean_Parser_Command_init__quot___elambda__1___closed__2(); @@ -70970,12 +76133,26 @@ l_Lean_Parser_Command_init__quot_formatter___closed__2 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_init__quot_formatter___closed__2); l_Lean_Parser_Command_init__quot_formatter___closed__3 = _init_l_Lean_Parser_Command_init__quot_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_init__quot_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_init__quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_init__quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_init__quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_init__quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_init__quot_parenthesizer___closed__1); l_Lean_Parser_Command_init__quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_init__quot_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_init__quot_parenthesizer___closed__2); l_Lean_Parser_Command_init__quot_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_init__quot_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_init__quot_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_init__quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_optionValue___elambda__1___closed__1 = _init_l_Lean_Parser_Command_optionValue___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_optionValue___elambda__1___closed__1); l_Lean_Parser_Command_optionValue___elambda__1___closed__2 = _init_l_Lean_Parser_Command_optionValue___elambda__1___closed__2(); @@ -71104,6 +76281,13 @@ l_Lean_Parser_Command_set__option_formatter___closed__6 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_set__option_formatter___closed__6); l_Lean_Parser_Command_set__option_formatter___closed__7 = _init_l_Lean_Parser_Command_set__option_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_set__option_formatter___closed__7); +l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_set__option_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_set__option_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_optionValue_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_optionValue_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_optionValue_parenthesizer___closed__1); l_Lean_Parser_Command_optionValue_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_optionValue_parenthesizer___closed__2(); @@ -71128,6 +76312,13 @@ l_Lean_Parser_Command_set__option_parenthesizer___closed__6 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Command_set__option_parenthesizer___closed__6); l_Lean_Parser_Command_set__option_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_set__option_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_set__option_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_set__option_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_eraseAttr___elambda__1___closed__1 = _init_l_Lean_Parser_Command_eraseAttr___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_eraseAttr___elambda__1___closed__1); l_Lean_Parser_Command_eraseAttr___elambda__1___closed__2 = _init_l_Lean_Parser_Command_eraseAttr___elambda__1___closed__2(); @@ -71282,6 +76473,13 @@ l_Lean_Parser_Command_eraseAttr_formatter___closed__4 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_eraseAttr_formatter___closed__4); l_Lean_Parser_Command_eraseAttr_formatter___closed__5 = _init_l_Lean_Parser_Command_eraseAttr_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_eraseAttr_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_eraseAttr_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_attribute_formatter___closed__1 = _init_l_Lean_Parser_Command_attribute_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_attribute_formatter___closed__1); l_Lean_Parser_Command_attribute_formatter___closed__2 = _init_l_Lean_Parser_Command_attribute_formatter___closed__2(); @@ -71304,8 +76502,13 @@ l_Lean_Parser_Command_attribute_formatter___closed__10 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_attribute_formatter___closed__10); l_Lean_Parser_Command_attribute_formatter___closed__11 = _init_l_Lean_Parser_Command_attribute_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_attribute_formatter___closed__11); -l_Lean_Parser_Command_attribute_formatter___closed__12 = _init_l_Lean_Parser_Command_attribute_formatter___closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_attribute_formatter___closed__12); +l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_attribute_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_attribute_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1); l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2(); @@ -71316,6 +76519,13 @@ l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__4 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__4); l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_eraseAttr_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_eraseAttr_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_attribute_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_attribute_parenthesizer___closed__1); l_Lean_Parser_Command_attribute_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__2(); @@ -71338,8 +76548,13 @@ l_Lean_Parser_Command_attribute_parenthesizer___closed__10 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_attribute_parenthesizer___closed__10); l_Lean_Parser_Command_attribute_parenthesizer___closed__11 = _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_attribute_parenthesizer___closed__11); -l_Lean_Parser_Command_attribute_parenthesizer___closed__12 = _init_l_Lean_Parser_Command_attribute_parenthesizer___closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_attribute_parenthesizer___closed__12); +l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_attribute_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_export___elambda__1___closed__1 = _init_l_Lean_Parser_Command_export___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_export___elambda__1___closed__1); l_Lean_Parser_Command_export___elambda__1___closed__2 = _init_l_Lean_Parser_Command_export___elambda__1___closed__2(); @@ -71442,6 +76657,13 @@ l_Lean_Parser_Command_export_formatter___closed__7 = _init_l_Lean_Parser_Command lean_mark_persistent(l_Lean_Parser_Command_export_formatter___closed__7); l_Lean_Parser_Command_export_formatter___closed__8 = _init_l_Lean_Parser_Command_export_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_export_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_export_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_export_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_export_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_export_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_export_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_export_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_export_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_export_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_export_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_export_parenthesizer___closed__1); l_Lean_Parser_Command_export_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_export_parenthesizer___closed__2(); @@ -71458,6 +76680,13 @@ l_Lean_Parser_Command_export_parenthesizer___closed__7 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_export_parenthesizer___closed__7); l_Lean_Parser_Command_export_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_export_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_export_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_export_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_export_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openHiding___elambda__1___closed__1 = _init_l_Lean_Parser_Command_openHiding___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openHiding___elambda__1___closed__1); l_Lean_Parser_Command_openHiding___elambda__1___closed__2 = _init_l_Lean_Parser_Command_openHiding___elambda__1___closed__2(); @@ -71806,6 +77035,13 @@ l_Lean_Parser_Command_openHiding_formatter___closed__8 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_openHiding_formatter___closed__8); l_Lean_Parser_Command_openHiding_formatter___closed__9 = _init_l_Lean_Parser_Command_openHiding_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_openHiding_formatter___closed__9); +l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openHiding_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openHiding_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openRenamingItem_formatter___closed__1 = _init_l_Lean_Parser_Command_openRenamingItem_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openRenamingItem_formatter___closed__1); l_Lean_Parser_Command_openRenamingItem_formatter___closed__2 = _init_l_Lean_Parser_Command_openRenamingItem_formatter___closed__2(); @@ -71816,6 +77052,13 @@ l_Lean_Parser_Command_openRenamingItem_formatter___closed__4 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Command_openRenamingItem_formatter___closed__4); l_Lean_Parser_Command_openRenamingItem_formatter___closed__5 = _init_l_Lean_Parser_Command_openRenamingItem_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_openRenamingItem_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openRenamingItem_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openRenaming_formatter___closed__1 = _init_l_Lean_Parser_Command_openRenaming_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openRenaming_formatter___closed__1); l_Lean_Parser_Command_openRenaming_formatter___closed__2 = _init_l_Lean_Parser_Command_openRenaming_formatter___closed__2(); @@ -71830,8 +77073,13 @@ l_Lean_Parser_Command_openRenaming_formatter___closed__6 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_openRenaming_formatter___closed__6); l_Lean_Parser_Command_openRenaming_formatter___closed__7 = _init_l_Lean_Parser_Command_openRenaming_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_openRenaming_formatter___closed__7); -l_Lean_Parser_Command_openRenaming_formatter___closed__8 = _init_l_Lean_Parser_Command_openRenaming_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_openRenaming_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openRenaming_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openRenaming_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openOnly_formatter___closed__1 = _init_l_Lean_Parser_Command_openOnly_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openOnly_formatter___closed__1); l_Lean_Parser_Command_openOnly_formatter___closed__2 = _init_l_Lean_Parser_Command_openOnly_formatter___closed__2(); @@ -71842,10 +77090,24 @@ l_Lean_Parser_Command_openOnly_formatter___closed__4 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_openOnly_formatter___closed__4); l_Lean_Parser_Command_openOnly_formatter___closed__5 = _init_l_Lean_Parser_Command_openOnly_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_openOnly_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openOnly_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openOnly_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openSimple_formatter___closed__1 = _init_l_Lean_Parser_Command_openSimple_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openSimple_formatter___closed__1); l_Lean_Parser_Command_openSimple_formatter___closed__2 = _init_l_Lean_Parser_Command_openSimple_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_openSimple_formatter___closed__2); +l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openSimple_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openSimple_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openScoped_formatter___closed__1 = _init_l_Lean_Parser_Command_openScoped_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openScoped_formatter___closed__1); l_Lean_Parser_Command_openScoped_formatter___closed__2 = _init_l_Lean_Parser_Command_openScoped_formatter___closed__2(); @@ -71854,22 +77116,19 @@ l_Lean_Parser_Command_openScoped_formatter___closed__3 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_openScoped_formatter___closed__3); l_Lean_Parser_Command_openScoped_formatter___closed__4 = _init_l_Lean_Parser_Command_openScoped_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_openScoped_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openScoped_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openScoped_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openDecl_formatter___closed__1 = _init_l_Lean_Parser_Command_openDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openDecl_formatter___closed__1); l_Lean_Parser_Command_openDecl_formatter___closed__2 = _init_l_Lean_Parser_Command_openDecl_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_openDecl_formatter___closed__2); l_Lean_Parser_Command_openDecl_formatter___closed__3 = _init_l_Lean_Parser_Command_openDecl_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_openDecl_formatter___closed__3); -l_Lean_Parser_Command_openDecl_formatter___closed__4 = _init_l_Lean_Parser_Command_openDecl_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_formatter___closed__4); -l_Lean_Parser_Command_openDecl_formatter___closed__5 = _init_l_Lean_Parser_Command_openDecl_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_formatter___closed__5); -l_Lean_Parser_Command_openDecl_formatter___closed__6 = _init_l_Lean_Parser_Command_openDecl_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_formatter___closed__6); -l_Lean_Parser_Command_openDecl_formatter___closed__7 = _init_l_Lean_Parser_Command_openDecl_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_formatter___closed__7); -l_Lean_Parser_Command_openDecl_formatter___closed__8 = _init_l_Lean_Parser_Command_openDecl_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_formatter___closed__8); l_Lean_Parser_Command_open_formatter___closed__1 = _init_l_Lean_Parser_Command_open_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_open_formatter___closed__1); l_Lean_Parser_Command_open_formatter___closed__2 = _init_l_Lean_Parser_Command_open_formatter___closed__2(); @@ -71882,6 +77141,13 @@ l_Lean_Parser_Command_open_formatter___closed__5 = _init_l_Lean_Parser_Command_o lean_mark_persistent(l_Lean_Parser_Command_open_formatter___closed__5); l_Lean_Parser_Command_open_formatter___closed__6 = _init_l_Lean_Parser_Command_open_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_open_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_open_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_open_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_open_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_open_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_open_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_open_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_open_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openHiding_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_openHiding_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openHiding_parenthesizer___closed__1); l_Lean_Parser_Command_openHiding_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_openHiding_parenthesizer___closed__2(); @@ -71900,6 +77166,13 @@ l_Lean_Parser_Command_openHiding_parenthesizer___closed__8 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_openHiding_parenthesizer___closed__8); l_Lean_Parser_Command_openHiding_parenthesizer___closed__9 = _init_l_Lean_Parser_Command_openHiding_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_openHiding_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openHiding_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1); l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2(); @@ -71910,6 +77183,13 @@ l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__4 = _init_l_Lean_ lean_mark_persistent(l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__4); l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openRenamingItem_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openRenaming_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openRenaming_parenthesizer___closed__1); l_Lean_Parser_Command_openRenaming_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__2(); @@ -71924,8 +77204,13 @@ l_Lean_Parser_Command_openRenaming_parenthesizer___closed__6 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Command_openRenaming_parenthesizer___closed__6); l_Lean_Parser_Command_openRenaming_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_openRenaming_parenthesizer___closed__7); -l_Lean_Parser_Command_openRenaming_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_openRenaming_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_openRenaming_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openRenaming_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openOnly_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_openOnly_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openOnly_parenthesizer___closed__1); l_Lean_Parser_Command_openOnly_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_openOnly_parenthesizer___closed__2(); @@ -71936,10 +77221,24 @@ l_Lean_Parser_Command_openOnly_parenthesizer___closed__4 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_openOnly_parenthesizer___closed__4); l_Lean_Parser_Command_openOnly_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_openOnly_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Command_openOnly_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openOnly_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openSimple_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_openSimple_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openSimple_parenthesizer___closed__1); l_Lean_Parser_Command_openSimple_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_openSimple_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_openSimple_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openSimple_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openScoped_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_openScoped_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openScoped_parenthesizer___closed__1); l_Lean_Parser_Command_openScoped_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_openScoped_parenthesizer___closed__2(); @@ -71948,22 +77247,19 @@ l_Lean_Parser_Command_openScoped_parenthesizer___closed__3 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_openScoped_parenthesizer___closed__3); l_Lean_Parser_Command_openScoped_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_openScoped_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_openScoped_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_openScoped_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_openDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_openDecl_parenthesizer___closed__1); l_Lean_Parser_Command_openDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_openDecl_parenthesizer___closed__2); l_Lean_Parser_Command_openDecl_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_openDecl_parenthesizer___closed__3); -l_Lean_Parser_Command_openDecl_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_parenthesizer___closed__4); -l_Lean_Parser_Command_openDecl_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_parenthesizer___closed__5); -l_Lean_Parser_Command_openDecl_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_parenthesizer___closed__6); -l_Lean_Parser_Command_openDecl_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_parenthesizer___closed__7); -l_Lean_Parser_Command_openDecl_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_openDecl_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_openDecl_parenthesizer___closed__8); l_Lean_Parser_Command_open_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_open_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_open_parenthesizer___closed__1); l_Lean_Parser_Command_open_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_open_parenthesizer___closed__2(); @@ -71976,6 +77272,13 @@ l_Lean_Parser_Command_open_parenthesizer___closed__5 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_open_parenthesizer___closed__5); l_Lean_Parser_Command_open_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_open_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_open_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_open_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_open_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_mutual___elambda__1___closed__1 = _init_l_Lean_Parser_Command_mutual___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_mutual___elambda__1___closed__1); l_Lean_Parser_Command_mutual___elambda__1___closed__2 = _init_l_Lean_Parser_Command_mutual___elambda__1___closed__2(); @@ -72100,6 +77403,13 @@ l_Lean_Parser_Command_mutual_formatter___closed__12 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_mutual_formatter___closed__12); l_Lean_Parser_Command_mutual_formatter___closed__13 = _init_l_Lean_Parser_Command_mutual_formatter___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_mutual_formatter___closed__13); +l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_mutual_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_mutual_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_mutual_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_mutual_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_mutual_parenthesizer___closed__1); l_Lean_Parser_Command_mutual_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_mutual_parenthesizer___closed__2(); @@ -72126,6 +77436,59 @@ l_Lean_Parser_Command_mutual_parenthesizer___closed__12 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_mutual_parenthesizer___closed__12); l_Lean_Parser_Command_mutual_parenthesizer___closed__13 = _init_l_Lean_Parser_Command_mutual_parenthesizer___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_mutual_parenthesizer___closed__13); +l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_mutual_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__1); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__2); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__3 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__3); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__4 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__4); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__5 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__5); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__6 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__6(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__6); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__7 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__7(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__7); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__8 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__8(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__8); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__9 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__9(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__9); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__10 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__10(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__10); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__11 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__11(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__11); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__12 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__12(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__12); +l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__13 = _init_l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__13(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___elambda__1___closed__13); +l_Lean_Parser_Command_initializeKeyword___closed__1 = _init_l_Lean_Parser_Command_initializeKeyword___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__1); +l_Lean_Parser_Command_initializeKeyword___closed__2 = _init_l_Lean_Parser_Command_initializeKeyword___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__2); +l_Lean_Parser_Command_initializeKeyword___closed__3 = _init_l_Lean_Parser_Command_initializeKeyword___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__3); +l_Lean_Parser_Command_initializeKeyword___closed__4 = _init_l_Lean_Parser_Command_initializeKeyword___closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__4); +l_Lean_Parser_Command_initializeKeyword___closed__5 = _init_l_Lean_Parser_Command_initializeKeyword___closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__5); +l_Lean_Parser_Command_initializeKeyword___closed__6 = _init_l_Lean_Parser_Command_initializeKeyword___closed__6(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__6); +l_Lean_Parser_Command_initializeKeyword___closed__7 = _init_l_Lean_Parser_Command_initializeKeyword___closed__7(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__7); +l_Lean_Parser_Command_initializeKeyword___closed__8 = _init_l_Lean_Parser_Command_initializeKeyword___closed__8(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__8); +l_Lean_Parser_Command_initializeKeyword___closed__9 = _init_l_Lean_Parser_Command_initializeKeyword___closed__9(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword___closed__9); +l_Lean_Parser_Command_initializeKeyword = _init_l_Lean_Parser_Command_initializeKeyword(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword); l_Lean_Parser_Command_initialize___elambda__1___closed__1 = _init_l_Lean_Parser_Command_initialize___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_initialize___elambda__1___closed__1); l_Lean_Parser_Command_initialize___elambda__1___closed__2 = _init_l_Lean_Parser_Command_initialize___elambda__1___closed__2(); @@ -72162,16 +77525,6 @@ l_Lean_Parser_Command_initialize___elambda__1___closed__17 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_initialize___elambda__1___closed__17); l_Lean_Parser_Command_initialize___elambda__1___closed__18 = _init_l_Lean_Parser_Command_initialize___elambda__1___closed__18(); lean_mark_persistent(l_Lean_Parser_Command_initialize___elambda__1___closed__18); -l_Lean_Parser_Command_initialize___elambda__1___closed__19 = _init_l_Lean_Parser_Command_initialize___elambda__1___closed__19(); -lean_mark_persistent(l_Lean_Parser_Command_initialize___elambda__1___closed__19); -l_Lean_Parser_Command_initialize___elambda__1___closed__20 = _init_l_Lean_Parser_Command_initialize___elambda__1___closed__20(); -lean_mark_persistent(l_Lean_Parser_Command_initialize___elambda__1___closed__20); -l_Lean_Parser_Command_initialize___elambda__1___closed__21 = _init_l_Lean_Parser_Command_initialize___elambda__1___closed__21(); -lean_mark_persistent(l_Lean_Parser_Command_initialize___elambda__1___closed__21); -l_Lean_Parser_Command_initialize___elambda__1___closed__22 = _init_l_Lean_Parser_Command_initialize___elambda__1___closed__22(); -lean_mark_persistent(l_Lean_Parser_Command_initialize___elambda__1___closed__22); -l_Lean_Parser_Command_initialize___elambda__1___closed__23 = _init_l_Lean_Parser_Command_initialize___elambda__1___closed__23(); -lean_mark_persistent(l_Lean_Parser_Command_initialize___elambda__1___closed__23); l_Lean_Parser_Command_initialize___closed__1 = _init_l_Lean_Parser_Command_initialize___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_initialize___closed__1); l_Lean_Parser_Command_initialize___closed__2 = _init_l_Lean_Parser_Command_initialize___closed__2(); @@ -72190,8 +77543,6 @@ l_Lean_Parser_Command_initialize___closed__8 = _init_l_Lean_Parser_Command_initi lean_mark_persistent(l_Lean_Parser_Command_initialize___closed__8); l_Lean_Parser_Command_initialize___closed__9 = _init_l_Lean_Parser_Command_initialize___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_initialize___closed__9); -l_Lean_Parser_Command_initialize___closed__10 = _init_l_Lean_Parser_Command_initialize___closed__10(); -lean_mark_persistent(l_Lean_Parser_Command_initialize___closed__10); l_Lean_Parser_Command_initialize = _init_l_Lean_Parser_Command_initialize(); lean_mark_persistent(l_Lean_Parser_Command_initialize); res = l___regBuiltin_Lean_Parser_Command_initialize(lean_io_mk_world()); @@ -72214,6 +77565,23 @@ lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initialize_declRange___c res = l___regBuiltin_Lean_Parser_Command_initialize_declRange(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l_Lean_Parser_Command_initializeKeyword_formatter___closed__1 = _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_formatter___closed__1); +l_Lean_Parser_Command_initializeKeyword_formatter___closed__2 = _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_formatter___closed__2); +l_Lean_Parser_Command_initializeKeyword_formatter___closed__3 = _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_formatter___closed__3); +l_Lean_Parser_Command_initializeKeyword_formatter___closed__4 = _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_formatter___closed__4); +l_Lean_Parser_Command_initializeKeyword_formatter___closed__5 = _init_l_Lean_Parser_Command_initializeKeyword_formatter___closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_formatter___closed__5); +l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_initializeKeyword_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_initialize_formatter___closed__1 = _init_l_Lean_Parser_Command_initialize_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_initialize_formatter___closed__1); l_Lean_Parser_Command_initialize_formatter___closed__2 = _init_l_Lean_Parser_Command_initialize_formatter___closed__2(); @@ -72236,8 +77604,30 @@ l_Lean_Parser_Command_initialize_formatter___closed__10 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_initialize_formatter___closed__10); l_Lean_Parser_Command_initialize_formatter___closed__11 = _init_l_Lean_Parser_Command_initialize_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_initialize_formatter___closed__11); -l_Lean_Parser_Command_initialize_formatter___closed__12 = _init_l_Lean_Parser_Command_initialize_formatter___closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_initialize_formatter___closed__12); +l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initialize_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_initialize_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1); +l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2); +l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__3); +l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__4); +l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_initializeKeyword_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_initialize_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_initialize_parenthesizer___closed__1); l_Lean_Parser_Command_initialize_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__2(); @@ -72260,94 +77650,13 @@ l_Lean_Parser_Command_initialize_parenthesizer___closed__10 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Command_initialize_parenthesizer___closed__10); l_Lean_Parser_Command_initialize_parenthesizer___closed__11 = _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_initialize_parenthesizer___closed__11); -l_Lean_Parser_Command_initialize_parenthesizer___closed__12 = _init_l_Lean_Parser_Command_initialize_parenthesizer___closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_initialize_parenthesizer___closed__12); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__1); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__2); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__3 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__3(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__3); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__4 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__4); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__5); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__6 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__6); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__7 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__7); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__8 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__8); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__9 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__9); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__10 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__10(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__10); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__11 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__11(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__11); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__12 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__12); -l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__13 = _init_l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__13(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___elambda__1___closed__13); -l_Lean_Parser_Command_builtin__initialize___closed__1 = _init_l_Lean_Parser_Command_builtin__initialize___closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__1); -l_Lean_Parser_Command_builtin__initialize___closed__2 = _init_l_Lean_Parser_Command_builtin__initialize___closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__2); -l_Lean_Parser_Command_builtin__initialize___closed__3 = _init_l_Lean_Parser_Command_builtin__initialize___closed__3(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__3); -l_Lean_Parser_Command_builtin__initialize___closed__4 = _init_l_Lean_Parser_Command_builtin__initialize___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__4); -l_Lean_Parser_Command_builtin__initialize___closed__5 = _init_l_Lean_Parser_Command_builtin__initialize___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__5); -l_Lean_Parser_Command_builtin__initialize___closed__6 = _init_l_Lean_Parser_Command_builtin__initialize___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__6); -l_Lean_Parser_Command_builtin__initialize___closed__7 = _init_l_Lean_Parser_Command_builtin__initialize___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__7); -l_Lean_Parser_Command_builtin__initialize___closed__8 = _init_l_Lean_Parser_Command_builtin__initialize___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__8); -l_Lean_Parser_Command_builtin__initialize___closed__9 = _init_l_Lean_Parser_Command_builtin__initialize___closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize___closed__9); -l_Lean_Parser_Command_builtin__initialize = _init_l_Lean_Parser_Command_builtin__initialize(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize); -res = l___regBuiltin_Lean_Parser_Command_builtin__initialize(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__1); -l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__2); -l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__3 = _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__3); -l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__4 = _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__4); -l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__5 = _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__5); -l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__6 = _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__6); -l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__7 = _init_l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange___closed__7); -res = l___regBuiltin_Lean_Parser_Command_builtin__initialize_declRange(lean_io_mk_world()); +l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_initialize_parenthesizer(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Parser_Command_builtin__initialize_formatter___closed__1 = _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_formatter___closed__1); -l_Lean_Parser_Command_builtin__initialize_formatter___closed__2 = _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_formatter___closed__2); -l_Lean_Parser_Command_builtin__initialize_formatter___closed__3 = _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__3(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_formatter___closed__3); -l_Lean_Parser_Command_builtin__initialize_formatter___closed__4 = _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_formatter___closed__4); -l_Lean_Parser_Command_builtin__initialize_formatter___closed__5 = _init_l_Lean_Parser_Command_builtin__initialize_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_formatter___closed__5); -l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__1); -l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__2); -l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__3(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__3); -l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__4); -l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_builtin__initialize_parenthesizer___closed__5); l_Lean_Parser_Command_in___elambda__1___closed__1 = _init_l_Lean_Parser_Command_in___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_in___elambda__1___closed__1); l_Lean_Parser_Command_in___elambda__1___closed__2 = _init_l_Lean_Parser_Command_in___elambda__1___closed__2(); @@ -72404,12 +77713,26 @@ l_Lean_Parser_Command_in_formatter___closed__2 = _init_l_Lean_Parser_Command_in_ lean_mark_persistent(l_Lean_Parser_Command_in_formatter___closed__2); l_Lean_Parser_Command_in_formatter___closed__3 = _init_l_Lean_Parser_Command_in_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_in_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_in_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_in_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_in_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_in_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_in_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_in_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_in_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_in_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_in_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_in_parenthesizer___closed__1); l_Lean_Parser_Command_in_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_in_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_in_parenthesizer___closed__2); l_Lean_Parser_Command_in_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_in_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_in_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_in_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_in_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__1 = _init_l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__1); l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__2 = _init_l_Lean_Parser_Command_genInjectiveTheorems___elambda__1___closed__2(); @@ -72480,6 +77803,13 @@ l_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__3 = _init_l_Lean_ lean_mark_persistent(l_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__3); l_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__4 = _init_l_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__4); +l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1); l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2(); @@ -72488,101 +77818,122 @@ l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__3 = _init_l_L lean_mark_persistent(l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__3); l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_genInjectiveTheorems_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_declModifiersF = _init_l_Lean_Parser_Command_declModifiersF(); lean_mark_persistent(l_Lean_Parser_Command_declModifiersF); l_Lean_Parser_Command_declModifiersT = _init_l_Lean_Parser_Command_declModifiersT(); lean_mark_persistent(l_Lean_Parser_Command_declModifiersT); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__1 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__1); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__2 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__2(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__2); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__3 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__3(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__3); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__4 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__4); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__5 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__5); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__6 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__6); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__7 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__7); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__8 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__8); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__9 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__9(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__9); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__10 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__10(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__10); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__11 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__11(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__11); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__12 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__12(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__12); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__13 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__13(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__13); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__14 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__14); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__15 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__15(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__15); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__16 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__16(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__16); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__17 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__17(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__17); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__18 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__18(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__18); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__19 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__19(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__19); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__20 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__20(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__20); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__21 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__21(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__21); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__22 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__22(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__22); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__23 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__23(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__23); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__24 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__24(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__24); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__25 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__25(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__25); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__26 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__26(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__26); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__27 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__27(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__27); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__28 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__28(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__28); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__29 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__29(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__29); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__30 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__30(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__30); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__31 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__31(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__31); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__32 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__32(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__32); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__33 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__33(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__33); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__34 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__34(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__34); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__35 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__35(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__35); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__36 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__36(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__36); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__37 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__37(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__37); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__38 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__38(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__38); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__39 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__39(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__39); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__40 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__40(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__40); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__41 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__41(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__41); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__42 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__42(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__42); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__43 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__43(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__43); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__44 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__44(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__44); -l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__45 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__45(); -lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493____closed__45); -res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2493_(lean_io_mk_world()); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__1 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__1(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__1); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__2 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__2(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__2); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__3 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__3(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__3); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__4 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__4(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__4); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__5 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__5(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__5); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__6 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__6(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__6); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__7 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__7(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__7); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__8 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__8(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__8); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__9 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__9(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__9); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__10 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__10(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__10); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__11 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__11(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__11); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__12 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__12(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__12); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__13 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__13(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__13); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__14 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__14(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__14); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__15 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__15(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__15); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__16 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__16(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__16); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__17 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__17(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__17); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__18 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__18(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__18); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__19 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__19(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__19); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__20 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__20(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__20); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__21 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__21(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__21); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__22 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__22(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__22); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__23 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__23(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__23); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__24 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__24(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__24); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__25 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__25(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__25); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__26 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__26(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__26); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__27 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__27(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__27); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__28 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__28(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__28); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__29 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__29(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__29); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__30 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__30(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__30); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__31 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__31(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__31); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__32 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__32(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__32); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__33 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__33(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__33); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__34 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__34(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__34); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__35 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__35(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__35); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__36 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__36(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__36); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__37 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__37(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__37); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__38 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__38(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__38); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__39 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__39(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__39); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__40 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__40(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__40); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__41 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__41(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__41); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__42 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__42(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__42); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__43 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__43(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__43); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__44 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__44(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__44); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__45 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__45(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__45); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__46 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__46(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__46); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__47 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__47(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__47); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__48 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__48(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__48); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__49 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__49(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__49); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__50 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__50(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__50); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__51 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__51(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__51); +l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__52 = _init_l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__52(); +lean_mark_persistent(l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474____closed__52); +res = l_Lean_Parser_Command_initFn____x40_Lean_Parser_Command___hyg_2474_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Parser_Term_open___elambda__1___closed__1 = _init_l_Lean_Parser_Term_open___elambda__1___closed__1(); @@ -72661,6 +78012,13 @@ l_Lean_Parser_Term_open_formatter___closed__5 = _init_l_Lean_Parser_Term_open_fo lean_mark_persistent(l_Lean_Parser_Term_open_formatter___closed__5); l_Lean_Parser_Term_open_formatter___closed__6 = _init_l_Lean_Parser_Term_open_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_open_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_open_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_open_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_open_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_open_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_open_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_open_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_open_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_open_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_open_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_open_parenthesizer___closed__1); l_Lean_Parser_Term_open_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_open_parenthesizer___closed__2(); @@ -72673,6 +78031,13 @@ l_Lean_Parser_Term_open_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_ope lean_mark_persistent(l_Lean_Parser_Term_open_parenthesizer___closed__5); l_Lean_Parser_Term_open_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_open_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_open_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_open_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_open_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_set__option___elambda__1___closed__1 = _init_l_Lean_Parser_Term_set__option___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_set__option___elambda__1___closed__1); l_Lean_Parser_Term_set__option___elambda__1___closed__2 = _init_l_Lean_Parser_Term_set__option___elambda__1___closed__2(); @@ -72753,6 +78118,13 @@ l_Lean_Parser_Term_set__option_formatter___closed__6 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_set__option_formatter___closed__6); l_Lean_Parser_Term_set__option_formatter___closed__7 = _init_l_Lean_Parser_Term_set__option_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_set__option_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_set__option_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_set__option_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_set__option_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_set__option_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_set__option_parenthesizer___closed__1); l_Lean_Parser_Term_set__option_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_set__option_parenthesizer___closed__2(); @@ -72767,6 +78139,13 @@ l_Lean_Parser_Term_set__option_parenthesizer___closed__6 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_set__option_parenthesizer___closed__6); l_Lean_Parser_Term_set__option_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_set__option_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_set__option_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_set__option_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_open___elambda__1___closed__1 = _init_l_Lean_Parser_Tactic_open___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_open___elambda__1___closed__1); l_Lean_Parser_Tactic_open___elambda__1___closed__2 = _init_l_Lean_Parser_Tactic_open___elambda__1___closed__2(); @@ -72847,6 +78226,13 @@ l_Lean_Parser_Tactic_open_formatter___closed__5 = _init_l_Lean_Parser_Tactic_ope lean_mark_persistent(l_Lean_Parser_Tactic_open_formatter___closed__5); l_Lean_Parser_Tactic_open_formatter___closed__6 = _init_l_Lean_Parser_Tactic_open_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Tactic_open_formatter___closed__6); +l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_open_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_open_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_open_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_open_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_open_parenthesizer___closed__1); l_Lean_Parser_Tactic_open_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_open_parenthesizer___closed__2(); @@ -72859,6 +78245,13 @@ l_Lean_Parser_Tactic_open_parenthesizer___closed__5 = _init_l_Lean_Parser_Tactic lean_mark_persistent(l_Lean_Parser_Tactic_open_parenthesizer___closed__5); l_Lean_Parser_Tactic_open_parenthesizer___closed__6 = _init_l_Lean_Parser_Tactic_open_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Tactic_open_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_open_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_set__option___elambda__1___closed__1 = _init_l_Lean_Parser_Tactic_set__option___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_set__option___elambda__1___closed__1); l_Lean_Parser_Tactic_set__option___elambda__1___closed__2 = _init_l_Lean_Parser_Tactic_set__option___elambda__1___closed__2(); @@ -72931,6 +78324,13 @@ l_Lean_Parser_Tactic_set__option_formatter___closed__5 = _init_l_Lean_Parser_Tac lean_mark_persistent(l_Lean_Parser_Tactic_set__option_formatter___closed__5); l_Lean_Parser_Tactic_set__option_formatter___closed__6 = _init_l_Lean_Parser_Tactic_set__option_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Tactic_set__option_formatter___closed__6); +l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_set__option_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_set__option_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_set__option_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_set__option_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_set__option_parenthesizer___closed__1); l_Lean_Parser_Tactic_set__option_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_set__option_parenthesizer___closed__2(); @@ -72943,6 +78343,13 @@ l_Lean_Parser_Tactic_set__option_parenthesizer___closed__5 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Tactic_set__option_parenthesizer___closed__5); l_Lean_Parser_Tactic_set__option_parenthesizer___closed__6 = _init_l_Lean_Parser_Tactic_set__option_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Tactic_set__option_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_set__option_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Parser/Do.c b/stage0/stdlib/Lean/Parser/Do.c index 4c6521284044..211484a8370f 100644 --- a/stage0/stdlib/Lean/Parser/Do.c +++ b/stage0/stdlib/Lean/Parser/Do.c @@ -20,6 +20,8 @@ static lean_object* l_Lean_Parser_Term_doLetElse___closed__10; static lean_object* l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_do_declRange___closed__6; static lean_object* l_Lean_Parser_Term_doExpr___closed__1; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__2; @@ -47,6 +49,7 @@ static lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__22; LEAN_EXPORT lean_object* l_Lean_Parser_doElemParser(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doDbgTrace_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doUnless_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doUnless(lean_object*); @@ -65,6 +68,7 @@ static lean_object* l_Lean_Parser_Term_doFinally_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doIf___closed__12; static lean_object* l_Lean_Parser_Term_doLet_formatter___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_declRange___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_declRange___closed__5; lean_object* l_Lean_Parser_tokenAntiquotFn(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__5; @@ -82,6 +86,7 @@ static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda static lean_object* l_Lean_Parser_Term_doIfProp___closed__1; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__21; lean_object* l_Lean_Parser_andthenInfo(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_doDbgTrace___closed__1; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__12; @@ -109,6 +114,7 @@ static lean_object* l_Lean_Parser_Term_doForDecl_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_do_parenthesizer(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doBreak___closed__7; static lean_object* l_Lean_Parser_Term_doTry_formatter___closed__1; @@ -127,8 +133,8 @@ static lean_object* l_Lean_Parser_Term_doCatch___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIf_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doSeqBracketed___closed__9; static lean_object* l_Lean_Parser_Term_doIfLet___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_doIfLet_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_doUnless___closed__6; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__20; static lean_object* l_Lean_Parser_Term_do___elambda__1___closed__8; @@ -173,13 +179,17 @@ static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_doIfLet___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doCatch___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doForDecl_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doNested_declRange___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doLet_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doExpr___closed__4; static lean_object* l_Lean_Parser_Term_doTry___closed__9; static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__1; static lean_object* l_Lean_Parser_Term_doContinue___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetArrow___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doContinue_parenthesizer___closed__3; @@ -220,6 +230,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetElse_parenthesizer(lean_object* lean_object* l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doExpr_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doFinally___closed__3; static lean_object* l_Lean_Parser_Term_doDbgTrace_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doMatchAlts; @@ -239,6 +250,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_declRange___closed static lean_object* l_Lean_Parser_Term_doForDecl___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doForDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doExpr___closed__8; static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1___closed__5; @@ -266,12 +278,15 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_do_declRange___closed__5; static lean_object* l_Lean_Parser_Term_doForDecl___closed__5; static lean_object* l_Lean_Parser_Term_termUnless_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1___closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doSeqItem_formatter___closed__6; static lean_object* l_Lean_Parser_Term_doIfLetPure_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doFinally___closed__5; static lean_object* l_Lean_Parser_Term_doIfProp_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doUnless___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_doMatch___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__1; extern lean_object* l_Lean_Parser_pushNone; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doBreak(lean_object*); static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__4; @@ -282,7 +297,6 @@ static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__25; static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__6; static lean_object* l_Lean_Parser_Term_doCatch___closed__6; -static lean_object* l_Lean_Parser_Term_doReassign_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassignArrow; static lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_declRange___closed__1; static lean_object* l_Lean_Parser_Term_doSeqBracketed___closed__8; @@ -290,7 +304,9 @@ static lean_object* l_Lean_Parser_Term_doUnless_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doHave_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_doAssert_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__33; +static lean_object* l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_declRange___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_declRange___closed__4; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__4; @@ -301,11 +317,13 @@ static lean_object* l_Lean_Parser_Term_doIfLet___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__6; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__16; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__22; static lean_object* l_Lean_Parser_Term_doFinally___elambda__1___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doReassign_parenthesizer___closed__6; -static lean_object* l_Lean_Parser_Term_doIfCond_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIdDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_declRange___closed__2; @@ -321,6 +339,7 @@ static lean_object* l_Lean_Parser_Term_termUnless___closed__3; static lean_object* l_Lean_Parser_Term_doIdDecl_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__3; lean_object* l_id___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doBreak___elambda__1(lean_object*, lean_object*); @@ -330,17 +349,20 @@ static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_do_declRange___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doCatch_formatter___closed__10; lean_object* l_Lean_Parser_ParserState_mkNode(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doUnless_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doFor___closed__1; static lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doHave___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_declRange___closed__7; -static lean_object* l_Lean_Parser_Term_doIfCond_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__1; extern lean_object* l_Lean_Parser_darrow; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doReassign___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doElem_quot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -357,6 +379,7 @@ static lean_object* l_Lean_Parser_Term_doIfLet_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_declRange___closed__7; static lean_object* l_Lean_Parser_Term_doLet_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doCatch_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_termReturn___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_termUnless___closed__5; @@ -374,6 +397,7 @@ static lean_object* l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_doIdDecl___closed__5; lean_object* l_Lean_Parser_pushNone___elambda__1___boxed(lean_object*); static lean_object* l_Lean_Parser_Term_doIdDecl___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__2; lean_object* l_Lean_Parser_notFollowedByFn(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfLet; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doBreak_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -385,20 +409,23 @@ static lean_object* l_Lean_Parser_Term_termTry___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_doElemParser_formatter(lean_object*); lean_object* l_Lean_Parser_orelseFn(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_registerBuiltinDynamicParserAttribute(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__2; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__28; static lean_object* l_Lean_Parser_Term_doIfLet___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__14; -static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Term_doHave___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__2; static lean_object* l_Lean_Parser_Term_doElem_quot_formatter___closed__3; -static lean_object* l_Lean_Parser_Term_doFor_formatter___closed__8; static lean_object* l_Lean_Parser_Term_doCatchMatch___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doTry_formatter___closed__8; static lean_object* l_Lean_Parser_Term_termReturn___closed__4; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Term_do_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIdDecl___closed__3; @@ -407,14 +434,18 @@ static lean_object* l_Lean_Parser_Term_doSeqBracketed_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doFor___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassignArrow___elambda__1___lambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfCond___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doReassignArrow___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doElem_quot___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfProp_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfLet___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassignArrow_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doHave___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_doReturn___closed__8; lean_object* l_Lean_Parser_addBuiltinParser(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); @@ -435,6 +466,7 @@ static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_doIdDecl___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doBreak___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doReturn_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doNested_formatter(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIdDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__22; @@ -444,12 +476,12 @@ static lean_object* l_Lean_Parser_Term_termUnless___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_declRange___closed__4; static lean_object* l_Lean_Parser_Term_doIfProp___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__1; static lean_object* l_Lean_Parser_Term_termFor___closed__6; static lean_object* l_Lean_Parser_Term_doFinally___closed__6; static lean_object* l_Lean_Parser_Term_doIf___closed__1; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__18; -static lean_object* l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doCatchMatch___closed__3; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__13; @@ -458,6 +490,7 @@ static lean_object* l_Lean_Parser_Term_doAssert___closed__1; lean_object* l_Lean_Parser_unicodeSymbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__2; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doSeqItem_formatter___closed__5; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__11; @@ -472,14 +505,15 @@ static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_elseIf_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_termTry___closed__6; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__46; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_termFor_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doElem_quot; static lean_object* l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doUnless_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_elseIf___closed__7; static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__5; -static lean_object* l_Lean_Parser_Term_doSeq_formatter___closed__3; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doReassign___closed__2; static lean_object* l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__9; @@ -507,6 +541,8 @@ static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_doSeqBracketed___closed__3; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doSeqBracketed_formatter___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_darrow_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -514,6 +550,7 @@ lean_object* l_Lean_Parser_mkAntiquot_formatter___boxed(lean_object*, lean_objec static lean_object* l_Lean_Parser_Term_doHave_formatter___closed__4; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__29; lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_doDbgTrace___closed__2; static lean_object* l_Lean_Parser_Term_doAssert___closed__8; @@ -532,14 +569,18 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassign; lean_object* l_Lean_Parser_checkColGeFn___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Term_haveDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___closed__5; +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doNested_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doIfLet_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doIfLet___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__19; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doTry_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__21; +static lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__2; lean_object* l_Lean_Parser_many_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__2; static lean_object* l_Lean_Parser_Term_do___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__8; @@ -557,7 +598,6 @@ static lean_object* l_Lean_Parser_Term_doReturn_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doElem_quot_formatter___closed__6; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_declRange(lean_object*); -static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_doUnless___elambda__1___closed__7; @@ -565,10 +605,10 @@ lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, le static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__18; -static lean_object* l_Lean_Parser_Term_doTry_formatter___closed__11; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__15; static lean_object* l_Lean_Parser_Term_doIf___closed__2; static lean_object* l_Lean_Parser_Term_doReassign___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Term_doSeq_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doIfLetPure___closed__4; @@ -577,6 +617,7 @@ static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_liftMethod___closed__5; static lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_elseIf___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIf; lean_object* l_Lean_Parser_checkPrecFn(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_atomic_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -585,6 +626,7 @@ lean_object* l_Lean_Parser_Term_motive_parenthesizer(lean_object*, lean_object*, static lean_object* l_Lean_Parser_Term_doIfProp___closed__4; lean_object* l_Lean_PrettyPrinter_Formatter_checkColGt_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfProp___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__22; static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_declRange___closed__7; @@ -614,15 +656,19 @@ static lean_object* l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_declRange___closed__6; static lean_object* l_Lean_Parser_Term_doSeqIndent___closed__1; static lean_object* l_Lean_Parser_Term_doReturn_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doTry_formatter___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_declRange(lean_object*); lean_object* l_Lean_Parser_Term_matchAlts_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLetArrow___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doMatchAlts_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__19; static lean_object* l_Lean_Parser_Term_doIf___closed__5; static lean_object* l_Lean_Parser_Term_doHave___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer(lean_object*); lean_object* l_Lean_Parser_Term_letRecDecls_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfProp___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doContinue_formatter___closed__3; @@ -630,6 +676,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassignArrow___elambda__1(lean_ob static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__11; lean_object* l_Lean_Parser_registerAliasCore___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIf___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doIdDecl___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Term_termTry___closed__3; @@ -646,12 +693,14 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_declRange___closed__2; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doSeq___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassignArrow_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_declRange___closed__6; -static lean_object* l_Lean_Parser_Term_doLetArrow_formatter___closed__7; static lean_object* l_Lean_Parser_Term_doIfLetPure___closed__1; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__27; static lean_object* l_Lean_Parser_Term_doUnless___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLet_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termFor___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doPatDecl_formatter___closed__5; @@ -667,8 +716,10 @@ static lean_object* l_Lean_Parser_Term_doBreak___elambda__1___closed__6; uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__22; static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__11; +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l_Lean_Parser_Term_doIfLetPure_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_liftMethod_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doAssert_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetRec___elambda__1(lean_object*, lean_object*); @@ -689,7 +740,6 @@ static lean_object* l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doReassign_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doIf___closed__8; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__16; -static lean_object* l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_doLetElse_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_do___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfLetBind___elambda__1(lean_object*, lean_object*); @@ -700,8 +750,12 @@ static lean_object* l_Lean_Parser_Term_doReturn___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_declRange___closed__6; static lean_object* l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__1; static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__14; static lean_object* l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_declRange___closed__4; static lean_object* l_Lean_Parser_Term_doSeq___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doForDecl___elambda__1(lean_object*, lean_object*); @@ -712,9 +766,11 @@ static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Do___hyg_19____close static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_termUnless_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__24; static lean_object* l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termTry_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_liftMethod___closed__7; static lean_object* l_Lean_Parser_Term_doLetElse_formatter___closed__5; static lean_object* l_Lean_Parser_Term_doSeqIndent_formatter___closed__2; @@ -729,6 +785,7 @@ static lean_object* l_Lean_Parser_Term_elseIf_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doDbgTrace___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfLetBind_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_do___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLet_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doUnless___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_declRange___closed__5; static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__5; @@ -740,6 +797,7 @@ static lean_object* l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doUnless_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_doContinue___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doCatch_formatter___closed__12; extern lean_object* l_Lean_Parser_Term_optType; @@ -750,11 +808,15 @@ static lean_object* l_Lean_Parser_Term_doFor_formatter___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIdDecl___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse___closed__5; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doTry_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_elseIf___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_doFor___closed__4; static lean_object* l_Lean_Parser_Term_doLetRec_formatter___closed__7; static lean_object* l_Lean_Parser_Term_termReturn_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termReturn(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFor(lean_object*); @@ -762,12 +824,15 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_elseIf; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doFor_parenthesizer___closed__7; lean_object* l_Lean_Parser_nodeInfo(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doReassign___elambda__1___closed__5; lean_object* l_Lean_Parser_darrow_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doReturn_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_doNested_parenthesizer___closed__1; @@ -778,6 +843,8 @@ static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed_ static lean_object* l_Lean_Parser_Term_doSeq___closed__1; static lean_object* l_Lean_Parser_Term_doSeqIndent___closed__2; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doIf___closed__7; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__42; static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_declRange___closed__6; @@ -797,11 +864,13 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_declRange___closed__ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doNested; static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__20; static lean_object* l_Lean_Parser_Term_doReturn___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_termUnless_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_termReturn___elambda__1___closed__1; extern lean_object* l_Lean_Parser_Term_letDecl; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__9; static lean_object* l_Lean_Parser_Term_doHave_formatter___closed__2; @@ -816,6 +885,7 @@ static lean_object* l_Lean_Parser_Term_doLet_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_doBreak___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_declRange___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termTry_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__5; @@ -826,6 +896,7 @@ static lean_object* l_Lean_Parser_Term_doSeq___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doCatch___closed__7; static lean_object* l_Lean_Parser_Term_doUnless___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doCatch_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doTry___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_declRange___closed__1; static lean_object* l_Lean_Parser_Term_doBreak_parenthesizer___closed__3; @@ -842,15 +913,19 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIf___elambda__1___lambda__1___boxe static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doExpr_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_elseIf___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doContinue___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termReturn___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIf_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doLetArrow___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___lambda__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__13; static lean_object* l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__4; @@ -869,15 +944,18 @@ static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetArrow; static lean_object* l_Lean_Parser_Term_termUnless___elambda__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doExpr_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doAssert_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doHave_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termTry; static lean_object* l___regBuiltin_Lean_Parser_Term_doHave_declRange___closed__4; static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termFor; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doAssert_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetArrow___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__3; @@ -908,6 +986,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIdDecl_parenthesizer(lean_object*, static lean_object* l_Lean_Parser_Term_doHave_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_doIfProp_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doNested_declRange___closed__1; static lean_object* l_Lean_Parser_Term_doSeqIndent___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_declRange___closed__2; @@ -918,6 +997,7 @@ static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__1; lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_node_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doCatchMatch___closed__6; @@ -926,6 +1006,9 @@ static lean_object* l_Lean_Parser_Term_termUnless___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__3; lean_object* l_Lean_PrettyPrinter_Parenthesizer_interpolatedStr_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__15; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doUnless___closed__4; @@ -949,12 +1032,14 @@ static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__19; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_declRange___closed__5; static lean_object* l_Lean_Parser_Term_doContinue___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_doIfProp___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doBreak___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_doFor_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doReassignArrow_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doLetRec_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetRec_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doForDecl_formatter___closed__8; static lean_object* l_Lean_Parser_Term_doCatch_formatter___closed__8; static lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1___closed__12; @@ -964,6 +1049,7 @@ static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doUnless___elambda__1___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_doFor_declRange___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_termFor_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__3; @@ -979,9 +1065,10 @@ static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Do___hyg_5____closed static lean_object* l_Lean_Parser_Term_termBeforeDo___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doLetRec_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_doSeqIndent___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doFor_formatter___closed__5; static lean_object* l_Lean_Parser_Term_doForDecl___closed__10; -static lean_object* l_Lean_Parser_Term_doSeq_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFor_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__16; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__7; @@ -1006,6 +1093,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___lambda__1 static lean_object* l___regBuiltin_Lean_Parser_Term_do_declRange___closed__4; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__32; static lean_object* l___regBuiltin_Lean_Parser_Term_doFor_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doLet_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doSeq___closed__2; static lean_object* l_Lean_Parser_Term_doDbgTrace_formatter___closed__4; @@ -1013,9 +1102,12 @@ static lean_object* l_Lean_Parser_Term_doLetRec___closed__3; static lean_object* l_Lean_Parser_Term_doSeq___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_doExpr_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__2; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__49; static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_declRange___closed__7; static lean_object* l_Lean_Parser_Term_doMatch___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__20; @@ -1030,11 +1122,15 @@ static lean_object* l_Lean_Parser_Term_doPatDecl_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doReturn_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_termTry___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doNested___closed__4; static lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doTry_formatter___closed__6; static lean_object* l_Lean_Parser_Term_doFinally___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doReturn_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_doHave_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_doCatch_formatter___closed__11; @@ -1047,6 +1143,7 @@ static lean_object* l_Lean_Parser_Term_doReturn___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_declRange___closed__5; static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__1; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__13; static lean_object* l___regBuiltin_Lean_Parser_Term_doHave_declRange___closed__1; @@ -1056,6 +1153,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_declRange___close static lean_object* l_Lean_Parser_Term_doIfCond___closed__2; static lean_object* l_Lean_Parser_Term_doForDecl_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_declRange___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doSeqBracketed_formatter___closed__4; static lean_object* l_Lean_Parser_Term_leftArrow___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__20; @@ -1067,6 +1165,7 @@ static lean_object* l_Lean_Parser_Term_doLetRec___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_termUnless___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termUnless___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_doMatchAlts_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doTry_declRange___closed__5; @@ -1085,6 +1184,7 @@ static lean_object* l_Lean_Parser_Term_doLetArrow___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfLetBind_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_doContinue___closed__6; +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; static lean_object* l_Lean_Parser_Term_doIfLetBind___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFor_declRange(lean_object*); uint32_t lean_string_utf8_get(lean_object*, lean_object*); @@ -1096,20 +1196,27 @@ static lean_object* l_Lean_Parser_Term_doIfLetBind_formatter___closed__2; lean_object* l_Lean_Parser_Term_letPatDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doMatch___closed__1; lean_object* l_Lean_Parser_interpolatedStr(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doPatDecl_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termFor_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doNested___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_do___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doReassign_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_doFor___closed__5; static lean_object* l_Lean_Parser_Term_leftArrow___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doReturn_formatter___closed__6; static lean_object* l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doBreak___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doExpr_formatter___closed__8; @@ -1132,8 +1239,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIdDecl; static lean_object* l_Lean_Parser_Term_doLetElse_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_doFor_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_doNested_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doHave_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doBreak___elambda__1___closed__9; -static lean_object* l_Lean_Parser_Term_doSeq_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doHave_declRange___closed__3; static lean_object* l_Lean_Parser_Term_doBreak___elambda__1___closed__8; @@ -1142,8 +1249,10 @@ static lean_object* l_Lean_Parser_Term_liftMethod___closed__1; static lean_object* l_Lean_Parser_Term_doPatDecl___closed__5; static lean_object* l_Lean_Parser_Term_doCatchMatch___closed__1; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__25; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termFor_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__13; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__21; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_doCatch_formatter___closed__1; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); @@ -1153,6 +1262,7 @@ static lean_object* l_Lean_Parser_Term_doCatch___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Term_doLet_declRange___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doBreak___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doFinally_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doForDecl_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_doSeqItem_formatter___closed__4; @@ -1160,12 +1270,16 @@ lean_object* l_Lean_PrettyPrinter_Parenthesizer_pushNone_parenthesizer___boxed(l static lean_object* l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_declRange___closed__7; extern lean_object* l_Lean_instInhabitedSyntax; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_declRange___closed__5; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__17; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doIdDecl_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReturn___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__1; static lean_object* l_Lean_Parser_Term_termFor___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_elseIf___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doContinue___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__17; @@ -1198,21 +1312,24 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_doFor_declRange___closed__7; static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doUnless_formatter___closed__5; static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__1; static lean_object* l_Lean_Parser_Term_leftArrow___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_liftMethod___closed__3; static lean_object* l_Lean_Parser_Term_termFor___closed__2; static lean_object* l_Lean_Parser_Term_termFor___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_declRange___closed__5; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__20; static lean_object* l_Lean_Parser_Term_doCatchMatch___closed__2; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__8; lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doFinally___elambda__1___closed__1; -static lean_object* l_Lean_Parser_Term_doIfCond_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doIfLetPure___closed__3; static lean_object* l_Lean_Parser_Term_doForDecl_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__1; lean_object* l_Lean_Parser_sepBy1_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_declRange___closed__1; @@ -1220,23 +1337,27 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termFor(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termTry(lean_object*); static lean_object* l_Lean_Parser_Term_doMatch___closed__8; static lean_object* l_Lean_Parser_Term_doIfProp_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doAssert___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doReturn___closed__5; static lean_object* l_Lean_Parser_Term_doLet_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_doHave_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doLetArrow_formatter___closed__3; -static lean_object* l_Lean_Parser_Term_doTry_formatter___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIf___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_termUnless___closed__4; static lean_object* l_Lean_Parser_Term_doReturn___closed__3; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__26; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfLetPure___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__15; +static lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___closed__1; lean_object* l_Lean_Parser_registerAlias(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_doUnless___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__6; @@ -1252,13 +1373,15 @@ static lean_object* l_Lean_Parser_Term_doCatchMatch___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_declRange___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_checkLineEq_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doLet___closed__5; lean_object* l_Lean_Parser_Term_binderIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__2; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_doBreak___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfProp___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_doIfLet_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__2; static lean_object* l_Lean_Parser_Term_termUnless___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_declRange___closed__2; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__5; @@ -1282,31 +1405,38 @@ static lean_object* l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken_formatter(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doReassign_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doSeqItem_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doReassign_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termTry_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__21; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__38; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doHave___closed__2; static lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___closed__6; static lean_object* l_Lean_Parser_Term_doIfProp_parenthesizer___closed__1; lean_object* l_Lean_Parser_many1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_doIdDecl_formatter___closed__7; static lean_object* l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doLetArrow_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReturn___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doFinally___closed__8; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__19; static lean_object* l_Lean_Parser_Term_doFinally___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doContinue___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doFor_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__16; static lean_object* l_Lean_Parser_Term_doTry___closed__7; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_leftArrow___elambda__1___closed__2; lean_object* l_Lean_Parser_checkLineEqFn___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfProp___elambda__1___closed__6; @@ -1324,11 +1454,11 @@ static lean_object* l_Lean_Parser_Term_doExpr_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_declRange___closed__7; static lean_object* l_Lean_Parser_Term_doIdDecl___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReturn; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doUnless_formatter___closed__3; lean_object* l_Lean_Parser_Term_haveDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_elseIf___closed__1; -static lean_object* l_Lean_Parser_Term_doSeq_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termBeforeDo; lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1347,6 +1477,7 @@ static lean_object* l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__23; static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_leftArrow___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_doLet_parenthesizer___closed__6; @@ -1358,6 +1489,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_declRange___closed__ static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__16; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_doLetElse_formatter___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doTry_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__41; @@ -1370,6 +1502,7 @@ static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda static lean_object* l_Lean_Parser_Term_doPatDecl_formatter___closed__7; static lean_object* l_Lean_Parser_Term_doLetElse___closed__13; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doFor_parenthesizer___closed__5; lean_object* l_Lean_Parser_Term_letPatDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1396,6 +1529,7 @@ static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_doFor_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doAssert_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFinally_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Term_leftArrow; static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__8; @@ -1405,6 +1539,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_declRange___close LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_declRange(lean_object*); lean_object* l_Lean_Parser_Term_ident___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doReassignArrow___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_declRange___closed__7; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_doHave___closed__8; @@ -1420,6 +1555,7 @@ static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__17; static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_declRange___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_declRange___closed__6; static lean_object* l_Lean_Parser_Term_doIfLet___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_do_declRange(lean_object*); lean_object* l_Lean_Parser_Term_optType_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1427,18 +1563,24 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqIndent; static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doAssert___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_liftMethod_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__18; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__20; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_elseIf___closed__2; static lean_object* l_Lean_Parser_Term_do___closed__7; static lean_object* l_Lean_Parser_Term_leftArrow___elambda__1___closed__3; extern lean_object* l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_declRange___closed__4; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__19; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doSeqBracketed___closed__6; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__11; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__18; static lean_object* l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__3; @@ -1457,6 +1599,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___lambda__1(l LEAN_EXPORT lean_object* l_Lean_Parser_Term_doBreak; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termTry___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doTry_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doAssert_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doMatch___closed__13; static lean_object* l_Lean_Parser_Term_doHave___closed__4; @@ -1465,6 +1608,7 @@ static lean_object* l_Lean_Parser_Term_doPatDecl___closed__9; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__20; LEAN_EXPORT lean_object* l_Lean_Parser_Term_leftArrow_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_doHave___elambda__1___closed__11; @@ -1477,6 +1621,7 @@ static lean_object* l_Lean_Parser_Term_doExpr_formatter___closed__5; static lean_object* l_Lean_Parser_Term_doLetElse___closed__8; static lean_object* l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_declRange___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_do_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_elseIf___closed__4; static lean_object* l_Lean_Parser_Term_doLetRec___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_declRange___closed__5; @@ -1486,7 +1631,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_declRange___close static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doTry_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_termReturn_formatter___closed__2; -static lean_object* l_Lean_Parser_Term_doSeqBracketed_formatter___closed__10; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_doNested___closed__5; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___closed__4; @@ -1500,6 +1644,7 @@ static lean_object* l_Lean_Parser_Term_doBreak___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_doBreak___closed__6; static lean_object* l_Lean_Parser_Term_doLetElse_formatter___closed__6; static lean_object* l_Lean_Parser_Term_doSeqBracketed___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse___closed__1; static lean_object* l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__9; @@ -1527,6 +1672,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_declRange___close lean_object* l_Lean_PrettyPrinter_Formatter_incQuotDepth_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doSeq___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReturn_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doMatch___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Term_termUnless; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__31; @@ -1535,10 +1681,10 @@ static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__19; static lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_declRange___closed__2; static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doElem_quot_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doIfLet_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doIfLet_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doIfLetBind___closed__6; @@ -1572,6 +1718,7 @@ static lean_object* l_Lean_Parser_Term_doIfLet___closed__7; lean_object* l_Lean_Parser_orelseFnCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); extern lean_object* l_Lean_Parser_epsilonInfo; static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doMatch(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIf_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doNested___elambda__1___closed__6; @@ -1583,15 +1730,18 @@ static lean_object* l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_declRange___closed__2; static lean_object* l_Lean_Parser_Term_doLetElse___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetElse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__11; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withForbidden_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_declRange___closed__3; static lean_object* l_Lean_Parser_Term_doReassign___elambda__1___closed__4; lean_object* l_Lean_Parser_Term_letDecl___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doCatch_formatter___closed__6; static lean_object* l_Lean_Parser_Term_doTry___closed__2; static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__2; @@ -1615,6 +1765,7 @@ static lean_object* l_Lean_Parser_Term_doIfCond___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doBreak_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doCatch_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_leftArrow___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_doIfProp___closed__2; static lean_object* l_Lean_Parser_Term_doTry_formatter___closed__5; @@ -1624,6 +1775,7 @@ static lean_object* l_Lean_Parser_Term_doSeqBracketed_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__35; static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_declRange___closed__2; static lean_object* l_Lean_Parser_Term_doForDecl___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doReassign_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doFinally___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doContinue___closed__7; @@ -1637,21 +1789,24 @@ static lean_object* l_Lean_Parser_Term_doSeqItem___closed__2; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doForDecl_formatter___closed__9; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__36; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfProp_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doDbgTrace___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow(lean_object*); static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__18; -static lean_object* l_Lean_Parser_Term_doIfCond_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doElem_quot___closed__4; static lean_object* l_Lean_Parser_Term_doAssert___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_doHave___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doReturn_formatter___closed__7; static lean_object* l_Lean_Parser_Term_doFor_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_declRange___closed__6; static lean_object* l_Lean_Parser_Term_doExpr_formatter___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doNested_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_declRange___closed__7; static lean_object* l_Lean_Parser_Term_doReassignArrow___closed__2; static lean_object* l_Lean_Parser_Term_doIfLet___elambda__1___closed__5; @@ -1666,6 +1821,7 @@ static lean_object* l_Lean_Parser_Term_doContinue___elambda__1___closed__5; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_declRange___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doUnless___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__35; lean_object* l_Lean_Parser_Term_optType_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1678,6 +1834,7 @@ static lean_object* l_Lean_Parser_Term_doUnless_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___closed__2; static lean_object* l_Lean_Parser_Term_doReassign_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doNested___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doFor___elambda__1(lean_object*, lean_object*); @@ -1694,21 +1851,25 @@ static lean_object* l_Lean_Parser_Term_doSeqBracketed_formatter___closed__5; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doHave___closed__3; static lean_object* l_Lean_Parser_Term_doLetElse_formatter___closed__4; static lean_object* l_Lean_Parser_Term_termUnless___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doExpr_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_do_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doTry___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__21; static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_declRange___closed__2; static lean_object* l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_doElem_quot___closed__6; lean_object* l_Lean_ppSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfLet___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doContinue___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfCond_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doTry; -static lean_object* l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_doLetElse_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_declRange___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_do_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1724,6 +1885,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeq_parenthesizer(lean_object*, le static lean_object* l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doPatDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassign_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_darrow___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__14; @@ -1738,20 +1900,23 @@ static lean_object* l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doPatDecl___closed__3; static lean_object* l_Lean_Parser_Term_doUnless_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__28; +static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__1; static lean_object* l_Lean_Parser_Term_termReturn___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doForDecl_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_doLetArrow___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doUnless_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doBreak_formatter___closed__2; -static lean_object* l_Lean_Parser_Term_doIfLet_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_doIfCond_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doElem_quot___closed__9; static lean_object* l_Lean_Parser_Term_doLetRec_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__7; static lean_object* l_Lean_Parser_Term_doCatch_parenthesizer___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__17; static lean_object* l_Lean_Parser_Term_doForDecl___closed__1; static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__2; static lean_object* l_Lean_Parser_Term_termReturn___closed__3; static lean_object* l_Lean_Parser_Term_doHave___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doHave___closed__5; @@ -1764,8 +1929,10 @@ static lean_object* l_Lean_Parser_Term_doContinue___elambda__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doAssert(lean_object*); static lean_object* l_Lean_Parser_Term_doLet___closed__4; static lean_object* l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2; lean_object* l_Lean_Parser_unicodeSymbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doUnless; static lean_object* l_Lean_Parser_Term_doIfLet_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__3; @@ -1788,11 +1955,13 @@ static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__21; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_doCatchMatch_formatter___closed__3; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Term_doIfLet_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doHave___closed__6; extern lean_object* l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; extern lean_object* l_Lean_Parser_Term_matchDiscr; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__2; static lean_object* l_Lean_Parser_Term_termFor___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_doIfLetBind___closed__2; @@ -1812,6 +1981,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_declRange(lean static lean_object* l_Lean_Parser_Term_doTry_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_termFor___closed__5; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_declRange___closed__1; lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1(lean_object*, lean_object*); @@ -1831,14 +2001,18 @@ static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__2; lean_object* l_Lean_Parser_mkAntiquot(lean_object*, lean_object*, uint8_t, uint8_t); static lean_object* l_Lean_Parser_Term_doNested___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doForDecl_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doIfLet___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIdDecl___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_elseIf_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_doIfProp___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfProp_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doForDecl_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_doLet_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken_parenthesizer___rarg(lean_object*); @@ -1848,12 +2022,17 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_declRange___clos static lean_object* l_Lean_Parser_Term_doElem_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doForDecl___closed__6; static lean_object* l_Lean_Parser_Term_do_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_termFor___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_doElemParser_formatter___boxed(lean_object*); static lean_object* l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doLetRec_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doLetElse_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__24; @@ -1862,7 +2041,7 @@ static lean_object* l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_doLet_declRange___closed__6; lean_object* l_Lean_Parser_many_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doMatch___closed__11; -static lean_object* l_Lean_Parser_Term_doTry_formatter___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doSeqIndent_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doContinue_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___closed__5; @@ -1871,6 +2050,7 @@ static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_doForDecl_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_doLet_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doFor_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLet_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doNested___elambda__1___closed__3; @@ -1878,12 +2058,15 @@ static lean_object* l_Lean_Parser_Term_doFor___closed__7; lean_object* l_Lean_PrettyPrinter_Formatter_interpolatedStr_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_liftMethod; static lean_object* l_Lean_Parser_Term_doLetRec_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doLetRec___closed__9; static lean_object* l_Lean_Parser_Term_doFor___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__21; static lean_object* l_Lean_Parser_Term_doContinue_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doIfLet_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_liftMethod_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doNested_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1901,6 +2084,7 @@ lean_object* l_Lean_PrettyPrinter_Parenthesizer_notFollowedBy_parenthesizer___bo static lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_declRange___closed__6; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_doIdDecl___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___closed__1; static lean_object* l_Lean_Parser_Term_elseIf_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_doFinally_formatter___closed__2; @@ -1914,6 +2098,7 @@ static lean_object* l_Lean_Parser_Term_termReturn___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doFinally_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_do___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doReturn___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doReassign___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__9; @@ -1942,9 +2127,12 @@ static lean_object* l_Lean_Parser_Term_doIfLetBind___closed__4; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__1; static lean_object* l_Lean_Parser_Term_termTry_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doTry_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_doPatDecl___closed__4; static lean_object* l_Lean_Parser_Term_doLetArrow_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doContinue___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_termTry_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doExpr(lean_object*); @@ -1953,16 +2141,19 @@ static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__16; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__23; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__6; lean_object* l_Lean_Parser_Term_matchAlts_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfLetPure_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__21; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___closed__2; static lean_object* l_Lean_Parser_Term_doBreak___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doCatch; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_doFor_declRange___closed__5; static lean_object* l_Lean_Parser_Term_doIfLetPure___closed__7; static lean_object* l_Lean_Parser_Term_doPatDecl___closed__6; static lean_object* l_Lean_Parser_Term_doPatDecl___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doLet___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_liftMethod___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_doIfLetBind___closed__1; @@ -1975,11 +2166,11 @@ static lean_object* l_Lean_Parser_Term_doSeqItem_formatter___closed__2; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__47; static lean_object* l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_declRange___closed__2; -static lean_object* l_Lean_Parser_Term_doFor_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_doForDecl_formatter___closed__10; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColGt_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doFinally___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_doSeqBracketed___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__2; lean_object* l_Lean_Parser_symbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfLetBind_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqBracketed_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1992,12 +2183,16 @@ lean_object* l_Lean_Parser_Term_binderIdent___elambda__1(lean_object*, lean_obje static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__20; static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_doDbgTrace___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_declRange___closed__4; static lean_object* l_Lean_Parser_Term_termReturn_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doExpr_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doExpr___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__19; static lean_object* l_Lean_Parser_Term_do___closed__5; @@ -2005,6 +2200,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_declRange___closed__ static lean_object* l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_declRange___closed__7; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__24; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doLetArrow_formatter___closed__2; @@ -2016,12 +2212,16 @@ static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__23; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassign_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doNested___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doForDecl___closed__8; static lean_object* l_Lean_Parser_Term_doReassign___closed__7; static lean_object* l_Lean_Parser_Term_elseIf_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doHave_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doBreak_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doReturn___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__4; @@ -2035,18 +2235,24 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_do___elambda__1(lean_object*, lean_o static lean_object* l___regBuiltin_Lean_Parser_Term_doIf_declRange___closed__5; static lean_object* l_Lean_Parser_Term_doIdDecl_formatter___closed__5; static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doMatch_formatter___closed__16; lean_object* l_Lean_Parser_symbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doBreak___closed__3; static lean_object* l_Lean_Parser_Term_doLetArrow_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__2; extern lean_object* l_Lean_Parser_Term_generalizingParam; static lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__2; lean_object* l_Lean_Parser_Term_haveDecl___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doCatchMatch_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_doUnless___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__22; static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_declRange___closed__1; static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__4; @@ -2054,6 +2260,7 @@ static lean_object* l_Lean_Parser_Term_liftMethod_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqBracketed; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLet; static lean_object* l_Lean_Parser_Term_doPatDecl___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doIfCond_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doExpr; static lean_object* l___regBuiltin_Lean_Parser_Term_doTry_declRange___closed__1; @@ -2063,8 +2270,10 @@ static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda lean_object* l_Lean_PrettyPrinter_Formatter_withoutPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lean_Parser_Term_doIfLetPure___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doLetElse_formatter___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_termReturn_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doIfLetBind_formatter___closed__4; static lean_object* l_Lean_Parser_Term_doHave___elambda__1___closed__3; @@ -2074,6 +2283,7 @@ static lean_object* l_Lean_Parser_Term_doExpr___closed__3; static lean_object* l_Lean_Parser_Term_doIdDecl___closed__1; static lean_object* l_Lean_Parser_Term_doElem_quot___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_leftArrow___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__3; static lean_object* l_Lean_Parser_Term_doElem_quot___elambda__1___closed__1; @@ -2085,6 +2295,7 @@ static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_declRange___closed__4; static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__2; lean_object* l_Lean_Parser_Term_optIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__27; lean_object* l_Lean_Parser_unicodeSymbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2101,12 +2312,14 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_doLet_declRange___closed__5; static lean_object* l_Lean_Parser_Term_do_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doPatDecl; lean_object* l_Lean_Parser_checkColGtFn___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doLet_formatter___closed__8; static lean_object* l_Lean_Parser_Term_doCatch___elambda__1___closed__17; static lean_object* l_Lean_Parser_Term_doMatch_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__17; static lean_object* l_Lean_Parser_Term_doFinally_formatter___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doLet___closed__9; static lean_object* l_Lean_Parser_Term_doCatch_formatter___closed__5; static lean_object* l_Lean_Parser_Term_liftMethod___closed__2; @@ -2130,6 +2343,7 @@ static lean_object* l_Lean_Parser_Term_doExpr___closed__5; static lean_object* l_Lean_Parser_Term_doIfLet___closed__6; static lean_object* l_Lean_Parser_Term_termUnless___closed__6; static lean_object* l_Lean_Parser_Term_doIf_parenthesizer___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Term_do_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__14; static lean_object* l_Lean_Parser_Term_doUnless_formatter___closed__8; static lean_object* l_Lean_Parser_Term_elseIf_formatter___closed__2; @@ -2143,11 +2357,14 @@ static lean_object* l_Lean_Parser_Term_doElem_quot___closed__1; static lean_object* l_Lean_Parser_Term_doLetElse___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_declRange___closed__4; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__44; +static lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doLetElse_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_declRange___closed__3; static lean_object* l_Lean_Parser_Term_doTry___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_declRange___closed__4; static lean_object* l_Lean_Parser_Term_doReassign_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doIf___closed__11; static lean_object* l_Lean_Parser_Term_termTry___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_doPatDecl___closed__8; @@ -2155,7 +2372,9 @@ static lean_object* l_Lean_Parser_Term_do_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doMatch___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken___elambda__1___closed__17; static lean_object* l_Lean_Parser_Term_doLetElse_parenthesizer___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__2; static lean_object* l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doNested___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_doCatch_formatter___closed__7; static lean_object* l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__5; @@ -2165,9 +2384,10 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_do_declRange___closed__7; lean_object* l_Lean_Parser_termParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ppDedent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLet_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer(lean_object*); extern lean_object* l_Lean_Parser_Term_ident; +static lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doForDecl___closed__9; -static lean_object* l_Lean_Parser_Term_doLetArrow_formatter___closed__8; static lean_object* l_Lean_Parser_Term_doIf_formatter___closed__5; static lean_object* l_Lean_Parser_Term_doIf___elambda__1___closed__34; static lean_object* l_Lean_Parser_Term_doCatch___closed__11; @@ -2182,15 +2402,16 @@ static lean_object* l_Lean_Parser_Term_doUnless_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doReassignArrow___closed__3; lean_object* l_Lean_Parser_setLhsPrecFn___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLet_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_categoryParser_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doLetElse___elambda__1___closed__2; lean_object* l_Lean_Parser_andthenFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doExpr___elambda__1___closed__9; -static lean_object* l_Lean_Parser_Term_doReassign_formatter___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqItem_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__1; static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Do___hyg_5____closed__1() { _start: { @@ -3028,6 +3249,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_liftMethod___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_liftMethod_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_liftMethod___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_leftArrow_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -3110,6 +3377,52 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_liftMethod___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_liftMethod_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_liftMethod___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqItem___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -4735,6 +5048,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doSeqItem___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqItem_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doSeqItem___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__1() { _start: { @@ -4766,32 +5109,24 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqItem_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__4; +x_1 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withoutPosition_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -4801,49 +5136,49 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doSeqItem_formatter___closed__6; -x_2 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__6; +x_2 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__5; -x_2 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__7; +x_1 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__4; +x_2 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__8; +x_2 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__9; +x_3 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -4856,11 +5191,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqBracketed_formatter(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__1; -x_7 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__10; +x_7 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__9; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqBracketed_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doSeqIndent_formatter___closed__1() { _start: { @@ -4883,7 +5248,7 @@ static lean_object* _init_l_Lean_Parser_Term_doSeqIndent_formatter___closed__2() _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doSeqBracketed_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1Indent_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -4913,6 +5278,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqIndent_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doSeq_formatter___closed__1() { _start: { @@ -4933,25 +5328,9 @@ return x_6; static lean_object* _init_l_Lean_Parser_Term_doSeq_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqBracketed_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doSeq_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqIndent_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doSeq_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doSeq_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doSeq_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -4963,7 +5342,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeq_formatter(lean_object* x_1, le { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doSeq_formatter___closed__1; -x_7 = l_Lean_Parser_Term_doSeq_formatter___closed__4; +x_7 = l_Lean_Parser_Term_doSeq_formatter___closed__2; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -5081,6 +5460,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doSeqItem___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqItem_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doSeqItem___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1() { _start: { @@ -5112,32 +5521,24 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqItem_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_withoutPosition_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -5147,49 +5548,49 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__7; +x_1 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__8; +x_2 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__9; +x_3 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -5202,11 +5603,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeqBracketed_parenthesizer(lean_ob { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__10; +x_7 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__9; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqBracketed_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doSeqBracketed___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1() { _start: { @@ -5229,7 +5660,7 @@ static lean_object* _init_l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed_ _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1Indent_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -5259,6 +5690,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqIndent_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doSeqIndent___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doSeq_parenthesizer___closed__1() { _start: { @@ -5279,25 +5740,9 @@ return x_6; static lean_object* _init_l_Lean_Parser_Term_doSeq_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqBracketed_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doSeq_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doSeqIndent_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doSeq_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doSeq_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doSeq_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -5309,7 +5754,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doSeq_parenthesizer(lean_object* x_1 { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doSeq_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_doSeq_parenthesizer___closed__4; +x_7 = l_Lean_Parser_Term_doSeq_parenthesizer___closed__2; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -6920,6 +7365,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doLet___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doLet_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLet_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doLet___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doLet_parenthesizer___closed__1() { _start: { @@ -7024,6 +7499,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doLet___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doLet_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doLet___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doLetElse___elambda__1___closed__1() { _start: { @@ -8037,6 +8542,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doLetElse___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doLetElse_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doLetElse___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doLetElse_parenthesizer___closed__1() { _start: { @@ -8179,6 +8714,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doLetElse___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doLetElse_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doLetElse___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetRec___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -8858,6 +9423,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doLetRec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doLetRec_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doLetRec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doLetRec_parenthesizer___closed__1() { _start: { @@ -8955,6 +9550,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doLetRec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doLetRec_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doLetRec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIdDecl___elambda__1___closed__1() { _start: { @@ -10578,6 +11203,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIdDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIdDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doIdDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doPatDecl_formatter___closed__1() { _start: { @@ -10676,6 +11331,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doPatDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doPatDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doPatDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__1() { _start: { @@ -10697,72 +11382,56 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIdDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doPatDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doLetArrow_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doLetArrow_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doLet_formatter___closed__4; -x_2 = l_Lean_Parser_Term_doLetArrow_formatter___closed__4; +x_2 = l_Lean_Parser_Term_doLetArrow_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doLet_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doLetArrow_formatter___closed__5; +x_2 = l_Lean_Parser_Term_doLetArrow_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doLetArrow_formatter___closed__6; +x_1 = l_Lean_Parser_Term_doLetArrow_formatter___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withPosition_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doLetArrow___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doLetArrow_formatter___closed__7; +x_3 = l_Lean_Parser_Term_doLetArrow_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -10775,11 +11444,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetArrow_formatter(lean_object* x_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doLetArrow_formatter___closed__1; -x_7 = l_Lean_Parser_Term_doLetArrow_formatter___closed__8; +x_7 = l_Lean_Parser_Term_doLetArrow_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doLetArrow___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doLetArrow_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doLetArrow___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1() { _start: { @@ -10904,6 +11603,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIdDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIdDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doIdDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1() { _start: { @@ -11026,6 +11755,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doPatDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doPatDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doPatDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1() { _start: { @@ -11047,72 +11806,56 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIdDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doPatDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doLet_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doLet_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doLetArrow___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -11125,11 +11868,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doLetArrow_parenthesizer(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__8; +x_7 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doLetArrow___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doLetArrow_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doLetArrow___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__1() { _start: { @@ -11841,6 +12614,54 @@ x_8 = l_Lean_PrettyPrinter_Formatter_node_formatter(x_6, x_7, x_1, x_2, x_3, x_4 return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("letIdDeclNoBinders", 18); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_liftMethod___elambda__1___closed__6; +x_2 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letIdDeclNoBinders_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__3; +x_5 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__1() { _start: { @@ -11863,31 +12684,23 @@ static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__2() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letIdDeclNoBinders_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__3() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letPatDecl_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doReassign_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doReassign_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__4; +x_2 = l_Lean_Parser_Term_doReassign_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__4() { _start: { lean_object* x_1; @@ -11895,25 +12708,25 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_notFollowedByRedefinedTermTo return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doReassign_formatter___closed__5; -x_2 = l_Lean_Parser_Term_doReassign_formatter___closed__4; +x_1 = l_Lean_Parser_Term_doReassign_formatter___closed__4; +x_2 = l_Lean_Parser_Term_doReassign_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doReassign_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doReassign___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doReassign_formatter___closed__6; +x_3 = l_Lean_Parser_Term_doReassign_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -11926,11 +12739,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassign_formatter(lean_object* x_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doReassign_formatter___closed__1; -x_7 = l_Lean_Parser_Term_doReassign_formatter___closed__7; +x_7 = l_Lean_Parser_Term_doReassign_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doReassign___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doReassign_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doReassign___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_notFollowedByRedefinedTermToken_parenthesizer___rarg(lean_object* x_1) { _start: { @@ -12038,6 +12881,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_node_parenthesizer(x_6, x_7, x_1, x_2, return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__1() { _start: { @@ -12060,31 +12933,23 @@ static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letPatDecl_parenthesizer), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__4() { _start: { lean_object* x_1; @@ -12092,25 +12957,25 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_notFollowedByRedefinedTermTo return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doReassign___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__6; +x_3 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -12123,11 +12988,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassign_parenthesizer(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__7; +x_7 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doReassign___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doReassign_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doReassign___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReassignArrow___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -12641,7 +13536,7 @@ static lean_object* _init_l_Lean_Parser_Term_doReassignArrow_formatter___closed_ _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doLetArrow_formatter___closed__4; +x_1 = l_Lean_Parser_Term_doLetArrow_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withPosition_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -12651,7 +13546,7 @@ static lean_object* _init_l_Lean_Parser_Term_doReassignArrow_formatter___closed_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doReassign_formatter___closed__5; +x_1 = l_Lean_Parser_Term_doReassign_formatter___closed__4; x_2 = l_Lean_Parser_Term_doReassignArrow_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -12683,6 +13578,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doReassignArrow_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1() { _start: { @@ -12705,7 +13630,7 @@ static lean_object* _init_l_Lean_Parser_Term_doReassignArrow_parenthesizer___clo _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -12715,7 +13640,7 @@ static lean_object* _init_l_Lean_Parser_Term_doReassignArrow_parenthesizer___clo _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__4; x_2 = l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -12747,6 +13672,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doReassignArrow_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doHave___elambda__1___closed__1() { _start: { @@ -13334,6 +14289,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doHave___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doHave_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doHave_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doHave___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doHave_parenthesizer___closed__1() { _start: { @@ -13406,6 +14391,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doHave___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doHave_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doHave___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_elseIf___elambda__1___lambda__1___closed__1() { _start: { @@ -17241,6 +18256,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLetPure_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfLetBind_formatter___closed__1() { _start: { @@ -17305,6 +18350,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLetBind_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__1() { _start: { @@ -17325,62 +18400,46 @@ return x_6; static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLetPure_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLetBind_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doIfLet_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doIfLet_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_liftMethod_formatter___closed__3; -x_2 = l_Lean_Parser_Term_doIfLet_formatter___closed__4; +x_2 = l_Lean_Parser_Term_doIfLet_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doLet_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doIfLet_formatter___closed__5; +x_2 = l_Lean_Parser_Term_doIfLet_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doIfLet_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doIfLet___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doIfLet_formatter___closed__6; +x_3 = l_Lean_Parser_Term_doIfLet_formatter___closed__4; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -17393,11 +18452,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfLet_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doIfLet_formatter___closed__1; -x_7 = l_Lean_Parser_Term_doIfLet_formatter___closed__7; +x_7 = l_Lean_Parser_Term_doIfLet_formatter___closed__5; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIfLet___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLet_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLet_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doIfLet___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfProp_formatter___closed__1() { _start: { @@ -17459,6 +18548,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIfProp___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfProp_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfProp_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doIfProp___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfCond_formatter___closed__1() { _start: { @@ -17480,25 +18599,9 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_doIfCond_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLet_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doIfCond_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfProp_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doIfCond_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doIfCond_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doIfCond_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -17510,7 +18613,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfCond_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doIfCond_formatter___closed__1; -x_7 = l_Lean_Parser_Term_doIfCond_formatter___closed__4; +x_7 = l_Lean_Parser_Term_doIfCond_formatter___closed__2; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -17844,6 +18947,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIf___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIf_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIf_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doIf___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1() { _start: { @@ -17898,6 +19031,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLetPure_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doIfLetPure___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1() { _start: { @@ -17962,6 +19125,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLetBind_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doIfLetBind___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__1() { _start: { @@ -17982,62 +19175,46 @@ return x_6; static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLetPure_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLetBind_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_liftMethod_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doLet_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doIfLet___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__6; +x_3 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__4; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -18050,11 +19227,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfLet_parenthesizer(lean_object* x { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__7; +x_7 = l_Lean_Parser_Term_doIfLet_parenthesizer___closed__5; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIfLet___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLet_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doIfLet___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfProp_parenthesizer___closed__1() { _start: { @@ -18116,6 +19323,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIfProp___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfProp_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doIfProp___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doIfCond_parenthesizer___closed__1() { _start: { @@ -18137,25 +19374,9 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_doIfCond_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfLet_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doIfCond_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIfProp_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doIfCond_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doIfCond_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doIfCond_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -18167,7 +19388,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doIfCond_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doIfCond_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_doIfCond_parenthesizer___closed__4; +x_7 = l_Lean_Parser_Term_doIfCond_parenthesizer___closed__2; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -18501,6 +19722,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doIf___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doIf_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doIf___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_doUnless___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -19279,6 +20530,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doUnless___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doUnless_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doUnless___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doUnless_parenthesizer___closed__1() { _start: { @@ -19387,6 +20668,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doUnless___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doUnless_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doUnless___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doForDecl___elambda__1___closed__1() { _start: { @@ -20728,6 +22039,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doForDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doForDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doForDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doForDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__1() { _start: { @@ -20769,16 +22110,8 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doForDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Term_doFor_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__2; x_2 = l_Lean_Parser_Term_doFor___elambda__1___closed__7; x_3 = l_Lean_Parser_Term_doFor_formatter___closed__3; x_4 = 0; @@ -20791,11 +22124,11 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doFor_formatter___closed__5; +x_1 = l_Lean_Parser_Term_doFor_formatter___closed__4; x_2 = l_Lean_Parser_Term_doUnless_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -20803,25 +22136,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doFor_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doFor_formatter___closed__6; +x_2 = l_Lean_Parser_Term_doFor_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_doFor_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doFor___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doFor_formatter___closed__7; +x_3 = l_Lean_Parser_Term_doFor_formatter___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -20834,11 +22167,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doFor_formatter(lean_object* x_1, le { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doFor_formatter___closed__1; -x_7 = l_Lean_Parser_Term_doFor_formatter___closed__8; +x_7 = l_Lean_Parser_Term_doFor_formatter___closed__7; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doFor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doFor_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFor_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doFor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doForDecl_parenthesizer___closed__1() { _start: { @@ -20969,6 +22332,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doForDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doForDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doForDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__1() { _start: { @@ -21010,16 +22403,8 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doForDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Term_doFor_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__2; x_2 = l_Lean_Parser_Term_doFor___elambda__1___closed__7; x_3 = l_Lean_Parser_Term_doFor_parenthesizer___closed__3; x_4 = 0; @@ -21032,11 +22417,11 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doFor_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Term_doFor_parenthesizer___closed__4; x_2 = l_Lean_Parser_Term_doUnless_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -21044,25 +22429,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doFor_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doFor_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_doFor_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doFor___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doFor_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Term_doFor_parenthesizer___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -21075,11 +22460,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doFor_parenthesizer(lean_object* x_1 { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doFor_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_doFor_parenthesizer___closed__8; +x_7 = l_Lean_Parser_Term_doFor_parenthesizer___closed__7; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doFor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doFor_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doFor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doMatchAlts___closed__1() { _start: { @@ -22098,6 +23513,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doMatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doMatch_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doMatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_doMatchAlts_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -22298,6 +23743,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doMatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doMatch_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doMatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doCatch___elambda__1___closed__1() { _start: { @@ -24372,6 +25847,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doCatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doCatch_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doCatch_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doCatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doCatchMatch_formatter___closed__1() { _start: { @@ -24426,6 +25931,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doCatchMatch_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doFinally_formatter___closed__1() { _start: { @@ -24490,6 +26025,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doFinally___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doFinally_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFinally_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doFinally___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__1() { _start: { @@ -24521,102 +26086,78 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doCatch_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doCatchMatch_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doTry_formatter___closed__3; -x_2 = l_Lean_Parser_Term_doTry_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doTry_formatter___closed__5; +x_1 = l_Lean_Parser_Term_doTry_formatter___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doFinally_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doTry_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doTry_formatter___closed__6; -x_2 = l_Lean_Parser_Term_doTry_formatter___closed__8; +x_1 = l_Lean_Parser_Term_doTry_formatter___closed__4; +x_2 = l_Lean_Parser_Term_doTry_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__6; -x_2 = l_Lean_Parser_Term_doTry_formatter___closed__9; +x_2 = l_Lean_Parser_Term_doTry_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doTry_formatter___closed__2; -x_2 = l_Lean_Parser_Term_doTry_formatter___closed__10; +x_2 = l_Lean_Parser_Term_doTry_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_doTry_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doTry___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doTry_formatter___closed__11; +x_3 = l_Lean_Parser_Term_doTry_formatter___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -24629,11 +26170,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doTry_formatter(lean_object* x_1, le { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doTry_formatter___closed__1; -x_7 = l_Lean_Parser_Term_doTry_formatter___closed__12; +x_7 = l_Lean_Parser_Term_doTry_formatter___closed__9; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doTry___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doTry_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doTry_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doTry___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doCatch_parenthesizer___closed__1() { _start: { @@ -24782,6 +26353,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doCatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doCatch_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doCatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1() { _start: { @@ -24836,6 +26437,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doCatchMatch_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doCatchMatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doFinally_parenthesizer___closed__1() { _start: { @@ -24900,6 +26531,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doFinally___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doFinally_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doFinally___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__1() { _start: { @@ -24931,102 +26592,78 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doCatch_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doCatchMatch_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doTry_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_doTry_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doTry_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Term_doTry_parenthesizer___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doFinally_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_doTry_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doTry_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Term_doTry_parenthesizer___closed__8; +x_1 = l_Lean_Parser_Term_doTry_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_doTry_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__9; -x_2 = l_Lean_Parser_Term_doTry_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Term_doTry_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_doTry_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_doTry_parenthesizer___closed__10; +x_2 = l_Lean_Parser_Term_doTry_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_doTry___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doTry_parenthesizer___closed__11; +x_3 = l_Lean_Parser_Term_doTry_parenthesizer___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -25039,11 +26676,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doTry_parenthesizer(lean_object* x_1 { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_doTry_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_doTry_parenthesizer___closed__12; +x_7 = l_Lean_Parser_Term_doTry_parenthesizer___closed__9; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doTry___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doTry_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doTry___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doBreak___elambda__1___closed__1() { _start: { @@ -25515,6 +27182,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doBreak___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doBreak_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doBreak___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doBreak_parenthesizer___closed__1() { _start: { @@ -25567,6 +27264,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doBreak___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doBreak_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doBreak___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doContinue___elambda__1___closed__1() { _start: { @@ -26038,6 +27765,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doContinue___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doContinue_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doContinue___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doContinue_parenthesizer___closed__1() { _start: { @@ -26090,6 +27847,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doContinue___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doContinue_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doContinue___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_doReturn___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -26921,6 +28708,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doReturn___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doReturn_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doReturn___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doReturn_parenthesizer___closed__1() { _start: { @@ -27017,6 +28834,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doReturn___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doReturn_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doReturn___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__1() { _start: { @@ -27656,6 +29503,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doDbgTrace_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1() { _start: { @@ -27742,6 +29619,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doDbgTrace_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doAssert___elambda__1___closed__1() { _start: { @@ -28317,6 +30224,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doAssert___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doAssert_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doAssert___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doAssert_parenthesizer___closed__1() { _start: { @@ -28381,6 +30318,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doAssert___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doAssert_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doAssert___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doExpr___elambda__1___closed__1() { _start: { @@ -29045,7 +31012,7 @@ static lean_object* _init_l_Lean_Parser_Term_doExpr_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doReassign_formatter___closed__5; +x_1 = l_Lean_Parser_Term_doReassign_formatter___closed__4; x_2 = l_Lean_Parser_Term_doExpr_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -29077,6 +31044,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doExpr___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doExpr_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doExpr___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doExpr_parenthesizer___closed__1() { _start: { @@ -29175,7 +31172,7 @@ static lean_object* _init_l_Lean_Parser_Term_doExpr_parenthesizer___closed__9() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Term_doReassign_parenthesizer___closed__4; x_2 = l_Lean_Parser_Term_doExpr_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -29207,6 +31204,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doExpr___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doExpr_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doExpr___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doNested___elambda__1___closed__1() { _start: { @@ -29676,6 +31703,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doNested___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doNested_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doNested_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doNested___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doNested_parenthesizer___closed__1() { _start: { @@ -29718,6 +31775,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doNested___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doNested_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doNested___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_do___elambda__1___closed__1() { _start: { @@ -30197,6 +32284,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_do_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_do___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_do_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_do_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_do_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_do___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_do_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_do_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_do_parenthesizer___closed__1() { _start: { @@ -30259,6 +32376,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_do___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_do_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_do_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_do___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doElem_quot___elambda__1___closed__1() { _start: { @@ -30999,6 +33146,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doElem_quot___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doElem_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doElem_quot___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1() { _start: { @@ -31095,6 +33272,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doElem_quot___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doElem_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doElem_quot___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_termUnless___elambda__1___closed__1() { _start: { @@ -31639,6 +33846,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_termUnless___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_termUnless_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_termUnless___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_termUnless_parenthesizer___closed__1() { _start: { @@ -31681,6 +33918,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_termUnless___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_termUnless_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_termUnless___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_termFor___elambda__1___closed__1() { _start: { @@ -32150,7 +34417,7 @@ static lean_object* _init_l_Lean_Parser_Term_termFor_formatter___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_termFor___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doFor_formatter___closed__7; +x_3 = l_Lean_Parser_Term_doFor_formatter___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -32168,6 +34435,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_termFor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_termFor_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termFor_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_termFor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_termFor_parenthesizer___closed__1() { _start: { @@ -32192,7 +34489,7 @@ static lean_object* _init_l_Lean_Parser_Term_termFor_parenthesizer___closed__2() lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_termFor___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doFor_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Term_doFor_parenthesizer___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -32210,6 +34507,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_termFor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_termFor_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_termFor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_termTry___elambda__1___closed__1() { _start: { @@ -32697,7 +35024,7 @@ static lean_object* _init_l_Lean_Parser_Term_termTry_formatter___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_termTry___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doTry_formatter___closed__11; +x_3 = l_Lean_Parser_Term_doTry_formatter___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -32715,6 +35042,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_termTry___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_termTry_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termTry_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_termTry___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_termTry_parenthesizer___closed__1() { _start: { @@ -32739,7 +35096,7 @@ static lean_object* _init_l_Lean_Parser_Term_termTry_parenthesizer___closed__2() lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_termTry___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_doTry_parenthesizer___closed__11; +x_3 = l_Lean_Parser_Term_doTry_parenthesizer___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -32757,6 +35114,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_termTry___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_termTry_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_termTry___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_termReturn___elambda__1___closed__1() { _start: { @@ -33282,6 +35669,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_termReturn___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_termReturn_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3; +x_3 = l_Lean_Parser_Term_termReturn___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_termReturn_parenthesizer___closed__1() { _start: { @@ -33324,6 +35741,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_termReturn___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_termReturn_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_termReturn___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Term(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -33469,6 +35916,17 @@ l_Lean_Parser_Term_liftMethod_formatter___closed__4 = _init_l_Lean_Parser_Term_l lean_mark_persistent(l_Lean_Parser_Term_liftMethod_formatter___closed__4); l_Lean_Parser_Term_liftMethod_formatter___closed__5 = _init_l_Lean_Parser_Term_liftMethod_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_liftMethod_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_liftMethod_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Term_liftMethod_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_liftMethod_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_liftMethod_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_liftMethod_parenthesizer___closed__1); l_Lean_Parser_Term_liftMethod_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_liftMethod_parenthesizer___closed__2(); @@ -33479,6 +35937,17 @@ l_Lean_Parser_Term_liftMethod_parenthesizer___closed__4 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_liftMethod_parenthesizer___closed__4); l_Lean_Parser_Term_liftMethod_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_liftMethod_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_liftMethod_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_Term_liftMethod_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doSeqItem___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doSeqItem___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doSeqItem___elambda__1___closed__1); l_Lean_Parser_Term_doSeqItem___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doSeqItem___elambda__1___closed__2(); @@ -33639,6 +36108,13 @@ l_Lean_Parser_Term_doSeqItem_formatter___closed__7 = _init_l_Lean_Parser_Term_do lean_mark_persistent(l_Lean_Parser_Term_doSeqItem_formatter___closed__7); l_Lean_Parser_Term_doSeqItem_formatter___closed__8 = _init_l_Lean_Parser_Term_doSeqItem_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_doSeqItem_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doSeqItem_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doSeqBracketed_formatter___closed__1 = _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doSeqBracketed_formatter___closed__1); l_Lean_Parser_Term_doSeqBracketed_formatter___closed__2 = _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__2(); @@ -33657,22 +36133,30 @@ l_Lean_Parser_Term_doSeqBracketed_formatter___closed__8 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_doSeqBracketed_formatter___closed__8); l_Lean_Parser_Term_doSeqBracketed_formatter___closed__9 = _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_doSeqBracketed_formatter___closed__9); -l_Lean_Parser_Term_doSeqBracketed_formatter___closed__10 = _init_l_Lean_Parser_Term_doSeqBracketed_formatter___closed__10(); -lean_mark_persistent(l_Lean_Parser_Term_doSeqBracketed_formatter___closed__10); +l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doSeqBracketed_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doSeqIndent_formatter___closed__1 = _init_l_Lean_Parser_Term_doSeqIndent_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doSeqIndent_formatter___closed__1); l_Lean_Parser_Term_doSeqIndent_formatter___closed__2 = _init_l_Lean_Parser_Term_doSeqIndent_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doSeqIndent_formatter___closed__2); l_Lean_Parser_Term_doSeqIndent_formatter___closed__3 = _init_l_Lean_Parser_Term_doSeqIndent_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doSeqIndent_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doSeqIndent_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doSeq_formatter___closed__1 = _init_l_Lean_Parser_Term_doSeq_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doSeq_formatter___closed__1); l_Lean_Parser_Term_doSeq_formatter___closed__2 = _init_l_Lean_Parser_Term_doSeq_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doSeq_formatter___closed__2); -l_Lean_Parser_Term_doSeq_formatter___closed__3 = _init_l_Lean_Parser_Term_doSeq_formatter___closed__3(); -lean_mark_persistent(l_Lean_Parser_Term_doSeq_formatter___closed__3); -l_Lean_Parser_Term_doSeq_formatter___closed__4 = _init_l_Lean_Parser_Term_doSeq_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Term_doSeq_formatter___closed__4); l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1); l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2(); @@ -33689,6 +36173,13 @@ l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__7 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__7); l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_doSeqItem_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doSeqItem_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1); l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2(); @@ -33707,22 +36198,30 @@ l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__8 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__8); l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__9); -l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__10 = _init_l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__10(); -lean_mark_persistent(l_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__10); +l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doSeqBracketed_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1); l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2); l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doSeqIndent_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doSeq_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doSeq_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doSeq_parenthesizer___closed__1); l_Lean_Parser_Term_doSeq_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doSeq_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doSeq_parenthesizer___closed__2); -l_Lean_Parser_Term_doSeq_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_doSeq_parenthesizer___closed__3(); -lean_mark_persistent(l_Lean_Parser_Term_doSeq_parenthesizer___closed__3); -l_Lean_Parser_Term_doSeq_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_doSeq_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Term_doSeq_parenthesizer___closed__4); l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__1 = _init_l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__1(); lean_mark_persistent(l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__1); l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__2 = _init_l_Lean_Parser_Term_initFn____x40_Lean_Parser_Do___hyg_163____closed__2(); @@ -33970,6 +36469,13 @@ l_Lean_Parser_Term_doLet_formatter___closed__7 = _init_l_Lean_Parser_Term_doLet_ lean_mark_persistent(l_Lean_Parser_Term_doLet_formatter___closed__7); l_Lean_Parser_Term_doLet_formatter___closed__8 = _init_l_Lean_Parser_Term_doLet_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_doLet_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLet_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doLet_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doLet_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doLet_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doLet_parenthesizer___closed__1); l_Lean_Parser_Term_doLet_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doLet_parenthesizer___closed__2(); @@ -33986,6 +36492,13 @@ l_Lean_Parser_Term_doLet_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_do lean_mark_persistent(l_Lean_Parser_Term_doLet_parenthesizer___closed__7); l_Lean_Parser_Term_doLet_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_doLet_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_doLet_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doLet_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doLetElse___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doLetElse___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doLetElse___elambda__1___closed__1); l_Lean_Parser_Term_doLetElse___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doLetElse___elambda__1___closed__2(); @@ -34106,6 +36619,13 @@ l_Lean_Parser_Term_doLetElse_formatter___closed__10 = _init_l_Lean_Parser_Term_d lean_mark_persistent(l_Lean_Parser_Term_doLetElse_formatter___closed__10); l_Lean_Parser_Term_doLetElse_formatter___closed__11 = _init_l_Lean_Parser_Term_doLetElse_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Term_doLetElse_formatter___closed__11); +l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetElse_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doLetElse_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doLetElse_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doLetElse_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doLetElse_parenthesizer___closed__1); l_Lean_Parser_Term_doLetElse_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doLetElse_parenthesizer___closed__2(); @@ -34128,6 +36648,13 @@ l_Lean_Parser_Term_doLetElse_parenthesizer___closed__10 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_doLetElse_parenthesizer___closed__10); l_Lean_Parser_Term_doLetElse_parenthesizer___closed__11 = _init_l_Lean_Parser_Term_doLetElse_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Term_doLetElse_parenthesizer___closed__11); +l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doLetElse_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doLetRec___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doLetRec___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doLetRec___elambda__1___closed__1); l_Lean_Parser_Term_doLetRec___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doLetRec___elambda__1___closed__2(); @@ -34204,6 +36731,13 @@ l_Lean_Parser_Term_doLetRec_formatter___closed__6 = _init_l_Lean_Parser_Term_doL lean_mark_persistent(l_Lean_Parser_Term_doLetRec_formatter___closed__6); l_Lean_Parser_Term_doLetRec_formatter___closed__7 = _init_l_Lean_Parser_Term_doLetRec_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doLetRec_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetRec_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doLetRec_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doLetRec_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doLetRec_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doLetRec_parenthesizer___closed__1); l_Lean_Parser_Term_doLetRec_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doLetRec_parenthesizer___closed__2(); @@ -34218,6 +36752,13 @@ l_Lean_Parser_Term_doLetRec_parenthesizer___closed__6 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_doLetRec_parenthesizer___closed__6); l_Lean_Parser_Term_doLetRec_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_doLetRec_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doLetRec_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doLetRec_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIdDecl___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doIdDecl___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIdDecl___elambda__1___closed__1); l_Lean_Parser_Term_doIdDecl___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doIdDecl___elambda__1___closed__2(); @@ -34378,6 +36919,13 @@ l_Lean_Parser_Term_doIdDecl_formatter___closed__9 = _init_l_Lean_Parser_Term_doI lean_mark_persistent(l_Lean_Parser_Term_doIdDecl_formatter___closed__9); l_Lean_Parser_Term_doIdDecl_formatter___closed__10 = _init_l_Lean_Parser_Term_doIdDecl_formatter___closed__10(); lean_mark_persistent(l_Lean_Parser_Term_doIdDecl_formatter___closed__10); +l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIdDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doPatDecl_formatter___closed__1 = _init_l_Lean_Parser_Term_doPatDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doPatDecl_formatter___closed__1); l_Lean_Parser_Term_doPatDecl_formatter___closed__2 = _init_l_Lean_Parser_Term_doPatDecl_formatter___closed__2(); @@ -34392,6 +36940,13 @@ l_Lean_Parser_Term_doPatDecl_formatter___closed__6 = _init_l_Lean_Parser_Term_do lean_mark_persistent(l_Lean_Parser_Term_doPatDecl_formatter___closed__6); l_Lean_Parser_Term_doPatDecl_formatter___closed__7 = _init_l_Lean_Parser_Term_doPatDecl_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doPatDecl_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doPatDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doLetArrow_formatter___closed__1 = _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_formatter___closed__1); l_Lean_Parser_Term_doLetArrow_formatter___closed__2 = _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__2(); @@ -34404,10 +36959,13 @@ l_Lean_Parser_Term_doLetArrow_formatter___closed__5 = _init_l_Lean_Parser_Term_d lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_formatter___closed__5); l_Lean_Parser_Term_doLetArrow_formatter___closed__6 = _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_formatter___closed__6); -l_Lean_Parser_Term_doLetArrow_formatter___closed__7 = _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_formatter___closed__7); -l_Lean_Parser_Term_doLetArrow_formatter___closed__8 = _init_l_Lean_Parser_Term_doLetArrow_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doLetArrow_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1); l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2(); @@ -34428,6 +36986,13 @@ l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__9 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__9); l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__10 = _init_l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__10(); lean_mark_persistent(l_Lean_Parser_Term_doIdDecl_parenthesizer___closed__10); +l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIdDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1); l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2(); @@ -34446,6 +37011,13 @@ l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__8 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__8); l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_doPatDecl_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doPatDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1); l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2(); @@ -34458,10 +37030,13 @@ l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__5 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__5); l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__6); -l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__7); -l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_doLetArrow_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doLetArrow_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__1 = _init_l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__1); l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__2 = _init_l_Lean_Parser_Term_letIdDeclNoBinders___elambda__1___closed__2(); @@ -34558,6 +37133,17 @@ l_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__5 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__5); l_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__6 = _init_l_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doReassign_formatter___closed__1 = _init_l_Lean_Parser_Term_doReassign_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doReassign_formatter___closed__1); l_Lean_Parser_Term_doReassign_formatter___closed__2 = _init_l_Lean_Parser_Term_doReassign_formatter___closed__2(); @@ -34570,8 +37156,13 @@ l_Lean_Parser_Term_doReassign_formatter___closed__5 = _init_l_Lean_Parser_Term_d lean_mark_persistent(l_Lean_Parser_Term_doReassign_formatter___closed__5); l_Lean_Parser_Term_doReassign_formatter___closed__6 = _init_l_Lean_Parser_Term_doReassign_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_doReassign_formatter___closed__6); -l_Lean_Parser_Term_doReassign_formatter___closed__7 = _init_l_Lean_Parser_Term_doReassign_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_doReassign_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReassign_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doReassign_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1); l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2(); @@ -34584,6 +37175,13 @@ l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__5 = _init_l_Lean_P lean_mark_persistent(l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__5); l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letIdDeclNoBinders_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doReassign_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doReassign_parenthesizer___closed__1); l_Lean_Parser_Term_doReassign_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__2(); @@ -34596,8 +37194,13 @@ l_Lean_Parser_Term_doReassign_parenthesizer___closed__5 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_doReassign_parenthesizer___closed__5); l_Lean_Parser_Term_doReassign_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_doReassign_parenthesizer___closed__6); -l_Lean_Parser_Term_doReassign_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_doReassign_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_doReassign_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doReassign_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__1); l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doReassignArrow___elambda__1___closed__2(); @@ -34658,6 +37261,13 @@ l_Lean_Parser_Term_doReassignArrow_formatter___closed__3 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_doReassignArrow_formatter___closed__3); l_Lean_Parser_Term_doReassignArrow_formatter___closed__4 = _init_l_Lean_Parser_Term_doReassignArrow_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doReassignArrow_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doReassignArrow_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1); l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2(); @@ -34666,6 +37276,13 @@ l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__3 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__3); l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doReassignArrow_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doHave___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doHave___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doHave___elambda__1___closed__1); l_Lean_Parser_Term_doHave___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doHave___elambda__1___closed__2(); @@ -34740,6 +37357,13 @@ l_Lean_Parser_Term_doHave_formatter___closed__4 = _init_l_Lean_Parser_Term_doHav lean_mark_persistent(l_Lean_Parser_Term_doHave_formatter___closed__4); l_Lean_Parser_Term_doHave_formatter___closed__5 = _init_l_Lean_Parser_Term_doHave_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_doHave_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doHave_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doHave_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doHave_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doHave_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doHave_parenthesizer___closed__1); l_Lean_Parser_Term_doHave_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doHave_parenthesizer___closed__2(); @@ -34750,6 +37374,13 @@ l_Lean_Parser_Term_doHave_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_d lean_mark_persistent(l_Lean_Parser_Term_doHave_parenthesizer___closed__4); l_Lean_Parser_Term_doHave_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_doHave_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_doHave_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doHave_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_elseIf___elambda__1___lambda__1___closed__1 = _init_l_Lean_Parser_Term_elseIf___elambda__1___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_elseIf___elambda__1___lambda__1___closed__1); l_Lean_Parser_Term_elseIf___elambda__1___closed__1 = _init_l_Lean_Parser_Term_elseIf___elambda__1___closed__1(); @@ -35058,6 +37689,13 @@ l_Lean_Parser_Term_doIfLetPure_formatter___closed__2 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_doIfLetPure_formatter___closed__2); l_Lean_Parser_Term_doIfLetPure_formatter___closed__3 = _init_l_Lean_Parser_Term_doIfLetPure_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doIfLetPure_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIfLetPure_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfLetBind_formatter___closed__1 = _init_l_Lean_Parser_Term_doIfLetBind_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfLetBind_formatter___closed__1); l_Lean_Parser_Term_doIfLetBind_formatter___closed__2 = _init_l_Lean_Parser_Term_doIfLetBind_formatter___closed__2(); @@ -35066,6 +37704,13 @@ l_Lean_Parser_Term_doIfLetBind_formatter___closed__3 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_doIfLetBind_formatter___closed__3); l_Lean_Parser_Term_doIfLetBind_formatter___closed__4 = _init_l_Lean_Parser_Term_doIfLetBind_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doIfLetBind_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIfLetBind_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfLet_formatter___closed__1 = _init_l_Lean_Parser_Term_doIfLet_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfLet_formatter___closed__1); l_Lean_Parser_Term_doIfLet_formatter___closed__2 = _init_l_Lean_Parser_Term_doIfLet_formatter___closed__2(); @@ -35076,10 +37721,13 @@ l_Lean_Parser_Term_doIfLet_formatter___closed__4 = _init_l_Lean_Parser_Term_doIf lean_mark_persistent(l_Lean_Parser_Term_doIfLet_formatter___closed__4); l_Lean_Parser_Term_doIfLet_formatter___closed__5 = _init_l_Lean_Parser_Term_doIfLet_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_doIfLet_formatter___closed__5); -l_Lean_Parser_Term_doIfLet_formatter___closed__6 = _init_l_Lean_Parser_Term_doIfLet_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_doIfLet_formatter___closed__6); -l_Lean_Parser_Term_doIfLet_formatter___closed__7 = _init_l_Lean_Parser_Term_doIfLet_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_doIfLet_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLet_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIfLet_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfProp_formatter___closed__1 = _init_l_Lean_Parser_Term_doIfProp_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfProp_formatter___closed__1); l_Lean_Parser_Term_doIfProp_formatter___closed__2 = _init_l_Lean_Parser_Term_doIfProp_formatter___closed__2(); @@ -35088,14 +37736,17 @@ l_Lean_Parser_Term_doIfProp_formatter___closed__3 = _init_l_Lean_Parser_Term_doI lean_mark_persistent(l_Lean_Parser_Term_doIfProp_formatter___closed__3); l_Lean_Parser_Term_doIfProp_formatter___closed__4 = _init_l_Lean_Parser_Term_doIfProp_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doIfProp_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfProp_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIfProp_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfCond_formatter___closed__1 = _init_l_Lean_Parser_Term_doIfCond_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfCond_formatter___closed__1); l_Lean_Parser_Term_doIfCond_formatter___closed__2 = _init_l_Lean_Parser_Term_doIfCond_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doIfCond_formatter___closed__2); -l_Lean_Parser_Term_doIfCond_formatter___closed__3 = _init_l_Lean_Parser_Term_doIfCond_formatter___closed__3(); -lean_mark_persistent(l_Lean_Parser_Term_doIfCond_formatter___closed__3); -l_Lean_Parser_Term_doIfCond_formatter___closed__4 = _init_l_Lean_Parser_Term_doIfCond_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Term_doIfCond_formatter___closed__4); l_Lean_Parser_Term_elseIf_formatter___closed__1 = _init_l_Lean_Parser_Term_elseIf_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_elseIf_formatter___closed__1); l_Lean_Parser_Term_elseIf_formatter___closed__2 = _init_l_Lean_Parser_Term_elseIf_formatter___closed__2(); @@ -35152,12 +37803,26 @@ l_Lean_Parser_Term_doIf_formatter___closed__21 = _init_l_Lean_Parser_Term_doIf_f lean_mark_persistent(l_Lean_Parser_Term_doIf_formatter___closed__21); l_Lean_Parser_Term_doIf_formatter___closed__22 = _init_l_Lean_Parser_Term_doIf_formatter___closed__22(); lean_mark_persistent(l_Lean_Parser_Term_doIf_formatter___closed__22); +l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIf_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIf_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1); l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2); l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIfLetPure_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1); l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2(); @@ -35166,6 +37831,13 @@ l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__3 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__3); l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIfLetBind_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfLet_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfLet_parenthesizer___closed__1); l_Lean_Parser_Term_doIfLet_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__2(); @@ -35176,10 +37848,13 @@ l_Lean_Parser_Term_doIfLet_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_doIfLet_parenthesizer___closed__4); l_Lean_Parser_Term_doIfLet_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_doIfLet_parenthesizer___closed__5); -l_Lean_Parser_Term_doIfLet_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_doIfLet_parenthesizer___closed__6); -l_Lean_Parser_Term_doIfLet_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_doIfLet_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_doIfLet_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIfLet_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfProp_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doIfProp_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfProp_parenthesizer___closed__1); l_Lean_Parser_Term_doIfProp_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doIfProp_parenthesizer___closed__2(); @@ -35188,14 +37863,17 @@ l_Lean_Parser_Term_doIfProp_parenthesizer___closed__3 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_doIfProp_parenthesizer___closed__3); l_Lean_Parser_Term_doIfProp_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_doIfProp_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doIfProp_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIfProp_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doIfCond_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doIfCond_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doIfCond_parenthesizer___closed__1); l_Lean_Parser_Term_doIfCond_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doIfCond_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doIfCond_parenthesizer___closed__2); -l_Lean_Parser_Term_doIfCond_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_doIfCond_parenthesizer___closed__3(); -lean_mark_persistent(l_Lean_Parser_Term_doIfCond_parenthesizer___closed__3); -l_Lean_Parser_Term_doIfCond_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_doIfCond_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Term_doIfCond_parenthesizer___closed__4); l_Lean_Parser_Term_elseIf_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_elseIf_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_elseIf_parenthesizer___closed__1); l_Lean_Parser_Term_elseIf_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_elseIf_parenthesizer___closed__2(); @@ -35252,6 +37930,13 @@ l_Lean_Parser_Term_doIf_parenthesizer___closed__21 = _init_l_Lean_Parser_Term_do lean_mark_persistent(l_Lean_Parser_Term_doIf_parenthesizer___closed__21); l_Lean_Parser_Term_doIf_parenthesizer___closed__22 = _init_l_Lean_Parser_Term_doIf_parenthesizer___closed__22(); lean_mark_persistent(l_Lean_Parser_Term_doIf_parenthesizer___closed__22); +l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doIf_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doUnless___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doUnless___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doUnless___elambda__1___closed__1); l_Lean_Parser_Term_doUnless___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doUnless___elambda__1___closed__2(); @@ -35340,6 +38025,13 @@ l_Lean_Parser_Term_doUnless_formatter___closed__7 = _init_l_Lean_Parser_Term_doU lean_mark_persistent(l_Lean_Parser_Term_doUnless_formatter___closed__7); l_Lean_Parser_Term_doUnless_formatter___closed__8 = _init_l_Lean_Parser_Term_doUnless_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_doUnless_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doUnless_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doUnless_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doUnless_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doUnless_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doUnless_parenthesizer___closed__1); l_Lean_Parser_Term_doUnless_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doUnless_parenthesizer___closed__2(); @@ -35356,6 +38048,13 @@ l_Lean_Parser_Term_doUnless_parenthesizer___closed__7 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_doUnless_parenthesizer___closed__7); l_Lean_Parser_Term_doUnless_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_doUnless_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_doUnless_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doUnless_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doForDecl___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doForDecl___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doForDecl___elambda__1___closed__1); l_Lean_Parser_Term_doForDecl___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doForDecl___elambda__1___closed__2(); @@ -35524,6 +38223,13 @@ l_Lean_Parser_Term_doForDecl_formatter___closed__9 = _init_l_Lean_Parser_Term_do lean_mark_persistent(l_Lean_Parser_Term_doForDecl_formatter___closed__9); l_Lean_Parser_Term_doForDecl_formatter___closed__10 = _init_l_Lean_Parser_Term_doForDecl_formatter___closed__10(); lean_mark_persistent(l_Lean_Parser_Term_doForDecl_formatter___closed__10); +l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doForDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doForDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doFor_formatter___closed__1 = _init_l_Lean_Parser_Term_doFor_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doFor_formatter___closed__1); l_Lean_Parser_Term_doFor_formatter___closed__2 = _init_l_Lean_Parser_Term_doFor_formatter___closed__2(); @@ -35538,8 +38244,13 @@ l_Lean_Parser_Term_doFor_formatter___closed__6 = _init_l_Lean_Parser_Term_doFor_ lean_mark_persistent(l_Lean_Parser_Term_doFor_formatter___closed__6); l_Lean_Parser_Term_doFor_formatter___closed__7 = _init_l_Lean_Parser_Term_doFor_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doFor_formatter___closed__7); -l_Lean_Parser_Term_doFor_formatter___closed__8 = _init_l_Lean_Parser_Term_doFor_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_doFor_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doFor_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doFor_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doForDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doForDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doForDecl_parenthesizer___closed__1); l_Lean_Parser_Term_doForDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doForDecl_parenthesizer___closed__2(); @@ -35560,6 +38271,13 @@ l_Lean_Parser_Term_doForDecl_parenthesizer___closed__9 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_doForDecl_parenthesizer___closed__9); l_Lean_Parser_Term_doForDecl_parenthesizer___closed__10 = _init_l_Lean_Parser_Term_doForDecl_parenthesizer___closed__10(); lean_mark_persistent(l_Lean_Parser_Term_doForDecl_parenthesizer___closed__10); +l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doForDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doFor_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doFor_parenthesizer___closed__1); l_Lean_Parser_Term_doFor_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__2(); @@ -35574,8 +38292,13 @@ l_Lean_Parser_Term_doFor_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_do lean_mark_persistent(l_Lean_Parser_Term_doFor_parenthesizer___closed__6); l_Lean_Parser_Term_doFor_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doFor_parenthesizer___closed__7); -l_Lean_Parser_Term_doFor_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_doFor_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_doFor_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doFor_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doMatchAlts___closed__1 = _init_l_Lean_Parser_Term_doMatchAlts___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doMatchAlts___closed__1); l_Lean_Parser_Term_doMatchAlts = _init_l_Lean_Parser_Term_doMatchAlts(); @@ -35714,6 +38437,13 @@ l_Lean_Parser_Term_doMatch_formatter___closed__15 = _init_l_Lean_Parser_Term_doM lean_mark_persistent(l_Lean_Parser_Term_doMatch_formatter___closed__15); l_Lean_Parser_Term_doMatch_formatter___closed__16 = _init_l_Lean_Parser_Term_doMatch_formatter___closed__16(); lean_mark_persistent(l_Lean_Parser_Term_doMatch_formatter___closed__16); +l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doMatch_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doMatch_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doMatch_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doMatch_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doMatch_parenthesizer___closed__1); l_Lean_Parser_Term_doMatch_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doMatch_parenthesizer___closed__2(); @@ -35746,6 +38476,13 @@ l_Lean_Parser_Term_doMatch_parenthesizer___closed__15 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_doMatch_parenthesizer___closed__15); l_Lean_Parser_Term_doMatch_parenthesizer___closed__16 = _init_l_Lean_Parser_Term_doMatch_parenthesizer___closed__16(); lean_mark_persistent(l_Lean_Parser_Term_doMatch_parenthesizer___closed__16); +l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doMatch_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doCatch___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doCatch___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doCatch___elambda__1___closed__1); l_Lean_Parser_Term_doCatch___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doCatch___elambda__1___closed__2(); @@ -35990,12 +38727,26 @@ l_Lean_Parser_Term_doCatch_formatter___closed__11 = _init_l_Lean_Parser_Term_doC lean_mark_persistent(l_Lean_Parser_Term_doCatch_formatter___closed__11); l_Lean_Parser_Term_doCatch_formatter___closed__12 = _init_l_Lean_Parser_Term_doCatch_formatter___closed__12(); lean_mark_persistent(l_Lean_Parser_Term_doCatch_formatter___closed__12); +l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doCatch_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doCatch_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doCatchMatch_formatter___closed__1 = _init_l_Lean_Parser_Term_doCatchMatch_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doCatchMatch_formatter___closed__1); l_Lean_Parser_Term_doCatchMatch_formatter___closed__2 = _init_l_Lean_Parser_Term_doCatchMatch_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doCatchMatch_formatter___closed__2); l_Lean_Parser_Term_doCatchMatch_formatter___closed__3 = _init_l_Lean_Parser_Term_doCatchMatch_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doCatchMatch_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doCatchMatch_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doFinally_formatter___closed__1 = _init_l_Lean_Parser_Term_doFinally_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doFinally_formatter___closed__1); l_Lean_Parser_Term_doFinally_formatter___closed__2 = _init_l_Lean_Parser_Term_doFinally_formatter___closed__2(); @@ -36004,6 +38755,13 @@ l_Lean_Parser_Term_doFinally_formatter___closed__3 = _init_l_Lean_Parser_Term_do lean_mark_persistent(l_Lean_Parser_Term_doFinally_formatter___closed__3); l_Lean_Parser_Term_doFinally_formatter___closed__4 = _init_l_Lean_Parser_Term_doFinally_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doFinally_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doFinally_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doFinally_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doTry_formatter___closed__1 = _init_l_Lean_Parser_Term_doTry_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doTry_formatter___closed__1); l_Lean_Parser_Term_doTry_formatter___closed__2 = _init_l_Lean_Parser_Term_doTry_formatter___closed__2(); @@ -36022,12 +38780,13 @@ l_Lean_Parser_Term_doTry_formatter___closed__8 = _init_l_Lean_Parser_Term_doTry_ lean_mark_persistent(l_Lean_Parser_Term_doTry_formatter___closed__8); l_Lean_Parser_Term_doTry_formatter___closed__9 = _init_l_Lean_Parser_Term_doTry_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_doTry_formatter___closed__9); -l_Lean_Parser_Term_doTry_formatter___closed__10 = _init_l_Lean_Parser_Term_doTry_formatter___closed__10(); -lean_mark_persistent(l_Lean_Parser_Term_doTry_formatter___closed__10); -l_Lean_Parser_Term_doTry_formatter___closed__11 = _init_l_Lean_Parser_Term_doTry_formatter___closed__11(); -lean_mark_persistent(l_Lean_Parser_Term_doTry_formatter___closed__11); -l_Lean_Parser_Term_doTry_formatter___closed__12 = _init_l_Lean_Parser_Term_doTry_formatter___closed__12(); -lean_mark_persistent(l_Lean_Parser_Term_doTry_formatter___closed__12); +l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doTry_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doTry_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doCatch_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doCatch_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doCatch_parenthesizer___closed__1); l_Lean_Parser_Term_doCatch_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doCatch_parenthesizer___closed__2(); @@ -36052,12 +38811,26 @@ l_Lean_Parser_Term_doCatch_parenthesizer___closed__11 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_doCatch_parenthesizer___closed__11); l_Lean_Parser_Term_doCatch_parenthesizer___closed__12 = _init_l_Lean_Parser_Term_doCatch_parenthesizer___closed__12(); lean_mark_persistent(l_Lean_Parser_Term_doCatch_parenthesizer___closed__12); +l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doCatch_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1); l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2); l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doCatchMatch_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doFinally_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doFinally_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doFinally_parenthesizer___closed__1); l_Lean_Parser_Term_doFinally_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doFinally_parenthesizer___closed__2(); @@ -36066,6 +38839,13 @@ l_Lean_Parser_Term_doFinally_parenthesizer___closed__3 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_doFinally_parenthesizer___closed__3); l_Lean_Parser_Term_doFinally_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_doFinally_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doFinally_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doFinally_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doTry_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doTry_parenthesizer___closed__1); l_Lean_Parser_Term_doTry_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__2(); @@ -36084,12 +38864,13 @@ l_Lean_Parser_Term_doTry_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_do lean_mark_persistent(l_Lean_Parser_Term_doTry_parenthesizer___closed__8); l_Lean_Parser_Term_doTry_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_doTry_parenthesizer___closed__9); -l_Lean_Parser_Term_doTry_parenthesizer___closed__10 = _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__10(); -lean_mark_persistent(l_Lean_Parser_Term_doTry_parenthesizer___closed__10); -l_Lean_Parser_Term_doTry_parenthesizer___closed__11 = _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__11(); -lean_mark_persistent(l_Lean_Parser_Term_doTry_parenthesizer___closed__11); -l_Lean_Parser_Term_doTry_parenthesizer___closed__12 = _init_l_Lean_Parser_Term_doTry_parenthesizer___closed__12(); -lean_mark_persistent(l_Lean_Parser_Term_doTry_parenthesizer___closed__12); +l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doTry_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doBreak___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doBreak___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doBreak___elambda__1___closed__1); l_Lean_Parser_Term_doBreak___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doBreak___elambda__1___closed__2(); @@ -36154,12 +38935,26 @@ l_Lean_Parser_Term_doBreak_formatter___closed__2 = _init_l_Lean_Parser_Term_doBr lean_mark_persistent(l_Lean_Parser_Term_doBreak_formatter___closed__2); l_Lean_Parser_Term_doBreak_formatter___closed__3 = _init_l_Lean_Parser_Term_doBreak_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doBreak_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doBreak_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doBreak_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doBreak_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doBreak_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doBreak_parenthesizer___closed__1); l_Lean_Parser_Term_doBreak_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doBreak_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doBreak_parenthesizer___closed__2); l_Lean_Parser_Term_doBreak_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_doBreak_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doBreak_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doBreak_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doContinue___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doContinue___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doContinue___elambda__1___closed__1); l_Lean_Parser_Term_doContinue___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doContinue___elambda__1___closed__2(); @@ -36224,12 +39019,26 @@ l_Lean_Parser_Term_doContinue_formatter___closed__2 = _init_l_Lean_Parser_Term_d lean_mark_persistent(l_Lean_Parser_Term_doContinue_formatter___closed__2); l_Lean_Parser_Term_doContinue_formatter___closed__3 = _init_l_Lean_Parser_Term_doContinue_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doContinue_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doContinue_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doContinue_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doContinue_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doContinue_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doContinue_parenthesizer___closed__1); l_Lean_Parser_Term_doContinue_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doContinue_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doContinue_parenthesizer___closed__2); l_Lean_Parser_Term_doContinue_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_doContinue_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_doContinue_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doContinue_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doReturn___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doReturn___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doReturn___elambda__1___closed__1); l_Lean_Parser_Term_doReturn___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doReturn___elambda__1___closed__2(); @@ -36306,6 +39115,13 @@ l_Lean_Parser_Term_doReturn_formatter___closed__6 = _init_l_Lean_Parser_Term_doR lean_mark_persistent(l_Lean_Parser_Term_doReturn_formatter___closed__6); l_Lean_Parser_Term_doReturn_formatter___closed__7 = _init_l_Lean_Parser_Term_doReturn_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doReturn_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReturn_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doReturn_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doReturn_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doReturn_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doReturn_parenthesizer___closed__1); l_Lean_Parser_Term_doReturn_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doReturn_parenthesizer___closed__2(); @@ -36320,6 +39136,13 @@ l_Lean_Parser_Term_doReturn_parenthesizer___closed__6 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_doReturn_parenthesizer___closed__6); l_Lean_Parser_Term_doReturn_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_doReturn_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doReturn_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doReturn_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__1); l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doDbgTrace___elambda__1___closed__2(); @@ -36400,6 +39223,13 @@ l_Lean_Parser_Term_doDbgTrace_formatter___closed__5 = _init_l_Lean_Parser_Term_d lean_mark_persistent(l_Lean_Parser_Term_doDbgTrace_formatter___closed__5); l_Lean_Parser_Term_doDbgTrace_formatter___closed__6 = _init_l_Lean_Parser_Term_doDbgTrace_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_doDbgTrace_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doDbgTrace_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1); l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2(); @@ -36412,6 +39242,13 @@ l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__5 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__5); l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doDbgTrace_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doAssert___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doAssert___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doAssert___elambda__1___closed__1); l_Lean_Parser_Term_doAssert___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doAssert___elambda__1___closed__2(); @@ -36482,6 +39319,13 @@ l_Lean_Parser_Term_doAssert_formatter___closed__3 = _init_l_Lean_Parser_Term_doA lean_mark_persistent(l_Lean_Parser_Term_doAssert_formatter___closed__3); l_Lean_Parser_Term_doAssert_formatter___closed__4 = _init_l_Lean_Parser_Term_doAssert_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doAssert_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doAssert_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doAssert_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doAssert_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doAssert_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doAssert_parenthesizer___closed__1); l_Lean_Parser_Term_doAssert_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doAssert_parenthesizer___closed__2(); @@ -36490,6 +39334,13 @@ l_Lean_Parser_Term_doAssert_parenthesizer___closed__3 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_doAssert_parenthesizer___closed__3); l_Lean_Parser_Term_doAssert_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_doAssert_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_doAssert_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doAssert_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doExpr___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doExpr___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doExpr___elambda__1___closed__1); l_Lean_Parser_Term_doExpr___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doExpr___elambda__1___closed__2(); @@ -36590,6 +39441,13 @@ l_Lean_Parser_Term_doExpr_formatter___closed__9 = _init_l_Lean_Parser_Term_doExp lean_mark_persistent(l_Lean_Parser_Term_doExpr_formatter___closed__9); l_Lean_Parser_Term_doExpr_formatter___closed__10 = _init_l_Lean_Parser_Term_doExpr_formatter___closed__10(); lean_mark_persistent(l_Lean_Parser_Term_doExpr_formatter___closed__10); +l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doExpr_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doExpr_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doExpr_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doExpr_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doExpr_parenthesizer___closed__1); l_Lean_Parser_Term_doExpr_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doExpr_parenthesizer___closed__2(); @@ -36610,6 +39468,13 @@ l_Lean_Parser_Term_doExpr_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_d lean_mark_persistent(l_Lean_Parser_Term_doExpr_parenthesizer___closed__9); l_Lean_Parser_Term_doExpr_parenthesizer___closed__10 = _init_l_Lean_Parser_Term_doExpr_parenthesizer___closed__10(); lean_mark_persistent(l_Lean_Parser_Term_doExpr_parenthesizer___closed__10); +l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doExpr_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doNested___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doNested___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doNested___elambda__1___closed__1); l_Lean_Parser_Term_doNested___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doNested___elambda__1___closed__2(); @@ -36660,10 +39525,24 @@ l_Lean_Parser_Term_doNested_formatter___closed__1 = _init_l_Lean_Parser_Term_doN lean_mark_persistent(l_Lean_Parser_Term_doNested_formatter___closed__1); l_Lean_Parser_Term_doNested_formatter___closed__2 = _init_l_Lean_Parser_Term_doNested_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doNested_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doNested_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doNested_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doNested_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doNested_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doNested_parenthesizer___closed__1); l_Lean_Parser_Term_doNested_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doNested_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_doNested_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doNested_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_do___elambda__1___closed__1 = _init_l_Lean_Parser_Term_do___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_do___elambda__1___closed__1); l_Lean_Parser_Term_do___elambda__1___closed__2 = _init_l_Lean_Parser_Term_do___elambda__1___closed__2(); @@ -36724,6 +39603,13 @@ l_Lean_Parser_Term_do_formatter___closed__3 = _init_l_Lean_Parser_Term_do_format lean_mark_persistent(l_Lean_Parser_Term_do_formatter___closed__3); l_Lean_Parser_Term_do_formatter___closed__4 = _init_l_Lean_Parser_Term_do_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_do_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_do_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_do_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_do_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_do_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_do_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_do_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_do_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_do_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_do_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_do_parenthesizer___closed__1); l_Lean_Parser_Term_do_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_do_parenthesizer___closed__2(); @@ -36732,6 +39618,13 @@ l_Lean_Parser_Term_do_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_do_pa lean_mark_persistent(l_Lean_Parser_Term_do_parenthesizer___closed__3); l_Lean_Parser_Term_do_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_do_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_do_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_do_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_do_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doElem_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doElem_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doElem_quot___elambda__1___closed__1); l_Lean_Parser_Term_doElem_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doElem_quot___elambda__1___closed__2(); @@ -36830,6 +39723,13 @@ l_Lean_Parser_Term_doElem_quot_formatter___closed__6 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_doElem_quot_formatter___closed__6); l_Lean_Parser_Term_doElem_quot_formatter___closed__7 = _init_l_Lean_Parser_Term_doElem_quot_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doElem_quot_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doElem_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1); l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__2(); @@ -36844,6 +39744,13 @@ l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__6 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__6); l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_doElem_quot_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doElem_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_termUnless___elambda__1___closed__1 = _init_l_Lean_Parser_Term_termUnless___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_termUnless___elambda__1___closed__1); l_Lean_Parser_Term_termUnless___elambda__1___closed__2 = _init_l_Lean_Parser_Term_termUnless___elambda__1___closed__2(); @@ -36898,10 +39805,24 @@ l_Lean_Parser_Term_termUnless_formatter___closed__1 = _init_l_Lean_Parser_Term_t lean_mark_persistent(l_Lean_Parser_Term_termUnless_formatter___closed__1); l_Lean_Parser_Term_termUnless_formatter___closed__2 = _init_l_Lean_Parser_Term_termUnless_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_termUnless_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termUnless_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_termUnless_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_termUnless_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_termUnless_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_termUnless_parenthesizer___closed__1); l_Lean_Parser_Term_termUnless_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_termUnless_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_termUnless_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_termUnless_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_termFor___elambda__1___closed__1 = _init_l_Lean_Parser_Term_termFor___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_termFor___elambda__1___closed__1); l_Lean_Parser_Term_termFor___elambda__1___closed__2 = _init_l_Lean_Parser_Term_termFor___elambda__1___closed__2(); @@ -36952,10 +39873,24 @@ l_Lean_Parser_Term_termFor_formatter___closed__1 = _init_l_Lean_Parser_Term_term lean_mark_persistent(l_Lean_Parser_Term_termFor_formatter___closed__1); l_Lean_Parser_Term_termFor_formatter___closed__2 = _init_l_Lean_Parser_Term_termFor_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_termFor_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termFor_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_termFor_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_termFor_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_termFor_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_termFor_parenthesizer___closed__1); l_Lean_Parser_Term_termFor_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_termFor_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_termFor_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_termFor_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_termTry___elambda__1___closed__1 = _init_l_Lean_Parser_Term_termTry___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_termTry___elambda__1___closed__1); l_Lean_Parser_Term_termTry___elambda__1___closed__2 = _init_l_Lean_Parser_Term_termTry___elambda__1___closed__2(); @@ -37006,10 +39941,24 @@ l_Lean_Parser_Term_termTry_formatter___closed__1 = _init_l_Lean_Parser_Term_term lean_mark_persistent(l_Lean_Parser_Term_termTry_formatter___closed__1); l_Lean_Parser_Term_termTry_formatter___closed__2 = _init_l_Lean_Parser_Term_termTry_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_termTry_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termTry_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_termTry_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_termTry_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_termTry_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_termTry_parenthesizer___closed__1); l_Lean_Parser_Term_termTry_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_termTry_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_termTry_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_termTry_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_termReturn___elambda__1___closed__1 = _init_l_Lean_Parser_Term_termReturn___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_termReturn___elambda__1___closed__1); l_Lean_Parser_Term_termReturn___elambda__1___closed__2 = _init_l_Lean_Parser_Term_termReturn___elambda__1___closed__2(); @@ -37062,10 +40011,24 @@ l_Lean_Parser_Term_termReturn_formatter___closed__1 = _init_l_Lean_Parser_Term_t lean_mark_persistent(l_Lean_Parser_Term_termReturn_formatter___closed__1); l_Lean_Parser_Term_termReturn_formatter___closed__2 = _init_l_Lean_Parser_Term_termReturn_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_termReturn_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termReturn_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_termReturn_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_termReturn_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_termReturn_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_termReturn_parenthesizer___closed__1); l_Lean_Parser_Term_termReturn_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_termReturn_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_termReturn_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_termReturn_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Parser/Extension.c b/stage0/stdlib/Lean/Parser/Extension.c index 525d8c04d364..7497d721cd62 100644 --- a/stage0/stdlib/Lean/Parser/Extension.c +++ b/stage0/stdlib/Lean/Parser/Extension.c @@ -19,7 +19,6 @@ uint8_t l_Lean_isRecCore(lean_object*, lean_object*); static lean_object* l_Lean_Parser_declareLeadingBuiltinParser___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_builtinTokenTable; static lean_object* l_Lean_Parser_parserOfStackFn___lambda__2___closed__5; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__4; lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContextCoreM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KVMap_setBool(lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Parser_getParserAliasInfo___closed__2; @@ -99,11 +98,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_mkParserState(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_addToken___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_6____closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__2; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_80____closed__9; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__1; extern lean_object* l_Lean_declRangeExt; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__4___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_registerBuiltinDynamicParserAttribute(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_getConstAlias___rarg___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_forM___at___private_Lean_Parser_Extension_0__Lean_Parser_ParserAttribute_add___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -125,7 +124,6 @@ static lean_object* l_Lean_findDeclarationRangesCore_x3f___at___private_Lean_Par static lean_object* l_Lean_Parser_isParserCategory___closed__1; LEAN_EXPORT uint8_t l_Std_PersistentHashMap_contains___at_Lean_Parser_isValidSyntaxNodeKind___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_declareBuiltinParser___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_registerAliasCore(lean_object*); static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_categoryParserFnImpl(lean_object*, lean_object*, lean_object*); @@ -134,13 +132,17 @@ static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3468 LEAN_EXPORT lean_object* l_IO_ofExcept___at_Lean_Parser_mkParserOfConstantUnsafe___spec__2___boxed(lean_object*, lean_object*); lean_object* l_Lean_Parser_checkPrecFn___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_leadingParserAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Parser_evalParserConstUnsafe___spec__1(lean_object*, lean_object*); size_t lean_usize_shift_right(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Parser_getParserAliasInfo___boxed(lean_object*, lean_object*); lean_object* l_Lean_ScopedEnvExtension_addScopedEntry___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Parser_Extension_0__Lean_Parser_ParserAttribute_add___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkParserState___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__1; static lean_object* l_Lean_Parser_parserOfStackFn___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_isParserCategory___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_foldlMAux___at_Lean_Parser_getSyntaxNodeKinds___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_evalInsideQuot___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_findDeclarationRangesCore_x3f___at___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -181,8 +183,8 @@ static lean_object* l_Lean_Parser_parserOfStack___closed__1; uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_throwUnknownParserCategory___rarg___closed__1; static lean_object* l_Lean_findDeclarationRanges_x3f___at___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___spec__1___lambda__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__4; lean_object* l_Lean_MapDeclarationExtension_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__2; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAux___at___private_Lean_Parser_Extension_0__Lean_Parser_addParserCategoryCore___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Parser_addToken___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_declareTrailingBuiltinParser___closed__2; @@ -191,11 +193,9 @@ static size_t l_Std_PersistentHashMap_containsAux___at___private_Lean_Parser_Ext LEAN_EXPORT lean_object* l_Lean_Parser_addSyntaxNodeKind(lean_object*, lean_object*); uint64_t l_Lean_Name_hash___override(lean_object*); LEAN_EXPORT lean_object* l_IO_ofExcept___at_Lean_Parser_mkParserOfConstantUnsafe___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_compileParserDescr_visit___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3419____closed__5; static lean_object* l_List_forM___at___private_Lean_Parser_Extension_0__Lean_Parser_ParserAttribute_add___spec__1___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__4; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__2___closed__17; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__4___closed__1; static lean_object* l_Lean_Parser_withOpenDeclFnCore___closed__4; @@ -204,7 +204,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_internal_parseQuotWithCurrentStage; lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Syntax_isNatLit_x3f(lean_object*); uint8_t l_Lean_Option_get___at_Lean_getSanitizeNames___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__3; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); uint8_t l___private_Lean_Attributes_0__Lean_beqAttributeKind____x40_Lean_Attributes___hyg_135_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Parser_getBinaryAlias___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -212,8 +211,12 @@ lean_object* l_Lean_Parser_nonReservedSymbolFnAux(lean_object*, lean_object*, le static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_updateBuiltinTokens___closed__2; static lean_object* l_Lean_Parser_declareLeadingBuiltinParser___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_ParserAttribute_add___boxed(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__3; +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1(lean_object*); static lean_object* l_Lean_Parser_ParserExtension_addEntryImpl___closed__4; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__3___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__4; LEAN_EXPORT lean_object* l_IO_ofExcept___at_Lean_Parser_mkParserOfConstantUnsafe___spec__2(lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_Parser_nodeInfo(lean_object*, lean_object*); @@ -234,7 +237,6 @@ static lean_object* l_Lean_Parser_mkParserOfConstantUnsafe___closed__1; lean_object* l_Lean_Parser_nonReservedSymbolInfo(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Parser_ParserExtension_instInhabitedState; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Parser_Extension_0__Lean_Parser_addParserCategoryCore___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__4; lean_object* l_Lean_mkRawNatLit(lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Parser_Extension_0__Lean_Parser_ParserAttribute_add___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_ParserContext_resolveName(lean_object*, lean_object*); @@ -249,16 +251,16 @@ LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3329_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3419_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3468_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_2028_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_1990_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_2066_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_189_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_6_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_80_(lean_object*); @@ -291,6 +293,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_Parser uint8_t l_Lean_Name_quickCmp(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_instCoeForAllParserParserAliasValue(lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3419____lambda__2___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__2; lean_object* l_Lean_Name_toExprAux(lean_object*); static lean_object* l_Lean_Parser_mkParserOfConstantUnsafe___closed__4; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_80____closed__13; @@ -300,9 +303,10 @@ LEAN_EXPORT lean_object* l_Lean_Parser_parserOfStackFn___lambda__1(lean_object*, LEAN_EXPORT lean_object* l_Lean_Parser_addToken(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ofExcept___at_Lean_Parser_addToken___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_categoryParserFnImpl___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_registerBuiltinParserAttribute___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_registerAlias___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__1; lean_object* l_Lean_Attribute_Builtin_getPrio(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_runParserCategory___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_parserAliasesRef; @@ -314,7 +318,6 @@ LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at_Lean_Parser_getCa LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_withNamespaces___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Parser_Extension_0__Lean_Parser_withNamespaces___spec__1(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Parser_Extension_0__Lean_Parser_addTrailingParserAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__1; static lean_object* l_Lean_Parser_mkParserAttributeImpl___closed__1; lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_registerAlias___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -346,7 +349,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_addParserTokens(lean_object*, lean_object uint32_t lean_string_utf8_get(lean_object*, lean_object*); static lean_object* l_Lean_findDeclarationRanges_x3f___at___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___spec__1___closed__1; static uint8_t l_Lean_Parser_isValidSyntaxNodeKind___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__2; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3641____closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_parserOfStack(lean_object*, lean_object*); static lean_object* l_Lean_Parser_registerAliasCore___rarg___closed__1; @@ -354,7 +356,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_getAlias(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_addParserCategory___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_registerBuiltinParserAttribute(lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3468____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_foldlMAux_traverse___at___private_Lean_Parser_Extension_0__Lean_Parser_ParserAttribute_add___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_80____closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -373,6 +374,7 @@ static lean_object* l_Lean_Parser_getParserPriority___closed__4; static lean_object* l_Lean_Parser_parserOfStackFn___lambda__1___closed__1; static lean_object* l_Lean_Parser_withOpenDeclFnCore___closed__6; static lean_object* l_Lean_Parser_mkParserOfConstantUnsafe___closed__6; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_parserAlias2kindRef; LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Parser_getParserAliasInfo___spec__1(lean_object*, lean_object*); size_t lean_usize_mul(size_t, size_t); @@ -392,6 +394,7 @@ LEAN_EXPORT uint8_t l_Std_PersistentHashMap_containsAtAux___at_Lean_Parser_isVal LEAN_EXPORT lean_object* l_Lean_Parser_isValidSyntaxNodeKind___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Parser_Extension_0__Lean_Parser_withNamespaces___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ParserExtension_instInhabitedEntry; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_registerAlias(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_isParserAlias___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Parser_addLeadingParser___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -404,6 +407,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_mkParserAttributeImpl___elambda__2___rarg lean_object* l_Lean_Parser_trailingNodeFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__2___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_addBuiltinLeadingParser(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__1; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3641____closed__3; lean_object* l_Lean_ScopedEnvExtension_getState___rarg(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); @@ -428,23 +432,29 @@ LEAN_EXPORT lean_object* l_Lean_Parser_declareLeadingBuiltinParser(lean_object*, LEAN_EXPORT lean_object* l_Lean_Parser_compileParserDescr_visit(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_registerParserCategory(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); lean_object* l_Lean_Parser_nodeWithAntiquot(lean_object*, lean_object*, lean_object*, uint8_t); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_getAlias___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_trailingLoop(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__1; uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l_Lean_Parser_throwUnknownParserCategory___rarg___closed__2; LEAN_EXPORT uint8_t l_Std_PersistentHashMap_containsAux___at___private_Lean_Parser_Extension_0__Lean_Parser_addParserCategoryCore___spec__2(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Parser_Extension_0__Lean_Parser_addParserCategoryCore___spec__6(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_getUnaryAlias___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__2; LEAN_EXPORT lean_object* l_List_forM___at_Lean_Parser_runParserAttributeHooks___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_parserOfStackFn___lambda__2___closed__7; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_withOpenDecl(lean_object*); static lean_object* l_Lean_Parser_registerAlias___closed__1; lean_object* l_Std_RBNode_find___at_Lean_findDeclarationRanges_x3f___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__1; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_80____closed__14; lean_object* l_Lean_Option_register___at_Std_Format_initFn____x40_Lean_Data_Format___hyg_57____spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_registerAliasCore___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3419____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_mkParserAttributeImpl___elambda__1___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getNumArgs(lean_object*); @@ -464,13 +474,12 @@ uint8_t lean_usize_dec_le(size_t, size_t); LEAN_EXPORT lean_object* l_IO_ofExcept___at___private_Lean_Parser_Extension_0__Lean_Parser_addBuiltinParserCategory___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Parser_categoryParser(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ensureConstantParserAlias(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__1; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__2___closed__14; lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__6; static lean_object* l_Lean_Parser_categoryParserFnImpl___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_mkParserAttributeImpl___elambda__1___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__1; LEAN_EXPORT uint8_t l_Std_PersistentHashMap_containsAux___at_Lean_Parser_isValidSyntaxNodeKind___spec__2(lean_object*, size_t, lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); LEAN_EXPORT uint8_t l_Lean_Parser_isValidSyntaxNodeKind(lean_object*, lean_object*); @@ -484,7 +493,7 @@ static lean_object* l_Lean_Parser_ParserExtension_addEntryImpl___closed__3; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__2___closed__13; uint8_t lean_is_aux_recursor(lean_object*, lean_object*); lean_object* l_Lean_Parser_symbolInfo(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_parserAttributeHooks; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Parser_withOpenDeclFnCore___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_updateBuiltinTokens(lean_object*, lean_object*, lean_object*); @@ -494,7 +503,6 @@ extern lean_object* l_Lean_instInhabitedDeclarationRanges; LEAN_EXPORT lean_object* l_Lean_Parser_ParserExtension_State_kinds___default; extern lean_object* l_Lean_Parser_epsilonInfo; LEAN_EXPORT lean_object* l_IO_ofExcept___at_Lean_Parser_mkParserOfConstantUnsafe___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_getParserPriority(lean_object*); static lean_object* l_Lean_Parser_ParserAliasInfo_stackSz_x3f___default___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_builtinSyntaxNodeKindSetRef; @@ -514,15 +522,14 @@ static lean_object* l_Std_PersistentHashMap_foldlMAux___at___private_Lean_Parser lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_findDeclarationRanges_x3f___at___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_runParserAttributeHooks(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__1; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Parser_ParserExtension_instInhabitedEntry___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Parser_Extension_0__Lean_Parser_ParserAttribute_add___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3419____closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__5; static lean_object* l_Lean_Parser_withOpenFn___closed__2; static lean_object* l_Lean_Parser_mkParserOfConstantUnsafe___closed__7; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Parser_Extension_0__Lean_Parser_withNamespaces___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_addTokenConfig___closed__1; LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Parser_addToken___spec__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_declareLeadingBuiltinParser___closed__3; @@ -593,17 +600,13 @@ static lean_object* l_Lean_Parser_mkParserOfConstantUnsafe___closed__5; extern lean_object* l_Lean_builtinDeclRanges; uint8_t lean_string_utf8_at_end(lean_object*, lean_object*); static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__2___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__1; LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_getAlias___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ParserExtension_Entry_toOLeanEntry(lean_object*); lean_object* l_Lean_ScopedEnvExtension_activateScoped___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__2; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_withOpenDeclFnCore(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__2; lean_object* l_Lean_Parser_Trie_find_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_getCategory(lean_object*, lean_object*); static lean_object* l_Lean_Parser_getConstAlias___rarg___closed__4; @@ -611,7 +614,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_instCoeForAllParserParserAliasValue__1(le LEAN_EXPORT lean_object* l_Std_PersistentHashMap_foldlMAux_traverse___at___private_Lean_Parser_Extension_0__Lean_Parser_ParserAttribute_add___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3468____lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_registerBuiltinNodeKind___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3419____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__2___closed__15; static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__2___closed__18; @@ -621,7 +623,6 @@ uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_evalInsideQuot(lean_object*, lean_object*); static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_addTokenConfig___closed__2; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_80____closed__10; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__3; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_contains___at_Lean_Parser_isValidSyntaxNodeKind___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_registerParserCategory___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); @@ -7910,58 +7911,162 @@ x_4 = lean_box(x_3); return x_4; } } +LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Parser_evalParserConstUnsafe___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +return x_1; +} +else +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_ctor_get(x_2, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_2, 1); +lean_inc(x_4); +lean_dec(x_2); +x_5 = lean_unsigned_to_nat(0u); +lean_inc(x_3); +x_6 = l_Lean_Parser_Trie_insert_loop___rarg(x_3, x_3, x_1, x_5); +lean_dec(x_3); +x_1 = x_6; +x_2 = x_4; +goto _start; +} +} +} LEAN_EXPORT lean_object* l_Lean_Parser_evalParserConstUnsafe(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_object* x_4; lean_object* x_5; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; x_4 = lean_ctor_get(x_2, 1); lean_inc(x_4); -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(x_4, 1); -lean_inc(x_6); +x_35 = lean_ctor_get(x_4, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_4, 1); +lean_inc(x_36); +x_37 = l_Lean_Parser_ParserExtension_instInhabitedState; +x_38 = l_Lean_Parser_isParserCategory___closed__1; +x_39 = l_Lean_ScopedEnvExtension_getState___rarg(x_37, x_38, x_35); +x_40 = lean_ctor_get(x_39, 2); +lean_inc(x_40); +lean_dec(x_39); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_35); +lean_ctor_set(x_41, 1, x_36); +x_42 = lean_box(0); +x_43 = l_Lean_Parser_mkParserOfConstant(x_40, x_1, x_41, x_42); +if (lean_obj_tag(x_43) == 0) +{ +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +lean_dec(x_43); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_5 = x_45; +goto block_34; +} +else +{ +lean_object* x_46; lean_object* x_47; +x_46 = lean_ctor_get(x_43, 0); +lean_inc(x_46); +lean_dec(x_43); +x_47 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_5 = x_47; +goto block_34; +} +block_34: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_dec(x_4); -x_7 = l_Lean_Parser_ParserExtension_instInhabitedState; -x_8 = l_Lean_Parser_isParserCategory___closed__1; -x_9 = l_Lean_ScopedEnvExtension_getState___rarg(x_7, x_8, x_5); -x_10 = lean_ctor_get(x_9, 2); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_5); -lean_ctor_set(x_11, 1, x_6); -x_12 = lean_box(0); -x_13 = l_Lean_Parser_mkParserOfConstant(x_10, x_1, x_11, x_12); -if (lean_obj_tag(x_13) == 0) +lean_dec(x_2); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_io_error_to_string(x_6); +x_8 = lean_box(0); +x_9 = l_Lean_Parser_ParserState_mkUnexpectedError(x_3, x_7, x_8); +return x_9; +} +else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_13, 0); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_2, 2); +lean_inc(x_13); +x_14 = lean_ctor_get(x_2, 3); lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_ctor_get(x_14, 1); +x_15 = lean_ctor_get(x_11, 0); lean_inc(x_15); -lean_dec(x_14); -x_16 = lean_ctor_get(x_15, 1); +x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); lean_dec(x_15); -x_17 = lean_apply_2(x_16, x_2, x_3); -return x_17; +x_17 = lean_box(0); +x_18 = lean_apply_1(x_16, x_17); +x_19 = l_List_foldl___at_Lean_Parser_evalParserConstUnsafe___spec__1(x_14, x_18); +x_20 = !lean_is_exclusive(x_2); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_21 = lean_ctor_get(x_2, 3); +lean_dec(x_21); +x_22 = lean_ctor_get(x_2, 2); +lean_dec(x_22); +x_23 = lean_ctor_get(x_2, 1); +lean_dec(x_23); +x_24 = lean_ctor_get(x_2, 0); +lean_dec(x_24); +lean_ctor_set(x_2, 3, x_19); +x_25 = lean_ctor_get(x_11, 1); +lean_inc(x_25); +lean_dec(x_11); +x_26 = lean_apply_2(x_25, x_2, x_3); +return x_26; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_27 = lean_ctor_get(x_2, 4); +x_28 = lean_ctor_get_uint8(x_2, sizeof(void*)*7); +x_29 = lean_ctor_get(x_2, 5); +x_30 = lean_ctor_get(x_2, 6); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_27); lean_dec(x_2); -x_18 = lean_ctor_get(x_13, 0); -lean_inc(x_18); -lean_dec(x_13); -x_19 = lean_io_error_to_string(x_18); -x_20 = lean_box(0); -x_21 = l_Lean_Parser_ParserState_mkUnexpectedError(x_3, x_19, x_20); -return x_21; +x_31 = lean_alloc_ctor(0, 7, 1); +lean_ctor_set(x_31, 0, x_12); +lean_ctor_set(x_31, 1, x_4); +lean_ctor_set(x_31, 2, x_13); +lean_ctor_set(x_31, 3, x_19); +lean_ctor_set(x_31, 4, x_27); +lean_ctor_set(x_31, 5, x_29); +lean_ctor_set(x_31, 6, x_30); +lean_ctor_set_uint8(x_31, sizeof(void*)*7, x_28); +x_32 = lean_ctor_get(x_11, 1); +lean_inc(x_32); +lean_dec(x_11); +x_33 = lean_apply_2(x_32, x_31, x_3); +return x_33; +} +} } } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__1() { _start: { lean_object* x_1; @@ -7969,17 +8074,17 @@ x_1 = lean_mk_string_from_bytes("internal", 8); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__1; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__3() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__3() { _start: { lean_object* x_1; @@ -7987,17 +8092,17 @@ x_1 = lean_mk_string_from_bytes("parseQuotWithCurrentStage", 25); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__4() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__2; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__3; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__2; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__5() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__5() { _start: { lean_object* x_1; @@ -8005,13 +8110,13 @@ x_1 = lean_mk_string_from_bytes("(Lean bootstrapping) use parsers from the curre return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__6() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__6() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 0; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__1; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__5; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__1; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__5; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -8020,12 +8125,12 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__4; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__6; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__4; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__6; x_4 = l_Lean_Option_register___at_Std_Format_initFn____x40_Lean_Data_Format___hyg_57____spec__1(x_2, x_3, x_1); return x_4; } @@ -8455,7 +8560,7 @@ return x_43; } } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__1() { _start: { lean_object* x_1; @@ -8463,7 +8568,7 @@ x_1 = l_Lean_Parser_categoryParserFnRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__2() { _start: { lean_object* x_1; @@ -8471,12 +8576,12 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_categoryParserFnImpl), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__1; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__2; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__1; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__2; x_4 = lean_st_ref_set(x_2, x_3, x_1); x_5 = !lean_is_exclusive(x_4); if (x_5 == 0) @@ -12357,7 +12462,7 @@ x_5 = l_Lean_registerBuiltinAttribute(x_4, x_3); return x_5; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -12365,23 +12470,23 @@ x_1 = lean_mk_string_from_bytes("invalid parser attribute implementation builder return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__1; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__1; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1(lean_object* x_1) { _start: { if (lean_obj_tag(x_1) == 0) { lean_object* x_2; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2; return x_2; } else @@ -12399,7 +12504,7 @@ if (lean_obj_tag(x_4) == 0) { lean_object* x_5; lean_dec(x_3); -x_5 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2; +x_5 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2; return x_5; } else @@ -12433,7 +12538,7 @@ lean_object* x_12; lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); -x_12 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2; +x_12 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2; return x_12; } } @@ -12443,7 +12548,7 @@ lean_object* x_13; lean_dec(x_6); lean_dec(x_4); lean_dec(x_3); -x_13 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2; +x_13 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2; return x_13; } } @@ -12453,13 +12558,13 @@ else lean_object* x_14; lean_dec(x_3); lean_dec(x_1); -x_14 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2; +x_14 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2; return x_14; } } } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__1() { _start: { lean_object* x_1; @@ -12467,30 +12572,30 @@ x_1 = lean_mk_string_from_bytes("parserAttr", 10); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__1; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__3() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__2; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__3; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__2; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__3; x_4 = l_Lean_registerAttributeImplBuilder(x_2, x_3, x_1); return x_4; } @@ -12522,7 +12627,7 @@ lean_ctor_set(x_13, 1, x_12); x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_10); lean_ctor_set(x_14, 1, x_13); -x_15 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__2; +x_15 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__2; x_16 = l_Lean_registerAttributeOfBuilder(x_8, x_15, x_14, x_9); return x_16; } @@ -12562,7 +12667,7 @@ x_7 = l_Lean_Parser_registerParserCategory(x_1, x_2, x_3, x_6, x_5); return x_7; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__1() { _start: { lean_object* x_1; @@ -12570,17 +12675,17 @@ x_1 = lean_mk_string_from_bytes("builtinTermParser", 17); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__1; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__3() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__3() { _start: { lean_object* x_1; @@ -12588,28 +12693,28 @@ x_1 = lean_mk_string_from_bytes("term", 4); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__4() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__3; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__2; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__4; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__2; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__4; x_4 = 0; x_5 = l_Lean_Parser_registerBuiltinParserAttribute(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__1() { _start: { lean_object* x_1; @@ -12617,27 +12722,27 @@ x_1 = lean_mk_string_from_bytes("termParser", 10); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__1; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__2; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__4; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__2; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__4; x_4 = l_Lean_Parser_registerBuiltinDynamicParserAttribute(x_2, x_3, x_1); return x_4; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__1() { _start: { lean_object* x_1; @@ -12645,17 +12750,17 @@ x_1 = lean_mk_string_from_bytes("builtinCommandParser", 20); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__1; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__3() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__3() { _start: { lean_object* x_1; @@ -12663,28 +12768,28 @@ x_1 = lean_mk_string_from_bytes("command", 7); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__4() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__3; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__2; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__4; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__2; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__4; x_4 = 0; x_5 = l_Lean_Parser_registerBuiltinParserAttribute(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__1() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__1() { _start: { lean_object* x_1; @@ -12692,22 +12797,22 @@ x_1 = lean_mk_string_from_bytes("commandParser", 13); return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__1; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__2; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__4; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__2; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__4; x_4 = l_Lean_Parser_registerBuiltinDynamicParserAttribute(x_2, x_3, x_1); return x_4; } @@ -12716,7 +12821,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_commandParser(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__4; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__4; x_3 = l_Lean_Parser_categoryParser(x_2, x_1); return x_3; } @@ -14292,19 +14397,19 @@ lean_mark_persistent(l_Lean_Parser_parserExtension); lean_dec_ref(res); }l_Lean_Parser_isParserCategory___closed__1 = _init_l_Lean_Parser_isParserCategory___closed__1(); lean_mark_persistent(l_Lean_Parser_isParserCategory___closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__3(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__3); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__4(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__4); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__5 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__5(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__5); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__6 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__6(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830____closed__6); -if (builtin) {res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3830_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__2); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__3(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__3); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__4(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__4); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__5 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__5(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__5); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__6 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__6(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861____closed__6); +if (builtin) {res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3861_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Parser_internal_parseQuotWithCurrentStage = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Parser_internal_parseQuotWithCurrentStage); @@ -14319,11 +14424,11 @@ l_Lean_Parser_categoryParserFnImpl___closed__3 = _init_l_Lean_Parser_categoryPar lean_mark_persistent(l_Lean_Parser_categoryParserFnImpl___closed__3); l_Lean_Parser_categoryParserFnImpl___closed__4 = _init_l_Lean_Parser_categoryParserFnImpl___closed__4(); lean_mark_persistent(l_Lean_Parser_categoryParserFnImpl___closed__4); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105____closed__2); -res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4105_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136____closed__2); +res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4136_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_ScopedEnvExtension_add___at_Lean_Parser_addToken___spec__3___closed__1 = _init_l_Lean_ScopedEnvExtension_add___at_Lean_Parser_addToken___spec__3___closed__1(); @@ -14443,53 +14548,53 @@ l_Lean_Parser_mkParserAttributeImpl___closed__1 = _init_l_Lean_Parser_mkParserAt lean_mark_persistent(l_Lean_Parser_mkParserAttributeImpl___closed__1); l_Lean_Parser_mkParserAttributeImpl___closed__2 = _init_l_Lean_Parser_mkParserAttributeImpl___closed__2(); lean_mark_persistent(l_Lean_Parser_mkParserAttributeImpl___closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____lambda__1___closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__3(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344____closed__3); -res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5344_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____lambda__1___closed__2); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__2); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__3(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375____closed__3); +res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5375_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__3(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__3); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__4(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456____closed__4); -res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5456_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__2); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__3(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__3); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__4(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487____closed__4); +res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5487_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470____closed__2); -res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5470_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501____closed__2); +res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5501_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__3(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__3); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__4(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484____closed__4); -res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5484_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__2); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__3(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__3); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__4(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515____closed__4); +res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5515_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498____closed__2); -res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5498_(lean_io_mk_world()); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529____closed__2); +res = l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5529_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Parser_withOpenDeclFnCore___closed__1 = _init_l_Lean_Parser_withOpenDeclFnCore___closed__1(); diff --git a/stage0/stdlib/Lean/Parser/Extra.c b/stage0/stdlib/Lean/Parser/Extra.c index 9e50f064a3ee..4c4c1fc4a1b1 100644 --- a/stage0/stdlib/Lean/Parser/Extra.c +++ b/stage0/stdlib/Lean/Parser/Extra.c @@ -31,6 +31,7 @@ static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___s lean_object* l_Lean_PrettyPrinter_Formatter_visitArgs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Parser_numLit___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__6; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__13; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__88; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealGroup_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -187,6 +188,7 @@ static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__5; lean_object* l_Lean_PrettyPrinter_Formatter_unicodeSymbolNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__23; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__8; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__24; LEAN_EXPORT lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__1___closed__7; @@ -197,10 +199,13 @@ static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____ lean_object* lean_string_utf8_byte_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquot_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1; static lean_object* l_Lean_Parser_scientificLit___closed__4; lean_object* l_Lean_Parser_checkColGeFn___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_nodeWithAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_many_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_nameLitFn(lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -208,6 +213,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_ppLine; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__116; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__16; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__112; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__2; static lean_object* l_Lean_Parser_strLit___closed__1; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_rawIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -215,7 +221,6 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le static lean_object* l_Lean_Parser_strLit_formatter___closed__3; static lean_object* l_Lean_Parser_leadingNode_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__37; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__3; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__61; LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_formatter___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -237,6 +242,7 @@ lean_object* l_Lean_PrettyPrinter_Parenthesizer_unicodeSymbolNoAntiquot_parenthe LEAN_EXPORT lean_object* l_Lean_Parser_optional(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_fill(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__7; static lean_object* l_Lean_Parser_sepByIndent___closed__5; static lean_object* l_Lean_Parser_numLit___closed__1; lean_object* l_Lean_Parser_rawIdentFn(lean_object*, lean_object*); @@ -248,7 +254,7 @@ lean_object* l_Lean_PrettyPrinter_Formatter_checkColGe_formatter___boxed(lean_ob LEAN_EXPORT lean_object* l_Lean_ppIndent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_symbolNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__36; +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealFill_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_setExpected_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_termParser_formatter___boxed(lean_object*); @@ -318,6 +324,7 @@ static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__25; LEAN_EXPORT lean_object* l_Lean_Parser_nodeWithAntiquot_formatter(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_sepBy(lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_manyIndent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__47; static lean_object* l_Lean_Parser_numLit_formatter___closed__1; @@ -360,6 +367,7 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_strLitFn(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__3; static lean_object* l_Lean_Parser_charLit___closed__3; lean_object* l_Lean_PrettyPrinter_Parenthesizer_charLitNoAntiquot_parenthesizer___boxed(lean_object*); static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__14; @@ -408,6 +416,7 @@ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Le LEAN_EXPORT lean_object* l_Lean_Parser_sepByIndent_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__44; lean_object* l_Lean_PrettyPrinter_Formatter_scientificLitNoAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; uint32_t lean_string_utf8_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_ppLine_parenthesizer___rarg(lean_object*); lean_object* l_Lean_Syntax_mkStrLit(lean_object*, lean_object*); @@ -423,12 +432,12 @@ static lean_object* l_Lean_Parser_optional_formatter___closed__3; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__5; static lean_object* l_Lean_Parser_sepByIndent___closed__4; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__42; -static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__53; LEAN_EXPORT lean_object* l_Lean_Parser_ppDedentIfGrouped_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_pushNone_parenthesizer___boxed(lean_object*); static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__8; static lean_object* l_Lean_Parser_rawIdent___elambda__1___closed__1; static lean_object* l_Lean_Parser_numLit_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4; static lean_object* l_Lean_Parser_scientificLit___closed__3; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__9; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__3; @@ -442,7 +451,6 @@ static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__11; lean_object* l_Lean_Syntax_MonadTraverser_goLeft___at_Lean_PrettyPrinter_Formatter_visitArgs___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__102; LEAN_EXPORT lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_antiquotExpr_parenthesizer___closed__4; static lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_formatter(lean_object*); @@ -466,7 +474,6 @@ static lean_object* l_Lean_Parser_rawIdent___closed__2; static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__27; static lean_object* l_Lean_Parser_antiquotNestedExpr_formatter___closed__6; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__14; -static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__54; LEAN_EXPORT lean_object* l_Lean_Parser_mkAntiquot_formatter(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ppHardSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_many1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -503,7 +510,6 @@ static lean_object* l_Lean_Parser_nameLit_parenthesizer___closed__1; lean_object* l_String_intercalate(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_numLit; static lean_object* l_Lean_Parser_many___closed__4; -static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__39; static lean_object* l_Lean_Parser_charLit_formatter___closed__1; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__27; static lean_object* l_Lean_Parser_antiquotExpr_parenthesizer___closed__3; @@ -537,7 +543,6 @@ static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____ static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_commandParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_scientificLit_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__5; static lean_object* l_Lean_Parser_mkAntiquot_formatter___closed__16; static lean_object* l_Lean_Parser_group_formatter___closed__1; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__24; @@ -612,6 +617,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1_formatter___boxed(lean_object*, le static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__2; uint8_t l_Lean_Syntax_isNone(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_numLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_ppSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__34; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__36; @@ -623,6 +629,7 @@ lean_object* l_Lean_PrettyPrinter_Formatter_fold(lean_object*, lean_object*, lea static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__50; lean_object* l_Lean_Parser_nodeFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__9; lean_object* l_Lean_Parser_optionalFn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__40; @@ -638,6 +645,7 @@ uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_rawIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__1; static lean_object* l_Lean_Parser_scientificLit_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__9; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__39; static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___spec__2___closed__3; extern lean_object* l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; @@ -662,7 +670,6 @@ lean_object* l_Lean_Parser_mkAntiquot(lean_object*, lean_object*, uint8_t, uint8 lean_object* l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_nameLit_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_ppGroup(lean_object*); -static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__38; static lean_object* l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__1___closed__5; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); @@ -678,6 +685,7 @@ static lean_object* l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___ static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__38; LEAN_EXPORT lean_object* l_Lean_Parser_ppRealFill___boxed(lean_object*); lean_object* lean_nat_mod(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter(lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__65; LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__35; @@ -727,6 +735,7 @@ static lean_object* l_List_forIn_loop___at_Lean_Parser_sepByIndent_formatter___s static lean_object* l_Lean_Parser_scientificLit___closed__2; static lean_object* l_Lean_Parser_many1Indent___closed__1; static lean_object* l_Lean_ppDedentIfGrouped_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_symbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__1___closed__10; static lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__48; @@ -761,6 +770,7 @@ static lean_object* l_Lean_Parser_strLit___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_ppDedent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_sepBy1Indent_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_notSymbol_formatter___rarg(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__3; static lean_object* l_Lean_Parser_antiquotExpr_formatter___closed__1; static lean_object* l_Lean_Parser_leadingNode_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_termParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1041,6 +1051,98 @@ x_8 = l_Lean_PrettyPrinter_Formatter_node_formatter(x_6, x_7, x_1, x_2, x_3, x_4 return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Lean", 4); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Parser", 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; +x_2 = l_Lean_Parser_antiquotNestedExpr_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__5; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__6; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_antiquotNestedExpr_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__8; +x_3 = l_Lean_Parser_antiquotNestedExpr_formatter___closed__2; +x_4 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__7; +x_5 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__9; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_antiquotExpr_formatter___closed__1() { _start: { @@ -1062,24 +1164,16 @@ return x_2; static lean_object* _init_l_Lean_Parser_antiquotExpr_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_antiquotNestedExpr_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_antiquotExpr_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_antiquotExpr_formatter___closed__2; -x_2 = l_Lean_Parser_antiquotExpr_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_antiquotExpr_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_antiquotExpr_formatter___closed__4() { _start: { lean_object* x_1; @@ -1091,8 +1185,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_antiquotExpr_formatter(lean_object* x_1, _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_antiquotExpr_formatter___closed__5; -x_7 = l_Lean_Parser_antiquotExpr_formatter___closed__4; +x_6 = l_Lean_Parser_antiquotExpr_formatter___closed__4; +x_7 = l_Lean_Parser_antiquotExpr_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -1494,17 +1588,33 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_node_parenthesizer(x_6, x_7, x_1, x_2, return x_8; } } -static lean_object* _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_antiquotExpr_formatter___closed__1; -x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_symbolNoAntiquot_parenthesizer___boxed), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; } } -static lean_object* _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__5; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4() { _start: { lean_object* x_1; @@ -1512,19 +1622,41 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_antiquotNestedExpr_parenthesizer) return x_1; } } -static lean_object* _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__3; +x_3 = l_Lean_Parser_antiquotNestedExpr_formatter___closed__2; +x_4 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_antiquotExpr_formatter___closed__1; +x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_symbolNoAntiquot_parenthesizer___boxed), 2, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_antiquotExpr_parenthesizer___closed__1; -x_2 = l_Lean_Parser_antiquotExpr_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__3() { _start: { lean_object* x_1; @@ -1536,8 +1668,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_antiquotExpr_parenthesizer(lean_object* x _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_antiquotExpr_parenthesizer___closed__4; -x_7 = l_Lean_Parser_antiquotExpr_parenthesizer___closed__3; +x_6 = l_Lean_Parser_antiquotExpr_parenthesizer___closed__3; +x_7 = l_Lean_Parser_antiquotExpr_parenthesizer___closed__2; x_8 = l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -2710,7 +2842,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_ident_formatter(lean_object* x_1, lean_ob { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_ident_formatter___closed__3; -x_7 = l_Lean_Parser_antiquotExpr_formatter___closed__5; +x_7 = l_Lean_Parser_antiquotExpr_formatter___closed__4; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -2738,7 +2870,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_ident_parenthesizer(lean_object* x_1, lea { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_ident_parenthesizer___closed__1; -x_7 = l_Lean_Parser_antiquotExpr_parenthesizer___closed__4; +x_7 = l_Lean_Parser_antiquotExpr_parenthesizer___closed__3; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -6361,7 +6493,7 @@ static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_ _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean", 4); +x_1 = lean_mk_string_from_bytes("termRegister_parser_alias(Kind:=_)____", 38); return x_1; } } @@ -6369,7 +6501,7 @@ static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -6379,7 +6511,7 @@ static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_ _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Parser", 6); +x_1 = lean_mk_string_from_bytes("andthen", 7); return x_1; } } @@ -6387,7 +6519,7 @@ static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__2; +x_1 = lean_box(0); x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -6397,57 +6529,21 @@ static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_ _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("termRegister_parser_alias(Kind:=_)____", 38); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("andthen", 7); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__7; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__9() { -_start: -{ -lean_object* x_1; x_1 = lean_mk_string_from_bytes("register_parser_alias", 21); return x_1; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__10() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__9; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__5; x_2 = lean_alloc_ctor(5, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__11() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__7() { _start: { lean_object* x_1; lean_object* x_2; @@ -6457,7 +6553,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__12() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8() { _start: { lean_object* x_1; @@ -6465,11 +6561,11 @@ x_1 = lean_mk_string_from_bytes("kind", 4); return x_1; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__13() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__9() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__12; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; x_2 = 0; x_3 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -6477,13 +6573,13 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__14() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__11; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__13; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__7; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__9; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6491,7 +6587,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__15() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__11() { _start: { lean_object* x_1; @@ -6499,23 +6595,23 @@ x_1 = lean_mk_string_from_bytes(" := ", 4); return x_1; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__16() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__15; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__11; x_2 = lean_alloc_ctor(5, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__17() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__14; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__16; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__10; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__12; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6523,7 +6619,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__18() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -6535,13 +6631,13 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__19() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__17; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__18; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__13; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__14; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6549,7 +6645,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__20() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__16() { _start: { lean_object* x_1; lean_object* x_2; @@ -6559,13 +6655,13 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__21() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__19; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__20; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__15; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__16; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6573,37 +6669,37 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__22() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_group_formatter___closed__2; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__21; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__17; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__23() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_optional_formatter___closed__2; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__22; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__18; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__24() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__10; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__23; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__6; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__19; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6611,7 +6707,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__25() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__21() { _start: { lean_object* x_1; @@ -6619,45 +6715,45 @@ x_1 = lean_mk_string_from_bytes("strLit", 6); return x_1; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__26() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__25; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__21; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__27() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__23() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__26; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__22; x_2 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__28() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_optional_formatter___closed__2; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__27; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__23; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__29() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__24; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__28; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__20; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__24; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6665,33 +6761,33 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__30() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__26() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_ident_formatter___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__31() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__27() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__30; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__26; x_2 = lean_alloc_ctor(8, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__32() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__28() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__29; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__31; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__25; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__27; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6699,7 +6795,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__33() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__29() { _start: { lean_object* x_1; @@ -6707,33 +6803,33 @@ x_1 = lean_mk_string_from_bytes("colGt", 5); return x_1; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__34() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__30() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__33; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__29; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__35() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__31() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__34; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__30; 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_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__36() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__32() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__35; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__18; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__31; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__14; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6741,25 +6837,25 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__37() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_optional_formatter___closed__2; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__36; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__32; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__38() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__34() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__8; -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__32; -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__37; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__28; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__33; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6767,13 +6863,13 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__39() { +static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__35() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__6; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__2; x_2 = lean_unsigned_to_nat(1022u); -x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__38; +x_3 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__34; x_4 = lean_alloc_ctor(3, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6785,7 +6881,7 @@ static lean_object* _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_ _start: { lean_object* x_1; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__39; +x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__35; return x_1; } } @@ -7052,7 +7148,7 @@ static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRul { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__3; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -7345,22 +7441,14 @@ return x_3; static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__41() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("formatter", 9); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__42() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__41; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__43() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__42() { _start: { lean_object* x_1; @@ -7368,22 +7456,22 @@ x_1 = lean_mk_string_from_bytes("PrettyPrinter.Parenthesizer.registerAlias", 41) return x_1; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__44() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__43() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__43; +x_1 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__42; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__45() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__44() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__43; +x_1 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__42; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__44; +x_3 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__43; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -7391,7 +7479,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__46() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__45() { _start: { lean_object* x_1; @@ -7399,45 +7487,37 @@ x_1 = lean_mk_string_from_bytes("Parenthesizer", 13); return x_1; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__47() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__46() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__37; -x_2 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__46; +x_2 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__45; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__48() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__47() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__47; +x_1 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__46; x_2 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__49() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("parenthesizer", 13); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__50() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__49; +x_2 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__51() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__49() { _start: { lean_object* x_1; lean_object* x_2; @@ -7446,7 +7526,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__52() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__50() { _start: { lean_object* x_1; @@ -7454,7 +7534,7 @@ x_1 = lean_mk_string_from_bytes("quotedName", 10); return x_1; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__53() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__51() { _start: { lean_object* x_1; @@ -7462,7 +7542,7 @@ x_1 = lean_mk_string_from_bytes(".", 1); return x_1; } } -static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__54() { +static lean_object* _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__52() { _start: { lean_object* x_1; @@ -7904,7 +7984,7 @@ lean_ctor_set(x_102, 0, x_32); lean_ctor_set(x_102, 1, x_101); lean_ctor_set(x_102, 2, x_93); lean_ctor_set(x_102, 3, x_100); -x_103 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__42; +x_103 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__41; x_104 = l_Lean_Name_append(x_16, x_103); lean_inc(x_11); x_105 = l_Lean_mkIdentFrom(x_11, x_104); @@ -7938,9 +8018,9 @@ x_119 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_119, 0, x_108); lean_ctor_set(x_119, 1, x_45); lean_ctor_set(x_119, 2, x_118); -x_120 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__48; +x_120 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__47; x_121 = l_Lean_addMacroScope(x_36, x_120, x_35); -x_122 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__46; +x_122 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__45; x_123 = l_Lean_Name_str___override(x_95, x_122); x_124 = l_Lean_Name_str___override(x_123, x_52); x_125 = lean_alloc_ctor(0, 2, 0); @@ -7949,13 +8029,13 @@ lean_ctor_set(x_125, 1, x_54); x_126 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_126, 0, x_125); lean_ctor_set(x_126, 1, x_54); -x_127 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__45; +x_127 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__44; x_128 = lean_alloc_ctor(3, 4, 0); lean_ctor_set(x_128, 0, x_32); lean_ctor_set(x_128, 1, x_127); lean_ctor_set(x_128, 2, x_121); lean_ctor_set(x_128, 3, x_126); -x_129 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__50; +x_129 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__48; x_130 = l_Lean_Name_append(x_16, x_129); lean_dec(x_16); x_131 = l_Lean_mkIdentFrom(x_11, x_130); @@ -8034,11 +8114,11 @@ lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; x_175 = lean_ctor_get(x_79, 0); lean_inc(x_175); lean_dec(x_79); -x_176 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__52; +x_176 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__50; x_177 = l_Lean_Name_str___override(x_38, x_176); -x_178 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__53; +x_178 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__51; x_179 = l_String_intercalate(x_178, x_175); -x_180 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__54; +x_180 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__52; x_181 = lean_string_append(x_180, x_179); lean_dec(x_179); x_182 = l_Lean_Syntax_mkNameLit(x_181, x_108); @@ -8103,7 +8183,7 @@ x_161 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_161, 0, x_108); lean_ctor_set(x_161, 1, x_45); lean_ctor_set(x_161, 2, x_160); -x_162 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__51; +x_162 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__49; x_163 = lean_array_push(x_162, x_161); x_164 = lean_array_push(x_163, x_119); x_165 = lean_array_push(x_164, x_141); @@ -8141,7 +8221,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser___aux__Lean__Parser__Extra______macroRule _start: { lean_object* x_4; uint8_t x_5; -x_4 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__6; +x_4 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__2; lean_inc(x_1); x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); if (x_5 == 0) @@ -8207,8 +8287,8 @@ x_21 = l_Lean_Syntax_getArg(x_15, x_20); lean_dec(x_15); x_22 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_22, 0, x_21); -x_23 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; -x_24 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__2; +x_23 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; +x_24 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__2; x_25 = lean_box(0); x_26 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2(x_1, x_23, x_24, x_25, x_22, x_2, x_3); lean_dec(x_1); @@ -8221,8 +8301,8 @@ else lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_dec(x_9); x_27 = lean_box(0); -x_28 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; -x_29 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__2; +x_28 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; +x_29 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__2; x_30 = lean_box(0); x_31 = l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2(x_1, x_28, x_29, x_30, x_27, x_2, x_3); lean_dec(x_1); @@ -8272,7 +8352,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_group_formatter___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -8394,7 +8474,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -8490,7 +8570,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__24; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -8564,7 +8644,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__32; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -8656,7 +8736,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__40; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -8760,7 +8840,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__51; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -8852,7 +8932,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__61; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -8944,7 +9024,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__71; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -9036,7 +9116,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__81; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -9128,7 +9208,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__91; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -9202,7 +9282,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__101; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -9276,7 +9356,7 @@ static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_16 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__4; +x_1 = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4; x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__109; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -10500,6 +10580,27 @@ l_Lean_Parser_antiquotNestedExpr_formatter___closed__9 = _init_l_Lean_Parser_ant lean_mark_persistent(l_Lean_Parser_antiquotNestedExpr_formatter___closed__9); l_Lean_Parser_antiquotNestedExpr_formatter___closed__10 = _init_l_Lean_Parser_antiquotNestedExpr_formatter___closed__10(); lean_mark_persistent(l_Lean_Parser_antiquotNestedExpr_formatter___closed__10); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__1); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__2); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__3); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__4); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__5 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__5); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__6 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__6); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__7 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__7); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__8 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__8); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__9 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__9(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter___closed__9); +res = l___regBuiltin_Lean_Parser_antiquotNestedExpr_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_antiquotExpr_formatter___closed__1 = _init_l_Lean_Parser_antiquotExpr_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_antiquotExpr_formatter___closed__1); l_Lean_Parser_antiquotExpr_formatter___closed__2 = _init_l_Lean_Parser_antiquotExpr_formatter___closed__2(); @@ -10508,8 +10609,6 @@ l_Lean_Parser_antiquotExpr_formatter___closed__3 = _init_l_Lean_Parser_antiquotE lean_mark_persistent(l_Lean_Parser_antiquotExpr_formatter___closed__3); l_Lean_Parser_antiquotExpr_formatter___closed__4 = _init_l_Lean_Parser_antiquotExpr_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_antiquotExpr_formatter___closed__4); -l_Lean_Parser_antiquotExpr_formatter___closed__5 = _init_l_Lean_Parser_antiquotExpr_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_antiquotExpr_formatter___closed__5); l_Lean_Parser_mkAntiquot_formatter___closed__1 = _init_l_Lean_Parser_mkAntiquot_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_mkAntiquot_formatter___closed__1); l_Lean_Parser_mkAntiquot_formatter___closed__2 = _init_l_Lean_Parser_mkAntiquot_formatter___closed__2(); @@ -10558,14 +10657,23 @@ l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__5 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__5); l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__6 = _init_l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_antiquotNestedExpr_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_antiquotExpr_parenthesizer___closed__1 = _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_antiquotExpr_parenthesizer___closed__1); l_Lean_Parser_antiquotExpr_parenthesizer___closed__2 = _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_antiquotExpr_parenthesizer___closed__2); l_Lean_Parser_antiquotExpr_parenthesizer___closed__3 = _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_antiquotExpr_parenthesizer___closed__3); -l_Lean_Parser_antiquotExpr_parenthesizer___closed__4 = _init_l_Lean_Parser_antiquotExpr_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_antiquotExpr_parenthesizer___closed__4); l_Lean_Parser_mkAntiquot_parenthesizer___closed__1 = _init_l_Lean_Parser_mkAntiquot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_mkAntiquot_parenthesizer___closed__1); l_Lean_Parser_mkAntiquot_parenthesizer___closed__2 = _init_l_Lean_Parser_mkAntiquot_parenthesizer___closed__2(); @@ -10942,14 +11050,6 @@ l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed lean_mark_persistent(l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__34); l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__35 = _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__35(); lean_mark_persistent(l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__35); -l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__36 = _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__36(); -lean_mark_persistent(l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__36); -l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__37 = _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__37(); -lean_mark_persistent(l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__37); -l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__38 = _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__38(); -lean_mark_persistent(l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__38); -l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__39 = _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__39(); -lean_mark_persistent(l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29___________closed__39); l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29________ = _init_l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29________(); lean_mark_persistent(l_Lean_Parser_termRegister__parser__alias_x28Kind_x3a_x3d___x29________); l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__1___closed__1 = _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__1___closed__1(); @@ -11080,10 +11180,6 @@ l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegi lean_mark_persistent(l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__51); l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__52 = _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__52(); lean_mark_persistent(l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__52); -l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__53 = _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__53(); -lean_mark_persistent(l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__53); -l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__54 = _init_l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__54(); -lean_mark_persistent(l_Lean_Parser___aux__Lean__Parser__Extra______macroRules__Lean__Parser__termRegister__parser__alias_x28Kind_x3a_x3d___x29__________1___lambda__2___closed__54); l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__1(); lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__1); l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Extra___hyg_1630____closed__2(); diff --git a/stage0/stdlib/Lean/Parser/Level.c b/stage0/stdlib/Lean/Parser/Level.c index d225a911f54a..a915aec82dae 100644 --- a/stage0/stdlib/Lean/Parser/Level.c +++ b/stage0/stdlib/Lean/Parser/Level.c @@ -44,6 +44,7 @@ static lean_object* l_Lean_Parser_Level_max___elambda__1___closed__6; static lean_object* l_Lean_Parser_Level_addLit_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Level_hole_declRange___closed__5; static lean_object* l_Lean_Parser_Level_max_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Level_imax_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_imax___elambda__1___closed__11; lean_object* l_Lean_Parser_symbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -59,11 +60,14 @@ static lean_object* l_Lean_Parser_Level_imax_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Level_imax_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Level_ident; static lean_object* l___regBuiltin_Lean_Parser_Level_max_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_imax_formatter(lean_object*); static lean_object* l_Lean_Parser_Level_hole_formatter___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_max_formatter___closed__4; extern lean_object* l_Lean_Parser_ident; static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Level_paren_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Level_imax_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_imax___closed__7; @@ -92,7 +96,10 @@ static lean_object* l_Lean_Parser_Level_max___elambda__1___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Level_max_declRange___closed__3; static lean_object* l_Lean_Parser_Level_max_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Level_paren___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_paren_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_hole_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Level_hole___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Level_paren___closed__3; lean_object* l_Lean_Parser_checkPrecFn___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__12; @@ -100,9 +107,14 @@ static lean_object* l_Lean_Parser_Level_max___elambda__1___closed__9; static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__2; static lean_object* l_Lean_Parser_Level_num___closed__1; static lean_object* l_Lean_Parser_Level_paren_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_max_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__1; lean_object* l_Lean_Parser_mkAntiquot_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_imax___closed__3; +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3; static lean_object* l_Lean_Parser_Level_addLit___elambda__1___closed__6; lean_object* l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkPrec_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -111,6 +123,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_paren_declRange(lean_o static lean_object* l___regBuiltin_Lean_Parser_Level_ident_declRange___closed__3; lean_object* l_Lean_Parser_checkPrecFn(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_ident_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Level_max___elambda__1___lambda__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Level_addLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_num_parenthesizer___closed__2; @@ -118,7 +131,9 @@ static lean_object* l_Lean_Parser_Level_max___closed__3; lean_object* l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Level_hole_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_max___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer(lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Level___hyg_5____closed__3; static lean_object* l_Lean_Parser_Level_imax___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Level_paren___elambda__1(lean_object*, lean_object*); @@ -127,11 +142,13 @@ static lean_object* l_Lean_Parser_Level_max___elambda__1___closed__8; static lean_object* l_Lean_Parser_Level_addLit_formatter___closed__1; static lean_object* l_Lean_Parser_Level_paren___elambda__1___lambda__1___closed__1; static lean_object* l_Lean_Parser_Level_imax___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Level_ident___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_addLit_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Level_num_declRange___closed__1; lean_object* l_Lean_Parser_nonReservedSymbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_imax_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1; lean_object* l_Lean_Parser_nodeInfo(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Level_addLit___elambda__1(lean_object*, lean_object*); lean_object* l_Lean_Parser_checkLhsPrecFn(lean_object*, lean_object*, lean_object*); @@ -140,15 +157,18 @@ static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Level___hyg_5____clo static lean_object* l_Lean_Parser_Level_max_formatter___closed__6; static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Level_ident_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__4; static lean_object* l_Lean_Parser_Level_imax___elambda__1___closed__8; lean_object* l_Lean_Parser_nonReservedSymbolInfo(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Parser_Level_paren; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_imax(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_checkPrec_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_addLit___elambda__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Level_num_declRange___closed__2; static lean_object* l_Lean_Parser_Level_paren_formatter___closed__7; static lean_object* l_Lean_Parser_Level_paren___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Level_num___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Level_num_declRange___closed__4; lean_object* l_Lean_Parser_many1_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -158,7 +178,9 @@ static lean_object* l_Lean_Parser_Level_max___closed__6; static lean_object* l_Lean_Parser_Level_addLit___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Level_imax; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Level___hyg_5____closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Level_paren_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Level_max_parenthesizer___closed__8; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Level___hyg_5____closed__2; static lean_object* l_Lean_Parser_Level_max_formatter___closed__1; @@ -181,7 +203,9 @@ static lean_object* l___regBuiltin_Lean_Parser_Level_paren_declRange___closed__3 LEAN_EXPORT lean_object* l_Lean_Parser_Level_paren___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_max_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Level_ident_declRange___closed__5; +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; uint32_t lean_string_utf8_get(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_max_formatter___closed__2; static lean_object* l_Lean_Parser_Level_ident___closed__1; static lean_object* l_Lean_Parser_Level_imax_formatter___closed__4; lean_object* l_Lean_Parser_registerBuiltinParserAttribute(lean_object*, lean_object*, uint8_t, lean_object*); @@ -196,6 +220,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Level_num_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Level_num_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Level_ident_declRange___closed__1; lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_max_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Level_addLit_declRange___closed__7; static lean_object* l_Lean_Parser_Level_paren___closed__4; static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__18; @@ -219,21 +244,27 @@ static lean_object* l___regBuiltin_Lean_Parser_Level_paren_declRange___closed__4 static lean_object* l___regBuiltin_Lean_Parser_Level_hole_declRange___closed__2; static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__15; static lean_object* l_Lean_Parser_Level_hole___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__2; lean_object* l_Lean_Parser_ident___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_max___closed__4; uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l_Lean_Parser_Level_hole___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_addLit_formatter(lean_object*); extern lean_object* l_Lean_Parser_numLit; static lean_object* l_Lean_Parser_Level_max___closed__8; static lean_object* l_Lean_Parser_Level_ident_formatter___closed__1; static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__3; lean_object* l_Lean_Parser_numLit___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Level_hole_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__20; static lean_object* l_Lean_Parser_Level_hole___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Level_max; LEAN_EXPORT lean_object* l_Lean_Parser_Level_num; lean_object* l_Lean_Parser_categoryParser(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Level_ident___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Level_ident_declRange___closed__2; static lean_object* l_Lean_Parser_Level_max___closed__5; @@ -281,9 +312,12 @@ static lean_object* l_Lean_Parser_Level_imax___closed__5; static lean_object* l_Lean_Parser_Level_addLit___closed__6; static lean_object* l_Lean_Parser_Level_addLit___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Level_num___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_max_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Level_addLit_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Level_num___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Level_max___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_hole_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Level_paren___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_ident(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Level_max_declRange___closed__4; @@ -291,11 +325,13 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Level_addLit; static lean_object* l_Lean_Parser_Level_hole___elambda__1___closed__11; lean_object* l_Lean_Parser_mkAntiquot(lean_object*, lean_object*, uint8_t, uint8_t); static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__13; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_imax_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Level_paren_formatter___closed__4; static lean_object* l_Lean_Parser_Level_max___elambda__1___closed__5; static lean_object* l_Lean_Parser_Level_paren_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Level_addLit_formatter___closed__2; static lean_object* l_Lean_Parser_Level_max___elambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_paren_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Level_imax_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Level_max_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_levelParser_formatter___boxed(lean_object*); @@ -329,6 +365,7 @@ static lean_object* l_Lean_Parser_Level_max_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Level_paren___closed__8; static lean_object* l_Lean_Parser_Level_paren___elambda__1___closed__4; static lean_object* l_Lean_Parser_Level_hole___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Level___hyg_5_(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Level_imax_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Level_addLit_declRange___closed__3; @@ -1225,6 +1262,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_paren___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_paren_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_paren_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Level_paren___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_levelParser_parenthesizer(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: { @@ -1330,6 +1413,52 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_paren___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_paren_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_paren_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Level_paren___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Level_max___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -2016,6 +2145,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_max_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_max___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_max_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_max_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_max_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Level_max___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Level_max_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_max_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Level_max_parenthesizer___closed__1() { _start: { @@ -2123,6 +2282,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_max___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_max_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_max_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Level_max___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Level_imax___elambda__1___closed__1() { _start: { @@ -2699,6 +2888,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_imax___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_imax_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_imax_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Level_imax___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Level_imax_parenthesizer___closed__1() { _start: { @@ -2766,6 +2985,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_imax___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_imax_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_imax_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Level_imax___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Level_hole___elambda__1___closed__1() { _start: { @@ -3236,6 +3485,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_hole___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_hole_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_hole_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Level_hole___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Level_hole_parenthesizer___closed__1() { _start: { @@ -3288,6 +3567,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_hole___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_hole_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_hole_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Level_hole___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Level_num___elambda__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -4236,6 +4545,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_addLit___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_addLit_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_addLit_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Level_addLit___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Level_addLit_parenthesizer___closed__1() { _start: { @@ -4270,6 +4609,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_addLit___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_addLit_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Level_addLit___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Extra(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -4394,6 +4763,17 @@ l_Lean_Parser_Level_paren_formatter___closed__6 = _init_l_Lean_Parser_Level_pare lean_mark_persistent(l_Lean_Parser_Level_paren_formatter___closed__6); l_Lean_Parser_Level_paren_formatter___closed__7 = _init_l_Lean_Parser_Level_paren_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Level_paren_formatter___closed__7); +l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__1); +l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__2); +l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__3); +l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_paren_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Level_paren_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_paren_parenthesizer___closed__1 = _init_l_Lean_Parser_Level_paren_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_paren_parenthesizer___closed__1); l_Lean_Parser_Level_paren_parenthesizer___closed__2 = _init_l_Lean_Parser_Level_paren_parenthesizer___closed__2(); @@ -4408,6 +4788,17 @@ l_Lean_Parser_Level_paren_parenthesizer___closed__6 = _init_l_Lean_Parser_Level_ lean_mark_persistent(l_Lean_Parser_Level_paren_parenthesizer___closed__6); l_Lean_Parser_Level_paren_parenthesizer___closed__7 = _init_l_Lean_Parser_Level_paren_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Level_paren_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_paren_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_Level_paren_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_max___elambda__1___closed__1 = _init_l_Lean_Parser_Level_max___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_max___elambda__1___closed__1); l_Lean_Parser_Level_max___elambda__1___closed__2 = _init_l_Lean_Parser_Level_max___elambda__1___closed__2(); @@ -4486,6 +4877,13 @@ l_Lean_Parser_Level_max_formatter___closed__6 = _init_l_Lean_Parser_Level_max_fo lean_mark_persistent(l_Lean_Parser_Level_max_formatter___closed__6); l_Lean_Parser_Level_max_formatter___closed__7 = _init_l_Lean_Parser_Level_max_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Level_max_formatter___closed__7); +l___regBuiltin_Lean_Parser_Level_max_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_max_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_max_formatter___closed__1); +l___regBuiltin_Lean_Parser_Level_max_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_max_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_max_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Level_max_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_max_parenthesizer___closed__1 = _init_l_Lean_Parser_Level_max_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_max_parenthesizer___closed__1); l_Lean_Parser_Level_max_parenthesizer___closed__2 = _init_l_Lean_Parser_Level_max_parenthesizer___closed__2(); @@ -4502,6 +4900,13 @@ l_Lean_Parser_Level_max_parenthesizer___closed__7 = _init_l_Lean_Parser_Level_ma lean_mark_persistent(l_Lean_Parser_Level_max_parenthesizer___closed__7); l_Lean_Parser_Level_max_parenthesizer___closed__8 = _init_l_Lean_Parser_Level_max_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Level_max_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_max_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Level_max_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_imax___elambda__1___closed__1 = _init_l_Lean_Parser_Level_imax___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_imax___elambda__1___closed__1); l_Lean_Parser_Level_imax___elambda__1___closed__2 = _init_l_Lean_Parser_Level_imax___elambda__1___closed__2(); @@ -4570,6 +4975,13 @@ l_Lean_Parser_Level_imax_formatter___closed__3 = _init_l_Lean_Parser_Level_imax_ lean_mark_persistent(l_Lean_Parser_Level_imax_formatter___closed__3); l_Lean_Parser_Level_imax_formatter___closed__4 = _init_l_Lean_Parser_Level_imax_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Level_imax_formatter___closed__4); +l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__1); +l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_imax_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Level_imax_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_imax_parenthesizer___closed__1 = _init_l_Lean_Parser_Level_imax_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_imax_parenthesizer___closed__1); l_Lean_Parser_Level_imax_parenthesizer___closed__2 = _init_l_Lean_Parser_Level_imax_parenthesizer___closed__2(); @@ -4578,6 +4990,13 @@ l_Lean_Parser_Level_imax_parenthesizer___closed__3 = _init_l_Lean_Parser_Level_i lean_mark_persistent(l_Lean_Parser_Level_imax_parenthesizer___closed__3); l_Lean_Parser_Level_imax_parenthesizer___closed__4 = _init_l_Lean_Parser_Level_imax_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Level_imax_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_imax_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Level_imax_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_hole___elambda__1___closed__1 = _init_l_Lean_Parser_Level_hole___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_hole___elambda__1___closed__1); l_Lean_Parser_Level_hole___elambda__1___closed__2 = _init_l_Lean_Parser_Level_hole___elambda__1___closed__2(); @@ -4642,12 +5061,26 @@ l_Lean_Parser_Level_hole_formatter___closed__2 = _init_l_Lean_Parser_Level_hole_ lean_mark_persistent(l_Lean_Parser_Level_hole_formatter___closed__2); l_Lean_Parser_Level_hole_formatter___closed__3 = _init_l_Lean_Parser_Level_hole_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Level_hole_formatter___closed__3); +l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__1); +l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_hole_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Level_hole_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_hole_parenthesizer___closed__1 = _init_l_Lean_Parser_Level_hole_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_hole_parenthesizer___closed__1); l_Lean_Parser_Level_hole_parenthesizer___closed__2 = _init_l_Lean_Parser_Level_hole_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Level_hole_parenthesizer___closed__2); l_Lean_Parser_Level_hole_parenthesizer___closed__3 = _init_l_Lean_Parser_Level_hole_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Level_hole_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_hole_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Level_hole_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_num___closed__1 = _init_l_Lean_Parser_Level_num___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_num___closed__1); l_Lean_Parser_Level_num___closed__2 = _init_l_Lean_Parser_Level_num___closed__2(); @@ -4778,10 +5211,24 @@ l_Lean_Parser_Level_addLit_formatter___closed__1 = _init_l_Lean_Parser_Level_add lean_mark_persistent(l_Lean_Parser_Level_addLit_formatter___closed__1); l_Lean_Parser_Level_addLit_formatter___closed__2 = _init_l_Lean_Parser_Level_addLit_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Level_addLit_formatter___closed__2); +l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__1); +l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_addLit_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Level_addLit_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_addLit_parenthesizer___closed__1 = _init_l_Lean_Parser_Level_addLit_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_addLit_parenthesizer___closed__1); l_Lean_Parser_Level_addLit_parenthesizer___closed__2 = _init_l_Lean_Parser_Level_addLit_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Level_addLit_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Level_addLit_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Parser/Module.c b/stage0/stdlib/Lean/Parser/Module.c index 80ba27188895..6a57eefc1734 100644 --- a/stage0/stdlib/Lean/Parser/Module.c +++ b/stage0/stdlib/Lean/Parser/Module.c @@ -14,11 +14,12 @@ extern "C" { #endif static lean_object* l_Lean_Parser_parseHeader___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__2; lean_object* l_String_csize(uint32_t); static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__5; static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__15; static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__14; -static lean_object* l_Lean_Parser_Module_header_parenthesizer___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Module_module_formatter___closed__2; static lean_object* l_Lean_Parser_Module_module_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Module_module_formatter___closed__2; static lean_object* l_Lean_Parser_Module_module___closed__5; @@ -55,7 +56,9 @@ static lean_object* l_Lean_Parser_Module_updateTokens___closed__4; static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__12; static lean_object* l___private_Lean_Parser_Module_0__Lean_Parser_mkEOI___closed__2; lean_object* l_Lean_Parser_symbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_module_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Parser_testParseModuleAux_parse___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Module_module_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_header_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Module_import_parenthesizer___closed__5; @@ -93,6 +96,7 @@ static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__1; static lean_object* l_Lean_Parser_Module_prelude_formatter___closed__1; static lean_object* l_Lean_Parser_Module_module_parenthesizer___closed__1; lean_object* lean_string_append(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3; LEAN_EXPORT lean_object* l_panic___at_Lean_Parser_Module_updateTokens___spec__1(lean_object*); static lean_object* l_Lean_Parser_Module_import_formatter___closed__8; lean_object* l_Lean_Parser_tokenFn(lean_object*, lean_object*, lean_object*); @@ -102,8 +106,10 @@ static lean_object* l_Lean_Parser_Module_import___closed__9; static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_isExitCommand___boxed(lean_object*); static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Module_module_formatter___closed__1; static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__3; static lean_object* l_Lean_Parser_Module_module_formatter___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Module_import_formatter___closed__1; lean_object* l_Lean_Parser_checkPrecFn___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Module_import_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_header_formatter___closed__6; @@ -115,9 +121,11 @@ lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_obje LEAN_EXPORT uint8_t l_Lean_Parser_ModuleParserState_recovering___default; LEAN_EXPORT lean_object* l_Lean_Parser_Module_prelude_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_prelude___closed__7; +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_import_parenthesizer___closed__3; lean_object* l_Lean_Parser_many_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_import_formatter___closed__2; static lean_object* l_Lean_Parser_Module_import_formatter___closed__4; static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__4; lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -131,10 +139,11 @@ static lean_object* l_Lean_Parser_Module_module___closed__4; lean_object* l_Lean_Parser_optional(lean_object*); static lean_object* l_Lean_Parser_Module_module_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Module_prelude_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Module_module_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__1; static lean_object* l_Lean_Parser_Module_module___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer(lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Parser_testParseModuleAux_parse___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_import_parenthesizer___closed__1; lean_object* l_Lean_Parser_initCacheForInput(lean_object*); @@ -147,11 +156,12 @@ static lean_object* l_Lean_Parser_testParseModuleAux_parse___closed__2; static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__2; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Parser_testParseModuleAux_parse___spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__13; -static lean_object* l_Lean_Parser_Module_header_formatter___closed__11; static lean_object* l_Lean_Parser_Module_header___closed__2; static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__8; lean_object* l_Lean_Parser_nodeInfo(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__17; static lean_object* l_Lean_Parser_Module_module___closed__6; static lean_object* l_Lean_Parser_Module_header_parenthesizer___closed__6; @@ -164,10 +174,12 @@ static lean_object* l_Lean_Parser_Module_header___closed__1; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Parser_parseCommand___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_import_parenthesizer___closed__8; static lean_object* l___private_Lean_Parser_Module_0__Lean_Parser_mkEOI___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_prelude_formatter(lean_object*); static lean_object* l_Lean_Parser_Module_module___elambda__1___closed__13; static lean_object* l___private_Lean_Parser_Module_0__Lean_Parser_mkErrorMessage___closed__1; static lean_object* l_Lean_Parser_Module_import_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Module_module___elambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_import_formatter(lean_object*); static lean_object* l_Lean_Parser_Module_import_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__11; lean_object* l_Lean_Syntax_updateLeading(lean_object*); @@ -191,6 +203,7 @@ lean_object* l_Array_back___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Parser_parseCommand___spec__1___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__7; static lean_object* l___private_Lean_Parser_Module_0__Lean_Parser_mkEOI___closed__5; +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; lean_object* l_Lean_Parser_addParserTokens(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_header_parenthesizer___closed__2; uint32_t lean_string_utf8_get(lean_object*, lean_object*); @@ -206,8 +219,9 @@ uint8_t l_Std_PersistentArray_isEmpty___rarg(lean_object*); extern lean_object* l_Lean_instInhabitedSyntax; static lean_object* l_Lean_Parser_Module_header_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Module_header_formatter___closed__9; -static lean_object* l_Lean_Parser_Module_module_formatter___closed__10; lean_object* l_Lean_Parser_whitespace(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_header_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Parser_testParseModuleAux_parse___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Module_module; static lean_object* l_Lean_Parser_Module_prelude_parenthesizer___closed__1; @@ -239,11 +253,13 @@ lean_object* lean_mk_empty_environment(uint32_t, lean_object*); lean_object* l_Lean_Parser_ident___elambda__1(lean_object*, lean_object*); uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l_Lean_Parser_Module_header_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Module_header_formatter___closed__2; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__7; lean_object* l_Lean_Parser_Error_toString(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_testParseFile(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_header_formatter(lean_object*); static lean_object* l_panic___at_Lean_Parser_Module_updateTokens___spec__1___closed__1; LEAN_EXPORT uint8_t l_Lean_Parser_isExitCommand(lean_object*); static lean_object* l_Lean_Parser_Module_module___elambda__1___closed__3; @@ -269,9 +285,10 @@ static lean_object* l_Lean_Parser_Module_module___elambda__1___closed__14; extern lean_object* l_Lean_Parser_epsilonInfo; static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__16; static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_module_formatter(lean_object*); lean_object* l_Lean_Parser_categoryParser___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Module_header_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Module_prelude___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Module_module_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__13; lean_object* l_Lean_Parser_ident_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -291,6 +308,7 @@ lean_object* l_Lean_mkListNode(lean_object*); static lean_object* l_Lean_Parser_Module_import___closed__5; static lean_object* l_Lean_Parser_Module_module_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Module_header_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Module_module___elambda__1___closed__7; lean_object* l_Lean_ppLine_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Parser_Module_0__Lean_Parser_consumeInput___closed__1; @@ -309,10 +327,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Module_prelude_parenthesizer(lean_object* LEAN_EXPORT lean_object* l_Lean_MessageLog_forM___at_Lean_Parser_testParseModuleAux_parse___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_many_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__20; +static lean_object* l___regBuiltin_Lean_Parser_Module_header_formatter___closed__1; static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__10; static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__3; static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__9; lean_object* l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__4; static lean_object* l_Lean_Parser_Module_header___elambda__1___closed__6; static lean_object* l_Lean_Parser_Module_header_formatter___closed__5; static lean_object* l_Lean_Parser_Module_import_formatter___closed__1; @@ -320,18 +340,22 @@ lean_object* l_Lean_Message_toString(lean_object*, uint8_t, lean_object*); lean_object* l_Lean_Parser_symbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__14; static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_import_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Module_header_formatter___closed__10; lean_object* l_Lean_Parser_ident_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Parser_parseCommand___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_utf8_at_end(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_header_formatter___closed__8; static lean_object* l_Lean_Parser_Module_module_formatter___closed__6; lean_object* l_Lean_Parser_symbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Module_prelude___elambda__1___closed__4; static lean_object* l_Lean_Parser_testParseModule___closed__1; static lean_object* l_Lean_Parser_Module_import___elambda__1___closed__6; static lean_object* l_Lean_Parser_Module_module___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_andthen_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_parseCommand(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_testParseModule(lean_object*, lean_object*, lean_object*, lean_object*); @@ -340,6 +364,7 @@ static lean_object* l_Lean_Parser_Module_header_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Module_import___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_isEOI___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Module_header___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__2; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Module_header_formatter___closed__4; lean_object* l_Lean_Parser_setLhsPrecFn___boxed(lean_object*, lean_object*, lean_object*); @@ -1682,6 +1707,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Module_prelude___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_prelude_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_prelude_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3; +x_3 = l_Lean_Parser_Module_prelude___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Module_import_formatter___closed__1() { _start: { @@ -1786,6 +1857,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_import_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Module_import___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_import_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_import_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_import_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3; +x_3 = l_Lean_Parser_Module_import___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Module_import_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Module_import_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__1() { _start: { @@ -1808,101 +1909,85 @@ static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_prelude_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__3() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_ppLine_formatter___boxed), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_header_formatter___closed__2; -x_2 = l_Lean_Parser_Module_header_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__4; +x_2 = l_Lean_Parser_Module_header_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Module_header_formatter___closed__4; +x_1 = l_Lean_Parser_Module_header_formatter___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_import_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_header_formatter___closed__6; -x_2 = l_Lean_Parser_Module_header_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Module_import_formatter___closed__2; +x_2 = l_Lean_Parser_Module_header_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Module_header_formatter___closed__7; +x_1 = l_Lean_Parser_Module_header_formatter___closed__5; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_header_formatter___closed__8; -x_2 = l_Lean_Parser_Module_header_formatter___closed__3; +x_1 = l_Lean_Parser_Module_header_formatter___closed__6; +x_2 = l_Lean_Parser_Module_header_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_header_formatter___closed__5; -x_2 = l_Lean_Parser_Module_header_formatter___closed__9; +x_1 = l_Lean_Parser_Module_header_formatter___closed__4; +x_2 = l_Lean_Parser_Module_header_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Module_header_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Module_header___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Module_header_formatter___closed__10; +x_3 = l_Lean_Parser_Module_header_formatter___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -1915,11 +2000,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Module_header_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Module_header_formatter___closed__1; -x_7 = l_Lean_Parser_Module_header_formatter___closed__11; +x_7 = l_Lean_Parser_Module_header_formatter___closed__9; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_header_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Module_header___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_header_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_header_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_header_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3; +x_3 = l_Lean_Parser_Module_header___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Module_header_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Module_header_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Module_module_formatter___closed__1() { _start: { @@ -1960,7 +2075,7 @@ static lean_object* _init_l_Lean_Parser_Module_module_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Module_header_formatter___closed__3; +x_1 = l_Lean_Parser_Module_header_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_2, 0, x_1); lean_closure_set(x_2, 1, x_1); @@ -2000,16 +2115,8 @@ return x_2; static lean_object* _init_l_Lean_Parser_Module_module_formatter___closed__8() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_header_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Module_module_formatter___closed__9() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_module_formatter___closed__8; +x_1 = l___regBuiltin_Lean_Parser_Module_header_formatter___closed__2; x_2 = l_Lean_Parser_Module_module_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -2017,13 +2124,13 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_module_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Module_module_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Module_module_formatter___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Module_module_formatter___closed__9; +x_3 = l_Lean_Parser_Module_module_formatter___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -2036,11 +2143,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Module_module_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Module_module_formatter___closed__3; -x_7 = l_Lean_Parser_Module_module_formatter___closed__10; +x_7 = l_Lean_Parser_Module_module_formatter___closed__9; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_module_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Module_module_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_module_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_module_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_module_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3; +x_3 = l_Lean_Parser_Module_module_formatter___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Module_module_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Module_module_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Module_prelude_parenthesizer___closed__1() { _start: { @@ -2093,6 +2230,52 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Module_prelude___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_prelude_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Module_prelude___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Module_import_parenthesizer___closed__1() { _start: { @@ -2197,6 +2380,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Module_import___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_import_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_import_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Module_import___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__1() { _start: { @@ -2219,101 +2432,85 @@ static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__2( _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_prelude_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppLine_parenthesizer___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Module_header_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Module_header_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_import_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Module_header_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Module_header_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__7; +x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__5; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__8; -x_2 = l_Lean_Parser_Module_header_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Module_header_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Module_header_parenthesizer___closed__9; +x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Module_header_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Module_header_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Module_header___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Module_header_parenthesizer___closed__10; +x_3 = l_Lean_Parser_Module_header_parenthesizer___closed__8; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -2326,11 +2523,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Module_header_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Module_header_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Module_header_parenthesizer___closed__11; +x_7 = l_Lean_Parser_Module_header_parenthesizer___closed__9; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Module_header___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_header_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_header_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Module_header___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Module_module_parenthesizer___closed__1() { _start: { @@ -2363,7 +2590,7 @@ static lean_object* _init_l_Lean_Parser_Module_module_parenthesizer___closed__3( _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Module_header_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_2, 0, x_1); lean_closure_set(x_2, 1, x_1); @@ -2395,16 +2622,8 @@ return x_2; static lean_object* _init_l_Lean_Parser_Module_module_parenthesizer___closed__6() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_header_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Module_module_parenthesizer___closed__7() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Module_module_parenthesizer___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__2; x_2 = l_Lean_Parser_Module_module_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -2412,13 +2631,13 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Module_module_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Module_module_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Module_module_formatter___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Module_module_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Module_module_parenthesizer___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -2431,11 +2650,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Module_module_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Module_module_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Module_module_parenthesizer___closed__8; +x_7 = l_Lean_Parser_Module_module_parenthesizer___closed__7; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Module_module_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Module_module_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Module_module_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Module_module_formatter___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Module_module___elambda__1___closed__1() { _start: { @@ -5234,6 +5483,17 @@ l_Lean_Parser_Module_prelude_formatter___closed__2 = _init_l_Lean_Parser_Module_ lean_mark_persistent(l_Lean_Parser_Module_prelude_formatter___closed__2); l_Lean_Parser_Module_prelude_formatter___closed__3 = _init_l_Lean_Parser_Module_prelude_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Module_prelude_formatter___closed__3); +l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__1); +l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__2); +l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__3); +l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_prelude_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Module_prelude_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Module_import_formatter___closed__1 = _init_l_Lean_Parser_Module_import_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Module_import_formatter___closed__1); l_Lean_Parser_Module_import_formatter___closed__2 = _init_l_Lean_Parser_Module_import_formatter___closed__2(); @@ -5250,6 +5510,13 @@ l_Lean_Parser_Module_import_formatter___closed__7 = _init_l_Lean_Parser_Module_i lean_mark_persistent(l_Lean_Parser_Module_import_formatter___closed__7); l_Lean_Parser_Module_import_formatter___closed__8 = _init_l_Lean_Parser_Module_import_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Module_import_formatter___closed__8); +l___regBuiltin_Lean_Parser_Module_import_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Module_import_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_import_formatter___closed__1); +l___regBuiltin_Lean_Parser_Module_import_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Module_import_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_import_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Module_import_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Module_header_formatter___closed__1 = _init_l_Lean_Parser_Module_header_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Module_header_formatter___closed__1); l_Lean_Parser_Module_header_formatter___closed__2 = _init_l_Lean_Parser_Module_header_formatter___closed__2(); @@ -5268,10 +5535,13 @@ l_Lean_Parser_Module_header_formatter___closed__8 = _init_l_Lean_Parser_Module_h lean_mark_persistent(l_Lean_Parser_Module_header_formatter___closed__8); l_Lean_Parser_Module_header_formatter___closed__9 = _init_l_Lean_Parser_Module_header_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Module_header_formatter___closed__9); -l_Lean_Parser_Module_header_formatter___closed__10 = _init_l_Lean_Parser_Module_header_formatter___closed__10(); -lean_mark_persistent(l_Lean_Parser_Module_header_formatter___closed__10); -l_Lean_Parser_Module_header_formatter___closed__11 = _init_l_Lean_Parser_Module_header_formatter___closed__11(); -lean_mark_persistent(l_Lean_Parser_Module_header_formatter___closed__11); +l___regBuiltin_Lean_Parser_Module_header_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Module_header_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_header_formatter___closed__1); +l___regBuiltin_Lean_Parser_Module_header_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Module_header_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_header_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Module_header_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Module_module_formatter___closed__1 = _init_l_Lean_Parser_Module_module_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Module_module_formatter___closed__1); l_Lean_Parser_Module_module_formatter___closed__2 = _init_l_Lean_Parser_Module_module_formatter___closed__2(); @@ -5290,14 +5560,30 @@ l_Lean_Parser_Module_module_formatter___closed__8 = _init_l_Lean_Parser_Module_m lean_mark_persistent(l_Lean_Parser_Module_module_formatter___closed__8); l_Lean_Parser_Module_module_formatter___closed__9 = _init_l_Lean_Parser_Module_module_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Module_module_formatter___closed__9); -l_Lean_Parser_Module_module_formatter___closed__10 = _init_l_Lean_Parser_Module_module_formatter___closed__10(); -lean_mark_persistent(l_Lean_Parser_Module_module_formatter___closed__10); +l___regBuiltin_Lean_Parser_Module_module_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Module_module_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_module_formatter___closed__1); +l___regBuiltin_Lean_Parser_Module_module_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Module_module_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_module_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Module_module_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Module_prelude_parenthesizer___closed__1 = _init_l_Lean_Parser_Module_prelude_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Module_prelude_parenthesizer___closed__1); l_Lean_Parser_Module_prelude_parenthesizer___closed__2 = _init_l_Lean_Parser_Module_prelude_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Module_prelude_parenthesizer___closed__2); l_Lean_Parser_Module_prelude_parenthesizer___closed__3 = _init_l_Lean_Parser_Module_prelude_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Module_prelude_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_Module_prelude_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Module_import_parenthesizer___closed__1 = _init_l_Lean_Parser_Module_import_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Module_import_parenthesizer___closed__1); l_Lean_Parser_Module_import_parenthesizer___closed__2 = _init_l_Lean_Parser_Module_import_parenthesizer___closed__2(); @@ -5314,6 +5600,13 @@ l_Lean_Parser_Module_import_parenthesizer___closed__7 = _init_l_Lean_Parser_Modu lean_mark_persistent(l_Lean_Parser_Module_import_parenthesizer___closed__7); l_Lean_Parser_Module_import_parenthesizer___closed__8 = _init_l_Lean_Parser_Module_import_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Module_import_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_import_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Module_import_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Module_header_parenthesizer___closed__1 = _init_l_Lean_Parser_Module_header_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Module_header_parenthesizer___closed__1); l_Lean_Parser_Module_header_parenthesizer___closed__2 = _init_l_Lean_Parser_Module_header_parenthesizer___closed__2(); @@ -5332,10 +5625,13 @@ l_Lean_Parser_Module_header_parenthesizer___closed__8 = _init_l_Lean_Parser_Modu lean_mark_persistent(l_Lean_Parser_Module_header_parenthesizer___closed__8); l_Lean_Parser_Module_header_parenthesizer___closed__9 = _init_l_Lean_Parser_Module_header_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Module_header_parenthesizer___closed__9); -l_Lean_Parser_Module_header_parenthesizer___closed__10 = _init_l_Lean_Parser_Module_header_parenthesizer___closed__10(); -lean_mark_persistent(l_Lean_Parser_Module_header_parenthesizer___closed__10); -l_Lean_Parser_Module_header_parenthesizer___closed__11 = _init_l_Lean_Parser_Module_header_parenthesizer___closed__11(); -lean_mark_persistent(l_Lean_Parser_Module_header_parenthesizer___closed__11); +l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_header_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Module_header_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Module_module_parenthesizer___closed__1 = _init_l_Lean_Parser_Module_module_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Module_module_parenthesizer___closed__1); l_Lean_Parser_Module_module_parenthesizer___closed__2 = _init_l_Lean_Parser_Module_module_parenthesizer___closed__2(); @@ -5350,8 +5646,13 @@ l_Lean_Parser_Module_module_parenthesizer___closed__6 = _init_l_Lean_Parser_Modu lean_mark_persistent(l_Lean_Parser_Module_module_parenthesizer___closed__6); l_Lean_Parser_Module_module_parenthesizer___closed__7 = _init_l_Lean_Parser_Module_module_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Module_module_parenthesizer___closed__7); -l_Lean_Parser_Module_module_parenthesizer___closed__8 = _init_l_Lean_Parser_Module_module_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Module_module_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Module_module_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Module_module_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Module_module___elambda__1___closed__1 = _init_l_Lean_Parser_Module_module___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Module_module___elambda__1___closed__1); l_Lean_Parser_Module_module___elambda__1___closed__2 = _init_l_Lean_Parser_Module_module___elambda__1___closed__2(); diff --git a/stage0/stdlib/Lean/Parser/Syntax.c b/stage0/stdlib/Lean/Parser/Syntax.c index d1b18f4c8f79..4dcfed6f0020 100644 --- a/stage0/stdlib/Lean/Parser/Syntax.c +++ b/stage0/stdlib/Lean/Parser/Syntax.c @@ -15,16 +15,19 @@ extern "C" { #endif static lean_object* l_Lean_Parser_Command_infixl___elambda__1___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_declRange(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__6; -static lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___lambda__1(lean_object*); static lean_object* l_Lean_Parser_Term_prio_quot___elambda__1___closed__15; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__1; static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__12; static lean_object* l_Lean_Parser_Syntax_cat___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntax_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_notation___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_declRange___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_mixfixKind___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_postfix___closed__6; @@ -35,6 +38,7 @@ static lean_object* l_Lean_Parser_Command_notationItem_parenthesizer___closed__1 static lean_object* l_Lean_Parser_Term_prec_quot___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_prefix___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_notationItem___closed__4; static lean_object* l_Lean_Parser_Command_macroTailTactic___elambda__1___closed__3; @@ -45,6 +49,7 @@ static lean_object* l_Lean_Parser_Command_prefix_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_infixl___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_notation_declRange___closed__7; static lean_object* l_Lean_Parser_Term_stx_quot_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_macro__rules___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_prio_quot; static lean_object* l_Lean_Parser_Command_syntaxCat___elambda__1___closed__5; @@ -59,6 +64,7 @@ static lean_object* l_Lean_Parser_Syntax_binary___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_elabTail_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_notation___closed__7; +static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__16; static lean_object* l_Lean_Parser_Syntax_binary___closed__5; static lean_object* l_Lean_Parser_Command_namedName_formatter___closed__1; static lean_object* l_Lean_Parser_Command_macroTailTactic___closed__1; @@ -82,12 +88,13 @@ static lean_object* l_Lean_Parser_Term_prec_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_macroTailTactic_formatter___closed__5; static lean_object* l_Lean_Parser_Command_optKind_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_syntaxParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_catBehavior_formatter___closed__8; static lean_object* l_Lean_Parser_Command_optKind___closed__13; static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_macroArg_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__2; lean_object* l_Lean_Parser_andthenInfo(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_elab___closed__13; static lean_object* l_Lean_Parser_Command_postfix_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mixfix; @@ -97,6 +104,10 @@ static lean_object* l_Lean_Parser_Command_catBehavior___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Syntax_numPrec___closed__3; static lean_object* l_Lean_Parser_Syntax_unary___elambda__1___closed__5; static lean_object* l_Lean_Parser_precedence___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__1; +static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__13; +lean_object* l_Lean_Parser_Term_attributes_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_macroTail_formatter___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -116,6 +127,7 @@ static lean_object* l_Lean_Parser_precedence___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_optKind_parenthesizer___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_declRange___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infix_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_macroRhs_formatter___closed__1; static lean_object* l_Lean_Parser_Term_prio_quot___closed__3; @@ -128,16 +140,19 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTailCommand_formatter(lean_o static lean_object* l_Lean_Parser_Term_stx_quot___closed__9; static lean_object* l_Lean_Parser_Command_macroTailTactic_formatter___closed__3; static lean_object* l_Lean_Parser_Command_macro__rules_formatter___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macroArg_formatter(lean_object*); static lean_object* l_Lean_Parser_Syntax_paren___closed__6; lean_object* l_Lean_Parser_Term_matchAlts(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntax___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macro_formatter___closed__6; static lean_object* l_Lean_Parser_Command_optKind_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_notation_declRange___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTail___elambda__1(lean_object*, lean_object*); lean_object* l_Lean_Parser_many(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules(lean_object*); static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_syntaxCat___elambda__1___closed__3; @@ -145,15 +160,17 @@ static lean_object* l_Lean_Parser_Command_elab_formatter___closed__7; static lean_object* l_Lean_Parser_Command_macroArg_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Syntax_nonReserved___closed__1; static lean_object* l_Lean_Parser_Syntax_sepBy1_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Syntax_nonReserved___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mixfix_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_setLhsPrecFn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_syntaxAbbrev___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_notationItem_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_stx_quot_parenthesizer___closed__5; static lean_object* l_Lean_Parser_precedence___elambda__1___closed__13; -static lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_namedName_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Syntax_unary___closed__1; @@ -200,8 +217,10 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_declRange(lean_ static lean_object* l_Lean_Parser_Syntax_cat___closed__4; static lean_object* l_Lean_Parser_Command_macroTail_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_sepBy1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__2; static lean_object* l_Lean_Parser_Command_infixr_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_macroTailTactic___closed__5; @@ -219,6 +238,7 @@ static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__20; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___closed__9; static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_macro__rules___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Syntax_paren_formatter___closed__4; static lean_object* l_Lean_Parser_Syntax_sepBy1_formatter___closed__2; static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__8; @@ -232,12 +252,12 @@ static lean_object* l_Lean_Parser_Syntax_binary_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__6; static lean_object* l_Lean_Parser_Syntax_unary___closed__2; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__12; -static lean_object* l_Lean_Parser_Command_macro_formatter___closed__13; static lean_object* l_Lean_Parser_Command_prefix___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_infixr_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macro__rules___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_namedName_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_identPrec___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroArg_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_declRange___closed__6; @@ -245,7 +265,9 @@ static lean_object* l_Lean_Parser_Term_stx_quot___closed__2; static lean_object* l_Lean_Parser_Term_prec_quot_formatter___closed__3; static lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_catBehavior_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_declRange___closed__1; static lean_object* l_Lean_Parser_Command_macroTailDefault_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -253,16 +275,19 @@ static lean_object* l_Lean_Parser_Command_mixfix_formatter___closed__3; static lean_object* l_Lean_Parser_Term_prec_quot_formatter___closed__5; static lean_object* l_Lean_Parser_Command_catBehavior_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_elab_declRange___closed__4; -static lean_object* l_Lean_Parser_Command_macro_formatter___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Syntax_paren_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_postfix_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroTailTactic___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_prefix; +static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__15; static lean_object* l_Lean_Parser_Command_elabTail_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_infixr___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroArg_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_elab__rules___closed__7; @@ -284,12 +309,14 @@ static lean_object* l_Lean_Parser_Command_notationItem___closed__3; static lean_object* l_Lean_Parser_Command_infixl_parenthesizer___closed__3; lean_object* l_Lean_Parser_withAntiquotFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macro_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__2; static lean_object* l_Lean_Parser_Command_namedName___closed__9; static lean_object* l_Lean_Parser_Command_mixfixKind___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_sepBy; static lean_object* l_Lean_Parser_Command_mixfix_formatter___closed__14; static lean_object* l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_paren; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_paren___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macro__rules___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_declRange___closed__6; @@ -305,23 +332,33 @@ static lean_object* l_Lean_Parser_Command_notation___closed__11; static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__16; static lean_object* l_Lean_Parser_Syntax_unary_parenthesizer___closed__1; extern lean_object* l_Lean_Parser_darrow; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_macroTailTactic_parenthesizer___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__1; static lean_object* l_Lean_Parser_Command_elab_formatter___closed__8; lean_object* l_Lean_Parser_priorityParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_declRange___closed__1; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__21; +static lean_object* l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__23; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_postfix_formatter(lean_object*); lean_object* l_Lean_Parser_Tactic_seq1_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehaviorSymbol___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__2; static lean_object* l_Lean_Parser_Command_elab_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mixfix___elambda__1___lambda__1___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Parser_Term_attributes_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_elabTail_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_optNamedName_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_declRange___closed__6; static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_numPrec___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_declRange___closed__1; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__13; static lean_object* l___regBuiltin_Lean_Parser_Syntax_numPrec___closed__4; @@ -360,14 +397,16 @@ static lean_object* l_Lean_Parser_Command_macroArg_formatter___closed__6; static lean_object* l_Lean_Parser_Command_identPrec_parenthesizer___closed__2; lean_object* l_Lean_Parser_addBuiltinParser(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroTail___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__1; static lean_object* l_Lean_Parser_Command_macroTail_formatter___closed__6; lean_object* l_Lean_Parser_optional_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_mixfixKind_formatter___closed__6; lean_object* lean_array_get_size(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_macro__rules_declRange___closed__6; static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infixr_formatter(lean_object*); extern lean_object* l_Lean_Parser_Tactic_seq1; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_paren_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__1; static lean_object* l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__9; @@ -379,16 +418,17 @@ static lean_object* l_Lean_Parser_Syntax_binary___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_infixr; static lean_object* l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_namedName___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_unary___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_elab_parenthesizer___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__4; static lean_object* l_Lean_Parser_Command_macroTailTactic_formatter___closed__2; -static lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_macro_declRange___closed__1; static lean_object* l_Lean_Parser_Command_infixl_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_declRange___closed__3; lean_object* l_Lean_Parser_mkAtomicInfo(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_macroArg_formatter___closed__2; static lean_object* l_Lean_Parser_Command_infixr___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mixfix___elambda__1___lambda__1(lean_object*, lean_object*); @@ -406,12 +446,13 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_declRange___closed lean_object* l_Lean_Parser_atomicFn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_elab___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__1; static lean_object* l_Lean_Parser_Command_catBehavior___closed__2; -static lean_object* l_Lean_Parser_Command_notationItem_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_macroTailTactic_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Syntax_numPrec___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__1; static lean_object* l_Lean_Parser_Syntax_cat_formatter___closed__2; static lean_object* l_Lean_Parser_Command_elab_formatter___closed__2; static lean_object* l_Lean_Parser_Command_notation_formatter___closed__5; @@ -431,9 +472,9 @@ static lean_object* l_Lean_Parser_Term_prec_quot___closed__7; static lean_object* l_Lean_Parser_precedence___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_optPrecedence; LEAN_EXPORT lean_object* l_Lean_Parser_Term_prec_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_infix___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_elab__rules___closed__10; -static lean_object* l_Lean_Parser_optPrecedence_formatter___closed__2; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_elab___closed__5; static lean_object* l_Lean_Parser_Command_postfix_parenthesizer___closed__1; @@ -455,11 +496,13 @@ static lean_object* l_Lean_Parser_Command_namedName___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_binary; LEAN_EXPORT lean_object* l_Lean_Parser_Command_elabArg; static lean_object* l_Lean_Parser_Command_macro__rules___closed__8; +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_infix; static lean_object* l_Lean_Parser_Command_macroRhs_formatter___closed__3; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__22; LEAN_EXPORT lean_object* l_Lean_Parser_Command_identPrec_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Syntax_numPrec___closed__2; static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__2; lean_object* l_Lean_Parser_many_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -470,8 +513,10 @@ static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__12; lean_object* l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_macro_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__2; static lean_object* l_Lean_Parser_Term_prio_quot___closed__6; static lean_object* l_Lean_Parser_Command_syntax___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__9; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_identPrec; @@ -485,7 +530,7 @@ static lean_object* l_Lean_Parser_Syntax_paren_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_mixfix___closed__12; static lean_object* l_Lean_Parser_Command_macroTailTactic_formatter___closed__1; static lean_object* l_Lean_Parser_Command_infixl___elambda__1___closed__1; -static lean_object* l_Lean_Parser_Command_optNamedName_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__2; lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_macroTailTactic_parenthesizer___closed__3; @@ -497,7 +542,9 @@ static lean_object* l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2 LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntaxAbbrev; LEAN_EXPORT lean_object* l_Lean_Parser_Command_notation_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_infix_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_postfix___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_macroArg___closed__5; @@ -512,6 +559,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_declRange___ static lean_object* l_Lean_Parser_Command_elab__rules___closed__5; static lean_object* l_Lean_Parser_Command_macro___closed__5; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__24; +static lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__2; static lean_object* l_Lean_Parser_optPrecedence_formatter___closed__1; lean_object* l_Lean_Parser_many1Fn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__2; @@ -528,6 +576,8 @@ static lean_object* l_Lean_Parser_Command_macroTailTactic_parenthesizer___closed static lean_object* l_Lean_Parser_Command_optKind___closed__16; static lean_object* l_Lean_Parser_Command_syntax___closed__5; static lean_object* l_Lean_Parser_Term_prio_quot___elambda__1___closed__13; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter(lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Syntax___hyg_5____closed__2; static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__12; lean_object* l_Lean_Parser_identEqFn(lean_object*, lean_object*, lean_object*); @@ -561,8 +611,11 @@ static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_declRange___closed__7; static lean_object* l_Lean_Parser_Command_macroTail___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_atom_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__1; lean_object* l_Lean_Parser_strLit___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_syntax___closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_precedence_formatter___closed__1; static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__11; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__16; @@ -579,19 +632,24 @@ LEAN_EXPORT lean_object* l_Lean_Parser_precedenceParser_formatter___rarg(lean_ob static lean_object* l_Lean_Parser_Command_macro__rules___elambda__1___closed__2; lean_object* l_Lean_Parser_Tactic_seq1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_infix___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_paren_formatter___closed__1; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__1; static lean_object* l_Lean_Parser_Command_elabTail___closed__8; static lean_object* l_Lean_Parser_Command_prefix___closed__4; static lean_object* l_Lean_Parser_Syntax_cat_formatter___closed__3; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_namedName_parenthesizer___closed__6; uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_infixl___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_declRange___closed__5; static lean_object* l_Lean_Parser_Syntax_paren___closed__9; static lean_object* l_Lean_Parser_Command_infix___elambda__1___closed__1; +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l_Lean_Parser_Term_stx_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_macro___closed__3; static lean_object* l_Lean_Parser_Syntax_cat___closed__1; @@ -601,14 +659,19 @@ static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_notation_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1; static lean_object* l_Lean_Parser_Term_prec_quot___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_macroArg___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_unary(lean_object*); static lean_object* l_Lean_Parser_Command_macroTailCommand_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__1; static lean_object* l_Lean_Parser_precedence_formatter___closed__2; static lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_formatter(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_withAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__3; @@ -621,6 +684,7 @@ static lean_object* l_Lean_Parser_Command_elab_parenthesizer___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Command_infixl; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_catBehaviorSymbol___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_stx_quot___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_prec_quot___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_macro__rules_formatter___closed__10; @@ -633,12 +697,14 @@ static lean_object* l_Lean_Parser_Command_postfix___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_prefix___elambda__1___closed__5; static lean_object* l_Lean_Parser_precedence___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_optKind___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_binary_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_numPrec_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_namedName___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_macroTail_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_infixl___elambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_optPrecedence_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__1; static lean_object* l_Lean_Parser_precedence_formatter___closed__4; static lean_object* l_Lean_Parser_Command_macro__rules___closed__1; static lean_object* l_Lean_Parser_Command_macroTail_formatter___closed__2; @@ -650,11 +716,13 @@ static lean_object* l_Lean_Parser_Command_infix_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_elabTail___closed__4; static lean_object* l_Lean_Parser_Command_mixfix___closed__11; static lean_object* l_Lean_Parser_Command_postfix___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mixfix_formatter___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macro(lean_object*); static lean_object* l_Lean_Parser_Term_stx_quot___elambda__1___closed__18; static lean_object* l_Lean_Parser_Command_macroTailCommand___closed__3; static lean_object* l_Lean_Parser_Command_elabTail___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_unary_formatter___closed__5; static lean_object* l_Lean_Parser_Command_macro__rules_formatter___closed__3; lean_object* l_Lean_Parser_nonReservedSymbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); @@ -662,6 +730,7 @@ static lean_object* l_Lean_Parser_Command_elabTail_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_mixfixKind___elambda__1___closed__1; static lean_object* l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_cat(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__16; static lean_object* l_Lean_Parser_Syntax_binary___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_declRange___closed__5; @@ -672,6 +741,9 @@ static lean_object* l_Lean_Parser_Command_macroTail_formatter___closed__4; static lean_object* l_Lean_Parser_Command_notation_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___closed__10; static lean_object* l_Lean_Parser_Syntax_binary___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_notation___closed__5; @@ -684,6 +756,8 @@ static lean_object* l_Lean_Parser_Command_notation_formatter___closed__6; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Syntax_paren_parenthesizer___closed__6; lean_object* l_Lean_Parser_nodeInfo(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_declRange___closed__4; static lean_object* l_Lean_Parser_Command_elabTail_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_infix___closed__1; @@ -720,6 +794,7 @@ static lean_object* l_Lean_Parser_Command_infix___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_macroTail___elambda__1___closed__3; static lean_object* l_Lean_Parser_Syntax_paren_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Syntax_binary___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_prefix___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_macroTailCommand_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_macro__rules___closed__4; @@ -728,11 +803,13 @@ lean_object* l_Lean_PrettyPrinter_Formatter_categoryParserOfStack_formatter___bo lean_object* l_Lean_PrettyPrinter_Parenthesizer_suppressInsideQuot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_prefix___closed__1; static lean_object* l_Lean_Parser_Command_infixl___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_formatter(lean_object*); lean_object* l_Lean_Parser_nonReservedSymbolInfo(lean_object*, uint8_t); static lean_object* l_Lean_Parser_Command_syntax___closed__15; lean_object* l_Lean_Parser_strLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_catBehaviorSymbol___elambda__1___closed__10; lean_object* l_Lean_Parser_checkNoWsBefore___elambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_checkPrec_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -750,6 +827,7 @@ static lean_object* l_Lean_Parser_Command_syntax___closed__3; static lean_object* l_Lean_Parser_Term_prec_quot_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__4; static lean_object* l_Lean_Parser_Command_optKind_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_declRange___closed__4; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__15; @@ -762,6 +840,7 @@ static lean_object* l_Lean_Parser_Command_elabTail_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_stx_quot_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_precedenceParser_formatter___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_stx_quot; +static lean_object* l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__1; static lean_object* l_Lean_Parser_Command_elab__rules___closed__6; static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__1; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__18; @@ -779,20 +858,25 @@ LEAN_EXPORT lean_object* l_Lean_Parser_optPrecedence_parenthesizer(lean_object*, static lean_object* l_Lean_Parser_Syntax_binary_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_catBehavior___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_elab_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_declRange___closed__6; static lean_object* l_Lean_Parser_Command_macro__rules___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_notation_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optKind_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_elab__rules; static lean_object* l_Lean_Parser_Command_macro__rules___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Command_macro_formatter___closed__1; static lean_object* l_Lean_Parser_Command_macroTailCommand___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macro_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_macroTailCommand_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_postfix___closed__5; @@ -834,6 +918,7 @@ static lean_object* l_Lean_Parser_Command_macro__rules_formatter___closed__5; static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_declRange___closed__3; static lean_object* l_Lean_Parser_Term_prec_quot___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_declRange___closed__1; static lean_object* l_Lean_Parser_Command_namedName___closed__12; static lean_object* l_Lean_Parser_Command_namedName_formatter___closed__4; @@ -841,7 +926,6 @@ static lean_object* l_Lean_Parser_Syntax_unary___elambda__1___closed__9; static lean_object* l_Lean_Parser_precedence___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_macroRhs___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__13; -static lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_identPrec___closed__3; static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_declRange___closed__4; @@ -859,6 +943,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_declRange___closed__1 static lean_object* l_Lean_Parser_Term_prec_quot___elambda__1___closed__4; static lean_object* l_Lean_Parser_Command_macroRhs___closed__1; static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__1; static lean_object* l_Lean_Parser_Term_stx_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_elab_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__6; @@ -875,9 +960,11 @@ static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_declRange___ static lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_declRange___closed__4; static lean_object* l_Lean_Parser_Command_catBehavior___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_elab_formatter___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_binary_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__18; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infix_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__19; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_unary_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Syntax_unary___closed__7; @@ -903,7 +990,6 @@ static lean_object* l_Lean_Parser_Term_prio_quot___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_cat; static lean_object* l_Lean_Parser_Command_macroTailDefault_formatter___closed__1; static lean_object* l_Lean_Parser_Command_catBehavior_formatter___closed__6; -static lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_declRange___closed__5; static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_binary___elambda__1(lean_object*, lean_object*); @@ -926,12 +1012,14 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntaxCat_parenthesizer(lean_obje static lean_object* l_Lean_Parser_Command_macroRhs___elambda__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_nonReserved_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macroTail_formatter(lean_object*); static lean_object* l_Lean_Parser_Syntax_nonReserved___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTailTactic; static lean_object* l_Lean_Parser_Command_catBehavior___closed__13; static lean_object* l_Lean_Parser_Command_namedName_formatter___closed__9; static lean_object* l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___closed__6; +extern lean_object* l_Lean_Parser_Term_attributes; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__5; static lean_object* l_Lean_Parser_Syntax_binary_formatter___closed__6; @@ -969,6 +1057,7 @@ static lean_object* l_Lean_Parser_Command_macro___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_declRange___closed__1; static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__9; lean_object* l_Lean_PrettyPrinter_Formatter_many1Unbox_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_declRange___closed__1; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__5; @@ -976,6 +1065,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_infixr_parenthesizer(lean_object* static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__13; static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__18; +static lean_object* l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_numPrec_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__13; @@ -984,6 +1074,7 @@ static lean_object* l_Lean_Parser_Term_prec_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_mixfixKind___closed__1; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_declRange___closed__7; +static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__28; static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__9; static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_catBehaviorSymbol___closed__4; @@ -999,6 +1090,7 @@ static lean_object* l_Lean_Parser_Syntax_numPrec___closed__3; static lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Command_macroTail_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_optKind___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_namedName_formatter___closed__8; static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__17; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__13; @@ -1013,6 +1105,7 @@ static lean_object* l_Lean_Parser_Command_catBehaviorBoth___closed__5; static lean_object* l_Lean_Parser_Term_prio_quot_parenthesizer___closed__7; extern lean_object* l_Lean_Parser_Command_optNamedPrio; static lean_object* l_Lean_Parser_Term_prio_quot___elambda__1___closed__6; +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; static lean_object* l_Lean_Parser_Command_macro__rules___elambda__1___closed__3; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_stx_quot_parenthesizer___closed__4; @@ -1020,6 +1113,7 @@ uint32_t lean_string_utf8_get(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mixfix_formatter___closed__8; static lean_object* l_Lean_Parser_Command_namedName_formatter___closed__5; static lean_object* l_Lean_Parser_Syntax_numPrec_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__1; static lean_object* l_Lean_Parser_Command_infixr___closed__5; static lean_object* l_Lean_Parser_Command_macroTailCommand_formatter___closed__3; static lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer___closed__2; @@ -1048,7 +1142,9 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehaviorBoth_formatter(lean_ob static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__13; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_macroTailCommand_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_precedence_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehaviorSymbol; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntax_formatter(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_declRange(lean_object*); static lean_object* l_Lean_Parser_precedence_parenthesizer___closed__4; lean_object* l_Lean_PrettyPrinter_Parenthesizer_many1Unbox_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1065,6 +1161,7 @@ static lean_object* l_Lean_Parser_Syntax_binary___elambda__1___closed__1; static lean_object* l_Lean_Parser_Syntax_cat___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_prefix___closed__2; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__26; +static lean_object* l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__2; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_infix_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_declRange___closed__6; @@ -1087,12 +1184,15 @@ static lean_object* l_Lean_Parser_Term_prec_quot___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehaviorBoth___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroTailDefault_parenthesizer___closed__3; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Syntax___hyg_5____closed__5; +static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__17; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_unary; static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_declRange___closed__4; static lean_object* l_Lean_Parser_Term_stx_quot_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_macroArg_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_prio_quot_formatter___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_formatter(lean_object*); static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__17; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_catBehaviorSymbol___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macro_declRange(lean_object*); @@ -1103,14 +1203,15 @@ static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Syntax___hyg_37____c static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Syntax_binary___closed__1; static lean_object* l_Lean_Parser_Syntax_numPrec___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat(lean_object*); static lean_object* l_Lean_Parser_Term_prio_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__3; static lean_object* l_Lean_Parser_Syntax_sepBy___closed__2; -static lean_object* l_Lean_Parser_Command_mixfixKind_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_notation_declRange___closed__4; static lean_object* l_Lean_Parser_Command_macroTail_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Command_mixfix_formatter___closed__4; @@ -1133,7 +1234,6 @@ static lean_object* l_Lean_Parser_Command_macroTailTactic_parenthesizer___closed LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedName___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__2; static lean_object* l_Lean_Parser_Syntax_numPrec___closed__1; -static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__13; static lean_object* l_Lean_Parser_Syntax_unary_formatter___closed__4; static lean_object* l_Lean_Parser_Command_macro___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_precedence_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1144,7 +1244,9 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_unary_parenthesizer(lean_object*, static lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_declRange___closed__1; static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_atom; +static lean_object* l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__2; static lean_object* l_Lean_Parser_Command_elab__rules___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_stx_quot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1___closed__8; static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__13; @@ -1157,7 +1259,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_declRange___closed_ static lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_declRange___closed__6; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___closed__10; static lean_object* l_Lean_Parser_Command_macroTailTactic___elambda__1___closed__2; -static lean_object* l_Lean_Parser_Command_catBehavior_formatter___closed__7; static lean_object* l_Lean_Parser_Syntax_cat_formatter___closed__1; static lean_object* l_Lean_Parser_Command_namedName_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_prec_quot___closed__5; @@ -1165,12 +1266,14 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_nonReserved; static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_macroTailCommand___closed__1; static lean_object* l_Lean_Parser_Command_identPrec___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__1; static lean_object* l_Lean_Parser_Syntax_paren_formatter___closed__7; static lean_object* l_Lean_Parser_Command_catBehaviorBoth_formatter___closed__1; static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_syntax___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Command_macro_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__5; static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__21; LEAN_EXPORT lean_object* l_Lean_Parser_Term_prio_quot___elambda__1(lean_object*, lean_object*); @@ -1185,6 +1288,7 @@ static lean_object* l_Lean_Parser_precedence___closed__3; static lean_object* l_Lean_Parser_Command_macroArg___closed__4; static lean_object* l_Lean_Parser_Command_notationItem___closed__1; static lean_object* l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_formatter(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_withPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__5; lean_object* l_Lean_Parser_withResultOfFn(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1196,11 +1300,14 @@ static lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer___closed__4 lean_object* l_Lean_Parser_many1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_namedName___elambda__1___closed__21; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_precedence_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_binary___closed__11; static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__2; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Syntax___hyg_5____closed__6; static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__1; static lean_object* l_Lean_Parser_Command_infixr_formatter___closed__1; static lean_object* l_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2; static lean_object* l_Lean_Parser_Command_macroRhs_parenthesizer___closed__1; @@ -1214,6 +1321,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_optNamedName_parenthesizer(lean_o static lean_object* l_Lean_Parser_Command_elab_formatter___closed__4; static lean_object* l_Lean_Parser_Command_macroArg_formatter___closed__5; static lean_object* l_Lean_Parser_Command_elab__rules___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_notation_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_syntax___closed__13; @@ -1222,6 +1330,7 @@ static lean_object* l_Lean_Parser_Command_macroTail___closed__8; static lean_object* l_Lean_Parser_Syntax_unary_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Syntax_unary___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_declRange___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1___closed__17; @@ -1230,11 +1339,16 @@ static lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer___closed__9 static lean_object* l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_postfix___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_precedence; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Syntax_binary_formatter___closed__1; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_macroTailTactic___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_declRange___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroRhs(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__2; lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_nonReserved_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1255,6 +1369,7 @@ static lean_object* l_Lean_Parser_Term_prio_quot___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_prio_quot_formatter___closed__3; static lean_object* l_Lean_Parser_Command_prefix_formatter___closed__3; static lean_object* l_Lean_Parser_Command_syntaxCat___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_infix___elambda__1___closed__6; @@ -1272,6 +1387,7 @@ lean_object* l_Lean_Parser_commandParser_formatter___rarg(lean_object*, lean_obj static lean_object* l_Lean_Parser_Command_macro_formatter___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_declRange___closed__1; lean_object* l_Lean_Parser_ident___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_macro__rules___elambda__1___closed__9; static lean_object* l_Lean_Parser_precedence___elambda__1___closed__10; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkNoWsBefore_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1286,6 +1402,7 @@ static lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_syntaxCat___elambda__1___closed__9; extern lean_object* l_Lean_Parser_numLit; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Syntax_paren___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mixfixKind___elambda__1(lean_object*, lean_object*); @@ -1293,6 +1410,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_numPrec_declRange(lea static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehaviorBoth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elabTail_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_macro_declRange___closed__5; static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__13; @@ -1309,12 +1427,14 @@ static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__3; lean_object* l_Lean_Parser_numLit___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_prio_quot___closed__10; static lean_object* l_Lean_Parser_Command_mixfix_formatter___closed__11; +static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Command_namedName___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__17; static lean_object* l_Lean_Parser_Syntax_atom___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_prio_quot___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macro; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_syntax___closed__6; static lean_object* l_Lean_Parser_Term_stx_quot___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_infix_parenthesizer___closed__1; @@ -1324,6 +1444,7 @@ static lean_object* l_Lean_Parser_Term_prio_quot___elambda__1___closed__4; lean_object* l_Lean_Syntax_getNumArgs(lean_object*); static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__1; static lean_object* l_Lean_Parser_precedence___closed__5; static lean_object* l_Lean_Parser_Command_notation_parenthesizer___closed__8; @@ -1331,6 +1452,7 @@ static lean_object* l_Lean_Parser_Command_macroRhs___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___lambda__1___boxed(lean_object*); extern lean_object* l_Lean_Parser_Term_attrKind; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_infixl___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroTailCommand_parenthesizer___closed__6; @@ -1342,6 +1464,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer(lean_ob static lean_object* l_Lean_Parser_Syntax_atom_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Command_macro_declRange___closed__3; static lean_object* l_Lean_Parser_Command_postfix___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__1; static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__18; static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__12; static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__10; @@ -1366,6 +1489,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_cat___elambda__1(lean_object*, lea static lean_object* l_Lean_Parser_Syntax_unary_formatter___closed__2; static lean_object* l_Lean_Parser_Term_prio_quot___elambda__1___closed__17; static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_binary___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__8; static lean_object* l_Lean_Parser_precedence___elambda__1___closed__11; @@ -1386,10 +1510,12 @@ static lean_object* l_Lean_Parser_Command_macroTail___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_macroRhs___closed__4; static lean_object* l_Lean_Parser_precedence_parenthesizer___closed__5; lean_object* l_Lean_Parser_commandParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Syntax_unary___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__2; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___closed__7; static lean_object* l_Lean_Parser_Command_namedName_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Syntax_binary___elambda__1___closed__13; @@ -1405,13 +1531,16 @@ static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_notationItem___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_infixl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Syntax_binary_formatter___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__2; static lean_object* l_Lean_Parser_Command_catBehavior___closed__10; static lean_object* l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_prec_quot___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_declRange___closed__5; static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Command_notation_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; static lean_object* l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__2; static lean_object* l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__9; static lean_object* l_Lean_Parser_Syntax_atom___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__4; @@ -1426,16 +1555,20 @@ static lean_object* l_Lean_Parser_Term_prio_quot___elambda__1___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_incQuotDepth_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroTailCommand_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_elab__rules___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2; static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__12; static lean_object* l_Lean_Parser_Command_syntaxCat___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__1; static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Command_elab_formatter___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntaxAbbrev_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_precedenceParser(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_macroRhs_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_macroTailTactic___closed__6; static lean_object* l_Lean_Parser_Command_notation___closed__1; @@ -1468,8 +1601,8 @@ static lean_object* l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_optKind___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_declRange___closed__6; -static lean_object* l_Lean_Parser_Command_notationItem_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_elabArg_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__2; extern lean_object* l_Lean_Parser_Command_docComment; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__14; lean_object* l_Lean_Parser_orelseFnCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); @@ -1502,12 +1635,14 @@ static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__20; lean_object* l_Lean_Parser_categoryParser___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__21; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_atom___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_postfix___closed__2; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_elab__rules___closed__9; static lean_object* l_Lean_Parser_Command_notation___closed__4; static lean_object* l_Lean_Parser_Term_prec_quot___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_optKind___closed__12; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_identPrec___closed__2; @@ -1518,9 +1653,9 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_declRange___closed static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__3; static lean_object* l_Lean_Parser_Command_syntaxCat___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__8; -static lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_syntaxCat_formatter___closed__6; static lean_object* l_Lean_Parser_Syntax_cat___closed__7; @@ -1528,11 +1663,13 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_cat_formatter(lean_object*, lean_o static lean_object* l_Lean_Parser_Command_syntaxCat___closed__8; static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_infix___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_infix_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_optKind___closed__9; static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__3; static lean_object* l_Lean_Parser_Command_mixfixKind_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_precedenceParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__5; static lean_object* l_Lean_Parser_Command_notation___closed__9; static lean_object* l_Lean_Parser_Command_notation_formatter___closed__3; @@ -1558,14 +1695,19 @@ static lean_object* l_Lean_Parser_Command_postfix___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroArg___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev(lean_object*); static lean_object* l_Lean_Parser_Syntax_paren___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Syntax_cat_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_notation_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__1; static lean_object* l_Lean_Parser_Command_infixl___closed__1; static lean_object* l_Lean_Parser_Syntax_unary___closed__5; static lean_object* l_Lean_Parser_Command_optKind___closed__4; +static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__27; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_declRange___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_syntax___closed__11; static lean_object* l_Lean_Parser_Command_macroTail___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Syntax_numPrec_declRange___closed__5; @@ -1581,7 +1723,7 @@ static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__15; static lean_object* l_Lean_Parser_Syntax_atom___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_mixfixKind___closed__6; -static lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_notation_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__4; @@ -1605,19 +1747,20 @@ static lean_object* l_Lean_Parser_Command_macro__rules_formatter___closed__8; static lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_macroRhs___closed__2; static lean_object* l_Lean_Parser_Command_postfix___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__2; lean_object* l_Lean_Parser_darrow___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_elab_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Command_macro__rules___elambda__1___closed__10; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_prec_quot___elambda__1___closed__11; lean_object* l_Lean_Parser_nodeFn(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Command_elab_parenthesizer___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_declRange___closed__2; static lean_object* l_Lean_Parser_Command_optKind_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_binary_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTailTactic___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__10; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_identPrec_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__16; static lean_object* l_Lean_Parser_Command_mixfixKind___closed__3; static lean_object* l_Lean_Parser_Command_infixr___elambda__1___closed__1; @@ -1636,6 +1779,7 @@ static lean_object* l_Lean_Parser_Command_namedName___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_macro__rules_formatter___closed__1; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_namedName___closed__7; static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_notationItem___closed__5; @@ -1648,12 +1792,15 @@ static lean_object* l_Lean_Parser_Command_postfix_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_elab___closed__9; static lean_object* l_Lean_Parser_Command_namedName___elambda__1___closed__14; static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_catBehaviorSymbol___closed__3; static lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Command_notation_declRange___closed__3; static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_stx_quot___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__3; static lean_object* l_Lean_Parser_Command_notation_parenthesizer___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Command_elabArg_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1661,16 +1808,19 @@ static lean_object* l_Lean_Parser_Command_namedName___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_macro___closed__8; static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__7; static lean_object* l_Lean_Parser_Command_macroTailDefault_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_mixfixKind___closed__4; static lean_object* l_Lean_Parser_Command_syntaxCat___closed__9; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__15; static lean_object* l_Lean_Parser_Command_mixfix___closed__14; static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_prefix_formatter(lean_object*); static lean_object* l_Lean_Parser_Syntax_numPrec_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedName_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Command_elab_declRange___closed__5; static lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_prec_quot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__3; @@ -1679,6 +1829,7 @@ static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__18; static lean_object* l_Lean_Parser_Command_notationItem_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Syntax_binary_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_identPrec___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__1; static lean_object* l_Lean_Parser_Command_infix___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__17; static lean_object* l_Lean_Parser_Command_macroArg_parenthesizer___closed__2; @@ -1686,11 +1837,14 @@ static lean_object* l_Lean_Parser_Command_macro__rules___closed__3; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__18; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Syntax___hyg_37____closed__3; static lean_object* l_Lean_Parser_Command_syntaxCat___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macro_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_prio_quot_formatter___closed__1; lean_object* l_Lean_Parser_mkAntiquot(lean_object*, lean_object*, uint8_t, uint8_t); static lean_object* l_Lean_Parser_Term_stx_quot___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Command_macro_declRange___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_precedence_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__1; static lean_object* l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__9; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__3; @@ -1727,6 +1881,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_declRange___closed_ static lean_object* l_Lean_Parser_Command_elab__rules___closed__11; static lean_object* l_Lean_Parser_Command_catBehaviorSymbol___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_macroTailTactic_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__2; static lean_object* l_Lean_Parser_Syntax_atom_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_notation_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_macroTailDefault___elambda__1___closed__2; @@ -1740,6 +1895,7 @@ static lean_object* l_Lean_Parser_Syntax_binary_formatter___closed__3; static lean_object* l_Lean_Parser_Syntax_nonReserved___closed__4; static lean_object* l_Lean_Parser_Command_elab___elambda__1___closed__10; static lean_object* l_Lean_Parser_Syntax_cat___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_notation_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_declRange___closed__4; @@ -1755,14 +1911,17 @@ static lean_object* l_Lean_Parser_Command_infix___elambda__1___closed__3; static lean_object* l_Lean_Parser_Syntax_unary___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_macro__rules___closed__2; static lean_object* l_Lean_Parser_Syntax_binary___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__2; static lean_object* l_Lean_Parser_Command_syntaxCat_formatter___closed__3; static lean_object* l_Lean_Parser_Command_namedName_formatter___closed__7; static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__22; static lean_object* l_Lean_Parser_Command_syntax___closed__9; static lean_object* l_Lean_Parser_Command_elabTail_formatter___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_notationItem___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_macroTailDefault___closed__2; static lean_object* l_Lean_Parser_Command_mixfix_parenthesizer___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infixl_formatter(lean_object*); static lean_object* l_Lean_Parser_Syntax_cat___elambda__1___closed__6; static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_declRange(lean_object*); @@ -1771,6 +1930,7 @@ static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__14; static lean_object* l_Lean_Parser_Syntax_atom___closed__2; static lean_object* l_Lean_Parser_precedence___closed__2; static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__2; static lean_object* l_Lean_Parser_Command_syntaxCat_formatter___closed__5; static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__10; @@ -1786,8 +1946,11 @@ static lean_object* l_Lean_Parser_Term_prec_quot___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_infix_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1; static lean_object* l_Lean_Parser_Command_namedName___elambda__1___closed__18; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namedName_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_syntaxParser_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_elab___closed__1; static lean_object* l_Lean_Parser_Command_macroTailDefault___elambda__1___closed__1; @@ -1799,6 +1962,8 @@ static lean_object* l_Lean_Parser_Command_identPrec___closed__1; static lean_object* l_Lean_Parser_Syntax_cat___closed__5; static lean_object* l_Lean_Parser_Command_macroRhs_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__2; lean_object* l_Lean_Parser_Term_matchAlts_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_catBehaviorBoth___closed__2; static lean_object* l_Lean_Parser_Syntax_sepBy_formatter___closed__4; @@ -1822,6 +1987,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Syntax_numPrec_declRange___closed static lean_object* l_Lean_Parser_Command_elab_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Syntax_paren___elambda__1___closed__20; lean_object* l_Lean_Parser_symbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_suppressInsideQuot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_syntax___closed__2; static lean_object* l_Lean_Parser_Command_macroTail___closed__6; @@ -1829,6 +1995,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy(lean_object*); static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_catBehaviorSymbol___closed__7; static lean_object* l_Lean_Parser_Command_elabTail___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__1; static lean_object* l_Lean_Parser_Command_optNamedName___closed__1; static lean_object* l_Lean_Parser_Command_mixfixKind___closed__5; static lean_object* l_Lean_Parser_Command_catBehavior___closed__11; @@ -1844,7 +2011,7 @@ static lean_object* l_Lean_Parser_Syntax_cat___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_syntaxCat___elambda__1___closed__13; static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__5; static lean_object* l_Lean_Parser_Command_syntax_parenthesizer___closed__7; -static lean_object* l_Lean_Parser_Command_mixfixKind_formatter___closed__7; +static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__14; static lean_object* l_Lean_Parser_Command_elab___closed__8; static lean_object* l_Lean_Parser_Command_elab__rules_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Command_macroTail_formatter___closed__7; @@ -1853,16 +2020,21 @@ static lean_object* l_Lean_Parser_Command_identPrec___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_macro__rules_formatter___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_precedenceParser_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_macro__rules_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTailCommand_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_prec_quot___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__2; static lean_object* l_Lean_Parser_Command_mixfix_formatter___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_namedName; lean_object* l_Lean_Parser_ident_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_infixr___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__1; static lean_object* l_Lean_Parser_Command_macro__rules_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_prefix_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntaxCat; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Syntax_cat___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_prio_quot_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_declRange___closed__7; @@ -1873,6 +2045,7 @@ static lean_object* l_Lean_Parser_Command_elab_formatter___closed__5; static lean_object* l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__5; static lean_object* l_Lean_Parser_Syntax_atom___closed__3; lean_object* l_Lean_PrettyPrinter_Parenthesizer_categoryParserOfStack_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__2; lean_object* l_Lean_Parser_withResultOfInfo(lean_object*); static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTailTactic_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1880,7 +2053,6 @@ static lean_object* l_Lean_Parser_Command_catBehavior___closed__12; static lean_object* l_Lean_Parser_Command_macroArg_formatter___closed__7; static lean_object* l_Lean_Parser_Command_notation___elambda__1___closed__14; static lean_object* l_Lean_Parser_Command_macroArg_parenthesizer___closed__7; -static lean_object* l_Lean_Parser_optPrecedence_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab(lean_object*); static lean_object* l_Lean_Parser_Command_elabTail___closed__3; static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__5; @@ -1902,6 +2074,7 @@ static lean_object* l_Lean_Parser_Command_prefix_formatter___closed__2; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Syntax___hyg_5____closed__3; static lean_object* l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_prefix___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__2; static lean_object* l_Lean_Parser_Command_macroTailTactic___closed__7; static lean_object* l_Lean_Parser_Syntax_binary___elambda__1___closed__12; static lean_object* l_Lean_Parser_Command_infixr___elambda__1___closed__2; @@ -1913,19 +2086,18 @@ static lean_object* l_Lean_Parser_Command_macroTail___closed__3; static lean_object* l_Lean_Parser_Command_elab__rules_formatter___closed__9; static lean_object* l_Lean_Parser_Command_catBehaviorSymbol___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_macroTail___closed__1; -static lean_object* l_Lean_Parser_Command_mixfixKind_formatter___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntax(lean_object*); static lean_object* l_Lean_Parser_Term_prec_quot___closed__6; lean_object* l_Lean_PrettyPrinter_Parenthesizer_identEq_parenthesizer___boxed(lean_object*, lean_object*); lean_object* l_Lean_Parser_Term_attrKind___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_macro__rules_declRange___closed__4; static lean_object* l_Lean_Parser_Command_infixl_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macro_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehaviorSymbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_mixfix___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_macroArg___elambda__1___closed__7; -static lean_object* l_Lean_Parser_Command_macro_parenthesizer___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_declRange___closed__7; static lean_object* l_Lean_Parser_Syntax_sepBy1___closed__7; static lean_object* l_Lean_Parser_Term_prio_quot___closed__7; @@ -1943,6 +2115,7 @@ static lean_object* l_Lean_Parser_Command_elab_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_namedName_formatter___closed__2; static lean_object* l_Lean_Parser_Command_elabTail_formatter___closed__1; static lean_object* l_Lean_Parser_Command_infixr___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__2; static lean_object* l_Lean_Parser_Command_syntax_formatter___closed__6; static lean_object* l_Lean_Parser_Command_elab___closed__2; static lean_object* l_Lean_Parser_Syntax_binary_parenthesizer___closed__6; @@ -1957,14 +2130,19 @@ static lean_object* l_Lean_Parser_Command_mixfix___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_declRange___closed__1; static lean_object* l_Lean_Parser_Command_prefix___elambda__1___closed__1; static lean_object* l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__2; +static lean_object* l_Lean_Parser_Command_syntax___closed__17; +static lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_syntaxCat___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Command_macro___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_prio_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_elab__rules___elambda__1___closed__16; static lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_declRange___closed__7; static lean_object* l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__11; static lean_object* l_Lean_Parser_Command_optKind___closed__14; -static lean_object* l_Lean_Parser_Command_elab_formatter___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_notationItem_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_notationItem; @@ -1976,16 +2154,18 @@ static lean_object* l_Lean_Parser_Command_namedName___elambda__1___closed__7; static lean_object* l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__6; lean_object* l_Lean_Parser_termParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_macro__rules_declRange___closed__3; -static lean_object* l_Lean_Parser_Command_mixfixKind_formatter___closed__8; static lean_object* l_Lean_Parser_Command_syntax___elambda__1___closed__11; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1(lean_object*); static lean_object* l_Lean_Parser_Command_infixr___elambda__1___closed__9; static lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_elab__rules___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroTailCommand___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_precedence_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__3; static lean_object* l_Lean_Parser_precedence___closed__8; static lean_object* l_Lean_Parser_Command_macroTailCommand_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__2; static lean_object* l_Lean_Parser_Command_macro___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_sepBy1_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Syntax_cat_parenthesizer___closed__4; @@ -1994,12 +2174,17 @@ lean_object* l_Lean_Parser_setLhsPrecFn___boxed(lean_object*, lean_object*, lean static lean_object* l_Lean_Parser_Command_elabTail___elambda__1___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntaxAbbrev_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_macroTail___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_syntaxParser(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_categoryParser_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_syntaxCat_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab_formatter(lean_object*); static lean_object* l_Lean_Parser_Command_macro__rules___closed__5; lean_object* l_Lean_Parser_andthenFn(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_notation_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_declRange___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_formatter(lean_object*); static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Syntax___hyg_5____closed__1() { _start: { @@ -3768,6 +3953,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_paren___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_paren_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Syntax_paren___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_syntaxParser_parenthesizer(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: { @@ -3883,6 +4114,52 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_paren___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_paren_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Syntax_paren___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_cat___elambda__1___closed__1() { _start: { @@ -4380,7 +4657,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_optPrecedence_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_precedence_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_precedence___elambda__1___closed__6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_precedence_formatter___closed__2() { _start: { lean_object* x_1; @@ -4388,11 +4675,23 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_precedence_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_optPrecedence_formatter___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_precedence_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_precedence___elambda__1___closed__6; +x_4 = l___regBuiltin_Lean_Parser_precedence_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_precedence_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_optPrecedence_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_optPrecedence_formatter___closed__1; +x_1 = l___regBuiltin_Lean_Parser_precedence_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_atomic_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -4402,7 +4701,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_optPrecedence_formatter(lean_object* x_1, _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_optPrecedence_formatter___closed__2; +x_6 = l_Lean_Parser_optPrecedence_formatter___closed__1; x_7 = l_Lean_Parser_optional_formatter(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -4477,6 +4776,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_cat___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_cat_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Syntax_cat___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_precedenceParser_parenthesizer(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: { @@ -4560,7 +4889,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_optPrecedence_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_precedence___elambda__1___closed__6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -4568,11 +4907,23 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_precedence_parenthesizer), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_optPrecedence_parenthesizer___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_precedence_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_precedence___elambda__1___closed__6; +x_4 = l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_optPrecedence_parenthesizer___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_optPrecedence_parenthesizer___closed__1; +x_1 = l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_atomic_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -4582,7 +4933,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_optPrecedence_parenthesizer(lean_object* _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_optPrecedence_parenthesizer___closed__2; +x_6 = l_Lean_Parser_optPrecedence_parenthesizer___closed__1; x_7 = l_Lean_Parser_optional_parenthesizer(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -4657,6 +5008,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_cat___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_cat_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Syntax_cat___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_unary___elambda__1___closed__1() { _start: { @@ -5322,6 +5703,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_unary___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_unary_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Syntax_unary___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_unary_parenthesizer___closed__1() { _start: { @@ -5396,6 +5807,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_unary___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_unary_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Syntax_unary___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_binary___elambda__1___closed__1() { _start: { @@ -6300,6 +6741,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_binary___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_binary_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Syntax_binary___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_binary_parenthesizer___closed__1() { _start: { @@ -6412,6 +6883,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_binary___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_binary_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Syntax_binary___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Syntax_sepBy___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -7338,6 +7839,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_sepBy___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_sepBy_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Syntax_sepBy___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1() { _start: { @@ -7527,6 +8058,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_sepBy___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_sepBy_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Syntax_sepBy___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__1() { _start: { @@ -8391,10 +8952,40 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_sepBy1_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_1 = l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__1; x_2 = l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__2; x_3 = 1; @@ -8455,6 +9046,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_sepBy1_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_atom___elambda__1___closed__1() { _start: { @@ -8824,6 +9445,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_atom___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_atom_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Syntax_atom___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_atom_parenthesizer___closed__1() { _start: { @@ -8866,6 +9517,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_atom___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_atom_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Syntax_atom___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__1() { _start: { @@ -9437,6 +10118,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_nonReserved_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1() { _start: { @@ -9501,6 +10212,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Syntax_nonReserved_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_stx_quot___elambda__1___closed__1() { _start: { @@ -10223,6 +10964,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_stx_quot___elambda__1___closed__5; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_stx_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Term_stx_quot___elambda__1___closed__5; +x_4 = l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_stx_quot_parenthesizer___closed__1() { _start: { @@ -10309,6 +11080,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_stx_quot___elambda__1___closed__5; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_stx_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_stx_quot___elambda__1___closed__5; +x_4 = l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_prec_quot___elambda__1___closed__1() { _start: { @@ -10988,6 +11789,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_prec_quot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_prec_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Term_prec_quot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_prec_quot_parenthesizer___closed__1() { _start: { @@ -11084,6 +11915,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_prec_quot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_prec_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_prec_quot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_prio_quot___elambda__1___closed__1() { _start: { @@ -11789,6 +12650,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_prio_quot___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_prio_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Term_prio_quot___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_prio_quot_parenthesizer___closed__1() { _start: { @@ -11885,6 +12776,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_prio_quot___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_prio_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_prio_quot___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_namedName___elambda__1___closed__1() { _start: { @@ -14874,22 +15795,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_infix_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Parser_Command_infix___elambda__1___closed__1; -x_2 = l_Lean_Parser_Command_infix___elambda__1___closed__2; -x_3 = 1; -x_4 = 0; -x_5 = lean_box(x_3); -x_6 = lean_box(x_4); -x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_formatter___boxed), 9, 4); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, x_2); -lean_closure_set(x_7, 2, x_5); -lean_closure_set(x_7, 3, x_6); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_prefix___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_prefix_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_prefix_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_prefix___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_infix_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; uint8_t x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Parser_Command_infix___elambda__1___closed__1; +x_2 = l_Lean_Parser_Command_infix___elambda__1___closed__2; +x_3 = 1; +x_4 = 0; +x_5 = lean_box(x_3); +x_6 = lean_box(x_4); +x_7 = lean_alloc_closure((void*)(l_Lean_Parser_mkAntiquot_formatter___boxed), 9, 4); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +lean_closure_set(x_7, 2, x_5); +lean_closure_set(x_7, 3, x_6); +return x_7; } } static lean_object* _init_l_Lean_Parser_Command_infix_formatter___closed__2() { @@ -14926,6 +15877,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_infix___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infix_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infix_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_infix___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_infixl_formatter___closed__1() { _start: { @@ -14978,6 +15959,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_infixl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infixl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infixl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_infixl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_infixr_formatter___closed__1() { _start: { @@ -15030,6 +16041,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_infixr___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infixr_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infixr_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_infixr___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_postfix_formatter___closed__1() { _start: { @@ -15082,15 +16123,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infixr_formatter), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_postfix___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__2() { _start: { lean_object* x_1; @@ -15098,72 +16141,60 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_postfix_formatter), 5, 0) return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_postfix_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_postfix___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfixKind_formatter___closed__1; -x_2 = l_Lean_Parser_Command_mixfixKind_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infixl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfixKind_formatter___closed__4; -x_2 = l_Lean_Parser_Command_mixfixKind_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__2; +x_2 = l_Lean_Parser_Command_mixfixKind_formatter___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infix_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfixKind_formatter___closed__6; -x_2 = l_Lean_Parser_Command_mixfixKind_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__2; +x_2 = l_Lean_Parser_Command_mixfixKind_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_prefix_formatter), 5, 0); -return x_1; -} -} LEAN_EXPORT lean_object* l_Lean_Parser_Command_mixfixKind_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_mixfixKind_formatter___closed__8; -x_7 = l_Lean_Parser_Command_mixfixKind_formatter___closed__7; +x_6 = l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__2; +x_7 = l_Lean_Parser_Command_mixfixKind_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -15291,7 +16322,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_optNamedName_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_namedName___elambda__1___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__2() { _start: { lean_object* x_1; @@ -15299,11 +16340,23 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_namedName_formatter), 5, return x_1; } } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namedName_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_namedName___elambda__1___closed__4; +x_4 = l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Command_optNamedName_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Command_optNamedName_formatter___closed__1; +x_6 = l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__2; x_7 = l_Lean_Parser_optional_formatter(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -15430,7 +16483,7 @@ static lean_object* _init_l_Lean_Parser_Command_mixfix_formatter___closed__12() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_optPrecedence_formatter___closed__1; +x_1 = l___regBuiltin_Lean_Parser_precedence_formatter___closed__2; x_2 = l_Lean_Parser_Command_mixfix_formatter___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -15502,6 +16555,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_mixfix___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_mixfix_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_mixfix___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_prefix_parenthesizer___closed__1() { _start: { @@ -15554,6 +16637,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_prefix___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_prefix_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_prefix___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_infix_parenthesizer___closed__1() { _start: { @@ -15606,6 +16719,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_infix___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infix_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infix_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_infix___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_infixl_parenthesizer___closed__1() { _start: { @@ -15658,6 +16801,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_infixl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infixl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_infixl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_infixr_parenthesizer___closed__1() { _start: { @@ -15710,6 +16883,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_infixr___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infixr_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_infixr___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_postfix_parenthesizer___closed__1() { _start: { @@ -15762,15 +16965,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infixr_parenthesizer), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_postfix___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -15778,72 +16983,60 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_postfix_parenthesizer), 5 return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_postfix___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__1; -x_2 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infixl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_infix_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_prefix_parenthesizer), 5, 0); -return x_1; -} -} LEAN_EXPORT lean_object* l_Lean_Parser_Command_mixfixKind_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__8; -x_7 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__7; +x_6 = l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__2; +x_7 = l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__3; x_8 = l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -15971,7 +17164,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_optNamedName_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_namedName___elambda__1___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -15979,11 +17182,23 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_namedName_parenthesizer), return x_1; } } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_namedName___elambda__1___closed__4; +x_4 = l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Command_optNamedName_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Command_optNamedName_parenthesizer___closed__1; +x_6 = l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__2; x_7 = l_Lean_Parser_optional_parenthesizer(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -16112,7 +17327,7 @@ static lean_object* _init_l_Lean_Parser_Command_mixfix_parenthesizer___closed__1 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_optPrecedence_parenthesizer___closed__1; +x_1 = l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -16184,6 +17399,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_mixfix___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_mixfix_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_mixfix___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_identPrec___elambda__1___closed__1() { _start: { @@ -17526,6 +18771,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_identPrec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_identPrec_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_identPrec_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_identPrec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_notationItem_formatter___closed__1() { _start: { @@ -17547,29 +18822,21 @@ return x_7; static lean_object* _init_l_Lean_Parser_Command_notationItem_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_identPrec_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_notationItem_formatter___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_sepBy_formatter___closed__10; -x_2 = l_Lean_Parser_Command_notationItem_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_notationItem_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_notationItem_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_notationItem_formatter___closed__1; -x_2 = l_Lean_Parser_Command_notationItem_formatter___closed__3; +x_2 = l_Lean_Parser_Command_notationItem_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withAntiquot_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -17581,7 +18848,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_notationItem_formatter(lean_objec { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_mixfix_formatter___closed__6; -x_7 = l_Lean_Parser_Command_notationItem_formatter___closed__4; +x_7 = l_Lean_Parser_Command_notationItem_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_andthen_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -17728,6 +18995,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_notation___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_notation_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_notation_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_notation___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_identPrec_parenthesizer___closed__1() { _start: { @@ -17770,6 +19067,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_identPrec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_identPrec_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_identPrec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__1() { _start: { @@ -17791,29 +19118,21 @@ return x_7; static lean_object* _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_identPrec_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__10; -x_2 = l_Lean_Parser_Command_notationItem_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_notationItem_parenthesizer___closed__1; -x_2 = l_Lean_Parser_Command_notationItem_parenthesizer___closed__3; +x_2 = l_Lean_Parser_Command_notationItem_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -17825,7 +19144,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_notationItem_parenthesizer(lean_o { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__6; -x_7 = l_Lean_Parser_Command_notationItem_parenthesizer___closed__4; +x_7 = l_Lean_Parser_Command_notationItem_parenthesizer___closed__3; x_8 = l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -17972,6 +19291,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_notation___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_notation_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_notation_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_notation___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_macro__rules___elambda__1___closed__1() { _start: { @@ -18835,31 +20184,40 @@ return x_5; static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__4() { _start: { +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Term_attributes; +x_2 = l_Lean_Parser_optional(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__5() { +_start: +{ lean_object* x_1; x_1 = lean_mk_string_from_bytes("syntax ", 7); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__4; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__5; x_2 = l_String_trim(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__5; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_precedence___elambda__1___lambda__1___boxed), 3, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -18869,16 +20227,16 @@ x_3 = l_Lean_Parser_categoryParser(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__7; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__8; x_2 = l_Lean_Parser_many1(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__10() { _start: { lean_object* x_1; @@ -18886,30 +20244,30 @@ x_1 = lean_mk_string_from_bytes(" : ", 3); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__9; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__10; x_2 = l_String_trim(x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__10; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__11; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_precedence___elambda__1___lambda__1___boxed), 3, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__11; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__12; x_2 = l_Lean_Parser_Syntax_cat___elambda__1___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); @@ -18917,117 +20275,131 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__8; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__9; x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__12; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__13; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_4, 0, x_2); lean_closure_set(x_4, 1, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_optNamedPrio; x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__13; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__14; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_4, 0, x_2); lean_closure_set(x_4, 1, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_optNamedName; x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__14; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__15; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_4, 0, x_2); lean_closure_set(x_4, 1, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__16() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_optPrecedence; x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__15; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__16; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_4, 0, x_2); lean_closure_set(x_4, 1, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__17() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__6; -x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__16; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__7; +x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__17; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__18() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix___elambda__1___closed__14; -x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__17; +x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__18; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__19() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__4; +x_2 = lean_ctor_get(x_1, 1); +lean_inc(x_2); +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__19; +x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); +lean_closure_set(x_4, 0, x_2); +lean_closure_set(x_4, 1, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_macro__rules___elambda__1___closed__4; x_2 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__18; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__20; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_4, 0, x_2); lean_closure_set(x_4, 1, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__20() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__19; +x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__21; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_nodeFn), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__21() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__20; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__22; x_2 = l_Lean_Parser_precedence___elambda__1___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); @@ -19035,53 +20407,53 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__22() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_precedence___elambda__1___closed__11; -x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__21; +x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__23; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__23() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_precedence___elambda__1___lambda__1___closed__1; -x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__5; +x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__6; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__24() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__26() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__23; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__25; x_2 = l_Lean_Parser_precedence___elambda__1___lambda__1___closed__1; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__25() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__27() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_precedence___elambda__1___lambda__1___closed__1; -x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__10; +x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__11; x_3 = lean_string_append(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__26() { +static lean_object* _init_l_Lean_Parser_Command_syntax___elambda__1___closed__28() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__25; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__27; x_2 = l_Lean_Parser_precedence___elambda__1___lambda__1___closed__1; x_3 = lean_string_append(x_1, x_2); return x_3; @@ -19090,8 +20462,8 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntax___elambda__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; 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; uint32_t x_18; uint32_t x_19; uint8_t x_20; -x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__8; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; 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; uint32_t x_20; uint32_t x_21; uint8_t x_22; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__9; x_4 = lean_ctor_get(x_3, 1); lean_inc(x_4); x_5 = l_Lean_Parser_Command_optNamedPrio; @@ -19103,285 +20475,275 @@ lean_inc(x_8); x_9 = l_Lean_Parser_optPrecedence; x_10 = lean_ctor_get(x_9, 1); lean_inc(x_10); -x_11 = l_Lean_Parser_Command_macro__rules___elambda__1___closed__4; +x_11 = l_Lean_Parser_Command_syntax___elambda__1___closed__4; x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); -x_13 = l_Lean_Parser_Command_syntax___elambda__1___closed__3; +x_13 = l_Lean_Parser_Command_macro__rules___elambda__1___closed__4; x_14 = lean_ctor_get(x_13, 1); lean_inc(x_14); -x_15 = lean_ctor_get(x_1, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 0); +x_15 = l_Lean_Parser_Command_syntax___elambda__1___closed__3; +x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_ctor_get(x_2, 2); +x_17 = lean_ctor_get(x_1, 0); lean_inc(x_17); -x_18 = lean_string_utf8_get(x_16, x_17); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); lean_dec(x_17); -x_19 = 36; -x_20 = lean_uint32_dec_eq(x_18, x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -lean_dec(x_14); -x_21 = lean_unsigned_to_nat(1024u); -x_22 = l_Lean_Parser_checkPrecFn(x_21, x_1, x_2); -x_23 = lean_ctor_get(x_22, 4); -lean_inc(x_23); -x_24 = lean_box(0); -x_25 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_23, x_24); -lean_dec(x_23); -if (x_25 == 0) +x_19 = lean_ctor_get(x_2, 2); +lean_inc(x_19); +x_20 = lean_string_utf8_get(x_18, x_19); +lean_dec(x_19); +x_21 = 36; +x_22 = lean_uint32_dec_eq(x_20, x_21); +if (x_22 == 0) { +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_dec(x_16); +x_23 = lean_unsigned_to_nat(1024u); +x_24 = l_Lean_Parser_checkPrecFn(x_23, x_1, x_2); +x_25 = lean_ctor_get(x_24, 4); +lean_inc(x_25); +x_26 = lean_box(0); +x_27 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_25, x_26); +lean_dec(x_25); +if (x_27 == 0) +{ +lean_dec(x_18); +lean_dec(x_14); lean_dec(x_12); lean_dec(x_10); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); lean_dec(x_1); -return x_22; +return x_24; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; -x_26 = lean_ctor_get(x_22, 0); -lean_inc(x_26); -x_27 = lean_array_get_size(x_26); -lean_dec(x_26); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; +x_28 = lean_ctor_get(x_24, 0); +lean_inc(x_28); +x_29 = lean_array_get_size(x_28); +lean_dec(x_28); lean_inc(x_1); -x_28 = lean_apply_2(x_12, x_1, x_22); -x_29 = lean_ctor_get(x_28, 4); -lean_inc(x_29); -x_30 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_29, x_24); -lean_dec(x_29); -if (x_30 == 0) +x_30 = lean_apply_2(x_14, x_1, x_24); +x_31 = lean_ctor_get(x_30, 4); +lean_inc(x_31); +x_32 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_31, x_26); +lean_dec(x_31); +if (x_32 == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -lean_dec(x_16); +lean_dec(x_18); +lean_dec(x_12); lean_dec(x_10); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); -x_38 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; -x_39 = l_Lean_Parser_ParserState_mkNode(x_28, x_38, x_27); -x_40 = lean_ctor_get(x_39, 4); -lean_inc(x_40); -x_41 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_40, x_24); -lean_dec(x_40); -if (x_41 == 0) -{ -lean_dec(x_1); -return x_39; +x_33 = x_30; +goto block_39; } else { -lean_object* x_42; -x_42 = l_Lean_Parser_setLhsPrecFn(x_21, x_1, x_39); -lean_dec(x_1); -return x_42; -} +lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_inc(x_1); +x_40 = lean_apply_2(x_12, x_1, x_30); +x_41 = lean_ctor_get(x_40, 4); +lean_inc(x_41); +x_42 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_41, x_26); +lean_dec(x_41); +if (x_42 == 0) +{ +lean_dec(x_18); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_4); +x_33 = x_40; +goto block_39; } else { lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_inc(x_1); -x_43 = l_Lean_Parser_Term_attrKind___elambda__1(x_1, x_28); +x_43 = l_Lean_Parser_Term_attrKind___elambda__1(x_1, x_40); x_44 = lean_ctor_get(x_43, 4); lean_inc(x_44); -x_45 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_44, x_24); +x_45 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_44, x_26); lean_dec(x_44); if (x_45 == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; -lean_dec(x_16); +lean_dec(x_18); lean_dec(x_10); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); -x_46 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; -x_47 = l_Lean_Parser_ParserState_mkNode(x_43, x_46, x_27); -x_48 = lean_ctor_get(x_47, 4); -lean_inc(x_48); -x_49 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_48, x_24); -lean_dec(x_48); -if (x_49 == 0) -{ -lean_dec(x_1); -return x_47; +x_33 = x_43; +goto block_39; } else { -lean_object* x_50; -x_50 = l_Lean_Parser_setLhsPrecFn(x_21, x_1, x_47); -lean_dec(x_1); -return x_50; -} -} -else -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint32_t x_55; uint32_t x_56; uint8_t x_57; lean_object* x_58; -x_51 = l_Lean_Parser_Command_syntax___elambda__1___closed__5; -x_52 = l_Lean_Parser_Command_syntax___elambda__1___closed__24; +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint32_t x_50; uint32_t x_51; uint8_t x_52; lean_object* x_53; +x_46 = l_Lean_Parser_Command_syntax___elambda__1___closed__6; +x_47 = l_Lean_Parser_Command_syntax___elambda__1___closed__26; lean_inc(x_1); -x_53 = l_Lean_Parser_symbolFnAux(x_51, x_52, x_1, x_43); -x_54 = lean_ctor_get(x_53, 2); -lean_inc(x_54); -x_55 = lean_string_utf8_get(x_16, x_54); -lean_dec(x_54); -x_56 = 37; -x_57 = lean_uint32_dec_eq(x_55, x_56); -if (x_57 == 0) +x_48 = l_Lean_Parser_symbolFnAux(x_46, x_47, x_1, x_43); +x_49 = lean_ctor_get(x_48, 2); +lean_inc(x_49); +x_50 = lean_string_utf8_get(x_18, x_49); +lean_dec(x_49); +x_51 = 37; +x_52 = lean_uint32_dec_eq(x_50, x_51); +if (x_52 == 0) { -x_58 = x_53; -goto block_86; +x_53 = x_48; +goto block_81; } else { -lean_object* x_87; +lean_object* x_82; lean_inc(x_1); -x_87 = l_Lean_Parser_tokenAntiquotFn(x_1, x_53); -x_58 = x_87; -goto block_86; +x_82 = l_Lean_Parser_tokenAntiquotFn(x_1, x_48); +x_53 = x_82; +goto block_81; } -block_86: +block_81: { -lean_object* x_59; uint8_t x_60; -x_59 = lean_ctor_get(x_58, 4); -lean_inc(x_59); -x_60 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_59, x_24); -lean_dec(x_59); -if (x_60 == 0) +lean_object* x_54; uint8_t x_55; +x_54 = lean_ctor_get(x_53, 4); +lean_inc(x_54); +x_55 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_54, x_26); +lean_dec(x_54); +if (x_55 == 0) { -lean_dec(x_16); +lean_dec(x_18); lean_dec(x_10); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); -x_31 = x_58; -goto block_37; +x_33 = x_53; +goto block_39; } else { -lean_object* x_61; lean_object* x_62; uint8_t x_63; +lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_inc(x_1); -x_61 = lean_apply_2(x_10, x_1, x_58); -x_62 = lean_ctor_get(x_61, 4); -lean_inc(x_62); -x_63 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_62, x_24); -lean_dec(x_62); -if (x_63 == 0) +x_56 = lean_apply_2(x_10, x_1, x_53); +x_57 = lean_ctor_get(x_56, 4); +lean_inc(x_57); +x_58 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_57, x_26); +lean_dec(x_57); +if (x_58 == 0) { -lean_dec(x_16); +lean_dec(x_18); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); -x_31 = x_61; -goto block_37; +x_33 = x_56; +goto block_39; } else { -lean_object* x_64; lean_object* x_65; uint8_t x_66; +lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_inc(x_1); -x_64 = lean_apply_2(x_8, x_1, x_61); -x_65 = lean_ctor_get(x_64, 4); -lean_inc(x_65); -x_66 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_65, x_24); -lean_dec(x_65); -if (x_66 == 0) +x_59 = lean_apply_2(x_8, x_1, x_56); +x_60 = lean_ctor_get(x_59, 4); +lean_inc(x_60); +x_61 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_60, x_26); +lean_dec(x_60); +if (x_61 == 0) { -lean_dec(x_16); +lean_dec(x_18); lean_dec(x_6); lean_dec(x_4); -x_31 = x_64; -goto block_37; +x_33 = x_59; +goto block_39; } else { -lean_object* x_67; lean_object* x_68; uint8_t x_69; +lean_object* x_62; lean_object* x_63; uint8_t x_64; lean_inc(x_1); -x_67 = lean_apply_2(x_6, x_1, x_64); -x_68 = lean_ctor_get(x_67, 4); -lean_inc(x_68); -x_69 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_68, x_24); -lean_dec(x_68); -if (x_69 == 0) +x_62 = lean_apply_2(x_6, x_1, x_59); +x_63 = lean_ctor_get(x_62, 4); +lean_inc(x_63); +x_64 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_63, x_26); +lean_dec(x_63); +if (x_64 == 0) { -lean_dec(x_16); +lean_dec(x_18); lean_dec(x_4); -x_31 = x_67; -goto block_37; +x_33 = x_62; +goto block_39; } else { -lean_object* x_70; lean_object* x_71; uint8_t x_72; +lean_object* x_65; lean_object* x_66; uint8_t x_67; lean_inc(x_1); -x_70 = lean_apply_2(x_4, x_1, x_67); -x_71 = lean_ctor_get(x_70, 4); -lean_inc(x_71); -x_72 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_71, x_24); -lean_dec(x_71); -if (x_72 == 0) +x_65 = lean_apply_2(x_4, x_1, x_62); +x_66 = lean_ctor_get(x_65, 4); +lean_inc(x_66); +x_67 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_66, x_26); +lean_dec(x_66); +if (x_67 == 0) { -lean_dec(x_16); -x_31 = x_70; -goto block_37; +lean_dec(x_18); +x_33 = x_65; +goto block_39; } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint32_t x_77; uint8_t x_78; -x_73 = l_Lean_Parser_Command_syntax___elambda__1___closed__10; -x_74 = l_Lean_Parser_Command_syntax___elambda__1___closed__26; +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint32_t x_72; uint8_t x_73; +x_68 = l_Lean_Parser_Command_syntax___elambda__1___closed__11; +x_69 = l_Lean_Parser_Command_syntax___elambda__1___closed__28; lean_inc(x_1); -x_75 = l_Lean_Parser_symbolFnAux(x_73, x_74, x_1, x_70); -x_76 = lean_ctor_get(x_75, 2); -lean_inc(x_76); -x_77 = lean_string_utf8_get(x_16, x_76); -lean_dec(x_76); -lean_dec(x_16); -x_78 = lean_uint32_dec_eq(x_77, x_56); -if (x_78 == 0) +x_70 = l_Lean_Parser_symbolFnAux(x_68, x_69, x_1, x_65); +x_71 = lean_ctor_get(x_70, 2); +lean_inc(x_71); +x_72 = lean_string_utf8_get(x_18, x_71); +lean_dec(x_71); +lean_dec(x_18); +x_73 = lean_uint32_dec_eq(x_72, x_51); +if (x_73 == 0) { -lean_object* x_79; uint8_t x_80; -x_79 = lean_ctor_get(x_75, 4); -lean_inc(x_79); -x_80 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_79, x_24); -lean_dec(x_79); -if (x_80 == 0) +lean_object* x_74; uint8_t x_75; +x_74 = lean_ctor_get(x_70, 4); +lean_inc(x_74); +x_75 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_74, x_26); +lean_dec(x_74); +if (x_75 == 0) { -x_31 = x_75; -goto block_37; +x_33 = x_70; +goto block_39; } else { -lean_object* x_81; +lean_object* x_76; lean_inc(x_1); -x_81 = l_Lean_Parser_ident___elambda__1(x_1, x_75); -x_31 = x_81; -goto block_37; +x_76 = l_Lean_Parser_ident___elambda__1(x_1, x_70); +x_33 = x_76; +goto block_39; } } else { -lean_object* x_82; lean_object* x_83; uint8_t x_84; +lean_object* x_77; lean_object* x_78; uint8_t x_79; lean_inc(x_1); -x_82 = l_Lean_Parser_tokenAntiquotFn(x_1, x_75); -x_83 = lean_ctor_get(x_82, 4); -lean_inc(x_83); -x_84 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_83, x_24); -lean_dec(x_83); -if (x_84 == 0) -{ -x_31 = x_82; -goto block_37; +x_77 = l_Lean_Parser_tokenAntiquotFn(x_1, x_70); +x_78 = lean_ctor_get(x_77, 4); +lean_inc(x_78); +x_79 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_78, x_26); +lean_dec(x_78); +if (x_79 == 0) +{ +x_33 = x_77; +goto block_39; } else { -lean_object* x_85; +lean_object* x_80; lean_inc(x_1); -x_85 = l_Lean_Parser_ident___elambda__1(x_1, x_82); -x_31 = x_85; -goto block_37; +x_80 = l_Lean_Parser_ident___elambda__1(x_1, x_77); +x_33 = x_80; +goto block_39; } } } @@ -19392,43 +20754,45 @@ goto block_37; } } } -block_37: +} +block_39: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; -x_33 = l_Lean_Parser_ParserState_mkNode(x_31, x_32, x_27); -x_34 = lean_ctor_get(x_33, 4); -lean_inc(x_34); -x_35 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_34, x_24); -lean_dec(x_34); -if (x_35 == 0) +lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_34 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; +x_35 = l_Lean_Parser_ParserState_mkNode(x_33, x_34, x_29); +x_36 = lean_ctor_get(x_35, 4); +lean_inc(x_36); +x_37 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(x_36, x_26); +lean_dec(x_36); +if (x_37 == 0) { lean_dec(x_1); -return x_33; +return x_35; } else { -lean_object* x_36; -x_36 = l_Lean_Parser_setLhsPrecFn(x_21, x_1, x_33); +lean_object* x_38; +x_38 = l_Lean_Parser_setLhsPrecFn(x_23, x_1, x_35); lean_dec(x_1); -return x_36; +return x_38; } } } } else { -lean_object* x_88; uint8_t x_89; lean_object* x_90; -lean_dec(x_16); +lean_object* x_83; uint8_t x_84; lean_object* x_85; +lean_dec(x_18); +lean_dec(x_14); lean_dec(x_12); lean_dec(x_10); lean_dec(x_8); lean_dec(x_6); lean_dec(x_4); -x_88 = l_Lean_Parser_Command_syntax___elambda__1___closed__22; -x_89 = 0; -x_90 = l_Lean_Parser_orelseFnCore(x_14, x_88, x_89, x_1, x_2); -return x_90; +x_83 = l_Lean_Parser_Command_syntax___elambda__1___closed__24; +x_84 = 0; +x_85 = l_Lean_Parser_orelseFnCore(x_16, x_83, x_84, x_1, x_2); +return x_85; } } } @@ -19436,7 +20800,7 @@ static lean_object* _init_l_Lean_Parser_Command_syntax___closed__1() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__5; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__6; x_2 = l_Lean_Parser_symbolInfo(x_1); return x_2; } @@ -19445,7 +20809,7 @@ static lean_object* _init_l_Lean_Parser_Command_syntax___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__10; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__11; x_2 = l_Lean_Parser_symbolInfo(x_1); return x_2; } @@ -19466,7 +20830,7 @@ static lean_object* _init_l_Lean_Parser_Command_syntax___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__8; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__9; x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); x_3 = l_Lean_Parser_Command_syntax___closed__3; @@ -19536,7 +20900,7 @@ static lean_object* _init_l_Lean_Parser_Command_syntax___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_macro__rules___elambda__1___closed__4; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__4; x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); x_3 = l_Lean_Parser_Command_syntax___closed__9; @@ -19547,46 +20911,58 @@ return x_4; static lean_object* _init_l_Lean_Parser_Command_syntax___closed__11() { _start: { +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_macro__rules___elambda__1___closed__4; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = l_Lean_Parser_Command_syntax___closed__10; +x_4 = l_Lean_Parser_andthenInfo(x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax___closed__12() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; -x_2 = l_Lean_Parser_Command_syntax___closed__10; +x_2 = l_Lean_Parser_Command_syntax___closed__11; x_3 = l_Lean_Parser_nodeInfo(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_syntax___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___closed__11; +x_1 = l_Lean_Parser_Command_syntax___closed__12; x_2 = l_Lean_Parser_epsilonInfo; x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_syntax___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_epsilonInfo; -x_2 = l_Lean_Parser_Command_syntax___closed__12; +x_2 = l_Lean_Parser_Command_syntax___closed__13; x_3 = l_Lean_Parser_andthenInfo(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_syntax___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__3; x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_syntax___closed__13; +x_3 = l_Lean_Parser_Command_syntax___closed__14; x_4 = l_Lean_Parser_orelseInfo(x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___closed__15() { +static lean_object* _init_l_Lean_Parser_Command_syntax___closed__16() { _start: { lean_object* x_1; @@ -19594,12 +20970,12 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_syntax___elambda__1), 2, return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_syntax___closed__16() { +static lean_object* _init_l_Lean_Parser_Command_syntax___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___closed__14; -x_2 = l_Lean_Parser_Command_syntax___closed__15; +x_1 = l_Lean_Parser_Command_syntax___closed__15; +x_2 = l_Lean_Parser_Command_syntax___closed__16; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -19610,7 +20986,7 @@ static lean_object* _init_l_Lean_Parser_Command_syntax() { _start: { lean_object* x_1; -x_1 = l_Lean_Parser_Command_syntax___closed__16; +x_1 = l_Lean_Parser_Command_syntax___closed__17; return x_1; } } @@ -19644,7 +21020,7 @@ static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntax_declRange___ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_unsigned_to_nat(72u); -x_2 = lean_unsigned_to_nat(208u); +x_2 = lean_unsigned_to_nat(240u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -19658,7 +21034,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l___regBuiltin_Lean_Parser_Command_syntax_declRange___closed__1; x_2 = lean_unsigned_to_nat(24u); x_3 = l___regBuiltin_Lean_Parser_Command_syntax_declRange___closed__2; -x_4 = lean_unsigned_to_nat(208u); +x_4 = lean_unsigned_to_nat(240u); x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -19750,28 +21126,46 @@ return x_7; static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__2() { _start: { +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attributes_formatter), 5, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__3() { +_start: +{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__4; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__2; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__5; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__9; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__10; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_formatter___closed__3; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__5; x_2 = l_Lean_Parser_Syntax_cat_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -19779,97 +21173,109 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_paren_formatter___closed__4; -x_2 = l_Lean_Parser_Command_syntax_formatter___closed__4; +x_2 = l_Lean_Parser_Command_syntax_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__8; -x_2 = l_Lean_Parser_Command_syntax_formatter___closed__5; +x_2 = l_Lean_Parser_Command_syntax_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__10; -x_2 = l_Lean_Parser_Command_syntax_formatter___closed__6; +x_2 = l_Lean_Parser_Command_syntax_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_cat_formatter___closed__3; -x_2 = l_Lean_Parser_Command_syntax_formatter___closed__7; +x_2 = l_Lean_Parser_Command_syntax_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_formatter___closed__2; -x_2 = l_Lean_Parser_Command_syntax_formatter___closed__8; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__4; +x_2 = l_Lean_Parser_Command_syntax_formatter___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__15; -x_2 = l_Lean_Parser_Command_syntax_formatter___closed__9; +x_2 = l_Lean_Parser_Command_syntax_formatter___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__3; +x_2 = l_Lean_Parser_Command_syntax_formatter___closed__12; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_macro__rules_formatter___closed__3; -x_2 = l_Lean_Parser_Command_syntax_formatter___closed__10; +x_2 = l_Lean_Parser_Command_syntax_formatter___closed__13; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_syntax_formatter___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_syntax_formatter___closed__11; +x_3 = l_Lean_Parser_Command_syntax_formatter___closed__14; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -19882,11 +21288,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntax_formatter(lean_object* x_1 { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_syntax_formatter___closed__1; -x_7 = l_Lean_Parser_Command_syntax_formatter___closed__12; +x_7 = l_Lean_Parser_Command_syntax_formatter___closed__15; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_syntax_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntax_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__1() { _start: { @@ -19908,14 +21344,32 @@ return x_7; static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__2() { _start: { +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attributes_parenthesizer), 5, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__3() { +_start: +{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__4; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__2; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__5; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__3() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -19925,31 +21379,31 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__5; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__9; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__10; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_symbol_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__7; x_2 = l_Lean_Parser_Syntax_cat_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -19957,97 +21411,109 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__8; -x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__7; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__10; -x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__8; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_cat_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__10; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__15; -x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__11; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__13; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__3; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__14; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_macro__rules_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__12; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__15; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_syntax_parenthesizer___closed__13; +x_3 = l_Lean_Parser_Command_syntax_parenthesizer___closed__16; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -20055,14 +21521,44 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntax_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Parser_Command_syntax_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = l_Lean_Parser_Command_syntax_parenthesizer___closed__1; +x_7 = l_Lean_Parser_Command_syntax_parenthesizer___closed__17; +x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_syntax_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer(lean_object* x_1) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Command_syntax_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_syntax_parenthesizer___closed__14; -x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); -return x_8; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } static lean_object* _init_l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__1() { @@ -20125,7 +21621,7 @@ static lean_object* _init_l_Lean_Parser_Command_syntaxAbbrev___elambda__1___clos _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__6; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__7; x_2 = l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); @@ -20266,8 +21762,8 @@ return x_36; else { lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint32_t x_41; uint32_t x_42; uint8_t x_43; lean_object* x_44; -x_37 = l_Lean_Parser_Command_syntax___elambda__1___closed__5; -x_38 = l_Lean_Parser_Command_syntax___elambda__1___closed__24; +x_37 = l_Lean_Parser_Command_syntax___elambda__1___closed__6; +x_38 = l_Lean_Parser_Command_syntax___elambda__1___closed__26; lean_inc(x_1); x_39 = l_Lean_Parser_symbolFnAux(x_37, x_38, x_1, x_22); x_40 = lean_ctor_get(x_39, 2); @@ -20696,7 +22192,7 @@ static lean_object* _init_l_Lean_Parser_Command_syntaxAbbrev_formatter___closed_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_formatter___closed__2; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__4; x_2 = l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -20740,6 +22236,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_syntaxAbbrev_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1() { _start: { @@ -20786,7 +22312,7 @@ static lean_object* _init_l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___clo _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__2; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__4; x_2 = l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -20830,6 +22356,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_syntaxAbbrev_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__1() { _start: { @@ -22204,6 +23760,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_catBehaviorBoth_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1() { _start: { @@ -22259,52 +23845,66 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1() { _start: { -lean_object* x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_catBehavior___closed__1; -x_2 = 0; -x_3 = lean_box(x_2); -x_4 = lean_alloc_closure((void*)(l_Lean_Parser_nonReservedSymbol_formatter___boxed), 7, 2); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_3); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_catBehaviorSymbol___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_catBehaviorBoth_formatter), 5, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_catBehaviorSymbol_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_catBehaviorSymbol_formatter), 5, 0); -return x_1; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_catBehaviorSymbol___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_catBehavior___closed__1; +x_2 = 0; +x_3 = lean_box(x_2); +x_4 = lean_alloc_closure((void*)(l_Lean_Parser_nonReservedSymbol_formatter___boxed), 7, 2); +lean_closure_set(x_4, 0, x_1); +lean_closure_set(x_4, 1, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_catBehavior_formatter___closed__2; -x_2 = l_Lean_Parser_Command_catBehavior_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_catBehavior_formatter___closed__4; +x_1 = l_Lean_Parser_Command_catBehavior_formatter___closed__2; x_2 = l_Lean_Parser_Syntax_paren_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -22312,36 +23912,36 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_namedName_formatter___closed__5; -x_2 = l_Lean_Parser_Command_catBehavior_formatter___closed__5; +x_2 = l_Lean_Parser_Command_catBehavior_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_catBehavior_formatter___closed__1; -x_2 = l_Lean_Parser_Command_catBehavior_formatter___closed__6; +x_2 = l_Lean_Parser_Command_catBehavior_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_paren_formatter___closed__2; -x_2 = l_Lean_Parser_Command_catBehavior_formatter___closed__7; +x_2 = l_Lean_Parser_Command_catBehavior_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -22352,7 +23952,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehavior_formatter(lean_object _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Command_catBehavior_formatter___closed__8; +x_6 = l_Lean_Parser_Command_catBehavior_formatter___closed__6; x_7 = l_Lean_Parser_optional_formatter(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -22441,6 +24041,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_syntaxCat___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_syntaxCat_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_syntaxCat___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1() { _start: { @@ -22496,6 +24126,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_catBehaviorBoth_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1() { _start: { @@ -22551,52 +24211,66 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1() { _start: { -lean_object* x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Command_catBehavior___closed__1; -x_2 = 0; -x_3 = lean_box(x_2); -x_4 = lean_alloc_closure((void*)(l_Lean_Parser_nonReservedSymbol_parenthesizer___boxed), 7, 2); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_3); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_catBehaviorSymbol___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_catBehaviorBoth_parenthesizer), 5, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer), 5, 0); -return x_1; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_catBehaviorSymbol___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Parser_Command_catBehavior___closed__1; +x_2 = 0; +x_3 = lean_box(x_2); +x_4 = lean_alloc_closure((void*)(l_Lean_Parser_nonReservedSymbol_parenthesizer___boxed), 7, 2); +lean_closure_set(x_4, 0, x_1); +lean_closure_set(x_4, 1, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__2; x_2 = l_Lean_Parser_Syntax_paren_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -22604,36 +24278,36 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_namedName_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__1; -x_2 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_paren_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__7; +x_2 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -22644,7 +24318,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_catBehavior_parenthesizer(lean_ob _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__8; +x_6 = l_Lean_Parser_Command_catBehavior_parenthesizer___closed__6; x_7 = l_Lean_Parser_optional_parenthesizer(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -22733,6 +24407,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_syntaxCat___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_syntaxCat_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_syntaxCat___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_macroArg___elambda__1___closed__1() { _start: { @@ -23050,7 +24754,7 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_obj x_1 = l_Lean_Parser_Command_macroArg___elambda__1___closed__13; x_2 = lean_ctor_get(x_1, 0); lean_inc(x_2); -x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__7; +x_3 = l_Lean_Parser_Command_syntax___elambda__1___closed__8; x_4 = lean_ctor_get(x_3, 0); lean_inc(x_4); x_5 = l_Lean_Parser_andthenInfo(x_2, x_4); @@ -23378,7 +25082,7 @@ static lean_object* _init_l_Lean_Parser_Command_macroTailTactic___elambda__1___c _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__11; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__12; x_2 = l_Lean_Parser_Command_macroTailTactic___elambda__1___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); @@ -23555,7 +25259,7 @@ static lean_object* _init_l_Lean_Parser_Command_macroTailCommand___elambda__1___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__11; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__12; x_2 = l_Lean_Parser_Command_macroTailCommand___elambda__1___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); @@ -23779,7 +25483,7 @@ lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_obj x_3 = l_Lean_Parser_Command_macroTailDefault___elambda__1___closed__2; x_4 = lean_ctor_get(x_3, 1); lean_inc(x_4); -x_5 = l_Lean_Parser_Command_syntax___elambda__1___closed__12; +x_5 = l_Lean_Parser_Command_syntax___elambda__1___closed__13; lean_inc(x_1); x_6 = l_Lean_Parser_atomicFn(x_5, x_1, x_2); x_7 = lean_ctor_get(x_6, 4); @@ -24789,6 +26493,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_macroArg___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macroArg_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macroArg_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_macroArg___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_macroRhs_formatter___closed__1() { _start: { @@ -24868,7 +26602,7 @@ static lean_object* _init_l_Lean_Parser_Command_macroTailTactic_formatter___clos _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_formatter___closed__3; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__5; x_2 = l_Lean_Parser_Command_macroTailTactic_formatter___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -24980,7 +26714,7 @@ static lean_object* _init_l_Lean_Parser_Command_macroTailDefault_formatter___clo _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax_formatter___closed__4; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_atomic_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -25118,6 +26852,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_macroTail___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macroTail_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macroTail_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_macroTail___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__1() { _start: { @@ -25149,130 +26913,114 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macroArg_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_macro_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macroTail_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_macro_formatter___closed__4; -x_2 = l_Lean_Parser_Command_macro_formatter___closed__5; +x_1 = l_Lean_Parser_Command_macro_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__8; -x_2 = l_Lean_Parser_Command_macro_formatter___closed__6; +x_2 = l_Lean_Parser_Command_macro_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__10; -x_2 = l_Lean_Parser_Command_macro_formatter___closed__7; +x_2 = l_Lean_Parser_Command_macro_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_cat_formatter___closed__3; -x_2 = l_Lean_Parser_Command_macro_formatter___closed__8; +x_2 = l_Lean_Parser_Command_macro_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_macro_formatter___closed__2; -x_2 = l_Lean_Parser_Command_macro_formatter___closed__9; +x_2 = l_Lean_Parser_Command_macro_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__15; -x_2 = l_Lean_Parser_Command_macro_formatter___closed__10; +x_2 = l_Lean_Parser_Command_macro_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_macro__rules_formatter___closed__3; -x_2 = l_Lean_Parser_Command_macro_formatter___closed__11; +x_2 = l_Lean_Parser_Command_macro_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_macro_formatter___closed__12; +x_1 = l_Lean_Parser_Command_macro_formatter___closed__10; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_suppressInsideQuot_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_macro_formatter___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_macro___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_macro_formatter___closed__13; +x_3 = l_Lean_Parser_Command_macro_formatter___closed__11; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -25285,11 +27033,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_macro_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_macro_formatter___closed__1; -x_7 = l_Lean_Parser_Command_macro_formatter___closed__14; +x_7 = l_Lean_Parser_Command_macro_formatter___closed__12; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_macro___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macro_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macro_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_macro___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_macroArg_parenthesizer___closed__1() { _start: { @@ -25357,7 +27135,7 @@ static lean_object* _init_l_Lean_Parser_Command_macroArg_parenthesizer___closed_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_macroArg_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__3; +x_2 = l_Lean_Parser_Command_syntax_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -25388,6 +27166,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_macroArg___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macroArg_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_macroArg___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_macroRhs_parenthesizer___closed__1() { _start: { @@ -25469,7 +27277,7 @@ static lean_object* _init_l_Lean_Parser_Command_macroTailTactic_parenthesizer___ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__7; x_2 = l_Lean_Parser_Command_macroTailTactic_parenthesizer___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -25541,7 +27349,7 @@ static lean_object* _init_l_Lean_Parser_Command_macroTailCommand_parenthesizer__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__7; x_2 = l_Lean_Parser_Command_macroTailCommand_parenthesizer___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -25615,7 +27423,7 @@ static lean_object* _init_l_Lean_Parser_Command_macroTailDefault_parenthesizer__ _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__8; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_atomic_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -25755,6 +27563,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_macroTail___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macroTail_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_macroTail___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__1() { _start: { @@ -25786,130 +27624,114 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macroArg_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_macro_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many1_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macroTail_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_macro_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_macro_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__8; -x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__10; -x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__7; +x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Syntax_cat_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__8; +x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_macro_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__15; -x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__10; +x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_macro__rules_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__11; +x_2 = l_Lean_Parser_Command_macro_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__13() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_macro_parenthesizer___closed__12; +x_1 = l_Lean_Parser_Command_macro_parenthesizer___closed__10; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_suppressInsideQuot_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_macro_parenthesizer___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_macro___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_macro_parenthesizer___closed__13; +x_3 = l_Lean_Parser_Command_macro_parenthesizer___closed__11; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -25922,11 +27744,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_macro_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_macro_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_macro_parenthesizer___closed__14; +x_7 = l_Lean_Parser_Command_macro_parenthesizer___closed__12; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_macro___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_macro_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_macro_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_macro___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_elab__rules___elambda__1___closed__1() { _start: { @@ -25981,7 +27833,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab__rules___elambda__1___close { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Command_syntax___closed__3; -x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__12; +x_2 = l_Lean_Parser_Command_syntax___elambda__1___closed__13; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -26579,7 +28431,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab__rules_formatter___closed__ _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax_formatter___closed__4; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -26723,6 +28575,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_elab__rules___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_elab__rules_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_elab__rules___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_elab__rules_parenthesizer___closed__1() { _start: { @@ -26755,7 +28637,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab__rules_parenthesizer___clos _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__8; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -26899,6 +28781,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_elab__rules___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_elab__rules_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_elab__rules___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_elabArg() { _start: { @@ -26988,7 +28900,7 @@ static lean_object* _init_l_Lean_Parser_Command_elabTail___elambda__1___closed__ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__11; +x_1 = l_Lean_Parser_Command_syntax___elambda__1___closed__12; x_2 = l_Lean_Parser_Command_elabTail___elambda__1___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_Parser_andthenFn), 4, 2); lean_closure_set(x_3, 0, x_1); @@ -27982,7 +29894,7 @@ static lean_object* _init_l_Lean_Parser_Command_elabTail_formatter___closed__3() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_formatter___closed__3; +x_1 = l_Lean_Parser_Command_syntax_formatter___closed__5; x_2 = l_Lean_Parser_Command_elabTail_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28048,6 +29960,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_elabTail___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_elabTail_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elabTail_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_elabTail___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__1() { _start: { @@ -28097,16 +30039,20 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_elabTail_formatter), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_elab_formatter___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; } } static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_elab_formatter___closed__4; +x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__8; x_2 = l_Lean_Parser_Command_elab_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28118,7 +30064,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__8; +x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__10; x_2 = l_Lean_Parser_Command_elab_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28130,7 +30076,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__10; +x_1 = l_Lean_Parser_Syntax_cat_formatter___closed__3; x_2 = l_Lean_Parser_Command_elab_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28142,7 +30088,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Syntax_cat_formatter___closed__3; +x_1 = l_Lean_Parser_Command_elab_formatter___closed__2; x_2 = l_Lean_Parser_Command_elab_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28154,7 +30100,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_elab_formatter___closed__2; +x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__15; x_2 = l_Lean_Parser_Command_elab_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28166,7 +30112,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfix_formatter___closed__15; +x_1 = l_Lean_Parser_Command_macro__rules_formatter___closed__3; x_2 = l_Lean_Parser_Command_elab_formatter___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28177,32 +30123,20 @@ return x_3; static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__12() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_macro__rules_formatter___closed__3; -x_2 = l_Lean_Parser_Command_elab_formatter___closed__11; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__13() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_elab_formatter___closed__12; +x_1 = l_Lean_Parser_Command_elab_formatter___closed__11; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_suppressInsideQuot_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_elab_formatter___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_elab___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_elab_formatter___closed__13; +x_3 = l_Lean_Parser_Command_elab_formatter___closed__12; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -28215,11 +30149,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_elab_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_elab_formatter___closed__1; -x_7 = l_Lean_Parser_Command_elab_formatter___closed__14; +x_7 = l_Lean_Parser_Command_elab_formatter___closed__13; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_elab___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_elab_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3; +x_3 = l_Lean_Parser_Command_elab___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Command_elabArg_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -28262,7 +30226,7 @@ static lean_object* _init_l_Lean_Parser_Command_elabTail_parenthesizer___closed_ _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Command_syntax_parenthesizer___closed__7; x_2 = l_Lean_Parser_Command_elabTail_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28328,6 +30292,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_elabTail___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_elabTail_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_elabTail___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__1() { _start: { @@ -28377,16 +30371,20 @@ return x_2; static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_elabTail_parenthesizer), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_elab_parenthesizer___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__2; +x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; } } static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_elab_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__8; x_2 = l_Lean_Parser_Command_elab_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28398,7 +30396,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__7() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__8; +x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__10; x_2 = l_Lean_Parser_Command_elab_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28410,7 +30408,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__8() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__10; +x_1 = l_Lean_Parser_Syntax_cat_parenthesizer___closed__3; x_2 = l_Lean_Parser_Command_elab_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28422,7 +30420,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__9() _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Syntax_cat_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Command_elab_parenthesizer___closed__2; x_2 = l_Lean_Parser_Command_elab_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28434,7 +30432,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__10( _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_elab_parenthesizer___closed__2; +x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__15; x_2 = l_Lean_Parser_Command_elab_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28446,7 +30444,7 @@ static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__11( _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_mixfix_parenthesizer___closed__15; +x_1 = l_Lean_Parser_Command_macro__rules_parenthesizer___closed__3; x_2 = l_Lean_Parser_Command_elab_parenthesizer___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -28457,32 +30455,20 @@ return x_3; static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__12() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Command_macro__rules_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Command_elab_parenthesizer___closed__11; -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__13() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Command_elab_parenthesizer___closed__12; +x_1 = l_Lean_Parser_Command_elab_parenthesizer___closed__11; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_suppressInsideQuot_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Command_elab_parenthesizer___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Command_elab___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Command_elab_parenthesizer___closed__13; +x_3 = l_Lean_Parser_Command_elab_parenthesizer___closed__12; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -28495,11 +30481,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_elab_parenthesizer(lean_object* x { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Command_elab_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Command_elab_parenthesizer___closed__14; +x_7 = l_Lean_Parser_Command_elab_parenthesizer___closed__13; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_elab___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_elab_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_elab_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_elab___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Command(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Tactic(uint8_t builtin, lean_object*); @@ -28747,6 +30763,17 @@ l_Lean_Parser_Syntax_paren_formatter___closed__7 = _init_l_Lean_Parser_Syntax_pa lean_mark_persistent(l_Lean_Parser_Syntax_paren_formatter___closed__7); l_Lean_Parser_Syntax_paren_formatter___closed__8 = _init_l_Lean_Parser_Syntax_paren_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Syntax_paren_formatter___closed__8); +l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__1); +l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__2); +l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__3); +l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_paren_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Syntax_paren_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_paren_parenthesizer___closed__1 = _init_l_Lean_Parser_Syntax_paren_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_paren_parenthesizer___closed__1); l_Lean_Parser_Syntax_paren_parenthesizer___closed__2 = _init_l_Lean_Parser_Syntax_paren_parenthesizer___closed__2(); @@ -28763,6 +30790,17 @@ l_Lean_Parser_Syntax_paren_parenthesizer___closed__7 = _init_l_Lean_Parser_Synta lean_mark_persistent(l_Lean_Parser_Syntax_paren_parenthesizer___closed__7); l_Lean_Parser_Syntax_paren_parenthesizer___closed__8 = _init_l_Lean_Parser_Syntax_paren_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Syntax_paren_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_Syntax_paren_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_cat___elambda__1___closed__1 = _init_l_Lean_Parser_Syntax_cat___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_cat___elambda__1___closed__1); l_Lean_Parser_Syntax_cat___elambda__1___closed__2 = _init_l_Lean_Parser_Syntax_cat___elambda__1___closed__2(); @@ -28825,10 +30863,15 @@ l_Lean_Parser_precedence_formatter___closed__4 = _init_l_Lean_Parser_precedence_ lean_mark_persistent(l_Lean_Parser_precedence_formatter___closed__4); l_Lean_Parser_precedence_formatter___closed__5 = _init_l_Lean_Parser_precedence_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_precedence_formatter___closed__5); +l___regBuiltin_Lean_Parser_precedence_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_precedence_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_precedence_formatter___closed__1); +l___regBuiltin_Lean_Parser_precedence_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_precedence_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_precedence_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_precedence_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_optPrecedence_formatter___closed__1 = _init_l_Lean_Parser_optPrecedence_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_optPrecedence_formatter___closed__1); -l_Lean_Parser_optPrecedence_formatter___closed__2 = _init_l_Lean_Parser_optPrecedence_formatter___closed__2(); -lean_mark_persistent(l_Lean_Parser_optPrecedence_formatter___closed__2); l_Lean_Parser_Syntax_cat_formatter___closed__1 = _init_l_Lean_Parser_Syntax_cat_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_cat_formatter___closed__1); l_Lean_Parser_Syntax_cat_formatter___closed__2 = _init_l_Lean_Parser_Syntax_cat_formatter___closed__2(); @@ -28839,6 +30882,13 @@ l_Lean_Parser_Syntax_cat_formatter___closed__4 = _init_l_Lean_Parser_Syntax_cat_ lean_mark_persistent(l_Lean_Parser_Syntax_cat_formatter___closed__4); l_Lean_Parser_Syntax_cat_formatter___closed__5 = _init_l_Lean_Parser_Syntax_cat_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Syntax_cat_formatter___closed__5); +l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__1); +l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_cat_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_cat_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_precedence_parenthesizer___closed__1 = _init_l_Lean_Parser_precedence_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_precedence_parenthesizer___closed__1); l_Lean_Parser_precedence_parenthesizer___closed__2 = _init_l_Lean_Parser_precedence_parenthesizer___closed__2(); @@ -28849,10 +30899,15 @@ l_Lean_Parser_precedence_parenthesizer___closed__4 = _init_l_Lean_Parser_precede lean_mark_persistent(l_Lean_Parser_precedence_parenthesizer___closed__4); l_Lean_Parser_precedence_parenthesizer___closed__5 = _init_l_Lean_Parser_precedence_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_precedence_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_precedence_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_precedence_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_optPrecedence_parenthesizer___closed__1 = _init_l_Lean_Parser_optPrecedence_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_optPrecedence_parenthesizer___closed__1); -l_Lean_Parser_optPrecedence_parenthesizer___closed__2 = _init_l_Lean_Parser_optPrecedence_parenthesizer___closed__2(); -lean_mark_persistent(l_Lean_Parser_optPrecedence_parenthesizer___closed__2); l_Lean_Parser_Syntax_cat_parenthesizer___closed__1 = _init_l_Lean_Parser_Syntax_cat_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_cat_parenthesizer___closed__1); l_Lean_Parser_Syntax_cat_parenthesizer___closed__2 = _init_l_Lean_Parser_Syntax_cat_parenthesizer___closed__2(); @@ -28863,6 +30918,13 @@ l_Lean_Parser_Syntax_cat_parenthesizer___closed__4 = _init_l_Lean_Parser_Syntax_ lean_mark_persistent(l_Lean_Parser_Syntax_cat_parenthesizer___closed__4); l_Lean_Parser_Syntax_cat_parenthesizer___closed__5 = _init_l_Lean_Parser_Syntax_cat_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Syntax_cat_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_cat_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_unary___elambda__1___closed__1 = _init_l_Lean_Parser_Syntax_unary___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_unary___elambda__1___closed__1); l_Lean_Parser_Syntax_unary___elambda__1___closed__2 = _init_l_Lean_Parser_Syntax_unary___elambda__1___closed__2(); @@ -28931,6 +30993,13 @@ l_Lean_Parser_Syntax_unary_formatter___closed__4 = _init_l_Lean_Parser_Syntax_un lean_mark_persistent(l_Lean_Parser_Syntax_unary_formatter___closed__4); l_Lean_Parser_Syntax_unary_formatter___closed__5 = _init_l_Lean_Parser_Syntax_unary_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Syntax_unary_formatter___closed__5); +l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__1); +l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_unary_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_unary_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_unary_parenthesizer___closed__1 = _init_l_Lean_Parser_Syntax_unary_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_unary_parenthesizer___closed__1); l_Lean_Parser_Syntax_unary_parenthesizer___closed__2 = _init_l_Lean_Parser_Syntax_unary_parenthesizer___closed__2(); @@ -28941,6 +31010,13 @@ l_Lean_Parser_Syntax_unary_parenthesizer___closed__4 = _init_l_Lean_Parser_Synta lean_mark_persistent(l_Lean_Parser_Syntax_unary_parenthesizer___closed__4); l_Lean_Parser_Syntax_unary_parenthesizer___closed__5 = _init_l_Lean_Parser_Syntax_unary_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Syntax_unary_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_unary_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_binary___elambda__1___closed__1 = _init_l_Lean_Parser_Syntax_binary___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_binary___elambda__1___closed__1); l_Lean_Parser_Syntax_binary___elambda__1___closed__2 = _init_l_Lean_Parser_Syntax_binary___elambda__1___closed__2(); @@ -29035,6 +31111,13 @@ l_Lean_Parser_Syntax_binary_formatter___closed__7 = _init_l_Lean_Parser_Syntax_b lean_mark_persistent(l_Lean_Parser_Syntax_binary_formatter___closed__7); l_Lean_Parser_Syntax_binary_formatter___closed__8 = _init_l_Lean_Parser_Syntax_binary_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Syntax_binary_formatter___closed__8); +l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__1); +l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_binary_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_binary_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_binary_parenthesizer___closed__1 = _init_l_Lean_Parser_Syntax_binary_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_binary_parenthesizer___closed__1); l_Lean_Parser_Syntax_binary_parenthesizer___closed__2 = _init_l_Lean_Parser_Syntax_binary_parenthesizer___closed__2(); @@ -29051,6 +31134,13 @@ l_Lean_Parser_Syntax_binary_parenthesizer___closed__7 = _init_l_Lean_Parser_Synt lean_mark_persistent(l_Lean_Parser_Syntax_binary_parenthesizer___closed__7); l_Lean_Parser_Syntax_binary_parenthesizer___closed__8 = _init_l_Lean_Parser_Syntax_binary_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Syntax_binary_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_binary_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_sepBy___elambda__1___closed__1 = _init_l_Lean_Parser_Syntax_sepBy___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_sepBy___elambda__1___closed__1); l_Lean_Parser_Syntax_sepBy___elambda__1___closed__2 = _init_l_Lean_Parser_Syntax_sepBy___elambda__1___closed__2(); @@ -29141,6 +31231,13 @@ l_Lean_Parser_Syntax_sepBy_formatter___closed__14 = _init_l_Lean_Parser_Syntax_s lean_mark_persistent(l_Lean_Parser_Syntax_sepBy_formatter___closed__14); l_Lean_Parser_Syntax_sepBy_formatter___closed__15 = _init_l_Lean_Parser_Syntax_sepBy_formatter___closed__15(); lean_mark_persistent(l_Lean_Parser_Syntax_sepBy_formatter___closed__15); +l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__1); +l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_sepBy_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1 = _init_l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1); l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2 = _init_l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2(); @@ -29171,6 +31268,13 @@ l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__14 = _init_l_Lean_Parser_Synt lean_mark_persistent(l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__14); l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__15 = _init_l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__15(); lean_mark_persistent(l_Lean_Parser_Syntax_sepBy_parenthesizer___closed__15); +l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_sepBy_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__1 = _init_l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__1); l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__2 = _init_l_Lean_Parser_Syntax_sepBy1___elambda__1___closed__2(); @@ -29269,6 +31373,13 @@ l_Lean_Parser_Syntax_sepBy1_formatter___closed__3 = _init_l_Lean_Parser_Syntax_s lean_mark_persistent(l_Lean_Parser_Syntax_sepBy1_formatter___closed__3); l_Lean_Parser_Syntax_sepBy1_formatter___closed__4 = _init_l_Lean_Parser_Syntax_sepBy1_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Syntax_sepBy1_formatter___closed__4); +l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__1); +l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_sepBy1_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1 = _init_l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1); l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2 = _init_l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2(); @@ -29277,6 +31388,13 @@ l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__3 = _init_l_Lean_Parser_Synt lean_mark_persistent(l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__3); l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__4 = _init_l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_sepBy1_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_atom___elambda__1___closed__1 = _init_l_Lean_Parser_Syntax_atom___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_atom___elambda__1___closed__1); l_Lean_Parser_Syntax_atom___elambda__1___closed__2 = _init_l_Lean_Parser_Syntax_atom___elambda__1___closed__2(); @@ -29327,10 +31445,24 @@ l_Lean_Parser_Syntax_atom_formatter___closed__1 = _init_l_Lean_Parser_Syntax_ato lean_mark_persistent(l_Lean_Parser_Syntax_atom_formatter___closed__1); l_Lean_Parser_Syntax_atom_formatter___closed__2 = _init_l_Lean_Parser_Syntax_atom_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Syntax_atom_formatter___closed__2); +l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__1); +l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_atom_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_atom_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_atom_parenthesizer___closed__1 = _init_l_Lean_Parser_Syntax_atom_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_atom_parenthesizer___closed__1); l_Lean_Parser_Syntax_atom_parenthesizer___closed__2 = _init_l_Lean_Parser_Syntax_atom_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Syntax_atom_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_atom_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__1 = _init_l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__1); l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__2 = _init_l_Lean_Parser_Syntax_nonReserved___elambda__1___closed__2(); @@ -29401,6 +31533,13 @@ l_Lean_Parser_Syntax_nonReserved_formatter___closed__3 = _init_l_Lean_Parser_Syn lean_mark_persistent(l_Lean_Parser_Syntax_nonReserved_formatter___closed__3); l_Lean_Parser_Syntax_nonReserved_formatter___closed__4 = _init_l_Lean_Parser_Syntax_nonReserved_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Syntax_nonReserved_formatter___closed__4); +l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__1); +l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_nonReserved_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1 = _init_l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1); l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__2 = _init_l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__2(); @@ -29409,6 +31548,13 @@ l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__3 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__3); l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__4 = _init_l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Syntax_nonReserved_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_stx_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_stx_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_stx_quot___elambda__1___closed__1); l_Lean_Parser_Term_stx_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_stx_quot___elambda__1___closed__2(); @@ -29503,6 +31649,13 @@ l_Lean_Parser_Term_stx_quot_formatter___closed__5 = _init_l_Lean_Parser_Term_stx lean_mark_persistent(l_Lean_Parser_Term_stx_quot_formatter___closed__5); l_Lean_Parser_Term_stx_quot_formatter___closed__6 = _init_l_Lean_Parser_Term_stx_quot_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_stx_quot_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_stx_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_stx_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_stx_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_stx_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_stx_quot_parenthesizer___closed__1); l_Lean_Parser_Term_stx_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_stx_quot_parenthesizer___closed__2(); @@ -29515,6 +31668,13 @@ l_Lean_Parser_Term_stx_quot_parenthesizer___closed__5 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_stx_quot_parenthesizer___closed__5); l_Lean_Parser_Term_stx_quot_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_stx_quot_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_stx_quot_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_stx_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_prec_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_prec_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_prec_quot___elambda__1___closed__1); l_Lean_Parser_Term_prec_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_prec_quot___elambda__1___closed__2(); @@ -29599,6 +31759,13 @@ l_Lean_Parser_Term_prec_quot_formatter___closed__5 = _init_l_Lean_Parser_Term_pr lean_mark_persistent(l_Lean_Parser_Term_prec_quot_formatter___closed__5); l_Lean_Parser_Term_prec_quot_formatter___closed__6 = _init_l_Lean_Parser_Term_prec_quot_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_prec_quot_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prec_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_prec_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_prec_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_prec_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_prec_quot_parenthesizer___closed__1); l_Lean_Parser_Term_prec_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_prec_quot_parenthesizer___closed__2(); @@ -29613,6 +31780,13 @@ l_Lean_Parser_Term_prec_quot_parenthesizer___closed__6 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_prec_quot_parenthesizer___closed__6); l_Lean_Parser_Term_prec_quot_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_prec_quot_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_prec_quot_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_prec_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_prio_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_prio_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_prio_quot___elambda__1___closed__1); l_Lean_Parser_Term_prio_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_prio_quot___elambda__1___closed__2(); @@ -29703,6 +31877,13 @@ l_Lean_Parser_Term_prio_quot_formatter___closed__6 = _init_l_Lean_Parser_Term_pr lean_mark_persistent(l_Lean_Parser_Term_prio_quot_formatter___closed__6); l_Lean_Parser_Term_prio_quot_formatter___closed__7 = _init_l_Lean_Parser_Term_prio_quot_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_prio_quot_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prio_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_prio_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_prio_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_prio_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_prio_quot_parenthesizer___closed__1); l_Lean_Parser_Term_prio_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_prio_quot_parenthesizer___closed__2(); @@ -29717,6 +31898,13 @@ l_Lean_Parser_Term_prio_quot_parenthesizer___closed__6 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_prio_quot_parenthesizer___closed__6); l_Lean_Parser_Term_prio_quot_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_prio_quot_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_prio_quot_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_prio_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_namedName___elambda__1___closed__1 = _init_l_Lean_Parser_Command_namedName___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_namedName___elambda__1___closed__1); l_Lean_Parser_Command_namedName___elambda__1___closed__2 = _init_l_Lean_Parser_Command_namedName___elambda__1___closed__2(); @@ -30087,46 +32275,71 @@ l_Lean_Parser_Command_prefix_formatter___closed__2 = _init_l_Lean_Parser_Command lean_mark_persistent(l_Lean_Parser_Command_prefix_formatter___closed__2); l_Lean_Parser_Command_prefix_formatter___closed__3 = _init_l_Lean_Parser_Command_prefix_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_prefix_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_prefix_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_prefix_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_infix_formatter___closed__1 = _init_l_Lean_Parser_Command_infix_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_infix_formatter___closed__1); l_Lean_Parser_Command_infix_formatter___closed__2 = _init_l_Lean_Parser_Command_infix_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_infix_formatter___closed__2); l_Lean_Parser_Command_infix_formatter___closed__3 = _init_l_Lean_Parser_Command_infix_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_infix_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infix_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_infix_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_infixl_formatter___closed__1 = _init_l_Lean_Parser_Command_infixl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_infixl_formatter___closed__1); l_Lean_Parser_Command_infixl_formatter___closed__2 = _init_l_Lean_Parser_Command_infixl_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_infixl_formatter___closed__2); l_Lean_Parser_Command_infixl_formatter___closed__3 = _init_l_Lean_Parser_Command_infixl_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_infixl_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infixl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_infixl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_infixr_formatter___closed__1 = _init_l_Lean_Parser_Command_infixr_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_infixr_formatter___closed__1); l_Lean_Parser_Command_infixr_formatter___closed__2 = _init_l_Lean_Parser_Command_infixr_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_infixr_formatter___closed__2); l_Lean_Parser_Command_infixr_formatter___closed__3 = _init_l_Lean_Parser_Command_infixr_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_infixr_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infixr_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_infixr_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_postfix_formatter___closed__1 = _init_l_Lean_Parser_Command_postfix_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_postfix_formatter___closed__1); l_Lean_Parser_Command_postfix_formatter___closed__2 = _init_l_Lean_Parser_Command_postfix_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_postfix_formatter___closed__2); l_Lean_Parser_Command_postfix_formatter___closed__3 = _init_l_Lean_Parser_Command_postfix_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_postfix_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_postfix_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_postfix_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_mixfixKind_formatter___closed__1 = _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_formatter___closed__1); l_Lean_Parser_Command_mixfixKind_formatter___closed__2 = _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_formatter___closed__2); l_Lean_Parser_Command_mixfixKind_formatter___closed__3 = _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_formatter___closed__3); -l_Lean_Parser_Command_mixfixKind_formatter___closed__4 = _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_formatter___closed__4); -l_Lean_Parser_Command_mixfixKind_formatter___closed__5 = _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_formatter___closed__5); -l_Lean_Parser_Command_mixfixKind_formatter___closed__6 = _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_formatter___closed__6); -l_Lean_Parser_Command_mixfixKind_formatter___closed__7 = _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_formatter___closed__7); -l_Lean_Parser_Command_mixfixKind_formatter___closed__8 = _init_l_Lean_Parser_Command_mixfixKind_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_formatter___closed__8); l_Lean_Parser_Command_namedName_formatter___closed__1 = _init_l_Lean_Parser_Command_namedName_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_namedName_formatter___closed__1); l_Lean_Parser_Command_namedName_formatter___closed__2 = _init_l_Lean_Parser_Command_namedName_formatter___closed__2(); @@ -30145,8 +32358,13 @@ l_Lean_Parser_Command_namedName_formatter___closed__8 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_namedName_formatter___closed__8); l_Lean_Parser_Command_namedName_formatter___closed__9 = _init_l_Lean_Parser_Command_namedName_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_namedName_formatter___closed__9); -l_Lean_Parser_Command_optNamedName_formatter___closed__1 = _init_l_Lean_Parser_Command_optNamedName_formatter___closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_optNamedName_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namedName_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_namedName_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_mixfix_formatter___closed__1 = _init_l_Lean_Parser_Command_mixfix_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_mixfix_formatter___closed__1); l_Lean_Parser_Command_mixfix_formatter___closed__2 = _init_l_Lean_Parser_Command_mixfix_formatter___closed__2(); @@ -30181,52 +32399,84 @@ l_Lean_Parser_Command_mixfix_formatter___closed__16 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_mixfix_formatter___closed__16); l_Lean_Parser_Command_mixfix_formatter___closed__17 = _init_l_Lean_Parser_Command_mixfix_formatter___closed__17(); lean_mark_persistent(l_Lean_Parser_Command_mixfix_formatter___closed__17); +l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_mixfix_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_mixfix_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_prefix_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_prefix_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_prefix_parenthesizer___closed__1); l_Lean_Parser_Command_prefix_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_prefix_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_prefix_parenthesizer___closed__2); l_Lean_Parser_Command_prefix_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_prefix_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_prefix_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_prefix_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_infix_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_infix_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_infix_parenthesizer___closed__1); l_Lean_Parser_Command_infix_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_infix_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_infix_parenthesizer___closed__2); l_Lean_Parser_Command_infix_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_infix_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_infix_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infix_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_infix_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_infixl_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_infixl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_infixl_parenthesizer___closed__1); l_Lean_Parser_Command_infixl_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_infixl_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_infixl_parenthesizer___closed__2); l_Lean_Parser_Command_infixl_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_infixl_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_infixl_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_infixl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_infixr_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_infixr_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_infixr_parenthesizer___closed__1); l_Lean_Parser_Command_infixr_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_infixr_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_infixr_parenthesizer___closed__2); l_Lean_Parser_Command_infixr_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_infixr_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_infixr_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_infixr_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_postfix_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_postfix_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_postfix_parenthesizer___closed__1); l_Lean_Parser_Command_postfix_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_postfix_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_postfix_parenthesizer___closed__2); l_Lean_Parser_Command_postfix_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_postfix_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_postfix_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_postfix_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__1); l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__2); l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__3); -l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__4); -l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__5 = _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__5); -l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__6); -l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__7); -l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_mixfixKind_parenthesizer___closed__8); l_Lean_Parser_Command_namedName_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_namedName_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_namedName_parenthesizer___closed__1); l_Lean_Parser_Command_namedName_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_namedName_parenthesizer___closed__2(); @@ -30245,8 +32495,13 @@ l_Lean_Parser_Command_namedName_parenthesizer___closed__8 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_namedName_parenthesizer___closed__8); l_Lean_Parser_Command_namedName_parenthesizer___closed__9 = _init_l_Lean_Parser_Command_namedName_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Command_namedName_parenthesizer___closed__9); -l_Lean_Parser_Command_optNamedName_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_optNamedName_parenthesizer___closed__1(); -lean_mark_persistent(l_Lean_Parser_Command_optNamedName_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_namedName_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_mixfix_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_mixfix_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_mixfix_parenthesizer___closed__1); l_Lean_Parser_Command_mixfix_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_mixfix_parenthesizer___closed__2(); @@ -30281,6 +32536,13 @@ l_Lean_Parser_Command_mixfix_parenthesizer___closed__16 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_mixfix_parenthesizer___closed__16); l_Lean_Parser_Command_mixfix_parenthesizer___closed__17 = _init_l_Lean_Parser_Command_mixfix_parenthesizer___closed__17(); lean_mark_persistent(l_Lean_Parser_Command_mixfix_parenthesizer___closed__17); +l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_mixfix_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_identPrec___elambda__1___closed__1 = _init_l_Lean_Parser_Command_identPrec___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_identPrec___elambda__1___closed__1); l_Lean_Parser_Command_identPrec___elambda__1___closed__2 = _init_l_Lean_Parser_Command_identPrec___elambda__1___closed__2(); @@ -30447,14 +32709,19 @@ l_Lean_Parser_Command_identPrec_formatter___closed__1 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_identPrec_formatter___closed__1); l_Lean_Parser_Command_identPrec_formatter___closed__2 = _init_l_Lean_Parser_Command_identPrec_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_identPrec_formatter___closed__2); +l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_identPrec_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_identPrec_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_notationItem_formatter___closed__1 = _init_l_Lean_Parser_Command_notationItem_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_notationItem_formatter___closed__1); l_Lean_Parser_Command_notationItem_formatter___closed__2 = _init_l_Lean_Parser_Command_notationItem_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_notationItem_formatter___closed__2); l_Lean_Parser_Command_notationItem_formatter___closed__3 = _init_l_Lean_Parser_Command_notationItem_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_notationItem_formatter___closed__3); -l_Lean_Parser_Command_notationItem_formatter___closed__4 = _init_l_Lean_Parser_Command_notationItem_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_notationItem_formatter___closed__4); l_Lean_Parser_Command_notation_formatter___closed__1 = _init_l_Lean_Parser_Command_notation_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_notation_formatter___closed__1); l_Lean_Parser_Command_notation_formatter___closed__2 = _init_l_Lean_Parser_Command_notation_formatter___closed__2(); @@ -30477,18 +32744,30 @@ l_Lean_Parser_Command_notation_formatter___closed__10 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_notation_formatter___closed__10); l_Lean_Parser_Command_notation_formatter___closed__11 = _init_l_Lean_Parser_Command_notation_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_notation_formatter___closed__11); +l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_notation_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_notation_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_identPrec_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_identPrec_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_identPrec_parenthesizer___closed__1); l_Lean_Parser_Command_identPrec_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_identPrec_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_identPrec_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_identPrec_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_notationItem_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_notationItem_parenthesizer___closed__1); l_Lean_Parser_Command_notationItem_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_notationItem_parenthesizer___closed__2); l_Lean_Parser_Command_notationItem_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_notationItem_parenthesizer___closed__3); -l_Lean_Parser_Command_notationItem_parenthesizer___closed__4 = _init_l_Lean_Parser_Command_notationItem_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Command_notationItem_parenthesizer___closed__4); l_Lean_Parser_Command_notation_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_notation_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_notation_parenthesizer___closed__1); l_Lean_Parser_Command_notation_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_notation_parenthesizer___closed__2(); @@ -30511,6 +32790,13 @@ l_Lean_Parser_Command_notation_parenthesizer___closed__10 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_notation_parenthesizer___closed__10); l_Lean_Parser_Command_notation_parenthesizer___closed__11 = _init_l_Lean_Parser_Command_notation_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Command_notation_parenthesizer___closed__11); +l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_notation_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_notation_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_macro__rules___elambda__1___closed__1 = _init_l_Lean_Parser_Command_macro__rules___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_macro__rules___elambda__1___closed__1); l_Lean_Parser_Command_macro__rules___elambda__1___closed__2 = _init_l_Lean_Parser_Command_macro__rules___elambda__1___closed__2(); @@ -30701,6 +32987,10 @@ l_Lean_Parser_Command_syntax___elambda__1___closed__25 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_syntax___elambda__1___closed__25); l_Lean_Parser_Command_syntax___elambda__1___closed__26 = _init_l_Lean_Parser_Command_syntax___elambda__1___closed__26(); lean_mark_persistent(l_Lean_Parser_Command_syntax___elambda__1___closed__26); +l_Lean_Parser_Command_syntax___elambda__1___closed__27 = _init_l_Lean_Parser_Command_syntax___elambda__1___closed__27(); +lean_mark_persistent(l_Lean_Parser_Command_syntax___elambda__1___closed__27); +l_Lean_Parser_Command_syntax___elambda__1___closed__28 = _init_l_Lean_Parser_Command_syntax___elambda__1___closed__28(); +lean_mark_persistent(l_Lean_Parser_Command_syntax___elambda__1___closed__28); l_Lean_Parser_Command_syntax___closed__1 = _init_l_Lean_Parser_Command_syntax___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_syntax___closed__1); l_Lean_Parser_Command_syntax___closed__2 = _init_l_Lean_Parser_Command_syntax___closed__2(); @@ -30733,6 +33023,8 @@ l_Lean_Parser_Command_syntax___closed__15 = _init_l_Lean_Parser_Command_syntax__ lean_mark_persistent(l_Lean_Parser_Command_syntax___closed__15); l_Lean_Parser_Command_syntax___closed__16 = _init_l_Lean_Parser_Command_syntax___closed__16(); lean_mark_persistent(l_Lean_Parser_Command_syntax___closed__16); +l_Lean_Parser_Command_syntax___closed__17 = _init_l_Lean_Parser_Command_syntax___closed__17(); +lean_mark_persistent(l_Lean_Parser_Command_syntax___closed__17); l_Lean_Parser_Command_syntax = _init_l_Lean_Parser_Command_syntax(); lean_mark_persistent(l_Lean_Parser_Command_syntax); res = l___regBuiltin_Lean_Parser_Command_syntax(lean_io_mk_world()); @@ -30779,6 +33071,19 @@ l_Lean_Parser_Command_syntax_formatter___closed__11 = _init_l_Lean_Parser_Comman lean_mark_persistent(l_Lean_Parser_Command_syntax_formatter___closed__11); l_Lean_Parser_Command_syntax_formatter___closed__12 = _init_l_Lean_Parser_Command_syntax_formatter___closed__12(); lean_mark_persistent(l_Lean_Parser_Command_syntax_formatter___closed__12); +l_Lean_Parser_Command_syntax_formatter___closed__13 = _init_l_Lean_Parser_Command_syntax_formatter___closed__13(); +lean_mark_persistent(l_Lean_Parser_Command_syntax_formatter___closed__13); +l_Lean_Parser_Command_syntax_formatter___closed__14 = _init_l_Lean_Parser_Command_syntax_formatter___closed__14(); +lean_mark_persistent(l_Lean_Parser_Command_syntax_formatter___closed__14); +l_Lean_Parser_Command_syntax_formatter___closed__15 = _init_l_Lean_Parser_Command_syntax_formatter___closed__15(); +lean_mark_persistent(l_Lean_Parser_Command_syntax_formatter___closed__15); +l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntax_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_syntax_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_syntax_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_syntax_parenthesizer___closed__1); l_Lean_Parser_Command_syntax_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__2(); @@ -30807,6 +33112,19 @@ l_Lean_Parser_Command_syntax_parenthesizer___closed__13 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_syntax_parenthesizer___closed__13); l_Lean_Parser_Command_syntax_parenthesizer___closed__14 = _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__14(); lean_mark_persistent(l_Lean_Parser_Command_syntax_parenthesizer___closed__14); +l_Lean_Parser_Command_syntax_parenthesizer___closed__15 = _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__15(); +lean_mark_persistent(l_Lean_Parser_Command_syntax_parenthesizer___closed__15); +l_Lean_Parser_Command_syntax_parenthesizer___closed__16 = _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__16(); +lean_mark_persistent(l_Lean_Parser_Command_syntax_parenthesizer___closed__16); +l_Lean_Parser_Command_syntax_parenthesizer___closed__17 = _init_l_Lean_Parser_Command_syntax_parenthesizer___closed__17(); +lean_mark_persistent(l_Lean_Parser_Command_syntax_parenthesizer___closed__17); +l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_syntax_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__1 = _init_l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__1); l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__2 = _init_l_Lean_Parser_Command_syntaxAbbrev___elambda__1___closed__2(); @@ -30881,6 +33199,13 @@ l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__5 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__5); l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__6 = _init_l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_syntaxAbbrev_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1); l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2(); @@ -30893,6 +33218,13 @@ l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__5 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__5); l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_syntaxAbbrev_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__1 = _init_l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__1); l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__2 = _init_l_Lean_Parser_Command_catBehaviorBoth___elambda__1___closed__2(); @@ -31075,12 +33407,26 @@ l_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2); l_Lean_Parser_Command_catBehaviorBoth_formatter___closed__3 = _init_l_Lean_Parser_Command_catBehaviorBoth_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorBoth_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1 = _init_l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1); l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2 = _init_l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2); l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__3 = _init_l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__3); +l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_catBehavior_formatter___closed__1 = _init_l_Lean_Parser_Command_catBehavior_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_catBehavior_formatter___closed__1); l_Lean_Parser_Command_catBehavior_formatter___closed__2 = _init_l_Lean_Parser_Command_catBehavior_formatter___closed__2(); @@ -31093,10 +33439,6 @@ l_Lean_Parser_Command_catBehavior_formatter___closed__5 = _init_l_Lean_Parser_Co lean_mark_persistent(l_Lean_Parser_Command_catBehavior_formatter___closed__5); l_Lean_Parser_Command_catBehavior_formatter___closed__6 = _init_l_Lean_Parser_Command_catBehavior_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_catBehavior_formatter___closed__6); -l_Lean_Parser_Command_catBehavior_formatter___closed__7 = _init_l_Lean_Parser_Command_catBehavior_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_catBehavior_formatter___closed__7); -l_Lean_Parser_Command_catBehavior_formatter___closed__8 = _init_l_Lean_Parser_Command_catBehavior_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_catBehavior_formatter___closed__8); l_Lean_Parser_Command_syntaxCat_formatter___closed__1 = _init_l_Lean_Parser_Command_syntaxCat_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_syntaxCat_formatter___closed__1); l_Lean_Parser_Command_syntaxCat_formatter___closed__2 = _init_l_Lean_Parser_Command_syntaxCat_formatter___closed__2(); @@ -31109,18 +33451,39 @@ l_Lean_Parser_Command_syntaxCat_formatter___closed__5 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_syntaxCat_formatter___closed__5); l_Lean_Parser_Command_syntaxCat_formatter___closed__6 = _init_l_Lean_Parser_Command_syntaxCat_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_syntaxCat_formatter___closed__6); +l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_syntaxCat_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1); l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2); l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_catBehaviorBoth_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1); l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2); l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__3 = _init_l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_catBehaviorSymbol_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_catBehavior_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_catBehavior_parenthesizer___closed__1); l_Lean_Parser_Command_catBehavior_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__2(); @@ -31133,10 +33496,6 @@ l_Lean_Parser_Command_catBehavior_parenthesizer___closed__5 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Command_catBehavior_parenthesizer___closed__5); l_Lean_Parser_Command_catBehavior_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_catBehavior_parenthesizer___closed__6); -l_Lean_Parser_Command_catBehavior_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Command_catBehavior_parenthesizer___closed__7); -l_Lean_Parser_Command_catBehavior_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_catBehavior_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Command_catBehavior_parenthesizer___closed__8); l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1); l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2(); @@ -31149,6 +33508,13 @@ l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__5 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__5); l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__6 = _init_l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Command_syntaxCat_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_syntaxCat_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_macroArg___elambda__1___closed__1 = _init_l_Lean_Parser_Command_macroArg___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_macroArg___elambda__1___closed__1); l_Lean_Parser_Command_macroArg___elambda__1___closed__2 = _init_l_Lean_Parser_Command_macroArg___elambda__1___closed__2(); @@ -31419,6 +33785,13 @@ l_Lean_Parser_Command_macroArg_formatter___closed__6 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_macroArg_formatter___closed__6); l_Lean_Parser_Command_macroArg_formatter___closed__7 = _init_l_Lean_Parser_Command_macroArg_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_macroArg_formatter___closed__7); +l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macroArg_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_macroArg_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_macroRhs_formatter___closed__1 = _init_l_Lean_Parser_Command_macroRhs_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_macroRhs_formatter___closed__1); l_Lean_Parser_Command_macroRhs_formatter___closed__2 = _init_l_Lean_Parser_Command_macroRhs_formatter___closed__2(); @@ -31467,6 +33840,13 @@ l_Lean_Parser_Command_macroTail_formatter___closed__6 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_macroTail_formatter___closed__6); l_Lean_Parser_Command_macroTail_formatter___closed__7 = _init_l_Lean_Parser_Command_macroTail_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_macroTail_formatter___closed__7); +l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macroTail_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_macroTail_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_macro_formatter___closed__1 = _init_l_Lean_Parser_Command_macro_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_macro_formatter___closed__1); l_Lean_Parser_Command_macro_formatter___closed__2 = _init_l_Lean_Parser_Command_macro_formatter___closed__2(); @@ -31491,10 +33871,13 @@ l_Lean_Parser_Command_macro_formatter___closed__11 = _init_l_Lean_Parser_Command lean_mark_persistent(l_Lean_Parser_Command_macro_formatter___closed__11); l_Lean_Parser_Command_macro_formatter___closed__12 = _init_l_Lean_Parser_Command_macro_formatter___closed__12(); lean_mark_persistent(l_Lean_Parser_Command_macro_formatter___closed__12); -l_Lean_Parser_Command_macro_formatter___closed__13 = _init_l_Lean_Parser_Command_macro_formatter___closed__13(); -lean_mark_persistent(l_Lean_Parser_Command_macro_formatter___closed__13); -l_Lean_Parser_Command_macro_formatter___closed__14 = _init_l_Lean_Parser_Command_macro_formatter___closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_macro_formatter___closed__14); +l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macro_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_macro_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_macroArg_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_macroArg_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_macroArg_parenthesizer___closed__1); l_Lean_Parser_Command_macroArg_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_macroArg_parenthesizer___closed__2(); @@ -31509,6 +33892,13 @@ l_Lean_Parser_Command_macroArg_parenthesizer___closed__6 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_macroArg_parenthesizer___closed__6); l_Lean_Parser_Command_macroArg_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_macroArg_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_macroArg_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_macroArg_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_macroRhs_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_macroRhs_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_macroRhs_parenthesizer___closed__1); l_Lean_Parser_Command_macroRhs_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_macroRhs_parenthesizer___closed__2(); @@ -31563,6 +33953,13 @@ l_Lean_Parser_Command_macroTail_parenthesizer___closed__6 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Command_macroTail_parenthesizer___closed__6); l_Lean_Parser_Command_macroTail_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_macroTail_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_macroTail_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_macroTail_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_macro_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_macro_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_macro_parenthesizer___closed__1); l_Lean_Parser_Command_macro_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_macro_parenthesizer___closed__2(); @@ -31587,10 +33984,13 @@ l_Lean_Parser_Command_macro_parenthesizer___closed__11 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_macro_parenthesizer___closed__11); l_Lean_Parser_Command_macro_parenthesizer___closed__12 = _init_l_Lean_Parser_Command_macro_parenthesizer___closed__12(); lean_mark_persistent(l_Lean_Parser_Command_macro_parenthesizer___closed__12); -l_Lean_Parser_Command_macro_parenthesizer___closed__13 = _init_l_Lean_Parser_Command_macro_parenthesizer___closed__13(); -lean_mark_persistent(l_Lean_Parser_Command_macro_parenthesizer___closed__13); -l_Lean_Parser_Command_macro_parenthesizer___closed__14 = _init_l_Lean_Parser_Command_macro_parenthesizer___closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_macro_parenthesizer___closed__14); +l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_macro_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_macro_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_elab__rules___elambda__1___closed__1 = _init_l_Lean_Parser_Command_elab__rules___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_elab__rules___elambda__1___closed__1); l_Lean_Parser_Command_elab__rules___elambda__1___closed__2 = _init_l_Lean_Parser_Command_elab__rules___elambda__1___closed__2(); @@ -31717,6 +34117,13 @@ l_Lean_Parser_Command_elab__rules_formatter___closed__13 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_elab__rules_formatter___closed__13); l_Lean_Parser_Command_elab__rules_formatter___closed__14 = _init_l_Lean_Parser_Command_elab__rules_formatter___closed__14(); lean_mark_persistent(l_Lean_Parser_Command_elab__rules_formatter___closed__14); +l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elab__rules_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_elab__rules_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_elab__rules_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_elab__rules_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_elab__rules_parenthesizer___closed__1); l_Lean_Parser_Command_elab__rules_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_elab__rules_parenthesizer___closed__2(); @@ -31745,6 +34152,13 @@ l_Lean_Parser_Command_elab__rules_parenthesizer___closed__13 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Command_elab__rules_parenthesizer___closed__13); l_Lean_Parser_Command_elab__rules_parenthesizer___closed__14 = _init_l_Lean_Parser_Command_elab__rules_parenthesizer___closed__14(); lean_mark_persistent(l_Lean_Parser_Command_elab__rules_parenthesizer___closed__14); +l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_elab__rules_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_elabArg = _init_l_Lean_Parser_Command_elabArg(); lean_mark_persistent(l_Lean_Parser_Command_elabArg); l_Lean_Parser_Command_elabTail___elambda__1___closed__1 = _init_l_Lean_Parser_Command_elabTail___elambda__1___closed__1(); @@ -31899,6 +34313,13 @@ l_Lean_Parser_Command_elabTail_formatter___closed__6 = _init_l_Lean_Parser_Comma lean_mark_persistent(l_Lean_Parser_Command_elabTail_formatter___closed__6); l_Lean_Parser_Command_elabTail_formatter___closed__7 = _init_l_Lean_Parser_Command_elabTail_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_elabTail_formatter___closed__7); +l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elabTail_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_elabTail_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_elab_formatter___closed__1 = _init_l_Lean_Parser_Command_elab_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_elab_formatter___closed__1); l_Lean_Parser_Command_elab_formatter___closed__2 = _init_l_Lean_Parser_Command_elab_formatter___closed__2(); @@ -31925,8 +34346,13 @@ l_Lean_Parser_Command_elab_formatter___closed__12 = _init_l_Lean_Parser_Command_ lean_mark_persistent(l_Lean_Parser_Command_elab_formatter___closed__12); l_Lean_Parser_Command_elab_formatter___closed__13 = _init_l_Lean_Parser_Command_elab_formatter___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_elab_formatter___closed__13); -l_Lean_Parser_Command_elab_formatter___closed__14 = _init_l_Lean_Parser_Command_elab_formatter___closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_elab_formatter___closed__14); +l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elab_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_elab_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_elabTail_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_elabTail_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_elabTail_parenthesizer___closed__1); l_Lean_Parser_Command_elabTail_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_elabTail_parenthesizer___closed__2(); @@ -31941,6 +34367,13 @@ l_Lean_Parser_Command_elabTail_parenthesizer___closed__6 = _init_l_Lean_Parser_C lean_mark_persistent(l_Lean_Parser_Command_elabTail_parenthesizer___closed__6); l_Lean_Parser_Command_elabTail_parenthesizer___closed__7 = _init_l_Lean_Parser_Command_elabTail_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Command_elabTail_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_elabTail_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_elab_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_elab_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_elab_parenthesizer___closed__1); l_Lean_Parser_Command_elab_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_elab_parenthesizer___closed__2(); @@ -31967,8 +34400,13 @@ l_Lean_Parser_Command_elab_parenthesizer___closed__12 = _init_l_Lean_Parser_Comm lean_mark_persistent(l_Lean_Parser_Command_elab_parenthesizer___closed__12); l_Lean_Parser_Command_elab_parenthesizer___closed__13 = _init_l_Lean_Parser_Command_elab_parenthesizer___closed__13(); lean_mark_persistent(l_Lean_Parser_Command_elab_parenthesizer___closed__13); -l_Lean_Parser_Command_elab_parenthesizer___closed__14 = _init_l_Lean_Parser_Command_elab_parenthesizer___closed__14(); -lean_mark_persistent(l_Lean_Parser_Command_elab_parenthesizer___closed__14); +l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_elab_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_elab_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Parser/Tactic.c b/stage0/stdlib/Lean/Parser/Tactic.c index 1467bddca164..32359296fe13 100644 --- a/stage0/stdlib/Lean/Parser/Tactic.c +++ b/stage0/stdlib/Lean/Parser/Tactic.c @@ -14,14 +14,17 @@ extern "C" { #endif static lean_object* l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Tactic_introMatch___closed__7; static lean_object* l_Lean_Parser_Tactic_unknown___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Tactic_nestedTactic_declRange___closed__3; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__10; lean_object* l_Lean_Parser_nonReservedSymbol_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_matchRhs_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_nestedTactic_declRange___closed__4; static lean_object* l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_match_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_declRange___closed__4; static lean_object* l_Lean_Parser_Tactic_unknown___closed__9; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_declRange(lean_object*); @@ -50,6 +53,7 @@ static lean_object* l_Lean_Parser_Tactic_decide___elambda__1___closed__3; static lean_object* l_Lean_Parser_Tactic_match___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_declRange___closed__4; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__2; lean_object* l_Lean_Parser_symbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_nativeDecide_formatter___closed__2; lean_object* l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -63,6 +67,7 @@ static lean_object* l_Lean_Parser_Tactic_match_formatter___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_declRange(lean_object*); lean_object* l_Lean_Parser_Term_hole___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_unknown___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_introMatch___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed; static lean_object* l_Lean_Parser_Tactic_initFn____x40_Lean_Parser_Tactic___hyg_6____closed__19; @@ -82,6 +87,7 @@ lean_object* l_Lean_Parser_ParserState_mkNode(lean_object*, lean_object*, lean_o static lean_object* l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_matchRhs___closed__1; static lean_object* l_Lean_Parser_Tactic_introMatch___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown(lean_object*); static lean_object* l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_declRange___closed__7; @@ -90,6 +96,7 @@ static lean_object* l_Lean_Parser_Tactic_decide___elambda__1___closed__5; lean_object* l_Lean_Parser_orelseFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_matchRhs_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_matchRhs_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_decide___closed__6; lean_object* l_Lean_Parser_addBuiltinParser(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_unknown___closed__2; @@ -119,6 +126,7 @@ static lean_object* l_Lean_Parser_Tactic_unknown___closed__1; lean_object* l_Lean_Parser_mkAntiquot_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_matchRhs___closed__4; +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_nestedTactic_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -131,6 +139,7 @@ static lean_object* l_Lean_Parser_Tactic_initFn____x40_Lean_Parser_Tactic___hyg_ static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__2; lean_object* l_Lean_Parser_checkPrecFn(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Term_motive_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_unknown_formatter___closed__6; static lean_object* l_Lean_Parser_Tactic_matchRhs_formatter___closed__3; lean_object* l_Lean_Parser_optional(lean_object*); @@ -145,9 +154,12 @@ static lean_object* l_Lean_Parser_Tactic_introMatch_formatter___closed__1; static lean_object* l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Tactic_initFn____x40_Lean_Parser_Tactic___hyg_6____closed__9; static lean_object* l_Lean_Parser_Tactic_decide___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_decide___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_match___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l___regBuiltin_Lean_Parser_Tactic_nestedTactic_declRange___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Tactic_match_declRange___closed__4; static lean_object* l_Lean_Parser_Tactic_unknown_formatter___closed__3; @@ -169,6 +181,7 @@ lean_object* l_Lean_Parser_nodeInfo(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_introMatch___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_unknown___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_decide_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Tactic_match_formatter___closed__12; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__16; lean_object* l_Lean_Parser_nonReservedSymbolInfo(lean_object*, uint8_t); @@ -185,6 +198,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_declRange___closed_ lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Tactic_introMatch___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_declRange___closed__3; static lean_object* l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Tactic_decide___elambda__1___closed__2; @@ -200,8 +214,10 @@ static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__18; static lean_object* l_Lean_Parser_Tactic_decide___closed__5; static lean_object* l_Lean_Parser_Tactic_initFn____x40_Lean_Parser_Tactic___hyg_6____closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__1; lean_object* l_Lean_Parser_Term_hole_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_orelseInfo(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Tactic_match___elambda__1___closed__14; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__5; @@ -210,9 +226,12 @@ static lean_object* l_Lean_Parser_Tactic_introMatch_formatter___closed__3; static lean_object* l_Lean_Parser_Tactic_decide___closed__3; static lean_object* l_Lean_Parser_Tactic_match___elambda__1___closed__5; lean_object* l_Lean_addBuiltinDeclarationRanges(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1; static lean_object* l_Lean_Parser_Tactic_match_formatter___closed__11; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_initFn____x40_Lean_Parser_Tactic___hyg_6____closed__1; +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; uint32_t lean_string_utf8_get(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_declRange___closed__3; @@ -228,6 +247,7 @@ static lean_object* l_Lean_Parser_Tactic_decide___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_nativeDecide_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_introMatch___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_matchRhs___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_declRange___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_nestedTactic_declRange___closed__7; lean_object* l_Lean_Parser_Term_syntheticHole_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -242,15 +262,19 @@ lean_object* l_Lean_Parser_registerAlias(lean_object*, lean_object*, lean_object lean_object* l_Lean_Parser_Term_generalizingParam_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_unknown_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_unknown___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_matchRhs_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_unknown___elambda__1___closed__7; lean_object* l_Lean_PrettyPrinter_Formatter_withPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_nativeDecide___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_unknown_formatter___closed__5; static lean_object* l_Lean_Parser_Tactic_unknown_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Tactic_match___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_unknown_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3; lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_match___closed__4; static lean_object* l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__3; @@ -260,29 +284,35 @@ static lean_object* l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__5; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Tactic_match___closed__1; static lean_object* l_Lean_Parser_Tactic_initFn____x40_Lean_Parser_Tactic___hyg_6____closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_matchRhs_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_ident___elambda__1(lean_object*, lean_object*); uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_declRange___closed__7; static lean_object* l_Lean_Parser_Tactic_match___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_unknown_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Tactic_unknown_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Tactic_decide_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_introMatch___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_decide___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_unknown_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Tactic_match_declRange___closed__3; extern lean_object* l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; static lean_object* l_Lean_Parser_Tactic_decide_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_match_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_declRange(lean_object*); static lean_object* l_Lean_Parser_Tactic_initFn____x40_Lean_Parser_Tactic___hyg_6____closed__7; static lean_object* l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__10; static lean_object* l_Lean_Parser_Tactic_introMatch_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Tactic_decide_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_match___elambda__1___closed__4; static lean_object* l_Lean_Parser_Tactic_matchRhs___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Tactic_match___elambda__1___closed__13; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_decide(lean_object*); static lean_object* l_Lean_Parser_Tactic_decide___elambda__1___closed__4; @@ -309,6 +339,7 @@ static lean_object* l_Lean_Parser_Tactic_unknown___elambda__1___closed__3; static lean_object* l_Lean_Parser_Tactic_introMatch_formatter___closed__4; static lean_object* l_Lean_Parser_Tactic_match_formatter___closed__13; static lean_object* l_Lean_Parser_Tactic_decide_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_formatter(lean_object*); lean_object* l_Lean_Parser_ident_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_nestedTactic_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_sepBy1_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -348,11 +379,15 @@ static lean_object* l_Lean_Parser_Tactic_match_formatter___closed__16; static lean_object* l_Lean_Parser_Tactic_unknown___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Tactic_nestedTactic___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_match_parenthesizer___closed__17; static lean_object* l_Lean_Parser_Tactic_match___elambda__1___closed__10; static lean_object* l_Lean_Parser_Tactic_decide___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__1; lean_object* l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_unknown___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer(lean_object*); lean_object* l_Lean_Parser_Term_matchAlts_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_match___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__7; @@ -361,8 +396,10 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_matchAlts; lean_object* l_Lean_Parser_symbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_match___elambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_match_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_decide_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_decide___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_match___elambda__1___lambda__1___closed__1; lean_object* l_Lean_Parser_ident_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_unknown___elambda__1___lambda__1(lean_object*, lean_object*); @@ -1300,6 +1337,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_unknown___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_unknown_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_unknown___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_unknown_parenthesizer___closed__1() { _start: { @@ -1385,6 +1468,52 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_unknown___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_unknown_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_unknown___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_nestedTactic() { _start: { @@ -2640,6 +2769,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_match___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_match_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_match_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_match___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_matchRhs_parenthesizer___closed__1() { _start: { @@ -2906,6 +3065,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_match___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_match_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_match___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_introMatch___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -3478,6 +3667,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_introMatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_introMatch_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_introMatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1() { _start: { @@ -3545,6 +3764,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_introMatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_introMatch_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_introMatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_decide___elambda__1___closed__1() { _start: { @@ -4011,6 +4260,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_decide___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_decide_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_decide___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_decide_parenthesizer___closed__1() { _start: { @@ -4066,6 +4345,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_decide___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_decide_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_decide___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__1() { _start: { @@ -4541,6 +4850,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_nativeDecide_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1() { _start: { @@ -4596,6 +4935,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_nativeDecide_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} lean_object* initialize_Init(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Parser_Term(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -4726,6 +5095,17 @@ l_Lean_Parser_Tactic_unknown_formatter___closed__5 = _init_l_Lean_Parser_Tactic_ lean_mark_persistent(l_Lean_Parser_Tactic_unknown_formatter___closed__5); l_Lean_Parser_Tactic_unknown_formatter___closed__6 = _init_l_Lean_Parser_Tactic_unknown_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Tactic_unknown_formatter___closed__6); +l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__2); +l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__3); +l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_unknown_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Tactic_unknown_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_unknown_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_unknown_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_unknown_parenthesizer___closed__1); l_Lean_Parser_Tactic_unknown_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_unknown_parenthesizer___closed__2(); @@ -4738,6 +5118,17 @@ l_Lean_Parser_Tactic_unknown_parenthesizer___closed__5 = _init_l_Lean_Parser_Tac lean_mark_persistent(l_Lean_Parser_Tactic_unknown_parenthesizer___closed__5); l_Lean_Parser_Tactic_unknown_parenthesizer___closed__6 = _init_l_Lean_Parser_Tactic_unknown_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Tactic_unknown_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_Tactic_unknown_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_nestedTactic = _init_l_Lean_Parser_Tactic_nestedTactic(); lean_mark_persistent(l_Lean_Parser_Tactic_nestedTactic); l___regBuiltin_Lean_Parser_Tactic_nestedTactic___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_nestedTactic___closed__1(); @@ -4898,6 +5289,13 @@ l_Lean_Parser_Tactic_match_formatter___closed__17 = _init_l_Lean_Parser_Tactic_m lean_mark_persistent(l_Lean_Parser_Tactic_match_formatter___closed__17); l_Lean_Parser_Tactic_match_formatter___closed__18 = _init_l_Lean_Parser_Tactic_match_formatter___closed__18(); lean_mark_persistent(l_Lean_Parser_Tactic_match_formatter___closed__18); +l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_match_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_match_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_matchRhs_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_matchRhs_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_matchRhs_parenthesizer___closed__1); l_Lean_Parser_Tactic_matchRhs_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_matchRhs_parenthesizer___closed__2(); @@ -4942,6 +5340,13 @@ l_Lean_Parser_Tactic_match_parenthesizer___closed__17 = _init_l_Lean_Parser_Tact lean_mark_persistent(l_Lean_Parser_Tactic_match_parenthesizer___closed__17); l_Lean_Parser_Tactic_match_parenthesizer___closed__18 = _init_l_Lean_Parser_Tactic_match_parenthesizer___closed__18(); lean_mark_persistent(l_Lean_Parser_Tactic_match_parenthesizer___closed__18); +l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_match_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_introMatch___elambda__1___closed__1 = _init_l_Lean_Parser_Tactic_introMatch___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_introMatch___elambda__1___closed__1); l_Lean_Parser_Tactic_introMatch___elambda__1___closed__2 = _init_l_Lean_Parser_Tactic_introMatch___elambda__1___closed__2(); @@ -5002,6 +5407,13 @@ l_Lean_Parser_Tactic_introMatch_formatter___closed__3 = _init_l_Lean_Parser_Tact lean_mark_persistent(l_Lean_Parser_Tactic_introMatch_formatter___closed__3); l_Lean_Parser_Tactic_introMatch_formatter___closed__4 = _init_l_Lean_Parser_Tactic_introMatch_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Tactic_introMatch_formatter___closed__4); +l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_introMatch_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1); l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__2(); @@ -5010,6 +5422,13 @@ l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__3 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__3); l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__4 = _init_l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Tactic_introMatch_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_introMatch_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_decide___elambda__1___closed__1 = _init_l_Lean_Parser_Tactic_decide___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_decide___elambda__1___closed__1); l_Lean_Parser_Tactic_decide___elambda__1___closed__2 = _init_l_Lean_Parser_Tactic_decide___elambda__1___closed__2(); @@ -5072,12 +5491,26 @@ l_Lean_Parser_Tactic_decide_formatter___closed__2 = _init_l_Lean_Parser_Tactic_d lean_mark_persistent(l_Lean_Parser_Tactic_decide_formatter___closed__2); l_Lean_Parser_Tactic_decide_formatter___closed__3 = _init_l_Lean_Parser_Tactic_decide_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_decide_formatter___closed__3); +l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_decide_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_decide_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_decide_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_decide_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_decide_parenthesizer___closed__1); l_Lean_Parser_Tactic_decide_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_decide_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Tactic_decide_parenthesizer___closed__2); l_Lean_Parser_Tactic_decide_parenthesizer___closed__3 = _init_l_Lean_Parser_Tactic_decide_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_decide_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_decide_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__1 = _init_l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__1); l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__2 = _init_l_Lean_Parser_Tactic_nativeDecide___elambda__1___closed__2(); @@ -5142,12 +5575,26 @@ l_Lean_Parser_Tactic_nativeDecide_formatter___closed__2 = _init_l_Lean_Parser_Ta lean_mark_persistent(l_Lean_Parser_Tactic_nativeDecide_formatter___closed__2); l_Lean_Parser_Tactic_nativeDecide_formatter___closed__3 = _init_l_Lean_Parser_Tactic_nativeDecide_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_nativeDecide_formatter___closed__3); +l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_nativeDecide_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1); l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2); l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__3 = _init_l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_nativeDecide_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Parser/Term.c b/stage0/stdlib/Lean/Parser/Term.c index 3605e7915be9..b002c8d13b15 100644 --- a/stage0/stdlib/Lean/Parser/Term.c +++ b/stage0/stdlib/Lean/Parser/Term.c @@ -18,6 +18,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_have_declRange___closed__6; static lean_object* l_Lean_Parser_Term_subst___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_binrel__no__prop_formatter___closed__2; static lean_object* l_Lean_Parser_Term_attr_quot___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__2; static lean_object* l_Lean_Parser_Term_dbgTrace_formatter___closed__7; static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__6; @@ -42,6 +43,7 @@ static lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_binop__lazy___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_binop___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_explicit_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1; static lean_object* l_Lean_Parser_Term_sufficesDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_tupleTail_parenthesizer___closed__2; @@ -53,17 +55,20 @@ static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_let__tmp___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_declRange___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_motive___closed__11; static lean_object* l_Lean_Parser_Term_binderTactic_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_basicFun___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveIdLhs_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchAlts_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_ident_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_declRange(lean_object*); static lean_object* l_Lean_Parser_Level_quot___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dynamicQuot; LEAN_EXPORT lean_object* l_Lean_Parser_Term_attr_quot; static lean_object* l_Lean_Parser_Term_proj___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer(lean_object*); lean_object* l_Lean_Parser_finishCommentBlock(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funImplicitBinder_formatter___closed__5; static lean_object* l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__4; @@ -72,6 +77,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_declRange___clo static lean_object* l_Lean_Parser_Term_letrec_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_structInst_declRange___closed__2; static lean_object* l_Lean_Parser_Term_dotIdent_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_paren_formatter___closed__5; static lean_object* l_Lean_Parser_Term_instBinder_formatter___closed__5; static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__9; @@ -83,16 +89,20 @@ static lean_object* l_Lean_Parser_Term_dbgTrace___closed__5; lean_object* l_Lean_Parser_nonReservedSymbol_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderType_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__10; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__47; static lean_object* l_Lean_Parser_Term_letMVar_parenthesizer___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_macroLastArg_formatter___closed__1; static lean_object* l_Lean_Parser_Term_have_formatter___closed__2; static lean_object* l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_attrKind_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attrKind_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_explicit___closed__9; static lean_object* l_Lean_Parser_Term_local___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__43; @@ -128,14 +138,15 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_pipeProj; static lean_object* l_Lean_Parser_Term_inaccessible___closed__8; static lean_object* l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_nomatch_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__21; static lean_object* l_Lean_Parser_Term_letPatDecl___closed__9; -static lean_object* l_Lean_Parser_Term_macroLastArg_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_trueVal_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_explicitUniv___elambda__1___closed__10; -static lean_object* l_Lean_Parser_Term_have_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doubleQuotedName_formatter___closed__3___boxed__const__1; static lean_object* l_Lean_Parser_Term_byTactic_formatter___closed__4; @@ -149,20 +160,24 @@ static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__32; static lean_object* l_Lean_Parser_Term_let__tmp_formatter___closed__4; static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__12; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__1; static lean_object* l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_structInstArrayRef___closed__9; static lean_object* l_Lean_Parser_Term_local___closed__2; static lean_object* l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_proj_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_letRecDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_letrec_formatter___closed__9; static lean_object* l_Lean_Parser_Term_namedPattern___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicit_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_noindex___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__4; lean_object* l_Lean_Parser_tokenAntiquotFn(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_cdot___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Term_letMVar_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_char___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forInMacro_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_suffices___closed__1; static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__6; @@ -172,13 +187,16 @@ static lean_object* l_Lean_Parser_Term_fromTerm___closed__3; static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Level_quot___closed__1; static lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_let__fun___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_namedArgument___elambda__1___closed__8; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__47; static lean_object* l_Lean_Parser_Term_binop__lazy___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_formatter___closed__1; static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_arrow_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_letRecDecl___closed__7; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__20; @@ -204,6 +222,8 @@ static lean_object* l_Lean_Parser_Term_num_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_typeOf___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_showRhs; static lean_object* l_Lean_Parser_Term_matchDiscr___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sorry_formatter(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__34; static lean_object* l_Lean_Parser_Term_anonymousCtor_formatter___closed__2; static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__8; static lean_object* l_Lean_Parser_Command_docComment___closed__3; @@ -218,13 +238,16 @@ static lean_object* l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__4; lean_object* l_Lean_Parser_ParserState_mkError(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_docComment___elambda__1___lambda__2(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_declRange___closed__4; static lean_object* l_Lean_Parser_Term_letRecDecl_formatter___closed__3; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binrel; static lean_object* l_Lean_Parser_Term_explicit_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_whereDecls_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_declRange___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_seq1_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_sort___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_binderTactic___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_docComment___elambda__1___lambda__2___boxed(lean_object*, lean_object*); @@ -239,17 +262,20 @@ static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___clo static lean_object* l_Lean_Parser_Term_pipeProj___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_suffices(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_declRange___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_scoped_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_borrowed___closed__4; static lean_object* l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_matchDiscr___closed__2; static lean_object* l_Lean_Parser_Term_arrow___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__15; static lean_object* l_Lean_Parser_darrow___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__25; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_binop___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_letRecDecls___closed__6; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___closed__6; @@ -259,7 +285,9 @@ static lean_object* l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__13 static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveEqnsDecl___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_argument___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_ident_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_letRecDecls___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_binrel_declRange___closed__4; @@ -287,7 +315,9 @@ static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_sorry___closed__6; static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letDecl_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_proj; +static lean_object* l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__23; LEAN_EXPORT lean_object* l_Lean_Parser_Term_funImplicitBinder; static lean_object* l_Lean_Parser_Tactic_quotSeq___closed__6; @@ -295,31 +325,35 @@ static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket_parenthesizer__ static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__5; static lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_funImplicitBinder_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer(lean_object*); lean_object* l_Lean_Parser_ppSpace_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letIdDecl___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_let__fun_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__1; static lean_object* l_Lean_Parser_Term_instBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_noImplicitLambda_formatter___closed__1; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket___closed__2; static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__1; static lean_object* l_Lean_Parser_Term_byTactic___closed__4; static lean_object* l_Lean_Parser_Term_structInstField___elambda__1___closed__7; lean_object* l_Lean_Parser_ppGroup_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_num_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_attrKind_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_show; static lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_proj_declRange___closed__5; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__17; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__34; static lean_object* l_Lean_Parser_Level_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_matchDiscr___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveIdLhs; static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__11; lean_object* l_Lean_Parser_parserOfStack___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_noImplicitLambda; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__1; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__7; @@ -339,15 +373,18 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_declRange LEAN_EXPORT lean_object* l_Lean_Parser_Term_fun_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_letDecl___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_explicitUniv_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_match_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Term_assert_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_instBinder; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___closed__4; static lean_object* l_Lean_Parser_Term_fun___closed__7; static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__18; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__2; static lean_object* l_Lean_Parser_Term_sufficesDecl_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_declRange___closed__4; static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__15; @@ -356,6 +393,7 @@ lean_object* l_Lean_PrettyPrinter_Formatter_checkLinebreakBefore_formatter___box static lean_object* l_Lean_Parser_Term_argument___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_ident_declRange___closed__6; static lean_object* l_Lean_Parser_Term_arrow___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__22; static lean_object* l_Lean_Parser_Term_inaccessible___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_semicolonOrLinebreak_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -365,6 +403,7 @@ static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27(lean_object*); static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__17; static lean_object* l_Lean_Parser_Term_funBinder_quot_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Command_docComment___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAlts(lean_object*); static lean_object* l_Lean_Parser_Term_let_formatter___closed__6; @@ -389,23 +428,25 @@ static lean_object* l_Lean_Parser_Term_letIdLhs___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_let__tmp___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_letRecDecl_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dotIdent___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_letDecl_formatter___closed__9; static lean_object* l_Lean_Parser_Term_explicit___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_let_formatter___closed__1; lean_object* l_Lean_Parser_many(lean_object*); static lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__19; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_byTactic_x27___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_bracketedBinder(uint8_t); static lean_object* l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_prop_declRange___closed__1; static lean_object* l_Lean_Parser_Term_structInst___closed__6; static lean_object* l_Lean_Parser_Level_quot_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_ensureExpectedType___closed__1; -static lean_object* l_Lean_Parser_Term_structInstField_formatter___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_hole_declRange___closed__1; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_basicFun_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_explicitUniv_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sorry(lean_object*); static lean_object* l_Lean_Parser_Term_letEqnsDecl___closed__2; @@ -415,7 +456,9 @@ static lean_object* l_Lean_Parser_Term_fun_formatter___closed__3; static lean_object* l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_hole___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__2; static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_declRange___closed__7; static lean_object* l_Lean_Parser_Term_quotedName_formatter___closed__3; @@ -427,23 +470,29 @@ static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__1 static lean_object* l_Lean_Parser_Term_binop__lazy___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_unreachable___closed__6; static lean_object* l_Lean_Parser_Term_letRecDecl___elambda__1___closed__9; -static lean_object* l_Lean_Parser_Term_let_formatter___closed__7; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__35; LEAN_EXPORT lean_object* l_Lean_Parser_Term_argument_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_tacticParser_formatter___boxed(lean_object*); static lean_object* l_Lean_Parser_Term_letDecl_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeSpec_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Level_quot_declRange___closed__1; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forall___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_optType_parenthesizer___closed__1; lean_object* l_Lean_Parser_setLhsPrecFn(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_completion_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letMVar_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__1; lean_object* l_Lean_PrettyPrinter_Parenthesizer_lookahead_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_argument___closed__7; static lean_object* l_Lean_Parser_Term_inaccessible___closed__9; static lean_object* l_Lean_Parser_Term_char___closed__3; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_match___closed__7; static lean_object* l_Lean_Parser_Term_tupleTail_parenthesizer___closed__3; @@ -456,7 +505,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_ellipsis_formatter(lean_object*, lea static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_num(lean_object*); static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__5; -static lean_object* l_Lean_Parser_Term_letRecDecl_formatter___closed__7; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Term_proj_declRange___closed__3; lean_object* l_Lean_PrettyPrinter_Parenthesizer_evalInsideQuot_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -464,8 +512,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_match_formatter(lean_object*, lean_o static lean_object* l_Lean_Parser_Tactic_seq1___elambda__1___closed__4; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkStackTop_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_pipeProj_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_trueVal_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__21; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_letEqnsDecl___closed__1; @@ -476,12 +527,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1(lean_object static lean_object* l_Lean_Parser_Term_instBinder___closed__5; static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_leading__parser_formatter___closed__6; -static lean_object* l_Lean_Parser_Term_parenSpecial_formatter___closed__2; static lean_object* l_Lean_Parser_Term_subst___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_completion_declRange___closed__4; static lean_object* l_Lean_Parser_Term_attrInstance_formatter___closed__3; static lean_object* l_Lean_Parser_Term_forInMacro_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__2; static lean_object* l_Lean_Parser_Term_inaccessible___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_attributes_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_namedArgument___closed__5; @@ -492,6 +543,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_declRange__ LEAN_EXPORT lean_object* l_Lean_Parser_Term_pipeProj___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_forall_declRange___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_typeOf___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_declRange___closed__7; static lean_object* l_Lean_Parser_Term_show___elambda__1___closed__8; @@ -508,6 +560,7 @@ static lean_object* l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_declRange___closed__7; static lean_object* l_Lean_Parser_Term_letRecDecl___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstField_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_proj_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_scientific___closed__2; static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__12; @@ -531,9 +584,11 @@ static lean_object* l_Lean_Parser_Term_trailing__parser___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfTypeMVar_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_semicolonOrLinebreak_formatter___closed__1; static lean_object* l_Lean_Parser_Term_typeOf___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_namedArgument___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicitUniv; +static lean_object* l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__1; static lean_object* l_Lean_Parser_Term_ident_parenthesizer___closed__1; lean_object* l_Lean_Parser_symbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___closed__7; @@ -543,8 +598,8 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_prop_declRange___closed__2; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__21; static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_declRange___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_inaccessible___closed__4; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__35; static lean_object* l_Lean_Parser_Term_match_formatter___closed__3; static lean_object* l_Lean_Parser_Term_subst_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_nomatch_formatter___closed__3; @@ -571,15 +626,18 @@ static lean_object* l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_prop_formatter___closed__3; static lean_object* l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__24; +static lean_object* l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__1; lean_object* l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_quot_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_binop_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Level_quot_formatter___closed__4; static lean_object* l_Lean_Parser_Term_byTactic___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchDiscr_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_match_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binderType___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__10; @@ -590,6 +648,7 @@ static lean_object* l_Lean_Parser_Term_suffices_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__7; static lean_object* l_Lean_Parser_Term_cdot___closed__8; static lean_object* l_Lean_Parser_Term_sort_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAlts___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sorry_declRange(lean_object*); @@ -597,17 +656,21 @@ static lean_object* l_Lean_Parser_Term_letDecl_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_structInst_declRange___closed__4; lean_object* l_Lean_Parser_sepBy_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_ellipsis___closed__5; static lean_object* l_Lean_Parser_Term_byTactic_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_forall_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderTactic_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_atomic_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binop_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_panic_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_letRecDecl___elambda__1___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fun_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_namedPattern___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_subst___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_funImplicitBinder___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_panic___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_prop; @@ -622,14 +685,16 @@ static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed_ static lean_object* l_Lean_Parser_Term_ellipsis___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_declRange___closed__7; static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_letrec___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__2; -static lean_object* l_Lean_Parser_Term_letDecl_formatter___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicit_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_declRange___closed__1; static lean_object* l_Lean_Parser_Term_attributes_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_hole___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_whereDecls_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_binderTactic___elambda__1___closed__3; @@ -637,11 +702,13 @@ static lean_object* l_Lean_Parser_Term_dotIdent___elambda__1___closed__6; lean_object* l_Lean_Parser_group_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_attrInstance___closed__1; static lean_object* l_Lean_Parser_Term_let__tmp___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_declRange___closed__3; static lean_object* l_Lean_Parser_Term_show_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_declRange___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_declRange___closed__5; static lean_object* l_Lean_Parser_Term_funBinder_quot___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_explicit___elambda__1___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Term_hole_declRange___closed__6; static lean_object* l_Lean_Parser_Level_quot___closed__4; @@ -649,17 +716,20 @@ static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_letIdLhs___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1; extern lean_object* l_Lean_Parser_minPrec; static lean_object* l_Lean_Parser_Term_letrec_formatter___closed__3; static lean_object* l_Lean_Parser_Term_subst_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__17; +static lean_object* l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_declRange___closed__3; static lean_object* l_Lean_Parser_Term_letPatDecl___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_completion_declRange___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar(lean_object*); static lean_object* l_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_fun_declRange___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_subst_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_letPatDecl; LEAN_EXPORT lean_object* l_Lean_Parser_Term_assert; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__delayed_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -674,6 +744,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeAscription___elambda__1(lean_obj static lean_object* l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__6; static lean_object* l_Lean_Parser_Term_show_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_declRange___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__1; static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__21; static lean_object* l_Lean_Parser_Term_implicitBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__7; @@ -681,6 +752,7 @@ static lean_object* l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicitUniv_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__1; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___closed__4; static lean_object* l_Lean_Parser_Term_explicitBinder___elambda__1___closed__3; static lean_object* l_Lean_Parser_semicolonOrLinebreak_formatter___closed__2; @@ -701,13 +773,17 @@ static lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer___closed__7 static lean_object* l_Lean_Parser_Term_let__tmp___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_declRange___closed__5; static lean_object* l_Lean_Parser_Term_haveDecl___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_paren_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_subst___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_borrowed___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fun_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_completion___closed__7; static lean_object* l_Lean_Parser_Term_fromTerm_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_haveDecl_formatter___closed__4; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__8; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__19; static lean_object* l_Lean_Parser_Term_letrec___closed__7; static lean_object* l_Lean_Parser_Term_basicFun_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_unreachable___elambda__1___closed__2; @@ -715,58 +791,62 @@ static lean_object* l_Lean_Parser_Term_forall_formatter___closed__5; static lean_object* l_Lean_Parser_Term_noindex___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_forInMacro_x27___closed__7; static lean_object* l_Lean_Parser_Level_quot___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__1; static lean_object* l_Lean_Parser_Term_forInMacro_x27_formatter___closed__3; static lean_object* l_Lean_Parser_Term_dotIdent_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed; static lean_object* l_Lean_Parser_Term_suffices_formatter___closed__7; static lean_object* l_Lean_Parser_Term_binderTactic___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_explicitUniv___elambda__1___closed__7; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__51; static lean_object* l_Lean_Parser_Term_show___elambda__1___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_cdot___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_type_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_pipeProj___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_implicitBinder_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_declRange___closed__7; static lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__12; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_formatter___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__19; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_paren_declRange(lean_object*); extern lean_object* l_Lean_Parser_scientificLit; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__14; LEAN_EXPORT lean_object* l_Lean_Parser_Term_completion___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__2; static lean_object* l_Lean_Parser_Term_type___closed__6; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_instBinder___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__27; +static lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_haveIdLhs___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_letIdBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_byTactic; static lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_declRange___closed__2; static lean_object* l_Lean_Parser_Term_falseVal___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_docComment_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_have___closed__3; static lean_object* l_Lean_Parser_Term_dbgTrace_formatter___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_declRange(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedArgument_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_binderDefault___closed__6; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__14; -static lean_object* l_Lean_Parser_Term_showRhs_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderTactic___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_declRange___closed__7; static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_declRange___closed__2; @@ -774,7 +854,6 @@ static lean_object* l_Lean_Parser_Term_cdot_parenthesizer___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_type(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__8; -static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__7; static lean_object* l_Lean_Parser_Term_proj___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_sort___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__3; @@ -783,10 +862,12 @@ static lean_object* l_Lean_Parser_Term_unreachable_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_declRange___closed__4; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__2; static lean_object* l_Lean_Parser_Term_dynamicQuot___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_declRange___closed__7; static lean_object* l_Lean_Parser_Term_attributes___closed__4; static lean_object* l_Lean_Parser_Term_namedPattern___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_orelse_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__9; static lean_object* l_Lean_Parser_Term_let__fun___elambda__1___closed__4; @@ -796,14 +877,15 @@ static lean_object* l_Lean_Parser_Term_namedArgument_formatter___closed__2; static lean_object* l_Lean_Parser_Term_assert___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_fun_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicitBinder_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_quotedName___closed__3; static lean_object* l_Lean_Parser_Term_pipeProj___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_subst___closed__6; -static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__19; extern lean_object* l_Lean_Parser_ident; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__40; static lean_object* l_Lean_Parser_Term_explicitUniv_formatter___closed__7; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__2; @@ -817,6 +899,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer( static lean_object* l_Lean_Parser_Term_optIdent___closed__1; static lean_object* l_Lean_Parser_semicolonOrLinebreak___closed__2; static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_letDecl_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_ensureTypeOf_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___closed__6; @@ -825,22 +908,25 @@ static lean_object* l_Lean_Parser_Term_forall___closed__3; static lean_object* l_Lean_Parser_Term_trailing__parser___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_app_declRange___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_scientific; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__1; lean_object* l_Lean_Parser_withAntiquotFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_unreachable___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_assert_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_pipeProj_formatter___closed__5; static lean_object* l_Lean_Parser_Term_letMVar___closed__2; static lean_object* l_Lean_Parser_Term_basicFun_formatter___closed__10; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicitUniv_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__27; static lean_object* l_Lean_Parser_Term_let__fun___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_bracketedBinder_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_id___rarg___boxed(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInstField___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_attrInstance___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_bracketedBinder_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___closed__7; -static lean_object* l_Lean_Parser_Term_showRhs_parenthesizer___closed__1; lean_object* l_Lean_Parser_checkLinebreakBefore___elambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_syntheticHole___elambda__1___closed__12; static lean_object* l_Lean_Parser_Level_quot_formatter___closed__2; @@ -857,6 +943,8 @@ static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_quotedName___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_strictImplicitRightBracket_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_trueVal___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_attributes___closed__9; static lean_object* l_Lean_Parser_Term_bracketedBinder_formatter___closed__2; @@ -864,8 +952,11 @@ static lean_object* l_Lean_Parser_Term_type_formatter___closed__6; static lean_object* l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_noImplicitLambda_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter(lean_object*); lean_object* l_Lean_Parser_ParserState_mkNode(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_generalizingParam_formatter___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__2; static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_ident___closed__1; @@ -876,23 +967,30 @@ static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_suffices___closed__9; static lean_object* l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_let__fun___elambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_inaccessible___elambda__1___closed__10; static lean_object* l_Lean_Parser_Command_commentBody___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prop_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_darrow; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_matchDiscr___closed__6; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__22; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__40; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_arrow___closed__2; static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__9; static lean_object* l_Lean_Parser_Term_noindex_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_completion_declRange___closed__3; static lean_object* l_Lean_Parser_Term_paren_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Command_docComment_formatter___closed__8; static lean_object* l_Lean_Parser_Term_dynamicQuot_formatter___closed__7; static lean_object* l_Lean_Parser_Level_quot_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__1; static lean_object* l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_let__tmp___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_sorry_formatter___closed__3; @@ -911,9 +1009,12 @@ static lean_object* l_Lean_Parser_Term_binop___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_binrel_declRange___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_optExprPrecedence___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_suffices___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noindex_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__1; static lean_object* l_Lean_Parser_Term_namedArgument___elambda__1___closed__1; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_Term_paren_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -923,6 +1024,7 @@ static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed_ static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_ellipsis___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__44; static lean_object* l_Lean_Parser_Term_inaccessible_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeOf; static lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__9; @@ -930,6 +1032,7 @@ static lean_object* l_Lean_Parser_Term_letPatDecl___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_declRange___closed__4; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket_parenthesizer___closed__3; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withoutPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_motive___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_attributes_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchDiscr___elambda__1(lean_object*, lean_object*); @@ -941,6 +1044,7 @@ static lean_object* l_Lean_Parser_Term_trailing__parser_formatter___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_binop___closed__2; static lean_object* l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__2; lean_object* l_Lean_Parser_pushNone___elambda__1___boxed(lean_object*); lean_object* l_Lean_Parser_notFollowedByFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__12; @@ -957,6 +1061,7 @@ static lean_object* l_Lean_Parser_Term_letRecDecl___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_assert___elambda__1___closed__7; static lean_object* l_Lean_Parser_Tactic_quotSeq_formatter___closed__4; static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_let__fun___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_local___closed__6; static lean_object* l_Lean_Parser_Term_attr_quot___closed__6; @@ -980,8 +1085,10 @@ static lean_object* l_Lean_Parser_Term_haveDecl___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_let__delayed_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_ensureTypeOf___closed__7; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_attributes_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_letRecDecls___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_optIdent_formatter___closed__1; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__19; @@ -991,12 +1098,14 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_ensureTypeOf_formatter(lean_object*, static lean_object* l_Lean_Parser_Term_scoped___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_binrel__no__prop_formatter___closed__4; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__36; +static lean_object* l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_quot_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_declRange___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prop_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_attrInstance___elambda__1___closed__10; lean_object* l_Lean_Parser_ParserState_mkTrailingNode(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_letPatDecl___closed__8; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__26; static lean_object* l___regBuiltin_Lean_Parser_Term_sort_declRange___closed__3; @@ -1007,6 +1116,8 @@ static lean_object* l_Lean_Parser_Term_letRecDecls_formatter___closed__2; static lean_object* l_Lean_Parser_Term_prop___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_fun_formatter___closed__6; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doubleQuotedName_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_declRange___closed__4; @@ -1017,6 +1128,7 @@ static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___closed__4; static lean_object* l_Lean_Parser_Term_let___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_suffices_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_forall_declRange___closed__3; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_assert_parenthesizer___closed__3; @@ -1026,13 +1138,17 @@ static lean_object* l_Lean_Parser_Term_binrel___closed__10; static lean_object* l_Lean_Parser_Term_trailing__parser_formatter___closed__2; static lean_object* l_Lean_Parser_Term_whereDecls_formatter___closed__6; static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__36; static lean_object* l_Lean_Parser_Term_doubleQuotedName___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_scientific_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_quotedName___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_semicolonOrLinebreak_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__3; lean_object* l_Lean_Parser_addBuiltinParser(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_prop___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_letRecDecls_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_type_declRange___closed__1; @@ -1047,7 +1163,7 @@ lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Parser_Term_binrel__no__prop___closed__3; static lean_object* l_Lean_Parser_Term_letRecDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__44; +static lean_object* l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_scientific_declRange___closed__7; static lean_object* l_Lean_Parser_Term_haveIdLhs___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstFieldAbbrev; @@ -1080,20 +1196,22 @@ static lean_object* l_Lean_Parser_Term_dbgTrace___closed__6; static lean_object* l_Lean_Parser_Term_forInMacro___elambda__1___closed__11; lean_object* l_Lean_PrettyPrinter_Formatter_checkWsBefore_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binop___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicit___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_sorry___closed__2; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket_formatter___closed__1; static lean_object* l_Lean_Parser_Term_nomatch___closed__7; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__1; static lean_object* l_Lean_Parser_Term_byTactic_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_completion_declRange___closed__5; static lean_object* l_Lean_Parser_Term_forInMacro___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__17; static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_attr_quot_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_sorry_formatter___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__25; static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_declRange___closed__2; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___closed__1; static lean_object* l_Lean_Parser_Term_hole_formatter___closed__2; @@ -1105,12 +1223,14 @@ static lean_object* l_Lean_Parser_Term_namedArgument___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_binop___closed__7; static lean_object* l_Lean_Parser_Term_type_formatter___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_completion_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_let__delayed___closed__9; lean_object* l_Lean_Parser_mkAtomicInfo(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_declRange___closed__7; static lean_object* l_Lean_Parser_Term_whereDecls_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInst_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_declRange___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_scoped___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_show___closed__6; static lean_object* l_Lean_Parser_Term_noImplicitLambda___closed__7; @@ -1118,10 +1238,12 @@ static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_typeAscription_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_attrInstance_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_scientific_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket_formatter___closed__2; static lean_object* l_Lean_Parser_Term_hole___closed__5; static lean_object* l_Lean_Parser_Term_optEllipsis___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fun_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_optType___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_declRange___closed__1; @@ -1130,6 +1252,7 @@ static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___clo LEAN_EXPORT lean_object* l_Lean_Parser_Term_funBinder; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_explicitUniv___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__2; lean_object* l_Lean_Parser_unicodeSymbol_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_attr_quot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1138,9 +1261,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1(lean_o LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quotedName(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_app_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_haveIdLhs___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__2; static lean_object* l_Lean_Parser_Term_instBinder_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_have_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___closed__10; @@ -1155,6 +1281,7 @@ static lean_object* l_Lean_Parser_Term_assert_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeq___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_suffices___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_scoped_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; static lean_object* l_Lean_Parser_Term_parenSpecial___closed__1; static lean_object* l_Lean_Parser_Term_argument___closed__5; static lean_object* l_Lean_Parser_Term_haveDecl___elambda__1___closed__3; @@ -1169,6 +1296,7 @@ static lean_object* l_Lean_Parser_Term_structInstArrayRef_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_pipeCompletion_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_type_declRange___closed__4; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_funBinder_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal___closed__9; static lean_object* l_Lean_Parser_Term_namedPattern___elambda__1___closed__3; @@ -1179,10 +1307,10 @@ static lean_object* l_Lean_Parser_Term_show___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_generalizingParam_formatter___closed__1; static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_tupleTail___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__2; static lean_object* l_Lean_Parser_Term_borrowed_formatter___closed__3; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_strictImplicitBinder_formatter___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__25; static lean_object* l_Lean_Parser_Term_leading__parser___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forall_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1196,9 +1324,11 @@ static lean_object* l_Lean_Parser_Term_namedPattern_formatter___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_depArrow___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_letMVar_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letEqnsDecl___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__2; static lean_object* l_Lean_Parser_Term_attr_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_let__delayed___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_declRange___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_basicFun___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_assert_declRange___closed__4; static lean_object* l_Lean_Parser_Term_depArrow_formatter___closed__4; @@ -1206,15 +1336,20 @@ static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_noImplicitLambda_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_quotedName___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_panic_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_declRange___closed__3; static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__1; lean_object* l_Lean_Parser_checkPrecFn___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_app_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binop_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_let__tmp_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__9; static lean_object* l_Lean_Parser_Term_sorry___closed__1; static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_paren_declRange___closed__7; static lean_object* l_Lean_Parser_Level_quot_formatter___closed__3; static lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__2; @@ -1224,6 +1359,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveIdDecl_formatter(lean_object*, l static lean_object* l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_declRange___closed__6; static lean_object* l_Lean_Parser_Term_falseVal___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_ident_declRange___closed__4; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__5; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__3; @@ -1233,11 +1369,14 @@ static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_attrKind___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveDecl_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_letRecDecls___closed__5; static lean_object* l_Lean_Parser_Term_noindex___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_basicFun_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_dotIdent_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__11; static lean_object* l_Lean_Parser_Term_dotIdent___elambda__1___closed__2; @@ -1256,7 +1395,9 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_sufficesDecl___elambda__1(lean_objec static lean_object* l___regBuiltin_Lean_Parser_Term_type_declRange___closed__2; static lean_object* l_Lean_Parser_Term_depArrow_formatter___closed__2; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_attr_quot___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_arrow_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_instBinder___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_declRange(lean_object*); static lean_object* l_Lean_Parser_Command_docComment___closed__2; @@ -1275,6 +1416,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_panic_declRange(lean_ob static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_declRange___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchDiscr_quot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_namedPattern_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1289,11 +1431,14 @@ lean_object* l_Lean_Parser_leadingNode_formatter___boxed(lean_object*, lean_obje static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_borrowed_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_declRange___closed__5; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doubleQuotedName_formatter___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderType(uint8_t); lean_object* l_Lean_PrettyPrinter_Parenthesizer_rawCh_parenthesizer___boxed(lean_object*, lean_object*); @@ -1306,6 +1451,7 @@ static lean_object* l_Lean_Parser_Term_binrel___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_declRange___closed__3; static lean_object* l_Lean_Parser_Term_optIdent___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstLVal_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__1; static lean_object* l_Lean_Parser_Term_ellipsis___closed__4; static lean_object* l_Lean_Parser_Term_assert_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_let__tmp___closed__4; @@ -1323,6 +1469,7 @@ static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__28; LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeAscription_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funBinder_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_prop_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_namedArgument_formatter___closed__1; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_paren_parenthesizer___closed__11; @@ -1335,6 +1482,7 @@ lean_object* l_Lean_Parser_checkColGeFn___boxed(lean_object*, lean_object*, lean static lean_object* l_Lean_Parser_Term_haveIdDecl___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_declRange___closed__1; +lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeq___closed__7; static lean_object* l_Lean_Parser_Term_forInMacro_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__12; @@ -1369,16 +1517,20 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeOf_formatter(lean_object*, lean_ static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_Term_str_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_unreachable___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___closed__5; -static lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter___closed__4; static lean_object* l_Lean_Parser_Term_noindex___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_ensureExpectedType___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_declRange___closed__7; lean_object* l_Lean_Parser_rawIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_have_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_declRange(lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__23; static lean_object* l_Lean_Parser_Term_suffices___elambda__1___closed__7; @@ -1392,10 +1544,12 @@ static lean_object* l_Lean_Parser_Term_generalizingParam_formatter___closed__6; static lean_object* l_Lean_Parser_Term_let__delayed___elambda__1___closed__10; lean_object* l_Lean_Parser_optional_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funBinder_quot___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_local___closed__1; static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_paren___closed__7; static lean_object* l_Lean_Parser_Term_unreachable___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_app_formatter___closed__1; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_namedArgument___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_binrel_formatter___closed__6; @@ -1403,12 +1557,14 @@ static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__7; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkPrec_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchDiscr_quot___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_app_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_sort___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_stateRefT___closed__7; static lean_object* l_Lean_Parser_Term_basicFun_formatter___closed__7; static lean_object* l_Lean_Parser_Term_letrec___closed__11; static lean_object* l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forInMacro_x27_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Term_optEllipsis___closed__2; @@ -1416,9 +1572,13 @@ static lean_object* l_Lean_Parser_Term_letDecl_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderTactic_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_stateRefT_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__15; +static lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Term_explicit___closed__4; static lean_object* l_Lean_Parser_Term_dbgTrace___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_cdot___closed__1; static lean_object* l_Lean_Parser_Term_namedPattern___closed__7; static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__4; @@ -1427,10 +1587,10 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_declRange___c static lean_object* l_Lean_Parser_Term_assert_formatter___closed__1; static lean_object* l_Lean_Parser_Term_syntheticHole___closed__1; static lean_object* l_Lean_Parser_Term_paren_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_num___closed__1; static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__13; -static lean_object* l_Lean_Parser_Term_leading__parser_formatter___closed__9; static lean_object* l_Lean_Parser_Term_noindex___closed__1; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___closed__2; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_63____closed__4; @@ -1446,7 +1606,9 @@ static lean_object* l_Lean_Parser_Term_funBinder_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_typeOf_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Command_docComment_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_atomic_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_let__fun_formatter___closed__5; static lean_object* l_Lean_Parser_Term_letIdLhs_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_let__fun___closed__3; @@ -1460,6 +1622,7 @@ static lean_object* l_Lean_Parser_Term_attr_quot_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_binderTactic___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_whereDecls_formatter___closed__2; static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_type_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_noindex___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_declRange___closed__1; static lean_object* l_Lean_Parser_Term_matchDiscr___elambda__1___closed__2; @@ -1475,15 +1638,16 @@ static lean_object* l_Lean_Parser_Term_sorry___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__17; static lean_object* l_Lean_Parser_Term_suffices___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_matchDiscr___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__1; static lean_object* l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_let___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_optEllipsis_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_completion(lean_object*); static lean_object* l_Lean_Parser_Term_cdot___elambda__1___closed__13; -static lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer___closed__9; lean_object* l_Lean_Parser_ppAllowUngrouped_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_binrel__no__prop; +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_declRange___closed__1; static lean_object* l_Lean_Parser_Term_attr_quot___elambda__1___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Term_suffices_declRange___closed__7; @@ -1493,6 +1657,7 @@ static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__19; LEAN_EXPORT lean_object* l_Lean_Parser_Command_docComment___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_argument_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__1; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_ensureTypeOf___closed__4; static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__7; @@ -1507,6 +1672,7 @@ static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_borrowed_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_sorry___closed__4; static lean_object* l_Lean_Parser_Term_dotIdent___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_implicitBinder_formatter(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__7; @@ -1525,7 +1691,9 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_declRange__ static lean_object* l_Lean_Parser_Term_explicitBinder_formatter___closed__4; static lean_object* l_Lean_Parser_Term_paren___closed__5; static lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__delayed___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attributes_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_prop_declRange___closed__3; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_sort___elambda__1___closed__3; @@ -1542,6 +1710,7 @@ static lean_object* l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed static lean_object* l___regBuiltin_Lean_Parser_Term_fun_declRange___closed__2; static lean_object* l_Lean_Parser_Term_sorry___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAlts_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_depArrow___closed__8; @@ -1550,6 +1719,7 @@ static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___close static lean_object* l_Lean_Parser_Term_completion___closed__2; static lean_object* l_Lean_Parser_Term_nomatch___closed__4; static lean_object* l_Lean_Parser_Term_whereDecls___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_hole___closed__6; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___closed__3; @@ -1559,6 +1729,7 @@ static lean_object* l_Lean_Parser_Tactic_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__22; LEAN_EXPORT lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_whereDecls_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_Term_basicFun_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1579,9 +1750,14 @@ static lean_object* l_Lean_Parser_Term_noindex___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_structInstField___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_funBinder_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_explicitUniv_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__2; static lean_object* l_Lean_Parser_semicolonOrLinebreak___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_have_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_bracketedBinder_quot; +static lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_trueVal___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_quot_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_binderTactic_formatter___closed__3; lean_object* l_Lean_PrettyPrinter_Parenthesizer_parserOfStack_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_scoped___elambda__1___closed__4; @@ -1592,6 +1768,8 @@ static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed_ lean_object* l_Lean_Parser_strLit___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letRecDecl___closed__6; static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_declRange___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_have_declRange___closed__4; static lean_object* l_Lean_Parser_Term_let__fun___closed__7; @@ -1609,6 +1787,8 @@ static lean_object* l_Lean_Parser_Term_prop___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeSpec_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__15; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_trueVal___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_panic(lean_object*); @@ -1623,7 +1803,6 @@ static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__18; static lean_object* l___regBuiltin_Lean_Parser_Term_noindex_declRange___closed__5; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_whereDecls___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__31; static lean_object* l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfTypeMVar___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_basicFun___closed__10; @@ -1633,6 +1812,7 @@ static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___close LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_seq1_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__5; static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__17; @@ -1647,14 +1827,18 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_declRange(l static lean_object* l_Lean_Parser_Term_forInMacro___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_trueVal___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letrec_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_ellipsis___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderType___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_num___closed__2; static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_suffices___elambda__1___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__39; static lean_object* l_Lean_Parser_Term_have___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_declRange___closed__1; lean_object* l_Lean_PrettyPrinter_Formatter_checkColGe_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -1662,6 +1846,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_declRange___cl LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__31; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_type_declRange(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_docString___closed__1; @@ -1670,6 +1855,7 @@ static lean_object* l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__3; static lean_object* l_Lean_Parser_Term_dbgTrace___closed__9; static lean_object* l_Lean_Parser_Term_letRecDecls___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_falseVal___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__12; lean_object* l_Lean_ppIndent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Parser_ParserState_hasError___spec__1(lean_object*, lean_object*); @@ -1682,12 +1868,15 @@ static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__15; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_binop_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__2; +extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___closed__1; static lean_object* l_Lean_Parser_Term_suffices___closed__4; static lean_object* l_Lean_Parser_Term_tupleTail_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_sorry___closed__7; static lean_object* l_Lean_Parser_Term_attr_quot___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__fun_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__1; static lean_object* l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_have_declRange___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_sorry_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1703,7 +1892,7 @@ static lean_object* l_Lean_Parser_Term_let___closed__2; static lean_object* l_Lean_Parser_Term_letIdDecl___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_binderTactic_formatter___closed__5; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__39; +static lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_let_declRange___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_show_declRange___closed__1; static lean_object* l_Lean_Parser_Term_binop_parenthesizer___closed__4; @@ -1717,12 +1906,14 @@ static lean_object* l_Lean_Parser_Term_dbgTrace___closed__1; static lean_object* l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_declRange___closed__5; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2; static lean_object* l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_haveIdDecl_formatter___closed__3; static lean_object* l_Lean_Parser_Term_hole___closed__4; static lean_object* l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_structInstLVal___closed__3; static lean_object* l_Lean_Parser_Term_fun___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__2; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__6; static lean_object* l_Lean_Parser_Tactic_quot___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_quotSeq_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1731,15 +1922,16 @@ static lean_object* l_Lean_Parser_Term_matchDiscr___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_num___closed__2; static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Term_argument_formatter___closed__5; static lean_object* l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_binrel__no__prop_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderDefault; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__28; static lean_object* l_Lean_Parser_Term_assert___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_namedPattern___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_local___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_paren_declRange___closed__4; lean_object* l_Lean_PrettyPrinter_Formatter_withAntiquot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letDecl___closed__6; @@ -1747,6 +1939,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_trailing__parser; static lean_object* l___regBuiltin_Lean_Parser_Term_ident_declRange___closed__7; static lean_object* l_Lean_Parser_Term_subst_formatter___closed__1; static lean_object* l_Lean_Parser_Term_binop__lazy___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__2; static lean_object* l_Lean_Parser_Term_sort___closed__1; static lean_object* l_Lean_Parser_Term_letMVar_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__6; @@ -1754,9 +1947,10 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_prop_declRange___closed__5; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__30; static lean_object* l___regBuiltin_Lean_Parser_Term_assert_declRange___closed__3; static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__11; -static lean_object* l_Lean_Parser_Term_have_formatter___closed__7; static lean_object* l_Lean_Parser_Term_paren___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfContainsMVar; +static lean_object* l___regBuiltin_Lean_Parser_Term_have_formatter___closed__1; static lean_object* l_Lean_Parser_Term_cdot_formatter___closed__4; static lean_object* l_Lean_Parser_Term_ensureTypeOf___closed__9; static lean_object* l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__3; @@ -1764,6 +1958,7 @@ static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_instBinder___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_letIdLhs_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_hole___elambda__1___closed__3; @@ -1775,9 +1970,13 @@ static lean_object* l_Lean_Parser_Term_let__tmp_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_let___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optEllipsis_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_panic_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeAscription; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letIdDecl___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__1; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__17; static lean_object* l___regBuiltin_Lean_Parser_Term_let_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_byTactic_x27_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1792,6 +1991,7 @@ static lean_object* l_Lean_Parser_Term_type_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInstField_formatter___closed__6; static lean_object* l_Lean_Parser_Term_funImplicitBinder_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_sort___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_seq1___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_haveDecl___elambda__1___closed__1; @@ -1803,12 +2003,15 @@ static lean_object* l_Lean_Parser_Term_typeOf___closed__5; static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__5; static lean_object* l_Lean_Parser_Term_type_formatter___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_quotedName___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_namedPattern; static lean_object* l___regBuiltin_Lean_Parser_Term_sort_declRange___closed__4; static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_motive_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__2; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_ident___closed__3; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__11; @@ -1816,16 +2019,20 @@ static lean_object* l_Lean_Parser_Term_unreachable___closed__7; static lean_object* l_Lean_Parser_Term_let__tmp_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_typeAscription_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_unreachable_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; static lean_object* l_Lean_Parser_Term_let__tmp_formatter___closed__5; static lean_object* l_Lean_Parser_Term_motive_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_letMVar_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_arrow; static lean_object* l_Lean_Parser_Term_arrow___closed__4; static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ellipsis_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_namedArgument_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letrec___closed__2; static lean_object* l_Lean_Parser_Term_letIdLhs___closed__5; @@ -1835,11 +2042,14 @@ static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___close static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dbgTrace; static lean_object* l_Lean_Parser_Term_dynamicQuot_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__2; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__15; static lean_object* l_Lean_Parser_Term_attributes___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Command_docComment___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_let__tmp___elambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAlt_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1849,6 +2059,7 @@ static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___closed__4; static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_declRange___closed__2; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__1; static lean_object* l_Lean_Parser_Tactic_quot_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_match___closed__6; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__2; @@ -1858,6 +2069,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_noImplicitLambda_parenthesizer(lean_ static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_prop___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_declRange___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_falseVal_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_structInstLVal_formatter___closed__9; @@ -1868,6 +2081,7 @@ static lean_object* l_Lean_Parser_Command_docComment___closed__4; static lean_object* l_Lean_Parser_Term_haveEqnsDecl___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_depArrow_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_have(lean_object*); @@ -1878,9 +2092,11 @@ static lean_object* l_Lean_Parser_Command_docComment___elambda__1___lambda__1___ static lean_object* l_Lean_Parser_Term_syntheticHole___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_namedArgument___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_declRange___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_explicitBinder_formatter___closed__2; lean_object* l_Lean_Parser_ppHardSpace_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_optIdent; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_paren___closed__2; static lean_object* l_Lean_Parser_Term_matchDiscr___closed__3; static lean_object* l_Lean_Parser_Term_suffices___elambda__1___closed__1; @@ -1899,16 +2115,20 @@ static lean_object* l_Lean_Parser_Command_docComment___closed__1; static lean_object* l_Lean_Parser_Term_noindex___closed__4; static lean_object* l_Lean_Parser_Term_noindex_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__16; +static lean_object* l___regBuiltin_Lean_Parser_Term_local_formatter___closed__1; static lean_object* l_Lean_Parser_Term_match_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_declRange___closed__2; static lean_object* l_Lean_Parser_Term_sorry___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_funBinder___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_let___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optType; static lean_object* l_Lean_Parser_Term_trueVal___closed__2; static lean_object* l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_funImplicitBinder_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_binderTactic___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__2; static lean_object* l_Lean_Parser_Term_tupleTail___closed__1; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_basicFun_parenthesizer___closed__11; @@ -1919,15 +2139,20 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_declRange___clos static lean_object* l_Lean_Parser_Term_assert_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letrec_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Command_commentBody_parenthesizer___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__2; static lean_object* l_Lean_Parser_Term_letMVar___closed__7; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_pipeProj___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_letEqnsDecl___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_str___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_parenSpecial_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_pipeCompletion_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1956,6 +2181,7 @@ static lean_object* l_Lean_Parser_Term_funBinder___elambda__1___closed__1; lean_object* l_Lean_Parser_lookaheadFn(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_proj___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__24; static lean_object* l_Lean_Parser_Term_char___closed__1; static lean_object* l_Lean_Parser_Term_stateRefT_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_fun; @@ -1963,19 +2189,19 @@ static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__4; lean_object* l_Lean_Parser_nodeInfo(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_let__tmp_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_structInst___closed__4; -static lean_object* l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_attributes_parenthesizer___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_suffices___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_arrow___closed__8; static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__12; lean_object* l_Lean_Parser_checkLhsPrecFn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_ensureTypeOf___closed__8; -static lean_object* l_Lean_Parser_Term_letRecDecls_formatter___closed__4; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___closed__5; static lean_object* l_Lean_Parser_Term_fromTerm___closed__2; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__2; static lean_object* l_Lean_Parser_Term_subst_formatter___closed__2; static lean_object* l_Lean_Parser_Term_completion___closed__6; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__5; @@ -1992,7 +2218,7 @@ static lean_object* l_Lean_Parser_Term_bracketedBinder_parenthesizer___closed__1 LEAN_EXPORT lean_object* l_Lean_Parser_darrow_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_charLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__2; -static lean_object* l_Lean_Parser_Term_letDecl_formatter___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicitUniv___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_falseVal___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1; @@ -2000,19 +2226,25 @@ static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed_ static lean_object* l_Lean_Parser_Term_binop__lazy___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_declRange___closed__4; static lean_object* l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter(lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__13; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_attributes___closed__5; static lean_object* l_Lean_Parser_Term_funBinder_parenthesizer___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_local_formatter___closed__2; static lean_object* l_Lean_Parser_Term_namedPattern___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_declRange___closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderTactic; static lean_object* l_Lean_Parser_Term_paren___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__4; static lean_object* l_Lean_Parser_Tactic_seq1___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_type_declRange___closed__7; static lean_object* l_Lean_Parser_Term_namedArgument___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__3; static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__2; static lean_object* l_Lean_Parser_Term_whereDecls_formatter___closed__8; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_proj___closed__8; @@ -2032,8 +2264,10 @@ static lean_object* l_Lean_Parser_Term_paren_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_hole_declRange___closed__7; static lean_object* l_Lean_Parser_Term_let__fun___closed__2; static lean_object* l_Lean_Parser_Term_byTactic_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_whereDecls___closed__4; static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_formatter(lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_typeSpec___closed__2; static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__7; @@ -2049,6 +2283,7 @@ static lean_object* l_Lean_Parser_Term_attributes_formatter___closed__4; static lean_object* l_Lean_Parser_Term_parenSpecial___closed__3; static lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dynamicQuot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__1; static lean_object* l_Lean_Parser_Term_attr_quot___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_quotedName_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_dynamicQuot_formatter___closed__3; @@ -2056,15 +2291,18 @@ static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_falseVal___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letDecl; lean_object* l_Lean_Parser_scientificLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__7; static lean_object* l_Lean_Parser_Term_completion___closed__5; static lean_object* l_Lean_Parser_Term_strictImplicitBinder___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_type_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_haveDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__1; static lean_object* l_Lean_Parser_Term_type_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__2; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_match_formatter___closed__9; static lean_object* l_Lean_Parser_Term_letrec_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__7; @@ -2073,11 +2311,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Command_commentBody_parenthesizer___boxed static lean_object* l_Lean_Parser_Term_sorry___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_explicitUniv___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_have_declRange___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__24; static lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_declRange___closed__6; lean_object* l_Lean_Parser_nonReservedSymbolInfo(lean_object*, uint8_t); static lean_object* l_Lean_Parser_Term_namedArgument_formatter___closed__4; static lean_object* l_Lean_Parser_Term_typeOf_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_sort; lean_object* l_Lean_Parser_strLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_let__tmp_formatter___closed__6; @@ -2086,6 +2324,7 @@ static lean_object* l_Lean_Parser_Term_scoped_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_strictImplicitBinder___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_declRange___closed__6; static lean_object* l_Lean_Parser_Term_bracketedBinder_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_attrKind___elambda__1___closed__10; @@ -2093,12 +2332,15 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_assert_declRange___closed__2 static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_byTactic_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_sufficesDecl___closed__5; static lean_object* l_Lean_Parser_Term_argument_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_let__delayed_formatter___closed__2; static lean_object* l_Lean_Parser_Term_ellipsis___closed__2; static lean_object* l_Lean_Parser_Term_cdot_formatter___closed__1; static lean_object* l_Lean_Parser_Term_forInMacro_x27___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_cdot___closed__9; lean_object* l_Lean_Parser_checkNoWsBefore___elambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Level_quot_parenthesizer___closed__3; @@ -2113,9 +2355,9 @@ static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed static lean_object* l_Lean_Parser_Term_letIdDecl___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_binop__lazy___closed__8; -static lean_object* l_Lean_Parser_Term_explicitBinder_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_declRange___closed__2; static lean_object* l_Lean_Parser_Term_explicitBinder___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__1; static lean_object* l_Lean_Parser_Term_match___closed__5; lean_object* l_Lean_Parser_checkWsBeforeFn(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_declRange___closed__7; @@ -2132,6 +2374,7 @@ static lean_object* l_Lean_Parser_Term_attrInstance___closed__8; static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_letEqnsDecl_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicitBinder___elambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__1; lean_object* l_Lean_Parser_sepBy(lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Parser_Term_letrec___closed__8; static lean_object* l_Lean_Parser_Term_optSemicolon_formatter___closed__1; @@ -2142,6 +2385,7 @@ static lean_object* l_Lean_Parser_Term_let__tmp_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_haveDecl_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_declRange___closed__6; static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_paren_formatter___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_char_declRange___closed__5; static lean_object* l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1; @@ -2153,12 +2397,10 @@ static lean_object* l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__3 static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_declRange___closed__3; static lean_object* l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__9; -static lean_object* l_Lean_Parser_Term_argument_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Tactic_quot___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_funImplicitBinder___closed__2; static lean_object* l_Lean_Parser_Term_funBinder___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__4; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__12; static lean_object* l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_explicitUniv___closed__5; @@ -2186,17 +2428,20 @@ static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_have; static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_letIdLhs___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_let_formatter___closed__2; static lean_object* l_Lean_Parser_Term_namedPattern___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeSpec; static lean_object* l_Lean_Parser_Term_hole_formatter___closed__3; static lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_leading__parser___closed__5; static lean_object* l_Lean_Parser_Tactic_quot_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_fun_declRange___closed__7; static lean_object* l_Lean_Parser_Term_let__delayed_formatter___closed__4; static lean_object* l_Lean_Parser_Term_paren___closed__8; static lean_object* l_Lean_Parser_Term_haveDecl___closed__3; static lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_letPatDecl___closed__5; static lean_object* l_Lean_Parser_Term_anonymousCtor_formatter___closed__1; @@ -2226,21 +2471,27 @@ static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__2; lean_object* l_Lean_PrettyPrinter_Formatter_visitAtom(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__1; static lean_object* l_Lean_Parser_Term_whereDecls___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__2; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__10; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Term_trueVal___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_quotedName___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_panic_declRange___closed__7; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_stateRefT___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letIdDecl___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_declRange___closed__4; static lean_object* l_Lean_Parser_Term_instBinder___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroArg_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_explicit_parenthesizer___closed__4; @@ -2255,14 +2506,18 @@ static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed_ static lean_object* l_Lean_Parser_Term_dbgTrace___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_byTactic_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__2; static lean_object* l_Lean_Parser_convParser___closed__1; static lean_object* l_Lean_Parser_Term_forInMacro_formatter___closed__1; static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_suffices_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_type_formatter___closed__1; static lean_object* l_Lean_Parser_Term_explicitBinder___closed__3; -static lean_object* l_Lean_Parser_Term_generalizingParam_formatter___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_have_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_suffices___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_dynamicQuot___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_letIdBinder___closed__1; static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__13; static lean_object* l_Lean_Parser_Term_panic___closed__8; @@ -2276,6 +2531,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letrec___elambda__1(lean_object*, le static lean_object* l_Lean_Parser_Term_sort___closed__8; static lean_object* l_Lean_Parser_Term_structInstField___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_haveDecl_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter(lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_63____closed__3; static lean_object* l_Lean_Parser_Term_paren___closed__4; static lean_object* l_Lean_Parser_Term_forInMacro_formatter___closed__4; @@ -2291,12 +2547,14 @@ static lean_object* l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket_parenthesizer___closed__1; lean_object* l_Lean_PrettyPrinter_Parenthesizer_incQuotDepth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_byTactic_formatter___closed__3; static lean_object* l_Lean_Parser_Term_optExprPrecedence___closed__6; static lean_object* l_Lean_Parser_Term_binderTactic_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_local; static lean_object* l_Lean_Parser_Term_matchAlt___closed__12; static lean_object* l_Lean_Parser_Term_let___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__4; static lean_object* l_Lean_Parser_Term_attr_quot_formatter___closed__3; static lean_object* l_Lean_Parser_Term_binop___elambda__1___closed__12; @@ -2321,7 +2579,9 @@ static lean_object* l_Lean_Parser_Term_syntheticHole___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_type_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___closed__5; static lean_object* l_Lean_Parser_Term_instBinder_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__13; +static lean_object* l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_bracketedBinder___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_unreachable___closed__5; static lean_object* l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__5; @@ -2336,13 +2596,16 @@ static lean_object* l_Lean_Parser_Term_falseVal_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_stateRefT___closed__2; static lean_object* l_Lean_Parser_Term_pipeProj___closed__5; static lean_object* l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__18; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_doubleQuotedName___closed__5; lean_object* l_Lean_Parser_sepByIndent_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_macroDollarArg___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_type_formatter___closed__2; static lean_object* l_Lean_Parser_Term_paren_formatter___closed__1; static lean_object* l_Lean_Parser_Term_pipeProj_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_declRange___closed__3; @@ -2352,6 +2615,7 @@ static lean_object* l_Lean_Parser_Term_fun___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_type_declRange___closed__3; static lean_object* l_Lean_Parser_Term_sorry___closed__5; static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_declRange___closed__1; static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_unreachable(lean_object*); @@ -2373,6 +2637,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer(lean LEAN_EXPORT lean_object* l_Lean_Parser_Term_attr_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_docString(lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_node_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dotIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__49; @@ -2390,8 +2655,11 @@ static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___elambda__1___cl static lean_object* l_Lean_Parser_Term_explicitUniv___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_defaultOrOfNonempty_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_cdot_formatter___closed__2; static lean_object* l_Lean_Parser_Term_binop__lazy___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_docComment_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_letMVar_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_declRange___closed__5; @@ -2405,13 +2673,16 @@ static lean_object* l_Lean_Parser_Term_let__tmp_formatter___closed__1; static lean_object* l_Lean_Parser_Term_panic___closed__4; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___closed__5; static lean_object* l_Lean_Parser_Term_whereDecls_formatter___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_have_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInst___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName(lean_object*); static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_attr_quot___closed__7; static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_matchDiscr___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_proj_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_scoped___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_implicitBinder_parenthesizer(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2427,7 +2698,6 @@ extern lean_object* l_Lean_Parser_argPrec; static lean_object* l_Lean_Parser_Term_fromTerm_parenthesizer___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_letRecDecls_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_byTactic_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_panic___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_structInstArrayRef___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_instCoeTSyntaxConsSyntaxNodeKindStrAnonymousNil__1___boxed(lean_object*); @@ -2437,6 +2707,7 @@ static lean_object* l_Lean_Parser_Term_type_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_structInstField_formatter___closed__2; static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Level_quot___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_fromTerm; static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_subst_declRange___closed__4; @@ -2444,15 +2715,19 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_funBinder___elambda__1(lean_object*, static lean_object* l_Lean_Parser_Term_tupleTail_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__9; static lean_object* l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_attrInstance___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_have_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_show___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_quotedName_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_char_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__2; static lean_object* l_Lean_Parser_Term_explicitBinder___closed__5; static lean_object* l_Lean_Parser_Term_letIdLhs___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_implicitBinder___elambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstField_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_declRange___closed__7; static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_declRange___closed__7; @@ -2480,7 +2755,6 @@ static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___closed__10; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_63____closed__5; static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_typeOf_formatter___closed__3; -static lean_object* l_Lean_Parser_Term_fun_formatter___closed__7; static lean_object* l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_tupleTail___closed__7; static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__5; @@ -2488,6 +2762,7 @@ static lean_object* l_Lean_Parser_Term_ensureExpectedType_formatter___closed__2; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__13; static lean_object* l_Lean_Parser_Tactic_quot___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_cdot___elambda__1___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trueVal_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_depArrow___closed__4; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__16; LEAN_EXPORT lean_object* l_Lean_Parser_Term_quotedName_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2496,6 +2771,7 @@ static lean_object* l_Lean_Parser_Term_byTactic_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_pipeProj___closed__3; static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_anonymousCtor_formatter___closed__5; static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__2; static lean_object* l_Lean_Parser_Tactic_quot___elambda__1___closed__1; @@ -2505,6 +2781,7 @@ static lean_object* l_Lean_Parser_Term_show_formatter___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser(lean_object*); static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_matchDiscr___elambda__1___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__4; static lean_object* l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_paren___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar(lean_object*); @@ -2515,16 +2792,19 @@ static lean_object* l_Lean_Parser_Term_subst___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_borrowed_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_show_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_showRhs_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_whereDecls; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withoutForbidden_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_subst_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_completion___closed__4; -static lean_object* l_Lean_Parser_Term_generalizingParam_formatter___closed__11; static lean_object* l_Lean_Parser_Term_trueVal_formatter___closed__3; static lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_haveDecl_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__1; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__10; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__26; +static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_declRange___closed__7; static lean_object* l_Lean_Parser_Term_structInstField___closed__8; static lean_object* l_Lean_Parser_Term_funImplicitBinder_parenthesizer___closed__4; @@ -2537,6 +2817,7 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_declRange(l static lean_object* l_Lean_Parser_Term_binderDefault___elambda__1___closed__5; lean_object* l_Lean_Parser_checkNoWsBeforeFn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letIdBinder___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal_formatter___closed__11; static lean_object* l_Lean_Parser_Term_have___closed__6; static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__11; @@ -2545,12 +2826,13 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_suffices_declRange(lean static lean_object* l_Lean_Parser_Term_assert_formatter___closed__4; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__34; static lean_object* l_Lean_Parser_Term_paren_parenthesizer___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__1; static lean_object* l_Lean_Parser_Term_let__tmp___closed__6; static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_scoped; static lean_object* l_Lean_Parser_Term_attrKind___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_fun___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_letrec_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___closed__4; @@ -2583,18 +2865,20 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_let_declRange___closed__2; lean_object* l_Lean_Parser_orelseInfo(lean_object*, lean_object*); lean_object* l_Lean_Parser_termParser_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_app_declRange___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_suffices___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_byTactic___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_trailing__parser___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroDollarArg_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__2; lean_object* l_Lean_Parser_scientificLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop(lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_type_formatter___closed__8; static lean_object* l_Lean_Parser_Term_typeSpec_formatter___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__4; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_nomatch___elambda__1(lean_object*, lean_object*); @@ -2608,6 +2892,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letEqnsDecl_formatter(lean_object*, static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__11; static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_declRange___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_falseVal; +static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_quotedName___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_forInMacro_x27___closed__3; static lean_object* l_Lean_Parser_Term_binop___closed__6; @@ -2617,9 +2902,12 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_show_declRange___closed__2; static lean_object* l_Lean_Parser_Term_structInstField_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_letMVar_formatter___closed__5; static lean_object* l_Lean_Parser_Term_attr_quot___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_pipeProj_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_declRange___closed__6; static lean_object* l_Lean_Parser_Term_forInMacro___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_ensureTypeOf___closed__1; static lean_object* l_Lean_Parser_Term_dotIdent_formatter___closed__2; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__13; @@ -2633,16 +2921,21 @@ static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__19; static lean_object* l_Lean_Parser_Term_have_formatter___closed__3; static lean_object* l_Lean_Parser_Term_explicit_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__41; +static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_structInst___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_attributes; static lean_object* l_Lean_Parser_Term_inaccessible___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_scoped___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binrel___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_falseVal___closed__6; static lean_object* l_Lean_Parser_Term_instBinder___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_letIdDecl_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_completion_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_borrowed_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_ensureTypeOf___closed__2; @@ -2656,6 +2949,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_declRange__ static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_letIdDecl_formatter___closed__4; static lean_object* l_Lean_Parser_Term_match___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_binderIdent___closed__2; static lean_object* l_Lean_Parser_Term_dbgTrace___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveEqnsDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2668,6 +2962,7 @@ static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__ static lean_object* l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__6; lean_object* l_Lean_PrettyPrinter_Formatter_withoutForbidden_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_subst___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_instBinder___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_show_declRange___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_declRange___closed__3; @@ -2676,9 +2971,9 @@ static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__3; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_scoped_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_ensureExpectedType_formatter___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__8; static lean_object* l_Lean_Parser_Level_quot___closed__2; static lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer(lean_object*); extern lean_object* l_Lean_Parser_maxPrec; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_local_formatter___closed__1; @@ -2695,11 +2990,14 @@ static lean_object* l_Lean_Parser_Term_explicit___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_whereDecls_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_declRange___closed__2; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Term_assert___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_local_formatter___closed__2; static lean_object* l_Lean_Parser_Term_explicit_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_quot___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_motive_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_ensureExpectedType___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_trailing__parser___closed__8; static lean_object* l_Lean_Parser_Term_sort_formatter___closed__1; @@ -2707,6 +3005,7 @@ static lean_object* l_Lean_Parser_Term_let__delayed___closed__2; lean_object* l_Lean_Parser_strLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__17; static lean_object* l_Lean_Parser_Term_whereDecls___closed__3; static lean_object* l_Lean_Parser_Term_optExprPrecedence_formatter___closed__2; static lean_object* l_Lean_Parser_Term_strictImplicitBinder_formatter___closed__2; @@ -2718,6 +3017,8 @@ lean_object* l_Array_back___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_str_declRange___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_binrel__no__prop___closed__6; static lean_object* l_Lean_Parser_Term_structInstField_formatter___closed__5; static lean_object* l_Lean_Parser_Term_fromTerm___closed__7; @@ -2731,6 +3032,7 @@ static lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_syntheticHole___closed__2; static lean_object* l_Lean_Parser_Term_prop_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_funImplicitBinder_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_app_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_declRange___closed__6; @@ -2751,18 +3053,20 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_forall_declRange___closed__2 static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_declRange___closed__4; static lean_object* l_Lean_Parser_Term_forInMacro_x27___closed__5; static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_declRange___closed__6; static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_declRange___closed__1; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__11; static lean_object* l_Lean_Parser_Term_optEllipsis_formatter___closed__3; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_show___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_declRange___closed__4; static lean_object* l_Lean_Parser_Term_depArrow___closed__1; -static lean_object* l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_declRange___closed__4; static lean_object* l_Lean_Parser_Term_proj___closed__5; static lean_object* l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__1; @@ -2777,6 +3081,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_argument_parenthesizer(lean_object*, static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_forall_formatter___closed__7; static lean_object* l_Lean_Parser_Term_sort_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__1; static lean_object* l_Lean_Parser_Term_match_formatter___closed__11; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_attrKind_parenthesizer___closed__2; @@ -2787,14 +3092,19 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_declRange___closed_ static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_attributes_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_paren_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_argument___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_proj_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__1; static lean_object* l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_inaccessible_formatter___closed__5; static lean_object* l_Lean_Parser_Term_binrel_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_suffices_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_haveDecl___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_declRange___closed__5; static lean_object* l_Lean_Parser_Term_paren_formatter___closed__4; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___closed__3; @@ -2802,7 +3112,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_structInst_declRange___close static lean_object* l_Lean_Parser_Term_suffices___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_sort___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_structInstField___closed__4; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__17; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_pipeProj_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_proj___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_declRange___closed__5; @@ -2815,22 +3125,25 @@ static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___clos static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__2; lean_object* l_Lean_Parser_sepByIndent_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_dbgTrace___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_implicitBinder(uint8_t); static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__16; static lean_object* l_Lean_Parser_Term_dotIdent___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_declRange___closed__1; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_namedPattern___closed__6; +extern lean_object* l_Lean_PrettyPrinter_formatterAttribute; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_panic___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_instCoeTSyntaxConsSyntaxNodeKindStrAnonymousNil___boxed(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_declRange___closed__7; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_optExprPrecedence_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prop_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_declRange___closed__3; uint32_t lean_string_utf8_get(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__43; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_haveDecl___closed__8; static lean_object* l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__6; @@ -2839,6 +3152,7 @@ static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_declRange___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_nomatch_formatter___closed__1; static lean_object* l_Lean_Parser_Term_haveDecl___closed__4; static lean_object* l_Lean_Parser_Term_let__delayed_formatter___closed__3; @@ -2849,7 +3163,9 @@ static lean_object* l_Lean_Parser_Term_depArrow___closed__5; static lean_object* l_Lean_Parser_Term_binderDefault_formatter___closed__2; static lean_object* l_Lean_Parser_Term_binop___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_explicitUniv___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___closed__3; static lean_object* l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_let__delayed___elambda__1___closed__2; @@ -2857,7 +3173,6 @@ static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_leading__parser___closed__9; lean_object* l_Lean_Parser_interpolatedStr(lean_object*); static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__2; -static lean_object* l_Lean_Parser_Term_haveDecl_formatter___closed__6; static lean_object* l_Lean_Parser_Term_letPatDecl___closed__7; static lean_object* l_Lean_Parser_Term_binrel__no__prop___closed__4; static lean_object* l_Lean_Parser_Term_structInstLVal_formatter___closed__1; @@ -2865,6 +3180,7 @@ static lean_object* l_Lean_Parser_Tactic_quot___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicitBinder___boxed(lean_object*); static lean_object* l_Lean_Parser_Term_dynamicQuot___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_structInst_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_declRange___closed__1; static lean_object* l_Lean_Parser_Term_binrel_formatter___closed__1; static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__12; @@ -2883,6 +3199,7 @@ lean_object* l_Lean_Parser_parserOfStack(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_argument_formatter___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_argument; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__fun___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__1; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_haveDecl___elambda__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_suffices_declRange___closed__6; @@ -2892,6 +3209,7 @@ static lean_object* l_Lean_Parser_Term_argument___elambda__1___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fun(lean_object*); static lean_object* l_Lean_Parser_Term_letDecl___closed__9; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__21; +static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__2; static lean_object* l_Lean_Parser_Term_ellipsis___elambda__1___closed__4; static lean_object* l_Lean_Parser_Tactic_tacticSeq___closed__4; static lean_object* l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__4; @@ -2912,6 +3230,7 @@ static lean_object* l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__5; static lean_object* l_Lean_Parser_Tactic_quot___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_show___elambda__1___closed__11; lean_object* l_Lean_Parser_registerBuiltinParserAttribute(lean_object*, lean_object*, uint8_t, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_tacticParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binderTactic___closed__1; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___closed__4; @@ -2934,6 +3253,7 @@ static lean_object* l_Lean_Parser_Term_panic_parenthesizer___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern(lean_object*); static lean_object* l_Lean_Parser_Term_structInst___closed__2; static lean_object* l_Lean_Parser_Term_explicitUniv___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__1; lean_object* l_Lean_Parser_evalInsideQuot___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_arrow(lean_object*); static lean_object* l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__4; @@ -2942,18 +3262,21 @@ static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__8; static lean_object* l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_sorry_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_leading__parser___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__1; static lean_object* l_Lean_Parser_Term_hole___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Command_commentBody___elambda__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_semicolonOrLinebreak_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_explicitUniv___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__delayed; LEAN_EXPORT lean_object* l_Lean_Parser_Term_strictImplicitRightBracket_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_hole_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_nomatch_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fromTerm_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_optExprPrecedence___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__2; static lean_object* l_Lean_Parser_Term_proj___closed__2; static lean_object* l_Lean_Parser_Term_trueVal___closed__4; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__32; static lean_object* l_Lean_Parser_Term_dynamicQuot_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_noindex_formatter___closed__3; @@ -2963,6 +3286,7 @@ lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_basicFun___closed__6; static lean_object* l_Lean_Parser_Term_fun___closed__4; static lean_object* l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_typeSpec___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_declRange___closed__2; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__10; @@ -2978,15 +3302,18 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_declRange___clo LEAN_EXPORT lean_object* l_Lean_Parser_Term_suffices___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_suffices_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_namedArgument___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__43; static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_ellipsis___elambda__1___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_panic_declRange___closed__5; static lean_object* l_Lean_Parser_Term_structInstField_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__13; static lean_object* l_Lean_Parser_Term_namedPattern_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__18; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_completion___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_arrow___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2997,6 +3324,7 @@ static lean_object* l_Lean_Parser_Term_explicit___closed__7; static lean_object* l_Lean_Parser_Term_completion___closed__1; static lean_object* l_Lean_Parser_Term_namedPattern___closed__5; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_show_formatter___closed__2; static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__12; lean_object* l_Lean_PrettyPrinter_Parenthesizer_pushNone_parenthesizer___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_app_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -3009,23 +3337,27 @@ static lean_object* l_Lean_Parser_Term_arrow___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__8; static lean_object* l_Lean_Parser_Term_noImplicitLambda___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doubleQuotedName; +static lean_object* l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_borrowed_formatter___closed__1; static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__15; -static lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter___closed__5; static lean_object* l_Lean_Parser_Term_noImplicitLambda___closed__5; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__2; extern lean_object* l_Lean_instInhabitedSyntax; static lean_object* l_Lean_Parser_Term_dbgTrace_formatter___closed__4; static lean_object* l_Lean_Parser_Term_optEllipsis___closed__5; static lean_object* l_Lean_Parser_Term_explicitUniv___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_leading__parser___closed__8; static lean_object* l_Lean_Parser_Tactic_quotSeq_formatter___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_local_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__1; static lean_object* l_Lean_Parser_Term_pipeCompletion___closed__3; static lean_object* l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_binop_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__1; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__47; static lean_object* l_Lean_Parser_Term_whereDecls_formatter___closed__11; static lean_object* l_Lean_Parser_Tactic_quotSeq_formatter___closed__5; @@ -3038,23 +3370,24 @@ static lean_object* l_Lean_Parser_Term_stateRefT_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_inaccessible_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_match_formatter___closed__4; -static lean_object* l_Lean_Parser_Term_showRhs_formatter___closed__1; -static lean_object* l_Lean_Parser_Term_attrKind_parenthesizer___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__8; static lean_object* l_Lean_Parser_Term_proj_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_declRange___closed__2; static lean_object* l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_char_declRange___closed__2; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_letrec___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__20; static lean_object* l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__1; static lean_object* l_Lean_Parser_Term_fromTerm_formatter___closed__1; static lean_object* l_Lean_Parser_Term_syntheticHole___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_trueVal_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_assert___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_inaccessible_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_inaccessible___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__7; @@ -3075,6 +3408,8 @@ static lean_object* l_Lean_Parser_Term_forInMacro_x27_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible(lean_object*); static lean_object* l_Lean_Parser_Term_sort_formatter___closed__4; static lean_object* l_Lean_Parser_Term_let___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_subst___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__12; static lean_object* l___regBuiltin_Lean_Parser_Term_str_declRange___closed__4; @@ -3084,7 +3419,11 @@ static lean_object* l_Lean_Parser_Term_structInstArrayRef_formatter___closed__3; static lean_object* l_Lean_Parser_Term_namedArgument___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_num_declRange___closed__2; static lean_object* l_Lean_Parser_Term_doubleQuotedName_formatter___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Term_cdot___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__2; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letEqnsDecl; static lean_object* l_Lean_Parser_Term_dbgTrace___elambda__1___closed__1; @@ -3092,7 +3431,6 @@ static lean_object* l_Lean_Parser_Term_generalizingParam_formatter___closed__5; static lean_object* l_Lean_Parser_Term_motive_formatter___closed__5; static lean_object* l_Lean_Parser_Term_letIdBinder_formatter___closed__1; lean_object* l_Lean_Parser_rawCh(uint32_t, uint8_t); -static lean_object* l_Lean_Parser_Term_structInstLVal_formatter___closed__12; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___elambda__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_nomatch(lean_object*); static lean_object* l_Lean_Parser_Term_forInMacro___elambda__1___closed__7; @@ -3102,6 +3440,7 @@ static lean_object* l_Lean_Parser_Term_app_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_assert_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_whereDecls_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_binderDefault___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letEqnsDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_have___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_declRange___closed__3; @@ -3118,7 +3457,6 @@ static lean_object* l_Lean_Parser_Term_quotedName___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letEqnsDecl___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__26; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__9; -static lean_object* l_Lean_Parser_Term_argument_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_scoped_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__6; @@ -3129,6 +3467,8 @@ static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__16; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___closed__3; static lean_object* l_Lean_Parser_Term_show_formatter___closed__4; static lean_object* l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_binop__lazy_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_haveIdDecl___closed__3; @@ -3140,21 +3480,21 @@ static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___close static lean_object* l_Lean_Parser_Term_letRecDecl___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binop___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_attributes___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_trailing__parser___closed__10; static lean_object* l_Lean_Parser_Term_attrInstance_formatter___closed__2; static lean_object* l_Lean_Parser_Term_letMVar_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__20; static lean_object* l_Lean_Parser_Term_sort_formatter___closed__2; static lean_object* l_Lean_Parser_Term_instBinder_formatter___closed__4; static lean_object* l_Lean_Parser_Term_leading__parser___closed__1; static lean_object* l_Lean_Parser_Term_instBinder___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__4; -static lean_object* l_Lean_Parser_Term_showRhs_formatter___closed__2; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_ellipsis___elambda__1___closed__1; lean_object* l_Lean_Parser_nonReservedSymbol_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_show___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_declRange___closed__5; static lean_object* l_Lean_Parser_Term_letMVar_formatter___closed__2; @@ -3162,16 +3502,21 @@ static lean_object* l_Lean_Parser_Term_borrowed_formatter___closed__2; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__15; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_str(lean_object*); static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optEllipsis; static lean_object* l_Lean_Parser_Term_have_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_namedPattern_parenthesizer___closed__7; lean_object* l_Lean_Parser_sepBy1_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sort_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_motive___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_typeSpec___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_pipeCompletion___closed__4; static lean_object* l_Lean_Parser_Term_tupleTail___elambda__1___closed__12; @@ -3182,8 +3527,12 @@ static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_local_formatter___closed__3; static lean_object* l_Lean_Parser_Term_letRecDecl___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forall; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_declRange___closed__6; static lean_object* l_Lean_Parser_Term_scoped___elambda__1___closed__7; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__32; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Term_app_declRange___closed__7; @@ -3197,6 +3546,7 @@ static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__4; lean_object* l_Lean_Parser_registerAlias(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_pipeProj___elambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_match_formatter___closed__6; static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1(lean_object*, lean_object*); @@ -3213,14 +3563,18 @@ static lean_object* l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_declRange___closed__1; static lean_object* l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__tmp_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_completion___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_depArrow_formatter___closed__1; static lean_object* l_Lean_Parser_Term_namedPattern_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_binrel___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_generalizingParam_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_show_declRange___closed__6; @@ -3234,9 +3588,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_let___elambda__1___lambda__1___boxed LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstField; static lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__37; static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_typeAscription___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__13; uint8_t l_Lean_Syntax_isAntiquot(lean_object*); static lean_object* l_Lean_Parser_Term_binrel___closed__2; @@ -3254,6 +3611,9 @@ static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___closed__15; lean_object* l_Lean_PrettyPrinter_Parenthesizer_fieldIdx_parenthesizer___boxed(lean_object*); static lean_object* l_Lean_Parser_Term_letIdDecl_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeOf(lean_object*); static lean_object* l_Lean_Parser_Term_haveIdDecl___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_declRange___closed__5; @@ -3262,6 +3622,7 @@ static lean_object* l_Lean_Parser_Term_generalizingParam___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_declRange___closed__2; static lean_object* l_Lean_Parser_Term_tupleTail_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_str_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_noindex; static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__3; @@ -3276,10 +3637,13 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_attrInstance; static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_declRange___closed__5; static lean_object* l_Lean_Parser_Term_forInMacro___closed__9; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_show_formatter___closed__1; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_explicitUniv___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_letMVar_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Level_quot___closed__7; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__12; @@ -3289,16 +3653,13 @@ static lean_object* l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_funImplicitBinder___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_declRange___closed__1; static lean_object* l_Lean_Parser_Term_attr_quot___elambda__1___closed__5; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__18; static lean_object* l___regBuiltin_Lean_Parser_Term_assert_declRange___closed__5; -static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__14; static lean_object* l_Lean_Parser_Term_proj_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_structInstField___elambda__1___closed__2; static lean_object* l_Lean_Parser_Command_docComment_formatter___closed__5; static lean_object* l_Lean_Parser_Term_typeOf_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letIdBinder___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_str___closed__1; static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__12; @@ -3317,6 +3678,7 @@ static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket_parenthesizer__ static lean_object* l_Lean_Parser_Term_funBinder_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_declRange___closed__1; static lean_object* l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInst_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_sorry___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1; @@ -3335,7 +3697,6 @@ static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__ static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__37; static lean_object* l_Lean_Parser_Term_binderTactic___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letrec___closed__4; @@ -3351,6 +3712,7 @@ static lean_object* l_Lean_Parser_Term_let__tmp_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_letDecl___closed__4; static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_forInMacro_x27___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_scientific(lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Term_char_declRange___closed__1; @@ -3381,14 +3743,17 @@ static lean_object* l_Lean_Parser_Term_attr_quot_formatter___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_declRange___closed__5; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_namedPattern___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_let__tmp_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_declRange___closed__4; static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__6; static lean_object* l_Lean_Parser_semicolonOrLinebreak___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Term_noindex_declRange___closed__2; static lean_object* l_Lean_Parser_Term_letIdLhs___closed__2; -static lean_object* l_Lean_Parser_Term_syntheticHole_formatter___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_show___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_completion; static lean_object* l___regBuiltin_Lean_Parser_Term_char_declRange___closed__3; @@ -3408,11 +3773,13 @@ static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___closed__3; static lean_object* l_Lean_Parser_Term_structInstLVal___closed__2; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binderTactic_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_letPatDecl___closed__10; static lean_object* l_Lean_Parser_Term_tupleTail_formatter___closed__5; static lean_object* l_Lean_Parser_Term_prop___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_have_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_cdot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_funBinder_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Term_explicitBinder___closed__6; @@ -3430,22 +3797,26 @@ static lean_object* l_Lean_Parser_Term_paren_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_noindex___closed__6; static lean_object* l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_typeAscription___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeAscription_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__15; static lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_paren_formatter___closed__11; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_declRange(lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__6; static lean_object* l_Lean_Parser_Term_attrKind_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__3; static lean_object* l_Lean_Parser_Term_nomatch___closed__1; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___closed__5; static lean_object* l_Lean_Parser_Term_whereDecls_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_matchAlt___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_motive_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_cdot___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_attr_quot___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__5; @@ -3476,6 +3847,7 @@ lean_object* l_Lean_Parser_mkAntiquot_parenthesizer___boxed(lean_object*, lean_o static lean_object* l___regBuiltin_Lean_Parser_Term_noindex_declRange___closed__4; static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_dynamicQuot___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__9; lean_object* l_Lean_Parser_sepBy1(lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__5; @@ -3486,43 +3858,48 @@ static lean_object* l_Lean_Parser_Term_namedPattern_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_instBinder___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_cdot_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_letDecl___closed__1; static lean_object* l_Lean_Parser_Term_ensureExpectedType___closed__5; static lean_object* l_Lean_Parser_Term_forall_formatter___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_declRange___closed__5; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__2; -static lean_object* l_Lean_Parser_Term_byTactic_formatter___closed__7; static lean_object* l_Lean_Parser_Term_argument_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_declRange___closed__6; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket___elambda__1___closed__5; lean_object* l_Lean_Parser_ppLine_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroDollarArg_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_match_declRange___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_let_formatter___closed__4; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__4; static lean_object* l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__15; static lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_declRange___closed__1; static lean_object* l_Lean_Parser_Term_depArrow_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_arrow___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_binop__lazy___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_ensureTypeOf_formatter___closed__3; static lean_object* l_Lean_Parser_Term_have___elambda__1___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__18; static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__7; lean_object* l_Lean_Parser_sepBy1Indent_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_inaccessible_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_trueVal___closed__5; static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__20; static lean_object* l_Lean_Parser_Term_haveIdDecl_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_let_declRange___closed__1; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__3; static lean_object* l_Lean_Parser_Tactic_seq1___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_namedArgument___closed__8; -static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__15; LEAN_EXPORT lean_object* l_Lean_Parser_Term_fromTerm_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__26; static lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_declRange___closed__1; @@ -3555,6 +3932,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letPatDecl_parenthesizer(lean_object static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_cdot___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_byTactic___closed__5; static lean_object* l_Lean_Parser_Term_proj___closed__7; static lean_object* l_Lean_Parser_Term_app_formatter___closed__1; @@ -3592,6 +3970,7 @@ static lean_object* l_Lean_Parser_Term_whereDecls___closed__6; static lean_object* l_Lean_Parser_Term_binop__lazy___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_forall_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_falseVal_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_forall_formatter___closed__6; lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkNoWsBefore_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_attr_quot___elambda__1___closed__6; @@ -3606,7 +3985,7 @@ static lean_object* l_Lean_Parser_Term_explicit___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_byTactic___closed__8; static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket___closed__3; static lean_object* l_Lean_Parser_Term_fromTerm___closed__4; -static lean_object* l_Lean_Parser_Term_attrKind_formatter___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Tactic_quot___closed__1; static lean_object* l_Lean_Parser_Term_falseVal___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_motive_parenthesizer___closed__8; @@ -3616,9 +3995,11 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1( static lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_declRange___closed__5; static lean_object* l_Lean_Parser_Term_matchAlt___closed__9; static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1; extern lean_object* l_Lean_Parser_numLit; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___closed__9; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__1; static lean_object* l_Lean_Parser_Term_panic___closed__6; static lean_object* l_Lean_Parser_Term_binop__lazy___elambda__1___closed__3; lean_object* l_Lean_PrettyPrinter_Formatter_parserOfStack_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -3633,14 +4014,18 @@ static lean_object* l_Lean_Parser_Term_inaccessible___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_namedPattern___closed__4; static lean_object* l_Lean_Parser_Term_matchAlt_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_trueVal___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_char_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_haveEqnsDecl___elambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_ident___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_syntheticHole___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__1; static lean_object* l_Lean_Parser_Term_binderTactic___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_num_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_forall___closed__1; static lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_funBinder_quot___closed__7; @@ -3656,14 +4041,19 @@ static lean_object* l_Lean_Parser_Term_dotIdent___closed__3; static lean_object* l_Lean_Parser_Term_let__delayed___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letrec___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_local_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__14; static lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__1; static lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_generalizingParam___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_declRange___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_let__fun_formatter___closed__6; static lean_object* l_Lean_Parser_Term_let___closed__5; @@ -3681,12 +4071,16 @@ static lean_object* l_Lean_Parser_Term_funBinder_quot_formatter___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optType_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_unreachable___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_panic; +static lean_object* l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__2; lean_object* l_Lean_Parser_numLit___elambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_funBinder_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sort_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_cdot___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__1; static lean_object* l_Lean_Parser_Term_falseVal_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__14; static lean_object* l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__3; @@ -3694,10 +4088,13 @@ static lean_object* l_Lean_Parser_Term_matchAlt___closed__4; static lean_object* l_Lean_Parser_Term_have___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_app; static lean_object* l_Lean_Parser_Term_depArrow_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_cdot_declRange___closed__6; static lean_object* l_Lean_Parser_Term_explicit_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_syntheticHole___closed__4; static lean_object* l_Lean_Parser_Term_proj_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Tactic_quotSeq___closed__3; static lean_object* l_Lean_Parser_Term_dotIdent___closed__5; static lean_object* l_Lean_Parser_Term_scoped___closed__5; @@ -3711,6 +4108,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_declRange__ static lean_object* l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__2; static lean_object* l_Lean_Parser_Term_noImplicitLambda___closed__4; static lean_object* l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInst_declRange(lean_object*); @@ -3721,6 +4119,7 @@ static lean_object* l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed_ static lean_object* l_Lean_Parser_Term_byTactic_x27_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_declRange(lean_object*); static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_match_formatter___closed__2; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__fun_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -3730,6 +4129,7 @@ static lean_object* l_Lean_Parser_Term_letMVar___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Term_sorry; static lean_object* l_Lean_Parser_Term_matchAlt_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_arrow_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_argument_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot(lean_object*); static lean_object* l_Lean_Parser_Term_syntheticHole___closed__8; @@ -3740,6 +4140,7 @@ static lean_object* l_Lean_Parser_Term_structInstLVal___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroArg_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAlt(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_letIdLhs_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sort_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_declRange___closed__2; @@ -3785,15 +4186,19 @@ static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__25; static lean_object* l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_char_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchAlt___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_letMVar_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_let__delayed_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__1; static lean_object* l_Lean_Parser_Term_namedArgument___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_attr_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Term_basicFun_formatter___closed__9; static lean_object* l_Lean_Parser_Term_binderDefault_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_depArrow_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_binderType___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__1; static lean_object* l_Lean_Parser_Term_fromTerm___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_optEllipsis_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_let__delayed___closed__3; static lean_object* l_Lean_Parser_Term_sort___closed__6; @@ -3806,6 +4211,7 @@ static lean_object* l_Lean_Parser_Term_cdot___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_structInstLVal___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_have___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_haveDecl_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_local___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___closed__6; @@ -3814,12 +4220,14 @@ static lean_object* l_Lean_Parser_Term_binop___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_sorry_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer___closed__8; lean_object* l_Lean_PrettyPrinter_Formatter_checkNoWsBefore_formatter___boxed(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__2; static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__23; static lean_object* l_Lean_Parser_Term_scoped___closed__6; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_declRange___closed__3; static lean_object* l_Lean_Parser_Term_tupleTail___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__17; LEAN_EXPORT lean_object* l_Lean_Parser_Level_quot; static lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_declRange___closed__4; @@ -3829,15 +4237,17 @@ static lean_object* l_Lean_Parser_Term_byTactic_parenthesizer___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_attrKind_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_funBinder_quot_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__2; lean_object* l_Lean_ppDedentIfGrouped_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_attr_quot___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__15; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_subst___closed__3; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_scoped___elambda__1___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_motive___closed__1; -static lean_object* l_Lean_Parser_Term_suffices_formatter___closed__8; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_let__fun_formatter___closed__4; static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__9; @@ -3854,6 +4264,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_declRange___clo static lean_object* l_Lean_Parser_Term_attrInstance___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_instBinder___closed__8; static lean_object* l_Lean_Parser_Term_funBinder_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_declRange___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_declRange___closed__4; static lean_object* l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__2; @@ -3881,7 +4292,6 @@ static lean_object* l_Lean_Parser_Term_forall___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dbgTrace___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_byTactic_x27_formatter___closed__1; -static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__11; static lean_object* l_Lean_Parser_Term_matchAlt___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_inaccessible_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_syntheticHole_formatter___closed__4; @@ -3893,13 +4303,14 @@ static lean_object* l_Lean_Parser_Term_let__fun_formatter___closed__1; static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_letrec_parenthesizer___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_num; +static lean_object* l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__1; static lean_object* l_Lean_Parser_Term_stateRefT_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_num_declRange___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__12; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__10; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__46; -static lean_object* l_Lean_Parser_Term_haveDecl_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Tactic_quotSeq___closed__5; static lean_object* l_Lean_Parser_Term_inaccessible___closed__7; static lean_object* l_Lean_Parser_Term_attrInstance___elambda__1___closed__8; @@ -3914,6 +4325,7 @@ static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__13; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_char_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__1; static lean_object* l_Lean_Parser_Term_let__fun___closed__10; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_attributes_parenthesizer___closed__4; @@ -3927,6 +4339,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Level_quot_declRange___closed__7; static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_unreachable_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__13; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_byTactic_x27; static lean_object* l_Lean_Parser_Term_inaccessible___closed__3; @@ -3936,6 +4349,8 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_declRange___c static lean_object* l_Lean_Parser_Term_motive_formatter___closed__7; static lean_object* l_Lean_Parser_Term_letIdLhs_formatter___closed__5; static lean_object* l_Lean_Parser_Term_funBinder_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letDecl_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_basicFun; static lean_object* l_Lean_Parser_Tactic_quot_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_sufficesDecl___closed__6; @@ -3950,6 +4365,7 @@ static lean_object* l_Lean_Parser_Term_forInMacro_x27_formatter___closed__4; static lean_object* l_Lean_Parser_Term_type_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_noindex___closed__3; static lean_object* l_Lean_Parser_Term_suffices___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_macroDollarArg___closed__2; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_hole___elambda__1___closed__2; @@ -3963,6 +4379,7 @@ static lean_object* l_Lean_Parser_Term_haveDecl_formatter___closed__3; static lean_object* l_Lean_Parser_Term_type_formatter___closed__11; static lean_object* l_Lean_Parser_Term_local___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_noindex___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letDecl_formatter___closed__5; static lean_object* l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroDollarArg; @@ -3988,8 +4405,10 @@ static lean_object* l_Lean_Parser_Term_let__tmp___closed__7; static lean_object* l_Lean_Parser_Term_suffices_formatter___closed__2; static lean_object* l_Lean_Parser_Term_haveIdDecl___closed__4; static lean_object* l_Lean_Parser_Term_syntheticHole___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType(lean_object*); static lean_object* l_Lean_Parser_Command_docComment_parenthesizer___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_prop___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_local_parenthesizer___closed__3; @@ -4000,17 +4419,21 @@ static lean_object* l_Lean_Parser_Term_letIdLhs___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_declRange___closed__5; lean_object* l_Lean_PrettyPrinter_Formatter_incQuotDepth_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__3; -static lean_object* l_Lean_Parser_Term_letDecl_parenthesizer___closed__9; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noindex_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_suffices_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_scientific_declRange___closed__1; static lean_object* l_Lean_Parser_Term_falseVal___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_matchAlt_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_depArrow___elambda__1___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_cdot_declRange___closed__1; static lean_object* l_Lean_Parser_Tactic_quot___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_match_declRange___closed__2; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_structInst___closed__13; @@ -4020,6 +4443,7 @@ static lean_object* l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__2; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_borrowed___closed__3; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__9; @@ -4031,17 +4455,16 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_declRange___close static lean_object* l_Lean_Parser_Term_depArrow___closed__6; static lean_object* l_Lean_Parser_Term_paren_formatter___closed__12; static lean_object* l_Lean_Parser_Term_sorry_parenthesizer___closed__2; -static lean_object* l_Lean_Parser_Term_attrKind_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_ellipsis_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_attributes___closed__1; static lean_object* l_Lean_Parser_Term_letIdLhs_parenthesizer___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forall_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_declRange___closed__7; static lean_object* l_Lean_Parser_Term_instBinder_formatter___closed__1; static lean_object* l_Lean_Parser_Term_assert___closed__3; static lean_object* l_Lean_Parser_Term_explicit___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_namedPattern___closed__1; static lean_object* l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__1; -static lean_object* l_Lean_Parser_Term_haveDecl_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_cdot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_assert___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__3; @@ -4049,6 +4472,7 @@ static lean_object* l_Lean_Parser_Term_match_formatter___closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_Term_ensureExpectedType_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__27; static lean_object* l_Lean_Parser_Term_ensureExpectedType___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__2; static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__10; static lean_object* l_Lean_Parser_Term_letDecl___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_subst_declRange___closed__7; @@ -4061,12 +4485,12 @@ static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___closed__8; static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_binderTactic_formatter___closed__2; static lean_object* l_Lean_Parser_Term_explicitBinder___closed__2; -static lean_object* l_Lean_Parser_Term_letDecl_parenthesizer___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_trailing__parser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__14; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__15; static lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_declRange___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_local_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_have___closed__1; static lean_object* l_Lean_Parser_darrow___closed__2; static lean_object* l_Lean_Parser_Term_typeSpec___closed__5; @@ -4078,14 +4502,15 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_scientific_declRange___close LEAN_EXPORT lean_object* l_Lean_Parser_Term_show___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_let__fun_parenthesizer___closed__3; -static lean_object* l_Lean_Parser_Term_letRecDecl_formatter___closed__8; static lean_object* l_Lean_Parser_Term_letRecDecl___elambda__1___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_declRange___closed__4; static lean_object* l_Lean_Parser_Term_type_parenthesizer___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__18; static lean_object* l_Lean_Parser_Term_letIdLhs_formatter___closed__7; static lean_object* l_Lean_Parser_Term_letrec___elambda__1___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_hole_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_local_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_instBinder___elambda__1___closed__3; @@ -4093,6 +4518,8 @@ static lean_object* l_Lean_Parser_Term_funBinder_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_funImplicitBinder___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_show(lean_object*); static lean_object* l_Lean_Parser_Term_typeSpec_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_binderTactic_formatter___closed__1; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___closed__1; @@ -4120,6 +4547,7 @@ static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___closed__8; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Term_basicFun_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderDefault_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_motive_formatter___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_declRange___closed__7; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___closed__11; @@ -4128,20 +4556,22 @@ lean_object* l_Lean_Parser_symbolInfo(lean_object*); static lean_object* l_Lean_Parser_Tactic_quot___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optIdent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_haveEqnsDecl___closed__6; -static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_explicit_formatter___closed__1; static lean_object* l_Lean_Parser_Term_match___closed__9; static lean_object* l_Lean_Parser_Term_tupleTail___closed__5; lean_object* l_Lean_Parser_charLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_hole_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__1; static lean_object* l_Lean_Parser_Term_generalizingParam___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_suffices_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__3; static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__5; static lean_object* l_Lean_Parser_Command_docComment___closed__10; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__19; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeq; +static lean_object* l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_namedArgument_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv(lean_object*); @@ -4165,36 +4595,44 @@ static lean_object* l_Lean_Parser_Term_str___closed__1; static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_fun___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Command_docComment; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_let__fun_formatter___closed__2; static lean_object* l_Lean_Parser_Term_argument_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_let__tmp___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer(lean_object*); lean_object* l_Lean_Parser_orelseFnCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_declRange___closed__6; -static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_explicitUniv___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_declRange___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_match(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_depArrow(lean_object*); static lean_object* l_Lean_Parser_Term_attrInstance___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_inaccessible___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_unreachable___elambda__1___closed__4; extern lean_object* l_Lean_Parser_epsilonInfo; static lean_object* l_Lean_Parser_Term_basicFun___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__2; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_funBinder_quot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_declRange___closed__5; static lean_object* l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_panic___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_fun_declRange___closed__4; static lean_object* l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_whereDecls_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__1; static lean_object* l_Lean_Parser_Term_have___closed__4; static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_hole___elambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___closed__8; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___closed__7; static lean_object* l_Lean_Parser_Term_pipeProj_formatter___closed__4; @@ -4203,6 +4641,7 @@ static lean_object* l_Lean_Parser_Term_pipeProj___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_anonymousCtor___closed__10; static lean_object* l_Lean_Parser_Term_num___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_scientific_declRange___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_declRange___closed__3; static lean_object* l_Lean_Parser_Term_fromTerm_formatter___closed__3; static lean_object* l_Lean_Parser_Term_haveIdLhs_formatter___closed__1; @@ -4227,14 +4666,15 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser(lean_ob static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__5; static lean_object* l_Lean_Parser_Term_letrec___closed__5; static lean_object* l_Lean_Parser_Term_let_parenthesizer___closed__6; -static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__16; static lean_object* l_Lean_Parser_Term_instBinder_formatter___closed__2; static lean_object* l_Lean_Parser_Term_let_formatter___closed__3; static lean_object* l_Lean_Parser_Term_matchAlt_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__10; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__26; static lean_object* l_Lean_Parser_Term_explicitUniv___closed__1; static lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__2; static lean_object* l_Lean_Parser_Term_dotIdent_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_quot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_typeAscription___closed__1; @@ -4243,7 +4683,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_declRange___closed_ static lean_object* l_Lean_Parser_Term_letRecDecl_formatter___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forInMacro___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_pipeCompletion___closed__1; -static lean_object* l_Lean_Parser_Term_letDecl_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1___closed__6; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_declRange(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_letDecl___elambda__1(lean_object*, lean_object*); @@ -4251,6 +4690,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_show_declRange___closed__5; static lean_object* l_Lean_Parser_Term_subst___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_haveIdDecl___closed__1; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__12; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_syntheticHole_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel(lean_object*); @@ -4261,6 +4701,7 @@ static lean_object* l_Lean_Parser_Term_letIdLhs___closed__4; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__9; static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_declRange___closed__1; static lean_object* l_Lean_Parser_Term_typeAscription_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__1; static lean_object* l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_hole___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letIdDecl_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -4294,6 +4735,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_declRange___closed_ static lean_object* l_Lean_Parser_Term_char_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_type; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binrel_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_structInstField___elambda__1___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_proj_declRange___closed__7; lean_object* l_Lean_PrettyPrinter_Formatter_pushNone_formatter___boxed(lean_object*); @@ -4301,10 +4743,11 @@ static lean_object* l_Lean_Parser_Term_binrel___closed__7; static lean_object* l_Lean_Parser_Term_pipeProj___closed__2; static lean_object* l_Lean_Parser_Term_letEqnsDecl_formatter___closed__3; static lean_object* l_Lean_Parser_Term_hole___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_quot_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Command_commentBody_parenthesizer(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_unreachable___elambda__1___closed__1; -static lean_object* l_Lean_Parser_Term_let_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__17; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__11; @@ -4316,15 +4759,17 @@ static lean_object* l_Lean_Parser_Term_subst___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_declRange___closed__6; static lean_object* l_Lean_Parser_Term_binderType___closed__4; static lean_object* l_Lean_Parser_Term_funImplicitBinder_parenthesizer___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__26; static lean_object* l_Lean_Parser_Term_falseVal_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_panic___closed__2; static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_let___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_attributes_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_haveIdDecl___closed__2; static lean_object* l_Lean_Parser_Term_letIdDecl_formatter___closed__6; static lean_object* l_Lean_Parser_Term_trueVal_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_declRange___closed__2; static lean_object* l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_declRange___closed__5; @@ -4343,7 +4788,9 @@ static lean_object* l_Lean_Parser_Term_scientific_formatter___closed__1; static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Term_show_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_have_declRange___closed__7; static lean_object* l_Lean_Parser_Term_macroDollarArg___closed__1; @@ -4357,34 +4804,43 @@ static lean_object* l_Lean_Parser_Term_typeAscription_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_depArrow_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_funImplicitBinder_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__2; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_implicitBinder_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_generalizingParam___closed__13; static lean_object* l_Lean_Parser_Term_fromTerm___closed__5; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__18; +static lean_object* l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_quotSeq___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dbgTrace_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_paren_declRange___closed__3; lean_object* l___private_Lean_Parser_Basic_0__Lean_Parser_rawAux(lean_object*, uint8_t, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__30; static lean_object* l_Lean_Parser_Term_trailing__parser_formatter___closed__6; static lean_object* l_Lean_Parser_Term_typeAscription_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letPatDecl_formatter___closed__4; static lean_object* l_Lean_Parser_Command_docComment_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Term_match_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_optSemicolon_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion(lean_object*); static lean_object* l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_declRange___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_declRange___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_declRange(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_declRange___closed__5; static lean_object* l_Lean_Parser_Term_attrInstance___elambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__5; static lean_object* l_Lean_Parser_Term_forall_parenthesizer___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letIdBinder___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_strictImplicitBinder_parenthesizer(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binderDefault___elambda__1___closed__1; @@ -4392,6 +4848,7 @@ static lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1; lean_object* l_Lean_Parser_withAntiquotSpliceAndSuffix(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_panic___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder___elambda__1___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_assert_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_basicFun___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfTypeMVar; @@ -4407,11 +4864,12 @@ static lean_object* l_Lean_Parser_Term_letIdDecl___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_binrel_declRange___closed__6; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_syntheticHole___elambda__1___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__5; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__28; static lean_object* l_Lean_Parser_Term_quotedName_formatter___closed__2; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_char; +static lean_object* l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__2; static lean_object* l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic___closed__1; static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__24; @@ -4419,6 +4877,7 @@ static lean_object* l_Lean_Parser_Term_structInstField___closed__5; lean_object* l_Lean_Parser_ident_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_arrow_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_dotIdent_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letIdDecl___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_scoped___closed__4; static lean_object* l_Lean_Parser_Term_letDecl_formatter___closed__7; @@ -4430,25 +4889,31 @@ static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__7; static lean_object* l_Lean_Parser_Term_panic___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_forall_declRange___closed__5; static lean_object* l_Lean_Parser_Term_have_parenthesizer___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__22; static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_sort_parenthesizer___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optType_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__1; static lean_object* l_Lean_Parser_Term_noImplicitLambda_formatter___closed__3; static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_fun_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_stateRefT_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_declRange___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_cdot_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_explicit_formatter___closed__3; static lean_object* l_Lean_Parser_Term_assert_formatter___closed__5; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__10; static lean_object* l_Lean_Parser_Tactic_seq1___closed__1; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___closed__3; static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_quot_parenthesizer(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_letPatDecl_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_declRange___closed__2; static lean_object* l_Lean_Parser_Term_letIdLhs_formatter___closed__1; static lean_object* l_Lean_Parser_Term_ellipsis_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__2; lean_object* l_Lean_Parser_levelParser_formatter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_syntheticHole___closed__3; static lean_object* l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__2; @@ -4458,8 +4923,11 @@ static lean_object* l_Lean_Parser_Term_showRhs___closed__1; static lean_object* l_Lean_Parser_Term_doubleQuotedName___closed__4; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___closed__6; static lean_object* l_Lean_Parser_Term_attributes_formatter___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__30; +static lean_object* l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__2; static lean_object* l_Lean_Parser_Term_subst___closed__2; static lean_object* l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_binrel___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_strictImplicitRightBracket; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__31; @@ -4470,17 +4938,19 @@ static lean_object* l_Lean_Parser_Term_typeOf_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_tupleTail_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstArrayRef; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__5; static lean_object* l_Lean_Parser_Term_dotIdent___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_sort_declRange___closed__7; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_assert(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_let__delayed___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_binop___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_declRange___closed__6; static lean_object* l_Lean_Parser_Term_typeAscription___closed__9; lean_object* l_Lean_Parser_sepBy1_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_leading__parser_formatter___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_let__tmp___closed__9; static lean_object* l_Lean_Parser_Term_explicit___elambda__1___closed__12; @@ -4489,6 +4959,7 @@ static lean_object* l_Lean_Parser_Term_subst___closed__1; static lean_object* l_Lean_Parser_Term_binderDefault___elambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_noindex_declRange___closed__3; static lean_object* l_Lean_Parser_Term_explicit___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_suffices___closed__5; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__13; @@ -4497,13 +4968,18 @@ static lean_object* l_Lean_Parser_Term_typeSpec___closed__4; static lean_object* l_Lean_Parser_Term_app___closed__6; static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_letRecDecl_formatter___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_noindex_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_declRange___closed__3; static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_declRange___closed__4; static lean_object* l_Lean_Parser_Term_binrel___closed__8; lean_object* l_Lean_Parser_numLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forall_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letIdDecl___elambda__1___closed__9; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_assert_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__6; @@ -4514,9 +4990,14 @@ static lean_object* l_Lean_Parser_Term_app___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_declRange___closed__4; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__3; static lean_object* l_Lean_Parser_Term_motive___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_have_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_unreachable_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__2; static lean_object* l_Lean_Parser_Term_panic_formatter___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__42; +static lean_object* l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__1; lean_object* l_Lean_Parser_levelParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_attrInstance_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchDiscr_quot; @@ -4530,8 +5011,12 @@ static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__1; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__1; static lean_object* l_Lean_Parser_Term_dotIdent_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__3; lean_object* l_Lean_ppSpace_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__15; @@ -4544,6 +5029,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_declRan LEAN_EXPORT lean_object* l_Lean_Parser_Term_arrow_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binderTactic_parenthesizer___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optSemicolon___elambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_declRange___closed__2; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_letIdDecl___closed__1; @@ -4557,27 +5043,33 @@ static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___clos static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_declRange___closed__2; static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_sorry___elambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_generalizingParam_formatter___closed__2; static lean_object* l_Lean_Parser_Term_matchAlt___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__33; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic(lean_object*); static lean_object* l_Lean_Parser_Term_parenSpecial___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__3; static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_tupleTail_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binderTactic___elambda__1___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_dotIdent___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_local___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_binop_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_unreachable___elambda__1___closed__8; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__22; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar___closed__7; static lean_object* l_Lean_Parser_Term_funBinder___closed__1; static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_binrel_formatter___closed__3; static lean_object* l_Lean_Parser_Term_type_formatter___closed__3; static lean_object* l_Lean_Parser_Term_binderDefault___elambda__1___closed__2; @@ -4591,12 +5083,13 @@ static lean_object* l_Lean_Parser_Term_ensureTypeOf_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optExprPrecedence; static lean_object* l_Lean_Parser_Term_panic___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_trailing__parser___closed__5; -static lean_object* l_Lean_Parser_Term_haveDecl_parenthesizer___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dotIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_subst_formatter___closed__3; static lean_object* l_Lean_Parser_Term_optExprPrecedence_formatter___closed__3; static lean_object* l_Lean_Parser_Term_hole_parenthesizer___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_declRange___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_darrow___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__10; @@ -4613,7 +5106,9 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_have_declRange(lean_obj static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_semicolonOrLinebreak; LEAN_EXPORT lean_object* l_Lean_Parser_Term_implicitBinder___boxed(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_matchDiscr_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_quot; static lean_object* l_Lean_Parser_Term_assert_formatter___closed__3; static lean_object* l_Lean_Parser_Term_binop__lazy___elambda__1___closed__6; @@ -4623,7 +5118,6 @@ static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___closed__1; static lean_object* l_Lean_Parser_Tactic_quot___closed__3; lean_object* l_Lean_Parser_nodeFn(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__16; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__42; static lean_object* l_Lean_Parser_Term_funBinder_formatter___closed__3; static lean_object* l_Lean_Parser_Term_typeSpec___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_declRange___closed__1; @@ -4643,18 +5137,21 @@ static lean_object* l_Lean_Parser_Term_generalizingParam_formatter___closed__8; static lean_object* l_Lean_Parser_Term_letIdLhs_formatter___closed__4; static lean_object* l_Lean_Parser_Term_namedArgument___closed__6; static lean_object* l_Lean_Parser_Command_docComment_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__1; static lean_object* l_Lean_Parser_Term_panic___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_local___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_funImplicitBinder_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__20; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__33; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_declRange(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_letPatDecl_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_falseVal___elambda__1(lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_declRange___closed__5; static lean_object* l_Lean_Parser_Term_typeAscription___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_byTactic___closed__3; static lean_object* l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__10; static lean_object* l___regBuiltin_Lean_Parser_Term_explicit_declRange___closed__1; @@ -4676,14 +5173,20 @@ static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__16; static lean_object* l_Lean_Parser_Term_basicFun_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_let__fun___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_app_declRange___closed__6; lean_object* l_Lean_Parser_nameLit_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_proj_parenthesizer___closed__2; static lean_object* l_Lean_Parser_semicolonOrLinebreak_formatter___closed__3; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__15; static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__18; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binderDefault_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_show_declRange___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__1; lean_object* l_Lean_Parser_unicodeSymbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__1; static lean_object* l_Lean_Parser_Term_panic___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_typeAscription_parenthesizer___closed__4; @@ -4696,47 +5199,54 @@ static lean_object* l_Lean_Parser_Term_letMVar___closed__8; static lean_object* l_Lean_Parser_Term_optIdent_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_let_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Tactic_quot___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_match_formatter___closed__1; static lean_object* l_Lean_Parser_Term_basicFun___closed__8; static lean_object* l_Lean_Parser_Term_suffices_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_instBinder___closed__4; static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__11; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__48; static lean_object* l_Lean_Parser_Term_local___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__3___boxed__const__1; static lean_object* l_Lean_Parser_Term_falseVal___closed__2; lean_object* l_Lean_Parser_rawIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_declRange___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_let__delayed___closed__5; static lean_object* l_Lean_Parser_Term_borrowed___closed__6; static lean_object* l_Lean_Parser_Term_binop___closed__5; static lean_object* l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_byTactic_parenthesizer___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_forall___closed__10; static lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_unreachable___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_matchAlt___closed__1; static lean_object* l_Lean_Parser_Term_doubleQuotedName___closed__2; static lean_object* l_Lean_Parser_Term_match_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letRecDecl___closed__3; static lean_object* l_Lean_Parser_Term_noImplicitLambda___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_tupleTail_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_declRange___closed__6; static lean_object* l_Lean_Parser_Term_trailing__parser___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_declRange___closed__3; static lean_object* l_Lean_Parser_Term_letRecDecl___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_assert_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_let_declRange___closed__3; extern lean_object* l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; +static lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchDiscr; static lean_object* l_Lean_Parser_Term_cdot___closed__7; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_prop_formatter___closed__2; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__14; +static lean_object* l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_assert___closed__7; static lean_object* l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__48; static lean_object* l_Lean_Parser_Term_depArrow_parenthesizer___closed__4; -static lean_object* l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_syntheticHole___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_cdot_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__2; @@ -4757,21 +5267,21 @@ static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___clos static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__16; static lean_object* l_Lean_Parser_Term_bracketedBinder___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___closed__6; -static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__20; static lean_object* l_Lean_Parser_Term_structInstField_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_attr_quot___closed__4; static lean_object* l_Lean_Parser_Term_basicFun_parenthesizer___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_sort_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_ellipsis___closed__6; static lean_object* l_Lean_Parser_Term_let__delayed_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_basicFun_formatter___closed__2; static lean_object* l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_let__fun___elambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_sort___elambda__1___closed__10; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_hole_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_type___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_attributes_formatter___closed__7; static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__2; @@ -4785,11 +5295,15 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_declRange___closed_ static lean_object* l_Lean_Parser_Level_quot___closed__6; static lean_object* l_Lean_Parser_Term_leading__parser_formatter___closed__7; lean_object* l_Lean_ppLine_formatter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__2; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_binop_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__1; static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_fun_declRange___closed__3; static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_motive___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_declRange___closed__7; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__4; @@ -4814,6 +5328,7 @@ static lean_object* l_Lean_Parser_Term_sorry___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__20; static lean_object* l_Lean_Parser_Term_binrel_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_attr_quot___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_binop___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__9; static lean_object* l_Lean_Parser_Tactic_quotSeq___closed__1; @@ -4825,6 +5340,7 @@ static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__4; static lean_object* l_Lean_Parser_Term_have___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doubleQuotedName_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_declRange___closed__4; static lean_object* l_Lean_Parser_Term_fun_parenthesizer___closed__2; @@ -4837,6 +5353,7 @@ static lean_object* l_Lean_Parser_Term_structInstField_parenthesizer___closed__1 LEAN_EXPORT lean_object* l_Lean_Parser_Term_syntheticHole___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___closed__5; static lean_object* l_Lean_Parser_Term_suffices_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_haveDecl___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_have_formatter___closed__4; @@ -4859,9 +5376,10 @@ static lean_object* l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_haveEqnsDecl___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_structInstArrayRef___closed__6; static lean_object* l_Lean_Parser_Term_letIdDecl___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_declRange___closed__4; static lean_object* l_Lean_Parser_Term_binop___elambda__1___closed__1; -static lean_object* l_Lean_Parser_Term_suffices_parenthesizer___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_hole_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_binderTactic___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_withAnonymousAntiquot; static lean_object* l_Lean_Parser_Term_macroDollarArg_formatter___closed__1; @@ -4877,6 +5395,7 @@ static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_ellipsis___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_motive_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter(lean_object*); lean_object* l_Lean_Parser_mkAntiquot(lean_object*, lean_object*, uint8_t, uint8_t); static lean_object* l_Lean_Parser_Term_funBinder___closed__2; static lean_object* l_Lean_Parser_Term_namedPattern_formatter___closed__5; @@ -4888,11 +5407,9 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_typeSpec_parenthesizer(lean_object*, static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__6; lean_object* l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__11; -static lean_object* l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_match_formatter___closed__10; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forInMacro_x27_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__13; static lean_object* l_Lean_Parser_Term_scientific___closed__1; static lean_object* l_Lean_Parser_Term_suffices_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__6; @@ -4902,15 +5419,14 @@ static lean_object* l_Lean_Parser_Term_dbgTrace___closed__10; static lean_object* l_Lean_Parser_Term_letRecDecls___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_declRange___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_explicit; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__41; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__22; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeq_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__13; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__45; static lean_object* l___regBuiltin_Lean_Parser_Term_have_declRange___closed__3; static lean_object* l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1; -static lean_object* l_Lean_Parser_Term_attrInstance_formatter___closed__6; static lean_object* l_Lean_Parser_Term_fun_formatter___closed__1; static lean_object* l_Lean_Parser_Term_let_parenthesizer___closed__5; lean_object* l_Lean_addBuiltinDocString(lean_object*, lean_object*, lean_object*); @@ -4919,22 +5435,24 @@ static lean_object* l_Lean_Parser_Term_nomatch___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_assert_formatter___closed__6; static lean_object* l_Lean_Parser_Term_paren_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_basicFun___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_noindex_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_attrInstance___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_declRange___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__23; static lean_object* l___regBuiltin_Lean_Parser_Term_suffices_declRange___closed__4; static lean_object* l_Lean_Parser_Term_typeAscription___closed__6; static lean_object* l_Lean_Parser_Term_panic_parenthesizer___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_declRange___closed__3; static lean_object* l_Lean_Parser_Term_byTactic_x27___closed__1; static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_namedPattern_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_attrKind___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_haveDecl___closed__6; static lean_object* l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__5; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__38; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__21; -static lean_object* l_Lean_Parser_Term_structInstField_parenthesizer___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__15; static lean_object* l_Lean_Parser_Term_matchAlt_formatter___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_declRange___closed__6; @@ -4956,18 +5474,18 @@ static lean_object* l_Lean_Parser_Term_pipeCompletion___closed__2; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__18; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__5; static lean_object* l_Lean_Parser_Tactic_seq1___closed__2; -static lean_object* l_Lean_Parser_Term_explicitBinder_formatter___closed__7; static lean_object* l_Lean_Parser_Term_byTactic___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optSemicolon_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_completion_declRange___closed__6; static lean_object* l_Lean_Parser_Term_strictImplicitBinder_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_structInstField___closed__3; static lean_object* l_Lean_Parser_Term_typeAscription___closed__8; static lean_object* l_Lean_Parser_Term_local___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__45; +static lean_object* l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__1; static lean_object* l_Lean_Parser_Term_macroDollarArg_formatter___closed__4; lean_object* l_Lean_Parser_many_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__1; static lean_object* l_Lean_Parser_Term_dbgTrace_formatter___closed__2; static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_byTactic___elambda__1___closed__16; @@ -4976,11 +5494,13 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_trueVal_parenthesizer(lean_object*, static lean_object* l___regBuiltin_Lean_Parser_Term_scientific_declRange___closed__3; static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_binrel___elambda__1___closed__7; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__13; static lean_object* l_Lean_Parser_Term_funBinder___closed__4; static lean_object* l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_leading__parser___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_declRange___closed__2; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__41; static lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_declRange___closed__1; static lean_object* l_Lean_Parser_Term_noindex___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_declRange___closed__2; @@ -4988,10 +5508,10 @@ static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_declRange___closed__7; static lean_object* l_Lean_Parser_Term_structInstArrayRef___closed__10; static lean_object* l_Lean_Parser_Term_let__delayed___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__1; static lean_object* l_Lean_Parser_Term_inaccessible_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_app_declRange___closed__3; static lean_object* l_Lean_Parser_Term_structInst_formatter___closed__10; -static lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_num_declRange___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_str_declRange___closed__3; static lean_object* l_Lean_Parser_Term_funBinder_quot___closed__3; @@ -5004,27 +5524,33 @@ static lean_object* l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_basicFun___closed__4; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_show_parenthesizer(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_letRecDecl___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_haveDecl___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_have___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__1; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_paren_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__38; static lean_object* l_Lean_Parser_Term_attrInstance___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_depArrow___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__15; lean_object* l_Lean_PrettyPrinter_Formatter_interpolatedStr_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__2; static lean_object* l_Lean_Parser_Term_typeSpec___elambda__1___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_declRange___closed__5; static lean_object* l_Lean_Parser_Term_letrec___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveIdDecl___elambda__1(lean_object*, lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__23; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__21; static lean_object* l_Lean_Parser_Term_falseVal___elambda__1___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_let__delayed_parenthesizer___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Command_commentBody_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_num_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_app_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_proj_formatter___closed__4; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_binderDefault___elambda__1___closed__6; @@ -5041,7 +5567,6 @@ static lean_object* l_Lean_Parser_Term_pipeProj_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_attr_quot___closed__9; static lean_object* l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_namedPattern___closed__2; -static lean_object* l_Lean_Parser_Term_attrKind_formatter___closed__6; static lean_object* l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letMVar___closed__4; @@ -5058,6 +5583,7 @@ static lean_object* l_Lean_Parser_Term_fun_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_optSemicolon_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binop__lazy_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_paren___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_explicitUniv___closed__11; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___closed__5; @@ -5070,17 +5596,19 @@ static lean_object* l_Lean_Parser_Term_namedArgument_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderDefault_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_binderDefault_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_match_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_macroLastArg___closed__3; static lean_object* l_Lean_Parser_Term_nomatch___closed__5; static lean_object* l_Lean_Parser_Term_fun___closed__2; static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__12; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ident(lean_object*); static lean_object* l_Lean_Parser_Term_subst___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__8; -static lean_object* l_Lean_Parser_Tactic_quotSeq_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_declRange___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_optEllipsis___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot(lean_object*); @@ -5090,18 +5618,21 @@ static lean_object* l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_local___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_paren_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_ident___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp(lean_object*); static lean_object* l_Lean_Parser_Term_falseVal___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letrec(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__1; static lean_object* l_Lean_Parser_Term_matchAlt_formatter___closed__3; static lean_object* l_Lean_Parser_Term_motive_formatter___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__delayed_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__46; static lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAltsWhereDecls; static lean_object* l_Lean_Parser_Term_matchAlts___elambda__1___closed__3; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__6; static lean_object* l_Lean_Parser_Term_show_formatter___closed__2; static lean_object* l_Lean_Parser_Term_type_parenthesizer___closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_basicFun_formatter(lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_notFollowedBy_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_subst___closed__7; static lean_object* l_Lean_Parser_Term_letMVar_parenthesizer___closed__5; @@ -5114,17 +5645,22 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_num_parenthesizer(lean_object*, lean static lean_object* l_Lean_Parser_Term_pipeProj___closed__10; static lean_object* l_Lean_Parser_Term_unreachable___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_char___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_binop_declRange___closed__2; static lean_object* l_Lean_Parser_Term_noindex_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__17; -static lean_object* l_Lean_Parser_Term_argument_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_prop_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_namedPattern_formatter___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_doubleQuotedName___closed__11; +static lean_object* l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_hole_declRange___closed__3; static lean_object* l_Lean_Parser_Term_sort___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_subst_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColGe_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_app___closed__2; @@ -5136,11 +5672,14 @@ static lean_object* l_Lean_Parser_Term_explicit___closed__5; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__1; static lean_object* l_Lean_Parser_Term_whereDecls_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_letrec___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_panic_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_formatter___closed__3; static lean_object* l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_declRange___closed__2; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__15; +static lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_byTactic_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__8; @@ -5152,11 +5691,13 @@ static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed_ static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__2; static lean_object* l_Lean_Parser_Term_trueVal_parenthesizer___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_scientific___elambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_attr_quot___closed__8; static lean_object* l_Lean_Parser_Term_binrel_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_funBinder_quot_formatter___closed__7; static lean_object* l_Lean_Parser_Term_typeOf___elambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__1; static lean_object* l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_quot___elambda__1___closed__10; lean_object* l_Lean_Parser_unicodeSymbolInfo(lean_object*, lean_object*); @@ -5173,6 +5714,7 @@ static lean_object* l_Lean_Parser_Term_doubleQuotedName_formatter___closed__3; static lean_object* l_Lean_Parser_Term_anonymousCtor_formatter___closed__7; static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__11; static lean_object* l_Lean_Parser_Term_borrowed___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_forInMacro_x27; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__25; static lean_object* l_Lean_Parser_Term_subst_parenthesizer___closed__3; @@ -5182,9 +5724,10 @@ static lean_object* l_Lean_Parser_Term_matchDiscr___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_funBinder_quot___closed__6; static lean_object* l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_type_formatter___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_tupleTail_formatter___closed__4; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__50; static lean_object* l_Lean_Parser_Term_dbgTrace___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_declRange___closed__1; @@ -5207,10 +5750,11 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_arrow_declRange___closed__4; static lean_object* l_Lean_Parser_Term_binrel__no__prop___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_cdot_declRange___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_declRange___closed__5; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__46; +static lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__1; static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_attr_quot___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__8; static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__11; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letIdLhs; @@ -5228,14 +5772,17 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_declRange___cl static lean_object* l_Lean_Parser_Term_dbgTrace___elambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_num___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__18; +static lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__2; static lean_object* l_Lean_Parser_Term_funBinder_formatter___closed__6; static lean_object* l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_sort___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_letDecl_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_stateRefT_formatter___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_declRange___closed__3; static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_inaccessible___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchDiscr___elambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAlts_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -5256,12 +5803,15 @@ static lean_object* l_Lean_Parser_Term_attributes___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_sufficesDecl___closed__4; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___closed__1; static lean_object* l_Lean_Parser_Term_noindex___elambda__1___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_structInstLVal_formatter___closed__6; static lean_object* l_Lean_Parser_Term_letDecl___closed__5; static lean_object* l_Lean_Parser_Term_letIdLhs_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_matchDiscr_formatter___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_letDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_let__fun___closed__11; @@ -5282,8 +5832,8 @@ lean_object* l_Lean_Parser_ParserState_mkUnexpectedError(lean_object*, lean_obje static lean_object* l_Lean_Parser_Term_inaccessible_formatter___closed__1; static lean_object* l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_binderTactic_formatter___closed__6; -static lean_object* l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_forInMacro___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_quot(lean_object*); static lean_object* l_Lean_Parser_Term_nomatch___closed__3; static lean_object* l_Lean_Parser_Term_argument___closed__4; @@ -5291,7 +5841,9 @@ lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColGt_parenthesizer___boxed static lean_object* l_Lean_Parser_Term_local___closed__7; static lean_object* l_Lean_Parser_Term_dbgTrace___closed__3; LEAN_EXPORT lean_object* l_Lean_Parser_Term_local_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_quotSeq_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__2; static lean_object* l_Lean_Parser_Term_ident_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__4; static lean_object* l_Lean_Parser_Term_quotedName_parenthesizer___closed__3; @@ -5299,6 +5851,7 @@ static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__22; static lean_object* l_Lean_Parser_Term_structInst___elambda__1___closed__27; static lean_object* l_Lean_Parser_Term_sufficesDecl_formatter___closed__7; static lean_object* l_Lean_Parser_Term_panic_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_trailing__parser___elambda__1___closed__13; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInst; @@ -5306,11 +5859,12 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_declRang lean_object* l_Lean_Parser_symbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_declRange___closed__2; static lean_object* l_Lean_Parser_Term_letEqnsDecl___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__tmp___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchAlt_formatter___closed__5; static lean_object* l_Lean_Parser_Term_let__fun_parenthesizer___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_declRange___closed__2; -static lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__2; static lean_object* l_Lean_Parser_Term_show___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_letMVar___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_match___elambda__1(lean_object*, lean_object*); @@ -5325,9 +5879,11 @@ static lean_object* l_Lean_Parser_Term_ensureTypeOf___closed__6; static lean_object* l_Lean_Parser_Term_let__fun___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_optEllipsis___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letIdBinder_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_letRecDecl___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__2; static lean_object* l_Lean_Parser_Term_noindex_formatter___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_paren_declRange___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_declRange___closed__2; @@ -5345,9 +5901,12 @@ static lean_object* l_Lean_Parser_Term_byTactic_x27___closed__5; static lean_object* l_Lean_Parser_Term_binrel_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_generalizingParam___closed__8; static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2; static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__19; static lean_object* l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__8; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_formatter(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_trailing__parser_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Command_docComment_parenthesizer___closed__6; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__8; @@ -5363,9 +5922,8 @@ static lean_object* l_Lean_Parser_Term_show_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_trueVal___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_sorry_declRange___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_63_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806_(lean_object*); static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__4; -static lean_object* l_Lean_Parser_Term_parenSpecial_formatter___closed__3; static lean_object* l_Lean_Parser_Term_noindex___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_typeAscription___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_doubleQuotedName___closed__7; @@ -5375,9 +5933,9 @@ static lean_object* l_Lean_Parser_Term_binop___elambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Parser_Term_binrel_declRange___closed__3; static lean_object* l_Lean_Parser_Term_dotIdent___elambda__1___closed__3; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_match_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_let__fun_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_doubleQuotedName_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_letDecl___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_ellipsis___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__3; @@ -5385,11 +5943,14 @@ static lean_object* l_Lean_Parser_Term_depArrow_formatter___closed__5; static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__9; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dbgTrace_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_binop__lazy; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_tupleTail_formatter___closed__1; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_matchAlt___closed__6; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_suffices_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveIdDecl; LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroLastArg_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_ensureTypeOf___closed__5; @@ -5412,6 +5973,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_declRange static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__4; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj(lean_object*); static lean_object* l_Lean_Parser_Term_binderDefault___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeAscription_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_cdot___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_borrowed___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_leading__parser_formatter___closed__1; @@ -5437,15 +5999,17 @@ static lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_declRange___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_subst_declRange___closed__6; static lean_object* l_Lean_Parser_Term_byTactic___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_attrKind___closed__5; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_type_parenthesizer(lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___closed__5; static lean_object* l_Lean_Parser_Term_letDecl___closed__3; static lean_object* l_Lean_Parser_Term_motive___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__8; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__9; -static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__22; static lean_object* l_Lean_Parser_Term_letrec_formatter___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop_formatter(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Level_quot_declRange___closed__6; static lean_object* l_Lean_Parser_Term_match___closed__10; lean_object* l_Lean_Parser_symbol_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -5454,9 +6018,11 @@ static lean_object* l_Lean_Parser_Term_forInMacro_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__19; static lean_object* l_Lean_Parser_Term_haveIdLhs___elambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__2; static lean_object* l_Lean_Parser_Term_whereDecls_parenthesizer___closed__7; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_63____closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_proj_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_attrInstance___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_generalizingParam; @@ -5479,7 +6045,9 @@ static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__3; static lean_object* l_Lean_Parser_Term_syntheticHole___elambda__1___closed__13; static lean_object* l_Lean_Parser_Term_sufficesDecl_formatter___closed__4; static lean_object* l_Lean_Parser_Term_tupleTail_parenthesizer___closed__4; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_ident_declRange___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__2; static lean_object* l_Lean_Parser_Term_namedPattern_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroLastArg_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_num_declRange(lean_object*); @@ -5498,8 +6066,8 @@ static lean_object* l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__4; lean_object* l_Lean_Parser_nameLit_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_formatter___closed__6; static lean_object* l_Lean_Parser_Term_namedArgument___closed__9; +static lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__2; static lean_object* l_Lean_Parser_Term_suffices___closed__6; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__29; static lean_object* l_Lean_Parser_Term_fun_formatter___closed__4; lean_object* l_Lean_PrettyPrinter_Formatter_withoutPosition_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); @@ -5513,6 +6081,7 @@ static lean_object* l_Lean_Parser_Tactic_tacticSeqBracketed___closed__11; static lean_object* l_Lean_Parser_Term_arrow___closed__3; static lean_object* l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__6; static lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_declRange___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_tupleTail_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_funBinder___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_fromTerm___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__3; @@ -5520,12 +6089,15 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar(lean_obj static lean_object* l_Lean_Parser_Term_binrel_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_match___closed__12; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_quotSeq___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__1; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__8; static lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_declRange___closed__7; static lean_object* l_Lean_Parser_Term_cdot_formatter___closed__5; static lean_object* l_Lean_Parser_Term_binderTactic___closed__3; static lean_object* l_Lean_Parser_Term_scoped_formatter___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_depArrow_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_letMVar___closed__3; static lean_object* l___regBuiltin_Lean_Parser_Term_match_declRange___closed__1; static lean_object* l_Lean_Parser_Term_sort___closed__7; @@ -5533,6 +6105,7 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_paren_declRange___closed__6; static lean_object* l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_ident___closed__1; static lean_object* l___regBuiltin_Lean_Parser_Term_subst_declRange___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__2; static lean_object* l_Lean_Parser_Term_fromTerm___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_namedPattern_formatter___closed__6; @@ -5546,8 +6119,8 @@ static lean_object* l_Lean_Parser_Term_ensureExpectedType___closed__6; static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__9; static lean_object* l_Lean_Parser_Term_type_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Term_str_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__1; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel_declRange(lean_object*); -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__16; static lean_object* l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_dotIdent___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_binderDefault___closed__5; @@ -5556,10 +6129,11 @@ static lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_proj_declRange___closed__4; static lean_object* l_Lean_Parser_Term_attrKind___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_structInstField___closed__7; +static lean_object* l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__2; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__14; LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstField_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_proj_formatter(lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_optIdent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_match_formatter___closed__16; static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__2; lean_object* l_Lean_Parser_unicodeSymbolFnAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_paren_formatter___closed__7; @@ -5567,7 +6141,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_declRange__ static lean_object* l_Lean_Parser_Term_have_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_haveIdDecl___closed__6; static lean_object* l_Lean_Parser_Term_letPatDecl___elambda__1___closed__10; -static lean_object* l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__12; static lean_object* l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_falseVal___elambda__1___closed__6; static lean_object* l_Lean_Parser_Term_hole___elambda__1___closed__11; @@ -5576,6 +6149,7 @@ static lean_object* l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__5; static lean_object* l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__3; static lean_object* l_Lean_Parser_Term_ensureExpectedType_formatter___closed__1; static lean_object* l_Lean_Parser_Term_letMVar___elambda__1___closed__6; +static lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__2; static lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_declRange___closed__6; static lean_object* l_Lean_Parser_Term_stateRefT___elambda__1___closed__9; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop_declRange(lean_object*); @@ -5583,8 +6157,11 @@ static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___close static lean_object* l_Lean_Parser_Term_sufficesDecl___closed__1; static lean_object* l_Lean_Parser_Term_letrec_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_paren___elambda__1___closed__14; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer(lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_forall___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_local___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__29; static lean_object* l_Lean_Parser_Level_quot_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_binop__lazy_formatter___closed__3; static lean_object* l_Lean_Parser_Term_basicFun_parenthesizer___closed__6; @@ -5599,6 +6176,7 @@ lean_object* l_Lean_Parser_checkColGtFn___boxed(lean_object*, lean_object*, lean LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_show_declRange(lean_object*); static lean_object* l_Lean_Parser_Term_namedArgument___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_semicolonOrLinebreak___elambda__1(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__1; static lean_object* l_Lean_Parser_Term_forInMacro_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__5; lean_object* l_Lean_Parser_rawIdent___elambda__1(lean_object*, lean_object*); @@ -5617,6 +6195,7 @@ static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___clos static lean_object* l___regBuiltin_Lean_Parser_Term_completion_declRange___closed__2; static lean_object* l_Lean_Parser_Term_let__fun_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_motive___closed__4; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__28; static lean_object* l_Lean_Parser_Term_fun___elambda__1___closed__20; static lean_object* l_Lean_Parser_Term_withAnonymousAntiquot___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_Term_trueVal; @@ -5634,28 +6213,31 @@ static lean_object* l_Lean_Parser_Level_quot___elambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__fun___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_Formatter_andthen_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_declRange___closed__7; -static lean_object* l_Lean_Parser_Term_optType_formatter___closed__1; static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__1; static lean_object* l_Lean_Parser_Term_forall_formatter___closed__9; static lean_object* l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_letIdLhs_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_whereDecls___elambda__1___closed__21; static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_binop__lazy___closed__3; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__14; static lean_object* l_Lean_Parser_Term_noindex_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__2; static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__5; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let; static lean_object* l_Lean_Parser_Term_type___elambda__1___closed__25; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_bracketedBinder___boxed(lean_object*); static lean_object* l_Lean_Parser_Term_depArrow___closed__3; static lean_object* l_Lean_Parser_Term_funImplicitBinder_formatter___closed__2; static lean_object* l_Lean_Parser_Term_sufficesDecl___closed__8; LEAN_EXPORT lean_object* l_Lean_Parser_Term_strictImplicitLeftBracket; static lean_object* l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer(lean_object*); static lean_object* l_Lean_Parser_Term_structInstLVal___elambda__1___closed__22; static lean_object* l_Lean_Parser_Tactic_quotSeq_formatter___closed__1; -static lean_object* l_Lean_Parser_Term_fun_parenthesizer___closed__7; static lean_object* l___regBuiltin_Lean_Parser_Term_match_declRange___closed__5; static lean_object* l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_basicFun___elambda__1___closed__11; @@ -5664,7 +6246,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Level_quot_parenthesizer(lean_object*, le lean_object* l_Lean_Parser_ppDedent_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_doubleQuotedName_formatter___closed__6; static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___closed__2; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__49; static lean_object* l_Lean_Parser_Term_funImplicitBinder___closed__6; static lean_object* l_Lean_Parser_Term_typeOf___closed__6; static lean_object* l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__8; @@ -5673,7 +6254,6 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_declRange___c static lean_object* l___regBuiltin_Lean_Parser_Term_char_declRange___closed__4; static lean_object* l_Lean_Parser_Term_letRecDecl___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_dbgTrace___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Parser_Term_match_formatter___closed__15; static lean_object* l_Lean_Parser_Command_docComment_formatter___closed__6; static lean_object* l_Lean_Parser_Term_forall___closed__6; static lean_object* l_Lean_Parser_Tactic_tacticSeq___closed__6; @@ -5696,7 +6276,6 @@ static lean_object* l_Lean_Parser_Term_let__delayed_parenthesizer___closed__5; static lean_object* l_Lean_Parser_Term_cdot_formatter___closed__3; static lean_object* l_Lean_Parser_Term_cdot_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_matchDiscr_quot___closed__5; -static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__14; LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_quot___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__14; static lean_object* l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__8; @@ -5717,8 +6296,12 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letrec_parenthesizer(lean_object*, l static lean_object* l_Lean_Parser_Term_let__delayed_parenthesizer___closed__3; static lean_object* l_Lean_Parser_Term_attrInstance_formatter___closed__5; static lean_object* l_Lean_Parser_Term_fromTerm_formatter___closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_show_formatter(lean_object*); static lean_object* l_Lean_Parser_Term_inaccessible_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__1; static lean_object* l_Lean_Parser_Term_ellipsis___elambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_match___elambda__1___closed__13; lean_object* l_Lean_Parser_termParser_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__5; @@ -5729,9 +6312,11 @@ static lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_declRange___closed_ LEAN_EXPORT lean_object* l_Lean_Parser_Term_whereDecls_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_Term_prop___elambda__1(lean_object*, lean_object*); static lean_object* l_Lean_Parser_semicolonOrLinebreak___elambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__1; lean_object* l_Lean_ppDedent_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_num_declRange___closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_Term_ident; +static lean_object* l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__1; static lean_object* l_Lean_Parser_Term_inaccessible___elambda__1___closed__4; static lean_object* l_Lean_Parser_Term_borrowed___closed__1; static lean_object* l_Lean_Parser_Term_suffices___closed__3; @@ -5739,11 +6324,13 @@ static lean_object* l_Lean_Parser_Command_docComment___elambda__1___closed__10; static lean_object* l_Lean_Parser_Term_leading__parser___elambda__1___closed__15; static lean_object* l_Lean_Parser_Term_explicit___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_prop___elambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_attr_quot_formatter___closed__4; static lean_object* l_Lean_Parser_Term_app___closed__3; static lean_object* l_Lean_Parser_Term_structInstLVal_formatter___closed__3; static lean_object* l_Lean_Parser_Tactic_quotSeq___closed__8; static lean_object* l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_Parser_Term_letrec; static lean_object* l_Lean_Parser_Term_structInst_parenthesizer___closed__16; static lean_object* l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__3; @@ -5755,6 +6342,7 @@ static lean_object* l_Lean_Parser_Term_funImplicitBinder_formatter___closed__4; static lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__9; static lean_object* l_Lean_Parser_Term_ident___closed__2; static lean_object* l_Lean_Parser_Term_binderTactic___closed__5; +static lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1; LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__tmp; static lean_object* l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__3; @@ -5763,13 +6351,16 @@ static lean_object* l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__11 lean_object* l_Lean_PrettyPrinter_Parenthesizer_node_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2; static lean_object* l_Lean_Parser_Term_binrel_formatter___closed__7; -static lean_object* l_Lean_Parser_Term_match_formatter___closed__14; static lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_declRange___closed__3; +static lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__2; static lean_object* l_Lean_Parser_Term_strictImplicitRightBracket___elambda__1___closed__5; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__49; static lean_object* l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__1; +static lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__2; static lean_object* l_Lean_Parser_Term_explicitBinder_formatter___closed__5; static lean_object* l_Lean_Parser_Term_namedArgument_formatter___closed__3; static lean_object* l_Lean_Parser_Term_argument___closed__2; +static lean_object* l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__1; static lean_object* l_Lean_Parser_Term_letrec_formatter___closed__8; static lean_object* l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__4; static lean_object* l___regBuiltin_Lean_Parser_Term_binop_declRange___closed__6; @@ -5798,7 +6389,9 @@ lean_object* l_Lean_Parser_andthenFn(lean_object*, lean_object*, lean_object*, l static lean_object* l_Lean_Parser_Term_haveEqnsDecl___elambda__1___closed__7; static lean_object* l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__7; static lean_object* l_Lean_Parser_Term_ellipsis_parenthesizer___closed__1; +static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__16; static lean_object* l___regBuiltin_Lean_Parser_Term_subst_declRange___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer(lean_object*); static lean_object* l___regBuiltin_Lean_Parser_Term_type_declRange___closed__6; LEAN_EXPORT lean_object* l_Lean_Parser_Term_syntheticHole; static lean_object* l_Lean_Parser_Term_basicFun_formatter___closed__6; @@ -8931,6 +9524,52 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("formatter", 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_formatterAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeqBracketed_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1() { _start: { @@ -8983,6 +9622,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeq1Indented_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__4; +x_4 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__1() { _start: { @@ -9004,38 +9673,22 @@ return x_7; static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeqBracketed_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeq1Indented_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_tacticSeq_formatter___closed__2; -x_2 = l_Lean_Parser_Tactic_tacticSeq_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Tactic_tacticSeq_formatter___closed__4; +x_3 = l_Lean_Parser_Tactic_tacticSeq_formatter___closed__2; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -9048,11 +9701,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeq_formatter(lean_object* x { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Tactic_tacticSeq_formatter___closed__1; -x_7 = l_Lean_Parser_Tactic_tacticSeq_formatter___closed__5; +x_7 = l_Lean_Parser_Tactic_tacticSeq_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeq_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__1() { _start: { @@ -9084,24 +9767,16 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeq_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_byTactic_formatter___closed__2; -x_2 = l_Lean_Parser_Term_byTactic_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__4() { _start: { lean_object* x_1; @@ -9109,25 +9784,25 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppAllowUngrouped_formatter___boxed), 1, return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_byTactic_formatter___closed__5; -x_2 = l_Lean_Parser_Term_byTactic_formatter___closed__4; +x_1 = l_Lean_Parser_Term_byTactic_formatter___closed__4; +x_2 = l_Lean_Parser_Term_byTactic_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_byTactic_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_byTactic___elambda__1___closed__4; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_byTactic_formatter___closed__6; +x_3 = l_Lean_Parser_Term_byTactic_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -9140,11 +9815,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_byTactic_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_byTactic_formatter___closed__1; -x_7 = l_Lean_Parser_Term_byTactic_formatter___closed__7; +x_7 = l_Lean_Parser_Term_byTactic_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_byTactic___elambda__1___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_byTactic_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_byTactic___elambda__1___closed__4; +x_4 = l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_tacticParser_parenthesizer(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: { @@ -9344,6 +10049,52 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("parenthesizer", 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PrettyPrinter_parenthesizerAttribute; +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_tacticSeqBracketed___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2; +x_5 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__4; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1() { _start: { @@ -9396,6 +10147,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_tacticSeq1Indented___elambda__1___closed__4; +x_4 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1() { _start: { @@ -9417,38 +10198,22 @@ return x_7; static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__4; +x_3 = l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -9461,11 +10226,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_tacticSeq_parenthesizer(lean_objec { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__5; +x_7 = l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__3; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeq_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_tacticSeq___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__1() { _start: { @@ -9497,24 +10292,16 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_tacticSeq_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__4() { _start: { lean_object* x_1; @@ -9522,25 +10309,25 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppAllowUngrouped_parenthesizer___ return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_byTactic___elambda__1___closed__4; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__6; +x_3 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -9553,11 +10340,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_byTactic_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__7; +x_7 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_byTactic___elambda__1___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_byTactic_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_byTactic___elambda__1___closed__4; +x_4 = l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__1() { _start: { @@ -11920,6 +12737,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_type_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_type___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_type_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_type_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_type_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_type___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_type_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_type_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_type_parenthesizer___closed__1() { _start: { @@ -12066,6 +12913,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_type___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_type_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_type_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_type___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_sort___elambda__1___closed__1() { _start: { @@ -12646,6 +13523,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_sort___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_sort_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sort_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_sort___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_sort_parenthesizer___closed__1() { _start: { @@ -12710,6 +13617,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_sort___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_sort_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sort_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_sort___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_prop___elambda__1___closed__1() { _start: { @@ -13181,6 +14118,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_prop___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_prop_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prop_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_prop___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_prop_parenthesizer___closed__1() { _start: { @@ -13233,6 +14200,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_prop___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_prop_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_prop_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_prop___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_hole___elambda__1___closed__1() { _start: { @@ -13704,6 +14701,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_hole___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_hole_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_hole_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_hole___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_hole_parenthesizer___closed__1() { _start: { @@ -13756,6 +14783,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_hole___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_hole_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_hole_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_hole___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_syntheticHole___elambda__1___closed__1() { _start: { @@ -14332,42 +15389,34 @@ return x_1; static lean_object* _init_l_Lean_Parser_Term_syntheticHole_formatter___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_hole_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_syntheticHole_formatter___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_syntheticHole_formatter___closed__3; -x_2 = l_Lean_Parser_Term_syntheticHole_formatter___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_syntheticHole_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_syntheticHole_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_syntheticHole_formatter___closed__2; -x_2 = l_Lean_Parser_Term_syntheticHole_formatter___closed__5; +x_2 = l_Lean_Parser_Term_syntheticHole_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_syntheticHole_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_syntheticHole_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_syntheticHole___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_syntheticHole_formatter___closed__6; +x_3 = l_Lean_Parser_Term_syntheticHole_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -14380,11 +15429,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_syntheticHole_formatter(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_syntheticHole_formatter___closed__1; -x_7 = l_Lean_Parser_Term_syntheticHole_formatter___closed__7; +x_7 = l_Lean_Parser_Term_syntheticHole_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_syntheticHole___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_syntheticHole_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_syntheticHole___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1() { _start: { @@ -14424,42 +15503,34 @@ return x_1; static lean_object* _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_hole_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__4; +x_2 = l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_syntheticHole___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__6; +x_3 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -14472,11 +15543,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_syntheticHole_parenthesizer(lean_obj { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__7; +x_7 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_syntheticHole___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_syntheticHole_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_syntheticHole___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_sorry___elambda__1___closed__1() { _start: { @@ -14940,6 +16041,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_sorry___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_sorry_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sorry_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_sorry___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_sorry_parenthesizer___closed__1() { _start: { @@ -14992,6 +16123,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_sorry___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_sorry_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_sorry___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_cdot___elambda__1___closed__1() { _start: { @@ -15488,6 +16649,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_cdot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_cdot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_cdot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_cdot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_cdot_parenthesizer___closed__1() { _start: { @@ -15562,6 +16753,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_cdot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_cdot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_cdot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_typeAscription___elambda__1___closed__1() { _start: { @@ -17255,6 +18476,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_tupleTail_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_tupleTail_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_typeAscription_formatter___closed__1() { _start: { @@ -17319,15 +18570,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_parenSpecial_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_tupleTail_formatter), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_typeAscription___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_parenSpecial_formatter___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__2() { _start: { lean_object* x_1; @@ -17335,12 +18588,24 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_typeAscription_formatter), 5 return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_parenSpecial_formatter___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeAscription_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_typeAscription___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Term_parenSpecial_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_parenSpecial_formatter___closed__1; -x_2 = l_Lean_Parser_Term_parenSpecial_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -17351,7 +18616,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_parenSpecial_formatter(lean_object* _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Term_parenSpecial_formatter___closed__3; +x_6 = l_Lean_Parser_Term_parenSpecial_formatter___closed__1; x_7 = l_Lean_Parser_optional_formatter(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -17502,6 +18767,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_paren___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_paren_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_paren_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_paren___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_tupleTail_parenthesizer___closed__1() { _start: { @@ -17593,6 +18888,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_tupleTail_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_typeAscription_parenthesizer___closed__1() { _start: { @@ -17657,15 +18982,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_tupleTail_parenthesizer), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_typeAscription___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -17673,12 +19000,24 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_typeAscription_parenthesizer return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_typeAscription___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__1; -x_2 = l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -17689,7 +19028,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_parenSpecial_parenthesizer(lean_obje _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__3; +x_6 = l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__1; x_7 = l_Lean_Parser_optional_parenthesizer(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -17840,6 +19179,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_paren___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_paren_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_paren_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_paren___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__1() { _start: { @@ -18574,6 +19943,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_anonymousCtor_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1() { _start: { @@ -18677,6 +20076,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_anonymousCtor_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_optIdent___closed__1() { _start: { @@ -20330,6 +21759,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_fromTerm___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_fromTerm_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fromTerm_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_fromTerm___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_byTactic_x27_formatter___closed__1() { _start: { @@ -20354,7 +21813,7 @@ static lean_object* _init_l_Lean_Parser_Term_byTactic_x27_formatter___closed__2( lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_byTactic_formatter___closed__4; +x_3 = l_Lean_Parser_Term_byTactic_formatter___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -20372,15 +21831,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_showRhs_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_fromTerm_formatter), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_showRhs_formatter___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__2() { _start: { lean_object* x_1; @@ -20388,12 +21849,24 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_byTactic_x27_formatter), 5, return x_1; } } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_showRhs_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Term_showRhs_formatter___closed__1; -x_7 = l_Lean_Parser_Term_showRhs_formatter___closed__2; +x_6 = l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__2; +x_7 = l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__2; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -20500,6 +21973,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_sufficesDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_semicolonOrLinebreak_formatter___closed__1() { _start: { @@ -20593,34 +22096,26 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_sufficesDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_suffices_formatter___closed__2; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_suffices_formatter___closed__4; +x_1 = l_Lean_Parser_Term_suffices_formatter___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withPosition_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -20630,25 +22125,25 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_suffices_formatter___closed__5; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_1 = l_Lean_Parser_Term_suffices_formatter___closed__4; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_suffices_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_suffices___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_suffices_formatter___closed__7; +x_3 = l_Lean_Parser_Term_suffices_formatter___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -20661,11 +22156,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_suffices_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_suffices_formatter___closed__1; -x_7 = l_Lean_Parser_Term_suffices_formatter___closed__8; +x_7 = l_Lean_Parser_Term_suffices_formatter___closed__7; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_suffices___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_suffices_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_suffices_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_suffices___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_optIdent_parenthesizer___closed__1() { _start: { @@ -20761,6 +22286,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_fromTerm___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_fromTerm_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_fromTerm___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1() { _start: { @@ -20785,7 +22340,7 @@ static lean_object* _init_l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__4; +x_3 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -20803,15 +22358,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_showRhs_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_fromTerm_parenthesizer), 5, 0); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_showRhs_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -20819,12 +22376,24 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_byTactic_x27_parenthesizer), return x_1; } } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_showRhs_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Term_showRhs_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_showRhs_parenthesizer___closed__2; +x_6 = l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__2; +x_7 = l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2; x_8 = l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -20931,6 +22500,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_sufficesDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_sufficesDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_semicolonOrLinebreak_parenthesizer___closed__1() { _start: { @@ -21021,34 +22620,26 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_sufficesDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_suffices_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_suffices_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_suffices_parenthesizer___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; @@ -21058,25 +22649,25 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_suffices_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_suffices___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_suffices_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -21089,11 +22680,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_suffices_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_suffices_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_suffices_parenthesizer___closed__8; +x_7 = l_Lean_Parser_Term_suffices_parenthesizer___closed__7; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_suffices___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_suffices_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_suffices___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_show___elambda__1___closed__1() { _start: { @@ -21657,6 +23278,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_show_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_show___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_show_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_show_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_show_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_show___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_show_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_show_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_show_parenthesizer___closed__1() { _start: { @@ -21721,6 +23372,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_show___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_show_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_show_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_show___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__1() { _start: { @@ -24899,6 +26580,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstFieldAbbrev_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInstArrayRef_formatter___closed__1() { _start: { @@ -24975,6 +26686,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstArrayRef_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__1() { _start: { @@ -25004,36 +26745,28 @@ return x_1; static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstArrayRef_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__2; -x_2 = l_Lean_Parser_Term_structInstLVal_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_syntheticHole_formatter___closed__3; -x_2 = l_Lean_Parser_Term_structInstLVal_formatter___closed__4; +x_2 = l_Lean_Parser_Term_structInstLVal_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -25045,69 +26778,69 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_cdot_formatter___closed__3; -x_2 = l_Lean_Parser_Term_structInstLVal_formatter___closed__6; +x_2 = l_Lean_Parser_Term_structInstLVal_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__7; +x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_group_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__8; -x_2 = l_Lean_Parser_Term_structInstLVal_formatter___closed__3; +x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__7; +x_2 = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__9; +x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__8; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__5; -x_2 = l_Lean_Parser_Term_structInstLVal_formatter___closed__10; +x_1 = l_Lean_Parser_Term_structInstLVal_formatter___closed__4; +x_2 = l_Lean_Parser_Term_structInstLVal_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_structInstLVal___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_structInstLVal_formatter___closed__11; +x_3 = l_Lean_Parser_Term_structInstLVal_formatter___closed__10; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -25120,11 +26853,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstLVal_formatter(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_structInstLVal_formatter___closed__1; -x_7 = l_Lean_Parser_Term_structInstLVal_formatter___closed__12; +x_7 = l_Lean_Parser_Term_structInstLVal_formatter___closed__11; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_structInstLVal___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstLVal_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_structInstLVal___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInstField_formatter___closed__1() { _start: { @@ -25168,16 +26931,8 @@ return x_3; static lean_object* _init_l_Lean_Parser_Term_structInstField_formatter___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstLVal_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_structInstField_formatter___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInstField_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__2; x_2 = l_Lean_Parser_Term_structInstField_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -25185,13 +26940,13 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstField_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_structInstField_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_structInstField___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_structInstField_formatter___closed__5; +x_3 = l_Lean_Parser_Term_structInstField_formatter___closed__4; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -25199,12 +26954,12 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Term_structInstField_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_structInstField_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInstField_formatter___closed__1; -x_2 = l_Lean_Parser_Term_structInstField_formatter___closed__6; +x_2 = l_Lean_Parser_Term_structInstField_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withAntiquot_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -25215,7 +26970,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstField_formatter(lean_objec _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Term_structInstField_formatter___closed__7; +x_6 = l_Lean_Parser_Term_structInstField_formatter___closed__6; x_7 = l_Lean_Parser_ppGroup_formatter(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -25282,6 +27037,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_optEllipsis___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_optEllipsis_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_optEllipsis___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__1() { _start: { @@ -25346,35 +27131,27 @@ static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__6() _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstFieldAbbrev_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__7() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstField_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_formatter___closed__6; -x_2 = l_Lean_Parser_Term_structInst_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__2; +x_2 = l_Lean_Parser_Term_structInst_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Parser_Term_structInst_formatter___closed__8; +x_1 = l_Lean_Parser_Term_structInst_formatter___closed__7; x_2 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__4; x_3 = l_Lean_Parser_Term_tupleTail_formatter___closed__2; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_sepByIndent_formatter___boxed), 8, 3); @@ -25384,7 +27161,7 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; @@ -25394,7 +27171,7 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; @@ -25404,63 +27181,55 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_formatter___closed__10; -x_2 = l_Lean_Parser_Term_structInst_formatter___closed__11; +x_1 = l_Lean_Parser_Term_structInst_formatter___closed__9; +x_2 = l_Lean_Parser_Term_structInst_formatter___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__13() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_optEllipsis_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__14() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_formatter___closed__13; -x_2 = l_Lean_Parser_Term_structInst_formatter___closed__12; +x_1 = l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__2; +x_2 = l_Lean_Parser_Term_structInst_formatter___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__15() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_formatter___closed__9; -x_2 = l_Lean_Parser_Term_structInst_formatter___closed__14; +x_1 = l_Lean_Parser_Term_structInst_formatter___closed__8; +x_2 = l_Lean_Parser_Term_structInst_formatter___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__16() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInst_formatter___closed__5; -x_2 = l_Lean_Parser_Term_structInst_formatter___closed__15; +x_2 = l_Lean_Parser_Term_structInst_formatter___closed__13; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__17() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__15() { _start: { lean_object* x_1; @@ -25468,37 +27237,37 @@ x_1 = lean_alloc_closure((void*)(l_Lean_ppHardSpace_formatter___boxed), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__18() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_formatter___closed__17; -x_2 = l_Lean_Parser_Term_structInst_formatter___closed__16; +x_1 = l_Lean_Parser_Term_structInst_formatter___closed__15; +x_2 = l_Lean_Parser_Term_structInst_formatter___closed__14; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__19() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__2; -x_2 = l_Lean_Parser_Term_structInst_formatter___closed__18; +x_2 = l_Lean_Parser_Term_structInst_formatter___closed__16; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__20() { +static lean_object* _init_l_Lean_Parser_Term_structInst_formatter___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_structInst___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_structInst_formatter___closed__19; +x_3 = l_Lean_Parser_Term_structInst_formatter___closed__17; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -25511,11 +27280,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInst_formatter(lean_object* x_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_structInst_formatter___closed__1; -x_7 = l_Lean_Parser_Term_structInst_formatter___closed__20; +x_7 = l_Lean_Parser_Term_structInst_formatter___closed__18; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_structInst___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInst_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInst_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_structInst___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1() { _start: { @@ -25634,6 +27433,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_structInstFieldAbbrev___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1() { _start: { @@ -25710,6 +27539,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstArrayRef_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1() { _start: { @@ -25739,36 +27598,28 @@ return x_1; static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstArrayRef_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -25780,69 +27631,69 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_cdot_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__7; +x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_group_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__8; -x_2 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__7; +x_2 = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__9; +x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__8; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_many_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__10; +x_1 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_structInstLVal___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__11; +x_3 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__10; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -25855,11 +27706,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstLVal_parenthesizer(lean_ob { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__12; +x_7 = l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__11; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_structInstLVal___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstLVal_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_structInstLVal___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__1() { _start: { @@ -25903,16 +27784,8 @@ return x_3; static lean_object* _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstLVal_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2; x_2 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -25920,13 +27793,13 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_structInstField___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__5; +x_3 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__4; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -25939,7 +27812,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInstField_parenthesizer(lean_o { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__6; +x_7 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__5; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -26006,6 +27879,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_optEllipsis___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_optEllipsis_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_optEllipsis___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__1() { _start: { @@ -26087,35 +27990,27 @@ static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__8() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInstField_parenthesizer), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__8; +x_1 = l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__9; +x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__8; x_2 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__4; x_3 = l_Lean_Parser_Term_tupleTail_parenthesizer___closed__2; x_4 = 1; @@ -26128,7 +28023,7 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -26140,17 +28035,17 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__11; +x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__10; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__13() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__12() { _start: { lean_object* x_1; lean_object* x_2; @@ -26160,63 +28055,55 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__12; -x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__13; +x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__11; +x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__12; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__15() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_optEllipsis_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__16() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__15; -x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__14; +x_1 = l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__13; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__17() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__10; -x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__16; +x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__14; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__18() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__17; +x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__15; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__19() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__17() { _start: { lean_object* x_1; @@ -26224,37 +28111,37 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_ppHardSpace_parenthesizer___boxed return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__20() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__19; -x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__18; +x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__17; +x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__16; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__21() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__20; +x_2 = l_Lean_Parser_Term_structInst_parenthesizer___closed__18; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__22() { +static lean_object* _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_structInst___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_structInst_parenthesizer___closed__21; +x_3 = l_Lean_Parser_Term_structInst_parenthesizer___closed__19; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -26267,11 +28154,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_structInst_parenthesizer(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_structInst_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_structInst_parenthesizer___closed__22; +x_7 = l_Lean_Parser_Term_structInst_parenthesizer___closed__20; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_structInst___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_structInst_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_structInst___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_typeSpec___elambda__1___closed__1() { _start: { @@ -27202,6 +29119,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_explicit___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_explicit_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicit_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_explicit___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_explicit_parenthesizer___closed__1() { _start: { @@ -27276,6 +29223,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_explicit___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_explicit_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_explicit___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_inaccessible___elambda__1___closed__1() { _start: { @@ -27909,6 +29886,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_inaccessible___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_inaccessible_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_inaccessible___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_inaccessible_parenthesizer___closed__1() { _start: { @@ -27985,6 +29992,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_inaccessible___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_inaccessible_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_inaccessible___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderIdent___elambda__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -30711,7 +32748,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderIdent_formatter(lean_object* x { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_syntheticHole_formatter___closed__3; -x_7 = l_Lean_Parser_Term_syntheticHole_formatter___closed__4; +x_7 = l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -30801,7 +32838,7 @@ static lean_object* _init_l_Lean_Parser_Term_binderTactic_formatter___closed__5( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_binderTactic_formatter___closed__4; -x_2 = l_Lean_Parser_Term_byTactic_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -30832,6 +32869,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binderTactic___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderTactic_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binderTactic_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_binderTactic___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binderDefault_formatter___closed__1() { _start: { @@ -30874,6 +32941,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binderDefault___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderDefault_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binderDefault_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_binderDefault___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__1() { _start: { @@ -30913,46 +33010,30 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderTactic_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderDefault_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_explicitBinder_formatter___closed__4; -x_2 = l_Lean_Parser_Term_explicitBinder_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_explicitBinder_formatter___closed__6; +x_1 = l_Lean_Parser_Term_explicitBinder_formatter___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_explicitBinder_formatter___closed__7; +x_1 = l_Lean_Parser_Term_explicitBinder_formatter___closed__5; x_2 = l_Lean_Parser_Term_paren_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -30967,7 +33048,7 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_ob x_7 = lean_box(x_1); x_8 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderType_formatter___boxed), 6, 1); lean_closure_set(x_8, 0, x_7); -x_9 = l_Lean_Parser_Term_explicitBinder_formatter___closed__8; +x_9 = l_Lean_Parser_Term_explicitBinder_formatter___closed__6; x_10 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_10, 0, x_8); lean_closure_set(x_10, 1, x_9); @@ -31472,12 +33553,42 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_depArrow___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_depArrow_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_depArrow___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_binderIdent_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__3; -x_7 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__4; +x_7 = l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2; x_8 = l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -31567,7 +33678,7 @@ static lean_object* _init_l_Lean_Parser_Term_binderTactic_parenthesizer___closed { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_binderTactic_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -31598,6 +33709,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binderTactic___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderTactic_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_binderTactic___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binderDefault_parenthesizer___closed__1() { _start: { @@ -31640,6 +33781,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binderDefault___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderDefault_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_binderDefault___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__1() { _start: { @@ -31679,46 +33850,30 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderTactic_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderDefault_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__4; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__7; +x_1 = l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__5; x_2 = l_Lean_Parser_Term_paren_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -31733,7 +33888,7 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_ob x_7 = lean_box(x_1); x_8 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binderType_parenthesizer___boxed), 6, 1); lean_closure_set(x_8, 0, x_7); -x_9 = l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__8; +x_9 = l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__6; x_10 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_10, 0, x_8); lean_closure_set(x_10, 1, x_9); @@ -32218,6 +34373,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_depArrow___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_depArrow_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_depArrow___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_forall___elambda__1___closed__1() { _start: { @@ -33011,7 +35196,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_optType_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_typeSpec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__2() { _start: { lean_object* x_1; @@ -33019,11 +35214,23 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_typeSpec_formatter), 5, 0); return x_1; } } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeSpec_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_typeSpec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_optType_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Term_optType_formatter___closed__1; +x_6 = l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__2; x_7 = l_Lean_Parser_optional_formatter(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -33183,6 +35390,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_forall___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_forall_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forall_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_forall___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_typeSpec_parenthesizer___closed__1() { _start: { @@ -33225,7 +35462,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_optType_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_typeSpec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -33233,11 +35480,23 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_typeSpec_parenthesizer), 5, return x_1; } } +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_typeSpec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_optType_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Term_optType_parenthesizer___closed__1; +x_6 = l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__2; x_7 = l_Lean_Parser_optional_parenthesizer(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -33397,6 +35656,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_forall___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_forall_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forall_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_forall___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_matchAlt___elambda__1___closed__1() { _start: { @@ -36545,6 +38834,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_trueVal___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_trueVal_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trueVal_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_trueVal___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_falseVal_formatter___closed__1() { _start: { @@ -36600,6 +38919,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_falseVal___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_falseVal_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_falseVal_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_falseVal___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__1() { _start: { @@ -36656,32 +39005,16 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_trueVal_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_falseVal_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__7() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_generalizingParam_formatter___closed__5; -x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -36693,49 +39026,49 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_generalizingParam_formatter___closed__7; -x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__8; +x_1 = l_Lean_Parser_Term_generalizingParam_formatter___closed__5; +x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInstField_formatter___closed__2; -x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__9; +x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_generalizingParam_formatter___closed__4; -x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__10; +x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_generalizingParam___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_generalizingParam_formatter___closed__11; +x_3 = l_Lean_Parser_Term_generalizingParam_formatter___closed__9; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -36748,11 +39081,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_generalizingParam_formatter(lean_obj { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_generalizingParam_formatter___closed__1; -x_7 = l_Lean_Parser_Term_generalizingParam_formatter___closed__12; +x_7 = l_Lean_Parser_Term_generalizingParam_formatter___closed__10; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_generalizingParam___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_generalizingParam_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_generalizingParam___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_motive_formatter___closed__1() { _start: { @@ -36823,7 +39186,7 @@ static lean_object* _init_l_Lean_Parser_Term_motive_formatter___closed__6() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_tupleTail_formatter___closed__3; -x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__8; +x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -36866,6 +39229,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_motive___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_motive_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_motive_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_motive___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_matchDiscr_formatter___closed__1() { _start: { @@ -36930,6 +39323,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_matchDiscr___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_matchDiscr_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_matchDiscr___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_darrow_formatter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -37116,52 +39539,28 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_generalizingParam_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_motive_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_matchDiscr_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Term_match_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2; x_2 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__4; x_3 = l_Lean_Parser_Term_tupleTail_formatter___closed__2; x_4 = 0; @@ -37174,7 +39573,7 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -37184,83 +39583,83 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_formatter___closed__9; +x_1 = l_Lean_Parser_Term_match_formatter___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_ppDedent_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInst_formatter___closed__2; -x_2 = l_Lean_Parser_Term_match_formatter___closed__10; +x_2 = l_Lean_Parser_Term_match_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_match_formatter___closed__8; -x_2 = l_Lean_Parser_Term_match_formatter___closed__11; +x_1 = l_Lean_Parser_Term_match_formatter___closed__5; +x_2 = l_Lean_Parser_Term_match_formatter___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__13() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_match_formatter___closed__6; -x_2 = l_Lean_Parser_Term_match_formatter___closed__12; +x_1 = l_Lean_Parser_Term_match_formatter___closed__4; +x_2 = l_Lean_Parser_Term_match_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__14() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_match_formatter___closed__4; -x_2 = l_Lean_Parser_Term_match_formatter___closed__13; +x_1 = l_Lean_Parser_Term_match_formatter___closed__3; +x_2 = l_Lean_Parser_Term_match_formatter___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__15() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_match_formatter___closed__2; -x_2 = l_Lean_Parser_Term_match_formatter___closed__14; +x_2 = l_Lean_Parser_Term_match_formatter___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__16() { +static lean_object* _init_l_Lean_Parser_Term_match_formatter___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_match___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_match_formatter___closed__15; +x_3 = l_Lean_Parser_Term_match_formatter___closed__12; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -37273,11 +39672,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_match_formatter(lean_object* x_1, le { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_match_formatter___closed__1; -x_7 = l_Lean_Parser_Term_match_formatter___closed__16; +x_7 = l_Lean_Parser_Term_match_formatter___closed__13; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_match_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_match___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_match_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_match_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_match_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_match___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_match_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_match_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_trueVal_parenthesizer___closed__1() { _start: { @@ -37333,6 +39762,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_trueVal___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_trueVal_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_trueVal___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_falseVal_parenthesizer___closed__1() { _start: { @@ -37388,6 +39847,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_falseVal___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_falseVal_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_falseVal___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1() { _start: { @@ -37444,32 +39933,16 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_trueVal_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_falseVal_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__7() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -37481,49 +39954,49 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__8; +x_1 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__10; +x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_generalizingParam___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__11; +x_3 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__9; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -37536,11 +40009,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_generalizingParam_parenthesizer(lean { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__12; +x_7 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__10; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_generalizingParam___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_generalizingParam_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_generalizingParam___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_motive_parenthesizer___closed__1() { _start: { @@ -37611,7 +40114,7 @@ static lean_object* _init_l_Lean_Parser_Term_motive_parenthesizer___closed__6() { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_tupleTail_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__8; +x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -37654,6 +40157,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_motive___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_motive_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_motive_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_motive___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1() { _start: { @@ -37718,6 +40251,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_matchDiscr___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_matchDiscr_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_matchDiscr___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_darrow_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -37904,52 +40467,28 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_generalizingParam_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_motive_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_matchDiscr_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2; x_2 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__4; x_3 = l_Lean_Parser_Term_tupleTail_parenthesizer___closed__2; x_4 = 0; @@ -37962,7 +40501,7 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; @@ -37972,83 +40511,83 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__9; +x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__6; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppDedent_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__11() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInst_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__10; +x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__12() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__8; -x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__11; +x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__8; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__13() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__12; +x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__14() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__13; +x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__3; +x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__10; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__15() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__14; +x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__11; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__16() { +static lean_object* _init_l_Lean_Parser_Term_match_parenthesizer___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_match___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_match_parenthesizer___closed__15; +x_3 = l_Lean_Parser_Term_match_parenthesizer___closed__12; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -38061,11 +40600,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_match_parenthesizer(lean_object* x_1 { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_match_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_match_parenthesizer___closed__16; +x_7 = l_Lean_Parser_Term_match_parenthesizer___closed__13; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_match___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_match_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_match_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_match___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_nomatch___elambda__1___closed__1() { _start: { @@ -38641,6 +41210,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_nomatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_nomatch_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_nomatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_nomatch_parenthesizer___closed__1() { _start: { @@ -38705,6 +41304,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_nomatch___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_nomatch_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_nomatch___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__1() { _start: { @@ -40755,6 +43384,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_basicFun___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_basicFun_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_basicFun_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_basicFun___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__1() { _start: { @@ -40788,54 +43447,46 @@ return x_3; static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_basicFun_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_fun_formatter___closed__3; -x_2 = l_Lean_Parser_Term_match_formatter___closed__9; +x_1 = l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__2; +x_2 = l_Lean_Parser_Term_match_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_fun_formatter___closed__2; -x_2 = l_Lean_Parser_Term_fun_formatter___closed__4; +x_2 = l_Lean_Parser_Term_fun_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_byTactic_formatter___closed__5; -x_2 = l_Lean_Parser_Term_fun_formatter___closed__5; +x_1 = l_Lean_Parser_Term_byTactic_formatter___closed__4; +x_2 = l_Lean_Parser_Term_fun_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_fun_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_fun___elambda__1___closed__2; x_2 = l_Lean_Parser_maxPrec; -x_3 = l_Lean_Parser_Term_fun_formatter___closed__6; +x_3 = l_Lean_Parser_Term_fun_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -40848,11 +43499,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_fun_formatter(lean_object* x_1, lean { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_fun_formatter___closed__1; -x_7 = l_Lean_Parser_Term_fun_formatter___closed__7; +x_7 = l_Lean_Parser_Term_fun_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_fun___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_fun_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fun_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_fun___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__1() { _start: { @@ -41237,6 +43918,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_basicFun___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_basicFun_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_basicFun___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__1() { _start: { @@ -41270,54 +43981,46 @@ return x_3; static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_basicFun_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_fun_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__9; +x_1 = l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_fun_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_fun_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_fun_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_fun_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Term_byTactic_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_fun_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_fun_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_fun___elambda__1___closed__2; x_2 = l_Lean_Parser_maxPrec; -x_3 = l_Lean_Parser_Term_fun_parenthesizer___closed__6; +x_3 = l_Lean_Parser_Term_fun_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -41330,11 +44033,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_fun_parenthesizer(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_fun_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_fun_parenthesizer___closed__7; +x_7 = l_Lean_Parser_Term_fun_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_fun___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_fun_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_fun_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_fun___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_optExprPrecedence___closed__1() { _start: { @@ -42572,7 +45305,7 @@ static lean_object* _init_l_Lean_Parser_Term_withAnonymousAntiquot_formatter___c { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__5; -x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__9; +x_2 = l_Lean_Parser_Term_generalizingParam_formatter___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -42603,6 +45336,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_withAnonymousAntiquot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__1() { _start: { @@ -42634,26 +45397,18 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_withAnonymousAntiquot_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__4; +x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__3; x_2 = l_Lean_Parser_Term_tupleTail_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -42661,7 +45416,7 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__5() { _start: { lean_object* x_1; @@ -42669,37 +45424,37 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_optExprPrecedence_formatter) return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__6; -x_2 = l_Lean_Parser_Term_leading__parser_formatter___closed__5; +x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__5; +x_2 = l_Lean_Parser_Term_leading__parser_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__2; -x_2 = l_Lean_Parser_Term_leading__parser_formatter___closed__7; +x_2 = l_Lean_Parser_Term_leading__parser_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_leading__parser___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_leading__parser_formatter___closed__8; +x_3 = l_Lean_Parser_Term_leading__parser_formatter___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -42712,11 +45467,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_leading__parser_formatter(lean_objec { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_leading__parser_formatter___closed__1; -x_7 = l_Lean_Parser_Term_leading__parser_formatter___closed__9; +x_7 = l_Lean_Parser_Term_leading__parser_formatter___closed__8; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_leading__parser___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_leading__parser_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_leading__parser___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_optExprPrecedence_parenthesizer___closed__1() { _start: { @@ -42828,7 +45613,7 @@ static lean_object* _init_l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__7; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -42859,6 +45644,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_withAnonymousAntiquot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__1() { _start: { @@ -42890,26 +45705,18 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__3; x_2 = l_Lean_Parser_Term_tupleTail_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -42917,7 +45724,7 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__5() { _start: { lean_object* x_1; @@ -42925,37 +45732,37 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_optExprPrecedence_parenthesi return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__5; +x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__7; +x_2 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_leading__parser___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__8; +x_3 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -42968,11 +45775,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_leading__parser_parenthesizer(lean_o { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__9; +x_7 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__8; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_leading__parser___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_leading__parser_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_leading__parser___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_trailing__parser___elambda__1___closed__1() { _start: { @@ -43595,7 +46432,7 @@ static lean_object* _init_l_Lean_Parser_Term_trailing__parser_formatter___closed _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__6; +x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__5; x_2 = l_Lean_Parser_Term_tupleTail_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -43607,7 +46444,7 @@ static lean_object* _init_l_Lean_Parser_Term_trailing__parser_formatter___closed _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__6; +x_1 = l_Lean_Parser_Term_leading__parser_formatter___closed__5; x_2 = l_Lean_Parser_Term_trailing__parser_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -43651,6 +46488,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_trailing__parser___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_trailing__parser_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_trailing__parser___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1() { _start: { @@ -43683,7 +46550,7 @@ static lean_object* _init_l_Lean_Parser_Term_trailing__parser_parenthesizer___cl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__5; x_2 = l_Lean_Parser_Term_tupleTail_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -43695,7 +46562,7 @@ static lean_object* _init_l_Lean_Parser_Term_trailing__parser_parenthesizer___cl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_leading__parser_parenthesizer___closed__5; x_2 = l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -43739,6 +46606,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_trailing__parser___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_trailing__parser_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_trailing__parser___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_borrowed___elambda__1___closed__1() { _start: { @@ -44336,6 +47233,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_borrowed___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_borrowed_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_borrowed___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_borrowed_parenthesizer___closed__1() { _start: { @@ -44410,6 +47337,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_borrowed___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_borrowed_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_borrowed___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_quotedName___elambda__1___closed__1() { _start: { @@ -44795,6 +47752,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_quotedName___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quotedName_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_quotedName___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_quotedName_parenthesizer___closed__1() { _start: { @@ -44845,6 +47832,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_quotedName___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_quotedName_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_quotedName___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__1() { _start: { @@ -45585,6 +48602,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doubleQuotedName_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1() { _start: { @@ -45700,6 +48747,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_doubleQuotedName_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letIdBinder___elambda__1___closed__1() { _start: { @@ -48202,6 +51279,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letIdDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letIdDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letIdDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letPatDecl_formatter___closed__1() { _start: { @@ -48301,6 +51408,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letPatDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letPatDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letPatDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letEqnsDecl_formatter___closed__1() { _start: { @@ -48323,7 +51460,7 @@ static lean_object* _init_l_Lean_Parser_Term_letEqnsDecl_formatter___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInstField_formatter___closed__2; -x_2 = l_Lean_Parser_Term_match_formatter___closed__9; +x_2 = l_Lean_Parser_Term_match_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -48366,6 +51503,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letEqnsDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__1() { _start: { @@ -48409,70 +51576,46 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letPatDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letEqnsDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letDecl_formatter___closed__4; -x_2 = l_Lean_Parser_Term_letDecl_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letIdDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letDecl_formatter___closed__7; -x_2 = l_Lean_Parser_Term_letDecl_formatter___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__2; +x_2 = l_Lean_Parser_Term_letDecl_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_letDecl_formatter___closed__3; -x_2 = l_Lean_Parser_Term_letDecl_formatter___closed__8; +x_2 = l_Lean_Parser_Term_letDecl_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_letDecl_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_letDecl___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_letDecl_formatter___closed__9; +x_3 = l_Lean_Parser_Term_letDecl_formatter___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -48485,11 +51628,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letDecl_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_letDecl_formatter___closed__1; -x_7 = l_Lean_Parser_Term_letDecl_formatter___closed__10; +x_7 = l_Lean_Parser_Term_letDecl_formatter___closed__7; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__1() { _start: { @@ -48521,52 +51694,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let_formatter___closed__2; -x_2 = l_Lean_Parser_Term_let_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_let_formatter___closed__4; +x_1 = l_Lean_Parser_Term_let_formatter___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withPosition_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_let_formatter___closed__5; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_1 = l_Lean_Parser_Term_let_formatter___closed__4; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_let_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_let___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_let_formatter___closed__6; +x_3 = l_Lean_Parser_Term_let_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -48579,11 +51744,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_let_formatter(lean_object* x_1, lean { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_let_formatter___closed__1; -x_7 = l_Lean_Parser_Term_let_formatter___closed__7; +x_7 = l_Lean_Parser_Term_let_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_let___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_let_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_let___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_let_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_let_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letIdBinder_parenthesizer___closed__1() { _start: { @@ -48780,6 +51975,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letIdDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letIdDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letIdDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1() { _start: { @@ -48879,6 +52104,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letPatDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letPatDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letPatDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1() { _start: { @@ -48901,7 +52156,7 @@ static lean_object* _init_l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_structInstField_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -48944,6 +52199,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letEqnsDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letEqnsDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__1() { _start: { @@ -48987,70 +52272,46 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letPatDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letEqnsDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letIdDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__6; +x_1 = l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__8; +x_2 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__10() { +static lean_object* _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_letDecl___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__9; +x_3 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -49063,11 +52324,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letDecl_parenthesizer(lean_object* x { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__10; +x_7 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__7; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__1() { _start: { @@ -49099,52 +52390,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_let_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_let_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_let_parenthesizer___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_let_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_let_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_let_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_let___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_let_parenthesizer___closed__6; +x_3 = l_Lean_Parser_Term_let_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -49157,11 +52440,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_let_parenthesizer(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_let_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_let_parenthesizer___closed__7; +x_7 = l_Lean_Parser_Term_let_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_let___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_let_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_let___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_let__fun___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -49824,7 +53137,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__fun_formatter___closed__5() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__fun_formatter___closed__4; -x_2 = l_Lean_Parser_Term_let_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -49846,7 +53159,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__fun_formatter___closed__7() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__fun_formatter___closed__6; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -49877,6 +53190,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_let__fun___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_let__fun_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_let__fun___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_let__fun_parenthesizer___closed__1() { _start: { @@ -49932,7 +53275,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__fun_parenthesizer___closed__5( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__fun_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_let_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -49954,7 +53297,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__fun_parenthesizer___closed__7( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__fun_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -49985,6 +53328,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_let__fun___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_let__fun_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_let__fun___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_let__delayed___elambda__1___closed__1() { _start: { @@ -50568,7 +53941,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__delayed_formatter___closed__3( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__delayed_formatter___closed__2; -x_2 = l_Lean_Parser_Term_let_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -50590,7 +53963,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__delayed_formatter___closed__5( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__delayed_formatter___closed__4; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -50621,6 +53994,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_let__delayed___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_let__delayed_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_let__delayed___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_let__delayed_parenthesizer___closed__1() { _start: { @@ -50654,7 +54057,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__delayed_parenthesizer___closed { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__delayed_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_let_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -50676,7 +54079,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__delayed_parenthesizer___closed { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__delayed_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -50707,6 +54110,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_let__delayed___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_let__delayed_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_let__delayed___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_let__tmp___elambda__1___closed__1() { _start: { @@ -51290,7 +54723,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__tmp_formatter___closed__3() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__tmp_formatter___closed__2; -x_2 = l_Lean_Parser_Term_let_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -51312,7 +54745,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__tmp_formatter___closed__5() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__tmp_formatter___closed__4; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -51343,6 +54776,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_let__tmp___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_let__tmp_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_let__tmp___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_let__tmp_parenthesizer___closed__1() { _start: { @@ -51376,7 +54839,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__tmp_parenthesizer___closed__3( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__tmp_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_let_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -51398,7 +54861,7 @@ static lean_object* _init_l_Lean_Parser_Term_let__tmp_parenthesizer___closed__5( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_let__tmp_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -51429,6 +54892,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_let__tmp___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_let__tmp_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_let__tmp___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_instCoeTSyntaxConsSyntaxNodeKindStrAnonymousNil__1(lean_object* x_1) { _start: { @@ -53200,6 +56693,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveIdDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1() { _start: { @@ -53222,7 +56745,7 @@ static lean_object* _init_l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_haveIdDecl_formatter___closed__2; -x_2 = l_Lean_Parser_Term_match_formatter___closed__9; +x_2 = l_Lean_Parser_Term_match_formatter___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -53253,6 +56776,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_haveEqnsDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveEqnsDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_haveEqnsDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_haveDecl_formatter___closed__1() { _start: { @@ -53273,50 +56826,34 @@ return x_6; static lean_object* _init_l_Lean_Parser_Term_haveDecl_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveEqnsDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_haveDecl_formatter___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letDecl_formatter___closed__4; -x_2 = l_Lean_Parser_Term_haveDecl_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_haveDecl_formatter___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveIdDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_haveDecl_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_haveDecl_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_haveDecl_formatter___closed__4; -x_2 = l_Lean_Parser_Term_haveDecl_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__2; +x_2 = l_Lean_Parser_Term_haveDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_haveDecl_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_haveDecl_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_haveDecl___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_haveDecl_formatter___closed__5; +x_3 = l_Lean_Parser_Term_haveDecl_formatter___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -53329,11 +56866,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveDecl_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_haveDecl_formatter___closed__1; -x_7 = l_Lean_Parser_Term_haveDecl_formatter___closed__6; +x_7 = l_Lean_Parser_Term_haveDecl_formatter___closed__4; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_haveDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_haveDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__1() { _start: { @@ -53365,52 +56932,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_have_formatter___closed__2; -x_2 = l_Lean_Parser_Term_have_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_have_formatter___closed__4; +x_1 = l_Lean_Parser_Term_have_formatter___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withPosition_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_have_formatter___closed__5; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_1 = l_Lean_Parser_Term_have_formatter___closed__4; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_have_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_have___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_have_formatter___closed__6; +x_3 = l_Lean_Parser_Term_have_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -53423,11 +56982,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_have_formatter(lean_object* x_1, lea { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_have_formatter___closed__1; -x_7 = l_Lean_Parser_Term_have_formatter___closed__7; +x_7 = l_Lean_Parser_Term_have_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_have_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_have___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_have_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_have_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_have_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_have___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_have_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_have_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_haveIdLhs_parenthesizer___closed__1() { _start: { @@ -53543,6 +57132,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveIdDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_haveIdDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1() { _start: { @@ -53565,7 +57184,7 @@ static lean_object* _init_l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__9; +x_2 = l_Lean_Parser_Term_match_parenthesizer___closed__6; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -53596,6 +57215,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_haveEqnsDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveEqnsDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_haveEqnsDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__1() { _start: { @@ -53616,50 +57265,34 @@ return x_6; static lean_object* _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveEqnsDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letDecl_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveIdDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_haveDecl___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__5; +x_3 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -53672,11 +57305,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_haveDecl_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__6; +x_7 = l_Lean_Parser_Term_haveDecl_parenthesizer___closed__4; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_haveDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_haveDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__1() { _start: { @@ -53708,52 +57371,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_haveDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_have_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_have_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_have_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_have_parenthesizer___closed__3; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_have_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_have_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_have_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_have___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_have_parenthesizer___closed__6; +x_3 = l_Lean_Parser_Term_have_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -53766,11 +57421,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_have_parenthesizer(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_have_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_have_parenthesizer___closed__7; +x_7 = l_Lean_Parser_Term_have_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_have___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_have_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_have_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_have___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_scoped___elambda__1___closed__1() { _start: { @@ -56998,6 +60683,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_docComment___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_docComment_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_docComment_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Command_docComment___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_scoped_formatter___closed__1() { _start: { @@ -57050,6 +60765,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_scoped___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_scoped_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_scoped_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_scoped___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_local_formatter___closed__1() { _start: { @@ -57102,6 +60847,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_local_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_local___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_local_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_local_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_local_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_local___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_local_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_local_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_attrKind_formatter___closed__1() { _start: { @@ -57123,48 +60898,32 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_attrKind_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_scoped_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_attrKind_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_local_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_attrKind_formatter___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_attrKind_formatter___closed__2; -x_2 = l_Lean_Parser_Term_attrKind_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_local_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_attrKind_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_attrKind_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_attrKind_formatter___closed__4; +x_1 = l_Lean_Parser_Term_attrKind_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_attrKind_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_attrKind_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_attrKind___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_attrKind_formatter___closed__5; +x_3 = l_Lean_Parser_Term_attrKind_formatter___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -57177,11 +60936,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_attrKind_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_attrKind_formatter___closed__1; -x_7 = l_Lean_Parser_Term_attrKind_formatter___closed__6; +x_7 = l_Lean_Parser_Term_attrKind_formatter___closed__4; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_attrKind___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attrKind_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attrKind_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_attrKind___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__1() { _start: { @@ -57204,37 +60993,29 @@ static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__2( _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attrKind_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__3() { -_start: -{ -lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Lean_Parser_attrParser_formatter___rarg), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_attrInstance_formatter___closed__2; -x_2 = l_Lean_Parser_Term_attrInstance_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__2; +x_2 = l_Lean_Parser_Term_attrInstance_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_attrInstance___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_attrInstance_formatter___closed__4; +x_3 = l_Lean_Parser_Term_attrInstance_formatter___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -57242,12 +61023,12 @@ lean_closure_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_attrInstance_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_attrInstance_formatter___closed__1; -x_2 = l_Lean_Parser_Term_attrInstance_formatter___closed__5; +x_2 = l_Lean_Parser_Term_attrInstance_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withAntiquot_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -57258,7 +61039,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_attrInstance_formatter(lean_object* _start: { lean_object* x_6; lean_object* x_7; -x_6 = l_Lean_Parser_Term_attrInstance_formatter___closed__6; +x_6 = l_Lean_Parser_Term_attrInstance_formatter___closed__5; x_7 = l_Lean_Parser_ppGroup_formatter(x_6, x_1, x_2, x_3, x_4, x_5); return x_7; } @@ -57364,6 +61145,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_attributes___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attributes_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attributes_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_attributes___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__1() { _start: { @@ -57385,70 +61196,54 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_docComment_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letRecDecl_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attributes_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letRecDecl_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letRecDecl_formatter___closed__5; -x_2 = l_Lean_Parser_Term_let_formatter___closed__3; +x_1 = l_Lean_Parser_Term_letRecDecl_formatter___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letRecDecl_formatter___closed__3; -x_2 = l_Lean_Parser_Term_letRecDecl_formatter___closed__6; +x_1 = l_Lean_Parser_Term_letRecDecl_formatter___closed__2; +x_2 = l_Lean_Parser_Term_letRecDecl_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_letRecDecl___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_letRecDecl_formatter___closed__7; +x_3 = l_Lean_Parser_Term_letRecDecl_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -57461,11 +61256,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letRecDecl_formatter(lean_object* x_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_letRecDecl_formatter___closed__1; -x_7 = l_Lean_Parser_Term_letRecDecl_formatter___closed__8; +x_7 = l_Lean_Parser_Term_letRecDecl_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letRecDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letRecDecl_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letRecDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__1() { _start: { @@ -57487,16 +61312,8 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letRecDecl_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Term_letRecDecls_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__2; x_2 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__4; x_3 = l_Lean_Parser_Term_tupleTail_formatter___closed__2; x_4 = 0; @@ -57509,13 +61326,13 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_letRecDecls___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_letRecDecls_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letRecDecls_formatter___closed__2; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -57528,11 +61345,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letRecDecls_formatter(lean_object* x { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_letRecDecls_formatter___closed__1; -x_7 = l_Lean_Parser_Term_letRecDecls_formatter___closed__4; +x_7 = l_Lean_Parser_Term_letRecDecls_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letRecDecls___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letRecDecls_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letRecDecls___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__1() { _start: { @@ -57589,52 +61436,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letRecDecls_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_letrec_formatter___closed__4; -x_2 = l_Lean_Parser_Term_letrec_formatter___closed__5; +x_2 = l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letrec_formatter___closed__6; +x_1 = l_Lean_Parser_Term_letrec_formatter___closed__5; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_withPosition_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letrec_formatter___closed__7; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_1 = l_Lean_Parser_Term_letrec_formatter___closed__6; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_letrec_formatter___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_letrec___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_letrec_formatter___closed__8; +x_3 = l_Lean_Parser_Term_letrec_formatter___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -57647,11 +61486,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letrec_formatter(lean_object* x_1, l { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_letrec_formatter___closed__1; -x_7 = l_Lean_Parser_Term_letrec_formatter___closed__9; +x_7 = l_Lean_Parser_Term_letrec_formatter___closed__8; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letrec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letrec_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letrec_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letrec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Command_docComment_parenthesizer___closed__1() { _start: { @@ -57758,6 +61627,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Command_docComment___elambda__1___closed__8; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_docComment_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Command_docComment___elambda__1___closed__8; +x_4 = l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_scoped_parenthesizer___closed__1() { _start: { @@ -57810,6 +61709,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_scoped___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_scoped_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_scoped___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_local_parenthesizer___closed__1() { _start: { @@ -57862,6 +61791,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_local___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_local_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_local_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_local___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__1() { _start: { @@ -57883,48 +61842,32 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_scoped_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_local_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__4; +x_1 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_attrKind___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__5; +x_3 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -57937,11 +61880,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_attrKind_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__6; +x_7 = l_Lean_Parser_Term_attrKind_parenthesizer___closed__4; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_attrKind___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attrKind_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_attrKind___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__1() { _start: { @@ -57973,16 +61946,8 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__3() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attrKind_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__4() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_attrInstance_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__2; x_2 = l_Lean_Parser_Term_attrInstance_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -57990,13 +61955,13 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_attrInstance___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_attrInstance_parenthesizer___closed__4; +x_3 = l_Lean_Parser_Term_attrInstance_parenthesizer___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -58009,7 +61974,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_attrInstance_parenthesizer(lean_obje { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_attrInstance_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_attrInstance_parenthesizer___closed__5; +x_7 = l_Lean_Parser_Term_attrInstance_parenthesizer___closed__4; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -58115,6 +62080,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_attributes___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attributes_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_attributes___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1() { _start: { @@ -58136,70 +62131,54 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Command_docComment_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attributes_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_let_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__3; -x_2 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_letRecDecl___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__7; +x_3 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -58212,11 +62191,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letRecDecl_parenthesizer(lean_object { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__8; +x_7 = l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__6; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letRecDecl___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letRecDecl_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letRecDecl___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1() { _start: { @@ -58238,16 +62247,8 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letRecDecl_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2; x_2 = l_Lean_Parser_Term_tupleTail___elambda__1___closed__4; x_3 = l_Lean_Parser_Term_tupleTail_parenthesizer___closed__2; x_4 = 0; @@ -58260,13 +62261,13 @@ lean_closure_set(x_6, 3, x_5); return x_6; } } -static lean_object* _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_letRecDecls___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -58279,11 +62280,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letRecDecls_parenthesizer(lean_objec { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__4; +x_7 = l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__3; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letRecDecls___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letRecDecls_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letRecDecls___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__1() { _start: { @@ -58340,52 +62371,44 @@ return x_2; static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__5() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letRecDecls_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_letrec_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_letrec_parenthesizer___closed__5; +x_2 = l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letrec_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_letrec_parenthesizer___closed__5; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_withPosition_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__8() { +static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_letrec_parenthesizer___closed__7; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_1 = l_Lean_Parser_Term_letrec_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__9() { +static lean_object* _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_letrec___elambda__1___closed__2; x_2 = l_Lean_Parser_leadPrec; -x_3 = l_Lean_Parser_Term_letrec_parenthesizer___closed__8; +x_3 = l_Lean_Parser_Term_letrec_parenthesizer___closed__7; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -58398,11 +62421,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_letrec_parenthesizer(lean_object* x_ { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_letrec_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_letrec_parenthesizer___closed__9; +x_7 = l_Lean_Parser_Term_letrec_parenthesizer___closed__8; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letrec___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letrec_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letrec___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_whereDecls_formatter___closed__1() { _start: { @@ -58461,7 +62514,7 @@ static lean_object* _init_l_Lean_Parser_Term_whereDecls_formatter___closed__6() _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letRecDecls_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -58535,6 +62588,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_whereDecls_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_whereDecls_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_whereDecls_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_whereDecls_formatter___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_whereDecls_parenthesizer___closed__1() { _start: { @@ -58567,7 +62650,7 @@ static lean_object* _init_l_Lean_Parser_Term_whereDecls_parenthesizer___closed__ _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_ppGroup_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -58636,6 +62719,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_whereDecls_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_whereDecls_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_whereDecls_formatter___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_whereDecls___elambda__1___closed__1() { _start: { @@ -59174,40 +63287,32 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_whereDecls_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_match_formatter___closed__9; -x_2 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__5; +x_1 = l_Lean_Parser_Term_match_formatter___closed__6; +x_2 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__4; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__7() { +static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__6; +x_3 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__5; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -59220,11 +63325,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_formatter(lean_o { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__3; -x_7 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__7; +x_7 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__6; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_matchAltsWhereDecls_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1() { _start: { @@ -59246,40 +63381,32 @@ return x_7; static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_whereDecls_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_Parser_optional_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__9; -x_2 = l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__4; +x_3 = l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__3; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -59292,11 +63419,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer(le { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__5; +x_7 = l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__4; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__1() { _start: { @@ -60146,6 +64303,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_noindex___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_noindex_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noindex_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_noindex___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_noindex_parenthesizer___closed__1() { _start: { @@ -60210,6 +64397,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_noindex___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_noindex_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_noindex___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binrel___elambda__1___closed__1() { _start: { @@ -60861,6 +65078,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binrel___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binrel_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_binrel___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binrel_parenthesizer___closed__1() { _start: { @@ -60960,6 +65207,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binrel___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binrel_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_binrel___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__1() { _start: { @@ -61525,6 +65802,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binrel__no__prop_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1() { _start: { @@ -61589,6 +65896,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binrel__no__prop_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binop___elambda__1___closed__1() { _start: { @@ -62136,6 +66473,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binop___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binop_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_binop___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binop_parenthesizer___closed__1() { _start: { @@ -62200,6 +66567,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binop___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binop_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_binop___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binop__lazy___elambda__1___closed__1() { _start: { @@ -62747,6 +67144,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binop__lazy___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binop__lazy_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_binop__lazy___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1() { _start: { @@ -62811,6 +67238,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_binop__lazy___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_binop__lazy_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_binop__lazy___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_forInMacro___elambda__1___closed__1() { _start: { @@ -63439,6 +67896,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_forInMacro___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_forInMacro_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_forInMacro___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_forInMacro_parenthesizer___closed__1() { _start: { @@ -63515,6 +68002,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_forInMacro___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_forInMacro_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_forInMacro___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__1() { _start: { @@ -64107,6 +68624,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_forInMacro_x27_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1() { _start: { @@ -64171,6 +68718,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_forInMacro_x27_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_typeOf___elambda__1___closed__1() { _start: { @@ -64746,6 +69323,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_typeOf___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_typeOf_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_typeOf___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_typeOf_parenthesizer___closed__1() { _start: { @@ -64810,6 +69417,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_typeOf___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_typeOf_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_typeOf___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__1() { _start: { @@ -65485,6 +70122,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_ensureTypeOf_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1() { _start: { @@ -65573,6 +70240,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_ensureTypeOf_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__1() { _start: { @@ -66159,6 +70856,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_ensureExpectedType_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1() { _start: { @@ -66235,6 +70962,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_ensureExpectedType_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__1() { _start: { @@ -66810,6 +71567,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_noImplicitLambda_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1() { _start: { @@ -66874,6 +71661,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_noImplicitLambda_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letMVar___elambda__1___closed__1() { _start: { @@ -67800,6 +72617,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letMVar___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letMVar_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_letMVar___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_letMVar_parenthesizer___closed__1() { _start: { @@ -67924,6 +72771,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_letMVar___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_letMVar_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_letMVar___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__1() { _start: { @@ -68648,6 +73525,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_waitIfTypeMVar_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1() { _start: { @@ -68748,6 +73655,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__1() { _start: { @@ -69390,6 +74327,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1() { _start: { @@ -69454,6 +74421,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__1() { _start: { @@ -70096,6 +75093,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_waitIfContainsMVar_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1() { _start: { @@ -70160,6 +75187,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__1() { _start: { @@ -70817,6 +75874,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_defaultOrOfNonempty_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1() { _start: { @@ -70901,6 +75988,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_namedArgument___elambda__1___closed__1() { _start: { @@ -72146,6 +77263,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_namedArgument___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_namedArgument_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedArgument_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_namedArgument___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_ellipsis_formatter___closed__1() { _start: { @@ -72187,7 +77334,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_argument_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_ellipsis___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__2() { _start: { lean_object* x_1; @@ -72195,11 +77352,23 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_ellipsis_formatter), 5, 0); return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_argument_formatter___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ellipsis_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_ellipsis___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Term_argument_formatter___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_argument_formatter___closed__1; +x_1 = l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__2; x_2 = l_Lean_Parser_Term_tupleTail_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -72207,32 +77376,24 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_argument_formatter___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_namedArgument_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_argument_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Term_argument_formatter___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_argument_formatter___closed__3; -x_2 = l_Lean_Parser_Term_argument_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__2; +x_2 = l_Lean_Parser_Term_argument_formatter___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_orelse_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_argument_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_argument_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_type_formatter___closed__3; -x_2 = l_Lean_Parser_Term_argument_formatter___closed__4; +x_2 = l_Lean_Parser_Term_argument_formatter___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -72244,7 +77405,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_argument_formatter(lean_object* x_1, { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_type_formatter___closed__7; -x_7 = l_Lean_Parser_Term_argument_formatter___closed__5; +x_7 = l_Lean_Parser_Term_argument_formatter___closed__3; x_8 = l_Lean_PrettyPrinter_Formatter_andthen_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -72279,6 +77440,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_app_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_app___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_app_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_app_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_app_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_app___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_app_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_app_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_namedArgument_parenthesizer___closed__1() { _start: { @@ -72366,6 +77557,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_namedArgument___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_namedArgument_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_namedArgument___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_ellipsis_parenthesizer___closed__1() { _start: { @@ -72407,17 +77628,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_argPrec; -x_2 = lean_alloc_closure((void*)(l_Lean_Parser_termParser_parenthesizer), 6, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_ellipsis___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__2() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -72425,11 +77646,33 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_ellipsis_parenthesizer), 5, return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__3() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_ellipsis___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Parser_argPrec; +x_2 = lean_alloc_closure((void*)(l_Lean_Parser_termParser_parenthesizer), 6, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_argument_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__2; x_2 = l_Lean_Parser_Term_argument_parenthesizer___closed__1; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -72437,32 +77680,24 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_namedArgument_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_argument_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_argument_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__2; +x_2 = l_Lean_Parser_Term_argument_parenthesizer___closed__2; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Term_argument_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_type_parenthesizer___closed__5; -x_2 = l_Lean_Parser_Term_argument_parenthesizer___closed__5; +x_2 = l_Lean_Parser_Term_argument_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -72474,7 +77709,7 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_argument_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Term_type_parenthesizer___closed__8; -x_7 = l_Lean_Parser_Term_argument_parenthesizer___closed__6; +x_7 = l_Lean_Parser_Term_argument_parenthesizer___closed__4; x_8 = l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -72509,6 +77744,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_app___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_app_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_app_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_app___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_proj___elambda__1___closed__1() { _start: { @@ -73021,6 +78286,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_proj___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_proj_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_proj_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_proj___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_proj_parenthesizer___closed__1() { _start: { @@ -73089,6 +78384,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_proj___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_proj_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_proj_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_proj___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_completion___elambda__1___closed__1() { _start: { @@ -73462,6 +78787,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_completion___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_completion_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_completion_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_completion___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_completion_parenthesizer___closed__1() { _start: { @@ -73486,6 +78841,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_completion___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_completion_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_completion_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_completion___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_arrow___elambda__1___closed__1() { _start: { @@ -73885,6 +79270,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_arrow___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_arrow_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_arrow_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_arrow___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_arrow_parenthesizer___closed__1() { _start: { @@ -73941,6 +79356,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_arrow___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_arrow_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_arrow___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT uint8_t l_Lean_Parser_Term_isIdent(lean_object* x_1) { _start: { @@ -74683,6 +80128,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_explicitUniv___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_explicitUniv_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_explicitUniv___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1() { _start: { @@ -74788,6 +80263,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_explicitUniv___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_explicitUniv_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_explicitUniv___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_namedPattern___elambda__1___closed__1() { _start: { @@ -75405,6 +80910,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_namedPattern___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_namedPattern_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_namedPattern___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_namedPattern_parenthesizer___closed__1() { _start: { @@ -75497,6 +81032,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_namedPattern___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_namedPattern_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_namedPattern___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_pipeProj___elambda__1___closed__1() { _start: { @@ -76056,6 +81621,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_pipeProj___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_pipeProj_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_pipeProj___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_pipeProj_parenthesizer___closed__1() { _start: { @@ -76124,6 +81719,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_pipeProj___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_pipeProj_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_pipeProj___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__1() { _start: { @@ -76442,6 +82067,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_pipeCompletion_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_pipeCompletion_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -76454,6 +82109,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_pipeCompletion_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_subst___elambda__1___closed__1() { _start: { @@ -76986,6 +82671,36 @@ x_10 = l_Lean_PrettyPrinter_Formatter_trailingNode_formatter(x_6, x_7, x_8, x_9, return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_subst___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_subst_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_subst_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_subst___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_subst_parenthesizer___closed__1() { _start: { @@ -77047,6 +82762,36 @@ x_10 = l_Lean_PrettyPrinter_Parenthesizer_trailingNode_parenthesizer(x_6, x_7, x return x_10; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_subst___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_subst_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_subst_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_subst___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__1() { _start: { @@ -77733,6 +83478,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_funBinder_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1() { _start: { @@ -77829,6 +83604,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_funBinder_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_bracketedBinderF() { _start: { @@ -78524,6 +84329,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_bracketedBinder_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1() { _start: { @@ -78620,6 +84455,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1() { _start: { @@ -79225,7 +85090,7 @@ static lean_object* _init_l_Lean_Parser_Term_matchDiscr_quot_formatter___closed_ _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_evalInsideQuot_formatter___rarg), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -79289,6 +85154,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_matchDiscr_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1() { _start: { @@ -79321,7 +85216,7 @@ static lean_object* _init_l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___clo _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_evalInsideQuot_parenthesizer___rarg), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -79385,6 +85280,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_matchDiscr_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_attr_quot___elambda__1___closed__1() { _start: { @@ -79988,7 +85913,7 @@ static lean_object* _init_l_Lean_Parser_Term_attr_quot_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_attrInstance_formatter___closed__3; +x_1 = l_Lean_Parser_Term_attrInstance_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_incQuotDepth_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; @@ -80042,6 +85967,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_attr_quot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attr_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_attr_quot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_attr_quot_parenthesizer___closed__1() { _start: { @@ -80128,6 +86083,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_attr_quot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_attr_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_attr_quot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_panic___elambda__1___closed__1() { _start: { @@ -80703,6 +86688,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_panic___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_panic_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_panic_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_panic___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_panic_parenthesizer___closed__1() { _start: { @@ -80767,6 +86782,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_panic___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_panic_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_panic_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_panic___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_unreachable___elambda__1___closed__1() { _start: { @@ -81238,6 +87283,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_unreachable___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_unreachable_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_unreachable___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_unreachable_parenthesizer___closed__1() { _start: { @@ -81290,6 +87365,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_unreachable___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_unreachable_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_unreachable___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_dbgTrace___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -82092,7 +88197,7 @@ static lean_object* _init_l_Lean_Parser_Term_dbgTrace_formatter___closed__7() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_dbgTrace_formatter___closed__6; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -82123,6 +88228,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_dbgTrace___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_dbgTrace_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_dbgTrace___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1() { _start: { @@ -82200,7 +88335,7 @@ static lean_object* _init_l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__7( { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__6; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -82231,6 +88366,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_dbgTrace___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_dbgTrace_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_dbgTrace___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_assert___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -82977,7 +89142,7 @@ static lean_object* _init_l_Lean_Parser_Term_assert_formatter___closed__5() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_assert_formatter___closed__4; -x_2 = l_Lean_Parser_Term_suffices_formatter___closed__6; +x_2 = l_Lean_Parser_Term_suffices_formatter___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -83008,6 +89173,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_assert___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_assert_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_assert_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_assert___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_assert_parenthesizer___closed__1() { _start: { @@ -83063,7 +89258,7 @@ static lean_object* _init_l_Lean_Parser_Term_assert_parenthesizer___closed__5() { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Term_assert_parenthesizer___closed__4; -x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__6; +x_2 = l_Lean_Parser_Term_suffices_parenthesizer___closed__5; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); @@ -83094,6 +89289,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_assert___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_assert_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_assert_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_assert___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_macroArg() { _start: { @@ -84175,7 +90400,17 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_macroLastArg_formatter___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__2() { _start: { lean_object* x_1; @@ -84183,7 +90418,19 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_macroDollarArg_formatter), 5 return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_macroLastArg_formatter___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Term_macroLastArg_formatter___closed__1() { _start: { lean_object* x_1; @@ -84195,8 +90442,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroLastArg_formatter(lean_object* _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Term_macroLastArg_formatter___closed__1; -x_7 = l_Lean_Parser_Term_macroLastArg_formatter___closed__2; +x_6 = l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__2; +x_7 = l_Lean_Parser_Term_macroLastArg_formatter___closed__1; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -84241,7 +90488,7 @@ static lean_object* _init_l_Lean_Parser_Term_stateRefT_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_macroLastArg_formatter___closed__2; +x_1 = l_Lean_Parser_Term_macroLastArg_formatter___closed__1; x_2 = l_Lean_Parser_Term_stateRefT_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -84285,6 +90532,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_stateRefT___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_stateRefT_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_stateRefT___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroArg_parenthesizer(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -84368,7 +90645,17 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2() { _start: { lean_object* x_1; @@ -84376,7 +90663,19 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_macroDollarArg_parenthesizer return x_1; } } -static lean_object* _init_l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__2() { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1() { _start: { lean_object* x_1; @@ -84388,8 +90687,8 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Term_macroLastArg_parenthesizer(lean_obje _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__2; +x_6 = l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2; +x_7 = l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1; x_8 = l_Lean_PrettyPrinter_Parenthesizer_orelse_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } @@ -84434,7 +90733,7 @@ static lean_object* _init_l_Lean_Parser_Term_stateRefT_parenthesizer___closed__4 _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__2; +x_1 = l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1; x_2 = l_Lean_Parser_Term_stateRefT_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -84478,6 +90777,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_stateRefT___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_stateRefT_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_stateRefT___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__1() { _start: { @@ -85347,6 +91676,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_dynamicQuot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1() { _start: { @@ -85469,6 +91828,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_dynamicQuot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_dotIdent___elambda__1___closed__1() { _start: { @@ -85997,6 +92386,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_dotIdent___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_dotIdent_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Term_dotIdent___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Term_dotIdent_parenthesizer___closed__1() { _start: { @@ -86063,6 +92482,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Term_dotIdent___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_dotIdent_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Term_dotIdent___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_quot___elambda__1___closed__1() { _start: { @@ -86710,6 +93159,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_quot___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_quot___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_quot_parenthesizer___closed__1() { _start: { @@ -86796,6 +93275,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_quot___elambda__1___closed__1; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_quot___elambda__1___closed__1; +x_4 = l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__1() { _start: { @@ -87346,6 +93855,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_node_formatter(x_6, x_7, x_1, x_2, x_3, x_4 return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_seq1___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_seq1_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_seq1_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_seq1___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__1() { _start: { @@ -87367,26 +93906,18 @@ return x_7; static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_seq1_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_incQuotDepth_formatter), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__4() { +static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__3; +x_1 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__2; x_2 = l_Lean_Parser_Term_paren_formatter___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -87394,25 +93925,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic_quot_formatter___closed__2; -x_2 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__4; +x_2 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Formatter_andthen_formatter), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__6() { +static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__5; +x_3 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__4; x_4 = lean_alloc_closure((void*)(l_Lean_Parser_leadingNode_formatter___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -87425,11 +93956,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_quotSeq_formatter(lean_object* x_1 { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__1; -x_7 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__6; +x_7 = l_Lean_Parser_Tactic_quotSeq_formatter___closed__5; x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_quotSeq_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_seq1_parenthesizer___closed__1() { _start: { @@ -87467,6 +94028,36 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_node_parenthesizer(x_6, x_7, x_1, x_2, return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_seq1___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_seq1_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_seq1___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1() { _start: { @@ -87488,26 +94079,18 @@ return x_7; static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_seq1_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__3() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__2; x_2 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_incQuotDepth_parenthesizer), 6, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__4() { +static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__3; +x_1 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2; x_2 = l_Lean_Parser_Term_paren_parenthesizer___closed__9; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); @@ -87515,25 +94098,25 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__5() { +static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Parser_Tactic_quot_parenthesizer___closed__2; -x_2 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__4; +x_2 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__3; x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_andthen_parenthesizer), 7, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__6() { +static lean_object* _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__5; +x_3 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__4; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_leadingNode_parenthesizer___boxed), 8, 3); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); @@ -87546,11 +94129,41 @@ LEAN_EXPORT lean_object* l_Lean_Parser_Tactic_quotSeq_parenthesizer(lean_object* { lean_object* x_6; lean_object* x_7; lean_object* x_8; x_6 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1; -x_7 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__6; +x_7 = l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__5; x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_1, x_2, x_3, x_4, x_5); return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Tactic_quotSeq_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2; +x_4 = l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Level_quot___elambda__1___closed__1() { _start: { @@ -88228,6 +94841,36 @@ x_8 = l_Lean_PrettyPrinter_Formatter_orelse_formatter(x_6, x_7, x_1, x_2, x_3, x return x_8; } } +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_quot___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_quot_formatter), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_quot_formatter(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3; +x_3 = l_Lean_Parser_Level_quot___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} static lean_object* _init_l_Lean_Parser_Level_quot_parenthesizer___closed__1() { _start: { @@ -88314,7 +94957,37 @@ x_8 = l_Lean_PrettyPrinter_Parenthesizer_withAntiquot_parenthesizer(x_6, x_7, x_ return x_8; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Parser_Level_quot___elambda__1___closed__3; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Level_quot_parenthesizer), 5, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Parser_Level_quot_parenthesizer(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3; +x_3 = l_Lean_Parser_Level_quot___elambda__1___closed__3; +x_4 = l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__1; +x_5 = l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__2; +x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88324,7 +94997,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__2() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__2() { _start: { lean_object* x_1; lean_object* x_2; @@ -88334,7 +95007,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__3() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -88344,7 +95017,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__4() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__4() { _start: { lean_object* x_1; lean_object* x_2; @@ -88354,11 +95027,11 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__5() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__5() { _start: { lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__4; +x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__4; x_2 = 1; x_3 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_3, 0, x_1); @@ -88366,17 +95039,17 @@ lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__6() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_let_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__7() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__7() { _start: { lean_object* x_1; @@ -88384,17 +95057,17 @@ x_1 = l_Lean_PrettyPrinter_Formatter_formatterAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__8() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_let_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__9() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__9() { _start: { lean_object* x_1; @@ -88402,7 +95075,7 @@ x_1 = l_Lean_PrettyPrinter_Parenthesizer_parenthesizerAliasesRef; return x_1; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__10() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88412,7 +95085,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__11() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__11() { _start: { lean_object* x_1; lean_object* x_2; @@ -88422,7 +95095,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__12() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__12() { _start: { lean_object* x_1; lean_object* x_2; @@ -88432,27 +95105,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__13() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_have_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__14() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__14() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_have_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__15() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88462,7 +95135,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__16() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__16() { _start: { lean_object* x_1; lean_object* x_2; @@ -88472,7 +95145,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__17() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__17() { _start: { lean_object* x_1; lean_object* x_2; @@ -88482,27 +95155,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__18() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__18() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_suffices_formatter___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__19() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__19() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_suffices_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__20() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88512,7 +95185,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__21() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__21() { _start: { lean_object* x_1; lean_object* x_2; @@ -88522,7 +95195,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__22() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__22() { _start: { lean_object* x_1; lean_object* x_2; @@ -88532,27 +95205,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__23() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__23() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letrec_formatter___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__24() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__24() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_letrec_parenthesizer___closed__5; +x_1 = l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__25() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88562,7 +95235,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__26() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__26() { _start: { lean_object* x_1; lean_object* x_2; @@ -88572,7 +95245,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__27() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__27() { _start: { lean_object* x_1; lean_object* x_2; @@ -88582,27 +95255,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__28() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__28() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_syntheticHole_formatter___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__29() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__29() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__4; +x_1 = l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__30() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__30() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88612,7 +95285,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__31() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__31() { _start: { lean_object* x_1; lean_object* x_2; @@ -88622,7 +95295,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__32() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__32() { _start: { lean_object* x_1; lean_object* x_2; @@ -88632,43 +95305,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__33() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_syntheticHole_formatter), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__34() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__33() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__33; +x_1 = l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__35() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Parser_Term_syntheticHole_parenthesizer), 5, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__36() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__34() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__35; +x_1 = l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__37() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__35() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88678,7 +95335,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__38() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__36() { _start: { lean_object* x_1; lean_object* x_2; @@ -88688,7 +95345,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__39() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__37() { _start: { lean_object* x_1; lean_object* x_2; @@ -88698,27 +95355,27 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__40() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__38() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_formatter___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__41() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__39() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_match_parenthesizer___closed__7; +x_1 = l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__42() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__40() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88728,7 +95385,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__43() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__41() { _start: { lean_object* x_1; lean_object* x_2; @@ -88738,7 +95395,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__44() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__42() { _start: { lean_object* x_1; lean_object* x_2; @@ -88748,7 +95405,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__45() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__43() { _start: { lean_object* x_1; lean_object* x_2; @@ -88758,7 +95415,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__46() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__44() { _start: { lean_object* x_1; lean_object* x_2; @@ -88768,7 +95425,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__47() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__45() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -88778,7 +95435,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__48() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__46() { _start: { lean_object* x_1; lean_object* x_2; @@ -88788,7 +95445,7 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__49() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__47() { _start: { lean_object* x_1; lean_object* x_2; @@ -88798,34 +95455,34 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__50() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__48() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_attrInstance_formatter___closed__2; +x_1 = l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__51() { +static lean_object* _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__49() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Parser_Term_attrInstance_parenthesizer___closed__3; +x_1 = l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__1; -x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__2; -x_4 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__3; -x_5 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__5; +x_2 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__1; +x_3 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__2; +x_4 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__3; +x_5 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__5; x_6 = l_Lean_Parser_registerAlias(x_2, x_3, x_4, x_5, x_1); if (lean_obj_tag(x_6) == 0) { @@ -88833,8 +95490,8 @@ lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); -x_8 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__7; -x_9 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__6; +x_8 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__7; +x_9 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__6; x_10 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_2, x_9, x_7); if (lean_obj_tag(x_10) == 0) { @@ -88842,8 +95499,8 @@ lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_10, 1); lean_inc(x_11); lean_dec(x_10); -x_12 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__9; -x_13 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__8; +x_12 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__9; +x_13 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__8; x_14 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_2, x_13, x_11); if (lean_obj_tag(x_14) == 0) { @@ -88851,9 +95508,9 @@ lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean x_15 = lean_ctor_get(x_14, 1); lean_inc(x_15); lean_dec(x_14); -x_16 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__10; -x_17 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__11; -x_18 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__12; +x_16 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__10; +x_17 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__11; +x_18 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__12; x_19 = l_Lean_Parser_registerAlias(x_16, x_17, x_18, x_5, x_15); if (lean_obj_tag(x_19) == 0) { @@ -88861,7 +95518,7 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; x_20 = lean_ctor_get(x_19, 1); lean_inc(x_20); lean_dec(x_19); -x_21 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__13; +x_21 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__13; x_22 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_16, x_21, x_20); if (lean_obj_tag(x_22) == 0) { @@ -88869,7 +95526,7 @@ 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 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__14; +x_24 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__14; x_25 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_16, x_24, x_23); if (lean_obj_tag(x_25) == 0) { @@ -88877,9 +95534,9 @@ lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean x_26 = lean_ctor_get(x_25, 1); lean_inc(x_26); lean_dec(x_25); -x_27 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__15; -x_28 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__16; -x_29 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__17; +x_27 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__15; +x_28 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__16; +x_29 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__17; x_30 = l_Lean_Parser_registerAlias(x_27, x_28, x_29, x_5, x_26); if (lean_obj_tag(x_30) == 0) { @@ -88887,7 +95544,7 @@ lean_object* x_31; lean_object* x_32; lean_object* x_33; x_31 = lean_ctor_get(x_30, 1); lean_inc(x_31); lean_dec(x_30); -x_32 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__18; +x_32 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__18; x_33 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_27, x_32, x_31); if (lean_obj_tag(x_33) == 0) { @@ -88895,7 +95552,7 @@ lean_object* x_34; lean_object* x_35; lean_object* x_36; x_34 = lean_ctor_get(x_33, 1); lean_inc(x_34); lean_dec(x_33); -x_35 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__19; +x_35 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__19; x_36 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_27, x_35, x_34); if (lean_obj_tag(x_36) == 0) { @@ -88903,9 +95560,9 @@ lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean x_37 = lean_ctor_get(x_36, 1); lean_inc(x_37); lean_dec(x_36); -x_38 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__20; -x_39 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__21; -x_40 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__22; +x_38 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__20; +x_39 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__21; +x_40 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__22; x_41 = l_Lean_Parser_registerAlias(x_38, x_39, x_40, x_5, x_37); if (lean_obj_tag(x_41) == 0) { @@ -88913,7 +95570,7 @@ lean_object* x_42; lean_object* x_43; lean_object* x_44; x_42 = lean_ctor_get(x_41, 1); lean_inc(x_42); lean_dec(x_41); -x_43 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__23; +x_43 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__23; x_44 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_38, x_43, x_42); if (lean_obj_tag(x_44) == 0) { @@ -88921,7 +95578,7 @@ lean_object* x_45; lean_object* x_46; lean_object* x_47; x_45 = lean_ctor_get(x_44, 1); lean_inc(x_45); lean_dec(x_44); -x_46 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__24; +x_46 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__24; x_47 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_38, x_46, x_45); if (lean_obj_tag(x_47) == 0) { @@ -88929,9 +95586,9 @@ lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean x_48 = lean_ctor_get(x_47, 1); lean_inc(x_48); lean_dec(x_47); -x_49 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__25; -x_50 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__26; -x_51 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__27; +x_49 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__25; +x_50 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__26; +x_51 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__27; x_52 = l_Lean_Parser_registerAlias(x_49, x_50, x_51, x_5, x_48); if (lean_obj_tag(x_52) == 0) { @@ -88939,7 +95596,7 @@ lean_object* x_53; lean_object* x_54; lean_object* x_55; x_53 = lean_ctor_get(x_52, 1); lean_inc(x_53); lean_dec(x_52); -x_54 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__28; +x_54 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__28; x_55 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_49, x_54, x_53); if (lean_obj_tag(x_55) == 0) { @@ -88947,7 +95604,7 @@ lean_object* x_56; lean_object* x_57; lean_object* x_58; x_56 = lean_ctor_get(x_55, 1); lean_inc(x_56); lean_dec(x_55); -x_57 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__29; +x_57 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__29; x_58 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_49, x_57, x_56); if (lean_obj_tag(x_58) == 0) { @@ -88955,9 +95612,9 @@ lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean x_59 = lean_ctor_get(x_58, 1); lean_inc(x_59); lean_dec(x_58); -x_60 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__30; -x_61 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__31; -x_62 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__32; +x_60 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__30; +x_61 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__31; +x_62 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__32; x_63 = l_Lean_Parser_registerAlias(x_60, x_61, x_62, x_5, x_59); if (lean_obj_tag(x_63) == 0) { @@ -88965,7 +95622,7 @@ lean_object* x_64; lean_object* x_65; lean_object* x_66; x_64 = lean_ctor_get(x_63, 1); lean_inc(x_64); lean_dec(x_63); -x_65 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__34; +x_65 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__33; x_66 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_60, x_65, x_64); if (lean_obj_tag(x_66) == 0) { @@ -88973,7 +95630,7 @@ lean_object* x_67; lean_object* x_68; lean_object* x_69; x_67 = lean_ctor_get(x_66, 1); lean_inc(x_67); lean_dec(x_66); -x_68 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__36; +x_68 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__34; x_69 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_60, x_68, x_67); if (lean_obj_tag(x_69) == 0) { @@ -88981,9 +95638,9 @@ lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean x_70 = lean_ctor_get(x_69, 1); lean_inc(x_70); lean_dec(x_69); -x_71 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__37; -x_72 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__38; -x_73 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__39; +x_71 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__35; +x_72 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__36; +x_73 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__37; x_74 = l_Lean_Parser_registerAlias(x_71, x_72, x_73, x_5, x_70); if (lean_obj_tag(x_74) == 0) { @@ -88991,7 +95648,7 @@ lean_object* x_75; lean_object* x_76; lean_object* x_77; x_75 = lean_ctor_get(x_74, 1); lean_inc(x_75); lean_dec(x_74); -x_76 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__40; +x_76 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__38; x_77 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_71, x_76, x_75); if (lean_obj_tag(x_77) == 0) { @@ -88999,7 +95656,7 @@ lean_object* x_78; lean_object* x_79; lean_object* x_80; x_78 = lean_ctor_get(x_77, 1); lean_inc(x_78); lean_dec(x_77); -x_79 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__41; +x_79 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__39; x_80 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_71, x_79, x_78); if (lean_obj_tag(x_80) == 0) { @@ -89007,9 +95664,9 @@ lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean x_81 = lean_ctor_get(x_80, 1); lean_inc(x_81); lean_dec(x_80); -x_82 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__42; -x_83 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__43; -x_84 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__44; +x_82 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__40; +x_83 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__41; +x_84 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__42; x_85 = l_Lean_Parser_registerAlias(x_82, x_83, x_84, x_5, x_81); if (lean_obj_tag(x_85) == 0) { @@ -89017,7 +95674,7 @@ lean_object* x_86; lean_object* x_87; lean_object* x_88; x_86 = lean_ctor_get(x_85, 1); lean_inc(x_86); lean_dec(x_85); -x_87 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__45; +x_87 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__43; x_88 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_82, x_87, x_86); if (lean_obj_tag(x_88) == 0) { @@ -89025,7 +95682,7 @@ lean_object* x_89; lean_object* x_90; lean_object* x_91; x_89 = lean_ctor_get(x_88, 1); lean_inc(x_89); lean_dec(x_88); -x_90 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__46; +x_90 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__44; x_91 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_82, x_90, x_89); if (lean_obj_tag(x_91) == 0) { @@ -89033,9 +95690,9 @@ lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean x_92 = lean_ctor_get(x_91, 1); lean_inc(x_92); lean_dec(x_91); -x_93 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__47; -x_94 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__48; -x_95 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__49; +x_93 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__45; +x_94 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__46; +x_95 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__47; x_96 = l_Lean_Parser_registerAlias(x_93, x_94, x_95, x_5, x_92); if (lean_obj_tag(x_96) == 0) { @@ -89043,7 +95700,7 @@ lean_object* x_97; lean_object* x_98; lean_object* x_99; x_97 = lean_ctor_get(x_96, 1); lean_inc(x_97); lean_dec(x_96); -x_98 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__50; +x_98 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__48; x_99 = l_Lean_Parser_registerAliasCore___rarg(x_8, x_93, x_98, x_97); if (lean_obj_tag(x_99) == 0) { @@ -89051,7 +95708,7 @@ lean_object* x_100; lean_object* x_101; lean_object* x_102; x_100 = lean_ctor_get(x_99, 1); lean_inc(x_100); lean_dec(x_99); -x_101 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__51; +x_101 = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__49; x_102 = l_Lean_Parser_registerAliasCore___rarg(x_12, x_93, x_101, x_100); return x_102; } @@ -90092,22 +96749,43 @@ l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__15 = _init_l_Lean_Pa lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__15); l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__16 = _init_l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__16(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__16); +l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__2); +l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__3); +l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__4 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter___closed__4); +res = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1 = _init_l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1); l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2 = _init_l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2); l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__3 = _init_l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__3); +l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_tacticSeq_formatter___closed__1 = _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_formatter___closed__1); l_Lean_Parser_Tactic_tacticSeq_formatter___closed__2 = _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_formatter___closed__2); l_Lean_Parser_Tactic_tacticSeq_formatter___closed__3 = _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_formatter___closed__3); -l_Lean_Parser_Tactic_tacticSeq_formatter___closed__4 = _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_formatter___closed__4); -l_Lean_Parser_Tactic_tacticSeq_formatter___closed__5 = _init_l_Lean_Parser_Tactic_tacticSeq_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_formatter___closed__5); +l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_byTactic_formatter___closed__1 = _init_l_Lean_Parser_Term_byTactic_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_formatter___closed__1); l_Lean_Parser_Term_byTactic_formatter___closed__2 = _init_l_Lean_Parser_Term_byTactic_formatter___closed__2(); @@ -90120,8 +96798,13 @@ l_Lean_Parser_Term_byTactic_formatter___closed__5 = _init_l_Lean_Parser_Term_byT lean_mark_persistent(l_Lean_Parser_Term_byTactic_formatter___closed__5); l_Lean_Parser_Term_byTactic_formatter___closed__6 = _init_l_Lean_Parser_Term_byTactic_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_formatter___closed__6); -l_Lean_Parser_Term_byTactic_formatter___closed__7 = _init_l_Lean_Parser_Term_byTactic_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_byTactic_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_byTactic_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_byTactic_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1); l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2(); @@ -90154,22 +96837,43 @@ l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__15 = _init_l_Lea lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__15); l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__16 = _init_l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__16(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__16); +l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__4 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer___closed__4); +res = l___regBuiltin_Lean_Parser_Tactic_tacticSeqBracketed_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1); l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2); l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__3 = _init_l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_tacticSeq1Indented_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1); l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2); l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__3 = _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__3); -l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__4 = _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__4); -l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__5 = _init_l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_tacticSeq_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_byTactic_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_parenthesizer___closed__1); l_Lean_Parser_Term_byTactic_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__2(); @@ -90182,8 +96886,13 @@ l_Lean_Parser_Term_byTactic_parenthesizer___closed__5 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_byTactic_parenthesizer___closed__5); l_Lean_Parser_Term_byTactic_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_parenthesizer___closed__6); -l_Lean_Parser_Term_byTactic_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_byTactic_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_byTactic_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_byTactic_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__1 = _init_l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__1); l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__2 = _init_l_Lean_Parser_Term_byTactic_x27___elambda__1___closed__2(); @@ -90510,6 +97219,13 @@ l_Lean_Parser_Term_type_formatter___closed__10 = _init_l_Lean_Parser_Term_type_f lean_mark_persistent(l_Lean_Parser_Term_type_formatter___closed__10); l_Lean_Parser_Term_type_formatter___closed__11 = _init_l_Lean_Parser_Term_type_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Term_type_formatter___closed__11); +l___regBuiltin_Lean_Parser_Term_type_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_type_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_type_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_type_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_type_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_type_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_type_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_type_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_type_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_type_parenthesizer___closed__1); l_Lean_Parser_Term_type_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_type_parenthesizer___closed__2(); @@ -90534,6 +97250,13 @@ l_Lean_Parser_Term_type_parenthesizer___closed__11 = _init_l_Lean_Parser_Term_ty lean_mark_persistent(l_Lean_Parser_Term_type_parenthesizer___closed__11); l_Lean_Parser_Term_type_parenthesizer___closed__12 = _init_l_Lean_Parser_Term_type_parenthesizer___closed__12(); lean_mark_persistent(l_Lean_Parser_Term_type_parenthesizer___closed__12); +l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_type_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_type_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_sort___elambda__1___closed__1 = _init_l_Lean_Parser_Term_sort___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_sort___elambda__1___closed__1); l_Lean_Parser_Term_sort___elambda__1___closed__2 = _init_l_Lean_Parser_Term_sort___elambda__1___closed__2(); @@ -90604,6 +97327,13 @@ l_Lean_Parser_Term_sort_formatter___closed__3 = _init_l_Lean_Parser_Term_sort_fo lean_mark_persistent(l_Lean_Parser_Term_sort_formatter___closed__3); l_Lean_Parser_Term_sort_formatter___closed__4 = _init_l_Lean_Parser_Term_sort_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_sort_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sort_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_sort_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_sort_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_sort_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_sort_parenthesizer___closed__1); l_Lean_Parser_Term_sort_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_sort_parenthesizer___closed__2(); @@ -90612,6 +97342,13 @@ l_Lean_Parser_Term_sort_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_sor lean_mark_persistent(l_Lean_Parser_Term_sort_parenthesizer___closed__3); l_Lean_Parser_Term_sort_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_sort_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_sort_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sort_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_sort_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_prop___elambda__1___closed__1 = _init_l_Lean_Parser_Term_prop___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_prop___elambda__1___closed__1); l_Lean_Parser_Term_prop___elambda__1___closed__2 = _init_l_Lean_Parser_Term_prop___elambda__1___closed__2(); @@ -90676,12 +97413,26 @@ l_Lean_Parser_Term_prop_formatter___closed__2 = _init_l_Lean_Parser_Term_prop_fo lean_mark_persistent(l_Lean_Parser_Term_prop_formatter___closed__2); l_Lean_Parser_Term_prop_formatter___closed__3 = _init_l_Lean_Parser_Term_prop_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_prop_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prop_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_prop_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_prop_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_prop_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_prop_parenthesizer___closed__1); l_Lean_Parser_Term_prop_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_prop_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_prop_parenthesizer___closed__2); l_Lean_Parser_Term_prop_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_prop_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_prop_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_prop_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_prop_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_hole___elambda__1___closed__1 = _init_l_Lean_Parser_Term_hole___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_hole___elambda__1___closed__1); l_Lean_Parser_Term_hole___elambda__1___closed__2 = _init_l_Lean_Parser_Term_hole___elambda__1___closed__2(); @@ -90746,12 +97497,26 @@ l_Lean_Parser_Term_hole_formatter___closed__2 = _init_l_Lean_Parser_Term_hole_fo lean_mark_persistent(l_Lean_Parser_Term_hole_formatter___closed__2); l_Lean_Parser_Term_hole_formatter___closed__3 = _init_l_Lean_Parser_Term_hole_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_hole_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_hole_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_hole_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_hole_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_hole_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_hole_parenthesizer___closed__1); l_Lean_Parser_Term_hole_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_hole_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_hole_parenthesizer___closed__2); l_Lean_Parser_Term_hole_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_hole_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_hole_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_hole_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_hole_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_syntheticHole___elambda__1___closed__1 = _init_l_Lean_Parser_Term_syntheticHole___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_syntheticHole___elambda__1___closed__1); l_Lean_Parser_Term_syntheticHole___elambda__1___closed__2 = _init_l_Lean_Parser_Term_syntheticHole___elambda__1___closed__2(); @@ -90830,8 +97595,13 @@ l_Lean_Parser_Term_syntheticHole_formatter___closed__5 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_syntheticHole_formatter___closed__5); l_Lean_Parser_Term_syntheticHole_formatter___closed__6 = _init_l_Lean_Parser_Term_syntheticHole_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_syntheticHole_formatter___closed__6); -l_Lean_Parser_Term_syntheticHole_formatter___closed__7 = _init_l_Lean_Parser_Term_syntheticHole_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_syntheticHole_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_syntheticHole_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1); l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2(); @@ -90844,8 +97614,13 @@ l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__5 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__5); l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__6); -l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_syntheticHole_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_syntheticHole_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_sorry___elambda__1___closed__1 = _init_l_Lean_Parser_Term_sorry___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_sorry___elambda__1___closed__1); l_Lean_Parser_Term_sorry___elambda__1___closed__2 = _init_l_Lean_Parser_Term_sorry___elambda__1___closed__2(); @@ -90908,12 +97683,26 @@ l_Lean_Parser_Term_sorry_formatter___closed__2 = _init_l_Lean_Parser_Term_sorry_ lean_mark_persistent(l_Lean_Parser_Term_sorry_formatter___closed__2); l_Lean_Parser_Term_sorry_formatter___closed__3 = _init_l_Lean_Parser_Term_sorry_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_sorry_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sorry_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_sorry_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_sorry_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_sorry_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_sorry_parenthesizer___closed__1); l_Lean_Parser_Term_sorry_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_sorry_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_sorry_parenthesizer___closed__2); l_Lean_Parser_Term_sorry_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_sorry_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_sorry_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_sorry_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_cdot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_cdot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_cdot___elambda__1___closed__1); l_Lean_Parser_Term_cdot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_cdot___elambda__1___closed__2(); @@ -90990,6 +97779,13 @@ l_Lean_Parser_Term_cdot_formatter___closed__4 = _init_l_Lean_Parser_Term_cdot_fo lean_mark_persistent(l_Lean_Parser_Term_cdot_formatter___closed__4); l_Lean_Parser_Term_cdot_formatter___closed__5 = _init_l_Lean_Parser_Term_cdot_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_cdot_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_cdot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_cdot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_cdot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_cdot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_cdot_parenthesizer___closed__1); l_Lean_Parser_Term_cdot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_cdot_parenthesizer___closed__2(); @@ -91000,6 +97796,13 @@ l_Lean_Parser_Term_cdot_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_cdo lean_mark_persistent(l_Lean_Parser_Term_cdot_parenthesizer___closed__4); l_Lean_Parser_Term_cdot_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_cdot_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_cdot_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_cdot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_typeAscription___elambda__1___closed__1 = _init_l_Lean_Parser_Term_typeAscription___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_typeAscription___elambda__1___closed__1); l_Lean_Parser_Term_typeAscription___elambda__1___closed__2 = _init_l_Lean_Parser_Term_typeAscription___elambda__1___closed__2(); @@ -91190,6 +97993,13 @@ l_Lean_Parser_Term_tupleTail_formatter___closed__5 = _init_l_Lean_Parser_Term_tu lean_mark_persistent(l_Lean_Parser_Term_tupleTail_formatter___closed__5); l_Lean_Parser_Term_tupleTail_formatter___closed__6 = _init_l_Lean_Parser_Term_tupleTail_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_tupleTail_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_tupleTail_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_tupleTail_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_typeAscription_formatter___closed__1 = _init_l_Lean_Parser_Term_typeAscription_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_typeAscription_formatter___closed__1); l_Lean_Parser_Term_typeAscription_formatter___closed__2 = _init_l_Lean_Parser_Term_typeAscription_formatter___closed__2(); @@ -91198,12 +98008,15 @@ l_Lean_Parser_Term_typeAscription_formatter___closed__3 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_typeAscription_formatter___closed__3); l_Lean_Parser_Term_typeAscription_formatter___closed__4 = _init_l_Lean_Parser_Term_typeAscription_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_typeAscription_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeAscription_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_typeAscription_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_parenSpecial_formatter___closed__1 = _init_l_Lean_Parser_Term_parenSpecial_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_parenSpecial_formatter___closed__1); -l_Lean_Parser_Term_parenSpecial_formatter___closed__2 = _init_l_Lean_Parser_Term_parenSpecial_formatter___closed__2(); -lean_mark_persistent(l_Lean_Parser_Term_parenSpecial_formatter___closed__2); -l_Lean_Parser_Term_parenSpecial_formatter___closed__3 = _init_l_Lean_Parser_Term_parenSpecial_formatter___closed__3(); -lean_mark_persistent(l_Lean_Parser_Term_parenSpecial_formatter___closed__3); l_Lean_Parser_Term_paren_formatter___closed__1 = _init_l_Lean_Parser_Term_paren_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_paren_formatter___closed__1); l_Lean_Parser_Term_paren_formatter___closed__2 = _init_l_Lean_Parser_Term_paren_formatter___closed__2(); @@ -91228,6 +98041,13 @@ l_Lean_Parser_Term_paren_formatter___closed__11 = _init_l_Lean_Parser_Term_paren lean_mark_persistent(l_Lean_Parser_Term_paren_formatter___closed__11); l_Lean_Parser_Term_paren_formatter___closed__12 = _init_l_Lean_Parser_Term_paren_formatter___closed__12(); lean_mark_persistent(l_Lean_Parser_Term_paren_formatter___closed__12); +l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_paren_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_paren_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_tupleTail_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_tupleTail_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_tupleTail_parenthesizer___closed__1); l_Lean_Parser_Term_tupleTail_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_tupleTail_parenthesizer___closed__2(); @@ -91240,6 +98060,13 @@ l_Lean_Parser_Term_tupleTail_parenthesizer___closed__5 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_tupleTail_parenthesizer___closed__5); l_Lean_Parser_Term_tupleTail_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_tupleTail_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_tupleTail_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_tupleTail_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_typeAscription_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_typeAscription_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_typeAscription_parenthesizer___closed__1); l_Lean_Parser_Term_typeAscription_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_typeAscription_parenthesizer___closed__2(); @@ -91248,12 +98075,15 @@ l_Lean_Parser_Term_typeAscription_parenthesizer___closed__3 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_typeAscription_parenthesizer___closed__3); l_Lean_Parser_Term_typeAscription_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_typeAscription_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_typeAscription_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_typeAscription_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__1); -l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__2(); -lean_mark_persistent(l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__2); -l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__3(); -lean_mark_persistent(l_Lean_Parser_Term_parenSpecial_parenthesizer___closed__3); l_Lean_Parser_Term_paren_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_paren_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_paren_parenthesizer___closed__1); l_Lean_Parser_Term_paren_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_paren_parenthesizer___closed__2(); @@ -91278,6 +98108,13 @@ l_Lean_Parser_Term_paren_parenthesizer___closed__11 = _init_l_Lean_Parser_Term_p lean_mark_persistent(l_Lean_Parser_Term_paren_parenthesizer___closed__11); l_Lean_Parser_Term_paren_parenthesizer___closed__12 = _init_l_Lean_Parser_Term_paren_parenthesizer___closed__12(); lean_mark_persistent(l_Lean_Parser_Term_paren_parenthesizer___closed__12); +l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_paren_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_paren_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__1 = _init_l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__1); l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__2 = _init_l_Lean_Parser_Term_anonymousCtor___elambda__1___closed__2(); @@ -91372,6 +98209,13 @@ l_Lean_Parser_Term_anonymousCtor_formatter___closed__6 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_anonymousCtor_formatter___closed__6); l_Lean_Parser_Term_anonymousCtor_formatter___closed__7 = _init_l_Lean_Parser_Term_anonymousCtor_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_anonymousCtor_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_anonymousCtor_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1); l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2(); @@ -91386,6 +98230,13 @@ l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__6 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__6); l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_anonymousCtor_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_optIdent___closed__1 = _init_l_Lean_Parser_Term_optIdent___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_optIdent___closed__1); l_Lean_Parser_Term_optIdent___closed__2 = _init_l_Lean_Parser_Term_optIdent___closed__2(); @@ -91554,14 +98405,24 @@ l_Lean_Parser_Term_fromTerm_formatter___closed__3 = _init_l_Lean_Parser_Term_fro lean_mark_persistent(l_Lean_Parser_Term_fromTerm_formatter___closed__3); l_Lean_Parser_Term_fromTerm_formatter___closed__4 = _init_l_Lean_Parser_Term_fromTerm_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_fromTerm_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_fromTerm_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_fromTerm_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_byTactic_x27_formatter___closed__1 = _init_l_Lean_Parser_Term_byTactic_x27_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_x27_formatter___closed__1); l_Lean_Parser_Term_byTactic_x27_formatter___closed__2 = _init_l_Lean_Parser_Term_byTactic_x27_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_x27_formatter___closed__2); -l_Lean_Parser_Term_showRhs_formatter___closed__1 = _init_l_Lean_Parser_Term_showRhs_formatter___closed__1(); -lean_mark_persistent(l_Lean_Parser_Term_showRhs_formatter___closed__1); -l_Lean_Parser_Term_showRhs_formatter___closed__2 = _init_l_Lean_Parser_Term_showRhs_formatter___closed__2(); -lean_mark_persistent(l_Lean_Parser_Term_showRhs_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_byTactic_x27_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_sufficesDecl_formatter___closed__1 = _init_l_Lean_Parser_Term_sufficesDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_sufficesDecl_formatter___closed__1); l_Lean_Parser_Term_sufficesDecl_formatter___closed__2 = _init_l_Lean_Parser_Term_sufficesDecl_formatter___closed__2(); @@ -91578,6 +98439,13 @@ l_Lean_Parser_Term_sufficesDecl_formatter___closed__7 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_sufficesDecl_formatter___closed__7); l_Lean_Parser_Term_sufficesDecl_formatter___closed__8 = _init_l_Lean_Parser_Term_sufficesDecl_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_sufficesDecl_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_sufficesDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_semicolonOrLinebreak_formatter___closed__1 = _init_l_Lean_Parser_semicolonOrLinebreak_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_semicolonOrLinebreak_formatter___closed__1); l_Lean_Parser_semicolonOrLinebreak_formatter___closed__2 = _init_l_Lean_Parser_semicolonOrLinebreak_formatter___closed__2(); @@ -91600,8 +98468,13 @@ l_Lean_Parser_Term_suffices_formatter___closed__6 = _init_l_Lean_Parser_Term_suf lean_mark_persistent(l_Lean_Parser_Term_suffices_formatter___closed__6); l_Lean_Parser_Term_suffices_formatter___closed__7 = _init_l_Lean_Parser_Term_suffices_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_suffices_formatter___closed__7); -l_Lean_Parser_Term_suffices_formatter___closed__8 = _init_l_Lean_Parser_Term_suffices_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_suffices_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_suffices_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_suffices_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_optIdent_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_optIdent_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_optIdent_parenthesizer___closed__1); l_Lean_Parser_Term_optIdent_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_optIdent_parenthesizer___closed__2(); @@ -91614,14 +98487,24 @@ l_Lean_Parser_Term_fromTerm_parenthesizer___closed__3 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_fromTerm_parenthesizer___closed__3); l_Lean_Parser_Term_fromTerm_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_fromTerm_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_fromTerm_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_fromTerm_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1); l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2); -l_Lean_Parser_Term_showRhs_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_showRhs_parenthesizer___closed__1(); -lean_mark_persistent(l_Lean_Parser_Term_showRhs_parenthesizer___closed__1); -l_Lean_Parser_Term_showRhs_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_showRhs_parenthesizer___closed__2(); -lean_mark_persistent(l_Lean_Parser_Term_showRhs_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_byTactic_x27_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1); l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2(); @@ -91638,6 +98521,13 @@ l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__7 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__7); l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_sufficesDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_semicolonOrLinebreak_parenthesizer___closed__1 = _init_l_Lean_Parser_semicolonOrLinebreak_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_semicolonOrLinebreak_parenthesizer___closed__1); l_Lean_Parser_semicolonOrLinebreak_parenthesizer___closed__2 = _init_l_Lean_Parser_semicolonOrLinebreak_parenthesizer___closed__2(); @@ -91660,8 +98550,13 @@ l_Lean_Parser_Term_suffices_parenthesizer___closed__6 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_suffices_parenthesizer___closed__6); l_Lean_Parser_Term_suffices_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_suffices_parenthesizer___closed__7); -l_Lean_Parser_Term_suffices_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_suffices_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_suffices_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_suffices_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_show___elambda__1___closed__1 = _init_l_Lean_Parser_Term_show___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_show___elambda__1___closed__1); l_Lean_Parser_Term_show___elambda__1___closed__2 = _init_l_Lean_Parser_Term_show___elambda__1___closed__2(); @@ -91732,6 +98627,13 @@ l_Lean_Parser_Term_show_formatter___closed__3 = _init_l_Lean_Parser_Term_show_fo lean_mark_persistent(l_Lean_Parser_Term_show_formatter___closed__3); l_Lean_Parser_Term_show_formatter___closed__4 = _init_l_Lean_Parser_Term_show_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_show_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_show_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_show_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_show_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_show_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_show_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_show_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_show_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_show_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_show_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_show_parenthesizer___closed__1); l_Lean_Parser_Term_show_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_show_parenthesizer___closed__2(); @@ -91740,6 +98642,13 @@ l_Lean_Parser_Term_show_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_sho lean_mark_persistent(l_Lean_Parser_Term_show_parenthesizer___closed__3); l_Lean_Parser_Term_show_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_show_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_show_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_show_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_show_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__1 = _init_l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__1); l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__2 = _init_l_Lean_Parser_Term_structInstArrayRef___elambda__1___closed__2(); @@ -92164,6 +99073,13 @@ l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__8 = _init_l_Lean_Pa lean_mark_persistent(l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__8); l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__9 = _init_l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__9); +l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInstArrayRef_formatter___closed__1 = _init_l_Lean_Parser_Term_structInstArrayRef_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInstArrayRef_formatter___closed__1); l_Lean_Parser_Term_structInstArrayRef_formatter___closed__2 = _init_l_Lean_Parser_Term_structInstArrayRef_formatter___closed__2(); @@ -92174,6 +99090,13 @@ l_Lean_Parser_Term_structInstArrayRef_formatter___closed__4 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_structInstArrayRef_formatter___closed__4); l_Lean_Parser_Term_structInstArrayRef_formatter___closed__5 = _init_l_Lean_Parser_Term_structInstArrayRef_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_structInstArrayRef_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInstLVal_formatter___closed__1 = _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInstLVal_formatter___closed__1); l_Lean_Parser_Term_structInstLVal_formatter___closed__2 = _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__2(); @@ -92196,8 +99119,13 @@ l_Lean_Parser_Term_structInstLVal_formatter___closed__10 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_structInstLVal_formatter___closed__10); l_Lean_Parser_Term_structInstLVal_formatter___closed__11 = _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Term_structInstLVal_formatter___closed__11); -l_Lean_Parser_Term_structInstLVal_formatter___closed__12 = _init_l_Lean_Parser_Term_structInstLVal_formatter___closed__12(); -lean_mark_persistent(l_Lean_Parser_Term_structInstLVal_formatter___closed__12); +l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_structInstLVal_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInstField_formatter___closed__1 = _init_l_Lean_Parser_Term_structInstField_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInstField_formatter___closed__1); l_Lean_Parser_Term_structInstField_formatter___closed__2 = _init_l_Lean_Parser_Term_structInstField_formatter___closed__2(); @@ -92210,8 +99138,6 @@ l_Lean_Parser_Term_structInstField_formatter___closed__5 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_structInstField_formatter___closed__5); l_Lean_Parser_Term_structInstField_formatter___closed__6 = _init_l_Lean_Parser_Term_structInstField_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_structInstField_formatter___closed__6); -l_Lean_Parser_Term_structInstField_formatter___closed__7 = _init_l_Lean_Parser_Term_structInstField_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_structInstField_formatter___closed__7); l_Lean_Parser_Term_optEllipsis_formatter___closed__1 = _init_l_Lean_Parser_Term_optEllipsis_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_optEllipsis_formatter___closed__1); l_Lean_Parser_Term_optEllipsis_formatter___closed__2 = _init_l_Lean_Parser_Term_optEllipsis_formatter___closed__2(); @@ -92220,6 +99146,13 @@ l_Lean_Parser_Term_optEllipsis_formatter___closed__3 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_optEllipsis_formatter___closed__3); l_Lean_Parser_Term_optEllipsis_formatter___closed__4 = _init_l_Lean_Parser_Term_optEllipsis_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_optEllipsis_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_optEllipsis_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInst_formatter___closed__1 = _init_l_Lean_Parser_Term_structInst_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInst_formatter___closed__1); l_Lean_Parser_Term_structInst_formatter___closed__2 = _init_l_Lean_Parser_Term_structInst_formatter___closed__2(); @@ -92256,10 +99189,13 @@ l_Lean_Parser_Term_structInst_formatter___closed__17 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_structInst_formatter___closed__17); l_Lean_Parser_Term_structInst_formatter___closed__18 = _init_l_Lean_Parser_Term_structInst_formatter___closed__18(); lean_mark_persistent(l_Lean_Parser_Term_structInst_formatter___closed__18); -l_Lean_Parser_Term_structInst_formatter___closed__19 = _init_l_Lean_Parser_Term_structInst_formatter___closed__19(); -lean_mark_persistent(l_Lean_Parser_Term_structInst_formatter___closed__19); -l_Lean_Parser_Term_structInst_formatter___closed__20 = _init_l_Lean_Parser_Term_structInst_formatter___closed__20(); -lean_mark_persistent(l_Lean_Parser_Term_structInst_formatter___closed__20); +l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInst_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_structInst_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1); l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2(); @@ -92278,6 +99214,13 @@ l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__8 = _init_l_Lea lean_mark_persistent(l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__8); l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_structInstFieldAbbrev_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1); l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2(); @@ -92288,6 +99231,13 @@ l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__4 = _init_l_Lean_P lean_mark_persistent(l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__4); l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_structInstArrayRef_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1); l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2(); @@ -92310,8 +99260,13 @@ l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__10 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__10); l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__11 = _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__11); -l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__12 = _init_l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__12(); -lean_mark_persistent(l_Lean_Parser_Term_structInstLVal_parenthesizer___closed__12); +l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_structInstLVal_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInstField_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInstField_parenthesizer___closed__1); l_Lean_Parser_Term_structInstField_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__2(); @@ -92322,8 +99277,6 @@ l_Lean_Parser_Term_structInstField_parenthesizer___closed__4 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Term_structInstField_parenthesizer___closed__4); l_Lean_Parser_Term_structInstField_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_structInstField_parenthesizer___closed__5); -l_Lean_Parser_Term_structInstField_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_structInstField_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_structInstField_parenthesizer___closed__6); l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1); l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2(); @@ -92332,6 +99285,13 @@ l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__3 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__3); l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_optEllipsis_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_optEllipsis_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_structInst_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_structInst_parenthesizer___closed__1); l_Lean_Parser_Term_structInst_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__2(); @@ -92372,10 +99332,13 @@ l_Lean_Parser_Term_structInst_parenthesizer___closed__19 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_structInst_parenthesizer___closed__19); l_Lean_Parser_Term_structInst_parenthesizer___closed__20 = _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__20(); lean_mark_persistent(l_Lean_Parser_Term_structInst_parenthesizer___closed__20); -l_Lean_Parser_Term_structInst_parenthesizer___closed__21 = _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__21(); -lean_mark_persistent(l_Lean_Parser_Term_structInst_parenthesizer___closed__21); -l_Lean_Parser_Term_structInst_parenthesizer___closed__22 = _init_l_Lean_Parser_Term_structInst_parenthesizer___closed__22(); -lean_mark_persistent(l_Lean_Parser_Term_structInst_parenthesizer___closed__22); +l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_structInst_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_typeSpec___elambda__1___closed__1 = _init_l_Lean_Parser_Term_typeSpec___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_typeSpec___elambda__1___closed__1); l_Lean_Parser_Term_typeSpec___elambda__1___closed__2 = _init_l_Lean_Parser_Term_typeSpec___elambda__1___closed__2(); @@ -92480,6 +99443,13 @@ l_Lean_Parser_Term_explicit_formatter___closed__3 = _init_l_Lean_Parser_Term_exp lean_mark_persistent(l_Lean_Parser_Term_explicit_formatter___closed__3); l_Lean_Parser_Term_explicit_formatter___closed__4 = _init_l_Lean_Parser_Term_explicit_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_explicit_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_explicit_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_explicit_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_explicit_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_explicit_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_explicit_parenthesizer___closed__1); l_Lean_Parser_Term_explicit_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_explicit_parenthesizer___closed__2(); @@ -92490,6 +99460,13 @@ l_Lean_Parser_Term_explicit_parenthesizer___closed__4 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_explicit_parenthesizer___closed__4); l_Lean_Parser_Term_explicit_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_explicit_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_explicit_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_explicit_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_inaccessible___elambda__1___closed__1 = _init_l_Lean_Parser_Term_inaccessible___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_inaccessible___elambda__1___closed__1); l_Lean_Parser_Term_inaccessible___elambda__1___closed__2 = _init_l_Lean_Parser_Term_inaccessible___elambda__1___closed__2(); @@ -92566,6 +99543,13 @@ l_Lean_Parser_Term_inaccessible_formatter___closed__4 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_inaccessible_formatter___closed__4); l_Lean_Parser_Term_inaccessible_formatter___closed__5 = _init_l_Lean_Parser_Term_inaccessible_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_inaccessible_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_inaccessible_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_inaccessible_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_inaccessible_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_inaccessible_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_inaccessible_parenthesizer___closed__1); l_Lean_Parser_Term_inaccessible_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_inaccessible_parenthesizer___closed__2(); @@ -92576,6 +99560,13 @@ l_Lean_Parser_Term_inaccessible_parenthesizer___closed__4 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_inaccessible_parenthesizer___closed__4); l_Lean_Parser_Term_inaccessible_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_inaccessible_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_inaccessible_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_inaccessible_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binderIdent___closed__1 = _init_l_Lean_Parser_Term_binderIdent___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binderIdent___closed__1); l_Lean_Parser_Term_binderIdent___closed__2 = _init_l_Lean_Parser_Term_binderIdent___closed__2(); @@ -92874,10 +99865,24 @@ l_Lean_Parser_Term_binderTactic_formatter___closed__5 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_binderTactic_formatter___closed__5); l_Lean_Parser_Term_binderTactic_formatter___closed__6 = _init_l_Lean_Parser_Term_binderTactic_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_binderTactic_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binderTactic_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binderTactic_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binderDefault_formatter___closed__1 = _init_l_Lean_Parser_Term_binderDefault_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binderDefault_formatter___closed__1); l_Lean_Parser_Term_binderDefault_formatter___closed__2 = _init_l_Lean_Parser_Term_binderDefault_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_binderDefault_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binderDefault_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binderDefault_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_explicitBinder_formatter___closed__1 = _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_formatter___closed__1); l_Lean_Parser_Term_explicitBinder_formatter___closed__2 = _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__2(); @@ -92890,10 +99895,6 @@ l_Lean_Parser_Term_explicitBinder_formatter___closed__5 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_formatter___closed__5); l_Lean_Parser_Term_explicitBinder_formatter___closed__6 = _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_formatter___closed__6); -l_Lean_Parser_Term_explicitBinder_formatter___closed__7 = _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_formatter___closed__7); -l_Lean_Parser_Term_explicitBinder_formatter___closed__8 = _init_l_Lean_Parser_Term_explicitBinder_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_formatter___closed__8); l_Lean_Parser_Term_strictImplicitLeftBracket_formatter___closed__1 = _init_l_Lean_Parser_Term_strictImplicitLeftBracket_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_strictImplicitLeftBracket_formatter___closed__1); l_Lean_Parser_Term_strictImplicitLeftBracket_formatter___closed__2 = _init_l_Lean_Parser_Term_strictImplicitLeftBracket_formatter___closed__2(); @@ -92944,6 +99945,13 @@ l_Lean_Parser_Term_depArrow_formatter___closed__5 = _init_l_Lean_Parser_Term_dep lean_mark_persistent(l_Lean_Parser_Term_depArrow_formatter___closed__5); l_Lean_Parser_Term_depArrow_formatter___closed__6 = _init_l_Lean_Parser_Term_depArrow_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_depArrow_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_depArrow_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_depArrow_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binderTactic_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_binderTactic_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binderTactic_parenthesizer___closed__1); l_Lean_Parser_Term_binderTactic_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_binderTactic_parenthesizer___closed__2(); @@ -92956,10 +99964,24 @@ l_Lean_Parser_Term_binderTactic_parenthesizer___closed__5 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_binderTactic_parenthesizer___closed__5); l_Lean_Parser_Term_binderTactic_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_binderTactic_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_binderTactic_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binderTactic_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binderDefault_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_binderDefault_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binderDefault_parenthesizer___closed__1); l_Lean_Parser_Term_binderDefault_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_binderDefault_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_binderDefault_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binderDefault_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__1); l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__2(); @@ -92972,10 +99994,6 @@ l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__5 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__5); l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__6); -l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__7); -l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_explicitBinder_parenthesizer___closed__8); l_Lean_Parser_Term_strictImplicitLeftBracket_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_strictImplicitLeftBracket_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_strictImplicitLeftBracket_parenthesizer___closed__1); l_Lean_Parser_Term_strictImplicitLeftBracket_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_strictImplicitLeftBracket_parenthesizer___closed__2(); @@ -93024,6 +100042,13 @@ l_Lean_Parser_Term_depArrow_parenthesizer___closed__5 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_depArrow_parenthesizer___closed__5); l_Lean_Parser_Term_depArrow_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_depArrow_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_depArrow_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_depArrow_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_forall___elambda__1___closed__1 = _init_l_Lean_Parser_Term_forall___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_forall___elambda__1___closed__1); l_Lean_Parser_Term_forall___elambda__1___closed__2 = _init_l_Lean_Parser_Term_forall___elambda__1___closed__2(); @@ -93124,8 +100149,13 @@ l_Lean_Parser_Term_typeSpec_formatter___closed__1 = _init_l_Lean_Parser_Term_typ lean_mark_persistent(l_Lean_Parser_Term_typeSpec_formatter___closed__1); l_Lean_Parser_Term_typeSpec_formatter___closed__2 = _init_l_Lean_Parser_Term_typeSpec_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_typeSpec_formatter___closed__2); -l_Lean_Parser_Term_optType_formatter___closed__1 = _init_l_Lean_Parser_Term_optType_formatter___closed__1(); -lean_mark_persistent(l_Lean_Parser_Term_optType_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeSpec_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_typeSpec_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_forall_formatter___closed__1 = _init_l_Lean_Parser_Term_forall_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_forall_formatter___closed__1); l_Lean_Parser_Term_forall_formatter___closed__2 = _init_l_Lean_Parser_Term_forall_formatter___closed__2(); @@ -93150,12 +100180,24 @@ l_Lean_Parser_Term_forall_formatter___closed__11 = _init_l_Lean_Parser_Term_fora lean_mark_persistent(l_Lean_Parser_Term_forall_formatter___closed__11); l_Lean_Parser_Term_forall_formatter___closed__12 = _init_l_Lean_Parser_Term_forall_formatter___closed__12(); lean_mark_persistent(l_Lean_Parser_Term_forall_formatter___closed__12); +l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forall_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_forall_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_typeSpec_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_typeSpec_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_typeSpec_parenthesizer___closed__1); l_Lean_Parser_Term_typeSpec_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_typeSpec_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_typeSpec_parenthesizer___closed__2); -l_Lean_Parser_Term_optType_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_optType_parenthesizer___closed__1(); -lean_mark_persistent(l_Lean_Parser_Term_optType_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_typeSpec_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_forall_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_forall_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_forall_parenthesizer___closed__1); l_Lean_Parser_Term_forall_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_forall_parenthesizer___closed__2(); @@ -93180,6 +100222,13 @@ l_Lean_Parser_Term_forall_parenthesizer___closed__11 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_forall_parenthesizer___closed__11); l_Lean_Parser_Term_forall_parenthesizer___closed__12 = _init_l_Lean_Parser_Term_forall_parenthesizer___closed__12(); lean_mark_persistent(l_Lean_Parser_Term_forall_parenthesizer___closed__12); +l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forall_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_forall_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchAlt___elambda__1___closed__1 = _init_l_Lean_Parser_Term_matchAlt___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchAlt___elambda__1___closed__1); l_Lean_Parser_Term_matchAlt___elambda__1___closed__2 = _init_l_Lean_Parser_Term_matchAlt___elambda__1___closed__2(); @@ -93524,12 +100573,26 @@ l_Lean_Parser_Term_trueVal_formatter___closed__2 = _init_l_Lean_Parser_Term_true lean_mark_persistent(l_Lean_Parser_Term_trueVal_formatter___closed__2); l_Lean_Parser_Term_trueVal_formatter___closed__3 = _init_l_Lean_Parser_Term_trueVal_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_trueVal_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_trueVal_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_trueVal_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_falseVal_formatter___closed__1 = _init_l_Lean_Parser_Term_falseVal_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_falseVal_formatter___closed__1); l_Lean_Parser_Term_falseVal_formatter___closed__2 = _init_l_Lean_Parser_Term_falseVal_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_falseVal_formatter___closed__2); l_Lean_Parser_Term_falseVal_formatter___closed__3 = _init_l_Lean_Parser_Term_falseVal_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_falseVal_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_falseVal_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_falseVal_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_generalizingParam_formatter___closed__1 = _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_formatter___closed__1); l_Lean_Parser_Term_generalizingParam_formatter___closed__2 = _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__2(); @@ -93550,10 +100613,13 @@ l_Lean_Parser_Term_generalizingParam_formatter___closed__9 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_formatter___closed__9); l_Lean_Parser_Term_generalizingParam_formatter___closed__10 = _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__10(); lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_formatter___closed__10); -l_Lean_Parser_Term_generalizingParam_formatter___closed__11 = _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__11(); -lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_formatter___closed__11); -l_Lean_Parser_Term_generalizingParam_formatter___closed__12 = _init_l_Lean_Parser_Term_generalizingParam_formatter___closed__12(); -lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_formatter___closed__12); +l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_generalizingParam_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_motive_formatter___closed__1 = _init_l_Lean_Parser_Term_motive_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_motive_formatter___closed__1); l_Lean_Parser_Term_motive_formatter___closed__2 = _init_l_Lean_Parser_Term_motive_formatter___closed__2(); @@ -93570,6 +100636,13 @@ l_Lean_Parser_Term_motive_formatter___closed__7 = _init_l_Lean_Parser_Term_motiv lean_mark_persistent(l_Lean_Parser_Term_motive_formatter___closed__7); l_Lean_Parser_Term_motive_formatter___closed__8 = _init_l_Lean_Parser_Term_motive_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_motive_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_motive_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_motive_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchDiscr_formatter___closed__1 = _init_l_Lean_Parser_Term_matchDiscr_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_formatter___closed__1); l_Lean_Parser_Term_matchDiscr_formatter___closed__2 = _init_l_Lean_Parser_Term_matchDiscr_formatter___closed__2(); @@ -93578,6 +100651,13 @@ l_Lean_Parser_Term_matchDiscr_formatter___closed__3 = _init_l_Lean_Parser_Term_m lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_formatter___closed__3); l_Lean_Parser_Term_matchDiscr_formatter___closed__4 = _init_l_Lean_Parser_Term_matchDiscr_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_matchDiscr_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchAlt_formatter___closed__1 = _init_l_Lean_Parser_Term_matchAlt_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchAlt_formatter___closed__1); l_Lean_Parser_Term_matchAlt_formatter___closed__2 = _init_l_Lean_Parser_Term_matchAlt_formatter___closed__2(); @@ -93618,24 +100698,39 @@ l_Lean_Parser_Term_match_formatter___closed__12 = _init_l_Lean_Parser_Term_match lean_mark_persistent(l_Lean_Parser_Term_match_formatter___closed__12); l_Lean_Parser_Term_match_formatter___closed__13 = _init_l_Lean_Parser_Term_match_formatter___closed__13(); lean_mark_persistent(l_Lean_Parser_Term_match_formatter___closed__13); -l_Lean_Parser_Term_match_formatter___closed__14 = _init_l_Lean_Parser_Term_match_formatter___closed__14(); -lean_mark_persistent(l_Lean_Parser_Term_match_formatter___closed__14); -l_Lean_Parser_Term_match_formatter___closed__15 = _init_l_Lean_Parser_Term_match_formatter___closed__15(); -lean_mark_persistent(l_Lean_Parser_Term_match_formatter___closed__15); -l_Lean_Parser_Term_match_formatter___closed__16 = _init_l_Lean_Parser_Term_match_formatter___closed__16(); -lean_mark_persistent(l_Lean_Parser_Term_match_formatter___closed__16); +l___regBuiltin_Lean_Parser_Term_match_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_match_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_match_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_match_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_match_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_match_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_match_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_trueVal_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_trueVal_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_trueVal_parenthesizer___closed__1); l_Lean_Parser_Term_trueVal_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_trueVal_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_trueVal_parenthesizer___closed__2); l_Lean_Parser_Term_trueVal_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_trueVal_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_trueVal_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_trueVal_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_falseVal_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_falseVal_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_falseVal_parenthesizer___closed__1); l_Lean_Parser_Term_falseVal_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_falseVal_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_falseVal_parenthesizer___closed__2); l_Lean_Parser_Term_falseVal_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_falseVal_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_falseVal_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_falseVal_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1); l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2(); @@ -93656,10 +100751,13 @@ l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__9 = _init_l_Lean_Pa lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__9); l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__10 = _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__10(); lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__10); -l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__11 = _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__11(); -lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__11); -l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__12 = _init_l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__12(); -lean_mark_persistent(l_Lean_Parser_Term_generalizingParam_parenthesizer___closed__12); +l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_generalizingParam_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_motive_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_motive_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_motive_parenthesizer___closed__1); l_Lean_Parser_Term_motive_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_motive_parenthesizer___closed__2(); @@ -93676,6 +100774,13 @@ l_Lean_Parser_Term_motive_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_m lean_mark_persistent(l_Lean_Parser_Term_motive_parenthesizer___closed__7); l_Lean_Parser_Term_motive_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_motive_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_motive_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_motive_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_motive_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1); l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2(); @@ -93684,6 +100789,13 @@ l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__3 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__3); l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_matchDiscr_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchAlt_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_matchAlt_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchAlt_parenthesizer___closed__1); l_Lean_Parser_Term_matchAlt_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_matchAlt_parenthesizer___closed__2(); @@ -93724,12 +100836,13 @@ l_Lean_Parser_Term_match_parenthesizer___closed__12 = _init_l_Lean_Parser_Term_m lean_mark_persistent(l_Lean_Parser_Term_match_parenthesizer___closed__12); l_Lean_Parser_Term_match_parenthesizer___closed__13 = _init_l_Lean_Parser_Term_match_parenthesizer___closed__13(); lean_mark_persistent(l_Lean_Parser_Term_match_parenthesizer___closed__13); -l_Lean_Parser_Term_match_parenthesizer___closed__14 = _init_l_Lean_Parser_Term_match_parenthesizer___closed__14(); -lean_mark_persistent(l_Lean_Parser_Term_match_parenthesizer___closed__14); -l_Lean_Parser_Term_match_parenthesizer___closed__15 = _init_l_Lean_Parser_Term_match_parenthesizer___closed__15(); -lean_mark_persistent(l_Lean_Parser_Term_match_parenthesizer___closed__15); -l_Lean_Parser_Term_match_parenthesizer___closed__16 = _init_l_Lean_Parser_Term_match_parenthesizer___closed__16(); -lean_mark_persistent(l_Lean_Parser_Term_match_parenthesizer___closed__16); +l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_match_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_match_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_nomatch___elambda__1___closed__1 = _init_l_Lean_Parser_Term_nomatch___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_nomatch___elambda__1___closed__1); l_Lean_Parser_Term_nomatch___elambda__1___closed__2 = _init_l_Lean_Parser_Term_nomatch___elambda__1___closed__2(); @@ -93800,6 +100913,13 @@ l_Lean_Parser_Term_nomatch_formatter___closed__3 = _init_l_Lean_Parser_Term_noma lean_mark_persistent(l_Lean_Parser_Term_nomatch_formatter___closed__3); l_Lean_Parser_Term_nomatch_formatter___closed__4 = _init_l_Lean_Parser_Term_nomatch_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_nomatch_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_nomatch_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_nomatch_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_nomatch_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_nomatch_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_nomatch_parenthesizer___closed__1); l_Lean_Parser_Term_nomatch_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_nomatch_parenthesizer___closed__2(); @@ -93808,6 +100928,13 @@ l_Lean_Parser_Term_nomatch_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_nomatch_parenthesizer___closed__3); l_Lean_Parser_Term_nomatch_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_nomatch_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_nomatch_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_nomatch_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__1 = _init_l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__1); l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__2 = _init_l_Lean_Parser_Term_funImplicitBinder___elambda__1___closed__2(); @@ -94092,6 +101219,13 @@ l_Lean_Parser_Term_basicFun_formatter___closed__10 = _init_l_Lean_Parser_Term_ba lean_mark_persistent(l_Lean_Parser_Term_basicFun_formatter___closed__10); l_Lean_Parser_Term_basicFun_formatter___closed__11 = _init_l_Lean_Parser_Term_basicFun_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Term_basicFun_formatter___closed__11); +l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_basicFun_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_basicFun_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_fun_formatter___closed__1 = _init_l_Lean_Parser_Term_fun_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_fun_formatter___closed__1); l_Lean_Parser_Term_fun_formatter___closed__2 = _init_l_Lean_Parser_Term_fun_formatter___closed__2(); @@ -94104,8 +101238,13 @@ l_Lean_Parser_Term_fun_formatter___closed__5 = _init_l_Lean_Parser_Term_fun_form lean_mark_persistent(l_Lean_Parser_Term_fun_formatter___closed__5); l_Lean_Parser_Term_fun_formatter___closed__6 = _init_l_Lean_Parser_Term_fun_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_fun_formatter___closed__6); -l_Lean_Parser_Term_fun_formatter___closed__7 = _init_l_Lean_Parser_Term_fun_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_fun_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_fun_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_fun_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__1); l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_funStrictImplicitBinder_parenthesizer___closed__2(); @@ -94166,6 +101305,13 @@ l_Lean_Parser_Term_basicFun_parenthesizer___closed__10 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_basicFun_parenthesizer___closed__10); l_Lean_Parser_Term_basicFun_parenthesizer___closed__11 = _init_l_Lean_Parser_Term_basicFun_parenthesizer___closed__11(); lean_mark_persistent(l_Lean_Parser_Term_basicFun_parenthesizer___closed__11); +l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_basicFun_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_fun_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_fun_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_fun_parenthesizer___closed__1); l_Lean_Parser_Term_fun_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_fun_parenthesizer___closed__2(); @@ -94178,8 +101324,13 @@ l_Lean_Parser_Term_fun_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_fun_ lean_mark_persistent(l_Lean_Parser_Term_fun_parenthesizer___closed__5); l_Lean_Parser_Term_fun_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_fun_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_fun_parenthesizer___closed__6); -l_Lean_Parser_Term_fun_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_fun_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_fun_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_fun_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_fun_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_optExprPrecedence___closed__1 = _init_l_Lean_Parser_Term_optExprPrecedence___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_optExprPrecedence___closed__1); l_Lean_Parser_Term_optExprPrecedence___closed__2 = _init_l_Lean_Parser_Term_optExprPrecedence___closed__2(); @@ -94338,6 +101489,13 @@ l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__6 = _init_l_Lean_Pa lean_mark_persistent(l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__6); l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__7 = _init_l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_leading__parser_formatter___closed__1 = _init_l_Lean_Parser_Term_leading__parser_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_leading__parser_formatter___closed__1); l_Lean_Parser_Term_leading__parser_formatter___closed__2 = _init_l_Lean_Parser_Term_leading__parser_formatter___closed__2(); @@ -94354,8 +101512,13 @@ l_Lean_Parser_Term_leading__parser_formatter___closed__7 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_leading__parser_formatter___closed__7); l_Lean_Parser_Term_leading__parser_formatter___closed__8 = _init_l_Lean_Parser_Term_leading__parser_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_leading__parser_formatter___closed__8); -l_Lean_Parser_Term_leading__parser_formatter___closed__9 = _init_l_Lean_Parser_Term_leading__parser_formatter___closed__9(); -lean_mark_persistent(l_Lean_Parser_Term_leading__parser_formatter___closed__9); +l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_leading__parser_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_leading__parser_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_optExprPrecedence_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_optExprPrecedence_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_optExprPrecedence_parenthesizer___closed__1); l_Lean_Parser_Term_optExprPrecedence_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_optExprPrecedence_parenthesizer___closed__2(); @@ -94376,6 +101539,13 @@ l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__6 = _init_l_Lea lean_mark_persistent(l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__6); l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_withAnonymousAntiquot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_leading__parser_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_leading__parser_parenthesizer___closed__1); l_Lean_Parser_Term_leading__parser_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__2(); @@ -94392,8 +101562,13 @@ l_Lean_Parser_Term_leading__parser_parenthesizer___closed__7 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Term_leading__parser_parenthesizer___closed__7); l_Lean_Parser_Term_leading__parser_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_leading__parser_parenthesizer___closed__8); -l_Lean_Parser_Term_leading__parser_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_leading__parser_parenthesizer___closed__9(); -lean_mark_persistent(l_Lean_Parser_Term_leading__parser_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_leading__parser_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_trailing__parser___elambda__1___closed__1 = _init_l_Lean_Parser_Term_trailing__parser___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_trailing__parser___elambda__1___closed__1); l_Lean_Parser_Term_trailing__parser___elambda__1___closed__2 = _init_l_Lean_Parser_Term_trailing__parser___elambda__1___closed__2(); @@ -94476,6 +101651,13 @@ l_Lean_Parser_Term_trailing__parser_formatter___closed__5 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_trailing__parser_formatter___closed__5); l_Lean_Parser_Term_trailing__parser_formatter___closed__6 = _init_l_Lean_Parser_Term_trailing__parser_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_trailing__parser_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_trailing__parser_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1); l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2(); @@ -94488,6 +101670,13 @@ l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__5 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__5); l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_trailing__parser_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_trailing__parser_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_borrowed___elambda__1___closed__1 = _init_l_Lean_Parser_Term_borrowed___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_borrowed___elambda__1___closed__1); l_Lean_Parser_Term_borrowed___elambda__1___closed__2 = _init_l_Lean_Parser_Term_borrowed___elambda__1___closed__2(); @@ -94562,6 +101751,13 @@ l_Lean_Parser_Term_borrowed_formatter___closed__3 = _init_l_Lean_Parser_Term_bor lean_mark_persistent(l_Lean_Parser_Term_borrowed_formatter___closed__3); l_Lean_Parser_Term_borrowed_formatter___closed__4 = _init_l_Lean_Parser_Term_borrowed_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_borrowed_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_borrowed_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_borrowed_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_borrowed_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_borrowed_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_borrowed_parenthesizer___closed__1); l_Lean_Parser_Term_borrowed_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_borrowed_parenthesizer___closed__2(); @@ -94572,6 +101768,13 @@ l_Lean_Parser_Term_borrowed_parenthesizer___closed__4 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_borrowed_parenthesizer___closed__4); l_Lean_Parser_Term_borrowed_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_borrowed_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_borrowed_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_borrowed_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_quotedName___elambda__1___closed__1 = _init_l_Lean_Parser_Term_quotedName___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_quotedName___elambda__1___closed__1); l_Lean_Parser_Term_quotedName___elambda__1___closed__2 = _init_l_Lean_Parser_Term_quotedName___elambda__1___closed__2(); @@ -94626,12 +101829,26 @@ l_Lean_Parser_Term_quotedName_formatter___closed__2 = _init_l_Lean_Parser_Term_q lean_mark_persistent(l_Lean_Parser_Term_quotedName_formatter___closed__2); l_Lean_Parser_Term_quotedName_formatter___closed__3 = _init_l_Lean_Parser_Term_quotedName_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_quotedName_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quotedName_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_quotedName_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_quotedName_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_quotedName_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_quotedName_parenthesizer___closed__1); l_Lean_Parser_Term_quotedName_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_quotedName_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_quotedName_parenthesizer___closed__2); l_Lean_Parser_Term_quotedName_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_quotedName_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_quotedName_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_quotedName_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__1 = _init_l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__1); l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__2 = _init_l_Lean_Parser_Term_doubleQuotedName___elambda__1___closed__2(); @@ -94730,6 +101947,13 @@ l_Lean_Parser_Term_doubleQuotedName_formatter___closed__7 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_doubleQuotedName_formatter___closed__7); l_Lean_Parser_Term_doubleQuotedName_formatter___closed__8 = _init_l_Lean_Parser_Term_doubleQuotedName_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_doubleQuotedName_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doubleQuotedName_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1); l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__2(); @@ -94748,6 +101972,13 @@ l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__7 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__7); l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_doubleQuotedName_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letIdBinder___elambda__1___closed__1 = _init_l_Lean_Parser_Term_letIdBinder___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letIdBinder___elambda__1___closed__1); l_Lean_Parser_Term_letIdBinder___elambda__1___closed__2 = _init_l_Lean_Parser_Term_letIdBinder___elambda__1___closed__2(); @@ -95030,6 +102261,13 @@ l_Lean_Parser_Term_letIdDecl_formatter___closed__5 = _init_l_Lean_Parser_Term_le lean_mark_persistent(l_Lean_Parser_Term_letIdDecl_formatter___closed__5); l_Lean_Parser_Term_letIdDecl_formatter___closed__6 = _init_l_Lean_Parser_Term_letIdDecl_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_letIdDecl_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letIdDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letPatDecl_formatter___closed__1 = _init_l_Lean_Parser_Term_letPatDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letPatDecl_formatter___closed__1); l_Lean_Parser_Term_letPatDecl_formatter___closed__2 = _init_l_Lean_Parser_Term_letPatDecl_formatter___closed__2(); @@ -95044,6 +102282,13 @@ l_Lean_Parser_Term_letPatDecl_formatter___closed__6 = _init_l_Lean_Parser_Term_l lean_mark_persistent(l_Lean_Parser_Term_letPatDecl_formatter___closed__6); l_Lean_Parser_Term_letPatDecl_formatter___closed__7 = _init_l_Lean_Parser_Term_letPatDecl_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_letPatDecl_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letPatDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letEqnsDecl_formatter___closed__1 = _init_l_Lean_Parser_Term_letEqnsDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letEqnsDecl_formatter___closed__1); l_Lean_Parser_Term_letEqnsDecl_formatter___closed__2 = _init_l_Lean_Parser_Term_letEqnsDecl_formatter___closed__2(); @@ -95052,6 +102297,13 @@ l_Lean_Parser_Term_letEqnsDecl_formatter___closed__3 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_letEqnsDecl_formatter___closed__3); l_Lean_Parser_Term_letEqnsDecl_formatter___closed__4 = _init_l_Lean_Parser_Term_letEqnsDecl_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_letEqnsDecl_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letEqnsDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letDecl_formatter___closed__1 = _init_l_Lean_Parser_Term_letDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letDecl_formatter___closed__1); l_Lean_Parser_Term_letDecl_formatter___closed__2 = _init_l_Lean_Parser_Term_letDecl_formatter___closed__2(); @@ -95066,12 +102318,13 @@ l_Lean_Parser_Term_letDecl_formatter___closed__6 = _init_l_Lean_Parser_Term_letD lean_mark_persistent(l_Lean_Parser_Term_letDecl_formatter___closed__6); l_Lean_Parser_Term_letDecl_formatter___closed__7 = _init_l_Lean_Parser_Term_letDecl_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_letDecl_formatter___closed__7); -l_Lean_Parser_Term_letDecl_formatter___closed__8 = _init_l_Lean_Parser_Term_letDecl_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_letDecl_formatter___closed__8); -l_Lean_Parser_Term_letDecl_formatter___closed__9 = _init_l_Lean_Parser_Term_letDecl_formatter___closed__9(); -lean_mark_persistent(l_Lean_Parser_Term_letDecl_formatter___closed__9); -l_Lean_Parser_Term_letDecl_formatter___closed__10 = _init_l_Lean_Parser_Term_letDecl_formatter___closed__10(); -lean_mark_persistent(l_Lean_Parser_Term_letDecl_formatter___closed__10); +l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_let_formatter___closed__1 = _init_l_Lean_Parser_Term_let_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_let_formatter___closed__1); l_Lean_Parser_Term_let_formatter___closed__2 = _init_l_Lean_Parser_Term_let_formatter___closed__2(); @@ -95084,8 +102337,13 @@ l_Lean_Parser_Term_let_formatter___closed__5 = _init_l_Lean_Parser_Term_let_form lean_mark_persistent(l_Lean_Parser_Term_let_formatter___closed__5); l_Lean_Parser_Term_let_formatter___closed__6 = _init_l_Lean_Parser_Term_let_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_let_formatter___closed__6); -l_Lean_Parser_Term_let_formatter___closed__7 = _init_l_Lean_Parser_Term_let_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_let_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_let_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_let_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_let_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_let_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_let_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letIdBinder_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letIdBinder_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letIdBinder_parenthesizer___closed__1); l_Lean_Parser_Term_letIdLhs_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letIdLhs_parenthesizer___closed__1(); @@ -95114,6 +102372,13 @@ l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__5 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__5); l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_letIdDecl_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letIdDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1); l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2(); @@ -95128,6 +102393,13 @@ l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__6 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__6); l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_letPatDecl_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letPatDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1); l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2(); @@ -95136,6 +102408,13 @@ l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__3 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__3); l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letEqnsDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letDecl_parenthesizer___closed__1); l_Lean_Parser_Term_letDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__2(); @@ -95150,12 +102429,13 @@ l_Lean_Parser_Term_letDecl_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_letDecl_parenthesizer___closed__6); l_Lean_Parser_Term_letDecl_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_letDecl_parenthesizer___closed__7); -l_Lean_Parser_Term_letDecl_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_letDecl_parenthesizer___closed__8); -l_Lean_Parser_Term_letDecl_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__9(); -lean_mark_persistent(l_Lean_Parser_Term_letDecl_parenthesizer___closed__9); -l_Lean_Parser_Term_letDecl_parenthesizer___closed__10 = _init_l_Lean_Parser_Term_letDecl_parenthesizer___closed__10(); -lean_mark_persistent(l_Lean_Parser_Term_letDecl_parenthesizer___closed__10); +l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_let_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_let_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_let_parenthesizer___closed__1); l_Lean_Parser_Term_let_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_let_parenthesizer___closed__2(); @@ -95168,8 +102448,13 @@ l_Lean_Parser_Term_let_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_let_ lean_mark_persistent(l_Lean_Parser_Term_let_parenthesizer___closed__5); l_Lean_Parser_Term_let_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_let_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_let_parenthesizer___closed__6); -l_Lean_Parser_Term_let_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_let_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_let_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_let_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_let__fun___elambda__1___closed__1 = _init_l_Lean_Parser_Term_let__fun___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_let__fun___elambda__1___closed__1); l_Lean_Parser_Term_let__fun___elambda__1___closed__2 = _init_l_Lean_Parser_Term_let__fun___elambda__1___closed__2(); @@ -95248,6 +102533,13 @@ l_Lean_Parser_Term_let__fun_formatter___closed__7 = _init_l_Lean_Parser_Term_let lean_mark_persistent(l_Lean_Parser_Term_let__fun_formatter___closed__7); l_Lean_Parser_Term_let__fun_formatter___closed__8 = _init_l_Lean_Parser_Term_let__fun_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_let__fun_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__fun_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_let__fun_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_let__fun_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_let__fun_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_let__fun_parenthesizer___closed__1); l_Lean_Parser_Term_let__fun_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_let__fun_parenthesizer___closed__2(); @@ -95264,6 +102556,13 @@ l_Lean_Parser_Term_let__fun_parenthesizer___closed__7 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_let__fun_parenthesizer___closed__7); l_Lean_Parser_Term_let__fun_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_let__fun_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_let__fun_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_let__fun_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_let__delayed___elambda__1___closed__1 = _init_l_Lean_Parser_Term_let__delayed___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_let__delayed___elambda__1___closed__1); l_Lean_Parser_Term_let__delayed___elambda__1___closed__2 = _init_l_Lean_Parser_Term_let__delayed___elambda__1___closed__2(); @@ -95340,6 +102639,13 @@ l_Lean_Parser_Term_let__delayed_formatter___closed__5 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_let__delayed_formatter___closed__5); l_Lean_Parser_Term_let__delayed_formatter___closed__6 = _init_l_Lean_Parser_Term_let__delayed_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_let__delayed_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__delayed_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_let__delayed_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_let__delayed_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_let__delayed_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_let__delayed_parenthesizer___closed__1); l_Lean_Parser_Term_let__delayed_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_let__delayed_parenthesizer___closed__2(); @@ -95352,6 +102658,13 @@ l_Lean_Parser_Term_let__delayed_parenthesizer___closed__5 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_let__delayed_parenthesizer___closed__5); l_Lean_Parser_Term_let__delayed_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_let__delayed_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_let__delayed_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_let__delayed_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_let__tmp___elambda__1___closed__1 = _init_l_Lean_Parser_Term_let__tmp___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_let__tmp___elambda__1___closed__1); l_Lean_Parser_Term_let__tmp___elambda__1___closed__2 = _init_l_Lean_Parser_Term_let__tmp___elambda__1___closed__2(); @@ -95428,6 +102741,13 @@ l_Lean_Parser_Term_let__tmp_formatter___closed__5 = _init_l_Lean_Parser_Term_let lean_mark_persistent(l_Lean_Parser_Term_let__tmp_formatter___closed__5); l_Lean_Parser_Term_let__tmp_formatter___closed__6 = _init_l_Lean_Parser_Term_let__tmp_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_let__tmp_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__tmp_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_let__tmp_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_let__tmp_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_let__tmp_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_let__tmp_parenthesizer___closed__1); l_Lean_Parser_Term_let__tmp_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_let__tmp_parenthesizer___closed__2(); @@ -95440,6 +102760,13 @@ l_Lean_Parser_Term_let__tmp_parenthesizer___closed__5 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_let__tmp_parenthesizer___closed__5); l_Lean_Parser_Term_let__tmp_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_let__tmp_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_let__tmp_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_let__tmp_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_haveIdLhs___elambda__1___closed__1 = _init_l_Lean_Parser_Term_haveIdLhs___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_haveIdLhs___elambda__1___closed__1); l_Lean_Parser_Term_haveIdLhs___elambda__1___closed__2 = _init_l_Lean_Parser_Term_haveIdLhs___elambda__1___closed__2(); @@ -95626,12 +102953,26 @@ l_Lean_Parser_Term_haveIdDecl_formatter___closed__5 = _init_l_Lean_Parser_Term_h lean_mark_persistent(l_Lean_Parser_Term_haveIdDecl_formatter___closed__5); l_Lean_Parser_Term_haveIdDecl_formatter___closed__6 = _init_l_Lean_Parser_Term_haveIdDecl_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_haveIdDecl_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_haveIdDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1 = _init_l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1); l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2 = _init_l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2); l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__3 = _init_l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_haveEqnsDecl_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_haveDecl_formatter___closed__1 = _init_l_Lean_Parser_Term_haveDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_haveDecl_formatter___closed__1); l_Lean_Parser_Term_haveDecl_formatter___closed__2 = _init_l_Lean_Parser_Term_haveDecl_formatter___closed__2(); @@ -95640,10 +102981,13 @@ l_Lean_Parser_Term_haveDecl_formatter___closed__3 = _init_l_Lean_Parser_Term_hav lean_mark_persistent(l_Lean_Parser_Term_haveDecl_formatter___closed__3); l_Lean_Parser_Term_haveDecl_formatter___closed__4 = _init_l_Lean_Parser_Term_haveDecl_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_haveDecl_formatter___closed__4); -l_Lean_Parser_Term_haveDecl_formatter___closed__5 = _init_l_Lean_Parser_Term_haveDecl_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_haveDecl_formatter___closed__5); -l_Lean_Parser_Term_haveDecl_formatter___closed__6 = _init_l_Lean_Parser_Term_haveDecl_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_haveDecl_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_haveDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_have_formatter___closed__1 = _init_l_Lean_Parser_Term_have_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_have_formatter___closed__1); l_Lean_Parser_Term_have_formatter___closed__2 = _init_l_Lean_Parser_Term_have_formatter___closed__2(); @@ -95656,8 +103000,13 @@ l_Lean_Parser_Term_have_formatter___closed__5 = _init_l_Lean_Parser_Term_have_fo lean_mark_persistent(l_Lean_Parser_Term_have_formatter___closed__5); l_Lean_Parser_Term_have_formatter___closed__6 = _init_l_Lean_Parser_Term_have_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_have_formatter___closed__6); -l_Lean_Parser_Term_have_formatter___closed__7 = _init_l_Lean_Parser_Term_have_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_have_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_have_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_have_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_have_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_have_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_have_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_have_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_have_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_haveIdLhs_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_haveIdLhs_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_haveIdLhs_parenthesizer___closed__1); l_Lean_Parser_Term_haveIdLhs_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_haveIdLhs_parenthesizer___closed__2(); @@ -95674,12 +103023,26 @@ l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__5 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__5); l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_haveIdDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1); l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2); l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_haveEqnsDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_haveDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_haveDecl_parenthesizer___closed__1); l_Lean_Parser_Term_haveDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__2(); @@ -95688,10 +103051,13 @@ l_Lean_Parser_Term_haveDecl_parenthesizer___closed__3 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_haveDecl_parenthesizer___closed__3); l_Lean_Parser_Term_haveDecl_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_haveDecl_parenthesizer___closed__4); -l_Lean_Parser_Term_haveDecl_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_haveDecl_parenthesizer___closed__5); -l_Lean_Parser_Term_haveDecl_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_haveDecl_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_haveDecl_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_haveDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_have_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_have_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_have_parenthesizer___closed__1); l_Lean_Parser_Term_have_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_have_parenthesizer___closed__2(); @@ -95704,8 +103070,13 @@ l_Lean_Parser_Term_have_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_hav lean_mark_persistent(l_Lean_Parser_Term_have_parenthesizer___closed__5); l_Lean_Parser_Term_have_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_have_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_have_parenthesizer___closed__6); -l_Lean_Parser_Term_have_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_have_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_have_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_have_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_have_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_scoped___elambda__1___closed__1 = _init_l_Lean_Parser_Term_scoped___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_scoped___elambda__1___closed__1); l_Lean_Parser_Term_scoped___elambda__1___closed__2 = _init_l_Lean_Parser_Term_scoped___elambda__1___closed__2(); @@ -96042,18 +103413,39 @@ l_Lean_Parser_Command_docComment_formatter___closed__7 = _init_l_Lean_Parser_Com lean_mark_persistent(l_Lean_Parser_Command_docComment_formatter___closed__7); l_Lean_Parser_Command_docComment_formatter___closed__8 = _init_l_Lean_Parser_Command_docComment_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_docComment_formatter___closed__8); +l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__1); +l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_docComment_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Command_docComment_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_scoped_formatter___closed__1 = _init_l_Lean_Parser_Term_scoped_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_scoped_formatter___closed__1); l_Lean_Parser_Term_scoped_formatter___closed__2 = _init_l_Lean_Parser_Term_scoped_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_scoped_formatter___closed__2); l_Lean_Parser_Term_scoped_formatter___closed__3 = _init_l_Lean_Parser_Term_scoped_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_scoped_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_scoped_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_scoped_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_local_formatter___closed__1 = _init_l_Lean_Parser_Term_local_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_local_formatter___closed__1); l_Lean_Parser_Term_local_formatter___closed__2 = _init_l_Lean_Parser_Term_local_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_local_formatter___closed__2); l_Lean_Parser_Term_local_formatter___closed__3 = _init_l_Lean_Parser_Term_local_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_local_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_local_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_local_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_local_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_local_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_local_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_local_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_local_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_attrKind_formatter___closed__1 = _init_l_Lean_Parser_Term_attrKind_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_attrKind_formatter___closed__1); l_Lean_Parser_Term_attrKind_formatter___closed__2 = _init_l_Lean_Parser_Term_attrKind_formatter___closed__2(); @@ -96062,10 +103454,13 @@ l_Lean_Parser_Term_attrKind_formatter___closed__3 = _init_l_Lean_Parser_Term_att lean_mark_persistent(l_Lean_Parser_Term_attrKind_formatter___closed__3); l_Lean_Parser_Term_attrKind_formatter___closed__4 = _init_l_Lean_Parser_Term_attrKind_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_attrKind_formatter___closed__4); -l_Lean_Parser_Term_attrKind_formatter___closed__5 = _init_l_Lean_Parser_Term_attrKind_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_attrKind_formatter___closed__5); -l_Lean_Parser_Term_attrKind_formatter___closed__6 = _init_l_Lean_Parser_Term_attrKind_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_attrKind_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attrKind_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_attrKind_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_attrInstance_formatter___closed__1 = _init_l_Lean_Parser_Term_attrInstance_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_attrInstance_formatter___closed__1); l_Lean_Parser_Term_attrInstance_formatter___closed__2 = _init_l_Lean_Parser_Term_attrInstance_formatter___closed__2(); @@ -96076,8 +103471,6 @@ l_Lean_Parser_Term_attrInstance_formatter___closed__4 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_attrInstance_formatter___closed__4); l_Lean_Parser_Term_attrInstance_formatter___closed__5 = _init_l_Lean_Parser_Term_attrInstance_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_attrInstance_formatter___closed__5); -l_Lean_Parser_Term_attrInstance_formatter___closed__6 = _init_l_Lean_Parser_Term_attrInstance_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_attrInstance_formatter___closed__6); l_Lean_Parser_Term_attributes_formatter___closed__1 = _init_l_Lean_Parser_Term_attributes_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_attributes_formatter___closed__1); l_Lean_Parser_Term_attributes_formatter___closed__2 = _init_l_Lean_Parser_Term_attributes_formatter___closed__2(); @@ -96092,6 +103485,13 @@ l_Lean_Parser_Term_attributes_formatter___closed__6 = _init_l_Lean_Parser_Term_a lean_mark_persistent(l_Lean_Parser_Term_attributes_formatter___closed__6); l_Lean_Parser_Term_attributes_formatter___closed__7 = _init_l_Lean_Parser_Term_attributes_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_attributes_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attributes_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_attributes_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letRecDecl_formatter___closed__1 = _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_formatter___closed__1); l_Lean_Parser_Term_letRecDecl_formatter___closed__2 = _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__2(); @@ -96104,18 +103504,26 @@ l_Lean_Parser_Term_letRecDecl_formatter___closed__5 = _init_l_Lean_Parser_Term_l lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_formatter___closed__5); l_Lean_Parser_Term_letRecDecl_formatter___closed__6 = _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_formatter___closed__6); -l_Lean_Parser_Term_letRecDecl_formatter___closed__7 = _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_formatter___closed__7); -l_Lean_Parser_Term_letRecDecl_formatter___closed__8 = _init_l_Lean_Parser_Term_letRecDecl_formatter___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letRecDecl_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letRecDecls_formatter___closed__1 = _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecls_formatter___closed__1); l_Lean_Parser_Term_letRecDecls_formatter___closed__2 = _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecls_formatter___closed__2); l_Lean_Parser_Term_letRecDecls_formatter___closed__3 = _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecls_formatter___closed__3); -l_Lean_Parser_Term_letRecDecls_formatter___closed__4 = _init_l_Lean_Parser_Term_letRecDecls_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Term_letRecDecls_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letRecDecls_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letrec_formatter___closed__1 = _init_l_Lean_Parser_Term_letrec_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letrec_formatter___closed__1); l_Lean_Parser_Term_letrec_formatter___closed__2 = _init_l_Lean_Parser_Term_letrec_formatter___closed__2(); @@ -96132,8 +103540,13 @@ l_Lean_Parser_Term_letrec_formatter___closed__7 = _init_l_Lean_Parser_Term_letre lean_mark_persistent(l_Lean_Parser_Term_letrec_formatter___closed__7); l_Lean_Parser_Term_letrec_formatter___closed__8 = _init_l_Lean_Parser_Term_letrec_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_letrec_formatter___closed__8); -l_Lean_Parser_Term_letrec_formatter___closed__9 = _init_l_Lean_Parser_Term_letrec_formatter___closed__9(); -lean_mark_persistent(l_Lean_Parser_Term_letrec_formatter___closed__9); +l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letrec_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letrec_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Command_docComment_parenthesizer___closed__1 = _init_l_Lean_Parser_Command_docComment_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Command_docComment_parenthesizer___closed__1); l_Lean_Parser_Command_docComment_parenthesizer___closed__2 = _init_l_Lean_Parser_Command_docComment_parenthesizer___closed__2(); @@ -96150,18 +103563,39 @@ l_Lean_Parser_Command_docComment_parenthesizer___closed__7 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Command_docComment_parenthesizer___closed__7); l_Lean_Parser_Command_docComment_parenthesizer___closed__8 = _init_l_Lean_Parser_Command_docComment_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Command_docComment_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Command_docComment_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_scoped_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_scoped_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_scoped_parenthesizer___closed__1); l_Lean_Parser_Term_scoped_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_scoped_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_scoped_parenthesizer___closed__2); l_Lean_Parser_Term_scoped_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_scoped_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_scoped_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_scoped_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_local_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_local_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_local_parenthesizer___closed__1); l_Lean_Parser_Term_local_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_local_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_local_parenthesizer___closed__2); l_Lean_Parser_Term_local_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_local_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_local_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_local_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_local_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_attrKind_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_attrKind_parenthesizer___closed__1); l_Lean_Parser_Term_attrKind_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__2(); @@ -96170,10 +103604,13 @@ l_Lean_Parser_Term_attrKind_parenthesizer___closed__3 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_attrKind_parenthesizer___closed__3); l_Lean_Parser_Term_attrKind_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_attrKind_parenthesizer___closed__4); -l_Lean_Parser_Term_attrKind_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_attrKind_parenthesizer___closed__5); -l_Lean_Parser_Term_attrKind_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_attrKind_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_attrKind_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_attrKind_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_attrInstance_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_attrInstance_parenthesizer___closed__1); l_Lean_Parser_Term_attrInstance_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__2(); @@ -96182,8 +103619,6 @@ l_Lean_Parser_Term_attrInstance_parenthesizer___closed__3 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_attrInstance_parenthesizer___closed__3); l_Lean_Parser_Term_attrInstance_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_attrInstance_parenthesizer___closed__4); -l_Lean_Parser_Term_attrInstance_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_attrInstance_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_attrInstance_parenthesizer___closed__5); l_Lean_Parser_Term_attributes_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_attributes_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_attributes_parenthesizer___closed__1); l_Lean_Parser_Term_attributes_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_attributes_parenthesizer___closed__2(); @@ -96198,6 +103633,13 @@ l_Lean_Parser_Term_attributes_parenthesizer___closed__6 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_attributes_parenthesizer___closed__6); l_Lean_Parser_Term_attributes_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_attributes_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_attributes_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_attributes_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1); l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2(); @@ -96210,18 +103652,26 @@ l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__5 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__5); l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__6); -l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__7); -l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__8(); -lean_mark_persistent(l_Lean_Parser_Term_letRecDecl_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letRecDecl_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1); l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2); l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__3); -l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__4(); -lean_mark_persistent(l_Lean_Parser_Term_letRecDecls_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letRecDecls_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letrec_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letrec_parenthesizer___closed__1); l_Lean_Parser_Term_letrec_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__2(); @@ -96238,8 +103688,13 @@ l_Lean_Parser_Term_letrec_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_l lean_mark_persistent(l_Lean_Parser_Term_letrec_parenthesizer___closed__7); l_Lean_Parser_Term_letrec_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_letrec_parenthesizer___closed__8); -l_Lean_Parser_Term_letrec_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_letrec_parenthesizer___closed__9(); -lean_mark_persistent(l_Lean_Parser_Term_letrec_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letrec_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_whereDecls_formatter___closed__1 = _init_l_Lean_Parser_Term_whereDecls_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_whereDecls_formatter___closed__1); l_Lean_Parser_Term_whereDecls_formatter___closed__2 = _init_l_Lean_Parser_Term_whereDecls_formatter___closed__2(); @@ -96262,6 +103717,13 @@ l_Lean_Parser_Term_whereDecls_formatter___closed__10 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_whereDecls_formatter___closed__10); l_Lean_Parser_Term_whereDecls_formatter___closed__11 = _init_l_Lean_Parser_Term_whereDecls_formatter___closed__11(); lean_mark_persistent(l_Lean_Parser_Term_whereDecls_formatter___closed__11); +l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_whereDecls_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_whereDecls_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_whereDecls_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_whereDecls_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_whereDecls_parenthesizer___closed__1); l_Lean_Parser_Term_whereDecls_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_whereDecls_parenthesizer___closed__2(); @@ -96276,6 +103738,13 @@ l_Lean_Parser_Term_whereDecls_parenthesizer___closed__6 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_whereDecls_parenthesizer___closed__6); l_Lean_Parser_Term_whereDecls_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_whereDecls_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_whereDecls_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_whereDecls_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_whereDecls___elambda__1___closed__1 = _init_l_Lean_Parser_Term_whereDecls___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_whereDecls___elambda__1___closed__1); l_Lean_Parser_Term_whereDecls___elambda__1___closed__2 = _init_l_Lean_Parser_Term_whereDecls___elambda__1___closed__2(); @@ -96348,8 +103817,13 @@ l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__5 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__5); l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__6 = _init_l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__6); -l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__7 = _init_l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__7(); -lean_mark_persistent(l_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1); l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2(); @@ -96358,8 +103832,13 @@ l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__3 = _init_l_Lean_ lean_mark_persistent(l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__3); l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__4); -l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_matchAltsWhereDecls_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__1 = _init_l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__1); l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__2 = _init_l_Lean_Parser_Term_matchAltsWhereDecls___elambda__1___closed__2(); @@ -96458,6 +103937,13 @@ l_Lean_Parser_Term_noindex_formatter___closed__3 = _init_l_Lean_Parser_Term_noin lean_mark_persistent(l_Lean_Parser_Term_noindex_formatter___closed__3); l_Lean_Parser_Term_noindex_formatter___closed__4 = _init_l_Lean_Parser_Term_noindex_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_noindex_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_noindex_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_noindex_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_noindex_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_noindex_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_noindex_parenthesizer___closed__1); l_Lean_Parser_Term_noindex_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_noindex_parenthesizer___closed__2(); @@ -96466,6 +103952,13 @@ l_Lean_Parser_Term_noindex_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_noindex_parenthesizer___closed__3); l_Lean_Parser_Term_noindex_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_noindex_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_noindex_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_noindex_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binrel___elambda__1___closed__1 = _init_l_Lean_Parser_Term_binrel___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binrel___elambda__1___closed__1); l_Lean_Parser_Term_binrel___elambda__1___closed__2 = _init_l_Lean_Parser_Term_binrel___elambda__1___closed__2(); @@ -96554,6 +104047,13 @@ l_Lean_Parser_Term_binrel_formatter___closed__6 = _init_l_Lean_Parser_Term_binre lean_mark_persistent(l_Lean_Parser_Term_binrel_formatter___closed__6); l_Lean_Parser_Term_binrel_formatter___closed__7 = _init_l_Lean_Parser_Term_binrel_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_binrel_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binrel_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binrel_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binrel_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_binrel_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binrel_parenthesizer___closed__1); l_Lean_Parser_Term_binrel_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_binrel_parenthesizer___closed__2(); @@ -96568,6 +104068,13 @@ l_Lean_Parser_Term_binrel_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_b lean_mark_persistent(l_Lean_Parser_Term_binrel_parenthesizer___closed__6); l_Lean_Parser_Term_binrel_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_binrel_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_binrel_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binrel_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__1 = _init_l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__1); l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__2 = _init_l_Lean_Parser_Term_binrel__no__prop___elambda__1___closed__2(); @@ -96643,6 +104150,13 @@ l_Lean_Parser_Term_binrel__no__prop_formatter___closed__3 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_binrel__no__prop_formatter___closed__3); l_Lean_Parser_Term_binrel__no__prop_formatter___closed__4 = _init_l_Lean_Parser_Term_binrel__no__prop_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_binrel__no__prop_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binrel__no__prop_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1); l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2(); @@ -96651,6 +104165,13 @@ l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__3 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__3); l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binrel__no__prop_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binop___elambda__1___closed__1 = _init_l_Lean_Parser_Term_binop___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binop___elambda__1___closed__1); l_Lean_Parser_Term_binop___elambda__1___closed__2 = _init_l_Lean_Parser_Term_binop___elambda__1___closed__2(); @@ -96721,6 +104242,13 @@ l_Lean_Parser_Term_binop_formatter___closed__3 = _init_l_Lean_Parser_Term_binop_ lean_mark_persistent(l_Lean_Parser_Term_binop_formatter___closed__3); l_Lean_Parser_Term_binop_formatter___closed__4 = _init_l_Lean_Parser_Term_binop_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_binop_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binop_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binop_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binop_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_binop_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binop_parenthesizer___closed__1); l_Lean_Parser_Term_binop_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_binop_parenthesizer___closed__2(); @@ -96729,6 +104257,13 @@ l_Lean_Parser_Term_binop_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_bi lean_mark_persistent(l_Lean_Parser_Term_binop_parenthesizer___closed__3); l_Lean_Parser_Term_binop_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_binop_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_binop_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binop_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binop_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binop__lazy___elambda__1___closed__1 = _init_l_Lean_Parser_Term_binop__lazy___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binop__lazy___elambda__1___closed__1); l_Lean_Parser_Term_binop__lazy___elambda__1___closed__2 = _init_l_Lean_Parser_Term_binop__lazy___elambda__1___closed__2(); @@ -96799,6 +104334,13 @@ l_Lean_Parser_Term_binop__lazy_formatter___closed__3 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_binop__lazy_formatter___closed__3); l_Lean_Parser_Term_binop__lazy_formatter___closed__4 = _init_l_Lean_Parser_Term_binop__lazy_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_binop__lazy_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binop__lazy_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1); l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2(); @@ -96807,6 +104349,13 @@ l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__3 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__3); l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_binop__lazy_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_binop__lazy_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_forInMacro___elambda__1___closed__1 = _init_l_Lean_Parser_Term_forInMacro___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_forInMacro___elambda__1___closed__1); l_Lean_Parser_Term_forInMacro___elambda__1___closed__2 = _init_l_Lean_Parser_Term_forInMacro___elambda__1___closed__2(); @@ -96883,6 +104432,13 @@ l_Lean_Parser_Term_forInMacro_formatter___closed__4 = _init_l_Lean_Parser_Term_f lean_mark_persistent(l_Lean_Parser_Term_forInMacro_formatter___closed__4); l_Lean_Parser_Term_forInMacro_formatter___closed__5 = _init_l_Lean_Parser_Term_forInMacro_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_forInMacro_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forInMacro_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_forInMacro_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_forInMacro_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_forInMacro_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_forInMacro_parenthesizer___closed__1); l_Lean_Parser_Term_forInMacro_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_forInMacro_parenthesizer___closed__2(); @@ -96893,6 +104449,13 @@ l_Lean_Parser_Term_forInMacro_parenthesizer___closed__4 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_forInMacro_parenthesizer___closed__4); l_Lean_Parser_Term_forInMacro_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_forInMacro_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_forInMacro_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_forInMacro_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__1 = _init_l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__1); l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__2 = _init_l_Lean_Parser_Term_forInMacro_x27___elambda__1___closed__2(); @@ -96963,6 +104526,13 @@ l_Lean_Parser_Term_forInMacro_x27_formatter___closed__3 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_forInMacro_x27_formatter___closed__3); l_Lean_Parser_Term_forInMacro_x27_formatter___closed__4 = _init_l_Lean_Parser_Term_forInMacro_x27_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_forInMacro_x27_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_forInMacro_x27_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1); l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2(); @@ -96971,6 +104541,13 @@ l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__3 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__3); l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_forInMacro_x27_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_typeOf___elambda__1___closed__1 = _init_l_Lean_Parser_Term_typeOf___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_typeOf___elambda__1___closed__1); l_Lean_Parser_Term_typeOf___elambda__1___closed__2 = _init_l_Lean_Parser_Term_typeOf___elambda__1___closed__2(); @@ -97041,6 +104618,13 @@ l_Lean_Parser_Term_typeOf_formatter___closed__3 = _init_l_Lean_Parser_Term_typeO lean_mark_persistent(l_Lean_Parser_Term_typeOf_formatter___closed__3); l_Lean_Parser_Term_typeOf_formatter___closed__4 = _init_l_Lean_Parser_Term_typeOf_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_typeOf_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeOf_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_typeOf_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_typeOf_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_typeOf_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_typeOf_parenthesizer___closed__1); l_Lean_Parser_Term_typeOf_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_typeOf_parenthesizer___closed__2(); @@ -97049,6 +104633,13 @@ l_Lean_Parser_Term_typeOf_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_t lean_mark_persistent(l_Lean_Parser_Term_typeOf_parenthesizer___closed__3); l_Lean_Parser_Term_typeOf_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_typeOf_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_typeOf_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_typeOf_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__1 = _init_l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__1); l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__2 = _init_l_Lean_Parser_Term_ensureTypeOf___elambda__1___closed__2(); @@ -97133,6 +104724,13 @@ l_Lean_Parser_Term_ensureTypeOf_formatter___closed__5 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_ensureTypeOf_formatter___closed__5); l_Lean_Parser_Term_ensureTypeOf_formatter___closed__6 = _init_l_Lean_Parser_Term_ensureTypeOf_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_ensureTypeOf_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_ensureTypeOf_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1); l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__2(); @@ -97145,6 +104743,13 @@ l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__5 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__5); l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_ensureTypeOf_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__1 = _init_l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__1); l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__2 = _init_l_Lean_Parser_Term_ensureExpectedType___elambda__1___closed__2(); @@ -97219,6 +104824,13 @@ l_Lean_Parser_Term_ensureExpectedType_formatter___closed__3 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_ensureExpectedType_formatter___closed__3); l_Lean_Parser_Term_ensureExpectedType_formatter___closed__4 = _init_l_Lean_Parser_Term_ensureExpectedType_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_ensureExpectedType_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_ensureExpectedType_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1); l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__2(); @@ -97229,6 +104841,13 @@ l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__4 = _init_l_Lean_P lean_mark_persistent(l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__4); l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_ensureExpectedType_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__1 = _init_l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__1); l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__2 = _init_l_Lean_Parser_Term_noImplicitLambda___elambda__1___closed__2(); @@ -97299,6 +104918,13 @@ l_Lean_Parser_Term_noImplicitLambda_formatter___closed__3 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_noImplicitLambda_formatter___closed__3); l_Lean_Parser_Term_noImplicitLambda_formatter___closed__4 = _init_l_Lean_Parser_Term_noImplicitLambda_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_noImplicitLambda_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_noImplicitLambda_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1); l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__2(); @@ -97307,6 +104933,13 @@ l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__3 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__3); l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_noImplicitLambda_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letMVar___elambda__1___closed__1 = _init_l_Lean_Parser_Term_letMVar___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letMVar___elambda__1___closed__1); l_Lean_Parser_Term_letMVar___elambda__1___closed__2 = _init_l_Lean_Parser_Term_letMVar___elambda__1___closed__2(); @@ -97411,6 +105044,13 @@ l_Lean_Parser_Term_letMVar_formatter___closed__8 = _init_l_Lean_Parser_Term_letM lean_mark_persistent(l_Lean_Parser_Term_letMVar_formatter___closed__8); l_Lean_Parser_Term_letMVar_formatter___closed__9 = _init_l_Lean_Parser_Term_letMVar_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_letMVar_formatter___closed__9); +l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letMVar_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letMVar_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_letMVar_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_letMVar_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_letMVar_parenthesizer___closed__1); l_Lean_Parser_Term_letMVar_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_letMVar_parenthesizer___closed__2(); @@ -97429,6 +105069,13 @@ l_Lean_Parser_Term_letMVar_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_letMVar_parenthesizer___closed__8); l_Lean_Parser_Term_letMVar_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_letMVar_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_letMVar_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_letMVar_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__1 = _init_l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__1); l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__2 = _init_l_Lean_Parser_Term_waitIfTypeMVar___elambda__1___closed__2(); @@ -97513,6 +105160,13 @@ l_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__5 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__5); l_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__6 = _init_l_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1); l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__2(); @@ -97527,6 +105181,13 @@ l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__6 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__6); l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_waitIfTypeMVar_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__1 = _init_l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__1); l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__2 = _init_l_Lean_Parser_Term_waitIfTypeContainsMVar___elambda__1___closed__2(); @@ -97597,6 +105258,13 @@ l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__3 = _init_l_Lean_P lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__3); l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__4 = _init_l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1); l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2(); @@ -97605,6 +105273,13 @@ l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__3 = _init_l_Le lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__3); l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_waitIfTypeContainsMVar_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__1 = _init_l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__1); l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__2 = _init_l_Lean_Parser_Term_waitIfContainsMVar___elambda__1___closed__2(); @@ -97675,6 +105350,13 @@ l_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__3 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__3); l_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__4 = _init_l_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1); l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2(); @@ -97683,6 +105365,13 @@ l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__3 = _init_l_Lean_P lean_mark_persistent(l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__3); l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_waitIfContainsMVar_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__1 = _init_l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__1); l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__2 = _init_l_Lean_Parser_Term_defaultOrOfNonempty___elambda__1___closed__2(); @@ -97769,6 +105458,13 @@ l_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__5 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__5); l_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__6 = _init_l_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1); l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2(); @@ -97781,6 +105477,13 @@ l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__5 = _init_l_Lean_ lean_mark_persistent(l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__5); l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_defaultOrOfNonempty_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_namedArgument___elambda__1___closed__1 = _init_l_Lean_Parser_Term_namedArgument___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_namedArgument___elambda__1___closed__1); l_Lean_Parser_Term_namedArgument___elambda__1___closed__2 = _init_l_Lean_Parser_Term_namedArgument___elambda__1___closed__2(); @@ -97927,24 +105630,41 @@ l_Lean_Parser_Term_namedArgument_formatter___closed__5 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_namedArgument_formatter___closed__5); l_Lean_Parser_Term_namedArgument_formatter___closed__6 = _init_l_Lean_Parser_Term_namedArgument_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_namedArgument_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_namedArgument_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_namedArgument_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_ellipsis_formatter___closed__1 = _init_l_Lean_Parser_Term_ellipsis_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_ellipsis_formatter___closed__1); l_Lean_Parser_Term_ellipsis_formatter___closed__2 = _init_l_Lean_Parser_Term_ellipsis_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_ellipsis_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ellipsis_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_ellipsis_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_argument_formatter___closed__1 = _init_l_Lean_Parser_Term_argument_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_argument_formatter___closed__1); l_Lean_Parser_Term_argument_formatter___closed__2 = _init_l_Lean_Parser_Term_argument_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_argument_formatter___closed__2); l_Lean_Parser_Term_argument_formatter___closed__3 = _init_l_Lean_Parser_Term_argument_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_argument_formatter___closed__3); -l_Lean_Parser_Term_argument_formatter___closed__4 = _init_l_Lean_Parser_Term_argument_formatter___closed__4(); -lean_mark_persistent(l_Lean_Parser_Term_argument_formatter___closed__4); -l_Lean_Parser_Term_argument_formatter___closed__5 = _init_l_Lean_Parser_Term_argument_formatter___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_argument_formatter___closed__5); l_Lean_Parser_Term_app_formatter___closed__1 = _init_l_Lean_Parser_Term_app_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_app_formatter___closed__1); l_Lean_Parser_Term_app_formatter___closed__2 = _init_l_Lean_Parser_Term_app_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_app_formatter___closed__2); +l___regBuiltin_Lean_Parser_Term_app_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_app_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_app_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_app_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_app_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_app_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_app_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_namedArgument_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_namedArgument_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_namedArgument_parenthesizer___closed__1); l_Lean_Parser_Term_namedArgument_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_namedArgument_parenthesizer___closed__2(); @@ -97957,10 +105677,24 @@ l_Lean_Parser_Term_namedArgument_parenthesizer___closed__5 = _init_l_Lean_Parser lean_mark_persistent(l_Lean_Parser_Term_namedArgument_parenthesizer___closed__5); l_Lean_Parser_Term_namedArgument_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_namedArgument_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_namedArgument_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_namedArgument_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_ellipsis_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_ellipsis_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_ellipsis_parenthesizer___closed__1); l_Lean_Parser_Term_ellipsis_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_ellipsis_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_ellipsis_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_ellipsis_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_argument_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_argument_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_argument_parenthesizer___closed__1); l_Lean_Parser_Term_argument_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_argument_parenthesizer___closed__2(); @@ -97969,14 +105703,17 @@ l_Lean_Parser_Term_argument_parenthesizer___closed__3 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_argument_parenthesizer___closed__3); l_Lean_Parser_Term_argument_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_argument_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_argument_parenthesizer___closed__4); -l_Lean_Parser_Term_argument_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_argument_parenthesizer___closed__5(); -lean_mark_persistent(l_Lean_Parser_Term_argument_parenthesizer___closed__5); -l_Lean_Parser_Term_argument_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_argument_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Term_argument_parenthesizer___closed__6); l_Lean_Parser_Term_app_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_app_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_app_parenthesizer___closed__1); l_Lean_Parser_Term_app_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_app_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_app_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_app_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_app_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_proj___elambda__1___closed__1 = _init_l_Lean_Parser_Term_proj___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_proj___elambda__1___closed__1); l_Lean_Parser_Term_proj___elambda__1___closed__2 = _init_l_Lean_Parser_Term_proj___elambda__1___closed__2(); @@ -98039,6 +105776,13 @@ l_Lean_Parser_Term_proj_formatter___closed__4 = _init_l_Lean_Parser_Term_proj_fo lean_mark_persistent(l_Lean_Parser_Term_proj_formatter___closed__4); l_Lean_Parser_Term_proj_formatter___closed__5 = _init_l_Lean_Parser_Term_proj_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_proj_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_proj_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_proj_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_proj_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_proj_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_proj_parenthesizer___closed__1); l_Lean_Parser_Term_proj_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_proj_parenthesizer___closed__2(); @@ -98049,6 +105793,13 @@ l_Lean_Parser_Term_proj_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_pro lean_mark_persistent(l_Lean_Parser_Term_proj_parenthesizer___closed__4); l_Lean_Parser_Term_proj_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_proj_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_proj_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_proj_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_proj_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_completion___elambda__1___closed__1 = _init_l_Lean_Parser_Term_completion___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_completion___elambda__1___closed__1); l_Lean_Parser_Term_completion___elambda__1___closed__2 = _init_l_Lean_Parser_Term_completion___elambda__1___closed__2(); @@ -98091,8 +105842,22 @@ if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Parser_Term_completion_formatter___closed__1 = _init_l_Lean_Parser_Term_completion_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_completion_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_completion_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_completion_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_completion_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_completion_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_completion_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_completion_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_completion_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_arrow___elambda__1___closed__1 = _init_l_Lean_Parser_Term_arrow___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_arrow___elambda__1___closed__1); l_Lean_Parser_Term_arrow___elambda__1___closed__2 = _init_l_Lean_Parser_Term_arrow___elambda__1___closed__2(); @@ -98139,6 +105904,13 @@ if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Parser_Term_arrow_formatter___closed__1 = _init_l_Lean_Parser_Term_arrow_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_arrow_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_arrow_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_arrow_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_arrow_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_arrow_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_arrow_parenthesizer___closed__1); l_Lean_Parser_Term_arrow_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_arrow_parenthesizer___closed__2(); @@ -98147,6 +105919,13 @@ l_Lean_Parser_Term_arrow_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_ar lean_mark_persistent(l_Lean_Parser_Term_arrow_parenthesizer___closed__3); l_Lean_Parser_Term_arrow_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_arrow_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_arrow_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_arrow_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_explicitUniv___elambda__1___closed__1 = _init_l_Lean_Parser_Term_explicitUniv___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_explicitUniv___elambda__1___closed__1); l_Lean_Parser_Term_explicitUniv___elambda__1___closed__2 = _init_l_Lean_Parser_Term_explicitUniv___elambda__1___closed__2(); @@ -98225,6 +106004,13 @@ l_Lean_Parser_Term_explicitUniv_formatter___closed__6 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_explicitUniv_formatter___closed__6); l_Lean_Parser_Term_explicitUniv_formatter___closed__7 = _init_l_Lean_Parser_Term_explicitUniv_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_explicitUniv_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_explicitUniv_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1); l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2(); @@ -98241,6 +106027,13 @@ l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__7 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__7); l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_explicitUniv_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_explicitUniv_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_namedPattern___elambda__1___closed__1 = _init_l_Lean_Parser_Term_namedPattern___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_namedPattern___elambda__1___closed__1); l_Lean_Parser_Term_namedPattern___elambda__1___closed__2 = _init_l_Lean_Parser_Term_namedPattern___elambda__1___closed__2(); @@ -98313,6 +106106,13 @@ l_Lean_Parser_Term_namedPattern_formatter___closed__6 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_namedPattern_formatter___closed__6); l_Lean_Parser_Term_namedPattern_formatter___closed__7 = _init_l_Lean_Parser_Term_namedPattern_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_namedPattern_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_namedPattern_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_namedPattern_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_namedPattern_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_namedPattern_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_namedPattern_parenthesizer___closed__1); l_Lean_Parser_Term_namedPattern_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_namedPattern_parenthesizer___closed__2(); @@ -98327,6 +106127,13 @@ l_Lean_Parser_Term_namedPattern_parenthesizer___closed__6 = _init_l_Lean_Parser_ lean_mark_persistent(l_Lean_Parser_Term_namedPattern_parenthesizer___closed__6); l_Lean_Parser_Term_namedPattern_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_namedPattern_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_namedPattern_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_namedPattern_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_pipeProj___elambda__1___closed__1 = _init_l_Lean_Parser_Term_pipeProj___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_pipeProj___elambda__1___closed__1); l_Lean_Parser_Term_pipeProj___elambda__1___closed__2 = _init_l_Lean_Parser_Term_pipeProj___elambda__1___closed__2(); @@ -98393,6 +106200,13 @@ l_Lean_Parser_Term_pipeProj_formatter___closed__4 = _init_l_Lean_Parser_Term_pip lean_mark_persistent(l_Lean_Parser_Term_pipeProj_formatter___closed__4); l_Lean_Parser_Term_pipeProj_formatter___closed__5 = _init_l_Lean_Parser_Term_pipeProj_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_pipeProj_formatter___closed__5); +l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeProj_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_pipeProj_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_pipeProj_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_pipeProj_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_pipeProj_parenthesizer___closed__1); l_Lean_Parser_Term_pipeProj_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_pipeProj_parenthesizer___closed__2(); @@ -98403,6 +106217,13 @@ l_Lean_Parser_Term_pipeProj_parenthesizer___closed__4 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_pipeProj_parenthesizer___closed__4); l_Lean_Parser_Term_pipeProj_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_pipeProj_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_pipeProj_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_pipeProj_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__1 = _init_l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__1); l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__2 = _init_l_Lean_Parser_Term_pipeCompletion___elambda__1___closed__2(); @@ -98441,6 +106262,20 @@ lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeCompletion_declRange___ res = l___regBuiltin_Lean_Parser_Term_pipeCompletion_declRange(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_pipeCompletion_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_pipeCompletion_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_subst___elambda__1___closed__1 = _init_l_Lean_Parser_Term_subst___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_subst___elambda__1___closed__1); l_Lean_Parser_Term_subst___elambda__1___closed__2 = _init_l_Lean_Parser_Term_subst___elambda__1___closed__2(); @@ -98505,6 +106340,13 @@ l_Lean_Parser_Term_subst_formatter___closed__2 = _init_l_Lean_Parser_Term_subst_ lean_mark_persistent(l_Lean_Parser_Term_subst_formatter___closed__2); l_Lean_Parser_Term_subst_formatter___closed__3 = _init_l_Lean_Parser_Term_subst_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_subst_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_subst_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_subst_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_subst_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_subst_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_subst_parenthesizer___closed__1); l_Lean_Parser_Term_subst_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_subst_parenthesizer___closed__2(); @@ -98513,6 +106355,13 @@ l_Lean_Parser_Term_subst_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_su lean_mark_persistent(l_Lean_Parser_Term_subst_parenthesizer___closed__3); l_Lean_Parser_Term_subst_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_subst_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_subst_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_subst_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_subst_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__1); l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_funBinder_quot___elambda__1___closed__2(); @@ -98599,6 +106448,13 @@ l_Lean_Parser_Term_funBinder_quot_formatter___closed__6 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_funBinder_quot_formatter___closed__6); l_Lean_Parser_Term_funBinder_quot_formatter___closed__7 = _init_l_Lean_Parser_Term_funBinder_quot_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_funBinder_quot_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_funBinder_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1); l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__2(); @@ -98613,6 +106469,13 @@ l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__6 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__6); l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_funBinder_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_bracketedBinderF = _init_l_Lean_Parser_Term_bracketedBinderF(); lean_mark_persistent(l_Lean_Parser_Term_bracketedBinderF); l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_bracketedBinder_quot___elambda__1___closed__1(); @@ -98701,6 +106564,13 @@ l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__6 = _init_l_Lean_Par lean_mark_persistent(l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__6); l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__7 = _init_l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1); l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__2(); @@ -98715,6 +106585,13 @@ l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__6 = _init_l_Lean lean_mark_persistent(l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__6); l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_bracketedBinder_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__1); l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_matchDiscr_quot___elambda__1___closed__2(); @@ -98797,6 +106674,13 @@ l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__6 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__6); l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__7 = _init_l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_quot_formatter___closed__7); +l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1); l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__2(); @@ -98811,6 +106695,13 @@ l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__6 = _init_l_Lean_Pars lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__6); l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__7 = _init_l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__7(); lean_mark_persistent(l_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__7); +l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_matchDiscr_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_attr_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_attr_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_attr_quot___elambda__1___closed__1); l_Lean_Parser_Term_attr_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_attr_quot___elambda__1___closed__2(); @@ -98891,6 +106782,13 @@ l_Lean_Parser_Term_attr_quot_formatter___closed__5 = _init_l_Lean_Parser_Term_at lean_mark_persistent(l_Lean_Parser_Term_attr_quot_formatter___closed__5); l_Lean_Parser_Term_attr_quot_formatter___closed__6 = _init_l_Lean_Parser_Term_attr_quot_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_attr_quot_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attr_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_attr_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_attr_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_attr_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_attr_quot_parenthesizer___closed__1); l_Lean_Parser_Term_attr_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_attr_quot_parenthesizer___closed__2(); @@ -98903,6 +106801,13 @@ l_Lean_Parser_Term_attr_quot_parenthesizer___closed__5 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_attr_quot_parenthesizer___closed__5); l_Lean_Parser_Term_attr_quot_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_attr_quot_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_attr_quot_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_attr_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_panic___elambda__1___closed__1 = _init_l_Lean_Parser_Term_panic___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_panic___elambda__1___closed__1); l_Lean_Parser_Term_panic___elambda__1___closed__2 = _init_l_Lean_Parser_Term_panic___elambda__1___closed__2(); @@ -98973,6 +106878,13 @@ l_Lean_Parser_Term_panic_formatter___closed__3 = _init_l_Lean_Parser_Term_panic_ lean_mark_persistent(l_Lean_Parser_Term_panic_formatter___closed__3); l_Lean_Parser_Term_panic_formatter___closed__4 = _init_l_Lean_Parser_Term_panic_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_panic_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_panic_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_panic_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_panic_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_panic_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_panic_parenthesizer___closed__1); l_Lean_Parser_Term_panic_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_panic_parenthesizer___closed__2(); @@ -98981,6 +106893,13 @@ l_Lean_Parser_Term_panic_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_pa lean_mark_persistent(l_Lean_Parser_Term_panic_parenthesizer___closed__3); l_Lean_Parser_Term_panic_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_panic_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_panic_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_panic_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_panic_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_unreachable___elambda__1___closed__1 = _init_l_Lean_Parser_Term_unreachable___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_unreachable___elambda__1___closed__1); l_Lean_Parser_Term_unreachable___elambda__1___closed__2 = _init_l_Lean_Parser_Term_unreachable___elambda__1___closed__2(); @@ -99045,12 +106964,26 @@ l_Lean_Parser_Term_unreachable_formatter___closed__2 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_unreachable_formatter___closed__2); l_Lean_Parser_Term_unreachable_formatter___closed__3 = _init_l_Lean_Parser_Term_unreachable_formatter___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_unreachable_formatter___closed__3); +l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_unreachable_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_unreachable_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_unreachable_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_unreachable_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_unreachable_parenthesizer___closed__1); l_Lean_Parser_Term_unreachable_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_unreachable_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Term_unreachable_parenthesizer___closed__2); l_Lean_Parser_Term_unreachable_parenthesizer___closed__3 = _init_l_Lean_Parser_Term_unreachable_parenthesizer___closed__3(); lean_mark_persistent(l_Lean_Parser_Term_unreachable_parenthesizer___closed__3); +l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_unreachable_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_dbgTrace___elambda__1___closed__1 = _init_l_Lean_Parser_Term_dbgTrace___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_dbgTrace___elambda__1___closed__1); l_Lean_Parser_Term_dbgTrace___elambda__1___closed__2 = _init_l_Lean_Parser_Term_dbgTrace___elambda__1___closed__2(); @@ -99125,6 +107058,13 @@ l_Lean_Parser_Term_dbgTrace_formatter___closed__7 = _init_l_Lean_Parser_Term_dbg lean_mark_persistent(l_Lean_Parser_Term_dbgTrace_formatter___closed__7); l_Lean_Parser_Term_dbgTrace_formatter___closed__8 = _init_l_Lean_Parser_Term_dbgTrace_formatter___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_dbgTrace_formatter___closed__8); +l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_dbgTrace_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1); l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2(); @@ -99141,6 +107081,13 @@ l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__7 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__7); l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__8 = _init_l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__8(); lean_mark_persistent(l_Lean_Parser_Term_dbgTrace_parenthesizer___closed__8); +l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_dbgTrace_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_assert___elambda__1___closed__1 = _init_l_Lean_Parser_Term_assert___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_assert___elambda__1___closed__1); l_Lean_Parser_Term_assert___elambda__1___closed__2 = _init_l_Lean_Parser_Term_assert___elambda__1___closed__2(); @@ -99207,6 +107154,13 @@ l_Lean_Parser_Term_assert_formatter___closed__5 = _init_l_Lean_Parser_Term_asser lean_mark_persistent(l_Lean_Parser_Term_assert_formatter___closed__5); l_Lean_Parser_Term_assert_formatter___closed__6 = _init_l_Lean_Parser_Term_assert_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_assert_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_assert_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_assert_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_assert_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_assert_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_assert_parenthesizer___closed__1); l_Lean_Parser_Term_assert_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_assert_parenthesizer___closed__2(); @@ -99219,6 +107173,13 @@ l_Lean_Parser_Term_assert_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_a lean_mark_persistent(l_Lean_Parser_Term_assert_parenthesizer___closed__5); l_Lean_Parser_Term_assert_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_assert_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_assert_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_assert_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_assert_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_macroArg = _init_l_Lean_Parser_Term_macroArg(); lean_mark_persistent(l_Lean_Parser_Term_macroArg); l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__1 = _init_l_Lean_Parser_Term_macroDollarArg___elambda__1___closed__1(); @@ -99349,10 +107310,15 @@ l_Lean_Parser_Term_macroDollarArg_formatter___closed__3 = _init_l_Lean_Parser_Te lean_mark_persistent(l_Lean_Parser_Term_macroDollarArg_formatter___closed__3); l_Lean_Parser_Term_macroDollarArg_formatter___closed__4 = _init_l_Lean_Parser_Term_macroDollarArg_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_macroDollarArg_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_macroDollarArg_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_macroLastArg_formatter___closed__1 = _init_l_Lean_Parser_Term_macroLastArg_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_macroLastArg_formatter___closed__1); -l_Lean_Parser_Term_macroLastArg_formatter___closed__2 = _init_l_Lean_Parser_Term_macroLastArg_formatter___closed__2(); -lean_mark_persistent(l_Lean_Parser_Term_macroLastArg_formatter___closed__2); l_Lean_Parser_Term_stateRefT_formatter___closed__1 = _init_l_Lean_Parser_Term_stateRefT_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_stateRefT_formatter___closed__1); l_Lean_Parser_Term_stateRefT_formatter___closed__2 = _init_l_Lean_Parser_Term_stateRefT_formatter___closed__2(); @@ -99365,6 +107331,13 @@ l_Lean_Parser_Term_stateRefT_formatter___closed__5 = _init_l_Lean_Parser_Term_st lean_mark_persistent(l_Lean_Parser_Term_stateRefT_formatter___closed__5); l_Lean_Parser_Term_stateRefT_formatter___closed__6 = _init_l_Lean_Parser_Term_stateRefT_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_stateRefT_formatter___closed__6); +l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_stateRefT_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_stateRefT_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1); l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2(); @@ -99375,10 +107348,15 @@ l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__4 = _init_l_Lean_Parse lean_mark_persistent(l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__4); l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__5 = _init_l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__5); +l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_macroDollarArg_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__1); -l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__2(); -lean_mark_persistent(l_Lean_Parser_Term_macroLastArg_parenthesizer___closed__2); l_Lean_Parser_Term_stateRefT_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_stateRefT_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_stateRefT_parenthesizer___closed__1); l_Lean_Parser_Term_stateRefT_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_stateRefT_parenthesizer___closed__2(); @@ -99391,6 +107369,13 @@ l_Lean_Parser_Term_stateRefT_parenthesizer___closed__5 = _init_l_Lean_Parser_Ter lean_mark_persistent(l_Lean_Parser_Term_stateRefT_parenthesizer___closed__5); l_Lean_Parser_Term_stateRefT_parenthesizer___closed__6 = _init_l_Lean_Parser_Term_stateRefT_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Term_stateRefT_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_stateRefT_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__1 = _init_l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__1); l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__2 = _init_l_Lean_Parser_Term_dynamicQuot___elambda__1___closed__2(); @@ -99493,6 +107478,13 @@ l_Lean_Parser_Term_dynamicQuot_formatter___closed__8 = _init_l_Lean_Parser_Term_ lean_mark_persistent(l_Lean_Parser_Term_dynamicQuot_formatter___closed__8); l_Lean_Parser_Term_dynamicQuot_formatter___closed__9 = _init_l_Lean_Parser_Term_dynamicQuot_formatter___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_dynamicQuot_formatter___closed__9); +l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_dynamicQuot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1); l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2(); @@ -99511,6 +107503,13 @@ l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__8 = _init_l_Lean_Parser_T lean_mark_persistent(l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__8); l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__9 = _init_l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__9(); lean_mark_persistent(l_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__9); +l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_dynamicQuot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_dotIdent___elambda__1___closed__1 = _init_l_Lean_Parser_Term_dotIdent___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_dotIdent___elambda__1___closed__1); l_Lean_Parser_Term_dotIdent___elambda__1___closed__2 = _init_l_Lean_Parser_Term_dotIdent___elambda__1___closed__2(); @@ -99573,6 +107572,13 @@ l_Lean_Parser_Term_dotIdent_formatter___closed__3 = _init_l_Lean_Parser_Term_dot lean_mark_persistent(l_Lean_Parser_Term_dotIdent_formatter___closed__3); l_Lean_Parser_Term_dotIdent_formatter___closed__4 = _init_l_Lean_Parser_Term_dotIdent_formatter___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_dotIdent_formatter___closed__4); +l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__1); +l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dotIdent_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Term_dotIdent_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Term_dotIdent_parenthesizer___closed__1 = _init_l_Lean_Parser_Term_dotIdent_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Term_dotIdent_parenthesizer___closed__1); l_Lean_Parser_Term_dotIdent_parenthesizer___closed__2 = _init_l_Lean_Parser_Term_dotIdent_parenthesizer___closed__2(); @@ -99581,6 +107587,13 @@ l_Lean_Parser_Term_dotIdent_parenthesizer___closed__3 = _init_l_Lean_Parser_Term lean_mark_persistent(l_Lean_Parser_Term_dotIdent_parenthesizer___closed__3); l_Lean_Parser_Term_dotIdent_parenthesizer___closed__4 = _init_l_Lean_Parser_Term_dotIdent_parenthesizer___closed__4(); lean_mark_persistent(l_Lean_Parser_Term_dotIdent_parenthesizer___closed__4); +l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Term_dotIdent_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Tactic_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_quot___elambda__1___closed__1); l_Lean_Parser_Tactic_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Tactic_quot___elambda__1___closed__2(); @@ -99659,6 +107672,13 @@ l_Lean_Parser_Tactic_quot_formatter___closed__5 = _init_l_Lean_Parser_Tactic_quo lean_mark_persistent(l_Lean_Parser_Tactic_quot_formatter___closed__5); l_Lean_Parser_Tactic_quot_formatter___closed__6 = _init_l_Lean_Parser_Tactic_quot_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Tactic_quot_formatter___closed__6); +l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_quot_parenthesizer___closed__1); l_Lean_Parser_Tactic_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_quot_parenthesizer___closed__2(); @@ -99671,6 +107691,13 @@ l_Lean_Parser_Tactic_quot_parenthesizer___closed__5 = _init_l_Lean_Parser_Tactic lean_mark_persistent(l_Lean_Parser_Tactic_quot_parenthesizer___closed__5); l_Lean_Parser_Tactic_quot_parenthesizer___closed__6 = _init_l_Lean_Parser_Tactic_quot_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Tactic_quot_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__1 = _init_l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__1); l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2 = _init_l_Lean_Parser_Tactic_quotSeq___elambda__1___closed__2(); @@ -99731,6 +107758,13 @@ l_Lean_Parser_Tactic_seq1_formatter___closed__1 = _init_l_Lean_Parser_Tactic_seq lean_mark_persistent(l_Lean_Parser_Tactic_seq1_formatter___closed__1); l_Lean_Parser_Tactic_seq1_formatter___closed__2 = _init_l_Lean_Parser_Tactic_seq1_formatter___closed__2(); lean_mark_persistent(l_Lean_Parser_Tactic_seq1_formatter___closed__2); +l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_seq1_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_seq1_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_quotSeq_formatter___closed__1 = _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq_formatter___closed__1); l_Lean_Parser_Tactic_quotSeq_formatter___closed__2 = _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__2(); @@ -99741,12 +107775,24 @@ l_Lean_Parser_Tactic_quotSeq_formatter___closed__4 = _init_l_Lean_Parser_Tactic_ lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq_formatter___closed__4); l_Lean_Parser_Tactic_quotSeq_formatter___closed__5 = _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__5(); lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq_formatter___closed__5); -l_Lean_Parser_Tactic_quotSeq_formatter___closed__6 = _init_l_Lean_Parser_Tactic_quotSeq_formatter___closed__6(); -lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq_formatter___closed__6); +l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__1); +l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_quotSeq_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_seq1_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_seq1_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_seq1_parenthesizer___closed__1); l_Lean_Parser_Tactic_seq1_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_seq1_parenthesizer___closed__2(); lean_mark_persistent(l_Lean_Parser_Tactic_seq1_parenthesizer___closed__2); +l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_seq1_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1 = _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1); l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2 = _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2(); @@ -99757,8 +107803,13 @@ l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__4 = _init_l_Lean_Parser_Tac lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__4); l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__5 = _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__5(); lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__5); -l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__6 = _init_l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__6(); -lean_mark_persistent(l_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__6); +l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Tactic_quotSeq_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_quot___elambda__1___closed__1 = _init_l_Lean_Parser_Level_quot___elambda__1___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_quot___elambda__1___closed__1); l_Lean_Parser_Level_quot___elambda__1___closed__2 = _init_l_Lean_Parser_Level_quot___elambda__1___closed__2(); @@ -99843,6 +107894,13 @@ l_Lean_Parser_Level_quot_formatter___closed__5 = _init_l_Lean_Parser_Level_quot_ lean_mark_persistent(l_Lean_Parser_Level_quot_formatter___closed__5); l_Lean_Parser_Level_quot_formatter___closed__6 = _init_l_Lean_Parser_Level_quot_formatter___closed__6(); lean_mark_persistent(l_Lean_Parser_Level_quot_formatter___closed__6); +l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__1); +l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_quot_formatter___closed__2); +res = l___regBuiltin_Lean_Parser_Level_quot_formatter(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_Parser_Level_quot_parenthesizer___closed__1 = _init_l_Lean_Parser_Level_quot_parenthesizer___closed__1(); lean_mark_persistent(l_Lean_Parser_Level_quot_parenthesizer___closed__1); l_Lean_Parser_Level_quot_parenthesizer___closed__2 = _init_l_Lean_Parser_Level_quot_parenthesizer___closed__2(); @@ -99855,109 +107913,112 @@ l_Lean_Parser_Level_quot_parenthesizer___closed__5 = _init_l_Lean_Parser_Level_q lean_mark_persistent(l_Lean_Parser_Level_quot_parenthesizer___closed__5); l_Lean_Parser_Level_quot_parenthesizer___closed__6 = _init_l_Lean_Parser_Level_quot_parenthesizer___closed__6(); lean_mark_persistent(l_Lean_Parser_Level_quot_parenthesizer___closed__6); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__1(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__1); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__2(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__2); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__3(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__3); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__4(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__4); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__5 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__5(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__5); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__6 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__6(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__6); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__7 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__7(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__7); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__8 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__8(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__8); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__9 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__9(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__9); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__10 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__10(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__10); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__11 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__11(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__11); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__12 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__12(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__12); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__13 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__13(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__13); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__14 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__14(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__14); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__15 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__15(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__15); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__16 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__16(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__16); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__17 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__17(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__17); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__18 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__18(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__18); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__19 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__19(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__19); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__20 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__20(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__20); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__21 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__21(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__21); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__22 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__22(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__22); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__23 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__23(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__23); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__24 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__24(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__24); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__25 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__25(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__25); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__26 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__26(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__26); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__27 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__27(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__27); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__28 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__28(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__28); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__29 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__29(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__29); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__30 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__30(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__30); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__31 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__31(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__31); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__32 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__32(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__32); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__33 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__33(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__33); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__34 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__34(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__34); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__35 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__35(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__35); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__36 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__36(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__36); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__37 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__37(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__37); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__38 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__38(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__38); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__39 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__39(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__39); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__40 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__40(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__40); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__41 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__41(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__41); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__42 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__42(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__42); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__43 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__43(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__43); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__44 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__44(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__44); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__45 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__45(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__45); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__46 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__46(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__46); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__47 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__47(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__47); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__48 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__48(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__48); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__49 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__49(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__49); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__50 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__50(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__50); -l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__51 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__51(); -lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808____closed__51); -res = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3808_(lean_io_mk_world()); +l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__1 = _init_l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__1); +l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__2 = _init_l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Parser_Level_quot_parenthesizer___closed__2); +res = l___regBuiltin_Lean_Parser_Level_quot_parenthesizer(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__1 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__1(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__1); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__2 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__2(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__2); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__3 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__3(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__3); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__4 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__4(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__4); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__5 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__5(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__5); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__6 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__6(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__6); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__7 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__7(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__7); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__8 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__8(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__8); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__9 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__9(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__9); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__10 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__10(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__10); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__11 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__11(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__11); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__12 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__12(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__12); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__13 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__13(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__13); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__14 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__14(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__14); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__15 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__15(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__15); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__16 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__16(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__16); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__17 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__17(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__17); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__18 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__18(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__18); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__19 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__19(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__19); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__20 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__20(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__20); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__21 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__21(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__21); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__22 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__22(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__22); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__23 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__23(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__23); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__24 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__24(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__24); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__25 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__25(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__25); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__26 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__26(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__26); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__27 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__27(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__27); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__28 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__28(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__28); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__29 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__29(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__29); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__30 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__30(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__30); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__31 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__31(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__31); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__32 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__32(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__32); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__33 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__33(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__33); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__34 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__34(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__34); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__35 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__35(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__35); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__36 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__36(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__36); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__37 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__37(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__37); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__38 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__38(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__38); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__39 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__39(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__39); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__40 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__40(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__40); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__41 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__41(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__41); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__42 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__42(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__42); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__43 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__43(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__43); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__44 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__44(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__44); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__45 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__45(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__45); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__46 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__46(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__46); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__47 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__47(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__47); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__48 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__48(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__48); +l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__49 = _init_l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__49(); +lean_mark_persistent(l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806____closed__49); +res = l_Lean_Parser_initFn____x40_Lean_Parser_Term___hyg_3806_(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/ParserCompiler.c b/stage0/stdlib/Lean/ParserCompiler.c index 78538245ff5f..69fff03ca12f 100644 --- a/stage0/stdlib/Lean/ParserCompiler.c +++ b/stage0/stdlib/Lean/ParserCompiler.c @@ -214,6 +214,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__16; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1(lean_object*, lean_object*); @@ -304,7 +305,6 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28___boxed(lean_object**); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__10; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48(lean_object*); @@ -1288,7 +1288,7 @@ else lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_dec(x_11); x_28 = lean_unsigned_to_nat(0u); -x_29 = l_Lean_Expr_getAppNumArgsAux(x_9, x_28); +x_29 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_28); x_30 = lean_nat_sub(x_29, x_28); lean_dec(x_29); x_31 = lean_unsigned_to_nat(1u); @@ -1359,7 +1359,7 @@ else lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_dec(x_11); x_48 = lean_unsigned_to_nat(0u); -x_49 = l_Lean_Expr_getAppNumArgsAux(x_9, x_48); +x_49 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_48); x_50 = lean_nat_sub(x_49, x_48); lean_dec(x_49); x_51 = lean_unsigned_to_nat(1u); @@ -1430,7 +1430,7 @@ else lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_dec(x_11); x_68 = lean_unsigned_to_nat(0u); -x_69 = l_Lean_Expr_getAppNumArgsAux(x_9, x_68); +x_69 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_68); x_70 = lean_nat_sub(x_69, x_68); lean_dec(x_69); x_71 = lean_unsigned_to_nat(1u); @@ -1501,7 +1501,7 @@ else lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_dec(x_11); x_88 = lean_unsigned_to_nat(0u); -x_89 = l_Lean_Expr_getAppNumArgsAux(x_9, x_88); +x_89 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_88); x_90 = lean_unsigned_to_nat(1u); x_91 = lean_nat_sub(x_89, x_90); lean_dec(x_89); @@ -1518,7 +1518,7 @@ else lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_dec(x_11); x_95 = lean_unsigned_to_nat(0u); -x_96 = l_Lean_Expr_getAppNumArgsAux(x_9, x_95); +x_96 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_95); x_97 = lean_unsigned_to_nat(1u); x_98 = lean_nat_sub(x_96, x_97); lean_dec(x_96); @@ -1846,7 +1846,7 @@ static lean_object* _init_l_Std_Range_forIn_loop___at_Lean_ParserCompiler_compil lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_Range_forIn_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___rarg___closed__1; x_2 = l_Std_Range_forIn_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___rarg___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_Range_forIn_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -21619,7 +21619,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -22296,7 +22296,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -22434,7 +22434,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -23059,7 +23059,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -23197,7 +23197,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -23822,7 +23822,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -23960,7 +23960,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -24585,7 +24585,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -24723,7 +24723,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -25348,7 +25348,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -25542,7 +25542,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -26167,7 +26167,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -26305,7 +26305,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -26930,7 +26930,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -27068,7 +27068,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -27693,7 +27693,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -27831,7 +27831,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -28456,7 +28456,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -28594,7 +28594,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -29219,7 +29219,7 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); diff --git a/stage0/stdlib/Lean/PrettyPrinter.c b/stage0/stdlib/Lean/PrettyPrinter.c index 9d88fd6d9a8a..e7c6c1373595 100644 --- a/stage0/stdlib/Lean/PrettyPrinter.c +++ b/stage0/stdlib/Lean/PrettyPrinter.c @@ -14,6 +14,7 @@ extern "C" { #endif lean_object* l_Lean_sanitizeSyntax(lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_ppCommand___closed__1; static lean_object* l_Lean_PrettyPrinter_ppExprLegacy___closed__1; size_t lean_usize_add(size_t, size_t); lean_object* lean_io_get_num_heartbeats(lean_object*); @@ -27,7 +28,6 @@ LEAN_EXPORT lean_object* l_Lean_PPContext_runMetaM___rarg(lean_object*, lean_obj static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__7; lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__16; -lean_object* l_Lean_PrettyPrinter_formatTerm(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_Parser_Module_module_formatter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_MetaM_run_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -36,20 +36,21 @@ lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -lean_object* l_Lean_PrettyPrinter_parenthesizeCommand(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_PrettyPrinter_parenthesizeTerm(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runMetaM___rarg___closed__4; uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_noContext___spec__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppCategory(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); lean_object* l_Lean_Meta_ppGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_ppConst___closed__1; -static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__3; +static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__5; LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__5; +static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__3; static lean_object* l_Lean_PPContext_runMetaM___rarg___closed__9; extern lean_object* l_Lean_PrettyPrinter_parenthesizerAttribute; static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__6; +lean_object* l_Lean_PrettyPrinter_formatCategory(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_toString(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppModule(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__14; @@ -61,10 +62,11 @@ static lean_object* l_Lean_PrettyPrinter_ppExpr___closed__1; static lean_object* l_Lean_PPContext_runMetaM___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppCommand(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runMetaM___rarg___closed__6; +lean_object* l_Lean_PrettyPrinter_parenthesizeCategory(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PPContext_runCoreM___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppTerm(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619_(lean_object*); static lean_object* l_Lean_PrettyPrinter_ppExprLegacy___closed__2; lean_object* l_Nat_repr(lean_object*); static lean_object* l_Lean_PrettyPrinter_registerParserCompilers___closed__2; @@ -87,70 +89,71 @@ static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__4; static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__8; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_registerParserCompilers(lean_object*); extern lean_object* l_Lean_firstFrontendMacroScope; +static lean_object* l_Lean_PrettyPrinter_ppCommand___closed__2; static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__17; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppTactic(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__2; LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_noContext(lean_object*); static lean_object* l_Lean_PrettyPrinter_registerParserCompilers___closed__9; static lean_object* l_Lean_PrettyPrinter_registerParserCompilers___closed__4; -static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__2; +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__9; size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lean_PPContext_runMetaM___rarg___closed__2; lean_object* l_Lean_PrettyPrinter_format(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppConst___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PPContext_runCoreM___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_registerParserCompilers___closed__6; -static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__1; +static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__1; static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__2; lean_object* l_Lean_PrettyPrinter_delab(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__1; lean_object* l_Lean_PrettyPrinter_Delaborator_delab(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_ppTerm___closed__2; static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__15; static lean_object* l_Lean_PPContext_runMetaM___rarg___closed__7; -lean_object* l_Lean_PrettyPrinter_formatCommand(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_ppModule___closed__2; LEAN_EXPORT lean_object* l_Lean_PPContext_runCoreM(lean_object*); static lean_object* l_Lean_PPContext_runMetaM___rarg___closed__8; +static lean_object* l_Lean_PrettyPrinter_ppTactic___closed__2; extern lean_object* l_Lean_PrettyPrinter_combinatorParenthesizerAttribute; static lean_object* l_Lean_PrettyPrinter_ppModule___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__5; +static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__4; LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___rarg___lambda__1(lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__3; -static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__4; +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext(lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__1___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_PrettyPrinter_parenthesizeTactic(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Module_module_parenthesizer(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___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_delabCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__12; lean_object* l_Lean_PrettyPrinter_Delaborator_delabConst(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_ppTactic___closed__1; extern lean_object* l_Lean_Expr_instBEqExpr; -LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____spec__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__3(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_ppTerm___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppUsing___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_noContext___spec__1(size_t, size_t, lean_object*); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__11; -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__2___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__1; static lean_object* l_Lean_PrettyPrinter_registerParserCompilers___closed__3; +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PPContext_runCoreM___rarg___closed__13; +static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__1; static lean_object* l_Lean_PPContext_runMetaM___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_PPContext_runMetaM(lean_object*); static lean_object* l_Lean_PrettyPrinter_registerParserCompilers___closed__5; static lean_object* l_Lean_PrettyPrinter_ppExprLegacy___closed__3; static lean_object* l_Lean_PrettyPrinter_registerParserCompilers___closed__10; -static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppExprWithInfos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalContext_sanitizeNames(lean_object*, lean_object*); -lean_object* l_Lean_PrettyPrinter_formatTactic(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__2; static lean_object* _init_l_Lean_PPContext_runCoreM___rarg___closed__1() { _start: { @@ -720,59 +723,88 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppTerm(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppCategory(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_5 = lean_ctor_get(x_2, 2); -lean_inc(x_5); -x_6 = lean_box(0); -x_7 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_7, 0, x_5); -lean_ctor_set(x_7, 1, x_6); -lean_ctor_set(x_7, 2, x_6); -x_8 = l_Lean_sanitizeSyntax(x_1, x_7); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -lean_dec(x_8); +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_6 = lean_ctor_get(x_3, 2); +lean_inc(x_6); +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_8, 0, x_6); +lean_ctor_set(x_8, 1, x_7); +lean_ctor_set(x_8, 2, x_7); +x_9 = l_Lean_sanitizeSyntax(x_2, x_8); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +lean_dec(x_9); +lean_inc(x_4); lean_inc(x_3); -lean_inc(x_2); -x_10 = l_Lean_PrettyPrinter_parenthesizeTerm(x_9, x_2, x_3, x_4); -if (lean_obj_tag(x_10) == 0) +lean_inc(x_1); +x_11 = l_Lean_PrettyPrinter_parenthesizeCategory(x_1, x_10, x_3, x_4, x_5); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_PrettyPrinter_formatTerm(x_11, x_2, x_3, x_12); -return x_13; +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_PrettyPrinter_formatCategory(x_1, x_12, x_3, x_4, x_13); +return x_14; } else { -uint8_t x_14; +uint8_t x_15; +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_14 = !lean_is_exclusive(x_10); -if (x_14 == 0) +lean_dec(x_1); +x_15 = !lean_is_exclusive(x_11); +if (x_15 == 0) { -return x_10; +return x_11; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_10, 0); -x_16 = lean_ctor_get(x_10, 1); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 0); +x_17 = lean_ctor_get(x_11, 1); +lean_inc(x_17); lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_10); -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -return x_17; +lean_dec(x_11); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +return x_18; +} +} +} +} +static lean_object* _init_l_Lean_PrettyPrinter_ppTerm___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("term", 4); +return x_1; +} +} +static lean_object* _init_l_Lean_PrettyPrinter_ppTerm___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_PrettyPrinter_ppTerm___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppTerm(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; +x_5 = l_Lean_PrettyPrinter_ppTerm___closed__2; +x_6 = l_Lean_PrettyPrinter_ppCategory(x_5, x_1, x_2, x_3, x_4); +return x_6; } } LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppUsing___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) { @@ -1490,92 +1522,58 @@ return x_18; } } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppTactic(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_PrettyPrinter_ppTactic___closed__1() { _start: { -lean_object* x_5; -lean_inc(x_3); -lean_inc(x_2); -x_5 = l_Lean_PrettyPrinter_parenthesizeTactic(x_1, x_2, x_3, x_4); -if (lean_obj_tag(x_5) == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_ctor_get(x_5, 1); -lean_inc(x_7); -lean_dec(x_5); -x_8 = l_Lean_PrettyPrinter_formatTactic(x_6, x_2, x_3, x_7); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("tactic", 6); +return x_1; } -else -{ -uint8_t x_9; -lean_dec(x_3); -lean_dec(x_2); -x_9 = !lean_is_exclusive(x_5); -if (x_9 == 0) -{ -return x_5; } -else +static lean_object* _init_l_Lean_PrettyPrinter_ppTactic___closed__2() { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_5, 0); -x_11 = lean_ctor_get(x_5, 1); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_5); -x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_11); -return x_12; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_PrettyPrinter_ppTactic___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppTactic(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; +x_5 = l_Lean_PrettyPrinter_ppTactic___closed__2; +x_6 = l_Lean_PrettyPrinter_ppCategory(x_5, x_1, x_2, x_3, x_4); +return x_6; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppCommand(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_PrettyPrinter_ppCommand___closed__1() { _start: { -lean_object* x_5; -lean_inc(x_3); -lean_inc(x_2); -x_5 = l_Lean_PrettyPrinter_parenthesizeCommand(x_1, x_2, x_3, x_4); -if (lean_obj_tag(x_5) == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_ctor_get(x_5, 1); -lean_inc(x_7); -lean_dec(x_5); -x_8 = l_Lean_PrettyPrinter_formatCommand(x_6, x_2, x_3, x_7); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("command", 7); +return x_1; } -else -{ -uint8_t x_9; -lean_dec(x_3); -lean_dec(x_2); -x_9 = !lean_is_exclusive(x_5); -if (x_9 == 0) -{ -return x_5; } -else +static lean_object* _init_l_Lean_PrettyPrinter_ppCommand___closed__2() { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_5, 0); -x_11 = lean_ctor_get(x_5, 1); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_5); -x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_11); -return x_12; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_PrettyPrinter_ppCommand___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_ppCommand(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; +x_5 = l_Lean_PrettyPrinter_ppCommand___closed__2; +x_6 = l_Lean_PrettyPrinter_ppCategory(x_5, x_1, x_2, x_3, x_4); +return x_6; } } static lean_object* _init_l_Lean_PrettyPrinter_ppModule___closed__1() { @@ -1934,7 +1932,7 @@ x_2 = lean_alloc_closure((void*)(l___private_Lean_PrettyPrinter_0__Lean_PrettyPr return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; @@ -2040,7 +2038,7 @@ return x_28; } } } -LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; @@ -2146,73 +2144,73 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_ppExpr), 6, 1); lean_closure_set(x_4, 0, x_2); -x_5 = lean_alloc_closure((void*)(l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____spec__1), 6, 1); +x_5 = lean_alloc_closure((void*)(l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____spec__1), 6, 1); lean_closure_set(x_5, 0, x_4); x_6 = l_Lean_PPContext_runMetaM___rarg(x_1, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_ppTerm), 4, 1); lean_closure_set(x_4, 0, x_2); -x_5 = lean_alloc_closure((void*)(l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____spec__2), 4, 1); +x_5 = lean_alloc_closure((void*)(l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____spec__2), 4, 1); lean_closure_set(x_5, 0, x_4); x_6 = l_Lean_PPContext_runCoreM___rarg(x_1, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_alloc_closure((void*)(l_Lean_Meta_ppGoal), 6, 1); lean_closure_set(x_4, 0, x_2); -x_5 = lean_alloc_closure((void*)(l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____spec__1), 6, 1); +x_5 = lean_alloc_closure((void*)(l___private_Lean_PrettyPrinter_0__Lean_PrettyPrinter_withoutContext___at_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____spec__1), 6, 1); lean_closure_set(x_5, 0, x_4); x_6 = l_Lean_PPContext_runMetaM___rarg(x_1, x_5, x_3); return x_6; } } -static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__1() { +static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__1___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__1___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__2() { +static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__2___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__2___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__3() { +static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__3___boxed), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__3___boxed), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__4() { +static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__1; -x_2 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__2; -x_3 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__3; +x_1 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__1; +x_2 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__2; +x_3 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__3; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -2220,7 +2218,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__5() { +static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__5() { _start: { lean_object* x_1; @@ -2228,12 +2226,12 @@ x_1 = l_Lean_ppFnsRef; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_2 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__5; -x_3 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__4; +x_2 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__5; +x_3 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__4; x_4 = lean_st_ref_set(x_2, x_3, x_1); x_5 = !lean_is_exclusive(x_4); if (x_5 == 0) @@ -2255,34 +2253,34 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__1(x_1, x_2, x_3); +x_4 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__1(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__2(x_1, x_2, x_3); +x_4 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__2(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____lambda__3(x_1, x_2, x_3); +x_4 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____lambda__3(x_1, x_2, x_3); lean_dec(x_1); return x_4; } } -static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__1() { +static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__1() { _start: { lean_object* x_1; @@ -2290,21 +2288,21 @@ x_1 = lean_mk_string_from_bytes("PrettyPrinter", 13); return x_1; } } -static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__2() { +static lean_object* _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__1; +x_2 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__2; +x_2 = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__2; x_3 = l_Lean_registerTraceClass(x_2, x_1); return x_3; } @@ -2500,6 +2498,10 @@ l_Lean_PPContext_runMetaM___rarg___closed__8 = _init_l_Lean_PPContext_runMetaM__ lean_mark_persistent(l_Lean_PPContext_runMetaM___rarg___closed__8); l_Lean_PPContext_runMetaM___rarg___closed__9 = _init_l_Lean_PPContext_runMetaM___rarg___closed__9(); lean_mark_persistent(l_Lean_PPContext_runMetaM___rarg___closed__9); +l_Lean_PrettyPrinter_ppTerm___closed__1 = _init_l_Lean_PrettyPrinter_ppTerm___closed__1(); +lean_mark_persistent(l_Lean_PrettyPrinter_ppTerm___closed__1); +l_Lean_PrettyPrinter_ppTerm___closed__2 = _init_l_Lean_PrettyPrinter_ppTerm___closed__2(); +lean_mark_persistent(l_Lean_PrettyPrinter_ppTerm___closed__2); l_Lean_PrettyPrinter_ppExpr___closed__1 = _init_l_Lean_PrettyPrinter_ppExpr___closed__1(); lean_mark_persistent(l_Lean_PrettyPrinter_ppExpr___closed__1); l_Lean_PrettyPrinter_ppExprWithInfos___lambda__1___closed__1 = _init_l_Lean_PrettyPrinter_ppExprWithInfos___lambda__1___closed__1(); @@ -2514,28 +2516,36 @@ l_Lean_PrettyPrinter_ppExprLegacy___closed__2 = _init_l_Lean_PrettyPrinter_ppExp lean_mark_persistent(l_Lean_PrettyPrinter_ppExprLegacy___closed__2); l_Lean_PrettyPrinter_ppExprLegacy___closed__3 = _init_l_Lean_PrettyPrinter_ppExprLegacy___closed__3(); lean_mark_persistent(l_Lean_PrettyPrinter_ppExprLegacy___closed__3); +l_Lean_PrettyPrinter_ppTactic___closed__1 = _init_l_Lean_PrettyPrinter_ppTactic___closed__1(); +lean_mark_persistent(l_Lean_PrettyPrinter_ppTactic___closed__1); +l_Lean_PrettyPrinter_ppTactic___closed__2 = _init_l_Lean_PrettyPrinter_ppTactic___closed__2(); +lean_mark_persistent(l_Lean_PrettyPrinter_ppTactic___closed__2); +l_Lean_PrettyPrinter_ppCommand___closed__1 = _init_l_Lean_PrettyPrinter_ppCommand___closed__1(); +lean_mark_persistent(l_Lean_PrettyPrinter_ppCommand___closed__1); +l_Lean_PrettyPrinter_ppCommand___closed__2 = _init_l_Lean_PrettyPrinter_ppCommand___closed__2(); +lean_mark_persistent(l_Lean_PrettyPrinter_ppCommand___closed__2); l_Lean_PrettyPrinter_ppModule___closed__1 = _init_l_Lean_PrettyPrinter_ppModule___closed__1(); lean_mark_persistent(l_Lean_PrettyPrinter_ppModule___closed__1); l_Lean_PrettyPrinter_ppModule___closed__2 = _init_l_Lean_PrettyPrinter_ppModule___closed__2(); lean_mark_persistent(l_Lean_PrettyPrinter_ppModule___closed__2); -l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__1 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__1(); -lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__1); -l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__2 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__2(); -lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__2); -l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__3 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__3(); -lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__3); -l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__4 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__4(); -lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__4); -l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__5 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__5(); -lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615____closed__5); -res = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_615_(lean_io_mk_world()); +l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__1 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__1(); +lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__1); +l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__2 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__2(); +lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__2); +l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__3 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__3(); +lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__3); +l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__4 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__4(); +lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__4); +l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__5 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__5(); +lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619____closed__5); +res = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_619_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__1 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__1(); -lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__1); -l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__2 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__2(); -lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666____closed__2); -res = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_666_(lean_io_mk_world()); +l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__1 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__1(); +lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__1); +l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__2 = _init_l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__2(); +lean_mark_persistent(l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670____closed__2); +res = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter___hyg_670_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_PrettyPrinter_registerParserCompilers___closed__1 = _init_l_Lean_PrettyPrinter_registerParserCompilers___closed__1(); diff --git a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c index 3159556fbb14..06e04e0af508 100644 --- a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c +++ b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/Builtins.c @@ -496,6 +496,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabProjectionApp___l static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__3___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabMVar___closed__5; static lean_object* l_Lean_PrettyPrinter_Delaborator_maybeAddBlockImplicit___closed__9; +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_delabFVar___closed__1; extern lean_object* l_Lean_PrettyPrinter_Delaborator_delabAttribute; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabForall___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -724,7 +725,6 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDoElems_prependAn lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PrettyPrinter_Delaborator_hasIdent(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapIdxM_map___at___private_Lean_PrettyPrinter_Delaborator_Builtins_0__Lean_PrettyPrinter_Delaborator_delabPatterns___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Array_foldrMUnsafe_fold___at_Lean_PrettyPrinter_Delaborator_delabForall___spec__1___closed__1; static lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_withMDatasOptions(lean_object*); @@ -5667,7 +5667,7 @@ lean_inc(x_10); lean_dec(x_8); x_11 = l_Lean_Expr_getAppFn(x_9); x_12 = lean_unsigned_to_nat(0u); -x_13 = l_Lean_Expr_getAppNumArgsAux(x_9, x_12); +x_13 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_12); x_14 = l_Lean_PrettyPrinter_Delaborator_getParamKinds___closed__1; lean_inc(x_13); x_15 = lean_mk_array(x_13, x_14); @@ -7397,7 +7397,7 @@ x_14 = lean_ctor_get(x_12, 1); lean_inc(x_14); lean_dec(x_12); x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_10, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_10, x_15); x_17 = l_Lean_SubExpr_Pos_pushNaryFn(x_16, x_13); lean_dec(x_13); lean_dec(x_16); @@ -7476,7 +7476,7 @@ static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg__ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_isRegularApp___spec__2___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_isRegularApp___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___at_Lean_PrettyPrinter_Delaborator_isRegularApp___spec__2___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -7494,7 +7494,7 @@ x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_11, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_13); x_15 = l_Lean_PrettyPrinter_Delaborator_getParamKinds___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -7851,7 +7851,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_isRegularApp___lambda_ { lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_1, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_10); x_12 = l_Lean_PrettyPrinter_Delaborator_unresolveNameGlobal___lambda__1___closed__1; x_13 = lean_unsigned_to_nat(1u); lean_inc(x_8); @@ -9681,7 +9681,7 @@ goto block_136; { lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; x_30 = lean_unsigned_to_nat(0u); -x_31 = l_Lean_Expr_getAppNumArgsAux(x_11, x_30); +x_31 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_30); x_32 = l_Lean_PrettyPrinter_Delaborator_getParamKinds___closed__1; lean_inc(x_31); x_33 = lean_mk_array(x_31, x_32); @@ -25202,7 +25202,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabOfScientific___la { lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Expr_getAppNumArgsAux(x_1, x_9); +x_10 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_9); x_11 = lean_unsigned_to_nat(5u); x_12 = lean_nat_dec_eq(x_10, x_11); if (x_12 == 0) @@ -26334,7 +26334,7 @@ if (x_22 == 0) { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; x_23 = lean_unsigned_to_nat(0u); -x_24 = l_Lean_Expr_getAppNumArgsAux(x_1, x_23); +x_24 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_23); x_25 = lean_ctor_get(x_21, 1); lean_inc(x_25); lean_dec(x_21); @@ -27107,7 +27107,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabDIte___lambda__1( { lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Expr_getAppNumArgsAux(x_1, x_9); +x_10 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_9); x_11 = lean_unsigned_to_nat(5u); x_12 = lean_nat_dec_eq(x_10, x_11); lean_dec(x_10); @@ -27515,7 +27515,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabCond___lambda__1( { lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Expr_getAppNumArgsAux(x_1, x_9); +x_10 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_9); x_11 = lean_unsigned_to_nat(4u); x_12 = lean_nat_dec_eq(x_10, x_11); lean_dec(x_10); @@ -27928,7 +27928,7 @@ x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_11, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_13); lean_dec(x_11); x_15 = lean_unsigned_to_nat(4u); x_16 = lean_nat_dec_eq(x_14, x_15); @@ -28997,7 +28997,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_delabSigmaCore___lambd { lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_10 = lean_unsigned_to_nat(0u); -x_11 = l_Lean_Expr_getAppNumArgsAux(x_2, x_10); +x_11 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_10); x_12 = lean_unsigned_to_nat(2u); x_13 = lean_nat_dec_eq(x_11, x_12); lean_dec(x_11); @@ -30257,7 +30257,7 @@ else { lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; lean_object* x_87; x_77 = lean_unsigned_to_nat(0u); -x_78 = l_Lean_Expr_getAppNumArgsAux(x_9, x_77); +x_78 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_9, x_77); x_79 = l_Lean_PrettyPrinter_Delaborator_getParamKinds___closed__1; lean_inc(x_78); x_80 = lean_mk_array(x_78, x_79); diff --git a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/SubExpr.c b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/SubExpr.c index c0fff7cbcd0a..0a51198353b9 100644 --- a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/SubExpr.c +++ b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/SubExpr.c @@ -119,6 +119,7 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_SubExpr_wit static lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withProj___rarg___lambda__1___closed__4; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_SubExpr_withLetVarType___spec__11(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody___spec__1(lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_SubExpr_withLetValue___spec__6(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_SubExpr_withMDataExpr___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_SubExpr_withLetBody___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -159,7 +160,6 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBod LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_SubExpr_withMDataExpr___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_nextExtraPos___rarg___lambda__2(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_SubExpr_withLetBody___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_SubExpr_withProj___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withLetBody___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2712,7 +2712,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryFn___r { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_5 = lean_unsigned_to_nat(0u); -x_6 = l_Lean_Expr_getAppNumArgsAux(x_1, x_5); +x_6 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_5); x_7 = l_Lean_SubExpr_Pos_pushNaryFn(x_6, x_4); lean_dec(x_6); x_8 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryFn___rarg___lambda__1___boxed), 3, 2); @@ -2812,7 +2812,7 @@ static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg__ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___rarg___lambda__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___rarg___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___rarg___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2874,7 +2874,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___ { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_8 = lean_unsigned_to_nat(0u); -x_9 = l_Lean_Expr_getAppNumArgsAux(x_7, x_8); +x_9 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_7, x_8); x_10 = l_Lean_PrettyPrinter_Delaborator_SubExpr_withNaryArg___rarg___lambda__3___closed__1; lean_inc(x_9); x_11 = lean_mk_array(x_9, x_10); diff --git a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/TopDownAnalyze.c b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/TopDownAnalyze.c index 96dd3d653e8f..63edc1458914 100644 --- a/stage0/stdlib/Lean/PrettyPrinter/Delaborator/TopDownAnalyze.c +++ b/stage0/stdlib/Lean/PrettyPrinter/Delaborator/TopDownAnalyze.c @@ -183,6 +183,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_isHighe LEAN_EXPORT uint8_t l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_nameNotRoundtrippable(lean_object*); LEAN_EXPORT uint8_t l_Lean_getPPAnalysisSkip(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams_inspectAux___lambda__1___closed__2; +uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyzeAppStagedCore_analyzeArg___lambda__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_SubExpr_withBindingBody___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyze_analyzeLam___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -358,6 +359,7 @@ static lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_isHBinOp___l LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams_inspectAux(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyze_analyzeLet___spec__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyze_analyzeLet___spec__35(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyzeAppStagedCore_maybeSetExplicit___spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_replaceLPsWithVars___spec__9(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_annotateBoolAt___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -477,7 +479,6 @@ LEAN_EXPORT lean_object* l_Lean_pp_analyze_trustOfScientific; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_instInhabitedContext; static lean_object* l_Lean_PrettyPrinter_Delaborator_initFn____x40_Lean_PrettyPrinter_Delaborator_TopDownAnalyze___hyg_9767____closed__1; LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyze_analyzeProj___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_loop___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyzeAppStagedCore_collectHigherOrders___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_isHBinOp(lean_object*); static lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_isFunLike___closed__1; @@ -539,7 +540,6 @@ static lean_object* l_Lean_initFn____x40_Lean_PrettyPrinter_Delaborator_TopDownA LEAN_EXPORT lean_object* l_panic___at_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_analyze_analyzeMData___spec__12(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_PrettyPrinter_Delaborator_TopDownAnalyze_analyzeAppStagedCore_collectHigherOrders___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_trySynthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); extern uint8_t l_instInhabitedBool; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_containsBadMax___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_pp_analyze_trustId; @@ -3249,7 +3249,7 @@ else { lean_object* x_9; lean_object* x_10; uint8_t x_11; x_9 = lean_unsigned_to_nat(0u); -x_10 = l_Lean_Expr_getAppNumArgsAux(x_1, x_9); +x_10 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_9); x_11 = lean_nat_dec_le(x_3, x_10); lean_dec(x_10); if (x_11 == 0) @@ -3571,7 +3571,7 @@ lean_inc(x_4); lean_dec(x_1); x_5 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_5, 0, x_4); -x_6 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_3, x_5); +x_6 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_3, x_5); lean_dec(x_5); lean_dec(x_3); return x_6; @@ -4480,7 +4480,7 @@ LEAN_EXPORT uint8_t l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_isHBinOp(lea { lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Expr_getAppNumArgsAux(x_1, x_2); +x_3 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_2); x_4 = lean_unsigned_to_nat(6u); x_5 = lean_nat_dec_eq(x_3, x_4); lean_dec(x_3); @@ -6664,7 +6664,7 @@ static lean_object* _init_l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspec lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams_inspectAux___lambda__1___closed__1; x_2 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams_inspectAux___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams_inspectAux___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -7299,7 +7299,7 @@ x_23 = lean_ctor_get(x_21, 1); lean_inc(x_23); lean_dec(x_21); x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_Expr_getAppNumArgsAux(x_11, x_24); +x_25 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_24); x_26 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams___closed__1; lean_inc(x_25); x_27 = lean_mk_array(x_25, x_26); @@ -7307,7 +7307,7 @@ x_28 = lean_unsigned_to_nat(1u); x_29 = lean_nat_sub(x_25, x_28); lean_dec(x_25); x_30 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_11, x_27, x_29); -x_31 = l_Lean_Expr_getAppNumArgsAux(x_14, x_24); +x_31 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_14, x_24); lean_inc(x_31); x_32 = lean_mk_array(x_31, x_26); x_33 = lean_nat_sub(x_31, x_28); @@ -9050,7 +9050,7 @@ LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_canBott 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_dec(x_5); x_13 = lean_unsigned_to_nat(0u); -x_14 = l_Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); x_15 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams___closed__1; lean_inc(x_14); x_16 = lean_mk_array(x_14, x_15); @@ -19920,7 +19920,7 @@ x_16 = lean_ctor_get(x_13, 1); lean_inc(x_16); lean_dec(x_13); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_15, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_15, x_17); x_19 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -21692,7 +21692,7 @@ x_14 = lean_ctor_get(x_12, 1); lean_inc(x_14); lean_dec(x_12); x_15 = lean_unsigned_to_nat(0u); -x_16 = l_Lean_Expr_getAppNumArgsAux(x_10, x_15); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_10, x_15); x_17 = l_Lean_SubExpr_Pos_pushNaryFn(x_16, x_13); lean_dec(x_13); lean_dec(x_16); @@ -25402,7 +25402,7 @@ lean_dec(x_13); x_16 = l_Lean_Expr_getAppFn(x_11); lean_dec(x_11); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_14, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_14, x_17); x_19 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -27129,7 +27129,7 @@ x_16 = lean_ctor_get(x_13, 1); lean_inc(x_16); lean_dec(x_13); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_15, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_15, x_17); x_19 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -27583,7 +27583,7 @@ if (x_19 == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_3, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_20); lean_dec(x_3); x_22 = lean_nat_add(x_21, x_2); lean_dec(x_21); @@ -27670,7 +27670,7 @@ if (x_41 == 0) { lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; x_42 = lean_unsigned_to_nat(0u); -x_43 = l_Lean_Expr_getAppNumArgsAux(x_3, x_42); +x_43 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_42); lean_dec(x_3); x_44 = lean_nat_add(x_43, x_2); lean_dec(x_43); @@ -28213,7 +28213,7 @@ x_16 = lean_ctor_get(x_13, 1); lean_inc(x_16); lean_dec(x_13); x_17 = lean_unsigned_to_nat(0u); -x_18 = l_Lean_Expr_getAppNumArgsAux(x_15, x_17); +x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_15, x_17); x_19 = l_Lean_PrettyPrinter_Delaborator_TopDownAnalyze_inspectOutParams___closed__1; lean_inc(x_18); x_20 = lean_mk_array(x_18, x_19); @@ -30136,7 +30136,7 @@ x_25 = lean_array_get_size(x_13); x_26 = lean_nat_dec_lt(x_1, x_25); lean_dec(x_25); x_27 = lean_unsigned_to_nat(0u); -x_28 = l_Lean_Expr_getAppNumArgsAux(x_11, x_27); +x_28 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_27); lean_dec(x_11); x_29 = lean_nat_add(x_28, x_1); lean_dec(x_28); diff --git a/stage0/stdlib/Lean/PrettyPrinter/Parenthesizer.c b/stage0/stdlib/Lean/PrettyPrinter/Parenthesizer.c index 5cb1cf408a01..21c161d01fbd 100644 --- a/stage0/stdlib/Lean/PrettyPrinter/Parenthesizer.c +++ b/stage0/stdlib/Lean/PrettyPrinter/Parenthesizer.c @@ -77,7 +77,6 @@ static lean_object* l_Lean_PrettyPrinter_mkCategoryParenthesizerAttribute___clos static lean_object* l_Lean_PrettyPrinter_mkParenthesizerAttribute___closed__10; static lean_object* l_Lean_PrettyPrinter_Parenthesizer_maybeParenthesize___closed__3; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_parenthesize___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_PrettyPrinter_parenthesizeCommand___closed__3; static lean_object* l___regBuiltin_Lean_PrettyPrinter_Parenthesizer_term_parenthesizer___closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_PrettyPrinter_parenthesize___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_maybeParenthesize___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -89,7 +88,7 @@ lean_object* lean_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_MonadTraverser_goUp___at_Lean_PrettyPrinter_Parenthesizer_visitArgs___spec__4___boxed(lean_object*); uint8_t l_Lean_checkTraceOption(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter_Parenthesizer___hyg_4162_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter_Parenthesizer___hyg_4159_(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_maybeParenthesize___lambda__9___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Syntax_MonadTraverser_setCur___at_Lean_PrettyPrinter_Parenthesizer_maybeParenthesize___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_Parenthesizer_term_parenthesizer___lambda__1___closed__6; @@ -172,7 +171,6 @@ LEAN_EXPORT lean_object* l_Nat_forM_loop___at_Lean_PrettyPrinter_Parenthesizer_m LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_unicodeSymbolNoAntiquot_parenthesizer___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_interpretParserDescr_x27___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Syntax_MonadTraverser_goLeft___at_Lean_PrettyPrinter_Parenthesizer_visitArgs___spec__2(lean_object*); -static lean_object* l_Lean_PrettyPrinter_parenthesizeTactic___closed__1; static lean_object* l_Lean_PrettyPrinter_Parenthesizer_term_parenthesizer___closed__1; static lean_object* l_Lean_PrettyPrinter_parenthesize___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_skip_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*); @@ -253,6 +251,7 @@ static lean_object* l_Lean_PrettyPrinter_mkParenthesizerAttribute___closed__12; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_incQuotDepth_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_PrettyPrinter_ParenthesizerM_orElse___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_categoryParserOfStack_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_parenthesizeCategory(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_instMonadTraverserParenthesizerM___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_manyNoAntiquot_parenthesizer(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_maybeParenthesize___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -527,7 +526,6 @@ lean_object* l_Nat_min(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_level_parenthesizer___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_PrettyPrinter_backtrackExceptionId; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_rawStx_parenthesizer(lean_object*, lean_object*); -static lean_object* l_Lean_PrettyPrinter_parenthesizeTerm___closed__1; static lean_object* l_Lean_PrettyPrinter_Parenthesizer_instMonadQuotationParenthesizerM___closed__3; static lean_object* l_Lean_PrettyPrinter_mkParenthesizerAttribute___closed__6; LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_Parenthesizer_checkColGt_parenthesizer___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -11165,45 +11163,33 @@ lean_dec(x_2); return x_5; } } -static lean_object* _init_l_Lean_PrettyPrinter_parenthesizeTerm___closed__1() { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_parenthesizeCategory(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_PrettyPrinter_Parenthesizer_term_parenthesizer___closed__2; -x_2 = lean_unsigned_to_nat(0u); -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_categoryParser_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_categoryParser_parenthesizer), 7, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_6); +x_8 = l_Lean_PrettyPrinter_parenthesize(x_7, x_2, x_3, x_4, x_5); +return x_8; } } LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_parenthesizeTerm(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_PrettyPrinter_parenthesizeTerm___closed__1; -x_6 = l_Lean_PrettyPrinter_parenthesize(x_5, x_1, x_2, x_3, x_4); +x_5 = l_Lean_PrettyPrinter_Parenthesizer_term_parenthesizer___closed__2; +x_6 = l_Lean_PrettyPrinter_parenthesizeCategory(x_5, x_1, x_2, x_3, x_4); return x_6; } } -static lean_object* _init_l_Lean_PrettyPrinter_parenthesizeTactic___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_PrettyPrinter_Parenthesizer_tactic_parenthesizer___closed__2; -x_2 = lean_unsigned_to_nat(0u); -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_categoryParser_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_parenthesizeTactic(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_PrettyPrinter_parenthesizeTactic___closed__1; -x_6 = l_Lean_PrettyPrinter_parenthesize(x_5, x_1, x_2, x_3, x_4); +x_5 = l_Lean_PrettyPrinter_Parenthesizer_tactic_parenthesizer___closed__2; +x_6 = l_Lean_PrettyPrinter_parenthesizeCategory(x_5, x_1, x_2, x_3, x_4); return x_6; } } @@ -11225,28 +11211,16 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_PrettyPrinter_parenthesizeCommand___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_PrettyPrinter_parenthesizeCommand___closed__2; -x_2 = lean_unsigned_to_nat(0u); -x_3 = lean_alloc_closure((void*)(l_Lean_PrettyPrinter_Parenthesizer_categoryParser_parenthesizer), 7, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_parenthesizeCommand(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_PrettyPrinter_parenthesizeCommand___closed__3; -x_6 = l_Lean_PrettyPrinter_parenthesize(x_5, x_1, x_2, x_3, x_4); +x_5 = l_Lean_PrettyPrinter_parenthesizeCommand___closed__2; +x_6 = l_Lean_PrettyPrinter_parenthesizeCategory(x_5, x_1, x_2, x_3, x_4); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter_Parenthesizer___hyg_4162_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter_Parenthesizer___hyg_4159_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -11659,17 +11633,11 @@ l_Lean_PrettyPrinter_parenthesize___closed__1 = _init_l_Lean_PrettyPrinter_paren lean_mark_persistent(l_Lean_PrettyPrinter_parenthesize___closed__1); l_Lean_PrettyPrinter_parenthesize___closed__2 = _init_l_Lean_PrettyPrinter_parenthesize___closed__2(); lean_mark_persistent(l_Lean_PrettyPrinter_parenthesize___closed__2); -l_Lean_PrettyPrinter_parenthesizeTerm___closed__1 = _init_l_Lean_PrettyPrinter_parenthesizeTerm___closed__1(); -lean_mark_persistent(l_Lean_PrettyPrinter_parenthesizeTerm___closed__1); -l_Lean_PrettyPrinter_parenthesizeTactic___closed__1 = _init_l_Lean_PrettyPrinter_parenthesizeTactic___closed__1(); -lean_mark_persistent(l_Lean_PrettyPrinter_parenthesizeTactic___closed__1); l_Lean_PrettyPrinter_parenthesizeCommand___closed__1 = _init_l_Lean_PrettyPrinter_parenthesizeCommand___closed__1(); lean_mark_persistent(l_Lean_PrettyPrinter_parenthesizeCommand___closed__1); l_Lean_PrettyPrinter_parenthesizeCommand___closed__2 = _init_l_Lean_PrettyPrinter_parenthesizeCommand___closed__2(); lean_mark_persistent(l_Lean_PrettyPrinter_parenthesizeCommand___closed__2); -l_Lean_PrettyPrinter_parenthesizeCommand___closed__3 = _init_l_Lean_PrettyPrinter_parenthesizeCommand___closed__3(); -lean_mark_persistent(l_Lean_PrettyPrinter_parenthesizeCommand___closed__3); -res = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter_Parenthesizer___hyg_4162_(lean_io_mk_world()); +res = l_Lean_PrettyPrinter_initFn____x40_Lean_PrettyPrinter_Parenthesizer___hyg_4159_(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/Server/FileWorker.c b/stage0/stdlib/Lean/Server/FileWorker.c index 12c5b378d2f2..556fd53da3a2 100644 --- a/stage0/stdlib/Lean/Server/FileWorker.c +++ b/stage0/stdlib/Lean/Server/FileWorker.c @@ -341,7 +341,7 @@ lean_object* lean_io_bind_task(lean_object*, lean_object*, lean_object*, lean_ob lean_object* l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(lean_object*); lean_object* lean_io_getenv(lean_object*, lean_object*); LEAN_EXPORT lean_object* lean_server_worker_main(lean_object*, lean_object*); -lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t); +lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_queueRequest(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_parseParams___rarg___closed__2; lean_object* l___private_Lean_Util_Paths_0__Lean_fromJsonLeanPaths____x40_Lean_Util_Paths___hyg_90_(lean_object*); @@ -373,7 +373,6 @@ static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_FileWorker_ini LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspResponse___at_Lean_Server_FileWorker_handleRequest___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_FileWorker_initAndRunWorker___spec__2___closed__71; static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_FileWorker_initAndRunWorker___spec__2___closed__7; -lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(lean_object*, uint64_t); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_parseParams___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_mainLoop___closed__2; lean_object* l_Lean_Json_mkObj(lean_object*); @@ -443,6 +442,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_compileHeader___lambda__3___bo static lean_object* l_Lean_Server_FileWorker_compileHeader___lambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_parseParams___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_System_FilePath_withExtension(lean_object*, lean_object*); +lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(lean_object*, uint64_t); lean_object* lean_get_stdin(lean_object*); uint8_t l_Std_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(lean_object*); static lean_object* l_Lean_Server_FileWorker_compileHeader___lambda__3___closed__1; @@ -816,7 +816,7 @@ return x_10; LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_0__Lean_Server_FileWorker_publishIleanInfo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_6 = lean_array_get_size(x_4); x_7 = lean_usize_of_nat(x_6); lean_dec(x_6); @@ -825,23 +825,24 @@ x_9 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight x_10 = lean_ctor_get(x_2, 2); lean_inc(x_10); x_11 = 1; -x_12 = l_Lean_Server_findModuleRefs(x_10, x_9, x_11); +x_12 = 0; +x_13 = l_Lean_Server_findModuleRefs(x_10, x_9, x_11, x_12); lean_dec(x_9); -x_13 = lean_ctor_get(x_2, 1); -lean_inc(x_13); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); lean_dec(x_2); -x_14 = l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(x_12); -x_15 = lean_box(0); -x_16 = l_List_mapTRAux___at___private_Lean_Server_FileWorker_0__Lean_Server_FileWorker_publishIleanInfo___spec__1(x_8, x_14, x_15); -x_17 = l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(x_16); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_13); -lean_ctor_set(x_18, 1, x_17); +x_15 = l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(x_13); +x_16 = lean_box(0); +x_17 = l_List_mapTRAux___at___private_Lean_Server_FileWorker_0__Lean_Server_FileWorker_publishIleanInfo___spec__1(x_8, x_15, x_16); +x_18 = l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(x_17); x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 0, x_14); lean_ctor_set(x_19, 1, x_18); -x_20 = l_IO_FS_Stream_writeLspNotification___at___private_Lean_Server_FileWorker_0__Lean_Server_FileWorker_publishIleanInfo___spec__2(x_3, x_19, x_5); -return x_20; +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_1); +lean_ctor_set(x_20, 1, x_19); +x_21 = l_IO_FS_Stream_writeLspNotification___at___private_Lean_Server_FileWorker_0__Lean_Server_FileWorker_publishIleanInfo___spec__2(x_3, x_20, x_5); +return x_21; } } LEAN_EXPORT lean_object* l_List_mapTRAux___at___private_Lean_Server_FileWorker_0__Lean_Server_FileWorker_publishIleanInfo___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { @@ -1784,7 +1785,7 @@ static lean_object* _init_l_Lean_Server_FileWorker_unfoldCmdSnaps___closed__4() lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Server_FileWorker_unfoldCmdSnaps___closed__1; x_2 = l_Lean_Server_FileWorker_unfoldCmdSnaps___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Server_FileWorker_unfoldCmdSnaps___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -8117,7 +8118,7 @@ x_9 = lean_ctor_get(x_7, 2); lean_inc(x_9); lean_dec(x_7); x_10 = lean_ctor_get_uint64(x_1, sizeof(void*)*2); -x_11 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(x_9, x_10); +x_11 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; @@ -8186,7 +8187,7 @@ x_33 = lean_ctor_get(x_31, 2); lean_inc(x_33); lean_dec(x_31); x_34 = lean_ctor_get_uint64(x_1, sizeof(void*)*2); -x_35 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(x_33, x_34); +x_35 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_33, x_34); if (lean_obj_tag(x_35) == 0) { lean_object* x_36; lean_object* x_37; @@ -8287,7 +8288,7 @@ x_9 = lean_ctor_get(x_7, 2); lean_inc(x_9); lean_dec(x_7); x_10 = lean_ctor_get_uint64(x_1, sizeof(void*)*1); -x_11 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(x_9, x_10); +x_11 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_9, x_10); if (lean_obj_tag(x_11) == 0) { lean_object* x_12; @@ -8350,7 +8351,7 @@ x_28 = lean_ctor_get(x_26, 2); lean_inc(x_28); lean_dec(x_26); x_29 = lean_ctor_get_uint64(x_1, sizeof(void*)*1); -x_30 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(x_28, x_29); +x_30 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_28, x_29); if (lean_obj_tag(x_30) == 0) { lean_object* x_31; lean_object* x_32; diff --git a/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c b/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c index f1903b86e5d6..4c0ffb00816a 100644 --- a/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c +++ b/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c @@ -14,20 +14,29 @@ extern "C" { #endif lean_object* l_List_reverse___rarg(lean_object*); +lean_object* l_Lean_initializing(lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Server_FileWorker_handleCompletion___spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__20___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__29___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_String_csize(uint32_t); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__2(lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__13; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__1(size_t, size_t, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_isImport___closed__4; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__1(lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__6; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokensRange(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__19(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__22(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__23___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__1(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__6; lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens___lambda__1___boxed(lean_object*, lean_object*); @@ -35,13 +44,11 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_go___closed__3; lean_object* l_Std_HashMapImp_find_x3f___at_Lean_Server_References_updateWorkerRefs___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleHover___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__2; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__17(size_t, size_t, lean_object*); lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonTextDocumentPositionParams____x40_Lean_Data_Lsp_Basic___hyg_2007_(lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__12___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_getInteractiveGoals___lambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_sectionLikeToDocumentSymbols___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_isImport___closed__1; static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_isImport___closed__2; @@ -50,72 +57,74 @@ lean_object* l_Lean_Syntax_getOptional_x3f(lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__2; lean_object* lean_io_error_to_string(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveTermGoal___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__33___boxed(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonHoverParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1781_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___boxed(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__7; lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonPlainGoalParams____x40_Lean_Data_Lsp_Extra___hyg_503_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; static lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__3___closed__7; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handlePlainTermGoal(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_sectionLikeToDocumentSymbols___closed__2; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__1; extern lean_object* l_Std_Format_defWidth; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_isImport___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__7; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__13___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleHover___closed__1; static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___closed__3; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__2; -static lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__2; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__1; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__23; +static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l_Lean_Server_FileWorker_handlePlainGoal___closed__2; static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__8; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__9___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Lsp_SemanticTokenType_toCtorIdx(uint8_t); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__10; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__11; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__4___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__26___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__2; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__14; static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_Completion_find_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_isImport___closed__3; -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__24; static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__12; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__6___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__5; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__18; lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__2(lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addCommandRange___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__2; uint8_t lean_name_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__20; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__3___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__1; -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__3___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__10; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__2; static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___closed__4; static lean_object* l_Lean_Server_FileWorker_handlePlainGoal___closed__1; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4___closed__1; static lean_object* l_Lean_Server_FileWorker_handlePlainTermGoal___closed__2; lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3___closed__1; lean_object* lean_array_get_size(lean_object*); lean_object* l_Lean_Server_Snapshots_Snapshot_infoTree(lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonPlainTermGoalParams____x40_Lean_Data_Lsp_Extra___hyg_724_(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___closed__1; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_sectionLikeToDocumentSymbols___closed__1; @@ -123,22 +132,21 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_addToken_ static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__5___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withPPInaccessibleNames___at_Lean_Server_FileWorker_getInteractiveGoals___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__8; lean_object* l_Lean_FileMap_lspPosToUtf8Pos(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__4; static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__11; lean_object* l_IO_sleep(uint32_t, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__2___closed__1; static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__9; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleCompletion___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__30___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Server_DocumentMeta_mkInputContext(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_isImport___closed__5; LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_handleWaitForDiagnostics___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__16; -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_join___rarg(lean_object*); @@ -147,48 +155,46 @@ LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveG static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__3; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRangeFromSyntax(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__3___closed__1; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__25; static lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__1___closed__1; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__24; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___boxed(lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__5; static lean_object* l_Lean_Server_FileWorker_handlePlainTermGoal___closed__3; -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__14; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__2(lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__20(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__18; -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__15; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_utf8PosToLspPos(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__20___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__2(lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__7; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__1(lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__15; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3___closed__1; lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonPlainTermGoal____x40_Lean_Data_Lsp_Extra___hyg_893_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_InfoTree_deepestNodes___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Server_FileWorker_handleSemanticTokens_go___spec__2(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_InteractiveGoal_pretty(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__5; static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addCommandRange___closed__2; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__2(lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__7; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics_waitLoop(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_FileMap_toPosition_loop___spec__1(lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__2(lean_object*, size_t, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens_highlightId___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Except_map___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2(lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonHover____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1682_(lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonWaitForDiagnosticsParams____x40_Lean_Data_Lsp_Extra___hyg_24_(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__3; @@ -196,19 +202,16 @@ static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addCommandRange_ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDefinition___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__11___closed__1; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__2; static lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__3___closed__6; lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__28(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__1(lean_object*); lean_object* l_Lean_Elab_InfoTree_findInfo_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addCommandRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Server_Snapshots_parseAhead(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__1(lean_object*); static lean_object* l_Lean_Server_FileWorker_handlePlainTermGoal___closed__1; uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__1; -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__3; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__22; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePlainGoal___spec__1___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_String_Range_contains(lean_object*, lean_object*, uint8_t); lean_object* l_Lean_Json_compress(lean_object*); @@ -217,49 +220,41 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___closed__2; static lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics___closed__1; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3___closed__1; lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonLocationLink____x40_Lean_Data_Lsp_Basic___hyg_1031_(lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instToJsonDocumentSymbol_go___spec__3(size_t, size_t, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Lsp_SemanticTokenType_toNat(uint8_t); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_isImport___closed__6; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__9(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveTermGoal___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_String_Range_toLspRange(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleCompletion___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRanges(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__10; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__2; -lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761_(lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__33(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__9___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addCommandRange___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePlainGoal___spec__2(size_t, size_t, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_sectionLikeToDocumentSymbols___closed__3; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___lambda__1___boxed(lean_object*); -LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__22(lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__2; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__1; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__10; lean_object* l_Std_PersistentHashMap_insert___at_Lean_Server_registerLspRequestHandler___spec__2(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__1(lean_object*); -lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3801_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__2(lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__22; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5383_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__2(lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__20; lean_object* l_IO_AsyncList_waitAll___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__33(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_documentUriFromModule(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_highlightKeyword(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDefinition___closed__1; @@ -267,19 +262,20 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_highlight LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleSemanticTokensFull___rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__3(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3616_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5167_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokensFull(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_highlightId___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4___closed__1; lean_object* lean_task_map(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePlainGoal___spec__2___closed__2; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__30(size_t, size_t, lean_object*); static lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__3___closed__3; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__9(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_handleWaitForDiagnostics___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__6___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__2___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Server_requestHandlers; @@ -287,37 +283,36 @@ lean_object* lean_format_pretty(lean_object*, lean_object*); lean_object* l_Lean_Server_RequestM_bindTask___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__5; lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__13(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveGoals(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__19(lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__16; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_highlightId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_PersistentHashMap_contains___at_Lean_Server_registerLspRequestHandler___spec__6(lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__25; static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__12; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePlainGoal___spec__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__3; -lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3530_(lean_object*); +lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5081_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handlePlainGoal(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_instCoeRefInfoRefInfo___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDefinition___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__36(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_RequestM_mapTask___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveGoals___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint32_t lean_string_utf8_get(lean_object*, lean_object*); -static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__4(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__1___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePlainGoal___spec__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__26(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleCompletion(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonPlainGoal____x40_Lean_Data_Lsp_Extra___hyg_673_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -325,139 +320,140 @@ lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDocu LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveTermGoal___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonDocumentHighlight____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2644_(lean_object*); lean_object* lean_local_ctx_pop(lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__21; static lean_object* l_Lean_Server_FileWorker_handleCompletion___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1(lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__12; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleCompletion___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__26(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokensFull___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___boxed(lean_object*); extern lean_object* l_Lean_instInhabitedSyntax; -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_stx(lean_object*); lean_object* l_Lean_Elab_Info_toElabInfo_x3f(lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__36___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__8(lean_object*); -extern lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__6; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__30(size_t, size_t, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__9; lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonCompletionParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1566_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__32(lean_object*); extern lean_object* l_Task_Priority_default; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_range_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__36___boxed(lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2(lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__1; static lean_object* l_Lean_Server_FileWorker_handleCompletion___closed__2; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__15; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__2(lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__3; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleCompletion___lambda__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleCompletion___lambda__1(lean_object*, lean_object*); uint8_t l_Char_isAlpha(uint32_t); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveTermGoal___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__1; -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__23; -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__35(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__5; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCompletionList____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1515_(lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__4; -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__26___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__20(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addCommandRange(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__7; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_handleSemanticTokens_go___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__5(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_panic___at_Lean_Elab_InfoTree_hoverableInfoAt_x3f___spec__1(lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__1; lean_object* l_List_drop___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__13; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_highlightId___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleCompletion___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_isIdOrAtom_x3f(lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__2; static lean_object* l_Lean_Server_FileWorker_handleCompletion___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__6___closed__1; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4___closed__1; static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__14; +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__11(lean_object*); static lean_object* l_Lean_Server_FileWorker_handlePlainGoal___closed__3; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__17___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__11; lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__17(size_t, size_t, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleHover(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__1(lean_object*); uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__2; lean_object* l_String_intercalate(lean_object*, lean_object*); lean_object* l_List_redLength___rarg(lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDefinition___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__1(lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__10; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__4; lean_object* l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__1(lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__9; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens_highlightId___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__36(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t, uint8_t); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokensFull___boxed(lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__2; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2(lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__2___closed__4; lean_object* l_Lean_Lsp_ModuleRefs_findAt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDefinition(uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleHover___lambda__1___boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__13___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__9; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__6(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4___closed__1; lean_object* l_Lean_Elab_Info_tailPos_x3f(lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); lean_object* l_Lean_Syntax_getRange_x3f(lean_object*, uint8_t); lean_object* l_Lean_Syntax_getKind(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__4; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__17___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__25(lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__5(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_sectionLikeToDocumentSymbols(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__16; -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__6(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__26; lean_object* l_Lean_Meta_withPPInaccessibleNamesImp___rarg(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__17; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__2(lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Server_RequestError_fileChanged; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__1; -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__8; lean_object* l_Lean_Elab_Info_fmtHover_x3f(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f(lean_object*, lean_object*, uint8_t, uint8_t); lean_object* lean_nat_shiftl(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__30___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_highlightKeyword___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Server_FileWorker_handleSemanticTokens_go___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__5(lean_object*); static lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__3___closed__2; -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__11; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__19; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f(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_Server_FileWorker_handleDocumentHighlight___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -466,28 +462,24 @@ lean_object* l_Lean_Server_Snapshots_Snapshot_endPos(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_addToken(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_go___closed__2; -lean_object* l_IO_AsyncList_waitFind_x3f___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handlePlainGoal___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__29___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRanges___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleHover___lambda__2___closed__2; lean_object* l_Lean_Expr_constName_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__32(lean_object*); lean_object* l_List_toArrayAux___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__16(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol(lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__9(lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__2; static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRanges___closed__2; lean_object* l_Option_map___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4(lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Server_GoTo_0__Lean_Server_beqGoToKind____x40_Lean_Server_GoTo___hyg_8_(uint8_t, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__9; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveGoals___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens_highlightId___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__7; @@ -496,94 +488,97 @@ static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightRe LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRange(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_noHighlightKinds; lean_object* l_Lean_Server_RequestM_withWaitFindSnap___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__1(lean_object*); static lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__3___closed__4; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleHover___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__9___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__16___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__13; lean_object* l_Lean_Syntax_getTailPos_x3f(lean_object*, uint8_t); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__6; static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__6; LEAN_EXPORT lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_contains___at_Lean_Server_FileWorker_handleSemanticTokens_go___spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleHover___lambda__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Server_FileWorker_handleSemanticTokens_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_io_initializing(lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__9; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveGoals___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_Server_locationLinksFromDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__5; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics(lean_object*, lean_object*, lean_object*); lean_object* lean_string_length(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__15(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handlePlainTermGoal___lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__23(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__29(lean_object*, lean_object*, lean_object*); lean_object* l_List_getLast_x21___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Server_FileWorker_handleCompletion___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__19; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3___closed__1; LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleHover___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePlainGoal___spec__1(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__12___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__13(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens_highlightId___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__11(lean_object*); lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__6; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handlePlainTermGoal___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__16(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__35(lean_object*); LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleFoldingRange_isImport(lean_object*); lean_object* l_Lean_Server_RequestM_asTask___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleSemanticTokens___lambda__2___closed__1; lean_object* l_Lean_Elab_Info_pos_x3f(lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__29(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__15(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Server_FileWorker_handleCompletion___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_spanAux___at_Lean_Server_FileWorker_handleFoldingRange_addRanges___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__23___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__17; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__1(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleHover___lambda__2___closed__4; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4___closed__1; LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleSemanticTokens___lambda__1(lean_object*, lean_object*); -lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922_(lean_object*); +lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__8; +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__21; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics_waitLoop___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_local_ctx_find(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__4; -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__25(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__1(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__8; static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__2; lean_object* l_Lean_Elab_Info_lctx(lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__12; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handlePlainGoal___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_go___closed__4; +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__28(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__11; +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__12(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_handleSemanticTokens_go___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handlePlainGoal___lambda__1___closed__3; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_ContextInfo_runMetaM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__8(lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_getInteractiveTermGoal(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__4(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_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__16___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___closed__5; static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__2; static lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_go___closed__1; @@ -594,38 +589,34 @@ static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightRe static lean_object* l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens___spec__1___lambda__1___closed__1; lean_object* l_IO_AsyncList_getFinishedPrefix___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleHover___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__23(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRangeFromSyntax___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withPPInaccessibleNames___at_Lean_Server_FileWorker_getInteractiveGoals___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__13; -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__12(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___closed__1; -lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__33___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__3___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__1(lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___boxed(lean_object*); lean_object* l_Lean_Syntax_reprint(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM___at_Lean_Server_FileWorker_getInteractiveGoals___spec__3___closed__5; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_RequestM_readDoc(lean_object*, lean_object*); lean_object* l_List_getLastD___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_IO_AsyncList_waitHead_x3f___rarg___lambda__1___boxed(lean_object*); -static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__26; -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__1; +static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__2; lean_object* l_Lean_Widget_goalToInteractive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__4; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___lambda__1(lean_object*); +static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__8; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__2; lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDocumentHighlightParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2503_(lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__2___closed__3; static lean_object* l_Lean_Server_FileWorker_handlePlainGoal___lambda__1___closed__1; @@ -8278,7 +8269,7 @@ x_10 = l_IO_AsyncList_getFinishedPrefix___rarg(x_9, x_8); x_11 = !lean_is_exclusive(x_10); if (x_11 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; size_t x_30; lean_object* x_31; uint8_t x_32; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; uint8_t x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; size_t x_31; lean_object* x_32; uint8_t x_33; x_12 = lean_ctor_get(x_10, 0); x_13 = lean_ctor_get(x_10, 1); x_14 = lean_ctor_get(x_12, 0); @@ -8294,112 +8285,114 @@ lean_dec(x_18); x_20 = 0; x_21 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__1(x_19, x_20, x_17); x_22 = 1; +x_23 = 0; lean_inc(x_3); -x_23 = l_Lean_Server_findModuleRefs(x_3, x_21, x_22); +x_24 = l_Lean_Server_findModuleRefs(x_3, x_21, x_22, x_23); lean_dec(x_21); -x_24 = l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(x_23); -x_25 = lean_box(0); -x_26 = l_List_mapTRAux___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__2(x_20, x_24, x_25); -x_27 = l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(x_26); -lean_inc(x_27); -x_28 = l_Lean_Lsp_ModuleRefs_findAt(x_27, x_5); -x_29 = lean_array_get_size(x_28); -x_30 = lean_usize_of_nat(x_29); -lean_dec(x_29); +x_25 = l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(x_24); +x_26 = lean_box(0); +x_27 = l_List_mapTRAux___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__2(x_20, x_25, x_26); +x_28 = l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(x_27); +lean_inc(x_28); +x_29 = l_Lean_Lsp_ModuleRefs_findAt(x_28, x_5); +x_30 = lean_array_get_size(x_29); +x_31 = lean_usize_of_nat(x_30); +lean_dec(x_30); lean_inc(x_2); -x_31 = l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__3(x_27, x_28, x_30, x_20, x_2); -lean_dec(x_28); -x_32 = l_Array_isEmpty___rarg(x_31); -if (x_32 == 0) +x_32 = l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__3(x_28, x_29, x_31, x_20, x_2); +lean_dec(x_29); +x_33 = l_Array_isEmpty___rarg(x_32); +if (x_33 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); lean_dec(x_2); -x_33 = lean_box(0); -x_34 = l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__2(x_31, x_20, x_33); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -lean_dec(x_34); -lean_ctor_set(x_10, 0, x_35); +x_34 = lean_box(0); +x_35 = l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__2(x_32, x_20, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +lean_dec(x_35); +lean_ctor_set(x_10, 0, x_36); return x_10; } else { -lean_object* x_36; lean_object* x_37; -lean_dec(x_31); +lean_object* x_37; lean_object* x_38; +lean_dec(x_32); lean_free_object(x_10); -x_36 = lean_box(0); -x_37 = l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__1(x_2, x_6, x_3, x_4, x_36, x_7, x_13); +x_37 = lean_box(0); +x_38 = l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__1(x_2, x_6, x_3, x_4, x_37, x_7, x_13); lean_dec(x_7); lean_dec(x_3); -return x_37; +return x_38; } } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; size_t x_45; size_t x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; size_t x_56; lean_object* x_57; uint8_t x_58; -x_38 = lean_ctor_get(x_10, 0); -x_39 = lean_ctor_get(x_10, 1); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; size_t x_46; size_t x_47; lean_object* x_48; uint8_t x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; size_t x_58; lean_object* x_59; uint8_t x_60; +x_39 = lean_ctor_get(x_10, 0); +x_40 = lean_ctor_get(x_10, 1); +lean_inc(x_40); lean_inc(x_39); -lean_inc(x_38); lean_dec(x_10); -x_40 = lean_ctor_get(x_38, 0); -lean_inc(x_40); -lean_dec(x_38); -x_41 = l_List_redLength___rarg(x_40); -x_42 = lean_mk_empty_array_with_capacity(x_41); -lean_dec(x_41); -x_43 = l_List_toArrayAux___rarg(x_40, x_42); -x_44 = lean_array_get_size(x_43); -x_45 = lean_usize_of_nat(x_44); -lean_dec(x_44); -x_46 = 0; -x_47 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__1(x_45, x_46, x_43); -x_48 = 1; +x_41 = lean_ctor_get(x_39, 0); +lean_inc(x_41); +lean_dec(x_39); +x_42 = l_List_redLength___rarg(x_41); +x_43 = lean_mk_empty_array_with_capacity(x_42); +lean_dec(x_42); +x_44 = l_List_toArrayAux___rarg(x_41, x_43); +x_45 = lean_array_get_size(x_44); +x_46 = lean_usize_of_nat(x_45); +lean_dec(x_45); +x_47 = 0; +x_48 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__1(x_46, x_47, x_44); +x_49 = 1; +x_50 = 0; lean_inc(x_3); -x_49 = l_Lean_Server_findModuleRefs(x_3, x_47, x_48); -lean_dec(x_47); -x_50 = l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(x_49); -x_51 = lean_box(0); -x_52 = l_List_mapTRAux___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__2(x_46, x_50, x_51); -x_53 = l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(x_52); -lean_inc(x_53); -x_54 = l_Lean_Lsp_ModuleRefs_findAt(x_53, x_5); -x_55 = lean_array_get_size(x_54); -x_56 = lean_usize_of_nat(x_55); -lean_dec(x_55); +x_51 = l_Lean_Server_findModuleRefs(x_3, x_48, x_49, x_50); +lean_dec(x_48); +x_52 = l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(x_51); +x_53 = lean_box(0); +x_54 = l_List_mapTRAux___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__2(x_47, x_52, x_53); +x_55 = l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(x_54); +lean_inc(x_55); +x_56 = l_Lean_Lsp_ModuleRefs_findAt(x_55, x_5); +x_57 = lean_array_get_size(x_56); +x_58 = lean_usize_of_nat(x_57); +lean_dec(x_57); lean_inc(x_2); -x_57 = l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__3(x_53, x_54, x_56, x_46, x_2); -lean_dec(x_54); -x_58 = l_Array_isEmpty___rarg(x_57); -if (x_58 == 0) +x_59 = l_Array_forInUnsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__3(x_55, x_56, x_58, x_47, x_2); +lean_dec(x_56); +x_60 = l_Array_isEmpty___rarg(x_59); +if (x_60 == 0) { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); lean_dec(x_2); -x_59 = lean_box(0); -x_60 = l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__2(x_57, x_46, x_59); -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -lean_dec(x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_39); -return x_62; +x_61 = lean_box(0); +x_62 = l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__2(x_59, x_47, x_61); +x_63 = lean_ctor_get(x_62, 0); +lean_inc(x_63); +lean_dec(x_62); +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_40); +return x_64; } else { -lean_object* x_63; lean_object* x_64; -lean_dec(x_57); -x_63 = lean_box(0); -x_64 = l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__1(x_2, x_6, x_3, x_4, x_63, x_7, x_39); +lean_object* x_65; lean_object* x_66; +lean_dec(x_59); +x_65 = lean_box(0); +x_66 = l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__1(x_2, x_6, x_3, x_4, x_65, x_7, x_40); lean_dec(x_7); lean_dec(x_3); -return x_64; +return x_66; } } } @@ -12819,179 +12812,48 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___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_EXPORT uint8_t l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1(lean_object* x_1) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_7 = l_Lean_Server_Snapshots_instInhabitedSnapshot; -x_8 = l_List_getLast_x21___rarg(x_7, x_1); -x_9 = lean_ctor_get(x_2, 0); -lean_inc(x_9); -lean_dec(x_2); -lean_inc(x_9); -x_10 = l_Lean_Server_DocumentMeta_mkInputContext(x_9); -x_11 = l_Lean_Server_Snapshots_parseAhead(x_10, x_8, x_6); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_array_to_list(lean_box(0), x_13); -x_15 = l_List_appendTR___rarg(x_3, x_14); -x_16 = lean_ctor_get(x_9, 2); -lean_inc(x_16); -lean_dec(x_9); -x_17 = l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols(x_16, x_15); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -lean_dec(x_17); -x_19 = l_List_redLength___rarg(x_18); -x_20 = lean_mk_empty_array_with_capacity(x_19); -lean_dec(x_19); -x_21 = l_List_toArrayAux___rarg(x_18, x_20); -lean_ctor_set(x_11, 0, x_21); -return x_11; -} -else -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_22 = lean_ctor_get(x_11, 0); -x_23 = lean_ctor_get(x_11, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_11); -x_24 = lean_array_to_list(lean_box(0), x_22); -x_25 = l_List_appendTR___rarg(x_3, x_24); -x_26 = lean_ctor_get(x_9, 2); -lean_inc(x_26); -lean_dec(x_9); -x_27 = l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols(x_26, x_25); -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -lean_dec(x_27); -x_29 = l_List_redLength___rarg(x_28); -x_30 = lean_mk_empty_array_with_capacity(x_29); -lean_dec(x_29); -x_31 = l_List_toArrayAux___rarg(x_28, x_30); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_23); -return x_32; -} +uint8_t x_2; +x_2 = 1; +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; -lean_dec(x_3); -x_6 = l_IO_AsyncList_getFinishedPrefix___rarg(x_1, x_5); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_7, 1); +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; 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_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_box(0); +x_7 = l_List_mapTRAux___at_Lean_Server_FileWorker_handleDocumentSymbol___spec__1(x_5, x_6); +x_8 = lean_ctor_get(x_1, 0); lean_inc(x_8); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_ctor_get(x_6, 1); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 2); lean_inc(x_9); -lean_dec(x_6); -x_10 = lean_ctor_get(x_7, 0); -lean_inc(x_10); -lean_dec(x_7); -x_11 = lean_box(0); -lean_inc(x_10); -x_12 = l_List_mapTRAux___at_Lean_Server_FileWorker_handleDocumentSymbol___spec__1(x_10, x_11); -x_13 = lean_box(0); -x_14 = l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1(x_10, x_2, x_12, x_13, x_4, x_9); -lean_dec(x_4); -return x_14; -} -else -{ -lean_object* x_15; -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_2); -x_15 = lean_ctor_get(x_8, 0); -lean_inc(x_15); lean_dec(x_8); -if (lean_obj_tag(x_15) == 0) -{ -uint8_t x_16; -x_16 = !lean_is_exclusive(x_6); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_6, 0); -lean_dec(x_17); -x_18 = l_Lean_Server_RequestError_fileChanged; -lean_ctor_set_tag(x_6, 1); -lean_ctor_set(x_6, 0, x_18); -return x_6; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_6, 1); -lean_inc(x_19); -lean_dec(x_6); -x_20 = l_Lean_Server_RequestError_fileChanged; -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -return x_21; -} -} -else -{ -uint8_t x_22; -x_22 = !lean_is_exclusive(x_6); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; -x_23 = lean_ctor_get(x_6, 0); -lean_dec(x_23); -x_24 = lean_ctor_get(x_15, 0); -lean_inc(x_24); -lean_dec(x_15); -x_25 = lean_io_error_to_string(x_24); -x_26 = 4; -x_27 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set_uint8(x_27, sizeof(void*)*1, x_26); -lean_ctor_set_tag(x_6, 1); -lean_ctor_set(x_6, 0, x_27); -return x_6; -} -else -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; -x_28 = lean_ctor_get(x_6, 1); -lean_inc(x_28); -lean_dec(x_6); -x_29 = lean_ctor_get(x_15, 0); -lean_inc(x_29); -lean_dec(x_15); -x_30 = lean_io_error_to_string(x_29); -x_31 = 4; -x_32 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set_uint8(x_32, sizeof(void*)*1, x_31); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_28); -return x_33; -} -} -} +x_10 = l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols(x_9, x_7); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +lean_dec(x_10); +x_12 = l_List_redLength___rarg(x_11); +x_13 = lean_mk_empty_array_with_capacity(x_12); +lean_dec(x_12); +x_14 = l_List_toArrayAux___rarg(x_11, x_13); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_4); +return x_15; } } static lean_object* _init_l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_IO_AsyncList_waitHead_x3f___rarg___lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1___boxed), 1, 0); return x_1; } } @@ -13008,16 +12870,14 @@ lean_dec(x_3); x_6 = lean_ctor_get(x_4, 1); lean_inc(x_6); x_7 = l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___closed__1; -lean_inc(x_6); -x_8 = l_IO_AsyncList_waitFind_x3f___rarg(x_7, x_6, x_5); +x_8 = l_IO_AsyncList_waitAll___rarg(x_7, x_6, x_5); x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); lean_dec(x_8); -x_11 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2), 5, 2); -lean_closure_set(x_11, 0, x_6); -lean_closure_set(x_11, 1, x_4); +x_11 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2___boxed), 4, 1); +lean_closure_set(x_11, 0, x_4); x_12 = l_Lean_Server_RequestM_mapTask___rarg(x_9, x_11, x_1, x_10); return x_12; } @@ -13030,14 +12890,23 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleDocumentSymbol__ return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1___boxed(lean_object* x_1) { _start: { -lean_object* x_7; -x_7 = l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_7; +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__1(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___lambda__2(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; } } LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol___boxed(lean_object* x_1) { @@ -13311,7 +13180,7 @@ lean_inc(x_37); lean_dec(x_36); x_38 = lean_nat_sub(x_37, x_34); lean_dec(x_37); -x_39 = l_Lean_Lsp_SemanticTokenType_toNat(x_2); +x_39 = l_Lean_Lsp_SemanticTokenType_toCtorIdx(x_2); x_40 = lean_ctor_get(x_4, 0); lean_inc(x_40); lean_dec(x_4); @@ -15111,43 +14980,53 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; x_7 = lean_ctor_get(x_4, 0); lean_inc(x_7); lean_dec(x_4); x_8 = lean_box(0); x_9 = l_Lean_Server_FileWorker_handleSemanticTokens___lambda__2___closed__1; x_10 = l_List_forIn_loop___at_Lean_Server_FileWorker_handleSemanticTokens___spec__1(x_1, x_2, x_3, x_7, x_8, x_9, x_5, x_6); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = !lean_is_exclusive(x_10); -if (x_13 == 0) +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_10, 0); -lean_dec(x_14); -x_15 = lean_ctor_get(x_12, 0); -lean_inc(x_15); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); lean_dec(x_12); -lean_ctor_set(x_10, 0, x_15); +x_14 = lean_box(0); +x_15 = lean_ctor_get(x_13, 0); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +lean_ctor_set(x_10, 0, x_16); return x_10; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); -lean_dec(x_10); -x_17 = lean_ctor_get(x_12, 0); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_17 = lean_ctor_get(x_10, 0); +x_18 = lean_ctor_get(x_10, 1); +lean_inc(x_18); lean_inc(x_17); -lean_dec(x_12); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_dec(x_10); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_box(0); +x_21 = lean_ctor_get(x_19, 0); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_18); +return x_23; } } } @@ -16566,15 +16445,7 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1(lean_object* x_1) { -_start: -{ -uint8_t x_2; -x_2 = 1; -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; @@ -16616,14 +16487,6 @@ return x_18; } } } -static lean_object* _init_l_Lean_Server_FileWorker_handleFoldingRange___rarg___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1___boxed), 1, 0); -return x_1; -} -} LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg(lean_object* x_1, lean_object* x_2) { _start: { @@ -16636,14 +16499,14 @@ lean_inc(x_5); lean_dec(x_3); x_6 = lean_ctor_get(x_4, 1); lean_inc(x_6); -x_7 = l_Lean_Server_FileWorker_handleFoldingRange___rarg___closed__1; +x_7 = l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___closed__1; x_8 = l_IO_AsyncList_waitAll___rarg(x_7, x_6, x_5); x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); x_10 = lean_ctor_get(x_8, 1); lean_inc(x_10); lean_dec(x_8); -x_11 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__2___boxed), 4, 1); +x_11 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1___boxed), 4, 1); lean_closure_set(x_11, 0, x_4); x_12 = l_Lean_Server_RequestM_mapTask___rarg(x_9, x_11, x_1, x_10); return x_12; @@ -16657,21 +16520,11 @@ x_2 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleFoldingRange___r return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___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_Server_FileWorker_handleFoldingRange___rarg___lambda__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_1); return x_5; @@ -16911,7 +16764,7 @@ lean_dec(x_4); x_7 = lean_ctor_get(x_5, 1); lean_inc(x_7); lean_dec(x_5); -x_8 = l_Lean_Server_FileWorker_handleFoldingRange___rarg___closed__1; +x_8 = l_Lean_Server_FileWorker_handleDocumentSymbol___rarg___closed__1; x_9 = l_IO_AsyncList_waitAll___rarg(x_8, x_7, x_6); x_10 = !lean_is_exclusive(x_9); if (x_10 == 0) @@ -17020,7 +16873,7 @@ lean_dec(x_1); return x_4; } } -static lean_object* _init_l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1() { +static lean_object* _init_l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1() { _start: { lean_object* x_1; @@ -17028,7 +16881,7 @@ x_1 = lean_mk_string_from_bytes("Cannot parse request params: ", 29); return x_1; } } -static lean_object* _init_l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2() { +static lean_object* _init_l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2() { _start: { lean_object* x_1; @@ -17036,7 +16889,7 @@ x_1 = lean_mk_string_from_bytes("\n", 1); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2(lean_object* x_1) { _start: { lean_object* x_2; @@ -17050,10 +16903,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -17073,10 +16926,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -17113,7 +16966,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -17138,11 +16991,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -17192,7 +17045,7 @@ return x_11; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -17201,38 +17054,38 @@ x_2 = l_Lean_Json_mkObj(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___closed__1; +x_2 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___closed__1; return x_2; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___boxed), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__3(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__3(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -17251,7 +17104,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -17265,7 +17118,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -17323,7 +17176,7 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -17331,28 +17184,28 @@ x_1 = l_Lean_Server_requestHandlers; return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__2; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__2; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -17378,7 +17231,7 @@ return x_17; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -17386,7 +17239,7 @@ x_1 = lean_mk_string_from_bytes("Failed to register LSP request handler for '", return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2() { _start: { lean_object* x_1; @@ -17394,12 +17247,12 @@ x_1 = lean_mk_string_from_bytes("': already registered", 21); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -17414,17 +17267,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -17447,17 +17300,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -17469,7 +17322,7 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1() { _start: { lean_object* x_1; @@ -17477,11 +17330,11 @@ x_1 = lean_mk_string_from_bytes("': only possible during initialization", 38); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -17496,10 +17349,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -17513,10 +17366,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -17533,12 +17386,12 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__5(lean_object* x_1) { _start: { lean_object* x_2; @@ -17552,10 +17405,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -17575,10 +17428,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -17615,7 +17468,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -17640,11 +17493,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__5(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__5(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -17694,7 +17547,7 @@ return x_11; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__1() { _start: { lean_object* x_1; @@ -17702,22 +17555,22 @@ x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__L return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__5(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__6(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__5(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__6(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -17736,7 +17589,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -17750,7 +17603,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -17808,28 +17661,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -17855,12 +17708,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -17875,17 +17728,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -17908,17 +17761,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -17930,11 +17783,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -17949,10 +17802,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -17966,10 +17819,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -17986,12 +17839,12 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__4(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__4(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__8(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__8(lean_object* x_1) { _start: { lean_object* x_2; @@ -18005,10 +17858,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -18028,10 +17881,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -18068,7 +17921,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -18093,11 +17946,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__8(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__8(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -18147,7 +18000,7 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__2(lean_object* x_1) { _start: { if (lean_obj_tag(x_1) == 0) @@ -18167,30 +18020,30 @@ return x_4; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__2), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__8(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__9(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__8(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__9(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -18209,7 +18062,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -18223,7 +18076,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -18281,28 +18134,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -18328,12 +18181,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -18348,17 +18201,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -18381,17 +18234,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -18403,11 +18256,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -18422,10 +18275,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -18439,10 +18292,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -18459,12 +18312,12 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__5(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__5(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__11(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__11(lean_object* x_1) { _start: { lean_object* x_2; @@ -18478,10 +18331,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -18501,10 +18354,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -18541,7 +18394,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -18566,7 +18419,7 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__13(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__13(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -18591,11 +18444,11 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__11(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__11(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -18645,7 +18498,7 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__2(lean_object* x_1) { _start: { lean_object* x_2; size_t x_3; size_t x_4; lean_object* x_5; lean_object* x_6; @@ -18653,36 +18506,36 @@ x_2 = lean_array_get_size(x_1); x_3 = lean_usize_of_nat(x_2); lean_dec(x_2); x_4 = 0; -x_5 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__13(x_3, x_4, x_1); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__13(x_3, x_4, x_1); x_6 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_6, 0, x_5); return x_6; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__2), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__11(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__12(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__11(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__12(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -18701,7 +18554,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -18715,7 +18568,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -18773,28 +18626,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -18820,12 +18673,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -18840,17 +18693,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -18873,17 +18726,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -18895,11 +18748,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -18914,10 +18767,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -18931,10 +18784,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -18951,12 +18804,12 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__5(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__5(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__15(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__15(lean_object* x_1) { _start: { lean_object* x_2; @@ -18970,10 +18823,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -18993,10 +18846,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -19033,7 +18886,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -19058,7 +18911,7 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__17(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__17(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -19083,11 +18936,11 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__15(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__15(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -19137,7 +18990,7 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__2(lean_object* x_1) { _start: { lean_object* x_2; size_t x_3; size_t x_4; lean_object* x_5; lean_object* x_6; @@ -19145,36 +18998,36 @@ x_2 = lean_array_get_size(x_1); x_3 = lean_usize_of_nat(x_2); lean_dec(x_2); x_4 = 0; -x_5 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__17(x_3, x_4, x_1); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__17(x_3, x_4, x_1); x_6 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_6, 0, x_5); return x_6; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__2), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__15(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__16(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__15(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__16(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -19193,7 +19046,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -19207,7 +19060,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -19265,28 +19118,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -19312,12 +19165,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -19332,17 +19185,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -19365,17 +19218,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -19387,11 +19240,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -19406,10 +19259,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -19423,10 +19276,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -19443,12 +19296,12 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__5(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__5(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__19(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__19(lean_object* x_1) { _start: { lean_object* x_2; @@ -19462,10 +19315,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -19485,10 +19338,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -19525,7 +19378,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__20(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -19550,11 +19403,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__19(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__19(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -19595,7 +19448,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__2(lean_object* x_1) { _start: { lean_object* x_2; size_t x_3; size_t x_4; lean_object* x_5; lean_object* x_6; @@ -19609,30 +19462,30 @@ lean_ctor_set(x_6, 0, x_5); return x_6; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__2), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__19(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__20(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__19(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__20(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -19651,7 +19504,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -19665,7 +19518,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -19723,28 +19576,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -19770,12 +19623,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -19790,17 +19643,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -19823,17 +19676,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -19845,11 +19698,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -19864,10 +19717,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -19881,10 +19734,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -19901,16 +19754,16 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__5(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__5(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__22(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__22(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3530_(x_1); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5081_(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -19920,10 +19773,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -19943,10 +19796,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -19983,7 +19836,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__23(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__23(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -20008,11 +19861,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__22(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__22(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -20053,30 +19906,30 @@ return x_8; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3761_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5339_), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__22(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__23(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__22(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__23(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -20095,7 +19948,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -20109,7 +19962,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -20167,28 +20020,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -20214,12 +20067,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -20234,17 +20087,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -20267,17 +20120,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -20289,11 +20142,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -20308,10 +20161,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -20325,10 +20178,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -20345,16 +20198,16 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__4(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__4(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__25(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__25(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3616_(x_1); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5167_(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -20364,10 +20217,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -20387,10 +20240,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -20427,7 +20280,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -20452,11 +20305,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__25(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__25(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -20506,12 +20359,12 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__25(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__26(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__25(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__26(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -20530,7 +20383,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -20544,7 +20397,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -20602,28 +20455,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__2), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__2), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -20649,12 +20502,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -20669,17 +20522,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -20702,17 +20555,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -20724,11 +20577,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -20743,10 +20596,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -20760,10 +20613,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -20780,16 +20633,16 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__4(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__4(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__28(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__28(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3801_(x_1); +x_2 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonFoldingRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5383_(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -20799,10 +20652,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -20822,10 +20675,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -20862,7 +20715,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__29(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__29(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -20887,7 +20740,7 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__30(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__30(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -20902,7 +20755,7 @@ lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x x_5 = lean_array_uget(x_3, x_2); x_6 = lean_unsigned_to_nat(0u); x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_3922_(x_5); +x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_5504_(x_5); x_9 = 1; x_10 = lean_usize_add(x_2, x_9); x_11 = lean_array_uset(x_7, x_2, x_8); @@ -20912,11 +20765,11 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__28(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__28(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -20957,7 +20810,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__2(lean_object* x_1) { _start: { lean_object* x_2; size_t x_3; size_t x_4; lean_object* x_5; lean_object* x_6; @@ -20965,36 +20818,36 @@ x_2 = lean_array_get_size(x_1); x_3 = lean_usize_of_nat(x_2); lean_dec(x_2); x_4 = 0; -x_5 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__30(x_3, x_4, x_1); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__30(x_3, x_4, x_1); x_6 = lean_alloc_ctor(4, 1, 0); lean_ctor_set(x_6, 0, x_5); return x_6; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__2), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__28(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__29(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__28(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__29(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -21013,7 +20866,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -21027,7 +20880,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -21085,28 +20938,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -21132,12 +20985,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -21152,17 +21005,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -21185,17 +21038,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -21207,11 +21060,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -21226,10 +21079,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -21243,10 +21096,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -21263,12 +21116,12 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__5(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__5(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__32(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__32(lean_object* x_1) { _start: { lean_object* x_2; @@ -21282,10 +21135,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -21305,10 +21158,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -21345,7 +21198,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__33(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__33(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -21370,11 +21223,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__32(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__32(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -21424,7 +21277,7 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__2(lean_object* x_1) { _start: { if (lean_obj_tag(x_1) == 0) @@ -21444,30 +21297,30 @@ return x_4; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__2), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__32(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__33(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__32(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__33(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -21486,7 +21339,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -21500,7 +21353,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -21558,28 +21411,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -21605,12 +21458,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -21625,17 +21478,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -21658,17 +21511,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -21680,11 +21533,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -21699,10 +21552,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -21716,10 +21569,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -21736,12 +21589,12 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__5(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__5(x_2, x_1, x_22, x_21); return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__35(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__35(lean_object* x_1) { _start: { lean_object* x_2; @@ -21755,10 +21608,10 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; x_4 = lean_ctor_get(x_2, 0); x_5 = l_Lean_Json_compress(x_1); -x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_string_append(x_9, x_4); lean_dec(x_4); @@ -21778,10 +21631,10 @@ x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); lean_dec(x_2); x_16 = l_Lean_Json_compress(x_1); -x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1; +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1; x_18 = lean_string_append(x_17, x_16); lean_dec(x_16); -x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2; +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2; x_20 = lean_string_append(x_18, x_19); x_21 = lean_string_append(x_20, x_15); lean_dec(x_15); @@ -21818,7 +21671,7 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__36(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__36(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -21843,11 +21696,11 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__35(x_1); +x_2 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__35(x_1); if (lean_obj_tag(x_2) == 0) { uint8_t x_3; @@ -21897,7 +21750,7 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__2(lean_object* x_1) { _start: { if (lean_obj_tag(x_1) == 0) @@ -21917,30 +21770,30 @@ return x_4; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__2), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__2() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__1; +x_1 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__1; x_2 = lean_alloc_closure((void*)(l_Except_map___rarg), 2, 1); lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__35(x_2); -x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__36(x_5, x_3, x_4); +x_5 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__35(x_2); +x_6 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__36(x_5, x_3, x_4); lean_dec(x_5); if (lean_obj_tag(x_6) == 0) { @@ -21959,7 +21812,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__2; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__2; x_13 = l_Task_Priority_default; x_14 = lean_task_map(x_12, x_11, x_13); lean_ctor_set(x_9, 0, x_14); @@ -21973,7 +21826,7 @@ x_16 = lean_ctor_get(x_9, 1); lean_inc(x_16); lean_inc(x_15); lean_dec(x_9); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__2; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__2; x_18 = l_Task_Priority_default; x_19 = lean_task_map(x_17, x_15, x_18); x_20 = lean_alloc_ctor(0, 2, 0); @@ -22031,28 +21884,28 @@ return x_28; } } } -static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__1), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__1), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3), 4, 1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3), 4, 1); lean_closure_set(x_5, 0, x_1); -x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_6 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); x_9 = lean_ctor_get(x_7, 1); lean_inc(x_9); lean_dec(x_7); -x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4___closed__1; +x_10 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4___closed__1; x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_5); @@ -22078,12 +21931,12 @@ return x_17; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_dec(x_3); -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1; +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1; x_6 = lean_st_ref_get(x_5, x_4); x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) @@ -22098,17 +21951,17 @@ if (x_10 == 0) lean_object* x_11; lean_object* x_12; lean_free_object(x_6); x_11 = lean_box(0); -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4(x_1, x_2, x_11, x_9); +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4(x_1, x_2, x_11, x_9); return x_12; } else { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_13 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_14 = lean_string_append(x_13, x_2); lean_dec(x_2); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_16 = lean_string_append(x_14, x_15); x_17 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_17, 0, x_16); @@ -22131,17 +21984,17 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4(x_1, x_2, x_21, x_19); +x_22 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4(x_1, x_2, x_21, x_19); return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_1); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_24 = lean_string_append(x_23, x_2); lean_dec(x_2); -x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2; +x_25 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2; x_26 = lean_string_append(x_24, x_25); x_27 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_27, 0, x_26); @@ -22153,11 +22006,11 @@ return x_28; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -22172,10 +22025,10 @@ if (x_7 == 0) lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_8 = lean_ctor_get(x_4, 0); lean_dec(x_8); -x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_9 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_10 = lean_string_append(x_9, x_1); lean_dec(x_1); -x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_11 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_12 = lean_string_append(x_10, x_11); x_13 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_13, 0, x_12); @@ -22189,10 +22042,10 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean x_14 = lean_ctor_get(x_4, 1); lean_inc(x_14); lean_dec(x_4); -x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1; +x_15 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1; x_16 = lean_string_append(x_15, x_1); lean_dec(x_1); -x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1; +x_17 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -22209,12 +22062,12 @@ x_21 = lean_ctor_get(x_4, 1); lean_inc(x_21); lean_dec(x_4); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__5(x_2, x_1, x_22, x_21); +x_23 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__5(x_2, x_1, x_22, x_21); return x_23; } } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__1() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__1() { _start: { lean_object* x_1; @@ -22222,7 +22075,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/waitForDiagnostics", 31); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__2() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__2() { _start: { lean_object* x_1; @@ -22230,7 +22083,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleWaitForDiagnosti return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__3() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__3() { _start: { lean_object* x_1; @@ -22238,7 +22091,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/completion", 23); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__4() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__4() { _start: { lean_object* x_1; @@ -22246,7 +22099,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleCompletion), 3, return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__5() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__5() { _start: { lean_object* x_1; @@ -22254,7 +22107,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/hover", 18); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__6() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__6() { _start: { lean_object* x_1; @@ -22262,7 +22115,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleHover), 3, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__7() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__7() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; @@ -22273,7 +22126,7 @@ lean_closure_set(x_3, 0, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__8() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__8() { _start: { lean_object* x_1; @@ -22281,7 +22134,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/declaration", 24); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__9() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__9() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; @@ -22292,7 +22145,7 @@ lean_closure_set(x_3, 0, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__10() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__10() { _start: { lean_object* x_1; @@ -22300,7 +22153,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/definition", 23); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__11() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__11() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; @@ -22311,7 +22164,7 @@ lean_closure_set(x_3, 0, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__12() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__12() { _start: { lean_object* x_1; @@ -22319,7 +22172,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/typeDefinition", 27); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__13() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__13() { _start: { lean_object* x_1; @@ -22327,7 +22180,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/documentHighlight", 30); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__14() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__14() { _start: { lean_object* x_1; @@ -22335,7 +22188,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleDocumentHighligh return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__15() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__15() { _start: { lean_object* x_1; @@ -22343,7 +22196,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/documentSymbol", 27); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__16() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__16() { _start: { lean_object* x_1; @@ -22351,7 +22204,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleDocumentSymbol__ return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__17() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__17() { _start: { lean_object* x_1; @@ -22359,7 +22212,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/semanticTokens/full", 32); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__18() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__18() { _start: { lean_object* x_1; @@ -22367,7 +22220,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleSemanticTokensFu return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__19() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__19() { _start: { lean_object* x_1; @@ -22375,7 +22228,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/semanticTokens/range", 33); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__20() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__20() { _start: { lean_object* x_1; @@ -22383,7 +22236,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleSemanticTokensRa return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__21() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__21() { _start: { lean_object* x_1; @@ -22391,7 +22244,7 @@ x_1 = lean_mk_string_from_bytes("textDocument/foldingRange", 25); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__22() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__22() { _start: { lean_object* x_1; @@ -22399,7 +22252,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handleFoldingRange___b return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__23() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__23() { _start: { lean_object* x_1; @@ -22407,7 +22260,7 @@ x_1 = lean_mk_string_from_bytes("$/lean/plainGoal", 16); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__24() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__24() { _start: { lean_object* x_1; @@ -22415,7 +22268,7 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handlePlainGoal), 3, 0 return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__25() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__25() { _start: { lean_object* x_1; @@ -22423,7 +22276,7 @@ x_1 = lean_mk_string_from_bytes("$/lean/plainTermGoal", 20); return x_1; } } -static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__26() { +static lean_object* _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__26() { _start: { lean_object* x_1; @@ -22431,121 +22284,121 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_handlePlainTermGoal), return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__1; -x_3 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__2; -x_4 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1(x_2, x_3, x_1); +x_2 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__1; +x_3 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__2; +x_4 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1(x_2, x_3, x_1); if (lean_obj_tag(x_4) == 0) { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_5 = lean_ctor_get(x_4, 1); lean_inc(x_5); lean_dec(x_4); -x_6 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__3; -x_7 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__4; -x_8 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4(x_6, x_7, x_5); +x_6 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__3; +x_7 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__4; +x_8 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4(x_6, x_7, x_5); if (lean_obj_tag(x_8) == 0) { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; x_9 = lean_ctor_get(x_8, 1); lean_inc(x_9); lean_dec(x_8); -x_10 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__5; -x_11 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__6; -x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7(x_10, x_11, x_9); +x_10 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__5; +x_11 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__6; +x_12 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7(x_10, x_11, x_9); if (lean_obj_tag(x_12) == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; x_13 = lean_ctor_get(x_12, 1); lean_inc(x_13); lean_dec(x_12); -x_14 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__8; -x_15 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__7; -x_16 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10(x_14, x_15, x_13); +x_14 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__8; +x_15 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__7; +x_16 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10(x_14, x_15, x_13); if (lean_obj_tag(x_16) == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_17 = lean_ctor_get(x_16, 1); lean_inc(x_17); lean_dec(x_16); -x_18 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__10; -x_19 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__9; -x_20 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10(x_18, x_19, x_17); +x_18 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__10; +x_19 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__9; +x_20 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10(x_18, x_19, x_17); if (lean_obj_tag(x_20) == 0) { lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; x_21 = lean_ctor_get(x_20, 1); lean_inc(x_21); lean_dec(x_20); -x_22 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__12; -x_23 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__11; -x_24 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10(x_22, x_23, x_21); +x_22 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__12; +x_23 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__11; +x_24 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10(x_22, x_23, x_21); if (lean_obj_tag(x_24) == 0) { lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; x_25 = lean_ctor_get(x_24, 1); lean_inc(x_25); lean_dec(x_24); -x_26 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__13; -x_27 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__14; -x_28 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14(x_26, x_27, x_25); +x_26 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__13; +x_27 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__14; +x_28 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14(x_26, x_27, x_25); if (lean_obj_tag(x_28) == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; x_29 = lean_ctor_get(x_28, 1); lean_inc(x_29); lean_dec(x_28); -x_30 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__15; -x_31 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__16; -x_32 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18(x_30, x_31, x_29); +x_30 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__15; +x_31 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__16; +x_32 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18(x_30, x_31, x_29); if (lean_obj_tag(x_32) == 0) { lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; x_33 = lean_ctor_get(x_32, 1); lean_inc(x_33); lean_dec(x_32); -x_34 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__17; -x_35 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__18; -x_36 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21(x_34, x_35, x_33); +x_34 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__17; +x_35 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__18; +x_36 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21(x_34, x_35, x_33); if (lean_obj_tag(x_36) == 0) { lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; x_37 = lean_ctor_get(x_36, 1); lean_inc(x_37); lean_dec(x_36); -x_38 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__19; -x_39 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__20; -x_40 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24(x_38, x_39, x_37); +x_38 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__19; +x_39 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__20; +x_40 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24(x_38, x_39, x_37); if (lean_obj_tag(x_40) == 0) { lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; x_41 = lean_ctor_get(x_40, 1); lean_inc(x_41); lean_dec(x_40); -x_42 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__21; -x_43 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__22; -x_44 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27(x_42, x_43, x_41); +x_42 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__21; +x_43 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__22; +x_44 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27(x_42, x_43, x_41); if (lean_obj_tag(x_44) == 0) { lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; x_45 = lean_ctor_get(x_44, 1); lean_inc(x_45); lean_dec(x_44); -x_46 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__23; -x_47 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__24; -x_48 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31(x_46, x_47, x_45); +x_46 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__23; +x_47 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__24; +x_48 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31(x_46, x_47, x_45); if (lean_obj_tag(x_48) == 0) { lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; x_49 = lean_ctor_get(x_48, 1); lean_inc(x_49); lean_dec(x_48); -x_50 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__25; -x_51 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__26; -x_52 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34(x_50, x_51, x_49); +x_50 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__25; +x_51 = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__26; +x_52 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34(x_50, x_51, x_49); return x_52; } else @@ -22825,83 +22678,83 @@ return x_100; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__3(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__3(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2(x_1); +x_2 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__6(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__6(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__9(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__9(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__12(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__12(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -22909,30 +22762,30 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__13(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__13(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__16(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__16(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -22940,87 +22793,87 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__17(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__17(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__20(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__20(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__23(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__23(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__26(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__26(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__29(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__29(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -23028,53 +22881,53 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__30(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__30(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__33___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__33___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__33(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__33(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__36___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__36___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__36(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__36(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -23346,143 +23199,141 @@ l_Lean_Server_FileWorker_handleFoldingRange_addRanges___closed__1 = _init_l_Lean lean_mark_persistent(l_Lean_Server_FileWorker_handleFoldingRange_addRanges___closed__1); l_Lean_Server_FileWorker_handleFoldingRange_addRanges___closed__2 = _init_l_Lean_Server_FileWorker_handleFoldingRange_addRanges___closed__2(); lean_mark_persistent(l_Lean_Server_FileWorker_handleFoldingRange_addRanges___closed__2); -l_Lean_Server_FileWorker_handleFoldingRange___rarg___closed__1 = _init_l_Lean_Server_FileWorker_handleFoldingRange___rarg___closed__1(); -lean_mark_persistent(l_Lean_Server_FileWorker_handleFoldingRange___rarg___closed__1); l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__1___closed__1 = _init_l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__1___closed__1); l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__2___closed__1 = _init_l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Server_FileWorker_handleWaitForDiagnostics___lambda__2___closed__1); l_Lean_Server_FileWorker_handleWaitForDiagnostics___closed__1 = _init_l_Lean_Server_FileWorker_handleWaitForDiagnostics___closed__1(); lean_mark_persistent(l_Lean_Server_FileWorker_handleWaitForDiagnostics___closed__1); -l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1 = _init_l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1(); -lean_mark_persistent(l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__1); -l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2 = _init_l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2(); -lean_mark_persistent(l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__2___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__2___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__3___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__4___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___lambda__5___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__1___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__2___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__4___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__3___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__7___lambda__4___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__3___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__10___lambda__4___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__3___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__14___lambda__4___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__3___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__18___lambda__4___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__2___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__21___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__24___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__3___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__27___lambda__4___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__3___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__31___lambda__4___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__1); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__3___closed__2); -l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____spec__34___lambda__4___closed__1); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__1 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__1(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__1); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__2 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__2(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__2); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__3 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__3(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__3); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__4 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__4(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__4); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__5 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__5(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__5); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__6 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__6(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__6); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__7 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__7(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__7); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__8 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__8(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__8); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__9 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__9(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__9); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__10 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__10(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__10); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__11 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__11(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__11); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__12 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__12(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__12); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__13 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__13(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__13); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__14 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__14(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__14); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__15 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__15(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__15); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__16 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__16(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__16); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__17 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__17(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__17); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__18 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__18(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__18); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__19 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__19(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__19); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__20 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__20(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__20); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__21 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__21(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__21); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__22 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__22(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__22); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__23 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__23(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__23); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__24 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__24(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__24); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__25 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__25(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__25); -l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__26 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__26(); -lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775____closed__26); -res = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9775_(lean_io_mk_world()); +l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1 = _init_l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1(); +lean_mark_persistent(l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__1); +l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2 = _init_l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2(); +lean_mark_persistent(l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__2___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__2___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__3___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__4___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___lambda__5___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__1___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__2___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__4___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__3___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__7___lambda__4___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__3___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__10___lambda__4___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__3___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__14___lambda__4___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__3___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__18___lambda__4___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__2___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__21___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__24___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__3___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__27___lambda__4___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__3___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__31___lambda__4___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__1); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__2 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__3___closed__2); +l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4___closed__1 = _init_l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__34___lambda__4___closed__1); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__1 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__1(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__1); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__2 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__2(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__2); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__3 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__3(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__3); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__4 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__4(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__4); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__5 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__5(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__5); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__6 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__6(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__6); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__7 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__7(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__7); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__8 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__8(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__8); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__9 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__9(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__9); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__10 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__10(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__10); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__11 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__11(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__11); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__12 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__12(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__12); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__13 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__13(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__13); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__14 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__14(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__14); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__15 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__15(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__15); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__16 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__16(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__16); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__17 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__17(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__17); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__18 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__18(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__18); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__19 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__19(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__19); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__20 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__20(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__20); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__21 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__21(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__21); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__22 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__22(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__22); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__23 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__23(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__23); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__24 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__24(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__24); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__25 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__25(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__25); +l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__26 = _init_l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__26(); +lean_mark_persistent(l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____closed__26); +res = l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629_(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/Server/FileWorker/WidgetRequests.c b/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c index 1bc849fe782d..52dc03436182 100644 --- a/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c +++ b/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c @@ -13,348 +13,526 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__9; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__1; -lean_object* l_Lean_instToJsonBool___boxed(lean_object*); -lean_object* l_Lean_Widget_TaggedText_instRpcEncodingTaggedText___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25(lean_object*); size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__9(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Lsp_instToJsonDiagnosticCode___boxed(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -lean_object* l_Lean_instToJsonOption___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15; +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__9; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__6(size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____closed__1; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311_(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__8; -extern lean_object* l_Lean_instFromJsonNat; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__8___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036_(lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__12; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -lean_object* l_Lean_instToJsonArray___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__32___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Widget_getInteractiveDiagnostics___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__13(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_ppExprTagged(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__2(lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__9(size_t, size_t, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); lean_object* lean_io_error_to_string(lean_object*); -lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__33___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__12(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoPopup___closed__1; -lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___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_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__22; -lean_object* l_Lean_Json_getObjValAs_x3f(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__4; -extern lean_object* l_Lean_Server_instFromJsonGoToKind; -LEAN_EXPORT lean_object* l_ReaderT_read___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__9___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Server_FileWorker_instMonadRpcSession___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__7; +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33(lean_object*); +lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__3; +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__1; lean_object* l_Lean_Elab_Info_type_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__17; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__4; +lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320_(lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__29___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__30(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1(lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__2; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__4; -lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__5(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__17(lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__3; extern lean_object* l_Lean_Server_builtinRpcProcedures; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__3; -static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; LEAN_EXPORT uint8_t l_Lean_Widget_getInteractiveDiagnostics___lambda__3(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__11; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__23(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__3; lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__38(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__8(lean_object*, lean_object*); -lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__5; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__8; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__9(lean_object*, lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__4___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__9___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_lspPosToUtf8Pos(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__7(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__17___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1563_(lean_object*); +lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845_(lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__7; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3; lean_object* l_List_join___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Lsp_instToJsonLocationLink; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1349_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_instToJsonNat(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__1(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__13; +uint8_t lean_usize_dec_lt(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__5; +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1074_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__30___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1074____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__3(lean_object*, lean_object*, uint64_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__3(lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23; -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedGetInteractiveDiagnosticsParams; -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__4; +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__5(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__4(uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2(lean_object*, lean_object*); -lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__7___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__24; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__3(lean_object*, lean_object*, uint64_t, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonLineRange____x40_Lean_Data_Lsp_Extra___hyg_1865_(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__1(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__6; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__2; -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__28(lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__10(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7(lean_object*, lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonPosition____x40_Lean_Data_Lsp_Basic___hyg_402____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); lean_object* l_List_getLast_x3f___rarg(lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__3; -LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1349____spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__1; +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__6; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__15(lean_object*, size_t, size_t, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__4(size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__7___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__8(lean_object*); +lean_object* l_Lean_Json_compress(lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); -extern lean_object* l_Lean_Lsp_instToJsonDiagnosticRelatedInformation; -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__18; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__2; -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__7___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__2(lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__26___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__10(size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__2(lean_object*, lean_object*, uint64_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__6(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__2; +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__2; +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34(lean_object*); static lean_object* l_Lean_Widget_getInteractiveDiagnostics___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__8___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__6(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__1(size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; lean_object* l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__26; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__9___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Lsp_instToJsonRpcRef; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__9(lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__9; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__9; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__5; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__6___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__31(lean_object*); lean_object* l_IO_AsyncList_waitAll___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__8; -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__8___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__1; +LEAN_EXPORT lean_object* l_ReaderT_read___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____lambda__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__8(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__8; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__22(lean_object*); static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__2(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__5; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_194____rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__3(lean_object*); lean_object* lean_task_map(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__4(lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2161____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__32(lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__5___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instToJsonGetInteractiveDiagnosticsParams___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_689____rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____rarg(lean_object*, lean_object*); -lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg(lean_object*); -lean_object* l_Lean_Server_instRpcEncoding___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__4___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +lean_object* l_Lean_Server_RequestM_bindTask___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__27(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__13(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_FileWorker_getInteractiveGoals(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____lambda__2(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Server_instRpcEncoding___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1(lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Lsp_instFromJsonRpcRef; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__4(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__3; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__9(lean_object*, size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +lean_object* l_Lean_Server_RequestM_mapTask___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedInfoPopup; lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3; static lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__1; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__3(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__8; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__14(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__19; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3___closed__1; -lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__10; +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__5(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1065_(size_t); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__8; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__31___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__4(size_t, size_t, lean_object*); static lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2; uint8_t l_Array_isEmpty___rarg(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__3; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__4; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__37___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__3(lean_object*, lean_object*, uint64_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__22___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__20___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__7(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonGetInteractiveDiagnosticsParams; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__7; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__6; +lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__32(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5(lean_object*); extern lean_object* l_Task_Priority_default; +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics(lean_object*, lean_object*, lean_object*); -lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2648____rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__6; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__36___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_msgToInteractive(lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; lean_object* l_Lean_Elab_Info_docString_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__5; -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__25; -lean_object* l_Lean_Widget_instToJsonMVarId(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__21; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15(lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24_(uint8_t); LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__2; +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4; +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__1; +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__3; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__4(uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__4___boxed(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; -static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -extern lean_object* l_Lean_Lsp_instFromJsonPlainTermGoalParams; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__5(lean_object*, lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__36(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedMsgToInteractive___closed__1; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__4(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__16; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__38___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_JsonNumber_fromNat(lean_object*); lean_object* l_Lean_Json_getObjValD(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__3___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__3; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1744_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_689_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_194_(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__5; -static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1___closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__14; +static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__5(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1390_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_115_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__9(lean_object*); +extern lean_object* l_Id_instMonadId; uint8_t lean_nat_dec_le(lean_object*, lean_object*); -lean_object* l_Lean_Server_instRpcEncodingOption___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__28; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__1(lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*); +static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; lean_object* l_Std_PersistentArray_toArray___rarg(lean_object*); -lean_object* l_Lean_Server_instRpcEncodingArray___rarg(lean_object*); static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1; -lean_object* l_Lean_instToJsonString(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__9; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__6; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__3(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__2(lean_object*, lean_object*, uint64_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__3; LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__2___boxed(lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__2; static lean_object* l_Lean_Widget_instInhabitedMsgToInteractive___closed__2; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__18(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__21(lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__1; +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__4; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__5___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_makePopup(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__8; +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__3; lean_object* l_Lean_Json_mkObj(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__1(uint8_t, lean_object*, size_t); +lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1027_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__2; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__12; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__20(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2131____spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__9___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_194____rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__19(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__2(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*); lean_object* l_Lean_Expr_constName_x3f(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__2; -static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__9; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); -lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1642____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__4___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_StateT_instMonadStateT___rarg(lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__3; +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__4(lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__8___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__16(lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__29(lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__1(lean_object*, lean_object*); lean_object* lean_io_initializing(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__20; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2(lean_object*, lean_object*); lean_object* l_Lean_Server_locationLinksFromDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__3; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__5; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__10; +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__5; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2; +static lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Lsp_instToJsonDiagnosticSeverity___boxed(lean_object*); -static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_instToJsonName(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Lsp_instToJsonRange; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__7___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__4(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__26(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__35(lean_object*); lean_object* l_Lean_Server_RequestM_asTask___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__7(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__3; +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__7; lean_object* l_Lean_Expr_getAppFn(lean_object*); -lean_object* l_Lean_Widget_instToJsonFVarId(lean_object*); +static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1; +lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__11(size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__2; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__3(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(lean_object*, uint64_t); +lean_object* l_instMonadStateOfStateT___rarg(lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2; +lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__4(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__37(lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__20(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__35(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Info_lctx(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__4; -static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1744____rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__6___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__1(lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_ContextInfo_runMetaM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___closed__3; static lean_object* l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Server_FileWorker_getInteractiveTermGoal(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__11; -lean_object* l_Lean_Server_wrapRpcProcedure___elambda__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___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__3; -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__7; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2; -lean_object* l_Lean_Lsp_instToJsonDiagnosticTag___boxed(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__6; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket(lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2; +static lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__7; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__3; LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__1; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4(lean_object*, lean_object*, uint64_t, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonLineRange____x40_Lean_Data_Lsp_Extra___hyg_1810_(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__1(lean_object*); -lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2236____rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569_(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__4___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_RequestM_readDoc(lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__27; -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Lsp_instFromJsonPlainGoalParams; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -extern lean_object* l_Lean_SubExpr_Pos_instToJsonPos; -static lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedMsgToInteractive; static lean_object* _init_l_Lean_Widget_instInhabitedMsgToInteractive___closed__1() { _start: @@ -386,7 +564,7 @@ x_1 = l_Lean_Widget_instInhabitedMsgToInteractive___closed__2; return x_1; } } -static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__1() { +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__1() { _start: { lean_object* x_1; @@ -394,7 +572,7 @@ x_1 = lean_mk_string_from_bytes("msg", 3); return x_1; } } -static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__2() { +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__2() { _start: { lean_object* x_1; @@ -402,190 +580,173 @@ x_1 = lean_mk_string_from_bytes("indent", 6); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60_(lean_object* x_1) { _start: { -lean_object* x_4; lean_object* x_5; -x_4 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__1; -x_5 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_1, x_4); -if (lean_obj_tag(x_5) == 0) +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1(x_1, x_2); +if (lean_obj_tag(x_3) == 0) { -uint8_t x_6; -lean_dec(x_2); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) { -return x_5; +return x_3; } else { -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -lean_dec(x_5); -x_10 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__2; -x_11 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_2, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +x_8 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__2; +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonPosition____x40_Lean_Data_Lsp_Basic___hyg_402____spec__1(x_1, x_8); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_12; -lean_dec(x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_10; +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -return x_11; +return x_9; } else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_11); -if (x_15 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_9); +if (x_13 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_11, 0); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_9); -lean_ctor_set(x_17, 1, x_16); -lean_ctor_set(x_11, 0, x_17); -return x_11; +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_9, 0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_7); +lean_ctor_set(x_15, 1, x_14); +lean_ctor_set(x_9, 0, x_15); +return x_9; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_11, 0); -lean_inc(x_18); -lean_dec(x_11); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_9); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_20, 0, x_19); -return x_20; -} -} +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_9, 0); +lean_inc(x_16); +lean_dec(x_9); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_7); +lean_ctor_set(x_17, 1, x_16); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; } } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___boxed), 3, 0); -return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____boxed(lean_object* x_1) { _start: { -lean_object* x_4; -x_4 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; +lean_object* x_2; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60_(x_1); +lean_dec(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__7___rarg(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__7___closed__1() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___boxed), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____boxed), 1, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__7(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__7() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__7___rarg), 2, 0); -return x_3; +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket__7___closed__1; +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_194____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_115_(lean_object* x_1) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); -x_5 = lean_apply_1(x_1, x_4); -x_6 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__1; -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_9, 0, x_7); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_ctor_get(x_3, 1); -lean_inc(x_10); -lean_dec(x_3); -x_11 = lean_apply_1(x_2, x_10); -x_12 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__2; +lean_object* x_2; size_t x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_4 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1065_(x_3); +x_5 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__1; +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_5); +lean_ctor_set(x_6, 1, x_4); +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_6); +lean_ctor_set(x_8, 1, x_7); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +lean_dec(x_1); +x_10 = l_Lean_JsonNumber_fromNat(x_9); +x_11 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__2; x_13 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_13, 0, x_12); lean_ctor_set(x_13, 1, x_11); x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_8); +lean_ctor_set(x_14, 1, x_7); x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_8); +lean_ctor_set(x_15, 1, x_7); x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_9); +lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l_List_join___rarg(x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_194_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_194____rarg), 3, 0); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__7___rarg(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__7___closed__1() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_194____rarg), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_115_), 1, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__7(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__7() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__7___rarg), 2, 0); -return x_3; +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket__7___closed__1; +return x_1; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -635,15 +796,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__1___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__1___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -693,3732 +854,25763 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__2___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__2___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; lean_dec(x_4); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_2); -lean_ctor_set(x_6, 1, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_1, 0); lean_inc(x_7); lean_dec(x_1); -x_8 = lean_ctor_get(x_2, 1); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); -lean_dec(x_2); -lean_inc(x_3); -x_9 = lean_apply_4(x_7, lean_box(0), x_3, x_4, x_8); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__1), 3, 2); -lean_closure_set(x_10, 0, x_3); -lean_closure_set(x_10, 1, x_6); -x_11 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_9, x_10); -return x_11; -} +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_7 = lean_ctor_get(x_4, 1); -lean_inc(x_7); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = lean_ctor_get(x_6, 0); -lean_inc(x_9); -lean_inc(x_5); -lean_inc(x_4); -x_10 = lean_apply_4(x_8, lean_box(0), x_4, x_5, x_9); -lean_inc(x_7); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__2), 6, 5); -lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, x_6); -lean_closure_set(x_11, 2, x_4); -lean_closure_set(x_11, 3, x_5); -lean_closure_set(x_11, 4, x_7); -x_12 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_10, x_11); -return x_12; +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_3); -x_5 = lean_ctor_get(x_2, 0); -lean_inc(x_5); -lean_dec(x_2); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); lean_dec(x_5); -x_7 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_7, 0, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__3(lean_object* x_1) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -lean_dec(x_1); -x_7 = lean_ctor_get(x_2, 1); -lean_inc(x_7); -lean_dec(x_2); -lean_inc(x_3); -x_8 = lean_apply_4(x_6, lean_box(0), x_3, x_4, x_7); -lean_inc(x_3); -x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__4), 3, 2); -lean_closure_set(x_9, 0, x_5); -lean_closure_set(x_9, 1, x_3); -x_10 = lean_ctor_get(x_3, 1); -lean_inc(x_10); -x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_11, 0, x_3); -lean_closure_set(x_11, 1, lean_box(0)); -lean_closure_set(x_11, 2, lean_box(0)); -lean_closure_set(x_11, 3, x_9); -x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); -return x_12; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__3___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_1, 1); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); lean_inc(x_7); lean_dec(x_1); -x_8 = lean_ctor_get(x_6, 0); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); -lean_inc(x_5); -lean_inc(x_4); -x_9 = lean_apply_4(x_7, lean_box(0), x_4, x_5, x_8); -lean_inc(x_4); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__5), 5, 4); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_6); -lean_closure_set(x_10, 2, x_4); -lean_closure_set(x_10, 3, x_5); -x_11 = lean_ctor_get(x_4, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_12, 0, x_4); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); -return x_13; +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +} +else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -lean_inc(x_3); -lean_inc(x_1); -x_4 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__3), 6, 2); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_3); -x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg___lambda__6), 6, 2); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_3); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_4); -lean_ctor_set(x_6, 1, x_5); -return x_6; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__4(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg), 3, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__4___rarg), 5, 0); return x_2; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncoding___lambda__1___boxed), 4, 0); -return x_1; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_box_usize(x_1); +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_2, lean_box(0), x_6); +return x_7; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__2(lean_object* x_1, lean_object* x_2, size_t x_3) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncoding___lambda__2___boxed), 4, 0); -return x_1; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__1___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__1; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__2; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_apply_4(x_6, lean_box(0), x_2, x_3, x_7); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__2___boxed), 3, 2); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_2); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__2___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__4() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_3 = l_Lean_Widget_instRpcEncodingMsgToInteractiveRpcEncodingPacket___rarg(x_1, lean_box(0), x_2); -return x_3; +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +x_6 = lean_apply_2(x_2, lean_box(0), x_5); +return x_6; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__5() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Lsp_instFromJsonRpcRef; -x_2 = l_Lean_instFromJsonNat; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___boxed), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__4), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__3___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__6() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_3 = l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg(x_1, lean_box(0), x_2); -return x_3; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_apply_4(x_6, lean_box(0), x_2, x_3, x_7); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__5___boxed), 3, 2); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_2); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgToInteractive___spec__4___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7() { +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__6; -x_2 = l_Lean_Widget_TaggedText_instRpcEncodingTaggedText___rarg(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__3), 4, 0); +return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8() { +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_2 = l_Lean_Server_instRpcEncodingArray___rarg(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__6), 4, 0); +return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__9() { +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg(x_1, lean_box(0), x_1, lean_box(0), x_2, lean_box(0), x_3); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__10() { +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgToInteractive() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__9; -x_2 = l_Lean_Server_instRpcEncodingArray___rarg(x_1); -return x_2; +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__3; +return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__11() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__10; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg(x_1, lean_box(0), x_2, lean_box(0), x_3, lean_box(0), x_3); -return x_4; +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__1(x_4, x_2, x_3); +return x_5; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__12() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__11; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; -x_5 = l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg(x_1, lean_box(0), x_2, lean_box(0), x_3, lean_box(0), x_3, lean_box(0), x_4); +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__2(x_1, x_2, x_4); +lean_dec(x_1); return x_5; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__13() { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__12; -x_2 = l_Lean_Widget_TaggedText_instRpcEncodingTaggedText___rarg(x_1); -return x_2; +lean_object* x_4; +x_4 = l_Lean_Widget_instRpcEncodingMsgToInteractive___lambda__5(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__14() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__4(size_t x_1, size_t x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Lsp_instToJsonRpcRef; -x_2 = l_Lean_SubExpr_Pos_instToJsonPos; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_194____rarg), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ return x_3; } -} -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__14; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__16() { +} +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_instToJsonName), 1, 0); +x_1 = lean_mk_string_from_bytes("text", 4); return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__17() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__16; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__18() { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonFVarId), 1, 0); +x_1 = lean_mk_string_from_bytes("append", 6); return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__19() { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__18; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); +x_1 = lean_unsigned_to_nat(2u); +x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__20() { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__4() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_instToJsonBool___boxed), 1, 0); +x_1 = lean_mk_string_from_bytes("tag", 3); return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__21() { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__17; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__19; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15; -x_4 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__20; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414____rarg), 5, 4); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_2); -lean_closure_set(x_5, 2, x_3); -lean_closure_set(x_5, 3, x_4); -return x_5; +switch (lean_obj_tag(x_1)) { +case 0: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +lean_dec(x_1); +x_3 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__1; +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_box(0); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_6); +x_8 = l_Lean_Json_mkObj(x_7); +return x_8; } +case 1: +{ +lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_9 = lean_ctor_get(x_1, 0); +lean_inc(x_9); +lean_dec(x_1); +x_10 = lean_array_get_size(x_9); +x_11 = lean_usize_of_nat(x_10); +lean_dec(x_10); +x_12 = 0; +x_13 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__4(x_11, x_12, x_9); +x_14 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__2; +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean_Json_mkObj(x_18); +return x_19; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__22() { -_start: +default: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__21; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_dec(x_1); +x_22 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320_(x_20); +x_23 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3(x_21); +x_24 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__3; +x_25 = lean_array_push(x_24, x_22); +x_26 = lean_array_push(x_25, x_23); +x_27 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_27, 0, x_26); +x_28 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__4; +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +x_30 = lean_box(0); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_Json_mkObj(x_31); +return x_32; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_instToJsonString), 1, 0); -return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__24() { +static lean_object* _init_l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonMVarId), 1, 0); +x_1 = lean_mk_string_from_bytes("Cannot parse request params: ", 29); return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__25() { +static lean_object* _init_l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__22; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23; -x_4 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__24; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237____rarg), 5, 4); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_2); -lean_closure_set(x_5, 2, x_3); -lean_closure_set(x_5, 3, x_4); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("\n", 1); +return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__26() { +static lean_object* _init_l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_instToJsonNat), 1, 0); +x_1 = lean_mk_string_from_bytes("", 0); return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__27() { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__25; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__26; -x_4 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__16; -x_5 = l_Lean_Lsp_instToJsonRpcRef; -x_6 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg), 6, 5); -lean_closure_set(x_6, 0, x_1); -lean_closure_set(x_6, 1, x_2); -lean_closure_set(x_6, 2, x_3); -lean_closure_set(x_6, 3, x_4); -lean_closure_set(x_6, 4, x_5); -return x_6; +lean_object* x_2; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60_(x_1); +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; +x_4 = lean_ctor_get(x_2, 0); +x_5 = l_Lean_Json_compress(x_1); +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +x_7 = lean_string_append(x_6, x_5); +lean_dec(x_5); +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; +x_9 = lean_string_append(x_7, x_8); +x_10 = lean_string_append(x_9, x_4); +lean_dec(x_4); +x_11 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_12 = lean_string_append(x_10, x_11); +x_13 = 0; +x_14 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set_uint8(x_14, sizeof(void*)*1, x_13); +lean_ctor_set(x_2, 0, x_14); +return x_2; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = l_Lean_Json_compress(x_1); +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +x_18 = lean_string_append(x_17, x_16); +lean_dec(x_16); +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; +x_20 = lean_string_append(x_18, x_19); +x_21 = lean_string_append(x_20, x_15); +lean_dec(x_15); +x_22 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_23 = lean_string_append(x_21, x_22); +x_24 = 0; +x_25 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set_uint8(x_25, sizeof(void*)*1, x_24); +x_26 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_26, 0, x_25); +return x_26; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__28() { -_start: +else +{ +uint8_t x_27; +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_2); +if (x_27 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__27; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); return x_2; } -} -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__4; -x_4 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__5; -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__13; -x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__28; -x_7 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___boxed), 14, 10); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, lean_box(0)); -lean_closure_set(x_7, 2, lean_box(0)); -lean_closure_set(x_7, 3, lean_box(0)); -lean_closure_set(x_7, 4, x_3); -lean_closure_set(x_7, 5, x_4); -lean_closure_set(x_7, 6, lean_box(0)); -lean_closure_set(x_7, 7, x_5); -lean_closure_set(x_7, 8, x_6); -lean_closure_set(x_7, 9, x_2); -return x_7; +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_2, 0); +lean_inc(x_28); +lean_dec(x_2); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; } } -static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Server_builtinRpcProcedures; -return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -lean_inc(x_1); -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2(x_1, x_2); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; -x_7 = lean_st_ref_take(x_6, x_4); -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_8, x_1, x_5); -x_11 = lean_st_ref_set(x_6, x_10, x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +if (lean_obj_tag(x_1) == 0) { -return x_11; +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +return x_5; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -return x_15; +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; } } } -static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__9(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("", 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2() { -_start: +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_3, x_2); +if (x_6 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(": already registered", 20); -return x_1; -} +lean_object* x_7; lean_object* x_8; +lean_dec(x_1); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_5); +return x_8; } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -lean_dec(x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; -x_7 = lean_st_ref_get(x_6, x_5); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) +else { -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_7, 1); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_array_uget(x_4, x_3); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_array_uset(x_4, x_3, x_10); lean_inc(x_1); -x_11 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_9, x_1); -if (x_11 == 0) +x_12 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_1, x_9, x_5); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_12; lean_object* x_13; -lean_free_object(x_7); -lean_dec(x_3); -x_12 = lean_box(0); -x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1(x_1, x_2, x_12, x_10); -return x_13; +uint8_t x_14; +lean_dec(x_11); +lean_dec(x_1); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) +{ +lean_object* x_15; uint8_t x_16; +x_15 = lean_ctor_get(x_12, 0); +lean_dec(x_15); +x_16 = !lean_is_exclusive(x_13); +if (x_16 == 0) +{ +return x_12; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -lean_dec(x_2); -lean_dec(x_1); -x_14 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_15 = lean_string_append(x_14, x_3); -lean_dec(x_3); -x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -x_17 = lean_string_append(x_15, x_16); -x_18 = lean_alloc_ctor(18, 1, 0); +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_13, 0); +lean_inc(x_17); +lean_dec(x_13); +x_18 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_18, 0, x_17); -lean_ctor_set_tag(x_7, 1); -lean_ctor_set(x_7, 0, x_18); -return x_7; +lean_ctor_set(x_12, 0, x_18); +return x_12; } } else { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_7, 0); -x_20 = lean_ctor_get(x_7, 1); -lean_inc(x_20); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_12, 1); lean_inc(x_19); -lean_dec(x_7); -lean_inc(x_1); -x_21 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_19, x_1); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -lean_dec(x_3); -x_22 = lean_box(0); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1(x_1, x_2, x_22, x_20); +lean_dec(x_12); +x_20 = lean_ctor_get(x_13, 0); +lean_inc(x_20); +if (lean_is_exclusive(x_13)) { + lean_ctor_release(x_13, 0); + x_21 = x_13; +} else { + lean_dec_ref(x_13); + x_21 = lean_box(0); +} +if (lean_is_scalar(x_21)) { + x_22 = lean_alloc_ctor(0, 1, 0); +} else { + x_22 = x_21; +} +lean_ctor_set(x_22, 0, x_20); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_19); return x_23; } +} else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_2); -lean_dec(x_1); -x_24 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_25 = lean_string_append(x_24, x_3); -lean_dec(x_3); -x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -x_27 = lean_string_append(x_25, x_26); -x_28 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_20); -return x_29; +lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; +x_24 = lean_ctor_get(x_12, 1); +lean_inc(x_24); +lean_dec(x_12); +x_25 = lean_ctor_get(x_13, 0); +lean_inc(x_25); +lean_dec(x_13); +x_26 = 1; +x_27 = lean_usize_add(x_3, x_26); +x_28 = lean_array_uset(x_11, x_3, x_25); +x_3 = x_27; +x_4 = x_28; +x_5 = x_24; +goto _start; } } } } -static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Failed to register builtin RPC call handler for '", 49); -return x_1; -} -} -static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2() { -_start: +switch (lean_obj_tag(x_2)) { +case 0: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("'", 1); -return x_1; -} +uint8_t x_4; +lean_dec(x_1); +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_2); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_5); +lean_ctor_set(x_6, 1, x_3); +return x_6; } -static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(": only possible during initialization", 37); -return x_1; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_3); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +case 1: { -uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_4 = 1; -lean_inc(x_1); -x_5 = l_Lean_Name_toString(x_1, x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1; -x_7 = lean_string_append(x_6, x_5); -lean_dec(x_5); -x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2; -x_9 = lean_string_append(x_7, x_8); -x_10 = lean_io_initializing(x_3); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_unbox(x_11); -lean_dec(x_11); -if (x_12 == 0) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_2); +if (x_11 == 0) { -uint8_t x_13; -lean_dec(x_2); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_10); -if (x_13 == 0) +lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; +x_12 = lean_ctor_get(x_2, 0); +x_13 = lean_array_get_size(x_12); +x_14 = lean_usize_of_nat(x_13); +lean_dec(x_13); +x_15 = 0; +x_16 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__9(x_1, x_14, x_15, x_12, x_3); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_ctor_get(x_10, 0); -lean_dec(x_14); -x_15 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_16 = lean_string_append(x_15, x_9); -lean_dec(x_9); -x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -x_18 = lean_string_append(x_16, x_17); -x_19 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set_tag(x_10, 1); -lean_ctor_set(x_10, 0, x_19); -return x_10; +uint8_t x_18; +lean_free_object(x_2); +x_18 = !lean_is_exclusive(x_16); +if (x_18 == 0) +{ +lean_object* x_19; uint8_t x_20; +x_19 = lean_ctor_get(x_16, 0); +lean_dec(x_19); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +return x_16; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_20 = lean_ctor_get(x_10, 1); -lean_inc(x_20); -lean_dec(x_10); -x_21 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_22 = lean_string_append(x_21, x_9); -lean_dec(x_9); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -x_24 = lean_string_append(x_22, x_23); -x_25 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_20); -return x_26; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_17, 0); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_16, 0, x_22); +return x_16; } } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_10, 1); -lean_inc(x_27); -lean_dec(x_10); -x_28 = lean_box(0); -x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); -return x_29; +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); +lean_dec(x_16); +x_24 = lean_ctor_get(x_17, 0); +lean_inc(x_24); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + x_25 = x_17; +} else { + lean_dec_ref(x_17); + x_25 = lean_box(0); +} +if (lean_is_scalar(x_25)) { + x_26 = lean_alloc_ctor(0, 1, 0); +} else { + x_26 = x_25; } +lean_ctor_set(x_26, 0, x_24); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_23); +return x_27; } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -uint8_t x_5; lean_object* x_6; -x_5 = 1; -x_6 = l_Lean_Widget_msgToInteractive(x_1, x_5, x_2, x_4); -if (lean_obj_tag(x_6) == 0) +uint8_t x_28; +x_28 = !lean_is_exclusive(x_16); +if (x_28 == 0) { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +lean_object* x_29; uint8_t x_30; +x_29 = lean_ctor_get(x_16, 0); +lean_dec(x_29); +x_30 = !lean_is_exclusive(x_17); +if (x_30 == 0) { -return x_6; +lean_object* x_31; +x_31 = lean_ctor_get(x_17, 0); +lean_ctor_set(x_2, 0, x_31); +lean_ctor_set(x_17, 0, x_2); +return x_16; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_inc(x_8); -lean_dec(x_6); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -return x_10; +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_17, 0); +lean_inc(x_32); +lean_dec(x_17); +lean_ctor_set(x_2, 0, x_32); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_2); +lean_ctor_set(x_16, 0, x_33); +return x_16; } } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_6); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_6, 0); -x_13 = lean_io_error_to_string(x_12); -x_14 = 4; -x_15 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set_uint8(x_15, sizeof(void*)*1, x_14); -lean_ctor_set(x_6, 0, x_15); -return x_6; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_34 = lean_ctor_get(x_16, 1); +lean_inc(x_34); +lean_dec(x_16); +x_35 = lean_ctor_get(x_17, 0); +lean_inc(x_35); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + x_36 = x_17; +} else { + lean_dec_ref(x_17); + x_36 = lean_box(0); } -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; -x_16 = lean_ctor_get(x_6, 0); -x_17 = lean_ctor_get(x_6, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_6); -x_18 = lean_io_error_to_string(x_16); -x_19 = 4; -x_20 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set_uint8(x_20, sizeof(void*)*1, x_19); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_17); -return x_21; +lean_ctor_set(x_2, 0, x_35); +if (lean_is_scalar(x_36)) { + x_37 = lean_alloc_ctor(1, 1, 0); +} else { + x_37 = x_36; } +lean_ctor_set(x_37, 0, x_2); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_34); +return x_38; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_1, 1); -lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_alloc_closure((void*)(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____lambda__1___boxed), 4, 2); -lean_closure_set(x_6, 0, x_4); -lean_closure_set(x_6, 1, x_5); -x_7 = l_Lean_Server_RequestM_asTask___rarg(x_6, x_2, x_3); -return x_7; +lean_object* x_39; lean_object* x_40; size_t x_41; size_t x_42; lean_object* x_43; lean_object* x_44; +x_39 = lean_ctor_get(x_2, 0); +lean_inc(x_39); +lean_dec(x_2); +x_40 = lean_array_get_size(x_39); +x_41 = lean_usize_of_nat(x_40); +lean_dec(x_40); +x_42 = 0; +x_43 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__9(x_1, x_41, x_42, x_39, x_3); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +if (lean_obj_tag(x_44) == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + x_46 = x_43; +} else { + lean_dec_ref(x_43); + x_46 = lean_box(0); +} +x_47 = lean_ctor_get(x_44, 0); +lean_inc(x_47); +if (lean_is_exclusive(x_44)) { + lean_ctor_release(x_44, 0); + x_48 = x_44; +} else { + lean_dec_ref(x_44); + x_48 = lean_box(0); } +if (lean_is_scalar(x_48)) { + x_49 = lean_alloc_ctor(0, 1, 0); +} else { + x_49 = x_48; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean", 4); -return x_1; +lean_ctor_set(x_49, 0, x_47); +if (lean_is_scalar(x_46)) { + x_50 = lean_alloc_ctor(0, 2, 0); +} else { + x_50 = x_46; } +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_45); +return x_50; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_51 = lean_ctor_get(x_43, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + x_52 = x_43; +} else { + lean_dec_ref(x_43); + x_52 = lean_box(0); +} +x_53 = lean_ctor_get(x_44, 0); +lean_inc(x_53); +if (lean_is_exclusive(x_44)) { + lean_ctor_release(x_44, 0); + x_54 = x_44; +} else { + lean_dec_ref(x_44); + x_54 = lean_box(0); } +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_53); +if (lean_is_scalar(x_54)) { + x_56 = lean_alloc_ctor(1, 1, 0); +} else { + x_56 = x_54; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Widget", 6); -return x_1; +lean_ctor_set(x_56, 0, x_55); +if (lean_is_scalar(x_52)) { + x_57 = lean_alloc_ctor(0, 2, 0); +} else { + x_57 = x_52; } +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_51); +return x_57; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__2; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__3; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__5() { -_start: +default: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("InteractiveDiagnostics", 22); -return x_1; -} +uint8_t x_58; +x_58 = !lean_is_exclusive(x_2); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_59 = lean_ctor_get(x_2, 0); +x_60 = lean_ctor_get(x_2, 1); +lean_inc(x_1); +x_61 = lean_apply_2(x_1, x_59, x_3); +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +if (lean_obj_tag(x_62) == 0) +{ +uint8_t x_63; +lean_free_object(x_2); +lean_dec(x_60); +lean_dec(x_1); +x_63 = !lean_is_exclusive(x_61); +if (x_63 == 0) +{ +lean_object* x_64; uint8_t x_65; +x_64 = lean_ctor_get(x_61, 0); +lean_dec(x_64); +x_65 = !lean_is_exclusive(x_62); +if (x_65 == 0) +{ +return x_61; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__6() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__5; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_66; lean_object* x_67; +x_66 = lean_ctor_get(x_62, 0); +lean_inc(x_66); +lean_dec(x_62); +x_67 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_61, 0, x_67); +return x_61; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__7() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("msgToInteractive", 16); -return x_1; +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_68 = lean_ctor_get(x_61, 1); +lean_inc(x_68); +lean_dec(x_61); +x_69 = lean_ctor_get(x_62, 0); +lean_inc(x_69); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + x_70 = x_62; +} else { + lean_dec_ref(x_62); + x_70 = lean_box(0); } +if (lean_is_scalar(x_70)) { + x_71 = lean_alloc_ctor(0, 1, 0); +} else { + x_71 = x_70; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__6; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__7; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_ctor_set(x_71, 0, x_69); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_68); +return x_72; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__9() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____lambda__2), 3, 0); -return x_1; -} +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_73 = lean_ctor_get(x_61, 1); +lean_inc(x_73); +lean_dec(x_61); +x_74 = lean_ctor_get(x_62, 0); +lean_inc(x_74); +lean_dec(x_62); +x_75 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_1, x_60, x_73); +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +if (lean_obj_tag(x_76) == 0) +{ +uint8_t x_77; +lean_dec(x_74); +lean_free_object(x_2); +x_77 = !lean_is_exclusive(x_75); +if (x_77 == 0) +{ +lean_object* x_78; uint8_t x_79; +x_78 = lean_ctor_get(x_75, 0); +lean_dec(x_78); +x_79 = !lean_is_exclusive(x_76); +if (x_79 == 0) +{ +return x_75; } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411_(lean_object* x_1) { -_start: +else { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__8; -x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__9; -x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1(x_2, x_3, x_1); -return x_4; +lean_object* x_80; lean_object* x_81; +x_80 = lean_ctor_get(x_76, 0); +lean_inc(x_80); +lean_dec(x_76); +x_81 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_75, 0, x_81); +return x_75; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -lean_object* x_5; -x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_82 = lean_ctor_get(x_75, 1); +lean_inc(x_82); +lean_dec(x_75); +x_83 = lean_ctor_get(x_76, 0); +lean_inc(x_83); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + x_84 = x_76; +} else { + lean_dec_ref(x_76); + x_84 = lean_box(0); } +if (lean_is_scalar(x_84)) { + x_85 = lean_alloc_ctor(0, 1, 0); +} else { + x_85 = x_84; } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____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_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_ctor_set(x_85, 0, x_83); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_82); +return x_86; } } -static lean_object* _init_l_Lean_Widget_instInhabitedInfoPopup___closed__1() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -lean_ctor_set(x_2, 2, x_1); -return x_2; -} +uint8_t x_87; +x_87 = !lean_is_exclusive(x_75); +if (x_87 == 0) +{ +lean_object* x_88; uint8_t x_89; +x_88 = lean_ctor_get(x_75, 0); +lean_dec(x_88); +x_89 = !lean_is_exclusive(x_76); +if (x_89 == 0) +{ +lean_object* x_90; +x_90 = lean_ctor_get(x_76, 0); +lean_ctor_set(x_2, 1, x_90); +lean_ctor_set(x_2, 0, x_74); +lean_ctor_set(x_76, 0, x_2); +return x_75; } -static lean_object* _init_l_Lean_Widget_instInhabitedInfoPopup() { -_start: +else { -lean_object* x_1; -x_1 = l_Lean_Widget_instInhabitedInfoPopup___closed__1; -return x_1; +lean_object* x_91; lean_object* x_92; +x_91 = lean_ctor_get(x_76, 0); +lean_inc(x_91); +lean_dec(x_76); +lean_ctor_set(x_2, 1, x_91); +lean_ctor_set(x_2, 0, x_74); +x_92 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_92, 0, x_2); +lean_ctor_set(x_75, 0, x_92); +return x_75; } } -static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("type", 4); -return x_1; +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_93 = lean_ctor_get(x_75, 1); +lean_inc(x_93); +lean_dec(x_75); +x_94 = lean_ctor_get(x_76, 0); +lean_inc(x_94); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + x_95 = x_76; +} else { + lean_dec_ref(x_76); + x_95 = lean_box(0); } +lean_ctor_set(x_2, 1, x_94); +lean_ctor_set(x_2, 0, x_74); +if (lean_is_scalar(x_95)) { + x_96 = lean_alloc_ctor(1, 1, 0); +} else { + x_96 = x_95; } -static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("exprExplicit", 12); -return x_1; +lean_ctor_set(x_96, 0, x_2); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_93); +return x_97; } } -static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("doc", 3); -return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; lean_object* x_5; -x_4 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__1; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_98 = lean_ctor_get(x_2, 0); +x_99 = lean_ctor_get(x_2, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_2); lean_inc(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_1, x_4); -if (lean_obj_tag(x_5) == 0) +x_100 = lean_apply_2(x_1, x_98, x_3); +x_101 = lean_ctor_get(x_100, 0); +lean_inc(x_101); +if (lean_obj_tag(x_101) == 0) { -uint8_t x_6; -lean_dec(x_2); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +lean_dec(x_99); lean_dec(x_1); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) -{ -return x_5; +x_102 = lean_ctor_get(x_100, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + x_103 = x_100; +} else { + lean_dec_ref(x_100); + x_103 = lean_box(0); +} +x_104 = lean_ctor_get(x_101, 0); +lean_inc(x_104); +if (lean_is_exclusive(x_101)) { + lean_ctor_release(x_101, 0); + x_105 = x_101; +} else { + lean_dec_ref(x_101); + x_105 = lean_box(0); } -else -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; +if (lean_is_scalar(x_105)) { + x_106 = lean_alloc_ctor(0, 1, 0); +} else { + x_106 = x_105; } +lean_ctor_set(x_106, 0, x_104); +if (lean_is_scalar(x_103)) { + x_107 = lean_alloc_ctor(0, 2, 0); +} else { + x_107 = x_103; } -else -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -lean_dec(x_5); -x_10 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__2; -x_11 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_1, x_10); -if (lean_obj_tag(x_11) == 0) -{ -uint8_t x_12; -lean_dec(x_9); -lean_dec(x_2); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -return x_11; +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set(x_107, 1, x_102); +return x_107; } else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; -} +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_108 = lean_ctor_get(x_100, 1); +lean_inc(x_108); +lean_dec(x_100); +x_109 = lean_ctor_get(x_101, 0); +lean_inc(x_109); +lean_dec(x_101); +x_110 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_1, x_99, x_108); +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +if (lean_obj_tag(x_111) == 0) +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +lean_dec(x_109); +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_113 = x_110; +} else { + lean_dec_ref(x_110); + x_113 = lean_box(0); +} +x_114 = lean_ctor_get(x_111, 0); +lean_inc(x_114); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + x_115 = x_111; +} else { + lean_dec_ref(x_111); + x_115 = lean_box(0); } -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_11, 0); -lean_inc(x_15); -lean_dec(x_11); -x_16 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__3; -x_17 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_2, x_16); -if (lean_obj_tag(x_17) == 0) -{ -uint8_t x_18; -lean_dec(x_15); -lean_dec(x_9); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -return x_17; +if (lean_is_scalar(x_115)) { + x_116 = lean_alloc_ctor(0, 1, 0); +} else { + x_116 = x_115; } -else -{ -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_17, 0); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_20, 0, x_19); -return x_20; +lean_ctor_set(x_116, 0, x_114); +if (lean_is_scalar(x_113)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_113; } +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_112); +return x_117; } else { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_17); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_17, 0); -x_23 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_23, 0, x_9); -lean_ctor_set(x_23, 1, x_15); -lean_ctor_set(x_23, 2, x_22); -lean_ctor_set(x_17, 0, x_23); -return x_17; +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_118 = lean_ctor_get(x_110, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_119 = x_110; +} else { + lean_dec_ref(x_110); + x_119 = lean_box(0); +} +x_120 = lean_ctor_get(x_111, 0); +lean_inc(x_120); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + x_121 = x_111; +} else { + lean_dec_ref(x_111); + x_121 = lean_box(0); +} +x_122 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_122, 0, x_109); +lean_ctor_set(x_122, 1, x_120); +if (lean_is_scalar(x_121)) { + x_123 = lean_alloc_ctor(1, 1, 0); +} else { + x_123 = x_121; } -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_17, 0); -lean_inc(x_24); -lean_dec(x_17); -x_25 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_25, 0, x_9); -lean_ctor_set(x_25, 1, x_15); -lean_ctor_set(x_25, 2, x_24); -x_26 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_26, 0, x_25); -return x_26; +lean_ctor_set(x_123, 0, x_122); +if (lean_is_scalar(x_119)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_119; } +lean_ctor_set(x_124, 0, x_123); +lean_ctor_set(x_124, 1, x_118); +return x_124; } } } } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___boxed), 3, 0); -return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__10(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_4; -x_4 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__8___rarg(lean_object* x_1, lean_object* x_2) { -_start: +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_2, x_1); +if (x_5 == 0) { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___boxed), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} +lean_object* x_6; lean_object* x_7; +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__8(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__8___rarg), 2, 0); -return x_3; +lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_8 = lean_array_uget(x_3, x_2); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_array_uset(x_3, x_2, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_2, x_11); +x_13 = lean_array_uset(x_10, x_2, x_8); +x_2 = x_12; +x_3 = x_13; +goto _start; +} } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_689____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__11(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); -lean_inc(x_1); -x_5 = lean_apply_1(x_1, x_4); -x_6 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__1; +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_2, x_1); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); x_7 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_9, 0, x_7); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_ctor_get(x_3, 1); -lean_inc(x_10); -x_11 = lean_apply_1(x_1, x_10); -x_12 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__2; -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_8); -x_15 = lean_ctor_get(x_3, 2); -lean_inc(x_15); -lean_dec(x_3); -x_16 = lean_apply_1(x_2, x_15); -x_17 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__3; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_8); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_8); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_14); -lean_ctor_set(x_21, 1, x_20); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_9); -lean_ctor_set(x_22, 1, x_21); -x_23 = l_List_join___rarg(x_22); -x_24 = l_Lean_Json_mkObj(x_23); -return x_24; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_689_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_689____rarg), 3, 0); -return x_3; -} +lean_ctor_set(x_7, 1, x_4); +return x_7; } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__8___rarg(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_689____rarg), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} +lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_8 = lean_array_uget(x_3, x_2); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_array_uset(x_3, x_2, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_2, x_11); +x_13 = lean_array_uset(x_10, x_2, x_8); +x_2 = x_12; +x_3 = x_13; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__8(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__8___rarg), 2, 0); -return x_3; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { if (lean_obj_tag(x_5) == 0) { -uint8_t x_6; +uint8_t x_7; lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_1, 0); lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_apply_3(x_9, lean_box(0), x_5, x_6); +return x_10; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_5, 0); lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); +lean_dec(x_5); +x_12 = lean_ctor_get(x_1, 0); lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_14, 0, x_11); +x_15 = lean_apply_3(x_13, lean_box(0), x_14, x_6); +return x_15; } } else { -lean_object* x_15; lean_object* x_16; +lean_object* x_16; lean_object* x_17; lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; +x_17 = lean_apply_2(x_4, x_16, x_6); +return x_17; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__1___rarg), 5, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_3, 1); +lean_inc(x_8); +lean_dec(x_3); +x_9 = lean_apply_5(x_6, lean_box(0), x_1, x_2, x_7, x_4); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 0) { -if (lean_obj_tag(x_5) == 0) +uint8_t x_11; +lean_dec(x_8); +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) { -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +lean_object* x_12; uint8_t x_13; +x_12 = lean_ctor_get(x_9, 0); +lean_dec(x_12); +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); return x_9; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_10, 0); +lean_inc(x_14); +lean_dec(x_10); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_9, 0, x_15); +return x_9; } } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; -} +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_9, 1); +lean_inc(x_16); +lean_dec(x_9); +x_17 = lean_ctor_get(x_10, 0); +lean_inc(x_17); +if (lean_is_exclusive(x_10)) { + lean_ctor_release(x_10, 0); + x_18 = x_10; +} else { + lean_dec_ref(x_10); + x_18 = lean_box(0); } +if (lean_is_scalar(x_18)) { + x_19 = lean_alloc_ctor(0, 1, 0); +} else { + x_19 = x_18; } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__2___rarg), 5, 0); -return x_2; +lean_ctor_set(x_19, 0, x_17); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_16); +return x_20; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -if (lean_obj_tag(x_5) == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_9); +if (x_21 == 0) { -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_9, 0); +lean_dec(x_22); +x_23 = !lean_is_exclusive(x_10); +if (x_23 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_10, 0); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_8); +lean_ctor_set(x_10, 0, x_25); return x_9; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_10, 0); +lean_inc(x_26); +lean_dec(x_10); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_8); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_9, 0, x_28); +return x_9; } } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_29 = lean_ctor_get(x_9, 1); +lean_inc(x_29); +lean_dec(x_9); +x_30 = lean_ctor_get(x_10, 0); +lean_inc(x_30); +if (lean_is_exclusive(x_10)) { + lean_ctor_release(x_10, 0); + x_31 = x_10; +} else { + lean_dec_ref(x_10); + x_31 = lean_box(0); +} +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_8); +if (lean_is_scalar(x_31)) { + x_33 = lean_alloc_ctor(1, 1, 0); +} else { + x_33 = x_31; } +lean_ctor_set(x_33, 0, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_29); +return x_34; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__3(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__3___rarg), 5, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; uint8_t x_10; lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_ctor_get(x_5, 1); +x_6 = lean_ctor_get(x_1, 1); lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_7, 0, x_2); -lean_ctor_set(x_7, 1, x_3); -lean_ctor_set(x_7, 2, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_ctor_get(x_1, 0); +x_7 = lean_ctor_get(x_1, 2); +lean_inc(x_7); +x_8 = lean_ctor_get(x_1, 3); lean_inc(x_8); +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_10 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); lean_dec(x_1); -x_9 = lean_ctor_get(x_2, 2); -lean_inc(x_9); -lean_dec(x_2); -lean_inc(x_3); -x_10 = lean_apply_4(x_8, lean_box(0), x_3, x_4, x_9); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__1), 4, 3); -lean_closure_set(x_11, 0, x_3); -lean_closure_set(x_11, 1, x_5); -lean_closure_set(x_11, 2, x_7); -x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); -lean_inc(x_4); -lean_inc(x_3); -x_9 = lean_apply_4(x_2, lean_box(0), x_3, x_4, x_8); -lean_inc(x_6); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__2), 7, 6); -lean_closure_set(x_10, 0, x_5); -lean_closure_set(x_10, 1, x_1); -lean_closure_set(x_10, 2, x_3); -lean_closure_set(x_10, 3, x_4); -lean_closure_set(x_10, 4, x_7); -lean_closure_set(x_10, 5, x_6); -x_11 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_9, x_10); +x_11 = lean_array_get_size(x_5); +x_12 = lean_usize_of_nat(x_11); +lean_dec(x_11); +x_13 = 0; +x_14 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__10(x_12, x_13, x_5, x_4); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_array_get_size(x_6); +x_19 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_20 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__11(x_19, x_13, x_6, x_16); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__1), 4, 2); +lean_closure_set(x_24, 0, x_2); +lean_closure_set(x_24, 1, x_3); +lean_inc(x_24); +x_25 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_24, x_7, x_22); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +if (lean_obj_tag(x_26) == 0) +{ +uint8_t x_27; +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_17); +lean_dec(x_8); +x_27 = !lean_is_exclusive(x_25); +if (x_27 == 0) +{ +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_25, 0); +lean_dec(x_28); +x_29 = !lean_is_exclusive(x_26); +if (x_29 == 0) +{ +return x_25; +} +else +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_26, 0); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_25, 0, x_31); +return x_25; +} +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_32 = lean_ctor_get(x_25, 1); +lean_inc(x_32); +lean_dec(x_25); +x_33 = lean_ctor_get(x_26, 0); +lean_inc(x_33); +if (lean_is_exclusive(x_26)) { + lean_ctor_release(x_26, 0); + x_34 = x_26; +} else { + lean_dec_ref(x_26); + x_34 = lean_box(0); +} +if (lean_is_scalar(x_34)) { + x_35 = lean_alloc_ctor(0, 1, 0); +} else { + x_35 = x_34; +} +lean_ctor_set(x_35, 0, x_33); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_32); +return x_36; +} +} +else +{ +if (lean_obj_tag(x_8) == 0) +{ +uint8_t x_37; +lean_dec(x_24); +x_37 = !lean_is_exclusive(x_25); +if (x_37 == 0) +{ +lean_object* x_38; uint8_t x_39; +x_38 = lean_ctor_get(x_25, 0); +lean_dec(x_38); +x_39 = !lean_is_exclusive(x_26); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_26, 0); +x_41 = lean_box(0); +x_42 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_42, 0, x_17); +lean_ctor_set(x_42, 1, x_23); +lean_ctor_set(x_42, 2, x_40); +lean_ctor_set(x_42, 3, x_41); +lean_ctor_set_uint8(x_42, sizeof(void*)*4, x_9); +lean_ctor_set_uint8(x_42, sizeof(void*)*4 + 1, x_10); +lean_ctor_set(x_26, 0, x_42); +return x_25; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_43 = lean_ctor_get(x_26, 0); +lean_inc(x_43); +lean_dec(x_26); +x_44 = lean_box(0); +x_45 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_45, 0, x_17); +lean_ctor_set(x_45, 1, x_23); +lean_ctor_set(x_45, 2, x_43); +lean_ctor_set(x_45, 3, x_44); +lean_ctor_set_uint8(x_45, sizeof(void*)*4, x_9); +lean_ctor_set_uint8(x_45, sizeof(void*)*4 + 1, x_10); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_25, 0, x_46); +return x_25; +} +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_47 = lean_ctor_get(x_25, 1); +lean_inc(x_47); +lean_dec(x_25); +x_48 = lean_ctor_get(x_26, 0); +lean_inc(x_48); +if (lean_is_exclusive(x_26)) { + lean_ctor_release(x_26, 0); + x_49 = x_26; +} else { + lean_dec_ref(x_26); + x_49 = lean_box(0); +} +x_50 = lean_box(0); +x_51 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_51, 0, x_17); +lean_ctor_set(x_51, 1, x_23); +lean_ctor_set(x_51, 2, x_48); +lean_ctor_set(x_51, 3, x_50); +lean_ctor_set_uint8(x_51, sizeof(void*)*4, x_9); +lean_ctor_set_uint8(x_51, sizeof(void*)*4 + 1, x_10); +if (lean_is_scalar(x_49)) { + x_52 = lean_alloc_ctor(1, 1, 0); +} else { + x_52 = x_49; +} +lean_ctor_set(x_52, 0, x_51); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_47); +return x_53; +} +} +else +{ +lean_object* x_54; lean_object* x_55; uint8_t x_56; +x_54 = lean_ctor_get(x_25, 1); +lean_inc(x_54); +lean_dec(x_25); +x_55 = lean_ctor_get(x_26, 0); +lean_inc(x_55); +lean_dec(x_26); +x_56 = !lean_is_exclusive(x_8); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_8, 0); +x_58 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_24, x_57, x_54); +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +if (lean_obj_tag(x_59) == 0) +{ +uint8_t x_60; +lean_free_object(x_8); +lean_dec(x_55); +lean_dec(x_23); +lean_dec(x_17); +x_60 = !lean_is_exclusive(x_58); +if (x_60 == 0) +{ +lean_object* x_61; uint8_t x_62; +x_61 = lean_ctor_get(x_58, 0); +lean_dec(x_61); +x_62 = !lean_is_exclusive(x_59); +if (x_62 == 0) +{ +return x_58; +} +else +{ +lean_object* x_63; lean_object* x_64; +x_63 = lean_ctor_get(x_59, 0); +lean_inc(x_63); +lean_dec(x_59); +x_64 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_58, 0, x_64); +return x_58; +} +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_65 = lean_ctor_get(x_58, 1); +lean_inc(x_65); +lean_dec(x_58); +x_66 = lean_ctor_get(x_59, 0); +lean_inc(x_66); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + x_67 = x_59; +} else { + lean_dec_ref(x_59); + x_67 = lean_box(0); +} +if (lean_is_scalar(x_67)) { + x_68 = lean_alloc_ctor(0, 1, 0); +} else { + x_68 = x_67; +} +lean_ctor_set(x_68, 0, x_66); +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_65); +return x_69; +} +} +else +{ +uint8_t x_70; +x_70 = !lean_is_exclusive(x_58); +if (x_70 == 0) +{ +lean_object* x_71; uint8_t x_72; +x_71 = lean_ctor_get(x_58, 0); +lean_dec(x_71); +x_72 = !lean_is_exclusive(x_59); +if (x_72 == 0) +{ +lean_object* x_73; lean_object* x_74; +x_73 = lean_ctor_get(x_59, 0); +lean_ctor_set(x_8, 0, x_73); +x_74 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_74, 0, x_17); +lean_ctor_set(x_74, 1, x_23); +lean_ctor_set(x_74, 2, x_55); +lean_ctor_set(x_74, 3, x_8); +lean_ctor_set_uint8(x_74, sizeof(void*)*4, x_9); +lean_ctor_set_uint8(x_74, sizeof(void*)*4 + 1, x_10); +lean_ctor_set(x_59, 0, x_74); +return x_58; +} +else +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_59, 0); +lean_inc(x_75); +lean_dec(x_59); +lean_ctor_set(x_8, 0, x_75); +x_76 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_76, 0, x_17); +lean_ctor_set(x_76, 1, x_23); +lean_ctor_set(x_76, 2, x_55); +lean_ctor_set(x_76, 3, x_8); +lean_ctor_set_uint8(x_76, sizeof(void*)*4, x_9); +lean_ctor_set_uint8(x_76, sizeof(void*)*4 + 1, x_10); +x_77 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_58, 0, x_77); +return x_58; +} +} +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_78 = lean_ctor_get(x_58, 1); +lean_inc(x_78); +lean_dec(x_58); +x_79 = lean_ctor_get(x_59, 0); +lean_inc(x_79); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + x_80 = x_59; +} else { + lean_dec_ref(x_59); + x_80 = lean_box(0); +} +lean_ctor_set(x_8, 0, x_79); +x_81 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_81, 0, x_17); +lean_ctor_set(x_81, 1, x_23); +lean_ctor_set(x_81, 2, x_55); +lean_ctor_set(x_81, 3, x_8); +lean_ctor_set_uint8(x_81, sizeof(void*)*4, x_9); +lean_ctor_set_uint8(x_81, sizeof(void*)*4 + 1, x_10); +if (lean_is_scalar(x_80)) { + x_82 = lean_alloc_ctor(1, 1, 0); +} else { + x_82 = x_80; +} +lean_ctor_set(x_82, 0, x_81); +x_83 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_83, 0, x_82); +lean_ctor_set(x_83, 1, x_78); +return x_83; +} +} +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_8, 0); +lean_inc(x_84); +lean_dec(x_8); +x_85 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_24, x_84, x_54); +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +if (lean_obj_tag(x_86) == 0) +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_dec(x_55); +lean_dec(x_23); +lean_dec(x_17); +x_87 = lean_ctor_get(x_85, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_88 = x_85; +} else { + lean_dec_ref(x_85); + x_88 = lean_box(0); +} +x_89 = lean_ctor_get(x_86, 0); +lean_inc(x_89); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + x_90 = x_86; +} else { + lean_dec_ref(x_86); + x_90 = lean_box(0); +} +if (lean_is_scalar(x_90)) { + x_91 = lean_alloc_ctor(0, 1, 0); +} else { + x_91 = x_90; +} +lean_ctor_set(x_91, 0, x_89); +if (lean_is_scalar(x_88)) { + x_92 = lean_alloc_ctor(0, 2, 0); +} else { + x_92 = x_88; +} +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_87); +return x_92; +} +else +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_93 = lean_ctor_get(x_85, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_94 = x_85; +} else { + lean_dec_ref(x_85); + x_94 = lean_box(0); +} +x_95 = lean_ctor_get(x_86, 0); +lean_inc(x_95); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + x_96 = x_86; +} else { + lean_dec_ref(x_86); + x_96 = lean_box(0); +} +x_97 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_97, 0, x_95); +x_98 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_98, 0, x_17); +lean_ctor_set(x_98, 1, x_23); +lean_ctor_set(x_98, 2, x_55); +lean_ctor_set(x_98, 3, x_97); +lean_ctor_set_uint8(x_98, sizeof(void*)*4, x_9); +lean_ctor_set_uint8(x_98, sizeof(void*)*4 + 1, x_10); +if (lean_is_scalar(x_96)) { + x_99 = lean_alloc_ctor(1, 1, 0); +} else { + x_99 = x_96; +} +lean_ctor_set(x_99, 0, x_98); +if (lean_is_scalar(x_94)) { + x_100 = lean_alloc_ctor(0, 2, 0); +} else { + x_100 = x_94; +} +lean_ctor_set(x_100, 0, x_99); +lean_ctor_set(x_100, 1, x_93); +return x_100; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__3(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; +x_8 = 1; +x_9 = lean_usize_add(x_1, x_8); +x_10 = lean_array_uset(x_2, x_1, x_6); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12(x_3, x_4, x_5, x_9, x_10, x_7); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_7 = lean_ctor_get(x_4, 1); -lean_inc(x_7); +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_4, x_3); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_2); x_8 = lean_ctor_get(x_1, 0); lean_inc(x_8); lean_dec(x_1); -x_9 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_8, 1); lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_5); -lean_inc(x_4); -x_10 = lean_apply_4(x_8, lean_box(0), x_4, x_5, x_9); -lean_inc(x_7); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__3), 7, 6); -lean_closure_set(x_11, 0, x_6); -lean_closure_set(x_11, 1, x_8); -lean_closure_set(x_11, 2, x_4); -lean_closure_set(x_11, 3, x_5); -lean_closure_set(x_11, 4, x_2); -lean_closure_set(x_11, 5, x_7); -x_12 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_10, x_11); -return x_12; +lean_dec(x_8); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_5); +x_11 = lean_apply_3(x_9, lean_box(0), x_10, x_6); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_12 = lean_array_uget(x_5, x_4); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_array_uset(x_5, x_4, x_13); +lean_inc(x_2); +lean_inc(x_1); +x_15 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__2), 4, 3); +lean_closure_set(x_15, 0, x_12); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +x_16 = lean_box_usize(x_4); +x_17 = lean_box_usize(x_3); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__3___boxed), 7, 5); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_14); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__13), 6, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_5(x_19, lean_box(0), lean_box(0), x_15, x_20, x_6); +return x_21; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1() { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_5 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_4); -x_6 = lean_ctor_get(x_3, 0); -lean_inc(x_6); -lean_dec(x_3); -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_8, 0, x_5); -x_9 = lean_apply_2(x_7, lean_box(0), x_8); -return x_9; +lean_object* x_1; lean_object* x_2; +x_1 = l_Id_instMonadId; +x_2 = l_StateT_instMonadStateT___rarg(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__2() { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_2, 2); -lean_inc(x_8); -lean_dec(x_2); -lean_inc(x_3); -x_9 = lean_apply_4(x_7, lean_box(0), x_3, x_4, x_8); -lean_inc(x_3); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__5), 4, 3); -lean_closure_set(x_10, 0, x_5); -lean_closure_set(x_10, 1, x_6); -lean_closure_set(x_10, 2, x_3); -x_11 = lean_ctor_get(x_3, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_12, 0, x_3); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); -return x_13; +lean_object* x_1; lean_object* x_2; +x_1 = l_Id_instMonadId; +x_2 = l_instMonadStateOfStateT___rarg(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3() { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -lean_inc(x_4); -lean_inc(x_3); -x_8 = lean_apply_4(x_2, lean_box(0), x_3, x_4, x_7); -lean_inc(x_3); -x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__6), 6, 5); -lean_closure_set(x_9, 0, x_5); -lean_closure_set(x_9, 1, x_1); -lean_closure_set(x_9, 2, x_3); -lean_closure_set(x_9, 3, x_4); -lean_closure_set(x_9, 4, x_6); -x_10 = lean_ctor_get(x_3, 1); -lean_inc(x_10); -x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_11, 0, x_3); -lean_closure_set(x_11, 1, lean_box(0)); -lean_closure_set(x_11, 2, lean_box(0)); -lean_closure_set(x_11, 3, x_9); -x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); -return x_12; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__2; +x_3 = l_Lean_Server_FileWorker_instMonadRpcSession___rarg(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); +lean_object* x_3; lean_object* x_4; +switch (lean_obj_tag(x_1)) { +case 0: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_19 = lean_ctor_get(x_1, 0); +lean_inc(x_19); lean_dec(x_1); -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_5); -lean_inc(x_4); -x_9 = lean_apply_4(x_7, lean_box(0), x_4, x_5, x_8); -lean_inc(x_4); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__7), 6, 5); -lean_closure_set(x_10, 0, x_6); -lean_closure_set(x_10, 1, x_7); -lean_closure_set(x_10, 2, x_4); -lean_closure_set(x_10, 3, x_5); -lean_closure_set(x_10, 4, x_2); -x_11 = lean_ctor_get(x_4, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___spec__3___rarg), 5, 4); -lean_closure_set(x_12, 0, x_4); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); -return x_13; +x_20 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_21 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_22 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__1), 4, 2); +lean_closure_set(x_22, 0, x_20); +lean_closure_set(x_22, 1, x_21); +x_23 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_22, x_19, x_2); +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +if (lean_obj_tag(x_24) == 0) +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_23); +if (x_25 == 0) +{ +lean_object* x_26; uint8_t x_27; +x_26 = lean_ctor_get(x_23, 0); +lean_dec(x_26); +x_27 = !lean_is_exclusive(x_24); +if (x_27 == 0) +{ +return x_23; +} +else +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_24, 0); +lean_inc(x_28); +lean_dec(x_24); +x_29 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_23, 0, x_29); +return x_23; +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = lean_ctor_get(x_23, 1); +lean_inc(x_30); +lean_dec(x_23); +x_31 = lean_ctor_get(x_24, 0); +lean_inc(x_31); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + x_32 = x_24; +} else { + lean_dec_ref(x_24); + x_32 = lean_box(0); +} +if (lean_is_scalar(x_32)) { + x_33 = lean_alloc_ctor(0, 1, 0); +} else { + x_33 = x_32; +} +lean_ctor_set(x_33, 0, x_31); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_30); +return x_34; +} +} +else +{ +uint8_t x_35; +x_35 = !lean_is_exclusive(x_23); +if (x_35 == 0) +{ +lean_object* x_36; uint8_t x_37; +x_36 = lean_ctor_get(x_23, 0); +lean_dec(x_36); +x_37 = !lean_is_exclusive(x_24); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_24, 0); +x_39 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_24, 0, x_39); +return x_23; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_24, 0); +lean_inc(x_40); +lean_dec(x_24); +x_41 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_41, 0, x_40); +x_42 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_23, 0, x_42); +return x_23; +} +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_43 = lean_ctor_get(x_23, 1); +lean_inc(x_43); +lean_dec(x_23); +x_44 = lean_ctor_get(x_24, 0); +lean_inc(x_44); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + x_45 = x_24; +} else { + lean_dec_ref(x_24); + x_45 = lean_box(0); +} +x_46 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_46, 0, x_44); +if (lean_is_scalar(x_45)) { + x_47 = lean_alloc_ctor(1, 1, 0); +} else { + x_47 = x_45; +} +lean_ctor_set(x_47, 0, x_46); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_43); +return x_48; +} +} +} +case 1: +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; size_t x_56; size_t x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_49 = lean_ctor_get(x_1, 0); +lean_inc(x_49); +lean_dec(x_1); +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +x_52 = lean_ctor_get(x_49, 2); +lean_inc(x_52); +x_53 = lean_ctor_get(x_49, 3); +lean_inc(x_53); +x_54 = lean_ctor_get(x_49, 4); +lean_inc(x_54); +lean_dec(x_49); +x_55 = lean_array_get_size(x_50); +x_56 = lean_usize_of_nat(x_55); +lean_dec(x_55); +x_57 = 0; +x_58 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_59 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_60 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12(x_58, x_59, x_56, x_57, x_50, x_2); +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +if (lean_obj_tag(x_61) == 0) +{ +lean_object* x_62; uint8_t x_63; +lean_dec(x_54); +lean_dec(x_53); +lean_dec(x_52); +lean_dec(x_51); +x_62 = lean_ctor_get(x_60, 1); +lean_inc(x_62); +lean_dec(x_60); +x_63 = !lean_is_exclusive(x_61); +if (x_63 == 0) +{ +x_3 = x_61; +x_4 = x_62; +goto block_18; +} +else +{ +lean_object* x_64; lean_object* x_65; +x_64 = lean_ctor_get(x_61, 0); +lean_inc(x_64); +lean_dec(x_61); +x_65 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_3 = x_65; +x_4 = x_62; +goto block_18; +} +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_66 = lean_ctor_get(x_60, 1); +lean_inc(x_66); +lean_dec(x_60); +x_67 = lean_ctor_get(x_61, 0); +lean_inc(x_67); +lean_dec(x_61); +x_68 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__1), 4, 2); +lean_closure_set(x_68, 0, x_58); +lean_closure_set(x_68, 1, x_59); +x_69 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_68, x_51, x_66); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +if (lean_obj_tag(x_70) == 0) +{ +lean_object* x_71; uint8_t x_72; +lean_dec(x_67); +lean_dec(x_54); +lean_dec(x_53); +lean_dec(x_52); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); +lean_dec(x_69); +x_72 = !lean_is_exclusive(x_70); +if (x_72 == 0) +{ +x_3 = x_70; +x_4 = x_71; +goto block_18; +} +else +{ +lean_object* x_73; lean_object* x_74; +x_73 = lean_ctor_get(x_70, 0); +lean_inc(x_73); +lean_dec(x_70); +x_74 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_74, 0, x_73); +x_3 = x_74; +x_4 = x_71; +goto block_18; +} +} +else +{ +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_75; uint8_t x_76; +x_75 = lean_ctor_get(x_69, 1); +lean_inc(x_75); +lean_dec(x_69); +x_76 = !lean_is_exclusive(x_70); +if (x_76 == 0) +{ +lean_object* x_77; lean_object* x_78; +x_77 = lean_ctor_get(x_70, 0); +x_78 = lean_box(0); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_79; +x_79 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_79, 0, x_67); +lean_ctor_set(x_79, 1, x_77); +lean_ctor_set(x_79, 2, x_78); +lean_ctor_set(x_79, 3, x_53); +lean_ctor_set(x_79, 4, x_78); +lean_ctor_set(x_70, 0, x_79); +x_3 = x_70; +x_4 = x_75; +goto block_18; +} +else +{ +uint8_t x_80; +x_80 = !lean_is_exclusive(x_54); +if (x_80 == 0) +{ +lean_object* x_81; +x_81 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_81, 0, x_67); +lean_ctor_set(x_81, 1, x_77); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set(x_81, 3, x_53); +lean_ctor_set(x_81, 4, x_54); +lean_ctor_set(x_70, 0, x_81); +x_3 = x_70; +x_4 = x_75; +goto block_18; +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_54, 0); +lean_inc(x_82); +lean_dec(x_54); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_82); +x_84 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_84, 0, x_67); +lean_ctor_set(x_84, 1, x_77); +lean_ctor_set(x_84, 2, x_78); +lean_ctor_set(x_84, 3, x_53); +lean_ctor_set(x_84, 4, x_83); +lean_ctor_set(x_70, 0, x_84); +x_3 = x_70; +x_4 = x_75; +goto block_18; +} +} +} +else +{ +lean_object* x_85; lean_object* x_86; +x_85 = lean_ctor_get(x_70, 0); +lean_inc(x_85); +lean_dec(x_70); +x_86 = lean_box(0); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_87; lean_object* x_88; +x_87 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_87, 0, x_67); +lean_ctor_set(x_87, 1, x_85); +lean_ctor_set(x_87, 2, x_86); +lean_ctor_set(x_87, 3, x_53); +lean_ctor_set(x_87, 4, x_86); +x_88 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_88, 0, x_87); +x_3 = x_88; +x_4 = x_75; +goto block_18; +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_89 = lean_ctor_get(x_54, 0); +lean_inc(x_89); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + x_90 = x_54; +} else { + lean_dec_ref(x_54); + x_90 = lean_box(0); +} +if (lean_is_scalar(x_90)) { + x_91 = lean_alloc_ctor(1, 1, 0); +} else { + x_91 = x_90; +} +lean_ctor_set(x_91, 0, x_89); +x_92 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_92, 0, x_67); +lean_ctor_set(x_92, 1, x_85); +lean_ctor_set(x_92, 2, x_86); +lean_ctor_set(x_92, 3, x_53); +lean_ctor_set(x_92, 4, x_91); +x_93 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_93, 0, x_92); +x_3 = x_93; +x_4 = x_75; +goto block_18; +} +} +} +else +{ +lean_object* x_94; uint8_t x_95; +x_94 = lean_ctor_get(x_69, 1); +lean_inc(x_94); +lean_dec(x_69); +x_95 = !lean_is_exclusive(x_70); +if (x_95 == 0) +{ +uint8_t x_96; +x_96 = !lean_is_exclusive(x_52); +if (x_96 == 0) +{ +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_70, 0); +x_98 = lean_box(0); +x_99 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_99, 0, x_67); +lean_ctor_set(x_99, 1, x_97); +lean_ctor_set(x_99, 2, x_52); +lean_ctor_set(x_99, 3, x_53); +lean_ctor_set(x_99, 4, x_98); +lean_ctor_set(x_70, 0, x_99); +x_3 = x_70; +x_4 = x_94; +goto block_18; +} +else +{ +uint8_t x_100; +x_100 = !lean_is_exclusive(x_54); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_70, 0); +x_102 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_102, 0, x_67); +lean_ctor_set(x_102, 1, x_101); +lean_ctor_set(x_102, 2, x_52); +lean_ctor_set(x_102, 3, x_53); +lean_ctor_set(x_102, 4, x_54); +lean_ctor_set(x_70, 0, x_102); +x_3 = x_70; +x_4 = x_94; +goto block_18; +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_103 = lean_ctor_get(x_70, 0); +x_104 = lean_ctor_get(x_54, 0); +lean_inc(x_104); +lean_dec(x_54); +x_105 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_105, 0, x_104); +x_106 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_106, 0, x_67); +lean_ctor_set(x_106, 1, x_103); +lean_ctor_set(x_106, 2, x_52); +lean_ctor_set(x_106, 3, x_53); +lean_ctor_set(x_106, 4, x_105); +lean_ctor_set(x_70, 0, x_106); +x_3 = x_70; +x_4 = x_94; +goto block_18; +} +} +} +else +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_70, 0); +x_108 = lean_ctor_get(x_52, 0); +lean_inc(x_108); +lean_dec(x_52); +x_109 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_109, 0, x_108); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_110; lean_object* x_111; +x_110 = lean_box(0); +x_111 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_111, 0, x_67); +lean_ctor_set(x_111, 1, x_107); +lean_ctor_set(x_111, 2, x_109); +lean_ctor_set(x_111, 3, x_53); +lean_ctor_set(x_111, 4, x_110); +lean_ctor_set(x_70, 0, x_111); +x_3 = x_70; +x_4 = x_94; +goto block_18; +} +else +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_112 = lean_ctor_get(x_54, 0); +lean_inc(x_112); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + x_113 = x_54; +} else { + lean_dec_ref(x_54); + x_113 = lean_box(0); +} +if (lean_is_scalar(x_113)) { + x_114 = lean_alloc_ctor(1, 1, 0); +} else { + x_114 = x_113; +} +lean_ctor_set(x_114, 0, x_112); +x_115 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_115, 0, x_67); +lean_ctor_set(x_115, 1, x_107); +lean_ctor_set(x_115, 2, x_109); +lean_ctor_set(x_115, 3, x_53); +lean_ctor_set(x_115, 4, x_114); +lean_ctor_set(x_70, 0, x_115); +x_3 = x_70; +x_4 = x_94; +goto block_18; +} +} +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_116 = lean_ctor_get(x_70, 0); +lean_inc(x_116); +lean_dec(x_70); +x_117 = lean_ctor_get(x_52, 0); +lean_inc(x_117); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + x_118 = x_52; +} else { + lean_dec_ref(x_52); + x_118 = lean_box(0); +} +if (lean_is_scalar(x_118)) { + x_119 = lean_alloc_ctor(1, 1, 0); +} else { + x_119 = x_118; +} +lean_ctor_set(x_119, 0, x_117); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_120 = lean_box(0); +x_121 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_121, 0, x_67); +lean_ctor_set(x_121, 1, x_116); +lean_ctor_set(x_121, 2, x_119); +lean_ctor_set(x_121, 3, x_53); +lean_ctor_set(x_121, 4, x_120); +x_122 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_122, 0, x_121); +x_3 = x_122; +x_4 = x_94; +goto block_18; +} +else +{ +lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_123 = lean_ctor_get(x_54, 0); +lean_inc(x_123); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + x_124 = x_54; +} else { + lean_dec_ref(x_54); + x_124 = lean_box(0); +} +if (lean_is_scalar(x_124)) { + x_125 = lean_alloc_ctor(1, 1, 0); +} else { + x_125 = x_124; +} +lean_ctor_set(x_125, 0, x_123); +x_126 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_126, 0, x_67); +lean_ctor_set(x_126, 1, x_116); +lean_ctor_set(x_126, 2, x_119); +lean_ctor_set(x_126, 3, x_53); +lean_ctor_set(x_126, 4, x_125); +x_127 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_127, 0, x_126); +x_3 = x_127; +x_4 = x_94; +goto block_18; +} +} +} +} +} +} +default: +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_128 = lean_ctor_get(x_1, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_1, 1); +lean_inc(x_129); +x_130 = lean_ctor_get(x_1, 2); +lean_inc(x_130); +lean_dec(x_1); +x_131 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; +x_132 = lean_ctor_get(x_131, 0); +lean_inc(x_132); +x_133 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_134 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_135 = lean_apply_5(x_132, lean_box(0), x_133, x_134, x_130, x_2); +x_136 = lean_ctor_get(x_135, 0); +lean_inc(x_136); +if (lean_obj_tag(x_136) == 0) +{ +uint8_t x_137; +lean_dec(x_129); +lean_dec(x_128); +x_137 = !lean_is_exclusive(x_135); +if (x_137 == 0) +{ +lean_object* x_138; uint8_t x_139; +x_138 = lean_ctor_get(x_135, 0); +lean_dec(x_138); +x_139 = !lean_is_exclusive(x_136); +if (x_139 == 0) +{ +return x_135; +} +else +{ +lean_object* x_140; lean_object* x_141; +x_140 = lean_ctor_get(x_136, 0); +lean_inc(x_140); +lean_dec(x_136); +x_141 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_141, 0, x_140); +lean_ctor_set(x_135, 0, x_141); +return x_135; +} +} +else +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_142 = lean_ctor_get(x_135, 1); +lean_inc(x_142); +lean_dec(x_135); +x_143 = lean_ctor_get(x_136, 0); +lean_inc(x_143); +if (lean_is_exclusive(x_136)) { + lean_ctor_release(x_136, 0); + x_144 = x_136; +} else { + lean_dec_ref(x_136); + x_144 = lean_box(0); +} +if (lean_is_scalar(x_144)) { + x_145 = lean_alloc_ctor(0, 1, 0); +} else { + x_145 = x_144; +} +lean_ctor_set(x_145, 0, x_143); +x_146 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_146, 0, x_145); +lean_ctor_set(x_146, 1, x_142); +return x_146; +} +} +else +{ +uint8_t x_147; +x_147 = !lean_is_exclusive(x_135); +if (x_147 == 0) +{ +lean_object* x_148; uint8_t x_149; +x_148 = lean_ctor_get(x_135, 0); +lean_dec(x_148); +x_149 = !lean_is_exclusive(x_136); +if (x_149 == 0) +{ +lean_object* x_150; lean_object* x_151; +x_150 = lean_ctor_get(x_136, 0); +x_151 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_151, 0, x_128); +lean_ctor_set(x_151, 1, x_129); +lean_ctor_set(x_151, 2, x_150); +lean_ctor_set(x_136, 0, x_151); +return x_135; +} +else +{ +lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_152 = lean_ctor_get(x_136, 0); +lean_inc(x_152); +lean_dec(x_136); +x_153 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_153, 0, x_128); +lean_ctor_set(x_153, 1, x_129); +lean_ctor_set(x_153, 2, x_152); +x_154 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_154, 0, x_153); +lean_ctor_set(x_135, 0, x_154); +return x_135; +} +} +else +{ +lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; +x_155 = lean_ctor_get(x_135, 1); +lean_inc(x_155); +lean_dec(x_135); +x_156 = lean_ctor_get(x_136, 0); +lean_inc(x_156); +if (lean_is_exclusive(x_136)) { + lean_ctor_release(x_136, 0); + x_157 = x_136; +} else { + lean_dec_ref(x_136); + x_157 = lean_box(0); +} +x_158 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_158, 0, x_128); +lean_ctor_set(x_158, 1, x_129); +lean_ctor_set(x_158, 2, x_156); +if (lean_is_scalar(x_157)) { + x_159 = lean_alloc_ctor(1, 1, 0); +} else { + x_159 = x_157; +} +lean_ctor_set(x_159, 0, x_158); +x_160 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_160, 0, x_159); +lean_ctor_set(x_160, 1, x_155); +return x_160; +} +} +} +} +block_18: +{ +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_5; +x_5 = !lean_is_exclusive(x_3); +if (x_5 == 0) +{ +lean_object* x_6; +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_4); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_4); +return x_9; +} +} +else +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_3); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_3, 0, x_12); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_3); +lean_ctor_set(x_13, 1, x_4); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_3, 0); +lean_inc(x_14); +lean_dec(x_3); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_4); +return x_17; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__15(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_3, x_2); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +lean_dec(x_1); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_5); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_array_uget(x_4, x_3); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_array_uset(x_4, x_3, x_10); +lean_inc(x_1); +x_12 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1, x_9, x_5); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +if (lean_obj_tag(x_13) == 0) +{ +uint8_t x_14; +lean_dec(x_11); +lean_dec(x_1); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) +{ +lean_object* x_15; uint8_t x_16; +x_15 = lean_ctor_get(x_12, 0); +lean_dec(x_15); +x_16 = !lean_is_exclusive(x_13); +if (x_16 == 0) +{ +return x_12; +} +else +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_13, 0); +lean_inc(x_17); +lean_dec(x_13); +x_18 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_12, 0, x_18); +return x_12; +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_12, 1); +lean_inc(x_19); +lean_dec(x_12); +x_20 = lean_ctor_get(x_13, 0); +lean_inc(x_20); +if (lean_is_exclusive(x_13)) { + lean_ctor_release(x_13, 0); + x_21 = x_13; +} else { + lean_dec_ref(x_13); + x_21 = lean_box(0); +} +if (lean_is_scalar(x_21)) { + x_22 = lean_alloc_ctor(0, 1, 0); +} else { + x_22 = x_21; +} +lean_ctor_set(x_22, 0, x_20); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_19); +return x_23; +} +} +else +{ +lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; lean_object* x_28; +x_24 = lean_ctor_get(x_12, 1); +lean_inc(x_24); +lean_dec(x_12); +x_25 = lean_ctor_get(x_13, 0); +lean_inc(x_25); +lean_dec(x_13); +x_26 = 1; +x_27 = lean_usize_add(x_3, x_26); +x_28 = lean_array_uset(x_11, x_3, x_25); +x_3 = x_27; +x_4 = x_28; +x_5 = x_24; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_2)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_1); +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_2); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_5); +lean_ctor_set(x_6, 1, x_3); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_3); +return x_10; +} +} +case 1: +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_2); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; +x_12 = lean_ctor_get(x_2, 0); +x_13 = lean_array_get_size(x_12); +x_14 = lean_usize_of_nat(x_13); +lean_dec(x_13); +x_15 = 0; +x_16 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__15(x_1, x_14, x_15, x_12, x_3); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +if (lean_obj_tag(x_17) == 0) +{ +uint8_t x_18; +lean_free_object(x_2); +x_18 = !lean_is_exclusive(x_16); +if (x_18 == 0) +{ +lean_object* x_19; uint8_t x_20; +x_19 = lean_ctor_get(x_16, 0); +lean_dec(x_19); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +return x_16; +} +else +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_17, 0); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_16, 0, x_22); +return x_16; +} +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); +lean_dec(x_16); +x_24 = lean_ctor_get(x_17, 0); +lean_inc(x_24); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + x_25 = x_17; +} else { + lean_dec_ref(x_17); + x_25 = lean_box(0); +} +if (lean_is_scalar(x_25)) { + x_26 = lean_alloc_ctor(0, 1, 0); +} else { + x_26 = x_25; +} +lean_ctor_set(x_26, 0, x_24); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_23); +return x_27; +} +} +else +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_16); +if (x_28 == 0) +{ +lean_object* x_29; uint8_t x_30; +x_29 = lean_ctor_get(x_16, 0); +lean_dec(x_29); +x_30 = !lean_is_exclusive(x_17); +if (x_30 == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_17, 0); +lean_ctor_set(x_2, 0, x_31); +lean_ctor_set(x_17, 0, x_2); +return x_16; +} +else +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_17, 0); +lean_inc(x_32); +lean_dec(x_17); +lean_ctor_set(x_2, 0, x_32); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_2); +lean_ctor_set(x_16, 0, x_33); +return x_16; +} +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_34 = lean_ctor_get(x_16, 1); +lean_inc(x_34); +lean_dec(x_16); +x_35 = lean_ctor_get(x_17, 0); +lean_inc(x_35); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + x_36 = x_17; +} else { + lean_dec_ref(x_17); + x_36 = lean_box(0); +} +lean_ctor_set(x_2, 0, x_35); +if (lean_is_scalar(x_36)) { + x_37 = lean_alloc_ctor(1, 1, 0); +} else { + x_37 = x_36; +} +lean_ctor_set(x_37, 0, x_2); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_34); +return x_38; +} +} +} +else +{ +lean_object* x_39; lean_object* x_40; size_t x_41; size_t x_42; lean_object* x_43; lean_object* x_44; +x_39 = lean_ctor_get(x_2, 0); +lean_inc(x_39); +lean_dec(x_2); +x_40 = lean_array_get_size(x_39); +x_41 = lean_usize_of_nat(x_40); +lean_dec(x_40); +x_42 = 0; +x_43 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__15(x_1, x_41, x_42, x_39, x_3); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +if (lean_obj_tag(x_44) == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + x_46 = x_43; +} else { + lean_dec_ref(x_43); + x_46 = lean_box(0); +} +x_47 = lean_ctor_get(x_44, 0); +lean_inc(x_47); +if (lean_is_exclusive(x_44)) { + lean_ctor_release(x_44, 0); + x_48 = x_44; +} else { + lean_dec_ref(x_44); + x_48 = lean_box(0); +} +if (lean_is_scalar(x_48)) { + x_49 = lean_alloc_ctor(0, 1, 0); +} else { + x_49 = x_48; +} +lean_ctor_set(x_49, 0, x_47); +if (lean_is_scalar(x_46)) { + x_50 = lean_alloc_ctor(0, 2, 0); +} else { + x_50 = x_46; +} +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_45); +return x_50; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_51 = lean_ctor_get(x_43, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + x_52 = x_43; +} else { + lean_dec_ref(x_43); + x_52 = lean_box(0); +} +x_53 = lean_ctor_get(x_44, 0); +lean_inc(x_53); +if (lean_is_exclusive(x_44)) { + lean_ctor_release(x_44, 0); + x_54 = x_44; +} else { + lean_dec_ref(x_44); + x_54 = lean_box(0); +} +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_53); +if (lean_is_scalar(x_54)) { + x_56 = lean_alloc_ctor(1, 1, 0); +} else { + x_56 = x_54; +} +lean_ctor_set(x_56, 0, x_55); +if (lean_is_scalar(x_52)) { + x_57 = lean_alloc_ctor(0, 2, 0); +} else { + x_57 = x_52; +} +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_51); +return x_57; +} +} +} +default: +{ +uint8_t x_58; +x_58 = !lean_is_exclusive(x_2); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_59 = lean_ctor_get(x_2, 0); +x_60 = lean_ctor_get(x_2, 1); +lean_inc(x_1); +x_61 = lean_apply_2(x_1, x_59, x_3); +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +if (lean_obj_tag(x_62) == 0) +{ +uint8_t x_63; +lean_free_object(x_2); +lean_dec(x_60); +lean_dec(x_1); +x_63 = !lean_is_exclusive(x_61); +if (x_63 == 0) +{ +lean_object* x_64; uint8_t x_65; +x_64 = lean_ctor_get(x_61, 0); +lean_dec(x_64); +x_65 = !lean_is_exclusive(x_62); +if (x_65 == 0) +{ +return x_61; +} +else +{ +lean_object* x_66; lean_object* x_67; +x_66 = lean_ctor_get(x_62, 0); +lean_inc(x_66); +lean_dec(x_62); +x_67 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_61, 0, x_67); +return x_61; +} +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_68 = lean_ctor_get(x_61, 1); +lean_inc(x_68); +lean_dec(x_61); +x_69 = lean_ctor_get(x_62, 0); +lean_inc(x_69); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + x_70 = x_62; +} else { + lean_dec_ref(x_62); + x_70 = lean_box(0); +} +if (lean_is_scalar(x_70)) { + x_71 = lean_alloc_ctor(0, 1, 0); +} else { + x_71 = x_70; +} +lean_ctor_set(x_71, 0, x_69); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_68); +return x_72; +} +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_73 = lean_ctor_get(x_61, 1); +lean_inc(x_73); +lean_dec(x_61); +x_74 = lean_ctor_get(x_62, 0); +lean_inc(x_74); +lean_dec(x_62); +x_75 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1, x_60, x_73); +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +if (lean_obj_tag(x_76) == 0) +{ +uint8_t x_77; +lean_dec(x_74); +lean_free_object(x_2); +x_77 = !lean_is_exclusive(x_75); +if (x_77 == 0) +{ +lean_object* x_78; uint8_t x_79; +x_78 = lean_ctor_get(x_75, 0); +lean_dec(x_78); +x_79 = !lean_is_exclusive(x_76); +if (x_79 == 0) +{ +return x_75; +} +else +{ +lean_object* x_80; lean_object* x_81; +x_80 = lean_ctor_get(x_76, 0); +lean_inc(x_80); +lean_dec(x_76); +x_81 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_75, 0, x_81); +return x_75; +} +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_82 = lean_ctor_get(x_75, 1); +lean_inc(x_82); +lean_dec(x_75); +x_83 = lean_ctor_get(x_76, 0); +lean_inc(x_83); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + x_84 = x_76; +} else { + lean_dec_ref(x_76); + x_84 = lean_box(0); +} +if (lean_is_scalar(x_84)) { + x_85 = lean_alloc_ctor(0, 1, 0); +} else { + x_85 = x_84; +} +lean_ctor_set(x_85, 0, x_83); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_82); +return x_86; +} +} +else +{ +uint8_t x_87; +x_87 = !lean_is_exclusive(x_75); +if (x_87 == 0) +{ +lean_object* x_88; uint8_t x_89; +x_88 = lean_ctor_get(x_75, 0); +lean_dec(x_88); +x_89 = !lean_is_exclusive(x_76); +if (x_89 == 0) +{ +lean_object* x_90; +x_90 = lean_ctor_get(x_76, 0); +lean_ctor_set(x_2, 1, x_90); +lean_ctor_set(x_2, 0, x_74); +lean_ctor_set(x_76, 0, x_2); +return x_75; +} +else +{ +lean_object* x_91; lean_object* x_92; +x_91 = lean_ctor_get(x_76, 0); +lean_inc(x_91); +lean_dec(x_76); +lean_ctor_set(x_2, 1, x_91); +lean_ctor_set(x_2, 0, x_74); +x_92 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_92, 0, x_2); +lean_ctor_set(x_75, 0, x_92); +return x_75; +} +} +else +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_93 = lean_ctor_get(x_75, 1); +lean_inc(x_93); +lean_dec(x_75); +x_94 = lean_ctor_get(x_76, 0); +lean_inc(x_94); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + x_95 = x_76; +} else { + lean_dec_ref(x_76); + x_95 = lean_box(0); +} +lean_ctor_set(x_2, 1, x_94); +lean_ctor_set(x_2, 0, x_74); +if (lean_is_scalar(x_95)) { + x_96 = lean_alloc_ctor(1, 1, 0); +} else { + x_96 = x_95; +} +lean_ctor_set(x_96, 0, x_2); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_93); +return x_97; +} +} +} +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_98 = lean_ctor_get(x_2, 0); +x_99 = lean_ctor_get(x_2, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_2); +lean_inc(x_1); +x_100 = lean_apply_2(x_1, x_98, x_3); +x_101 = lean_ctor_get(x_100, 0); +lean_inc(x_101); +if (lean_obj_tag(x_101) == 0) +{ +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +lean_dec(x_99); +lean_dec(x_1); +x_102 = lean_ctor_get(x_100, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + x_103 = x_100; +} else { + lean_dec_ref(x_100); + x_103 = lean_box(0); +} +x_104 = lean_ctor_get(x_101, 0); +lean_inc(x_104); +if (lean_is_exclusive(x_101)) { + lean_ctor_release(x_101, 0); + x_105 = x_101; +} else { + lean_dec_ref(x_101); + x_105 = lean_box(0); +} +if (lean_is_scalar(x_105)) { + x_106 = lean_alloc_ctor(0, 1, 0); +} else { + x_106 = x_105; +} +lean_ctor_set(x_106, 0, x_104); +if (lean_is_scalar(x_103)) { + x_107 = lean_alloc_ctor(0, 2, 0); +} else { + x_107 = x_103; +} +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set(x_107, 1, x_102); +return x_107; +} +else +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_108 = lean_ctor_get(x_100, 1); +lean_inc(x_108); +lean_dec(x_100); +x_109 = lean_ctor_get(x_101, 0); +lean_inc(x_109); +lean_dec(x_101); +x_110 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1, x_99, x_108); +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +if (lean_obj_tag(x_111) == 0) +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +lean_dec(x_109); +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_113 = x_110; +} else { + lean_dec_ref(x_110); + x_113 = lean_box(0); +} +x_114 = lean_ctor_get(x_111, 0); +lean_inc(x_114); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + x_115 = x_111; +} else { + lean_dec_ref(x_111); + x_115 = lean_box(0); +} +if (lean_is_scalar(x_115)) { + x_116 = lean_alloc_ctor(0, 1, 0); +} else { + x_116 = x_115; +} +lean_ctor_set(x_116, 0, x_114); +if (lean_is_scalar(x_113)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_113; +} +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_112); +return x_117; +} +else +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_118 = lean_ctor_get(x_110, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_119 = x_110; +} else { + lean_dec_ref(x_110); + x_119 = lean_box(0); +} +x_120 = lean_ctor_get(x_111, 0); +lean_inc(x_120); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + x_121 = x_111; +} else { + lean_dec_ref(x_111); + x_121 = lean_box(0); +} +x_122 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_122, 0, x_109); +lean_ctor_set(x_122, 1, x_120); +if (lean_is_scalar(x_121)) { + x_123 = lean_alloc_ctor(1, 1, 0); +} else { + x_123 = x_121; +} +lean_ctor_set(x_123, 0, x_122); +if (lean_is_scalar(x_119)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_119; +} +lean_ctor_set(x_124, 0, x_123); +lean_ctor_set(x_124, 1, x_118); +return x_124; +} +} +} +} +} +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Cannot decode params in RPC call '", 34); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("(", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(")'\n", 3); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; uint8_t x_8; +x_7 = lean_st_ref_get(x_1, x_6); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_9 = lean_ctor_get(x_7, 0); +x_10 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +x_12 = lean_ctor_get(x_4, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_4, 1); +lean_inc(x_13); +lean_dec(x_4); +x_14 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_15 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_16 = lean_apply_5(x_11, lean_box(0), x_14, x_15, x_12, x_9); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +lean_dec(x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; +lean_dec(x_13); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +lean_dec(x_17); +x_19 = 1; +x_20 = l_Lean_Name_toString(x_2, x_19); +x_21 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1; +x_22 = lean_string_append(x_21, x_20); +lean_dec(x_20); +x_23 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2; +x_24 = lean_string_append(x_22, x_23); +x_25 = l_Lean_Json_compress(x_3); +x_26 = lean_string_append(x_24, x_25); +lean_dec(x_25); +x_27 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3; +x_28 = lean_string_append(x_26, x_27); +x_29 = lean_string_append(x_28, x_18); +lean_dec(x_18); +x_30 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_31 = lean_string_append(x_29, x_30); +x_32 = 3; +x_33 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); +lean_ctor_set_tag(x_7, 1); +lean_ctor_set(x_7, 0, x_33); +return x_7; +} +else +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_3); +lean_dec(x_2); +x_34 = lean_ctor_get(x_17, 0); +lean_inc(x_34); +lean_dec(x_17); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_13); +lean_ctor_set(x_7, 0, x_35); +return x_7; +} +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_36 = lean_ctor_get(x_7, 0); +x_37 = lean_ctor_get(x_7, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_7); +x_38 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +x_40 = lean_ctor_get(x_4, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_4, 1); +lean_inc(x_41); +lean_dec(x_4); +x_42 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_43 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_44 = lean_apply_5(x_39, lean_box(0), x_42, x_43, x_40, x_36); +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +lean_dec(x_44); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; uint8_t 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; uint8_t x_60; lean_object* x_61; lean_object* x_62; +lean_dec(x_41); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +lean_dec(x_45); +x_47 = 1; +x_48 = l_Lean_Name_toString(x_2, x_47); +x_49 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1; +x_50 = lean_string_append(x_49, x_48); +lean_dec(x_48); +x_51 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2; +x_52 = lean_string_append(x_50, x_51); +x_53 = l_Lean_Json_compress(x_3); +x_54 = lean_string_append(x_52, x_53); +lean_dec(x_53); +x_55 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3; +x_56 = lean_string_append(x_54, x_55); +x_57 = lean_string_append(x_56, x_46); +lean_dec(x_46); +x_58 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_59 = lean_string_append(x_57, x_58); +x_60 = 3; +x_61 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set_uint8(x_61, sizeof(void*)*1, x_60); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_37); +return x_62; +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_3); +lean_dec(x_2); +x_63 = lean_ctor_get(x_45, 0); +lean_inc(x_63); +lean_dec(x_45); +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_41); +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_37); +return x_65; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_5; lean_object* x_6; +lean_dec(x_3); +lean_dec(x_1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_6, 0, x_5); +lean_ctor_set(x_6, 1, x_4); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_apply_3(x_1, x_7, x_3, x_4); +return x_8; +} +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Cannot encode result of RPC call '", 34); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("'\n", 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7), 2, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_2); +x_25 = lean_ctor_get(x_3, 0); +lean_inc(x_25); +lean_dec(x_3); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_5); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_27 = lean_ctor_get(x_3, 0); +lean_inc(x_27); +lean_dec(x_3); +x_28 = lean_st_ref_take(x_1, x_5); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +lean_inc(x_29); +x_32 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_31, x_27, x_29); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +if (lean_obj_tag(x_33) == 0) +{ +uint8_t x_34; +lean_dec(x_32); +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +x_35 = lean_st_ref_set(x_1, x_29, x_30); +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +lean_dec(x_35); +x_6 = x_33; +x_7 = x_36; +goto block_24; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = lean_ctor_get(x_33, 0); +lean_inc(x_37); +lean_dec(x_33); +x_38 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = lean_st_ref_set(x_1, x_29, x_30); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_6 = x_38; +x_7 = x_40; +goto block_24; +} +} +else +{ +lean_object* x_41; uint8_t x_42; +lean_dec(x_29); +x_41 = lean_ctor_get(x_32, 1); +lean_inc(x_41); +lean_dec(x_32); +x_42 = !lean_is_exclusive(x_33); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; +x_43 = lean_st_ref_set(x_1, x_41, x_30); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +x_6 = x_33; +x_7 = x_44; +goto block_24; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_45 = lean_ctor_get(x_33, 0); +lean_inc(x_45); +lean_dec(x_33); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = lean_st_ref_set(x_1, x_41, x_30); +x_48 = lean_ctor_get(x_47, 1); +lean_inc(x_48); +lean_dec(x_47); +x_6 = x_46; +x_7 = x_48; +goto block_24; +} +} +} +block_24: +{ +if (lean_obj_tag(x_6) == 0) +{ +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; uint8_t x_18; lean_object* x_19; lean_object* x_20; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +x_9 = 1; +x_10 = l_Lean_Name_toString(x_2, x_9); +x_11 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_string_append(x_14, x_8); +lean_dec(x_8); +x_16 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_17 = lean_string_append(x_15, x_16); +x_18 = 3; +x_19 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_18); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_7); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_2); +x_21 = lean_ctor_get(x_6, 0); +lean_inc(x_21); +lean_dec(x_6); +x_22 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3(x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_7); +return x_23; +} +} +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Outdated RPC session", 20); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2() { +_start: +{ +uint8_t x_1; lean_object* x_2; lean_object* x_3; +x_1 = 9; +x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__1; +x_3 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4(lean_object* x_1, lean_object* x_2, uint64_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +x_8 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_7, x_3); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2; +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_11 = lean_ctor_get(x_8, 0); +lean_inc(x_11); +lean_dec(x_8); +lean_inc(x_4); +x_12 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5(x_4); +x_13 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__6___boxed), 3, 1); +lean_closure_set(x_13, 0, x_12); +lean_inc(x_1); +lean_inc(x_11); +x_14 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___boxed), 6, 3); +lean_closure_set(x_14, 0, x_11); +lean_closure_set(x_14, 1, x_1); +lean_closure_set(x_14, 2, x_4); +x_15 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 2); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_14); +lean_inc(x_5); +x_16 = l_Lean_Server_RequestM_asTask___rarg(x_15, x_5, x_6); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__2), 4, 1); +lean_closure_set(x_19, 0, x_2); +lean_inc(x_5); +x_20 = l_Lean_Server_RequestM_bindTask___rarg(x_17, x_19, x_5, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___boxed), 5, 2); +lean_closure_set(x_23, 0, x_11); +lean_closure_set(x_23, 1, x_1); +x_24 = l_Lean_Server_RequestM_mapTask___rarg(x_21, x_23, x_5, x_22); +return x_24; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___boxed), 6, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Server_builtinRpcProcedures; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +lean_inc(x_1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___boxed), 6, 2); +lean_closure_set(x_5, 0, x_1); +lean_closure_set(x_5, 1, x_2); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +x_7 = lean_st_ref_take(x_6, x_4); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_8, x_1, x_5); +x_11 = lean_st_ref_set(x_6, x_10, x_9); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +return x_11; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +} +static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(": already registered", 20); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +lean_dec(x_4); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +x_7 = lean_st_ref_get(x_6, x_5); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get(x_7, 1); +lean_inc(x_1); +x_11 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_9, x_1); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_free_object(x_7); +lean_dec(x_3); +x_12 = lean_box(0); +x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1(x_1, x_2, x_12, x_10); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_2); +lean_dec(x_1); +x_14 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_15 = lean_string_append(x_14, x_3); +lean_dec(x_3); +x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; +x_17 = lean_string_append(x_15, x_16); +x_18 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set_tag(x_7, 1); +lean_ctor_set(x_7, 0, x_18); +return x_7; +} +} +else +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_7, 0); +x_20 = lean_ctor_get(x_7, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_7); +lean_inc(x_1); +x_21 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_19, x_1); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_3); +x_22 = lean_box(0); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1(x_1, x_2, x_22, x_20); +return x_23; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_2); +lean_dec(x_1); +x_24 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_25 = lean_string_append(x_24, x_3); +lean_dec(x_3); +x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; +x_27 = lean_string_append(x_25, x_26); +x_28 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_28, 0, x_27); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_20); +return x_29; +} +} +} +} +static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Failed to register builtin RPC call handler for '", 49); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("'", 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(": only possible during initialization", 37); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_4 = 1; +lean_inc(x_1); +x_5 = l_Lean_Name_toString(x_1, x_4); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1; +x_7 = lean_string_append(x_6, x_5); +lean_dec(x_5); +x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2; +x_9 = lean_string_append(x_7, x_8); +x_10 = lean_io_initializing(x_3); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +uint8_t x_13; +lean_dec(x_2); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_10, 0); +lean_dec(x_14); +x_15 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_16 = lean_string_append(x_15, x_9); +lean_dec(x_9); +x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; +x_18 = lean_string_append(x_16, x_17); +x_19 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set_tag(x_10, 1); +lean_ctor_set(x_10, 0, x_19); +return x_10; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_10, 1); +lean_inc(x_20); +lean_dec(x_10); +x_21 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_22 = lean_string_append(x_21, x_9); +lean_dec(x_9); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; +x_24 = lean_string_append(x_22, x_23); +x_25 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_20); +return x_26; +} +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_10, 1); +lean_inc(x_27); +lean_dec(x_10); +x_28 = lean_box(0); +x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); +return x_29; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; lean_object* x_6; +x_5 = 1; +x_6 = l_Lean_Widget_msgToInteractive(x_1, x_5, x_2, x_4); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) +{ +return x_6; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_6, 1); +lean_inc(x_9); +lean_inc(x_8); +lean_dec(x_6); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +return x_10; +} +} +else +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_6); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_6, 0); +x_13 = lean_io_error_to_string(x_12); +x_14 = 4; +x_15 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set_uint8(x_15, sizeof(void*)*1, x_14); +lean_ctor_set(x_6, 0, x_15); +return x_6; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; +x_16 = lean_ctor_get(x_6, 0); +x_17 = lean_ctor_get(x_6, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_6); +x_18 = lean_io_error_to_string(x_16); +x_19 = 4; +x_20 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*1, x_19); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_17); +return x_21; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____lambda__1___boxed), 4, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_5); +x_7 = l_Lean_Server_RequestM_asTask___rarg(x_6, x_2, x_3); +return x_7; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Lean", 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Widget", 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__2; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("InteractiveDiagnostics", 22); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__5; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("msgToInteractive", 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__6; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__7; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____lambda__2), 3, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__8; +x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__9; +x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__4(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__6(x_1, x_2, x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__9(x_1, x_6, x_7, x_4, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__10(x_5, x_6, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__11(x_5, x_6, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; +x_8 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_9 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__3(x_8, x_2, x_3, x_4, x_9, x_6, x_7); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12(x_1, x_2, x_7, x_8, x_5, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__15(x_1, x_6, x_7, x_4, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint64_t x_7; lean_object* x_8; +x_7 = lean_unbox_uint64(x_3); +lean_dec(x_3); +x_8 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4(x_1, x_2, x_7, x_4, x_5, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____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_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedInfoPopup___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +lean_ctor_set(x_2, 2, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedInfoPopup() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instInhabitedInfoPopup___closed__1; +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("type", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("exprExplicit", 12); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("doc", 3); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +x_8 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__2; +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8(x_1, x_8); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3; +x_15 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2161____spec__1(x_1, x_14); +if (lean_obj_tag(x_15) == 0) +{ +uint8_t x_16; +lean_dec(x_13); +lean_dec(x_7); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +return x_15; +} +else +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_15); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_15, 0); +x_21 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_21, 0, x_7); +lean_ctor_set(x_21, 1, x_13); +lean_ctor_set(x_21, 2, x_20); +lean_ctor_set(x_15, 0, x_21); +return x_15; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 0); +lean_inc(x_22); +lean_dec(x_15); +x_23 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_23, 0, x_7); +lean_ctor_set(x_23, 1, x_13); +lean_ctor_set(x_23, 2, x_22); +x_24 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_24, 0, x_23); +return x_24; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403_(x_1); +lean_dec(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__8() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket__8___closed__1; +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__2; +x_2 = lean_box(0); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__1; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3; +x_2 = lean_box(0); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__3; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____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___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__2; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__5; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = lean_box(0); +x_4 = lean_ctor_get(x_1, 1); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +lean_dec(x_1); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_46; +x_46 = lean_box(0); +x_6 = x_46; +goto block_45; +} +else +{ +lean_object* x_47; lean_object* x_48; +x_47 = lean_ctor_get(x_2, 0); +lean_inc(x_47); +lean_dec(x_2); +x_48 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_47); +x_6 = x_48; +goto block_45; +} +block_45: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__1; +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_6); +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_3); +if (lean_obj_tag(x_4) == 0) +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__6; +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = l_List_join___rarg(x_11); +x_13 = l_Lean_Json_mkObj(x_12); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +x_15 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_15, 0, x_14); +x_16 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3; +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_3); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_3); +x_20 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__2; +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_9); +lean_ctor_set(x_22, 1, x_21); +x_23 = l_List_join___rarg(x_22); +x_24 = l_Lean_Json_mkObj(x_23); +return x_24; +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_25 = lean_ctor_get(x_4, 0); +lean_inc(x_25); +lean_dec(x_4); +x_26 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_25); +x_27 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__2; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_3); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__5; +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_9); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_List_join___rarg(x_32); +x_34 = l_Lean_Json_mkObj(x_33); +return x_34; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_35 = lean_ctor_get(x_5, 0); +lean_inc(x_35); +lean_dec(x_5); +x_36 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_36, 0, x_35); +x_37 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3; +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_3); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_3); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_29); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_9); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_List_join___rarg(x_42); +x_44 = l_Lean_Json_mkObj(x_43); +return x_44; +} +} +} +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__8() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket__8___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__1___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__2___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__3___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__7(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__7___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__7___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__8(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__8___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__9(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__9___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__10(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__10___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_4 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__9___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__8___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__3), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__10___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__11___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__12___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__12(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__12___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__13___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__13(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__13___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__16___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__16(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__16___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__16___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__17___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__17(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__17___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__18___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__18(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__18___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__19___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__19(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__19___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__18___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__17___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__19___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__20(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__20___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__21(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__21___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__22___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__22(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__22___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__23___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__23(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__23___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__26___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__26(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__26___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__26___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__27(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__27___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__28___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__28(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__28___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__29___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__29(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__29___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__28___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__27___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__29___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__30___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__30(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__30___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__31___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__31(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__31___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__32___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__32(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__32___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__35___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__35(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__35___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__35___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__36___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__36(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__36___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__37___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__37(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__37___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__38___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__38(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__38___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__37___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__36___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__38___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___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; +x_5 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_4); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_dec(x_3); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_5); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; +x_4 = lean_apply_2(x_1, lean_box(0), x_2); +return x_4; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_1, lean_box(0), x_6); +return x_7; +} +} +else +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_2); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_2, 0, x_10); +x_11 = lean_apply_2(x_1, lean_box(0), x_2); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); +lean_dec(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = lean_apply_2(x_1, lean_box(0), x_14); +return x_15; +} +} +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_3); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__1), 4, 3); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_4); +lean_closure_set(x_6, 2, x_3); +x_7 = lean_ctor_get(x_3, 1); +lean_inc(x_7); +lean_inc(x_3); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__1___rarg), 5, 4); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_ctor_get(x_5, 0); +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +lean_inc(x_14); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_14); +lean_inc(x_16); +x_18 = lean_apply_2(x_16, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__2), 2, 1); +lean_closure_set(x_19, 0, x_16); +lean_inc(x_7); +x_20 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_20, x_8); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__4(size_t x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_box_usize(x_1); +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_2, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +lean_inc(x_5); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_5); +lean_inc(x_7); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +x_10 = lean_box_usize(x_4); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__4___boxed), 3, 2); +lean_closure_set(x_11, 0, x_10); +lean_closure_set(x_11, 1, x_7); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__3___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_11); +x_13 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +lean_inc(x_1); +x_8 = lean_apply_4(x_6, lean_box(0), x_1, x_2, x_7); +lean_inc(x_3); +lean_inc(x_1); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__5___boxed), 4, 3); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_1); +lean_closure_set(x_9, 2, x_3); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__4___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_9); +x_11 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_8, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__7(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_apply_2(x_5, lean_box(0), x_2); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_7); +x_11 = lean_apply_2(x_9, lean_box(0), x_10); +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_2); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_2, 0); +x_14 = lean_ctor_get(x_1, 0); +lean_inc(x_14); +lean_dec(x_1); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_13); +lean_ctor_set(x_2, 0, x_16); +x_17 = lean_apply_2(x_15, lean_box(0), x_2); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +lean_dec(x_2); +x_19 = lean_ctor_get(x_1, 0); +lean_inc(x_19); +lean_dec(x_1); +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_21, 0, x_18); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = lean_apply_2(x_20, lean_box(0), x_22); +return x_23; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___boxed), 4, 3); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_4); +lean_closure_set(x_6, 2, x_2); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__2___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_3); +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +lean_inc(x_7); +lean_inc(x_2); +x_15 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__6), 4, 3); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_3); +lean_closure_set(x_15, 2, x_7); +lean_inc(x_2); +x_16 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__5___rarg(x_2, x_15, x_14); +x_17 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__7), 2, 1); +lean_closure_set(x_17, 0, x_2); +lean_inc(x_7); +x_18 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_16, x_17); +x_19 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_8); +return x_19; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +lean_inc(x_5); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_5); +lean_inc(x_7); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +x_10 = lean_box_usize(x_4); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__4___boxed), 3, 2); +lean_closure_set(x_11, 0, x_10); +lean_closure_set(x_11, 1, x_7); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__12___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_11); +x_13 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +lean_inc(x_1); +x_8 = lean_apply_4(x_6, lean_box(0), x_1, x_2, x_7); +lean_inc(x_3); +lean_inc(x_1); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__9___boxed), 4, 3); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_1); +lean_closure_set(x_9, 2, x_3); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__13___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_9); +x_11 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_8, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__11(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; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +lean_inc(x_3); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__8), 4, 3); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_2); +lean_closure_set(x_6, 2, x_3); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__11___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_3); +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +lean_inc(x_7); +lean_inc(x_2); +x_15 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__10), 4, 3); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_3); +lean_closure_set(x_15, 2, x_7); +lean_inc(x_2); +x_16 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__14___rarg(x_2, x_15, x_14); +x_17 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__7), 2, 1); +lean_closure_set(x_17, 0, x_2); +lean_inc(x_7); +x_18 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_16, x_17); +x_19 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_8); +return x_19; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__12(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; +x_5 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_4); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_dec(x_3); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_5); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_3); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__12), 4, 3); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_4); +lean_closure_set(x_6, 2, x_3); +x_7 = lean_ctor_get(x_3, 1); +lean_inc(x_7); +lean_inc(x_3); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__20___rarg), 5, 4); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_ctor_get(x_5, 0); +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +lean_inc(x_14); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_14); +lean_inc(x_16); +x_18 = lean_apply_2(x_16, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__2), 2, 1); +lean_closure_set(x_19, 0, x_16); +lean_inc(x_7); +x_20 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_20, x_8); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +x_6 = lean_apply_2(x_2, lean_box(0), x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +lean_inc(x_5); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_5); +lean_inc(x_7); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__14), 3, 2); +lean_closure_set(x_10, 0, x_4); +lean_closure_set(x_10, 1, x_7); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__22___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_10); +x_12 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_9, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +lean_inc(x_1); +x_8 = lean_apply_4(x_6, lean_box(0), x_1, x_2, x_7); +lean_inc(x_3); +lean_inc(x_1); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__15___boxed), 4, 3); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_1); +lean_closure_set(x_9, 2, x_3); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__23___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_9); +x_11 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_8, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__17(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; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__13___boxed), 4, 3); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_4); +lean_closure_set(x_6, 2, x_2); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__21___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_3); +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +lean_inc(x_7); +lean_inc(x_2); +x_15 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__16), 4, 3); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_3); +lean_closure_set(x_15, 2, x_7); +lean_inc(x_2); +x_16 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__24___rarg(x_2, x_15, x_14); +x_17 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__7), 2, 1); +lean_closure_set(x_17, 0, x_2); +lean_inc(x_7); +x_18 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_16, x_17); +x_19 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_8); +return x_19; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_5 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +lean_inc(x_5); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_5); +lean_inc(x_7); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__14), 3, 2); +lean_closure_set(x_10, 0, x_4); +lean_closure_set(x_10, 1, x_7); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__31___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_10); +x_12 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_9, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +lean_inc(x_1); +x_8 = lean_apply_4(x_6, lean_box(0), x_1, x_2, x_7); +lean_inc(x_3); +lean_inc(x_1); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__18___boxed), 4, 3); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_1); +lean_closure_set(x_9, 2, x_3); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__32___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_9); +x_11 = lean_apply_4(x_3, lean_box(0), lean_box(0), x_8, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__20(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; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +lean_inc(x_3); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__17), 4, 3); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_2); +lean_closure_set(x_6, 2, x_3); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInfoPopup___spec__30___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_3); +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +lean_inc(x_7); +lean_inc(x_2); +x_15 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__19), 4, 3); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, x_3); +lean_closure_set(x_15, 2, x_7); +lean_inc(x_2); +x_16 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInfoPopup___spec__33___rarg(x_2, x_15, x_14); +x_17 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__7), 2, 1); +lean_closure_set(x_17, 0, x_2); +lean_inc(x_7); +x_18 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_16, x_17); +x_19 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_8); +return x_19; +} +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInfoPopup___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__11), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInfoPopup___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__20), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInfoPopup___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingInfoPopup___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingInfoPopup___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInfoPopup() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingInfoPopup___closed__3; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__6___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__15___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__25___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInfoPopup___spec__34___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__4(x_4, x_2, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; lean_object* x_6; +x_5 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_6 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__5(x_1, x_2, x_3, x_5); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; lean_object* x_6; +x_5 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_6 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__9(x_1, x_2, x_3, x_5); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__13(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__15___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_Widget_instRpcEncodingInfoPopup___lambda__15(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopup___lambda__18___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_Widget_instRpcEncodingInfoPopup___lambda__18(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Info_docString_x3f(x_1, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +x_12 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_12, 0, x_2); +lean_ctor_set(x_12, 1, x_3); +lean_ctor_set(x_12, 2, x_11); +lean_ctor_set(x_9, 0, x_12); +return x_9; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_9, 0); +x_14 = lean_ctor_get(x_9, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_9); +x_15 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_3); +lean_ctor_set(x_15, 2, x_13); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; +} +} +else +{ +uint8_t x_17; +lean_dec(x_3); +lean_dec(x_2); +x_17 = !lean_is_exclusive(x_9); +if (x_17 == 0) +{ +return x_9; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_9, 0); +x_19 = lean_ctor_get(x_9, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_9); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +return x_20; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +switch (lean_obj_tag(x_1)) { +case 1: +{ +lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 3); +lean_inc(x_9); +lean_dec(x_8); +x_10 = 1; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_11 = l_Lean_Widget_ppExprTagged(x_9, x_10, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 2) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +x_16 = l_Lean_Widget_makePopup___lambda__1(x_1, x_2, x_15, x_3, x_4, x_5, x_6, x_13); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_11, 1); +lean_inc(x_17); +lean_dec(x_11); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_12); +x_19 = l_Lean_Widget_makePopup___lambda__1(x_1, x_2, x_18, x_3, x_4, x_5, x_6, x_17); +return x_19; +} +} +else +{ +uint8_t x_20; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_11); +if (x_20 == 0) +{ +return x_11; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_11, 0); +x_22 = lean_ctor_get(x_11, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_11); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +case 4: +{ +lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_1, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = 1; +x_27 = l_Lean_Name_toString(x_25, x_26); +x_28 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_28, 0, x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +x_30 = l_Lean_Widget_makePopup___lambda__1(x_1, x_2, x_29, x_3, x_4, x_5, x_6, x_7); +return x_30; +} +default: +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_box(0); +x_32 = l_Lean_Widget_makePopup___lambda__1(x_1, x_2, x_31, x_3, x_4, x_5, x_6, x_7); +return x_32; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_7 = l_Lean_Elab_Info_type_x3f(x_1, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = lean_box(0); +x_11 = l_Lean_Widget_makePopup___lambda__2(x_1, x_10, x_2, x_3, x_4, x_5, x_9); +return x_11; +} +else +{ +lean_object* x_12; uint8_t x_13; +x_12 = lean_ctor_get(x_7, 1); +lean_inc(x_12); +lean_dec(x_7); +x_13 = !lean_is_exclusive(x_8); +if (x_13 == 0) +{ +lean_object* x_14; uint8_t x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_8, 0); +x_15 = 0; +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_16 = l_Lean_Widget_ppExprTagged(x_14, x_15, x_2, x_3, x_4, x_5, x_12); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_ctor_set(x_8, 0, x_17); +x_19 = l_Lean_Widget_makePopup___lambda__2(x_1, x_8, x_2, x_3, x_4, x_5, x_18); +return x_19; +} +else +{ +uint8_t x_20; +lean_free_object(x_8); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_16); +if (x_20 == 0) +{ +return x_16; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_16, 0); +x_22 = lean_ctor_get(x_16, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_16); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +else +{ +lean_object* x_24; uint8_t x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_8, 0); +lean_inc(x_24); +lean_dec(x_8); +x_25 = 0; +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_26 = l_Lean_Widget_ppExprTagged(x_24, x_25, x_2, x_3, x_4, x_5, x_12); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_27); +x_30 = l_Lean_Widget_makePopup___lambda__2(x_1, x_29, x_2, x_3, x_4, x_5, x_28); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_31 = lean_ctor_get(x_26, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_26, 1); +lean_inc(x_32); +if (lean_is_exclusive(x_26)) { + lean_ctor_release(x_26, 0); + lean_ctor_release(x_26, 1); + x_33 = x_26; +} else { + lean_dec_ref(x_26); + x_33 = lean_box(0); +} +if (lean_is_scalar(x_33)) { + x_34 = lean_alloc_ctor(1, 2, 0); +} else { + x_34 = x_33; +} +lean_ctor_set(x_34, 0, x_31); +lean_ctor_set(x_34, 1, x_32); +return x_34; +} +} +} +} +else +{ +uint8_t x_35; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_35 = !lean_is_exclusive(x_7); +if (x_35 == 0) +{ +return x_7; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_7, 0); +x_37 = lean_ctor_get(x_7, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_7); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Elab_ContextInfo_runMetaM___rarg(x_1, x_2, x_3, x_5); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) +{ +return x_6; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_6, 1); +lean_inc(x_9); +lean_inc(x_8); +lean_dec(x_6); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +return x_10; +} +} +else +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_6); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_6, 0); +x_13 = lean_io_error_to_string(x_12); +x_14 = 4; +x_15 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set_uint8(x_15, sizeof(void*)*1, x_14); +lean_ctor_set(x_6, 0, x_15); +return x_6; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; +x_16 = lean_ctor_get(x_6, 0); +x_17 = lean_ctor_get(x_6, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_6); +x_18 = lean_io_error_to_string(x_16); +x_19 = 4; +x_20 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*1, x_19); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_17); +return x_21; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_makePopup(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_dec(x_1); +x_6 = l_Lean_Elab_Info_lctx(x_5); +x_7 = lean_alloc_closure((void*)(l_Lean_Widget_makePopup___lambda__3), 6, 1); +lean_closure_set(x_7, 0, x_5); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_makePopup___lambda__4___boxed), 5, 3); +lean_closure_set(x_8, 0, x_4); +lean_closure_set(x_8, 1, x_6); +lean_closure_set(x_8, 2, x_7); +x_9 = l_Lean_Server_RequestM_asTask___rarg(x_8, x_2, x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Widget_makePopup___lambda__4(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +lean_inc(x_1); +x_2 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1027_(x_1); +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; +x_4 = lean_ctor_get(x_2, 0); +x_5 = l_Lean_Json_compress(x_1); +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +x_7 = lean_string_append(x_6, x_5); +lean_dec(x_5); +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; +x_9 = lean_string_append(x_7, x_8); +x_10 = lean_string_append(x_9, x_4); +lean_dec(x_4); +x_11 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_12 = lean_string_append(x_10, x_11); +x_13 = 0; +x_14 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set_uint8(x_14, sizeof(void*)*1, x_13); +lean_ctor_set(x_2, 0, x_14); +return x_2; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = l_Lean_Json_compress(x_1); +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +x_18 = lean_string_append(x_17, x_16); +lean_dec(x_16); +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; +x_20 = lean_string_append(x_18, x_19); +x_21 = lean_string_append(x_20, x_15); +lean_dec(x_15); +x_22 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_23 = lean_string_append(x_21, x_22); +x_24 = 0; +x_25 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set_uint8(x_25, sizeof(void*)*1, x_24); +x_26 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_26, 0, x_25); +return x_26; +} +} +else +{ +uint8_t x_27; +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_2); +if (x_27 == 0) +{ +return x_2; +} +else +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_2, 0); +lean_inc(x_28); +lean_dec(x_2); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} +} +} +} +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_7 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +x_9 = lean_st_ref_get(x_1, x_6); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_11 = lean_ctor_get(x_9, 0); +x_12 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_13 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_14 = lean_box_usize(x_4); +x_15 = lean_apply_5(x_8, lean_box(0), x_12, x_13, x_14, x_11); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_dec(x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +lean_dec(x_16); +x_18 = 1; +x_19 = l_Lean_Name_toString(x_2, x_18); +x_20 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1; +x_21 = lean_string_append(x_20, x_19); +lean_dec(x_19); +x_22 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2; +x_23 = lean_string_append(x_21, x_22); +x_24 = l_Lean_Json_compress(x_3); +x_25 = lean_string_append(x_23, x_24); +lean_dec(x_24); +x_26 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3; +x_27 = lean_string_append(x_25, x_26); +x_28 = lean_string_append(x_27, x_17); +lean_dec(x_17); +x_29 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_30 = lean_string_append(x_28, x_29); +x_31 = 3; +x_32 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set_uint8(x_32, sizeof(void*)*1, x_31); +lean_ctor_set_tag(x_9, 1); +lean_ctor_set(x_9, 0, x_32); +return x_9; +} +else +{ +lean_object* x_33; +lean_dec(x_3); +lean_dec(x_2); +x_33 = lean_ctor_get(x_16, 0); +lean_inc(x_33); +lean_dec(x_16); +lean_ctor_set(x_9, 0, x_33); +return x_9; +} +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_34 = lean_ctor_get(x_9, 0); +x_35 = lean_ctor_get(x_9, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_9); +x_36 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_37 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_38 = lean_box_usize(x_4); +x_39 = lean_apply_5(x_8, lean_box(0), x_36, x_37, x_38, x_34); +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +lean_dec(x_39); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +lean_dec(x_40); +x_42 = 1; +x_43 = l_Lean_Name_toString(x_2, x_42); +x_44 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1; +x_45 = lean_string_append(x_44, x_43); +lean_dec(x_43); +x_46 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2; +x_47 = lean_string_append(x_45, x_46); +x_48 = l_Lean_Json_compress(x_3); +x_49 = lean_string_append(x_47, x_48); +lean_dec(x_48); +x_50 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3; +x_51 = lean_string_append(x_49, x_50); +x_52 = lean_string_append(x_51, x_41); +lean_dec(x_41); +x_53 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_54 = lean_string_append(x_52, x_53); +x_55 = 3; +x_56 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set_uint8(x_56, sizeof(void*)*1, x_55); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_35); +return x_57; +} +else +{ +lean_object* x_58; lean_object* x_59; +lean_dec(x_3); +lean_dec(x_2); +x_58 = lean_ctor_get(x_40, 0); +lean_inc(x_58); +lean_dec(x_40); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_35); +return x_59; +} +} +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_3 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__1), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +lean_ctor_set(x_2, 2, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__2; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_2); +x_25 = lean_ctor_get(x_3, 0); +lean_inc(x_25); +lean_dec(x_3); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_5); +return x_26; +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_3); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_49; lean_object* x_50; lean_object* x_128; +x_28 = lean_ctor_get(x_3, 0); +x_29 = lean_st_ref_take(x_1, x_5); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_128 = lean_ctor_get(x_28, 0); +lean_inc(x_128); +if (lean_obj_tag(x_128) == 0) +{ +lean_object* x_129; lean_object* x_130; +x_129 = lean_box(0); +x_130 = lean_ctor_get(x_28, 1); +lean_inc(x_130); +if (lean_obj_tag(x_130) == 0) +{ +lean_object* x_131; +x_131 = lean_ctor_get(x_28, 2); +lean_inc(x_131); +lean_dec(x_28); +if (lean_obj_tag(x_131) == 0) +{ +lean_object* x_132; +lean_free_object(x_3); +x_132 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__3; +lean_inc(x_30); +x_32 = x_132; +x_33 = x_30; +goto block_48; +} +else +{ +uint8_t x_133; +x_133 = !lean_is_exclusive(x_131); +if (x_133 == 0) +{ +lean_object* x_134; +x_134 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_134, 0, x_129); +lean_ctor_set(x_134, 1, x_129); +lean_ctor_set(x_134, 2, x_131); +lean_ctor_set(x_3, 0, x_134); +lean_inc(x_30); +x_32 = x_3; +x_33 = x_30; +goto block_48; +} +else +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_135 = lean_ctor_get(x_131, 0); +lean_inc(x_135); +lean_dec(x_131); +x_136 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_136, 0, x_135); +x_137 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_137, 0, x_129); +lean_ctor_set(x_137, 1, x_129); +lean_ctor_set(x_137, 2, x_136); +lean_ctor_set(x_3, 0, x_137); +lean_inc(x_30); +x_32 = x_3; +x_33 = x_30; +goto block_48; +} +} +} +else +{ +uint8_t x_138; +lean_free_object(x_3); +x_138 = !lean_is_exclusive(x_130); +if (x_138 == 0) +{ +lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_139 = lean_ctor_get(x_130, 0); +x_140 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +lean_inc(x_30); +x_141 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_140, x_139, x_30); +x_142 = lean_ctor_get(x_141, 0); +lean_inc(x_142); +if (lean_obj_tag(x_142) == 0) +{ +lean_object* x_143; uint8_t x_144; +lean_free_object(x_130); +lean_dec(x_28); +x_143 = lean_ctor_get(x_141, 1); +lean_inc(x_143); +lean_dec(x_141); +x_144 = !lean_is_exclusive(x_142); +if (x_144 == 0) +{ +x_32 = x_142; +x_33 = x_143; +goto block_48; +} +else +{ +lean_object* x_145; lean_object* x_146; +x_145 = lean_ctor_get(x_142, 0); +lean_inc(x_145); +lean_dec(x_142); +x_146 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_146, 0, x_145); +x_32 = x_146; +x_33 = x_143; +goto block_48; +} +} +else +{ +lean_object* x_147; uint8_t x_148; +x_147 = lean_ctor_get(x_141, 1); +lean_inc(x_147); +lean_dec(x_141); +x_148 = !lean_is_exclusive(x_142); +if (x_148 == 0) +{ +lean_object* x_149; lean_object* x_150; +x_149 = lean_ctor_get(x_142, 0); +lean_ctor_set(x_130, 0, x_149); +x_150 = lean_ctor_get(x_28, 2); +lean_inc(x_150); +lean_dec(x_28); +if (lean_obj_tag(x_150) == 0) +{ +lean_object* x_151; +x_151 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_151, 0, x_129); +lean_ctor_set(x_151, 1, x_130); +lean_ctor_set(x_151, 2, x_129); +lean_ctor_set(x_142, 0, x_151); +x_32 = x_142; +x_33 = x_147; +goto block_48; +} +else +{ +uint8_t x_152; +x_152 = !lean_is_exclusive(x_150); +if (x_152 == 0) +{ +lean_object* x_153; +x_153 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_153, 0, x_129); +lean_ctor_set(x_153, 1, x_130); +lean_ctor_set(x_153, 2, x_150); +lean_ctor_set(x_142, 0, x_153); +x_32 = x_142; +x_33 = x_147; +goto block_48; +} +else +{ +lean_object* x_154; lean_object* x_155; lean_object* x_156; +x_154 = lean_ctor_get(x_150, 0); +lean_inc(x_154); +lean_dec(x_150); +x_155 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_155, 0, x_154); +x_156 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_156, 0, x_129); +lean_ctor_set(x_156, 1, x_130); +lean_ctor_set(x_156, 2, x_155); +lean_ctor_set(x_142, 0, x_156); +x_32 = x_142; +x_33 = x_147; +goto block_48; +} +} +} +else +{ +lean_object* x_157; lean_object* x_158; +x_157 = lean_ctor_get(x_142, 0); +lean_inc(x_157); +lean_dec(x_142); +lean_ctor_set(x_130, 0, x_157); +x_158 = lean_ctor_get(x_28, 2); +lean_inc(x_158); +lean_dec(x_28); +if (lean_obj_tag(x_158) == 0) +{ +lean_object* x_159; lean_object* x_160; +x_159 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_159, 0, x_129); +lean_ctor_set(x_159, 1, x_130); +lean_ctor_set(x_159, 2, x_129); +x_160 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_160, 0, x_159); +x_32 = x_160; +x_33 = x_147; +goto block_48; +} +else +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_161 = lean_ctor_get(x_158, 0); +lean_inc(x_161); +if (lean_is_exclusive(x_158)) { + lean_ctor_release(x_158, 0); + x_162 = x_158; +} else { + lean_dec_ref(x_158); + x_162 = lean_box(0); +} +if (lean_is_scalar(x_162)) { + x_163 = lean_alloc_ctor(1, 1, 0); +} else { + x_163 = x_162; +} +lean_ctor_set(x_163, 0, x_161); +x_164 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_164, 0, x_129); +lean_ctor_set(x_164, 1, x_130); +lean_ctor_set(x_164, 2, x_163); +x_165 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_165, 0, x_164); +x_32 = x_165; +x_33 = x_147; +goto block_48; +} +} +} +} +else +{ +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_166 = lean_ctor_get(x_130, 0); +lean_inc(x_166); +lean_dec(x_130); +x_167 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +lean_inc(x_30); +x_168 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_167, x_166, x_30); +x_169 = lean_ctor_get(x_168, 0); +lean_inc(x_169); +if (lean_obj_tag(x_169) == 0) +{ +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +lean_dec(x_28); +x_170 = lean_ctor_get(x_168, 1); +lean_inc(x_170); +lean_dec(x_168); +x_171 = lean_ctor_get(x_169, 0); +lean_inc(x_171); +if (lean_is_exclusive(x_169)) { + lean_ctor_release(x_169, 0); + x_172 = x_169; +} else { + lean_dec_ref(x_169); + x_172 = lean_box(0); +} +if (lean_is_scalar(x_172)) { + x_173 = lean_alloc_ctor(0, 1, 0); +} else { + x_173 = x_172; +} +lean_ctor_set(x_173, 0, x_171); +x_32 = x_173; +x_33 = x_170; +goto block_48; +} +else +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; +x_174 = lean_ctor_get(x_168, 1); +lean_inc(x_174); +lean_dec(x_168); +x_175 = lean_ctor_get(x_169, 0); +lean_inc(x_175); +if (lean_is_exclusive(x_169)) { + lean_ctor_release(x_169, 0); + x_176 = x_169; +} else { + lean_dec_ref(x_169); + x_176 = lean_box(0); +} +x_177 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_177, 0, x_175); +x_178 = lean_ctor_get(x_28, 2); +lean_inc(x_178); +lean_dec(x_28); +if (lean_obj_tag(x_178) == 0) +{ +lean_object* x_179; lean_object* x_180; +x_179 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_179, 0, x_129); +lean_ctor_set(x_179, 1, x_177); +lean_ctor_set(x_179, 2, x_129); +if (lean_is_scalar(x_176)) { + x_180 = lean_alloc_ctor(1, 1, 0); +} else { + x_180 = x_176; +} +lean_ctor_set(x_180, 0, x_179); +x_32 = x_180; +x_33 = x_174; +goto block_48; +} +else +{ +lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; +x_181 = lean_ctor_get(x_178, 0); +lean_inc(x_181); +if (lean_is_exclusive(x_178)) { + lean_ctor_release(x_178, 0); + x_182 = x_178; +} else { + lean_dec_ref(x_178); + x_182 = lean_box(0); +} +if (lean_is_scalar(x_182)) { + x_183 = lean_alloc_ctor(1, 1, 0); +} else { + x_183 = x_182; +} +lean_ctor_set(x_183, 0, x_181); +x_184 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_184, 0, x_129); +lean_ctor_set(x_184, 1, x_177); +lean_ctor_set(x_184, 2, x_183); +if (lean_is_scalar(x_176)) { + x_185 = lean_alloc_ctor(1, 1, 0); +} else { + x_185 = x_176; +} +lean_ctor_set(x_185, 0, x_184); +x_32 = x_185; +x_33 = x_174; +goto block_48; +} +} +} +} +} +else +{ +uint8_t x_186; +lean_free_object(x_3); +x_186 = !lean_is_exclusive(x_128); +if (x_186 == 0) +{ +lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_187 = lean_ctor_get(x_128, 0); +x_188 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +lean_inc(x_30); +x_189 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_188, x_187, x_30); +x_190 = lean_ctor_get(x_189, 0); +lean_inc(x_190); +if (lean_obj_tag(x_190) == 0) +{ +lean_object* x_191; uint8_t x_192; +lean_free_object(x_128); +x_191 = lean_ctor_get(x_189, 1); +lean_inc(x_191); +lean_dec(x_189); +x_192 = !lean_is_exclusive(x_190); +if (x_192 == 0) +{ +x_49 = x_190; +x_50 = x_191; +goto block_127; +} +else +{ +lean_object* x_193; lean_object* x_194; +x_193 = lean_ctor_get(x_190, 0); +lean_inc(x_193); +lean_dec(x_190); +x_194 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_194, 0, x_193); +x_49 = x_194; +x_50 = x_191; +goto block_127; +} +} +else +{ +lean_object* x_195; uint8_t x_196; +x_195 = lean_ctor_get(x_189, 1); +lean_inc(x_195); +lean_dec(x_189); +x_196 = !lean_is_exclusive(x_190); +if (x_196 == 0) +{ +lean_object* x_197; +x_197 = lean_ctor_get(x_190, 0); +lean_ctor_set(x_128, 0, x_197); +lean_ctor_set(x_190, 0, x_128); +x_49 = x_190; +x_50 = x_195; +goto block_127; +} +else +{ +lean_object* x_198; lean_object* x_199; +x_198 = lean_ctor_get(x_190, 0); +lean_inc(x_198); +lean_dec(x_190); +lean_ctor_set(x_128, 0, x_198); +x_199 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_199, 0, x_128); +x_49 = x_199; +x_50 = x_195; +goto block_127; +} +} +} +else +{ +lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +x_200 = lean_ctor_get(x_128, 0); +lean_inc(x_200); +lean_dec(x_128); +x_201 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +lean_inc(x_30); +x_202 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_201, x_200, x_30); +x_203 = lean_ctor_get(x_202, 0); +lean_inc(x_203); +if (lean_obj_tag(x_203) == 0) +{ +lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_204 = lean_ctor_get(x_202, 1); +lean_inc(x_204); +lean_dec(x_202); +x_205 = lean_ctor_get(x_203, 0); +lean_inc(x_205); +if (lean_is_exclusive(x_203)) { + lean_ctor_release(x_203, 0); + x_206 = x_203; +} else { + lean_dec_ref(x_203); + x_206 = lean_box(0); +} +if (lean_is_scalar(x_206)) { + x_207 = lean_alloc_ctor(0, 1, 0); +} else { + x_207 = x_206; +} +lean_ctor_set(x_207, 0, x_205); +x_49 = x_207; +x_50 = x_204; +goto block_127; +} +else +{ +lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_208 = lean_ctor_get(x_202, 1); +lean_inc(x_208); +lean_dec(x_202); +x_209 = lean_ctor_get(x_203, 0); +lean_inc(x_209); +if (lean_is_exclusive(x_203)) { + lean_ctor_release(x_203, 0); + x_210 = x_203; +} else { + lean_dec_ref(x_203); + x_210 = lean_box(0); +} +x_211 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_211, 0, x_209); +if (lean_is_scalar(x_210)) { + x_212 = lean_alloc_ctor(1, 1, 0); +} else { + x_212 = x_210; +} +lean_ctor_set(x_212, 0, x_211); +x_49 = x_212; +x_50 = x_208; +goto block_127; +} +} +} +block_48: +{ +if (lean_obj_tag(x_32) == 0) +{ +uint8_t x_34; +lean_dec(x_33); +x_34 = !lean_is_exclusive(x_32); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +x_35 = lean_st_ref_set(x_1, x_30, x_31); +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +lean_dec(x_35); +x_6 = x_32; +x_7 = x_36; +goto block_24; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = lean_ctor_get(x_32, 0); +lean_inc(x_37); +lean_dec(x_32); +x_38 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = lean_st_ref_set(x_1, x_30, x_31); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_6 = x_38; +x_7 = x_40; +goto block_24; +} +} +else +{ +uint8_t x_41; +lean_dec(x_30); +x_41 = !lean_is_exclusive(x_32); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +x_42 = lean_st_ref_set(x_1, x_33, x_31); +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +x_6 = x_32; +x_7 = x_43; +goto block_24; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_32, 0); +lean_inc(x_44); +lean_dec(x_32); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_46 = lean_st_ref_set(x_1, x_33, x_31); +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +x_6 = x_45; +x_7 = x_47; +goto block_24; +} +} +} +block_127: +{ +if (lean_obj_tag(x_49) == 0) +{ +uint8_t x_51; +lean_dec(x_28); +x_51 = !lean_is_exclusive(x_49); +if (x_51 == 0) +{ +x_32 = x_49; +x_33 = x_50; +goto block_48; +} +else +{ +lean_object* x_52; lean_object* x_53; +x_52 = lean_ctor_get(x_49, 0); +lean_inc(x_52); +lean_dec(x_49); +x_53 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_53, 0, x_52); +x_32 = x_53; +x_33 = x_50; +goto block_48; +} +} +else +{ +lean_object* x_54; +x_54 = lean_ctor_get(x_28, 1); +lean_inc(x_54); +if (lean_obj_tag(x_54) == 0) +{ +uint8_t x_55; +x_55 = !lean_is_exclusive(x_49); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_49, 0); +x_57 = lean_box(0); +x_58 = lean_ctor_get(x_28, 2); +lean_inc(x_58); +lean_dec(x_28); +if (lean_obj_tag(x_58) == 0) +{ +lean_object* x_59; +x_59 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_59, 0, x_56); +lean_ctor_set(x_59, 1, x_57); +lean_ctor_set(x_59, 2, x_57); +lean_ctor_set(x_49, 0, x_59); +x_32 = x_49; +x_33 = x_50; +goto block_48; +} +else +{ +uint8_t x_60; +x_60 = !lean_is_exclusive(x_58); +if (x_60 == 0) +{ +lean_object* x_61; +x_61 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_57); +lean_ctor_set(x_61, 2, x_58); +lean_ctor_set(x_49, 0, x_61); +x_32 = x_49; +x_33 = x_50; +goto block_48; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_58, 0); +lean_inc(x_62); +lean_dec(x_58); +x_63 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_63, 0, x_62); +x_64 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_64, 0, x_56); +lean_ctor_set(x_64, 1, x_57); +lean_ctor_set(x_64, 2, x_63); +lean_ctor_set(x_49, 0, x_64); +x_32 = x_49; +x_33 = x_50; +goto block_48; +} +} +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_49, 0); +lean_inc(x_65); +lean_dec(x_49); +x_66 = lean_box(0); +x_67 = lean_ctor_get(x_28, 2); +lean_inc(x_67); +lean_dec(x_28); +if (lean_obj_tag(x_67) == 0) +{ +lean_object* x_68; lean_object* x_69; +x_68 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_68, 0, x_65); +lean_ctor_set(x_68, 1, x_66); +lean_ctor_set(x_68, 2, x_66); +x_69 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_32 = x_69; +x_33 = x_50; +goto block_48; +} +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_70 = lean_ctor_get(x_67, 0); +lean_inc(x_70); +if (lean_is_exclusive(x_67)) { + lean_ctor_release(x_67, 0); + x_71 = x_67; +} else { + lean_dec_ref(x_67); + x_71 = lean_box(0); +} +if (lean_is_scalar(x_71)) { + x_72 = lean_alloc_ctor(1, 1, 0); +} else { + x_72 = x_71; +} +lean_ctor_set(x_72, 0, x_70); +x_73 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_73, 0, x_65); +lean_ctor_set(x_73, 1, x_66); +lean_ctor_set(x_73, 2, x_72); +x_74 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_74, 0, x_73); +x_32 = x_74; +x_33 = x_50; +goto block_48; +} +} +} +else +{ +lean_object* x_75; uint8_t x_76; +x_75 = lean_ctor_get(x_49, 0); +lean_inc(x_75); +lean_dec(x_49); +x_76 = !lean_is_exclusive(x_54); +if (x_76 == 0) +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_77 = lean_ctor_get(x_54, 0); +x_78 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +x_79 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_78, x_77, x_50); +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; uint8_t x_82; +lean_free_object(x_54); +lean_dec(x_75); +lean_dec(x_28); +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +lean_dec(x_79); +x_82 = !lean_is_exclusive(x_80); +if (x_82 == 0) +{ +x_32 = x_80; +x_33 = x_81; +goto block_48; +} +else +{ +lean_object* x_83; lean_object* x_84; +x_83 = lean_ctor_get(x_80, 0); +lean_inc(x_83); +lean_dec(x_80); +x_84 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_84, 0, x_83); +x_32 = x_84; +x_33 = x_81; +goto block_48; +} +} +else +{ +lean_object* x_85; uint8_t x_86; +x_85 = lean_ctor_get(x_79, 1); +lean_inc(x_85); +lean_dec(x_79); +x_86 = !lean_is_exclusive(x_80); +if (x_86 == 0) +{ +lean_object* x_87; lean_object* x_88; +x_87 = lean_ctor_get(x_80, 0); +lean_ctor_set(x_54, 0, x_87); +x_88 = lean_ctor_get(x_28, 2); +lean_inc(x_88); +lean_dec(x_28); +if (lean_obj_tag(x_88) == 0) +{ +lean_object* x_89; lean_object* x_90; +x_89 = lean_box(0); +x_90 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_90, 0, x_75); +lean_ctor_set(x_90, 1, x_54); +lean_ctor_set(x_90, 2, x_89); +lean_ctor_set(x_80, 0, x_90); +x_32 = x_80; +x_33 = x_85; +goto block_48; +} +else +{ +uint8_t x_91; +x_91 = !lean_is_exclusive(x_88); +if (x_91 == 0) +{ +lean_object* x_92; +x_92 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_92, 0, x_75); +lean_ctor_set(x_92, 1, x_54); +lean_ctor_set(x_92, 2, x_88); +lean_ctor_set(x_80, 0, x_92); +x_32 = x_80; +x_33 = x_85; +goto block_48; +} +else +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_88, 0); +lean_inc(x_93); +lean_dec(x_88); +x_94 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_94, 0, x_93); +x_95 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_95, 0, x_75); +lean_ctor_set(x_95, 1, x_54); +lean_ctor_set(x_95, 2, x_94); +lean_ctor_set(x_80, 0, x_95); +x_32 = x_80; +x_33 = x_85; +goto block_48; +} +} +} +else +{ +lean_object* x_96; lean_object* x_97; +x_96 = lean_ctor_get(x_80, 0); +lean_inc(x_96); +lean_dec(x_80); +lean_ctor_set(x_54, 0, x_96); +x_97 = lean_ctor_get(x_28, 2); +lean_inc(x_97); +lean_dec(x_28); +if (lean_obj_tag(x_97) == 0) +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_box(0); +x_99 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_99, 0, x_75); +lean_ctor_set(x_99, 1, x_54); +lean_ctor_set(x_99, 2, x_98); +x_100 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_100, 0, x_99); +x_32 = x_100; +x_33 = x_85; +goto block_48; +} +else +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_101 = lean_ctor_get(x_97, 0); +lean_inc(x_101); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + x_102 = x_97; +} else { + lean_dec_ref(x_97); + x_102 = lean_box(0); +} +if (lean_is_scalar(x_102)) { + x_103 = lean_alloc_ctor(1, 1, 0); +} else { + x_103 = x_102; +} +lean_ctor_set(x_103, 0, x_101); +x_104 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_104, 0, x_75); +lean_ctor_set(x_104, 1, x_54); +lean_ctor_set(x_104, 2, x_103); +x_105 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_105, 0, x_104); +x_32 = x_105; +x_33 = x_85; +goto block_48; +} +} +} +} +else +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_106 = lean_ctor_get(x_54, 0); +lean_inc(x_106); +lean_dec(x_54); +x_107 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +x_108 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_107, x_106, x_50); +x_109 = lean_ctor_get(x_108, 0); +lean_inc(x_109); +if (lean_obj_tag(x_109) == 0) +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +lean_dec(x_75); +lean_dec(x_28); +x_110 = lean_ctor_get(x_108, 1); +lean_inc(x_110); +lean_dec(x_108); +x_111 = lean_ctor_get(x_109, 0); +lean_inc(x_111); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + x_112 = x_109; +} else { + lean_dec_ref(x_109); + x_112 = lean_box(0); +} +if (lean_is_scalar(x_112)) { + x_113 = lean_alloc_ctor(0, 1, 0); +} else { + x_113 = x_112; +} +lean_ctor_set(x_113, 0, x_111); +x_32 = x_113; +x_33 = x_110; +goto block_48; +} +else +{ +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_114 = lean_ctor_get(x_108, 1); +lean_inc(x_114); +lean_dec(x_108); +x_115 = lean_ctor_get(x_109, 0); +lean_inc(x_115); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + x_116 = x_109; +} else { + lean_dec_ref(x_109); + x_116 = lean_box(0); +} +x_117 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_117, 0, x_115); +x_118 = lean_ctor_get(x_28, 2); +lean_inc(x_118); +lean_dec(x_28); +if (lean_obj_tag(x_118) == 0) +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_box(0); +x_120 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_120, 0, x_75); +lean_ctor_set(x_120, 1, x_117); +lean_ctor_set(x_120, 2, x_119); +if (lean_is_scalar(x_116)) { + x_121 = lean_alloc_ctor(1, 1, 0); +} else { + x_121 = x_116; +} +lean_ctor_set(x_121, 0, x_120); +x_32 = x_121; +x_33 = x_114; +goto block_48; +} +else +{ +lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_122 = lean_ctor_get(x_118, 0); +lean_inc(x_122); +if (lean_is_exclusive(x_118)) { + lean_ctor_release(x_118, 0); + x_123 = x_118; +} else { + lean_dec_ref(x_118); + x_123 = lean_box(0); +} +if (lean_is_scalar(x_123)) { + x_124 = lean_alloc_ctor(1, 1, 0); +} else { + x_124 = x_123; +} +lean_ctor_set(x_124, 0, x_122); +x_125 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_125, 0, x_75); +lean_ctor_set(x_125, 1, x_117); +lean_ctor_set(x_125, 2, x_124); +if (lean_is_scalar(x_116)) { + x_126 = lean_alloc_ctor(1, 1, 0); +} else { + x_126 = x_116; +} +lean_ctor_set(x_126, 0, x_125); +x_32 = x_126; +x_33 = x_114; +goto block_48; +} +} +} +} +} +} +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_230; lean_object* x_231; lean_object* x_271; +x_213 = lean_ctor_get(x_3, 0); +lean_inc(x_213); +lean_dec(x_3); +x_214 = lean_st_ref_take(x_1, x_5); +x_215 = lean_ctor_get(x_214, 0); +lean_inc(x_215); +x_216 = lean_ctor_get(x_214, 1); +lean_inc(x_216); +lean_dec(x_214); +x_271 = lean_ctor_get(x_213, 0); +lean_inc(x_271); +if (lean_obj_tag(x_271) == 0) +{ +lean_object* x_272; lean_object* x_273; +x_272 = lean_box(0); +x_273 = lean_ctor_get(x_213, 1); +lean_inc(x_273); +if (lean_obj_tag(x_273) == 0) +{ +lean_object* x_274; +x_274 = lean_ctor_get(x_213, 2); +lean_inc(x_274); +lean_dec(x_213); +if (lean_obj_tag(x_274) == 0) +{ +lean_object* x_275; +x_275 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__3; +lean_inc(x_215); +x_217 = x_275; +x_218 = x_215; +goto block_229; +} +else +{ +lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; +x_276 = lean_ctor_get(x_274, 0); +lean_inc(x_276); +if (lean_is_exclusive(x_274)) { + lean_ctor_release(x_274, 0); + x_277 = x_274; +} else { + lean_dec_ref(x_274); + x_277 = lean_box(0); +} +if (lean_is_scalar(x_277)) { + x_278 = lean_alloc_ctor(1, 1, 0); +} else { + x_278 = x_277; +} +lean_ctor_set(x_278, 0, x_276); +x_279 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_279, 0, x_272); +lean_ctor_set(x_279, 1, x_272); +lean_ctor_set(x_279, 2, x_278); +x_280 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_280, 0, x_279); +lean_inc(x_215); +x_217 = x_280; +x_218 = x_215; +goto block_229; +} +} +else +{ +lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; +x_281 = lean_ctor_get(x_273, 0); +lean_inc(x_281); +if (lean_is_exclusive(x_273)) { + lean_ctor_release(x_273, 0); + x_282 = x_273; +} else { + lean_dec_ref(x_273); + x_282 = lean_box(0); +} +x_283 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +lean_inc(x_215); +x_284 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_283, x_281, x_215); +x_285 = lean_ctor_get(x_284, 0); +lean_inc(x_285); +if (lean_obj_tag(x_285) == 0) +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; +lean_dec(x_282); +lean_dec(x_213); +x_286 = lean_ctor_get(x_284, 1); +lean_inc(x_286); +lean_dec(x_284); +x_287 = lean_ctor_get(x_285, 0); +lean_inc(x_287); +if (lean_is_exclusive(x_285)) { + lean_ctor_release(x_285, 0); + x_288 = x_285; +} else { + lean_dec_ref(x_285); + x_288 = lean_box(0); +} +if (lean_is_scalar(x_288)) { + x_289 = lean_alloc_ctor(0, 1, 0); +} else { + x_289 = x_288; +} +lean_ctor_set(x_289, 0, x_287); +x_217 = x_289; +x_218 = x_286; +goto block_229; +} +else +{ +lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; +x_290 = lean_ctor_get(x_284, 1); +lean_inc(x_290); +lean_dec(x_284); +x_291 = lean_ctor_get(x_285, 0); +lean_inc(x_291); +if (lean_is_exclusive(x_285)) { + lean_ctor_release(x_285, 0); + x_292 = x_285; +} else { + lean_dec_ref(x_285); + x_292 = lean_box(0); +} +if (lean_is_scalar(x_282)) { + x_293 = lean_alloc_ctor(1, 1, 0); +} else { + x_293 = x_282; +} +lean_ctor_set(x_293, 0, x_291); +x_294 = lean_ctor_get(x_213, 2); +lean_inc(x_294); +lean_dec(x_213); +if (lean_obj_tag(x_294) == 0) +{ +lean_object* x_295; lean_object* x_296; +x_295 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_295, 0, x_272); +lean_ctor_set(x_295, 1, x_293); +lean_ctor_set(x_295, 2, x_272); +if (lean_is_scalar(x_292)) { + x_296 = lean_alloc_ctor(1, 1, 0); +} else { + x_296 = x_292; +} +lean_ctor_set(x_296, 0, x_295); +x_217 = x_296; +x_218 = x_290; +goto block_229; +} +else +{ +lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; +x_297 = lean_ctor_get(x_294, 0); +lean_inc(x_297); +if (lean_is_exclusive(x_294)) { + lean_ctor_release(x_294, 0); + x_298 = x_294; +} else { + lean_dec_ref(x_294); + x_298 = lean_box(0); +} +if (lean_is_scalar(x_298)) { + x_299 = lean_alloc_ctor(1, 1, 0); +} else { + x_299 = x_298; +} +lean_ctor_set(x_299, 0, x_297); +x_300 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_300, 0, x_272); +lean_ctor_set(x_300, 1, x_293); +lean_ctor_set(x_300, 2, x_299); +if (lean_is_scalar(x_292)) { + x_301 = lean_alloc_ctor(1, 1, 0); +} else { + x_301 = x_292; +} +lean_ctor_set(x_301, 0, x_300); +x_217 = x_301; +x_218 = x_290; +goto block_229; +} +} +} +} +else +{ +lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +x_302 = lean_ctor_get(x_271, 0); +lean_inc(x_302); +if (lean_is_exclusive(x_271)) { + lean_ctor_release(x_271, 0); + x_303 = x_271; +} else { + lean_dec_ref(x_271); + x_303 = lean_box(0); +} +x_304 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +lean_inc(x_215); +x_305 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_304, x_302, x_215); +x_306 = lean_ctor_get(x_305, 0); +lean_inc(x_306); +if (lean_obj_tag(x_306) == 0) +{ +lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; +lean_dec(x_303); +x_307 = lean_ctor_get(x_305, 1); +lean_inc(x_307); +lean_dec(x_305); +x_308 = lean_ctor_get(x_306, 0); +lean_inc(x_308); +if (lean_is_exclusive(x_306)) { + lean_ctor_release(x_306, 0); + x_309 = x_306; +} else { + lean_dec_ref(x_306); + x_309 = lean_box(0); +} +if (lean_is_scalar(x_309)) { + x_310 = lean_alloc_ctor(0, 1, 0); +} else { + x_310 = x_309; +} +lean_ctor_set(x_310, 0, x_308); +x_230 = x_310; +x_231 = x_307; +goto block_270; +} +else +{ +lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; +x_311 = lean_ctor_get(x_305, 1); +lean_inc(x_311); +lean_dec(x_305); +x_312 = lean_ctor_get(x_306, 0); +lean_inc(x_312); +if (lean_is_exclusive(x_306)) { + lean_ctor_release(x_306, 0); + x_313 = x_306; +} else { + lean_dec_ref(x_306); + x_313 = lean_box(0); +} +if (lean_is_scalar(x_303)) { + x_314 = lean_alloc_ctor(1, 1, 0); +} else { + x_314 = x_303; +} +lean_ctor_set(x_314, 0, x_312); +if (lean_is_scalar(x_313)) { + x_315 = lean_alloc_ctor(1, 1, 0); +} else { + x_315 = x_313; +} +lean_ctor_set(x_315, 0, x_314); +x_230 = x_315; +x_231 = x_311; +goto block_270; +} +} +block_229: +{ +if (lean_obj_tag(x_217) == 0) +{ +lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; +lean_dec(x_218); +x_219 = lean_ctor_get(x_217, 0); +lean_inc(x_219); +if (lean_is_exclusive(x_217)) { + lean_ctor_release(x_217, 0); + x_220 = x_217; +} else { + lean_dec_ref(x_217); + x_220 = lean_box(0); +} +if (lean_is_scalar(x_220)) { + x_221 = lean_alloc_ctor(0, 1, 0); +} else { + x_221 = x_220; +} +lean_ctor_set(x_221, 0, x_219); +x_222 = lean_st_ref_set(x_1, x_215, x_216); +x_223 = lean_ctor_get(x_222, 1); +lean_inc(x_223); +lean_dec(x_222); +x_6 = x_221; +x_7 = x_223; +goto block_24; +} +else +{ +lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; +lean_dec(x_215); +x_224 = lean_ctor_get(x_217, 0); +lean_inc(x_224); +if (lean_is_exclusive(x_217)) { + lean_ctor_release(x_217, 0); + x_225 = x_217; +} else { + lean_dec_ref(x_217); + x_225 = lean_box(0); +} +if (lean_is_scalar(x_225)) { + x_226 = lean_alloc_ctor(1, 1, 0); +} else { + x_226 = x_225; +} +lean_ctor_set(x_226, 0, x_224); +x_227 = lean_st_ref_set(x_1, x_218, x_216); +x_228 = lean_ctor_get(x_227, 1); +lean_inc(x_228); +lean_dec(x_227); +x_6 = x_226; +x_7 = x_228; +goto block_24; +} +} +block_270: +{ +if (lean_obj_tag(x_230) == 0) +{ +lean_object* x_232; lean_object* x_233; lean_object* x_234; +lean_dec(x_213); +x_232 = lean_ctor_get(x_230, 0); +lean_inc(x_232); +if (lean_is_exclusive(x_230)) { + lean_ctor_release(x_230, 0); + x_233 = x_230; +} else { + lean_dec_ref(x_230); + x_233 = lean_box(0); +} +if (lean_is_scalar(x_233)) { + x_234 = lean_alloc_ctor(0, 1, 0); +} else { + x_234 = x_233; +} +lean_ctor_set(x_234, 0, x_232); +x_217 = x_234; +x_218 = x_231; +goto block_229; +} +else +{ +lean_object* x_235; +x_235 = lean_ctor_get(x_213, 1); +lean_inc(x_235); +if (lean_obj_tag(x_235) == 0) +{ +lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; +x_236 = lean_ctor_get(x_230, 0); +lean_inc(x_236); +if (lean_is_exclusive(x_230)) { + lean_ctor_release(x_230, 0); + x_237 = x_230; +} else { + lean_dec_ref(x_230); + x_237 = lean_box(0); +} +x_238 = lean_box(0); +x_239 = lean_ctor_get(x_213, 2); +lean_inc(x_239); +lean_dec(x_213); +if (lean_obj_tag(x_239) == 0) +{ +lean_object* x_240; lean_object* x_241; +x_240 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_240, 0, x_236); +lean_ctor_set(x_240, 1, x_238); +lean_ctor_set(x_240, 2, x_238); +if (lean_is_scalar(x_237)) { + x_241 = lean_alloc_ctor(1, 1, 0); +} else { + x_241 = x_237; +} +lean_ctor_set(x_241, 0, x_240); +x_217 = x_241; +x_218 = x_231; +goto block_229; +} +else +{ +lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +if (lean_is_exclusive(x_239)) { + lean_ctor_release(x_239, 0); + x_243 = x_239; +} else { + lean_dec_ref(x_239); + x_243 = lean_box(0); +} +if (lean_is_scalar(x_243)) { + x_244 = lean_alloc_ctor(1, 1, 0); +} else { + x_244 = x_243; +} +lean_ctor_set(x_244, 0, x_242); +x_245 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_245, 0, x_236); +lean_ctor_set(x_245, 1, x_238); +lean_ctor_set(x_245, 2, x_244); +if (lean_is_scalar(x_237)) { + x_246 = lean_alloc_ctor(1, 1, 0); +} else { + x_246 = x_237; +} +lean_ctor_set(x_246, 0, x_245); +x_217 = x_246; +x_218 = x_231; +goto block_229; +} +} +else +{ +lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; +x_247 = lean_ctor_get(x_230, 0); +lean_inc(x_247); +lean_dec(x_230); +x_248 = lean_ctor_get(x_235, 0); +lean_inc(x_248); +if (lean_is_exclusive(x_235)) { + lean_ctor_release(x_235, 0); + x_249 = x_235; +} else { + lean_dec_ref(x_235); + x_249 = lean_box(0); +} +x_250 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +x_251 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_250, x_248, x_231); +x_252 = lean_ctor_get(x_251, 0); +lean_inc(x_252); +if (lean_obj_tag(x_252) == 0) +{ +lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; +lean_dec(x_249); +lean_dec(x_247); +lean_dec(x_213); +x_253 = lean_ctor_get(x_251, 1); +lean_inc(x_253); +lean_dec(x_251); +x_254 = lean_ctor_get(x_252, 0); +lean_inc(x_254); +if (lean_is_exclusive(x_252)) { + lean_ctor_release(x_252, 0); + x_255 = x_252; +} else { + lean_dec_ref(x_252); + x_255 = lean_box(0); +} +if (lean_is_scalar(x_255)) { + x_256 = lean_alloc_ctor(0, 1, 0); +} else { + x_256 = x_255; +} +lean_ctor_set(x_256, 0, x_254); +x_217 = x_256; +x_218 = x_253; +goto block_229; +} +else +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; +x_257 = lean_ctor_get(x_251, 1); +lean_inc(x_257); +lean_dec(x_251); +x_258 = lean_ctor_get(x_252, 0); +lean_inc(x_258); +if (lean_is_exclusive(x_252)) { + lean_ctor_release(x_252, 0); + x_259 = x_252; +} else { + lean_dec_ref(x_252); + x_259 = lean_box(0); +} +if (lean_is_scalar(x_249)) { + x_260 = lean_alloc_ctor(1, 1, 0); +} else { + x_260 = x_249; +} +lean_ctor_set(x_260, 0, x_258); +x_261 = lean_ctor_get(x_213, 2); +lean_inc(x_261); +lean_dec(x_213); +if (lean_obj_tag(x_261) == 0) +{ +lean_object* x_262; lean_object* x_263; lean_object* x_264; +x_262 = lean_box(0); +x_263 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_263, 0, x_247); +lean_ctor_set(x_263, 1, x_260); +lean_ctor_set(x_263, 2, x_262); +if (lean_is_scalar(x_259)) { + x_264 = lean_alloc_ctor(1, 1, 0); +} else { + x_264 = x_259; +} +lean_ctor_set(x_264, 0, x_263); +x_217 = x_264; +x_218 = x_257; +goto block_229; +} +else +{ +lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; +x_265 = lean_ctor_get(x_261, 0); +lean_inc(x_265); +if (lean_is_exclusive(x_261)) { + lean_ctor_release(x_261, 0); + x_266 = x_261; +} else { + lean_dec_ref(x_261); + x_266 = lean_box(0); +} +if (lean_is_scalar(x_266)) { + x_267 = lean_alloc_ctor(1, 1, 0); +} else { + x_267 = x_266; +} +lean_ctor_set(x_267, 0, x_265); +x_268 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_268, 0, x_247); +lean_ctor_set(x_268, 1, x_260); +lean_ctor_set(x_268, 2, x_267); +if (lean_is_scalar(x_259)) { + x_269 = lean_alloc_ctor(1, 1, 0); +} else { + x_269 = x_259; +} +lean_ctor_set(x_269, 0, x_268); +x_217 = x_269; +x_218 = x_257; +goto block_229; +} +} +} +} +} +} +} +block_24: +{ +if (lean_obj_tag(x_6) == 0) +{ +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; uint8_t x_18; lean_object* x_19; lean_object* x_20; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +x_9 = 1; +x_10 = l_Lean_Name_toString(x_2, x_9); +x_11 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_string_append(x_14, x_8); +lean_dec(x_8); +x_16 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_17 = lean_string_append(x_15, x_16); +x_18 = 3; +x_19 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_18); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_7); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_2); +x_21 = lean_ctor_get(x_6, 0); +lean_inc(x_21); +lean_dec(x_6); +x_22 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475_(x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_7); +return x_23; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__3(lean_object* x_1, lean_object* x_2, uint64_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +x_8 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_7, x_3); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2; +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_11 = lean_ctor_get(x_8, 0); +lean_inc(x_11); +lean_dec(x_8); +lean_inc(x_4); +x_12 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__3(x_4); +x_13 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__4___boxed), 3, 1); +lean_closure_set(x_13, 0, x_12); +lean_inc(x_1); +lean_inc(x_11); +x_14 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__1___boxed), 6, 3); +lean_closure_set(x_14, 0, x_11); +lean_closure_set(x_14, 1, x_1); +lean_closure_set(x_14, 2, x_4); +x_15 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 2); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_14); +lean_inc(x_5); +x_16 = l_Lean_Server_RequestM_asTask___rarg(x_15, x_5, x_6); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__2), 4, 1); +lean_closure_set(x_19, 0, x_2); +lean_inc(x_5); +x_20 = l_Lean_Server_RequestM_bindTask___rarg(x_17, x_19, x_5, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___boxed), 5, 2); +lean_closure_set(x_23, 0, x_11); +lean_closure_set(x_23, 1, x_1); +x_24 = l_Lean_Server_RequestM_mapTask___rarg(x_21, x_23, x_5, x_22); +return x_24; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__3___boxed), 6, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +lean_inc(x_1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__3___boxed), 6, 2); +lean_closure_set(x_5, 0, x_1); +lean_closure_set(x_5, 1, x_2); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +x_7 = lean_st_ref_take(x_6, x_4); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_8, x_1, x_5); +x_11 = lean_st_ref_set(x_6, x_10, x_9); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +return x_11; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +lean_dec(x_4); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +x_7 = lean_st_ref_get(x_6, x_5); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get(x_7, 1); +lean_inc(x_1); +x_11 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_9, x_1); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_free_object(x_7); +lean_dec(x_3); +x_12 = lean_box(0); +x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__1(x_1, x_2, x_12, x_10); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_2); +lean_dec(x_1); +x_14 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_15 = lean_string_append(x_14, x_3); +lean_dec(x_3); +x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; +x_17 = lean_string_append(x_15, x_16); +x_18 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set_tag(x_7, 1); +lean_ctor_set(x_7, 0, x_18); +return x_7; +} +} +else +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_7, 0); +x_20 = lean_ctor_get(x_7, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_7); +lean_inc(x_1); +x_21 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_19, x_1); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_3); +x_22 = lean_box(0); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__1(x_1, x_2, x_22, x_20); +return x_23; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_2); +lean_dec(x_1); +x_24 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_25 = lean_string_append(x_24, x_3); +lean_dec(x_3); +x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; +x_27 = lean_string_append(x_25, x_26); +x_28 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_28, 0, x_27); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_20); +return x_29; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_4 = 1; +lean_inc(x_1); +x_5 = l_Lean_Name_toString(x_1, x_4); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1; +x_7 = lean_string_append(x_6, x_5); +lean_dec(x_5); +x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2; +x_9 = lean_string_append(x_7, x_8); +x_10 = lean_io_initializing(x_3); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +uint8_t x_13; +lean_dec(x_2); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_10, 0); +lean_dec(x_14); +x_15 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_16 = lean_string_append(x_15, x_9); +lean_dec(x_9); +x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; +x_18 = lean_string_append(x_16, x_17); +x_19 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set_tag(x_10, 1); +lean_ctor_set(x_10, 0, x_19); +return x_10; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_10, 1); +lean_inc(x_20); +lean_dec(x_10); +x_21 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_22 = lean_string_append(x_21, x_9); +lean_dec(x_9); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; +x_24 = lean_string_append(x_22, x_23); +x_25 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_20); +return x_26; +} +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_10, 1); +lean_inc(x_27); +lean_dec(x_10); +x_28 = lean_box(0); +x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); +return x_29; +} +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("infoToInteractive", 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__6; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_makePopup), 3, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__2; +x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__3; +x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__4(x_1, x_2, x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; lean_object* x_8; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__1(x_1, x_2, x_3, x_7, x_5, x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint64_t x_7; lean_object* x_8; +x_7 = lean_unbox_uint64(x_3); +lean_dec(x_3); +x_8 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__3(x_1, x_2, x_7, x_4, x_5, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__1___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_7; +lean_dec(x_4); +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_apply_3(x_9, lean_box(0), x_5, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_5, 0); +lean_inc(x_11); +lean_dec(x_5); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_14, 0, x_11); +x_15 = lean_apply_3(x_13, lean_box(0), x_14, x_6); +return x_15; +} +} +else +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_1); +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +lean_dec(x_5); +x_17 = lean_apply_2(x_4, x_16, x_6); +return x_17; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; +x_8 = 1; +x_9 = lean_usize_add(x_1, x_8); +x_10 = lean_array_uset(x_2, x_1, x_6); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3(x_3, x_4, x_5, x_9, x_10, x_7); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_4, x_3); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_5); +x_11 = lean_apply_3(x_9, lean_box(0), x_10, x_6); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_12 = lean_array_uget(x_5, x_4); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_array_uset(x_5, x_4, x_13); +lean_inc(x_2); +lean_inc(x_1); +x_15 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__2), 4, 3); +lean_closure_set(x_15, 0, x_12); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +x_16 = lean_box_usize(x_4); +x_17 = lean_box_usize(x_3); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3___lambda__1___boxed), 7, 5); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_14); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__4), 6, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_5(x_19, lean_box(0), lean_box(0), x_15, x_20, x_6); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_7; +lean_dec(x_4); +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_apply_3(x_9, lean_box(0), x_5, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_5, 0); +lean_inc(x_11); +lean_dec(x_5); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_14, 0, x_11); +x_15 = lean_apply_3(x_13, lean_box(0), x_14, x_6); +return x_15; +} +} +else +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_1); +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +lean_dec(x_5); +x_17 = lean_apply_2(x_4, x_16, x_6); +return x_17; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; lean_object* x_14; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_1, 2); +lean_inc(x_7); +x_8 = lean_ctor_get(x_1, 3); +lean_inc(x_8); +x_9 = lean_ctor_get(x_1, 4); +lean_inc(x_9); +lean_dec(x_1); +x_10 = lean_array_get_size(x_5); +x_11 = lean_usize_of_nat(x_10); +lean_dec(x_10); +x_12 = 0; +lean_inc(x_3); +lean_inc(x_2); +x_13 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3(x_2, x_3, x_11, x_12, x_5, x_4); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +x_15 = !lean_is_exclusive(x_13); +if (x_15 == 0) +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_ctor_get(x_13, 0); +lean_dec(x_16); +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) +{ +return x_13; +} +else +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_14, 0); +lean_inc(x_18); +lean_dec(x_14); +x_19 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_13, 0, x_19); +return x_13; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_20 = lean_ctor_get(x_13, 1); +lean_inc(x_20); +lean_dec(x_13); +x_21 = lean_ctor_get(x_14, 0); +lean_inc(x_21); +if (lean_is_exclusive(x_14)) { + lean_ctor_release(x_14, 0); + x_22 = x_14; +} else { + lean_dec_ref(x_14); + x_22 = lean_box(0); +} +if (lean_is_scalar(x_22)) { + x_23 = lean_alloc_ctor(0, 1, 0); +} else { + x_23 = x_22; +} +lean_ctor_set(x_23, 0, x_21); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_20); +return x_24; +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_25 = lean_ctor_get(x_13, 1); +lean_inc(x_25); +lean_dec(x_13); +x_26 = lean_ctor_get(x_14, 0); +lean_inc(x_26); +lean_dec(x_14); +x_27 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__1), 4, 2); +lean_closure_set(x_27, 0, x_2); +lean_closure_set(x_27, 1, x_3); +x_28 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_27, x_6, x_25); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +if (lean_obj_tag(x_29) == 0) +{ +uint8_t x_30; +lean_dec(x_26); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_30 = !lean_is_exclusive(x_28); +if (x_30 == 0) +{ +lean_object* x_31; uint8_t x_32; +x_31 = lean_ctor_get(x_28, 0); +lean_dec(x_31); +x_32 = !lean_is_exclusive(x_29); +if (x_32 == 0) +{ +return x_28; +} +else +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_29, 0); +lean_inc(x_33); +lean_dec(x_29); +x_34 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_28, 0, x_34); +return x_28; +} +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_35 = lean_ctor_get(x_28, 1); +lean_inc(x_35); +lean_dec(x_28); +x_36 = lean_ctor_get(x_29, 0); +lean_inc(x_36); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + x_37 = x_29; +} else { + lean_dec_ref(x_29); + x_37 = lean_box(0); +} +if (lean_is_scalar(x_37)) { + x_38 = lean_alloc_ctor(0, 1, 0); +} else { + x_38 = x_37; +} +lean_ctor_set(x_38, 0, x_36); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_35); +return x_39; +} +} +else +{ +if (lean_obj_tag(x_7) == 0) +{ +uint8_t x_40; +x_40 = !lean_is_exclusive(x_28); +if (x_40 == 0) +{ +lean_object* x_41; uint8_t x_42; +x_41 = lean_ctor_get(x_28, 0); +lean_dec(x_41); +x_42 = !lean_is_exclusive(x_29); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_29, 0); +x_44 = lean_box(0); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_45; +x_45 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_45, 0, x_26); +lean_ctor_set(x_45, 1, x_43); +lean_ctor_set(x_45, 2, x_44); +lean_ctor_set(x_45, 3, x_8); +lean_ctor_set(x_45, 4, x_44); +lean_ctor_set(x_29, 0, x_45); +return x_28; +} +else +{ +uint8_t x_46; +x_46 = !lean_is_exclusive(x_9); +if (x_46 == 0) +{ +lean_object* x_47; +x_47 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_47, 0, x_26); +lean_ctor_set(x_47, 1, x_43); +lean_ctor_set(x_47, 2, x_44); +lean_ctor_set(x_47, 3, x_8); +lean_ctor_set(x_47, 4, x_9); +lean_ctor_set(x_29, 0, x_47); +return x_28; +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_9, 0); +lean_inc(x_48); +lean_dec(x_9); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +x_50 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_50, 0, x_26); +lean_ctor_set(x_50, 1, x_43); +lean_ctor_set(x_50, 2, x_44); +lean_ctor_set(x_50, 3, x_8); +lean_ctor_set(x_50, 4, x_49); +lean_ctor_set(x_29, 0, x_50); +return x_28; +} +} +} +else +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_29, 0); +lean_inc(x_51); +lean_dec(x_29); +x_52 = lean_box(0); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_53; lean_object* x_54; +x_53 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_53, 0, x_26); +lean_ctor_set(x_53, 1, x_51); +lean_ctor_set(x_53, 2, x_52); +lean_ctor_set(x_53, 3, x_8); +lean_ctor_set(x_53, 4, x_52); +x_54 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_28, 0, x_54); +return x_28; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_55 = lean_ctor_get(x_9, 0); +lean_inc(x_55); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_56 = x_9; +} else { + lean_dec_ref(x_9); + x_56 = lean_box(0); +} +if (lean_is_scalar(x_56)) { + x_57 = lean_alloc_ctor(1, 1, 0); +} else { + x_57 = x_56; +} +lean_ctor_set(x_57, 0, x_55); +x_58 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_58, 0, x_26); +lean_ctor_set(x_58, 1, x_51); +lean_ctor_set(x_58, 2, x_52); +lean_ctor_set(x_58, 3, x_8); +lean_ctor_set(x_58, 4, x_57); +x_59 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_28, 0, x_59); +return x_28; +} +} +} +else +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_60 = lean_ctor_get(x_28, 1); +lean_inc(x_60); +lean_dec(x_28); +x_61 = lean_ctor_get(x_29, 0); +lean_inc(x_61); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + x_62 = x_29; +} else { + lean_dec_ref(x_29); + x_62 = lean_box(0); +} +x_63 = lean_box(0); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_64, 0, x_26); +lean_ctor_set(x_64, 1, x_61); +lean_ctor_set(x_64, 2, x_63); +lean_ctor_set(x_64, 3, x_8); +lean_ctor_set(x_64, 4, x_63); +if (lean_is_scalar(x_62)) { + x_65 = lean_alloc_ctor(1, 1, 0); +} else { + x_65 = x_62; +} +lean_ctor_set(x_65, 0, x_64); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_60); +return x_66; +} +else +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_67 = lean_ctor_get(x_9, 0); +lean_inc(x_67); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_68 = x_9; +} else { + lean_dec_ref(x_9); + x_68 = lean_box(0); +} +if (lean_is_scalar(x_68)) { + x_69 = lean_alloc_ctor(1, 1, 0); +} else { + x_69 = x_68; +} +lean_ctor_set(x_69, 0, x_67); +x_70 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_70, 0, x_26); +lean_ctor_set(x_70, 1, x_61); +lean_ctor_set(x_70, 2, x_63); +lean_ctor_set(x_70, 3, x_8); +lean_ctor_set(x_70, 4, x_69); +if (lean_is_scalar(x_62)) { + x_71 = lean_alloc_ctor(1, 1, 0); +} else { + x_71 = x_62; +} +lean_ctor_set(x_71, 0, x_70); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_60); +return x_72; +} +} +} +else +{ +uint8_t x_73; +x_73 = !lean_is_exclusive(x_28); +if (x_73 == 0) +{ +lean_object* x_74; uint8_t x_75; +x_74 = lean_ctor_get(x_28, 0); +lean_dec(x_74); +x_75 = !lean_is_exclusive(x_29); +if (x_75 == 0) +{ +uint8_t x_76; +x_76 = !lean_is_exclusive(x_7); +if (x_76 == 0) +{ +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_29, 0); +x_78 = lean_box(0); +x_79 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_79, 0, x_26); +lean_ctor_set(x_79, 1, x_77); +lean_ctor_set(x_79, 2, x_7); +lean_ctor_set(x_79, 3, x_8); +lean_ctor_set(x_79, 4, x_78); +lean_ctor_set(x_29, 0, x_79); +return x_28; +} +else +{ +uint8_t x_80; +x_80 = !lean_is_exclusive(x_9); +if (x_80 == 0) +{ +lean_object* x_81; lean_object* x_82; +x_81 = lean_ctor_get(x_29, 0); +x_82 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_82, 0, x_26); +lean_ctor_set(x_82, 1, x_81); +lean_ctor_set(x_82, 2, x_7); +lean_ctor_set(x_82, 3, x_8); +lean_ctor_set(x_82, 4, x_9); +lean_ctor_set(x_29, 0, x_82); +return x_28; +} +else +{ +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_83 = lean_ctor_get(x_29, 0); +x_84 = lean_ctor_get(x_9, 0); +lean_inc(x_84); +lean_dec(x_9); +x_85 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_85, 0, x_84); +x_86 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_86, 0, x_26); +lean_ctor_set(x_86, 1, x_83); +lean_ctor_set(x_86, 2, x_7); +lean_ctor_set(x_86, 3, x_8); +lean_ctor_set(x_86, 4, x_85); +lean_ctor_set(x_29, 0, x_86); +return x_28; +} +} +} +else +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_29, 0); +x_88 = lean_ctor_get(x_7, 0); +lean_inc(x_88); +lean_dec(x_7); +x_89 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_89, 0, x_88); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_90; lean_object* x_91; +x_90 = lean_box(0); +x_91 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_91, 0, x_26); +lean_ctor_set(x_91, 1, x_87); +lean_ctor_set(x_91, 2, x_89); +lean_ctor_set(x_91, 3, x_8); +lean_ctor_set(x_91, 4, x_90); +lean_ctor_set(x_29, 0, x_91); +return x_28; +} +else +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_92 = lean_ctor_get(x_9, 0); +lean_inc(x_92); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_93 = x_9; +} else { + lean_dec_ref(x_9); + x_93 = lean_box(0); +} +if (lean_is_scalar(x_93)) { + x_94 = lean_alloc_ctor(1, 1, 0); +} else { + x_94 = x_93; +} +lean_ctor_set(x_94, 0, x_92); +x_95 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_95, 0, x_26); +lean_ctor_set(x_95, 1, x_87); +lean_ctor_set(x_95, 2, x_89); +lean_ctor_set(x_95, 3, x_8); +lean_ctor_set(x_95, 4, x_94); +lean_ctor_set(x_29, 0, x_95); +return x_28; +} +} +} +else +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_96 = lean_ctor_get(x_29, 0); +lean_inc(x_96); +lean_dec(x_29); +x_97 = lean_ctor_get(x_7, 0); +lean_inc(x_97); +if (lean_is_exclusive(x_7)) { + lean_ctor_release(x_7, 0); + x_98 = x_7; +} else { + lean_dec_ref(x_7); + x_98 = lean_box(0); +} +if (lean_is_scalar(x_98)) { + x_99 = lean_alloc_ctor(1, 1, 0); +} else { + x_99 = x_98; +} +lean_ctor_set(x_99, 0, x_97); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_box(0); +x_101 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_101, 0, x_26); +lean_ctor_set(x_101, 1, x_96); +lean_ctor_set(x_101, 2, x_99); +lean_ctor_set(x_101, 3, x_8); +lean_ctor_set(x_101, 4, x_100); +x_102 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_102, 0, x_101); +lean_ctor_set(x_28, 0, x_102); +return x_28; +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_103 = lean_ctor_get(x_9, 0); +lean_inc(x_103); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_104 = x_9; +} else { + lean_dec_ref(x_9); + x_104 = lean_box(0); +} +if (lean_is_scalar(x_104)) { + x_105 = lean_alloc_ctor(1, 1, 0); +} else { + x_105 = x_104; +} +lean_ctor_set(x_105, 0, x_103); +x_106 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_106, 0, x_26); +lean_ctor_set(x_106, 1, x_96); +lean_ctor_set(x_106, 2, x_99); +lean_ctor_set(x_106, 3, x_8); +lean_ctor_set(x_106, 4, x_105); +x_107 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set(x_28, 0, x_107); +return x_28; +} +} +} +else +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_108 = lean_ctor_get(x_28, 1); +lean_inc(x_108); +lean_dec(x_28); +x_109 = lean_ctor_get(x_29, 0); +lean_inc(x_109); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + x_110 = x_29; +} else { + lean_dec_ref(x_29); + x_110 = lean_box(0); +} +x_111 = lean_ctor_get(x_7, 0); +lean_inc(x_111); +if (lean_is_exclusive(x_7)) { + lean_ctor_release(x_7, 0); + x_112 = x_7; +} else { + lean_dec_ref(x_7); + x_112 = lean_box(0); +} +if (lean_is_scalar(x_112)) { + x_113 = lean_alloc_ctor(1, 1, 0); +} else { + x_113 = x_112; +} +lean_ctor_set(x_113, 0, x_111); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_114 = lean_box(0); +x_115 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_115, 0, x_26); +lean_ctor_set(x_115, 1, x_109); +lean_ctor_set(x_115, 2, x_113); +lean_ctor_set(x_115, 3, x_8); +lean_ctor_set(x_115, 4, x_114); +if (lean_is_scalar(x_110)) { + x_116 = lean_alloc_ctor(1, 1, 0); +} else { + x_116 = x_110; +} +lean_ctor_set(x_116, 0, x_115); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_108); +return x_117; +} +else +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; +x_118 = lean_ctor_get(x_9, 0); +lean_inc(x_118); +if (lean_is_exclusive(x_9)) { + lean_ctor_release(x_9, 0); + x_119 = x_9; +} else { + lean_dec_ref(x_9); + x_119 = lean_box(0); +} +if (lean_is_scalar(x_119)) { + x_120 = lean_alloc_ctor(1, 1, 0); +} else { + x_120 = x_119; +} +lean_ctor_set(x_120, 0, x_118); +x_121 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_121, 0, x_26); +lean_ctor_set(x_121, 1, x_109); +lean_ctor_set(x_121, 2, x_113); +lean_ctor_set(x_121, 3, x_8); +lean_ctor_set(x_121, 4, x_120); +if (lean_is_scalar(x_110)) { + x_122 = lean_alloc_ctor(1, 1, 0); +} else { + x_122 = x_110; +} +lean_ctor_set(x_122, 0, x_121); +x_123 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_123, 0, x_122); +lean_ctor_set(x_123, 1, x_108); +return x_123; +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__2(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; +x_8 = 1; +x_9 = lean_usize_add(x_1, x_8); +x_10 = lean_array_uset(x_2, x_1, x_6); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5(x_3, x_4, x_5, x_9, x_10, x_7); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_4, x_3); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_5); +x_11 = lean_apply_3(x_9, lean_box(0), x_10, x_6); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_12 = lean_array_uget(x_5, x_4); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_array_uset(x_5, x_4, x_13); +lean_inc(x_2); +lean_inc(x_1); +x_15 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__1), 4, 3); +lean_closure_set(x_15, 0, x_12); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +x_16 = lean_box_usize(x_4); +x_17 = lean_box_usize(x_3); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__2___boxed), 7, 5); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_14); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__6), 6, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_5(x_19, lean_box(0), lean_box(0), x_15, x_20, x_6); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; uint8_t x_6; +x_5 = lean_st_ref_get(x_1, x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; +x_7 = lean_ctor_get(x_5, 0); +lean_dec(x_7); +lean_ctor_set(x_5, 0, x_2); +return x_5; +} +else +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_5, 1); +lean_inc(x_8); +lean_dec(x_5); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_2); +lean_ctor_set(x_9, 1, x_8); +return x_9; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_2); +x_28 = lean_ctor_get(x_3, 0); +lean_inc(x_28); +lean_dec(x_3); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_5); +return x_29; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_30 = lean_ctor_get(x_3, 0); +lean_inc(x_30); +lean_dec(x_3); +x_31 = lean_st_ref_take(x_1, x_5); +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); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_51; +x_51 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +lean_inc(x_32); +x_34 = x_51; +x_35 = x_32; +goto block_50; +} +else +{ +uint8_t x_52; +x_52 = !lean_is_exclusive(x_30); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; size_t x_55; size_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_53 = lean_ctor_get(x_30, 0); +x_54 = lean_array_get_size(x_53); +x_55 = lean_usize_of_nat(x_54); +lean_dec(x_54); +x_56 = 0; +x_57 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_58 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +lean_inc(x_32); +x_59 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5(x_57, x_58, x_55, x_56, x_53, x_32); +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; uint8_t x_62; +lean_free_object(x_30); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = !lean_is_exclusive(x_60); +if (x_62 == 0) +{ +x_34 = x_60; +x_35 = x_61; +goto block_50; +} +else +{ +lean_object* x_63; lean_object* x_64; +x_63 = lean_ctor_get(x_60, 0); +lean_inc(x_63); +lean_dec(x_60); +x_64 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_64, 0, x_63); +x_34 = x_64; +x_35 = x_61; +goto block_50; +} +} +else +{ +lean_object* x_65; uint8_t x_66; +x_65 = lean_ctor_get(x_59, 1); +lean_inc(x_65); +lean_dec(x_59); +x_66 = !lean_is_exclusive(x_60); +if (x_66 == 0) +{ +lean_object* x_67; +x_67 = lean_ctor_get(x_60, 0); +lean_ctor_set(x_30, 0, x_67); +lean_ctor_set(x_60, 0, x_30); +x_34 = x_60; +x_35 = x_65; +goto block_50; +} +else +{ +lean_object* x_68; lean_object* x_69; +x_68 = lean_ctor_get(x_60, 0); +lean_inc(x_68); +lean_dec(x_60); +lean_ctor_set(x_30, 0, x_68); +x_69 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_69, 0, x_30); +x_34 = x_69; +x_35 = x_65; +goto block_50; +} +} +} +else +{ +lean_object* x_70; lean_object* x_71; size_t x_72; size_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_70 = lean_ctor_get(x_30, 0); +lean_inc(x_70); +lean_dec(x_30); +x_71 = lean_array_get_size(x_70); +x_72 = lean_usize_of_nat(x_71); +lean_dec(x_71); +x_73 = 0; +x_74 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_75 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +lean_inc(x_32); +x_76 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5(x_74, x_75, x_72, x_73, x_70, x_32); +x_77 = lean_ctor_get(x_76, 0); +lean_inc(x_77); +if (lean_obj_tag(x_77) == 0) +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_78 = lean_ctor_get(x_76, 1); +lean_inc(x_78); +lean_dec(x_76); +x_79 = lean_ctor_get(x_77, 0); +lean_inc(x_79); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + x_80 = x_77; +} else { + lean_dec_ref(x_77); + x_80 = lean_box(0); +} +if (lean_is_scalar(x_80)) { + x_81 = lean_alloc_ctor(0, 1, 0); +} else { + x_81 = x_80; +} +lean_ctor_set(x_81, 0, x_79); +x_34 = x_81; +x_35 = x_78; +goto block_50; +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_82 = lean_ctor_get(x_76, 1); +lean_inc(x_82); +lean_dec(x_76); +x_83 = lean_ctor_get(x_77, 0); +lean_inc(x_83); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + x_84 = x_77; +} else { + lean_dec_ref(x_77); + x_84 = lean_box(0); +} +x_85 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_85, 0, x_83); +if (lean_is_scalar(x_84)) { + x_86 = lean_alloc_ctor(1, 1, 0); +} else { + x_86 = x_84; +} +lean_ctor_set(x_86, 0, x_85); +x_34 = x_86; +x_35 = x_82; +goto block_50; +} +} +} +block_50: +{ +if (lean_obj_tag(x_34) == 0) +{ +uint8_t x_36; +lean_dec(x_35); +x_36 = !lean_is_exclusive(x_34); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; +x_37 = lean_st_ref_set(x_1, x_32, x_33); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_6 = x_34; +x_7 = x_38; +goto block_27; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_34, 0); +lean_inc(x_39); +lean_dec(x_34); +x_40 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_40, 0, x_39); +x_41 = lean_st_ref_set(x_1, x_32, x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_6 = x_40; +x_7 = x_42; +goto block_27; +} +} +else +{ +uint8_t x_43; +lean_dec(x_32); +x_43 = !lean_is_exclusive(x_34); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +x_44 = lean_st_ref_set(x_1, x_35, x_33); +x_45 = lean_ctor_get(x_44, 1); +lean_inc(x_45); +lean_dec(x_44); +x_6 = x_34; +x_7 = x_45; +goto block_27; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_46 = lean_ctor_get(x_34, 0); +lean_inc(x_46); +lean_dec(x_34); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = lean_st_ref_set(x_1, x_35, x_33); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_6 = x_47; +x_7 = x_49; +goto block_27; +} +} +} +} +block_27: +{ +if (lean_obj_tag(x_6) == 0) +{ +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; uint8_t x_18; lean_object* x_19; lean_object* x_20; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +x_9 = 1; +x_10 = l_Lean_Name_toString(x_2, x_9); +x_11 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_string_append(x_14, x_8); +lean_dec(x_8); +x_16 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_17 = lean_string_append(x_15, x_16); +x_18 = 3; +x_19 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_18); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_7); +return x_20; +} +else +{ +lean_object* x_21; +lean_dec(x_2); +x_21 = lean_ctor_get(x_6, 0); +lean_inc(x_21); +lean_dec(x_6); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_7); +return x_23; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 0); +lean_inc(x_24); +lean_dec(x_21); +x_25 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845_(x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_7); +return x_26; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__3(lean_object* x_1, lean_object* x_2, uint64_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +x_8 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_7, x_3); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2; +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_11 = lean_ctor_get(x_8, 0); +lean_inc(x_11); +lean_dec(x_8); +x_12 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__32(x_4); +x_13 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__33___boxed), 3, 1); +lean_closure_set(x_13, 0, x_12); +lean_inc(x_11); +x_14 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__1___boxed), 4, 1); +lean_closure_set(x_14, 0, x_11); +x_15 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 2); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_14); +lean_inc(x_5); +x_16 = l_Lean_Server_RequestM_asTask___rarg(x_15, x_5, x_6); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__2), 4, 1); +lean_closure_set(x_19, 0, x_1); +lean_inc(x_5); +x_20 = l_Lean_Server_RequestM_bindTask___rarg(x_17, x_19, x_5, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__2___boxed), 5, 2); +lean_closure_set(x_23, 0, x_11); +lean_closure_set(x_23, 1, x_2); +x_24 = l_Lean_Server_RequestM_mapTask___rarg(x_21, x_23, x_5, x_22); +return x_24; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__3___boxed), 6, 2); +lean_closure_set(x_3, 0, x_2); +lean_closure_set(x_3, 1, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +lean_inc(x_1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__3___boxed), 6, 2); +lean_closure_set(x_5, 0, x_2); +lean_closure_set(x_5, 1, x_1); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +x_7 = lean_st_ref_take(x_6, x_4); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_8, x_1, x_5); +x_11 = lean_st_ref_set(x_6, x_10, x_9); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +return x_11; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +lean_dec(x_4); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +x_7 = lean_st_ref_get(x_6, x_5); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get(x_7, 1); +lean_inc(x_1); +x_11 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_9, x_1); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_free_object(x_7); +lean_dec(x_3); +x_12 = lean_box(0); +x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__1(x_1, x_2, x_12, x_10); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_2); +lean_dec(x_1); +x_14 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_15 = lean_string_append(x_14, x_3); +lean_dec(x_3); +x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; +x_17 = lean_string_append(x_15, x_16); +x_18 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set_tag(x_7, 1); +lean_ctor_set(x_7, 0, x_18); +return x_7; +} +} +else +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_7, 0); +x_20 = lean_ctor_get(x_7, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_7); +lean_inc(x_1); +x_21 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_19, x_1); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_3); +x_22 = lean_box(0); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__1(x_1, x_2, x_22, x_20); +return x_23; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_2); +lean_dec(x_1); +x_24 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_25 = lean_string_append(x_24, x_3); +lean_dec(x_3); +x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; +x_27 = lean_string_append(x_25, x_26); +x_28 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_28, 0, x_27); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_20); +return x_29; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_4 = 1; +lean_inc(x_1); +x_5 = l_Lean_Name_toString(x_1, x_4); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1; +x_7 = lean_string_append(x_6, x_5); +lean_dec(x_5); +x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2; +x_9 = lean_string_append(x_7, x_8); +x_10 = lean_io_initializing(x_3); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +uint8_t x_13; +lean_dec(x_2); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_10, 0); +lean_dec(x_14); +x_15 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_16 = lean_string_append(x_15, x_9); +lean_dec(x_9); +x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; +x_18 = lean_string_append(x_16, x_17); +x_19 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set_tag(x_10, 1); +lean_ctor_set(x_10, 0, x_19); +return x_10; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_10, 1); +lean_inc(x_20); +lean_dec(x_10); +x_21 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_22 = lean_string_append(x_21, x_9); +lean_dec(x_9); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; +x_24 = lean_string_append(x_22, x_23); +x_25 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_20); +return x_26; +} +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_10, 1); +lean_inc(x_27); +lean_dec(x_10); +x_28 = lean_box(0); +x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); +return x_29; +} +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("getInteractiveGoals", 19); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_getInteractiveGoals), 3, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__2; +x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__3; +x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; +x_8 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_9 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3___lambda__1(x_8, x_2, x_3, x_4, x_9, x_6, x_7); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__3(x_1, x_2, x_7, x_8, x_5, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; +x_8 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_9 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___lambda__2(x_8, x_2, x_3, x_4, x_9, x_6, x_7); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__5(x_1, x_2, x_7, x_8, x_5, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___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_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint64_t x_7; lean_object* x_8; +x_7 = lean_unbox_uint64(x_3); +lean_dec(x_3); +x_8 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__3(x_1, x_2, x_7, x_4, x_5, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__1___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_7; +lean_dec(x_4); +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_apply_3(x_9, lean_box(0), x_5, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_5, 0); +lean_inc(x_11); +lean_dec(x_5); +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_14, 0, x_11); +x_15 = lean_apply_3(x_13, lean_box(0), x_14, x_6); +return x_15; +} +} +else +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_1); +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +lean_dec(x_5); +x_17 = lean_apply_2(x_4, x_16, x_6); +return x_17; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; +x_8 = 1; +x_9 = lean_usize_add(x_1, x_8); +x_10 = lean_array_uset(x_2, x_1, x_6); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3(x_3, x_4, x_5, x_9, x_10, x_7); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_4, x_3); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_5); +x_11 = lean_apply_3(x_9, lean_box(0), x_10, x_6); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_12 = lean_array_uget(x_5, x_4); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_array_uset(x_5, x_4, x_13); +lean_inc(x_2); +lean_inc(x_1); +x_15 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__12___lambda__2), 4, 3); +lean_closure_set(x_15, 0, x_12); +lean_closure_set(x_15, 1, x_1); +lean_closure_set(x_15, 2, x_2); +x_16 = lean_box_usize(x_4); +x_17 = lean_box_usize(x_3); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3___lambda__1___boxed), 7, 5); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_14); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__4), 6, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_5(x_19, lean_box(0), lean_box(0), x_15, x_20, x_6); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_2); +x_28 = lean_ctor_get(x_3, 0); +lean_inc(x_28); +lean_dec(x_3); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_5); +return x_29; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_30 = lean_ctor_get(x_3, 0); +lean_inc(x_30); +lean_dec(x_3); +x_31 = lean_st_ref_take(x_1, x_5); +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); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_51; +x_51 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +lean_inc(x_32); +x_34 = x_51; +x_35 = x_32; +goto block_50; +} +else +{ +uint8_t x_52; +x_52 = !lean_is_exclusive(x_30); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; size_t x_58; size_t x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_53 = lean_ctor_get(x_30, 0); +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +x_56 = lean_ctor_get(x_53, 2); +lean_inc(x_56); +lean_dec(x_53); +x_57 = lean_array_get_size(x_54); +x_58 = lean_usize_of_nat(x_57); +lean_dec(x_57); +x_59 = 0; +x_60 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_61 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +lean_inc(x_32); +x_62 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3(x_60, x_61, x_58, x_59, x_54, x_32); +x_63 = lean_ctor_get(x_62, 0); +lean_inc(x_63); +if (lean_obj_tag(x_63) == 0) +{ +lean_object* x_64; uint8_t x_65; +lean_dec(x_56); +lean_dec(x_55); +lean_free_object(x_30); +x_64 = lean_ctor_get(x_62, 1); +lean_inc(x_64); +lean_dec(x_62); +x_65 = !lean_is_exclusive(x_63); +if (x_65 == 0) +{ +x_34 = x_63; +x_35 = x_64; +goto block_50; +} +else +{ +lean_object* x_66; lean_object* x_67; +x_66 = lean_ctor_get(x_63, 0); +lean_inc(x_66); +lean_dec(x_63); +x_67 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_67, 0, x_66); +x_34 = x_67; +x_35 = x_64; +goto block_50; +} +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_68 = lean_ctor_get(x_62, 1); +lean_inc(x_68); +lean_dec(x_62); +x_69 = lean_ctor_get(x_63, 0); +lean_inc(x_69); +lean_dec(x_63); +x_70 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +x_71 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_70, x_55, x_68); +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +if (lean_obj_tag(x_72) == 0) +{ +lean_object* x_73; uint8_t x_74; +lean_dec(x_69); +lean_dec(x_56); +lean_free_object(x_30); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = !lean_is_exclusive(x_72); +if (x_74 == 0) +{ +x_34 = x_72; +x_35 = x_73; +goto block_50; +} +else +{ +lean_object* x_75; lean_object* x_76; +x_75 = lean_ctor_get(x_72, 0); +lean_inc(x_75); +lean_dec(x_72); +x_76 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_76, 0, x_75); +x_34 = x_76; +x_35 = x_73; +goto block_50; +} +} +else +{ +lean_object* x_77; uint8_t x_78; +x_77 = lean_ctor_get(x_71, 1); +lean_inc(x_77); +lean_dec(x_71); +x_78 = !lean_is_exclusive(x_72); +if (x_78 == 0) +{ +lean_object* x_79; lean_object* x_80; +x_79 = lean_ctor_get(x_72, 0); +x_80 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_80, 0, x_69); +lean_ctor_set(x_80, 1, x_79); +lean_ctor_set(x_80, 2, x_56); +lean_ctor_set(x_30, 0, x_80); +lean_ctor_set(x_72, 0, x_30); +x_34 = x_72; +x_35 = x_77; +goto block_50; +} +else +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_72, 0); +lean_inc(x_81); +lean_dec(x_72); +x_82 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_82, 0, x_69); +lean_ctor_set(x_82, 1, x_81); +lean_ctor_set(x_82, 2, x_56); +lean_ctor_set(x_30, 0, x_82); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_30); +x_34 = x_83; +x_35 = x_77; +goto block_50; +} +} +} +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; size_t x_89; size_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_84 = lean_ctor_get(x_30, 0); +lean_inc(x_84); +lean_dec(x_30); +x_85 = lean_ctor_get(x_84, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_84, 1); +lean_inc(x_86); +x_87 = lean_ctor_get(x_84, 2); +lean_inc(x_87); +lean_dec(x_84); +x_88 = lean_array_get_size(x_85); +x_89 = lean_usize_of_nat(x_88); +lean_dec(x_88); +x_90 = 0; +x_91 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_92 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +lean_inc(x_32); +x_93 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3(x_91, x_92, x_89, x_90, x_85, x_32); +x_94 = lean_ctor_get(x_93, 0); +lean_inc(x_94); +if (lean_obj_tag(x_94) == 0) +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_87); +lean_dec(x_86); +x_95 = lean_ctor_get(x_93, 1); +lean_inc(x_95); +lean_dec(x_93); +x_96 = lean_ctor_get(x_94, 0); +lean_inc(x_96); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + x_97 = x_94; +} else { + lean_dec_ref(x_94); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(0, 1, 0); +} else { + x_98 = x_97; +} +lean_ctor_set(x_98, 0, x_96); +x_34 = x_98; +x_35 = x_95; +goto block_50; +} +else +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_99 = lean_ctor_get(x_93, 1); +lean_inc(x_99); +lean_dec(x_93); +x_100 = lean_ctor_get(x_94, 0); +lean_inc(x_100); +lean_dec(x_94); +x_101 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1; +x_102 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__8(x_101, x_86, x_99); +x_103 = lean_ctor_get(x_102, 0); +lean_inc(x_103); +if (lean_obj_tag(x_103) == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +lean_dec(x_100); +lean_dec(x_87); +x_104 = lean_ctor_get(x_102, 1); +lean_inc(x_104); +lean_dec(x_102); +x_105 = lean_ctor_get(x_103, 0); +lean_inc(x_105); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + x_106 = x_103; +} else { + lean_dec_ref(x_103); + x_106 = lean_box(0); +} +if (lean_is_scalar(x_106)) { + x_107 = lean_alloc_ctor(0, 1, 0); +} else { + x_107 = x_106; +} +lean_ctor_set(x_107, 0, x_105); +x_34 = x_107; +x_35 = x_104; +goto block_50; +} +else +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_108 = lean_ctor_get(x_102, 1); +lean_inc(x_108); +lean_dec(x_102); +x_109 = lean_ctor_get(x_103, 0); +lean_inc(x_109); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + x_110 = x_103; +} else { + lean_dec_ref(x_103); + x_110 = lean_box(0); +} +x_111 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_111, 0, x_100); +lean_ctor_set(x_111, 1, x_109); +lean_ctor_set(x_111, 2, x_87); +x_112 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_112, 0, x_111); +if (lean_is_scalar(x_110)) { + x_113 = lean_alloc_ctor(1, 1, 0); +} else { + x_113 = x_110; +} +lean_ctor_set(x_113, 0, x_112); +x_34 = x_113; +x_35 = x_108; +goto block_50; +} +} +} +} +block_50: +{ +if (lean_obj_tag(x_34) == 0) +{ +uint8_t x_36; +lean_dec(x_35); +x_36 = !lean_is_exclusive(x_34); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; +x_37 = lean_st_ref_set(x_1, x_32, x_33); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_6 = x_34; +x_7 = x_38; +goto block_27; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_34, 0); +lean_inc(x_39); +lean_dec(x_34); +x_40 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_40, 0, x_39); +x_41 = lean_st_ref_set(x_1, x_32, x_33); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_6 = x_40; +x_7 = x_42; +goto block_27; +} +} +else +{ +uint8_t x_43; +lean_dec(x_32); +x_43 = !lean_is_exclusive(x_34); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +x_44 = lean_st_ref_set(x_1, x_35, x_33); +x_45 = lean_ctor_get(x_44, 1); +lean_inc(x_45); +lean_dec(x_44); +x_6 = x_34; +x_7 = x_45; +goto block_27; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_46 = lean_ctor_get(x_34, 0); +lean_inc(x_46); +lean_dec(x_34); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = lean_st_ref_set(x_1, x_35, x_33); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_6 = x_47; +x_7 = x_49; +goto block_27; +} +} +} +} +block_27: +{ +if (lean_obj_tag(x_6) == 0) +{ +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; uint8_t x_18; lean_object* x_19; lean_object* x_20; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +x_9 = 1; +x_10 = l_Lean_Name_toString(x_2, x_9); +x_11 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_string_append(x_14, x_8); +lean_dec(x_8); +x_16 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_17 = lean_string_append(x_15, x_16); +x_18 = 3; +x_19 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_18); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_7); +return x_20; +} +else +{ +lean_object* x_21; +lean_dec(x_2); +x_21 = lean_ctor_get(x_6, 0); +lean_inc(x_21); +lean_dec(x_6); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_7); +return x_23; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 0); +lean_inc(x_24); +lean_dec(x_21); +x_25 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1563_(x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_7); +return x_26; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__2(lean_object* x_1, lean_object* x_2, uint64_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +x_8 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_7, x_3); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2; +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_11 = lean_ctor_get(x_8, 0); +lean_inc(x_11); +lean_dec(x_8); +x_12 = l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__35(x_4); +x_13 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__36___boxed), 3, 1); +lean_closure_set(x_13, 0, x_12); +lean_inc(x_11); +x_14 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__1___boxed), 4, 1); +lean_closure_set(x_14, 0, x_11); +x_15 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 2); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_14); +lean_inc(x_5); +x_16 = l_Lean_Server_RequestM_asTask___rarg(x_15, x_5, x_6); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__2), 4, 1); +lean_closure_set(x_19, 0, x_1); +lean_inc(x_5); +x_20 = l_Lean_Server_RequestM_bindTask___rarg(x_17, x_19, x_5, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__1___boxed), 5, 2); +lean_closure_set(x_23, 0, x_11); +lean_closure_set(x_23, 1, x_2); +x_24 = l_Lean_Server_RequestM_mapTask___rarg(x_21, x_23, x_5, x_22); +return x_24; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__2___boxed), 6, 2); +lean_closure_set(x_3, 0, x_2); +lean_closure_set(x_3, 1, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +lean_inc(x_1); +x_5 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__2___boxed), 6, 2); +lean_closure_set(x_5, 0, x_2); +lean_closure_set(x_5, 1, x_1); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +x_7 = lean_st_ref_take(x_6, x_4); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_8, x_1, x_5); +x_11 = lean_st_ref_set(x_6, x_10, x_9); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +return x_11; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +lean_dec(x_4); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; +x_7 = lean_st_ref_get(x_6, x_5); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get(x_7, 1); +lean_inc(x_1); +x_11 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_9, x_1); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_free_object(x_7); +lean_dec(x_3); +x_12 = lean_box(0); +x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__1(x_1, x_2, x_12, x_10); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_2); +lean_dec(x_1); +x_14 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_15 = lean_string_append(x_14, x_3); +lean_dec(x_3); +x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; +x_17 = lean_string_append(x_15, x_16); +x_18 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set_tag(x_7, 1); +lean_ctor_set(x_7, 0, x_18); +return x_7; +} +} +else +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_7, 0); +x_20 = lean_ctor_get(x_7, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_7); +lean_inc(x_1); +x_21 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_19, x_1); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_3); +x_22 = lean_box(0); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__1(x_1, x_2, x_22, x_20); +return x_23; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_2); +lean_dec(x_1); +x_24 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_25 = lean_string_append(x_24, x_3); +lean_dec(x_3); +x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; +x_27 = lean_string_append(x_25, x_26); +x_28 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_28, 0, x_27); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_20); +return x_29; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_4 = 1; +lean_inc(x_1); +x_5 = l_Lean_Name_toString(x_1, x_4); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1; +x_7 = lean_string_append(x_6, x_5); +lean_dec(x_5); +x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2; +x_9 = lean_string_append(x_7, x_8); +x_10 = lean_io_initializing(x_3); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +uint8_t x_13; +lean_dec(x_2); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_10); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_14 = lean_ctor_get(x_10, 0); +lean_dec(x_14); +x_15 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_16 = lean_string_append(x_15, x_9); +lean_dec(x_9); +x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; +x_18 = lean_string_append(x_16, x_17); +x_19 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set_tag(x_10, 1); +lean_ctor_set(x_10, 0, x_19); +return x_10; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_10, 1); +lean_inc(x_20); +lean_dec(x_10); +x_21 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_22 = lean_string_append(x_21, x_9); +lean_dec(x_9); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; +x_24 = lean_string_append(x_22, x_23); +x_25 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_20); +return x_26; +} +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_10, 1); +lean_inc(x_27); +lean_dec(x_10); +x_28 = lean_box(0); +x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); +return x_29; +} +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("getInteractiveTermGoal", 22); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_getInteractiveTermGoal), 3, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__2; +x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__3; +x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; +x_8 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_9 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3___lambda__1(x_8, x_2, x_3, x_4, x_9, x_6, x_7); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__3(x_1, x_2, x_7, x_8, x_5, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint64_t x_7; lean_object* x_8; +x_7 = lean_unbox_uint64(x_3); +lean_dec(x_3); +x_8 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__2___lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____spec__1___lambda__1(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedGetInteractiveDiagnosticsParams() { +_start: +{ +lean_object* x_1; +x_1 = lean_box(0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; +x_4 = l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1; +return x_4; +} +else +{ +lean_object* x_5; +x_5 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonLineRange____x40_Lean_Data_Lsp_Extra___hyg_1810_(x_3); +lean_dec(x_3); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +return x_5; +} +else +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +return x_8; +} +} +else +{ +uint8_t x_9; +x_9 = !lean_is_exclusive(x_5); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_5, 0); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_5, 0, x_11); +return x_5; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_5, 0); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +return x_14; +} +} +} +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("lineRange", 9); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____spec__1(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +else +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_3); +if (x_7 == 0) +{ +return x_3; +} +else +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +lean_dec(x_3); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +return x_9; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036_(x_1); +lean_dec(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1074____spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +lean_dec(x_1); +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_4 = lean_ctor_get(x_2, 0); +lean_inc(x_4); +lean_dec(x_2); +x_5 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonLineRange____x40_Lean_Data_Lsp_Extra___hyg_1865_(x_4); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_1); +lean_ctor_set(x_6, 1, x_5); +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_6); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1074_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____closed__1; +x_3 = l_Lean_Json_opt___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1074____spec__1(x_2, x_1); +x_4 = lean_box(0); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_3); +lean_ctor_set(x_5, 1, x_4); +x_6 = l_List_join___rarg(x_5); +x_7 = l_Lean_Json_mkObj(x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonGetInteractiveDiagnosticsParams___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1074_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonGetInteractiveDiagnosticsParams() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonGetInteractiveDiagnosticsParams___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_eq(x_3, x_4); +if (x_6 == 0) +{ +lean_object* x_7; size_t x_8; size_t x_9; +x_7 = lean_array_uget(x_2, x_3); +x_8 = 1; +x_9 = lean_usize_add(x_3, x_8); +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_10; +x_10 = lean_array_push(x_5, x_7); +x_3 = x_9; +x_5 = x_10; +goto _start; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_12 = lean_ctor_get(x_1, 0); +x_13 = lean_ctor_get(x_12, 0); +x_14 = lean_ctor_get(x_12, 1); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +lean_dec(x_16); +x_18 = lean_nat_dec_le(x_13, x_17); +if (x_18 == 0) +{ +uint8_t x_19; +x_19 = lean_nat_dec_le(x_17, x_13); +lean_dec(x_17); +if (x_19 == 0) +{ +lean_dec(x_15); +lean_dec(x_7); +x_3 = x_9; +goto _start; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); +lean_dec(x_15); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +lean_dec(x_21); +x_23 = lean_nat_dec_lt(x_13, x_22); +lean_dec(x_22); +if (x_23 == 0) +{ +lean_dec(x_7); +x_3 = x_9; +goto _start; +} +else +{ +lean_object* x_25; +x_25 = lean_array_push(x_5, x_7); +x_3 = x_9; +x_5 = x_25; +goto _start; +} +} +} +else +{ +uint8_t x_27; +x_27 = lean_nat_dec_lt(x_17, x_14); +if (x_27 == 0) +{ +uint8_t x_28; +x_28 = lean_nat_dec_le(x_17, x_13); +lean_dec(x_17); +if (x_28 == 0) +{ +lean_dec(x_15); +lean_dec(x_7); +x_3 = x_9; +goto _start; +} +else +{ +lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_30 = lean_ctor_get(x_15, 1); +lean_inc(x_30); +lean_dec(x_15); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +lean_dec(x_30); +x_32 = lean_nat_dec_lt(x_13, x_31); +lean_dec(x_31); +if (x_32 == 0) +{ +lean_dec(x_7); +x_3 = x_9; +goto _start; +} +else +{ +lean_object* x_34; +x_34 = lean_array_push(x_5, x_7); +x_3 = x_9; +x_5 = x_34; +goto _start; +} +} +} +else +{ +lean_object* x_36; +lean_dec(x_17); +lean_dec(x_15); +x_36 = lean_array_push(x_5, x_7); +x_3 = x_9; +x_5 = x_36; +goto _start; +} +} +} +} +else +{ +return x_5; +} +} +} +static lean_object* _init_l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__1; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = lean_ctor_get(x_2, 0); +lean_inc(x_3); +lean_dec(x_2); +x_4 = l_List_getLast_x3f___rarg(x_3); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; +x_5 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2; +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_ctor_get(x_6, 4); +lean_inc(x_7); +lean_dec(x_6); +x_8 = l_Std_PersistentArray_toArray___rarg(x_7); +x_9 = lean_array_get_size(x_8); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_lt(x_10, x_9); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_9); +lean_dec(x_8); +x_12 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2; +return x_12; +} +else +{ +uint8_t x_13; +x_13 = lean_nat_dec_le(x_9, x_9); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_9); +lean_dec(x_8); +x_14 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2; +return x_14; +} +else +{ +size_t x_15; size_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = 0; +x_16 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_17 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__1; +x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1(x_1, x_8, x_15, x_16, x_17); +lean_dec(x_8); +x_19 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_19, 0, x_18); +return x_19; +} +} +} +} +} +LEAN_EXPORT uint8_t l_Lean_Widget_getInteractiveDiagnostics___lambda__2(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = 1; +return x_2; +} +} +LEAN_EXPORT uint8_t l_Lean_Widget_getInteractiveDiagnostics___lambda__3(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; uint8_t x_4; +x_3 = lean_ctor_get(x_2, 0); +x_4 = lean_nat_dec_lt(x_3, x_1); +return x_4; +} +} +static lean_object* _init_l_Lean_Widget_getInteractiveDiagnostics___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_getInteractiveDiagnostics___lambda__2___boxed), 1, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_4 = l_Lean_Server_RequestM_readDoc(x_2, x_3); +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_4, 1); +lean_inc(x_6); +if (lean_is_exclusive(x_4)) { + lean_ctor_release(x_4, 0); + lean_ctor_release(x_4, 1); + x_7 = x_4; +} else { + lean_dec_ref(x_4); + x_7 = lean_box(0); +} +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_5, 1); +lean_inc(x_15); +lean_dec(x_5); +x_16 = l_Lean_Widget_getInteractiveDiagnostics___closed__1; +x_17 = l_IO_AsyncList_waitAll___rarg(x_16, x_15, x_6); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_8 = x_18; +x_9 = x_19; +goto block_14; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_20 = lean_ctor_get(x_5, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_5, 0); +lean_inc(x_22); +lean_dec(x_5); +x_23 = lean_ctor_get(x_22, 2); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_unsigned_to_nat(0u); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_FileMap_lspPosToUtf8Pos(x_23, x_26); +lean_dec(x_23); +x_28 = lean_alloc_closure((void*)(l_Lean_Widget_getInteractiveDiagnostics___lambda__3___boxed), 2, 1); +lean_closure_set(x_28, 0, x_27); +x_29 = l_IO_AsyncList_waitAll___rarg(x_28, x_20, x_6); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_8 = x_30; +x_9 = x_31; +goto block_14; +} +block_14: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_getInteractiveDiagnostics___lambda__1___boxed), 2, 1); +lean_closure_set(x_10, 0, x_1); +x_11 = l_Task_Priority_default; +x_12 = lean_task_map(x_10, x_8, x_11); +if (lean_is_scalar(x_7)) { + x_13 = lean_alloc_ctor(0, 2, 0); +} else { + x_13 = x_7; +} +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_9); +return x_13; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__2___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Widget_getInteractiveDiagnostics___lambda__2(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__3___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Lean_Widget_getInteractiveDiagnostics___lambda__3(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Widget_getInteractiveDiagnostics(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("range", 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("fullRange", 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("severity", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("code", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("source", 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("message", 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("tags", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("relatedInformation", 18); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; 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; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(x_2); +x_4 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__1; +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_box(0); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_6); +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); +x_9 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(x_8); +x_10 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__2; +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +x_12 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_6); +x_13 = lean_ctor_get(x_1, 2); +lean_inc(x_13); +x_14 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__3; +x_15 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__1(x_14, x_13); +lean_dec(x_13); +x_16 = lean_ctor_get(x_1, 3); +lean_inc(x_16); +x_17 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__4; +x_18 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__2(x_17, x_16); +lean_dec(x_16); +x_19 = lean_ctor_get(x_1, 4); +lean_inc(x_19); +x_20 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__5; +x_21 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2131____spec__1(x_20, x_19); +lean_dec(x_19); +x_22 = lean_ctor_get(x_1, 5); +lean_inc(x_22); +x_23 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3(x_22); +x_24 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__6; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_6); +x_27 = lean_ctor_get(x_1, 6); +lean_inc(x_27); +x_28 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__7; +x_29 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__3(x_28, x_27); +x_30 = lean_ctor_get(x_1, 7); +lean_inc(x_30); +lean_dec(x_1); +x_31 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__8; +x_32 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__5(x_31, x_30); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_6); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_29); +lean_ctor_set(x_34, 1, x_33); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_26); +lean_ctor_set(x_35, 1, x_34); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_21); +lean_ctor_set(x_36, 1, x_35); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_18); +lean_ctor_set(x_37, 1, x_36); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_15); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_12); +lean_ctor_set(x_39, 1, x_38); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_7); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_List_join___rarg(x_40); +x_42 = l_Lean_Json_mkObj(x_41); +return x_42; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__4(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036_(x_1); +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; +x_4 = lean_ctor_get(x_2, 0); +x_5 = l_Lean_Json_compress(x_1); +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +x_7 = lean_string_append(x_6, x_5); +lean_dec(x_5); +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; +x_9 = lean_string_append(x_7, x_8); +x_10 = lean_string_append(x_9, x_4); +lean_dec(x_4); +x_11 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_12 = lean_string_append(x_10, x_11); +x_13 = 0; +x_14 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set_uint8(x_14, sizeof(void*)*1, x_13); +lean_ctor_set(x_2, 0, x_14); +return x_2; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = l_Lean_Json_compress(x_1); +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +x_18 = lean_string_append(x_17, x_16); +lean_dec(x_16); +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; +x_20 = lean_string_append(x_18, x_19); +x_21 = lean_string_append(x_20, x_15); +lean_dec(x_15); +x_22 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_23 = lean_string_append(x_21, x_22); +x_24 = 0; +x_25 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set_uint8(x_25, sizeof(void*)*1, x_24); +x_26 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_26, 0, x_25); +return x_26; +} +} +else +{ +uint8_t x_27; +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_2); +if (x_27 == 0) +{ +return x_2; +} +else +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_2, 0); +lean_inc(x_28); +lean_dec(x_2); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} +} +} +} +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_2, x_1); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_8 = lean_array_uget(x_3, x_2); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_array_uset(x_3, x_2, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_2, x_11); +x_13 = lean_array_uset(x_10, x_2, x_8); +x_2 = x_12; +x_3 = x_13; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_2, x_1); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_8 = lean_array_uget(x_3, x_2); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_array_uset(x_3, x_2, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_2, x_11); +x_13 = lean_array_uset(x_10, x_2, x_8); +x_2 = x_12; +x_3 = x_13; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__9(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_2, x_1); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_30; +x_8 = lean_array_uget(x_3, x_2); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_array_uset(x_3, x_2, x_9); +x_30 = lean_ctor_get(x_8, 2); +lean_inc(x_30); +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; lean_object* x_37; lean_object* x_38; +x_31 = lean_ctor_get(x_8, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_8, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_8, 3); +lean_inc(x_33); +x_34 = lean_ctor_get(x_8, 4); +lean_inc(x_34); +x_35 = lean_ctor_get(x_8, 5); +lean_inc(x_35); +x_36 = lean_ctor_get(x_8, 6); +lean_inc(x_36); +x_37 = lean_ctor_get(x_8, 7); +lean_inc(x_37); +lean_dec(x_8); +x_38 = lean_box(0); +if (lean_obj_tag(x_33) == 0) +{ +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_40 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_39, x_35, x_4); +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +if (lean_obj_tag(x_41) == 0) +{ +uint8_t x_42; +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_32); +lean_dec(x_31); +x_42 = !lean_is_exclusive(x_40); +if (x_42 == 0) +{ +lean_object* x_43; uint8_t x_44; +x_43 = lean_ctor_get(x_40, 0); +lean_dec(x_43); +x_44 = !lean_is_exclusive(x_41); +if (x_44 == 0) +{ +x_11 = x_40; +goto block_29; +} +else +{ +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_41, 0); +lean_inc(x_45); +lean_dec(x_41); +x_46 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_40, 0, x_46); +x_11 = x_40; +goto block_29; +} +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_47 = lean_ctor_get(x_40, 1); +lean_inc(x_47); +lean_dec(x_40); +x_48 = lean_ctor_get(x_41, 0); +lean_inc(x_48); +if (lean_is_exclusive(x_41)) { + lean_ctor_release(x_41, 0); + x_49 = x_41; +} else { + lean_dec_ref(x_41); + x_49 = lean_box(0); +} +if (lean_is_scalar(x_49)) { + x_50 = lean_alloc_ctor(0, 1, 0); +} else { + x_50 = x_49; +} +lean_ctor_set(x_50, 0, x_48); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_47); +x_11 = x_51; +goto block_29; +} +} +else +{ +lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_52 = lean_ctor_get(x_40, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_53 = x_40; +} else { + lean_dec_ref(x_40); + x_53 = lean_box(0); +} +x_54 = !lean_is_exclusive(x_41); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_41, 0); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_53); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_103; lean_object* x_104; +x_103 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_103, 0, x_31); +lean_ctor_set(x_103, 1, x_32); +lean_ctor_set(x_103, 2, x_38); +lean_ctor_set(x_103, 3, x_38); +lean_ctor_set(x_103, 4, x_38); +lean_ctor_set(x_103, 5, x_55); +lean_ctor_set(x_103, 6, x_38); +lean_ctor_set(x_103, 7, x_38); +lean_ctor_set(x_41, 0, x_103); +x_104 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_104, 0, x_41); +lean_ctor_set(x_104, 1, x_52); +x_11 = x_104; +goto block_29; +} +else +{ +uint8_t x_105; +lean_free_object(x_41); +x_105 = !lean_is_exclusive(x_37); +if (x_105 == 0) +{ +lean_object* x_106; lean_object* x_107; size_t x_108; size_t x_109; lean_object* x_110; uint8_t x_111; +x_106 = lean_ctor_get(x_37, 0); +x_107 = lean_array_get_size(x_106); +x_108 = lean_usize_of_nat(x_107); +lean_dec(x_107); +x_109 = 0; +x_110 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_108, x_109, x_106, x_52); +x_111 = !lean_is_exclusive(x_110); +if (x_111 == 0) +{ +lean_object* x_112; uint8_t x_113; +x_112 = lean_ctor_get(x_110, 0); +x_113 = !lean_is_exclusive(x_112); +if (x_113 == 0) +{ +lean_object* x_114; lean_object* x_115; +x_114 = lean_ctor_get(x_112, 0); +lean_ctor_set(x_37, 0, x_114); +x_115 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_115, 0, x_31); +lean_ctor_set(x_115, 1, x_32); +lean_ctor_set(x_115, 2, x_38); +lean_ctor_set(x_115, 3, x_38); +lean_ctor_set(x_115, 4, x_38); +lean_ctor_set(x_115, 5, x_55); +lean_ctor_set(x_115, 6, x_38); +lean_ctor_set(x_115, 7, x_37); +lean_ctor_set(x_112, 0, x_115); +x_11 = x_110; +goto block_29; +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_112, 0); +lean_inc(x_116); +lean_dec(x_112); +lean_ctor_set(x_37, 0, x_116); +x_117 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_117, 0, x_31); +lean_ctor_set(x_117, 1, x_32); +lean_ctor_set(x_117, 2, x_38); +lean_ctor_set(x_117, 3, x_38); +lean_ctor_set(x_117, 4, x_38); +lean_ctor_set(x_117, 5, x_55); +lean_ctor_set(x_117, 6, x_38); +lean_ctor_set(x_117, 7, x_37); +x_118 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_118, 0, x_117); +lean_ctor_set(x_110, 0, x_118); +x_11 = x_110; +goto block_29; +} +} +else +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_119 = lean_ctor_get(x_110, 0); +x_120 = lean_ctor_get(x_110, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_110); +x_121 = lean_ctor_get(x_119, 0); +lean_inc(x_121); +if (lean_is_exclusive(x_119)) { + lean_ctor_release(x_119, 0); + x_122 = x_119; +} else { + lean_dec_ref(x_119); + x_122 = lean_box(0); +} +lean_ctor_set(x_37, 0, x_121); +x_123 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_123, 0, x_31); +lean_ctor_set(x_123, 1, x_32); +lean_ctor_set(x_123, 2, x_38); +lean_ctor_set(x_123, 3, x_38); +lean_ctor_set(x_123, 4, x_38); +lean_ctor_set(x_123, 5, x_55); +lean_ctor_set(x_123, 6, x_38); +lean_ctor_set(x_123, 7, x_37); +if (lean_is_scalar(x_122)) { + x_124 = lean_alloc_ctor(1, 1, 0); +} else { + x_124 = x_122; +} +lean_ctor_set(x_124, 0, x_123); +x_125 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_125, 0, x_124); +lean_ctor_set(x_125, 1, x_120); +x_11 = x_125; +goto block_29; +} +} +else +{ +lean_object* x_126; lean_object* x_127; size_t x_128; size_t 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; +x_126 = lean_ctor_get(x_37, 0); +lean_inc(x_126); +lean_dec(x_37); +x_127 = lean_array_get_size(x_126); +x_128 = lean_usize_of_nat(x_127); +lean_dec(x_127); +x_129 = 0; +x_130 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_128, x_129, x_126, x_52); +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_130, 1); +lean_inc(x_132); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_133 = x_130; +} else { + lean_dec_ref(x_130); + x_133 = lean_box(0); +} +x_134 = lean_ctor_get(x_131, 0); +lean_inc(x_134); +if (lean_is_exclusive(x_131)) { + lean_ctor_release(x_131, 0); + x_135 = x_131; +} else { + lean_dec_ref(x_131); + x_135 = lean_box(0); +} +x_136 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_136, 0, x_134); +x_137 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_137, 0, x_31); +lean_ctor_set(x_137, 1, x_32); +lean_ctor_set(x_137, 2, x_38); +lean_ctor_set(x_137, 3, x_38); +lean_ctor_set(x_137, 4, x_38); +lean_ctor_set(x_137, 5, x_55); +lean_ctor_set(x_137, 6, x_38); +lean_ctor_set(x_137, 7, x_136); +if (lean_is_scalar(x_135)) { + x_138 = lean_alloc_ctor(1, 1, 0); +} else { + x_138 = x_135; +} +lean_ctor_set(x_138, 0, x_137); +if (lean_is_scalar(x_133)) { + x_139 = lean_alloc_ctor(0, 2, 0); +} else { + x_139 = x_133; +} +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_132); +x_11 = x_139; +goto block_29; +} +} +} +else +{ +uint8_t x_140; +lean_free_object(x_41); +x_140 = !lean_is_exclusive(x_36); +if (x_140 == 0) +{ +lean_object* x_141; lean_object* x_142; size_t x_143; size_t x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; uint8_t x_148; +x_141 = lean_ctor_get(x_36, 0); +x_142 = lean_array_get_size(x_141); +x_143 = lean_usize_of_nat(x_142); +lean_dec(x_142); +x_144 = 0; +x_145 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_143, x_144, x_141, x_52); +x_146 = lean_ctor_get(x_145, 0); +lean_inc(x_146); +x_147 = lean_ctor_get(x_145, 1); +lean_inc(x_147); +lean_dec(x_145); +x_148 = !lean_is_exclusive(x_146); +if (x_148 == 0) +{ +lean_object* x_149; +x_149 = lean_ctor_get(x_146, 0); +lean_ctor_set(x_36, 0, x_149); +lean_ctor_set(x_146, 0, x_36); +x_56 = x_146; +x_57 = x_147; +goto block_102; +} +else +{ +lean_object* x_150; lean_object* x_151; +x_150 = lean_ctor_get(x_146, 0); +lean_inc(x_150); +lean_dec(x_146); +lean_ctor_set(x_36, 0, x_150); +x_151 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_151, 0, x_36); +x_56 = x_151; +x_57 = x_147; +goto block_102; +} +} +else +{ +lean_object* x_152; lean_object* x_153; size_t x_154; size_t x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_152 = lean_ctor_get(x_36, 0); +lean_inc(x_152); +lean_dec(x_36); +x_153 = lean_array_get_size(x_152); +x_154 = lean_usize_of_nat(x_153); +lean_dec(x_153); +x_155 = 0; +x_156 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_154, x_155, x_152, x_52); +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_159 = lean_ctor_get(x_157, 0); +lean_inc(x_159); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + x_160 = x_157; +} else { + lean_dec_ref(x_157); + x_160 = lean_box(0); +} +x_161 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_161, 0, x_159); +if (lean_is_scalar(x_160)) { + x_162 = lean_alloc_ctor(1, 1, 0); +} else { + x_162 = x_160; +} +lean_ctor_set(x_162, 0, x_161); +x_56 = x_162; +x_57 = x_158; +goto block_102; +} +} +block_102: +{ +if (lean_obj_tag(x_37) == 0) +{ +uint8_t x_58; +x_58 = !lean_is_exclusive(x_56); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_56, 0); +x_60 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_60, 0, x_31); +lean_ctor_set(x_60, 1, x_32); +lean_ctor_set(x_60, 2, x_38); +lean_ctor_set(x_60, 3, x_38); +lean_ctor_set(x_60, 4, x_38); +lean_ctor_set(x_60, 5, x_55); +lean_ctor_set(x_60, 6, x_59); +lean_ctor_set(x_60, 7, x_38); +lean_ctor_set(x_56, 0, x_60); +if (lean_is_scalar(x_53)) { + x_61 = lean_alloc_ctor(0, 2, 0); +} else { + x_61 = x_53; +} +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_57); +x_11 = x_61; +goto block_29; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_62 = lean_ctor_get(x_56, 0); +lean_inc(x_62); +lean_dec(x_56); +x_63 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_63, 0, x_31); +lean_ctor_set(x_63, 1, x_32); +lean_ctor_set(x_63, 2, x_38); +lean_ctor_set(x_63, 3, x_38); +lean_ctor_set(x_63, 4, x_38); +lean_ctor_set(x_63, 5, x_55); +lean_ctor_set(x_63, 6, x_62); +lean_ctor_set(x_63, 7, x_38); +x_64 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_64, 0, x_63); +if (lean_is_scalar(x_53)) { + x_65 = lean_alloc_ctor(0, 2, 0); +} else { + x_65 = x_53; +} +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_57); +x_11 = x_65; +goto block_29; +} +} +else +{ +lean_object* x_66; uint8_t x_67; +lean_dec(x_53); +x_66 = lean_ctor_get(x_56, 0); +lean_inc(x_66); +lean_dec(x_56); +x_67 = !lean_is_exclusive(x_37); +if (x_67 == 0) +{ +lean_object* x_68; lean_object* x_69; size_t x_70; size_t x_71; lean_object* x_72; uint8_t x_73; +x_68 = lean_ctor_get(x_37, 0); +x_69 = lean_array_get_size(x_68); +x_70 = lean_usize_of_nat(x_69); +lean_dec(x_69); +x_71 = 0; +x_72 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_70, x_71, x_68, x_57); +x_73 = !lean_is_exclusive(x_72); +if (x_73 == 0) +{ +lean_object* x_74; uint8_t x_75; +x_74 = lean_ctor_get(x_72, 0); +x_75 = !lean_is_exclusive(x_74); +if (x_75 == 0) +{ +lean_object* x_76; lean_object* x_77; +x_76 = lean_ctor_get(x_74, 0); +lean_ctor_set(x_37, 0, x_76); +x_77 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_77, 0, x_31); +lean_ctor_set(x_77, 1, x_32); +lean_ctor_set(x_77, 2, x_38); +lean_ctor_set(x_77, 3, x_38); +lean_ctor_set(x_77, 4, x_38); +lean_ctor_set(x_77, 5, x_55); +lean_ctor_set(x_77, 6, x_66); +lean_ctor_set(x_77, 7, x_37); +lean_ctor_set(x_74, 0, x_77); +x_11 = x_72; +goto block_29; +} +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_74, 0); +lean_inc(x_78); +lean_dec(x_74); +lean_ctor_set(x_37, 0, x_78); +x_79 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_79, 0, x_31); +lean_ctor_set(x_79, 1, x_32); +lean_ctor_set(x_79, 2, x_38); +lean_ctor_set(x_79, 3, x_38); +lean_ctor_set(x_79, 4, x_38); +lean_ctor_set(x_79, 5, x_55); +lean_ctor_set(x_79, 6, x_66); +lean_ctor_set(x_79, 7, x_37); +x_80 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_80, 0, x_79); +lean_ctor_set(x_72, 0, x_80); +x_11 = x_72; +goto block_29; +} +} +else +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_81 = lean_ctor_get(x_72, 0); +x_82 = lean_ctor_get(x_72, 1); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_72); +x_83 = lean_ctor_get(x_81, 0); +lean_inc(x_83); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + x_84 = x_81; +} else { + lean_dec_ref(x_81); + x_84 = lean_box(0); +} +lean_ctor_set(x_37, 0, x_83); +x_85 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_85, 0, x_31); +lean_ctor_set(x_85, 1, x_32); +lean_ctor_set(x_85, 2, x_38); +lean_ctor_set(x_85, 3, x_38); +lean_ctor_set(x_85, 4, x_38); +lean_ctor_set(x_85, 5, x_55); +lean_ctor_set(x_85, 6, x_66); +lean_ctor_set(x_85, 7, x_37); +if (lean_is_scalar(x_84)) { + x_86 = lean_alloc_ctor(1, 1, 0); +} else { + x_86 = x_84; +} +lean_ctor_set(x_86, 0, x_85); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_82); +x_11 = x_87; +goto block_29; +} +} +else +{ +lean_object* x_88; lean_object* x_89; size_t x_90; size_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_88 = lean_ctor_get(x_37, 0); +lean_inc(x_88); +lean_dec(x_37); +x_89 = lean_array_get_size(x_88); +x_90 = lean_usize_of_nat(x_89); +lean_dec(x_89); +x_91 = 0; +x_92 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_90, x_91, x_88, x_57); +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_95 = x_92; +} else { + lean_dec_ref(x_92); + x_95 = lean_box(0); +} +x_96 = lean_ctor_get(x_93, 0); +lean_inc(x_96); +if (lean_is_exclusive(x_93)) { + lean_ctor_release(x_93, 0); + x_97 = x_93; +} else { + lean_dec_ref(x_93); + x_97 = lean_box(0); +} +x_98 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_98, 0, x_96); +x_99 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_99, 0, x_31); +lean_ctor_set(x_99, 1, x_32); +lean_ctor_set(x_99, 2, x_38); +lean_ctor_set(x_99, 3, x_38); +lean_ctor_set(x_99, 4, x_38); +lean_ctor_set(x_99, 5, x_55); +lean_ctor_set(x_99, 6, x_66); +lean_ctor_set(x_99, 7, x_98); +if (lean_is_scalar(x_97)) { + x_100 = lean_alloc_ctor(1, 1, 0); +} else { + x_100 = x_97; +} +lean_ctor_set(x_100, 0, x_99); +if (lean_is_scalar(x_95)) { + x_101 = lean_alloc_ctor(0, 2, 0); +} else { + x_101 = x_95; +} +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_94); +x_11 = x_101; +goto block_29; +} +} +} +} +else +{ +lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_163 = lean_ctor_get(x_41, 0); +lean_inc(x_163); +lean_dec(x_41); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_53); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_188 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_188, 0, x_31); +lean_ctor_set(x_188, 1, x_32); +lean_ctor_set(x_188, 2, x_38); +lean_ctor_set(x_188, 3, x_38); +lean_ctor_set(x_188, 4, x_38); +lean_ctor_set(x_188, 5, x_163); +lean_ctor_set(x_188, 6, x_38); +lean_ctor_set(x_188, 7, x_38); +x_189 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_189, 0, x_188); +x_190 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_190, 0, x_189); +lean_ctor_set(x_190, 1, x_52); +x_11 = x_190; +goto block_29; +} +else +{ +lean_object* x_191; lean_object* x_192; lean_object* x_193; size_t x_194; size_t x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; +x_191 = lean_ctor_get(x_37, 0); +lean_inc(x_191); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_192 = x_37; +} else { + lean_dec_ref(x_37); + x_192 = lean_box(0); +} +x_193 = lean_array_get_size(x_191); +x_194 = lean_usize_of_nat(x_193); +lean_dec(x_193); +x_195 = 0; +x_196 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_194, x_195, x_191, x_52); +x_197 = lean_ctor_get(x_196, 0); +lean_inc(x_197); +x_198 = lean_ctor_get(x_196, 1); +lean_inc(x_198); +if (lean_is_exclusive(x_196)) { + lean_ctor_release(x_196, 0); + lean_ctor_release(x_196, 1); + x_199 = x_196; +} else { + lean_dec_ref(x_196); + x_199 = lean_box(0); +} +x_200 = lean_ctor_get(x_197, 0); +lean_inc(x_200); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + x_201 = x_197; +} else { + lean_dec_ref(x_197); + x_201 = lean_box(0); +} +if (lean_is_scalar(x_192)) { + x_202 = lean_alloc_ctor(1, 1, 0); +} else { + x_202 = x_192; +} +lean_ctor_set(x_202, 0, x_200); +x_203 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_203, 0, x_31); +lean_ctor_set(x_203, 1, x_32); +lean_ctor_set(x_203, 2, x_38); +lean_ctor_set(x_203, 3, x_38); +lean_ctor_set(x_203, 4, x_38); +lean_ctor_set(x_203, 5, x_163); +lean_ctor_set(x_203, 6, x_38); +lean_ctor_set(x_203, 7, x_202); +if (lean_is_scalar(x_201)) { + x_204 = lean_alloc_ctor(1, 1, 0); +} else { + x_204 = x_201; +} +lean_ctor_set(x_204, 0, x_203); +if (lean_is_scalar(x_199)) { + x_205 = lean_alloc_ctor(0, 2, 0); +} else { + x_205 = x_199; +} +lean_ctor_set(x_205, 0, x_204); +lean_ctor_set(x_205, 1, x_198); +x_11 = x_205; +goto block_29; +} +} +else +{ +lean_object* x_206; lean_object* x_207; lean_object* x_208; size_t x_209; size_t x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; +x_206 = lean_ctor_get(x_36, 0); +lean_inc(x_206); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_207 = x_36; +} else { + lean_dec_ref(x_36); + x_207 = lean_box(0); +} +x_208 = lean_array_get_size(x_206); +x_209 = lean_usize_of_nat(x_208); +lean_dec(x_208); +x_210 = 0; +x_211 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_209, x_210, x_206, x_52); +x_212 = lean_ctor_get(x_211, 0); +lean_inc(x_212); +x_213 = lean_ctor_get(x_211, 1); +lean_inc(x_213); +lean_dec(x_211); +x_214 = lean_ctor_get(x_212, 0); +lean_inc(x_214); +if (lean_is_exclusive(x_212)) { + lean_ctor_release(x_212, 0); + x_215 = x_212; +} else { + lean_dec_ref(x_212); + x_215 = lean_box(0); +} +if (lean_is_scalar(x_207)) { + x_216 = lean_alloc_ctor(1, 1, 0); +} else { + x_216 = x_207; +} +lean_ctor_set(x_216, 0, x_214); +if (lean_is_scalar(x_215)) { + x_217 = lean_alloc_ctor(1, 1, 0); +} else { + x_217 = x_215; +} +lean_ctor_set(x_217, 0, x_216); +x_164 = x_217; +x_165 = x_213; +goto block_187; +} +block_187: +{ +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; +x_166 = lean_ctor_get(x_164, 0); +lean_inc(x_166); +if (lean_is_exclusive(x_164)) { + lean_ctor_release(x_164, 0); + x_167 = x_164; +} else { + lean_dec_ref(x_164); + x_167 = lean_box(0); +} +x_168 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_168, 0, x_31); +lean_ctor_set(x_168, 1, x_32); +lean_ctor_set(x_168, 2, x_38); +lean_ctor_set(x_168, 3, x_38); +lean_ctor_set(x_168, 4, x_38); +lean_ctor_set(x_168, 5, x_163); +lean_ctor_set(x_168, 6, x_166); +lean_ctor_set(x_168, 7, x_38); +if (lean_is_scalar(x_167)) { + x_169 = lean_alloc_ctor(1, 1, 0); +} else { + x_169 = x_167; +} +lean_ctor_set(x_169, 0, x_168); +if (lean_is_scalar(x_53)) { + x_170 = lean_alloc_ctor(0, 2, 0); +} else { + x_170 = x_53; +} +lean_ctor_set(x_170, 0, x_169); +lean_ctor_set(x_170, 1, x_165); +x_11 = x_170; +goto block_29; +} +else +{ +lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; size_t x_175; size_t 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_dec(x_53); +x_171 = lean_ctor_get(x_164, 0); +lean_inc(x_171); +lean_dec(x_164); +x_172 = lean_ctor_get(x_37, 0); +lean_inc(x_172); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_173 = x_37; +} else { + lean_dec_ref(x_37); + x_173 = lean_box(0); +} +x_174 = lean_array_get_size(x_172); +x_175 = lean_usize_of_nat(x_174); +lean_dec(x_174); +x_176 = 0; +x_177 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_175, x_176, x_172, x_165); +x_178 = lean_ctor_get(x_177, 0); +lean_inc(x_178); +x_179 = lean_ctor_get(x_177, 1); +lean_inc(x_179); +if (lean_is_exclusive(x_177)) { + lean_ctor_release(x_177, 0); + lean_ctor_release(x_177, 1); + x_180 = x_177; +} else { + lean_dec_ref(x_177); + x_180 = lean_box(0); +} +x_181 = lean_ctor_get(x_178, 0); +lean_inc(x_181); +if (lean_is_exclusive(x_178)) { + lean_ctor_release(x_178, 0); + x_182 = x_178; +} else { + lean_dec_ref(x_178); + x_182 = lean_box(0); +} +if (lean_is_scalar(x_173)) { + x_183 = lean_alloc_ctor(1, 1, 0); +} else { + x_183 = x_173; +} +lean_ctor_set(x_183, 0, x_181); +x_184 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_184, 0, x_31); +lean_ctor_set(x_184, 1, x_32); +lean_ctor_set(x_184, 2, x_38); +lean_ctor_set(x_184, 3, x_38); +lean_ctor_set(x_184, 4, x_38); +lean_ctor_set(x_184, 5, x_163); +lean_ctor_set(x_184, 6, x_171); +lean_ctor_set(x_184, 7, x_183); +if (lean_is_scalar(x_182)) { + x_185 = lean_alloc_ctor(1, 1, 0); +} else { + x_185 = x_182; +} +lean_ctor_set(x_185, 0, x_184); +if (lean_is_scalar(x_180)) { + x_186 = lean_alloc_ctor(0, 2, 0); +} else { + x_186 = x_180; +} +lean_ctor_set(x_186, 0, x_185); +lean_ctor_set(x_186, 1, x_179); +x_11 = x_186; +goto block_29; +} +} +} +} +} +else +{ +uint8_t x_218; +x_218 = !lean_is_exclusive(x_34); +if (x_218 == 0) +{ +lean_object* x_219; lean_object* x_220; lean_object* x_221; +x_219 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_220 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_219, x_35, x_4); +x_221 = lean_ctor_get(x_220, 0); +lean_inc(x_221); +if (lean_obj_tag(x_221) == 0) +{ +uint8_t x_222; +lean_dec(x_34); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_32); +lean_dec(x_31); +x_222 = !lean_is_exclusive(x_220); +if (x_222 == 0) +{ +lean_object* x_223; uint8_t x_224; +x_223 = lean_ctor_get(x_220, 0); +lean_dec(x_223); +x_224 = !lean_is_exclusive(x_221); +if (x_224 == 0) +{ +x_11 = x_220; +goto block_29; +} +else +{ +lean_object* x_225; lean_object* x_226; +x_225 = lean_ctor_get(x_221, 0); +lean_inc(x_225); +lean_dec(x_221); +x_226 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_226, 0, x_225); +lean_ctor_set(x_220, 0, x_226); +x_11 = x_220; +goto block_29; +} +} +else +{ +lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; +x_227 = lean_ctor_get(x_220, 1); +lean_inc(x_227); +lean_dec(x_220); +x_228 = lean_ctor_get(x_221, 0); +lean_inc(x_228); +if (lean_is_exclusive(x_221)) { + lean_ctor_release(x_221, 0); + x_229 = x_221; +} else { + lean_dec_ref(x_221); + x_229 = lean_box(0); +} +if (lean_is_scalar(x_229)) { + x_230 = lean_alloc_ctor(0, 1, 0); +} else { + x_230 = x_229; +} +lean_ctor_set(x_230, 0, x_228); +x_231 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_231, 0, x_230); +lean_ctor_set(x_231, 1, x_227); +x_11 = x_231; +goto block_29; +} +} +else +{ +lean_object* x_232; lean_object* x_233; uint8_t x_234; +x_232 = lean_ctor_get(x_220, 1); +lean_inc(x_232); +if (lean_is_exclusive(x_220)) { + lean_ctor_release(x_220, 0); + lean_ctor_release(x_220, 1); + x_233 = x_220; +} else { + lean_dec_ref(x_220); + x_233 = lean_box(0); +} +x_234 = !lean_is_exclusive(x_221); +if (x_234 == 0) +{ +lean_object* x_235; lean_object* x_236; lean_object* x_237; +x_235 = lean_ctor_get(x_221, 0); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_233); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_283; lean_object* x_284; +x_283 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_283, 0, x_31); +lean_ctor_set(x_283, 1, x_32); +lean_ctor_set(x_283, 2, x_38); +lean_ctor_set(x_283, 3, x_38); +lean_ctor_set(x_283, 4, x_34); +lean_ctor_set(x_283, 5, x_235); +lean_ctor_set(x_283, 6, x_38); +lean_ctor_set(x_283, 7, x_38); +lean_ctor_set(x_221, 0, x_283); +x_284 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_284, 0, x_221); +lean_ctor_set(x_284, 1, x_232); +x_11 = x_284; +goto block_29; +} +else +{ +uint8_t x_285; +lean_free_object(x_221); +x_285 = !lean_is_exclusive(x_37); +if (x_285 == 0) +{ +lean_object* x_286; lean_object* x_287; size_t x_288; size_t x_289; lean_object* x_290; uint8_t x_291; +x_286 = lean_ctor_get(x_37, 0); +x_287 = lean_array_get_size(x_286); +x_288 = lean_usize_of_nat(x_287); +lean_dec(x_287); +x_289 = 0; +x_290 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_288, x_289, x_286, x_232); +x_291 = !lean_is_exclusive(x_290); +if (x_291 == 0) +{ +lean_object* x_292; uint8_t x_293; +x_292 = lean_ctor_get(x_290, 0); +x_293 = !lean_is_exclusive(x_292); +if (x_293 == 0) +{ +lean_object* x_294; lean_object* x_295; +x_294 = lean_ctor_get(x_292, 0); +lean_ctor_set(x_37, 0, x_294); +x_295 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_295, 0, x_31); +lean_ctor_set(x_295, 1, x_32); +lean_ctor_set(x_295, 2, x_38); +lean_ctor_set(x_295, 3, x_38); +lean_ctor_set(x_295, 4, x_34); +lean_ctor_set(x_295, 5, x_235); +lean_ctor_set(x_295, 6, x_38); +lean_ctor_set(x_295, 7, x_37); +lean_ctor_set(x_292, 0, x_295); +x_11 = x_290; +goto block_29; +} +else +{ +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_292, 0); +lean_inc(x_296); +lean_dec(x_292); +lean_ctor_set(x_37, 0, x_296); +x_297 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_297, 0, x_31); +lean_ctor_set(x_297, 1, x_32); +lean_ctor_set(x_297, 2, x_38); +lean_ctor_set(x_297, 3, x_38); +lean_ctor_set(x_297, 4, x_34); +lean_ctor_set(x_297, 5, x_235); +lean_ctor_set(x_297, 6, x_38); +lean_ctor_set(x_297, 7, x_37); +x_298 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_298, 0, x_297); +lean_ctor_set(x_290, 0, x_298); +x_11 = x_290; +goto block_29; +} +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; +x_299 = lean_ctor_get(x_290, 0); +x_300 = lean_ctor_get(x_290, 1); +lean_inc(x_300); +lean_inc(x_299); +lean_dec(x_290); +x_301 = lean_ctor_get(x_299, 0); +lean_inc(x_301); +if (lean_is_exclusive(x_299)) { + lean_ctor_release(x_299, 0); + x_302 = x_299; +} else { + lean_dec_ref(x_299); + x_302 = lean_box(0); +} +lean_ctor_set(x_37, 0, x_301); +x_303 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_303, 0, x_31); +lean_ctor_set(x_303, 1, x_32); +lean_ctor_set(x_303, 2, x_38); +lean_ctor_set(x_303, 3, x_38); +lean_ctor_set(x_303, 4, x_34); +lean_ctor_set(x_303, 5, x_235); +lean_ctor_set(x_303, 6, x_38); +lean_ctor_set(x_303, 7, x_37); +if (lean_is_scalar(x_302)) { + x_304 = lean_alloc_ctor(1, 1, 0); +} else { + x_304 = x_302; +} +lean_ctor_set(x_304, 0, x_303); +x_305 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_305, 0, x_304); +lean_ctor_set(x_305, 1, x_300); +x_11 = x_305; +goto block_29; +} +} +else +{ +lean_object* x_306; lean_object* x_307; size_t x_308; size_t x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; +x_306 = lean_ctor_get(x_37, 0); +lean_inc(x_306); +lean_dec(x_37); +x_307 = lean_array_get_size(x_306); +x_308 = lean_usize_of_nat(x_307); +lean_dec(x_307); +x_309 = 0; +x_310 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_308, x_309, x_306, x_232); +x_311 = lean_ctor_get(x_310, 0); +lean_inc(x_311); +x_312 = lean_ctor_get(x_310, 1); +lean_inc(x_312); +if (lean_is_exclusive(x_310)) { + lean_ctor_release(x_310, 0); + lean_ctor_release(x_310, 1); + x_313 = x_310; +} else { + lean_dec_ref(x_310); + x_313 = lean_box(0); +} +x_314 = lean_ctor_get(x_311, 0); +lean_inc(x_314); +if (lean_is_exclusive(x_311)) { + lean_ctor_release(x_311, 0); + x_315 = x_311; +} else { + lean_dec_ref(x_311); + x_315 = lean_box(0); +} +x_316 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_316, 0, x_314); +x_317 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_317, 0, x_31); +lean_ctor_set(x_317, 1, x_32); +lean_ctor_set(x_317, 2, x_38); +lean_ctor_set(x_317, 3, x_38); +lean_ctor_set(x_317, 4, x_34); +lean_ctor_set(x_317, 5, x_235); +lean_ctor_set(x_317, 6, x_38); +lean_ctor_set(x_317, 7, x_316); +if (lean_is_scalar(x_315)) { + x_318 = lean_alloc_ctor(1, 1, 0); +} else { + x_318 = x_315; +} +lean_ctor_set(x_318, 0, x_317); +if (lean_is_scalar(x_313)) { + x_319 = lean_alloc_ctor(0, 2, 0); +} else { + x_319 = x_313; +} +lean_ctor_set(x_319, 0, x_318); +lean_ctor_set(x_319, 1, x_312); +x_11 = x_319; +goto block_29; +} +} +} +else +{ +uint8_t x_320; +lean_free_object(x_221); +x_320 = !lean_is_exclusive(x_36); +if (x_320 == 0) +{ +lean_object* x_321; lean_object* x_322; size_t x_323; size_t x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; uint8_t x_328; +x_321 = lean_ctor_get(x_36, 0); +x_322 = lean_array_get_size(x_321); +x_323 = lean_usize_of_nat(x_322); +lean_dec(x_322); +x_324 = 0; +x_325 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_323, x_324, x_321, x_232); +x_326 = lean_ctor_get(x_325, 0); +lean_inc(x_326); +x_327 = lean_ctor_get(x_325, 1); +lean_inc(x_327); +lean_dec(x_325); +x_328 = !lean_is_exclusive(x_326); +if (x_328 == 0) +{ +lean_object* x_329; +x_329 = lean_ctor_get(x_326, 0); +lean_ctor_set(x_36, 0, x_329); +lean_ctor_set(x_326, 0, x_36); +x_236 = x_326; +x_237 = x_327; +goto block_282; +} +else +{ +lean_object* x_330; lean_object* x_331; +x_330 = lean_ctor_get(x_326, 0); +lean_inc(x_330); +lean_dec(x_326); +lean_ctor_set(x_36, 0, x_330); +x_331 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_331, 0, x_36); +x_236 = x_331; +x_237 = x_327; +goto block_282; +} +} +else +{ +lean_object* x_332; lean_object* x_333; size_t x_334; size_t x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; +x_332 = lean_ctor_get(x_36, 0); +lean_inc(x_332); +lean_dec(x_36); +x_333 = lean_array_get_size(x_332); +x_334 = lean_usize_of_nat(x_333); +lean_dec(x_333); +x_335 = 0; +x_336 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_334, x_335, x_332, x_232); +x_337 = lean_ctor_get(x_336, 0); +lean_inc(x_337); +x_338 = lean_ctor_get(x_336, 1); +lean_inc(x_338); +lean_dec(x_336); +x_339 = lean_ctor_get(x_337, 0); +lean_inc(x_339); +if (lean_is_exclusive(x_337)) { + lean_ctor_release(x_337, 0); + x_340 = x_337; +} else { + lean_dec_ref(x_337); + x_340 = lean_box(0); +} +x_341 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_341, 0, x_339); +if (lean_is_scalar(x_340)) { + x_342 = lean_alloc_ctor(1, 1, 0); +} else { + x_342 = x_340; +} +lean_ctor_set(x_342, 0, x_341); +x_236 = x_342; +x_237 = x_338; +goto block_282; +} +} +block_282: +{ +if (lean_obj_tag(x_37) == 0) +{ +uint8_t x_238; +x_238 = !lean_is_exclusive(x_236); +if (x_238 == 0) +{ +lean_object* x_239; lean_object* x_240; lean_object* x_241; +x_239 = lean_ctor_get(x_236, 0); +x_240 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_240, 0, x_31); +lean_ctor_set(x_240, 1, x_32); +lean_ctor_set(x_240, 2, x_38); +lean_ctor_set(x_240, 3, x_38); +lean_ctor_set(x_240, 4, x_34); +lean_ctor_set(x_240, 5, x_235); +lean_ctor_set(x_240, 6, x_239); +lean_ctor_set(x_240, 7, x_38); +lean_ctor_set(x_236, 0, x_240); +if (lean_is_scalar(x_233)) { + x_241 = lean_alloc_ctor(0, 2, 0); +} else { + x_241 = x_233; +} +lean_ctor_set(x_241, 0, x_236); +lean_ctor_set(x_241, 1, x_237); +x_11 = x_241; +goto block_29; +} +else +{ +lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; +x_242 = lean_ctor_get(x_236, 0); +lean_inc(x_242); +lean_dec(x_236); +x_243 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_243, 0, x_31); +lean_ctor_set(x_243, 1, x_32); +lean_ctor_set(x_243, 2, x_38); +lean_ctor_set(x_243, 3, x_38); +lean_ctor_set(x_243, 4, x_34); +lean_ctor_set(x_243, 5, x_235); +lean_ctor_set(x_243, 6, x_242); +lean_ctor_set(x_243, 7, x_38); +x_244 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_244, 0, x_243); +if (lean_is_scalar(x_233)) { + x_245 = lean_alloc_ctor(0, 2, 0); +} else { + x_245 = x_233; +} +lean_ctor_set(x_245, 0, x_244); +lean_ctor_set(x_245, 1, x_237); +x_11 = x_245; +goto block_29; +} +} +else +{ +lean_object* x_246; uint8_t x_247; +lean_dec(x_233); +x_246 = lean_ctor_get(x_236, 0); +lean_inc(x_246); +lean_dec(x_236); +x_247 = !lean_is_exclusive(x_37); +if (x_247 == 0) +{ +lean_object* x_248; lean_object* x_249; size_t x_250; size_t x_251; lean_object* x_252; uint8_t x_253; +x_248 = lean_ctor_get(x_37, 0); +x_249 = lean_array_get_size(x_248); +x_250 = lean_usize_of_nat(x_249); +lean_dec(x_249); +x_251 = 0; +x_252 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_250, x_251, x_248, x_237); +x_253 = !lean_is_exclusive(x_252); +if (x_253 == 0) +{ +lean_object* x_254; uint8_t x_255; +x_254 = lean_ctor_get(x_252, 0); +x_255 = !lean_is_exclusive(x_254); +if (x_255 == 0) +{ +lean_object* x_256; lean_object* x_257; +x_256 = lean_ctor_get(x_254, 0); +lean_ctor_set(x_37, 0, x_256); +x_257 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_257, 0, x_31); +lean_ctor_set(x_257, 1, x_32); +lean_ctor_set(x_257, 2, x_38); +lean_ctor_set(x_257, 3, x_38); +lean_ctor_set(x_257, 4, x_34); +lean_ctor_set(x_257, 5, x_235); +lean_ctor_set(x_257, 6, x_246); +lean_ctor_set(x_257, 7, x_37); +lean_ctor_set(x_254, 0, x_257); +x_11 = x_252; +goto block_29; +} +else +{ +lean_object* x_258; lean_object* x_259; lean_object* x_260; +x_258 = lean_ctor_get(x_254, 0); +lean_inc(x_258); +lean_dec(x_254); +lean_ctor_set(x_37, 0, x_258); +x_259 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_259, 0, x_31); +lean_ctor_set(x_259, 1, x_32); +lean_ctor_set(x_259, 2, x_38); +lean_ctor_set(x_259, 3, x_38); +lean_ctor_set(x_259, 4, x_34); +lean_ctor_set(x_259, 5, x_235); +lean_ctor_set(x_259, 6, x_246); +lean_ctor_set(x_259, 7, x_37); +x_260 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_260, 0, x_259); +lean_ctor_set(x_252, 0, x_260); +x_11 = x_252; +goto block_29; +} +} +else +{ +lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; +x_261 = lean_ctor_get(x_252, 0); +x_262 = lean_ctor_get(x_252, 1); +lean_inc(x_262); +lean_inc(x_261); +lean_dec(x_252); +x_263 = lean_ctor_get(x_261, 0); +lean_inc(x_263); +if (lean_is_exclusive(x_261)) { + lean_ctor_release(x_261, 0); + x_264 = x_261; +} else { + lean_dec_ref(x_261); + x_264 = lean_box(0); +} +lean_ctor_set(x_37, 0, x_263); +x_265 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_265, 0, x_31); +lean_ctor_set(x_265, 1, x_32); +lean_ctor_set(x_265, 2, x_38); +lean_ctor_set(x_265, 3, x_38); +lean_ctor_set(x_265, 4, x_34); +lean_ctor_set(x_265, 5, x_235); +lean_ctor_set(x_265, 6, x_246); +lean_ctor_set(x_265, 7, x_37); +if (lean_is_scalar(x_264)) { + x_266 = lean_alloc_ctor(1, 1, 0); +} else { + x_266 = x_264; +} +lean_ctor_set(x_266, 0, x_265); +x_267 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_267, 0, x_266); +lean_ctor_set(x_267, 1, x_262); +x_11 = x_267; +goto block_29; +} +} +else +{ +lean_object* x_268; lean_object* x_269; size_t x_270; size_t x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_268 = lean_ctor_get(x_37, 0); +lean_inc(x_268); +lean_dec(x_37); +x_269 = lean_array_get_size(x_268); +x_270 = lean_usize_of_nat(x_269); +lean_dec(x_269); +x_271 = 0; +x_272 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_270, x_271, x_268, x_237); +x_273 = lean_ctor_get(x_272, 0); +lean_inc(x_273); +x_274 = lean_ctor_get(x_272, 1); +lean_inc(x_274); +if (lean_is_exclusive(x_272)) { + lean_ctor_release(x_272, 0); + lean_ctor_release(x_272, 1); + x_275 = x_272; +} else { + lean_dec_ref(x_272); + x_275 = lean_box(0); +} +x_276 = lean_ctor_get(x_273, 0); +lean_inc(x_276); +if (lean_is_exclusive(x_273)) { + lean_ctor_release(x_273, 0); + x_277 = x_273; +} else { + lean_dec_ref(x_273); + x_277 = lean_box(0); +} +x_278 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_278, 0, x_276); +x_279 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_279, 0, x_31); +lean_ctor_set(x_279, 1, x_32); +lean_ctor_set(x_279, 2, x_38); +lean_ctor_set(x_279, 3, x_38); +lean_ctor_set(x_279, 4, x_34); +lean_ctor_set(x_279, 5, x_235); +lean_ctor_set(x_279, 6, x_246); +lean_ctor_set(x_279, 7, x_278); +if (lean_is_scalar(x_277)) { + x_280 = lean_alloc_ctor(1, 1, 0); +} else { + x_280 = x_277; +} +lean_ctor_set(x_280, 0, x_279); +if (lean_is_scalar(x_275)) { + x_281 = lean_alloc_ctor(0, 2, 0); +} else { + x_281 = x_275; +} +lean_ctor_set(x_281, 0, x_280); +lean_ctor_set(x_281, 1, x_274); +x_11 = x_281; +goto block_29; +} +} +} +} +else +{ +lean_object* x_343; lean_object* x_344; lean_object* x_345; +x_343 = lean_ctor_get(x_221, 0); +lean_inc(x_343); +lean_dec(x_221); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_233); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_368; lean_object* x_369; lean_object* x_370; +x_368 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_368, 0, x_31); +lean_ctor_set(x_368, 1, x_32); +lean_ctor_set(x_368, 2, x_38); +lean_ctor_set(x_368, 3, x_38); +lean_ctor_set(x_368, 4, x_34); +lean_ctor_set(x_368, 5, x_343); +lean_ctor_set(x_368, 6, x_38); +lean_ctor_set(x_368, 7, x_38); +x_369 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_369, 0, x_368); +x_370 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_370, 0, x_369); +lean_ctor_set(x_370, 1, x_232); +x_11 = x_370; +goto block_29; +} +else +{ +lean_object* x_371; lean_object* x_372; lean_object* x_373; size_t x_374; size_t x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; +x_371 = lean_ctor_get(x_37, 0); +lean_inc(x_371); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_372 = x_37; +} else { + lean_dec_ref(x_37); + x_372 = lean_box(0); +} +x_373 = lean_array_get_size(x_371); +x_374 = lean_usize_of_nat(x_373); +lean_dec(x_373); +x_375 = 0; +x_376 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_374, x_375, x_371, x_232); +x_377 = lean_ctor_get(x_376, 0); +lean_inc(x_377); +x_378 = lean_ctor_get(x_376, 1); +lean_inc(x_378); +if (lean_is_exclusive(x_376)) { + lean_ctor_release(x_376, 0); + lean_ctor_release(x_376, 1); + x_379 = x_376; +} else { + lean_dec_ref(x_376); + x_379 = lean_box(0); +} +x_380 = lean_ctor_get(x_377, 0); +lean_inc(x_380); +if (lean_is_exclusive(x_377)) { + lean_ctor_release(x_377, 0); + x_381 = x_377; +} else { + lean_dec_ref(x_377); + x_381 = lean_box(0); +} +if (lean_is_scalar(x_372)) { + x_382 = lean_alloc_ctor(1, 1, 0); +} else { + x_382 = x_372; +} +lean_ctor_set(x_382, 0, x_380); +x_383 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_383, 0, x_31); +lean_ctor_set(x_383, 1, x_32); +lean_ctor_set(x_383, 2, x_38); +lean_ctor_set(x_383, 3, x_38); +lean_ctor_set(x_383, 4, x_34); +lean_ctor_set(x_383, 5, x_343); +lean_ctor_set(x_383, 6, x_38); +lean_ctor_set(x_383, 7, x_382); +if (lean_is_scalar(x_381)) { + x_384 = lean_alloc_ctor(1, 1, 0); +} else { + x_384 = x_381; +} +lean_ctor_set(x_384, 0, x_383); +if (lean_is_scalar(x_379)) { + x_385 = lean_alloc_ctor(0, 2, 0); +} else { + x_385 = x_379; +} +lean_ctor_set(x_385, 0, x_384); +lean_ctor_set(x_385, 1, x_378); +x_11 = x_385; +goto block_29; +} +} +else +{ +lean_object* x_386; lean_object* x_387; lean_object* x_388; size_t x_389; size_t x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; +x_386 = lean_ctor_get(x_36, 0); +lean_inc(x_386); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_387 = x_36; +} else { + lean_dec_ref(x_36); + x_387 = lean_box(0); +} +x_388 = lean_array_get_size(x_386); +x_389 = lean_usize_of_nat(x_388); +lean_dec(x_388); +x_390 = 0; +x_391 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_389, x_390, x_386, x_232); +x_392 = lean_ctor_get(x_391, 0); +lean_inc(x_392); +x_393 = lean_ctor_get(x_391, 1); +lean_inc(x_393); +lean_dec(x_391); +x_394 = lean_ctor_get(x_392, 0); +lean_inc(x_394); +if (lean_is_exclusive(x_392)) { + lean_ctor_release(x_392, 0); + x_395 = x_392; +} else { + lean_dec_ref(x_392); + x_395 = lean_box(0); +} +if (lean_is_scalar(x_387)) { + x_396 = lean_alloc_ctor(1, 1, 0); +} else { + x_396 = x_387; +} +lean_ctor_set(x_396, 0, x_394); +if (lean_is_scalar(x_395)) { + x_397 = lean_alloc_ctor(1, 1, 0); +} else { + x_397 = x_395; +} +lean_ctor_set(x_397, 0, x_396); +x_344 = x_397; +x_345 = x_393; +goto block_367; +} +block_367: +{ +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; +x_346 = lean_ctor_get(x_344, 0); +lean_inc(x_346); +if (lean_is_exclusive(x_344)) { + lean_ctor_release(x_344, 0); + x_347 = x_344; +} else { + lean_dec_ref(x_344); + x_347 = lean_box(0); +} +x_348 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_348, 0, x_31); +lean_ctor_set(x_348, 1, x_32); +lean_ctor_set(x_348, 2, x_38); +lean_ctor_set(x_348, 3, x_38); +lean_ctor_set(x_348, 4, x_34); +lean_ctor_set(x_348, 5, x_343); +lean_ctor_set(x_348, 6, x_346); +lean_ctor_set(x_348, 7, x_38); +if (lean_is_scalar(x_347)) { + x_349 = lean_alloc_ctor(1, 1, 0); +} else { + x_349 = x_347; +} +lean_ctor_set(x_349, 0, x_348); +if (lean_is_scalar(x_233)) { + x_350 = lean_alloc_ctor(0, 2, 0); +} else { + x_350 = x_233; +} +lean_ctor_set(x_350, 0, x_349); +lean_ctor_set(x_350, 1, x_345); +x_11 = x_350; +goto block_29; +} +else +{ +lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; size_t x_355; size_t x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; +lean_dec(x_233); +x_351 = lean_ctor_get(x_344, 0); +lean_inc(x_351); +lean_dec(x_344); +x_352 = lean_ctor_get(x_37, 0); +lean_inc(x_352); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_353 = x_37; +} else { + lean_dec_ref(x_37); + x_353 = lean_box(0); +} +x_354 = lean_array_get_size(x_352); +x_355 = lean_usize_of_nat(x_354); +lean_dec(x_354); +x_356 = 0; +x_357 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_355, x_356, x_352, x_345); +x_358 = lean_ctor_get(x_357, 0); +lean_inc(x_358); +x_359 = lean_ctor_get(x_357, 1); +lean_inc(x_359); +if (lean_is_exclusive(x_357)) { + lean_ctor_release(x_357, 0); + lean_ctor_release(x_357, 1); + x_360 = x_357; +} else { + lean_dec_ref(x_357); + x_360 = lean_box(0); +} +x_361 = lean_ctor_get(x_358, 0); +lean_inc(x_361); +if (lean_is_exclusive(x_358)) { + lean_ctor_release(x_358, 0); + x_362 = x_358; +} else { + lean_dec_ref(x_358); + x_362 = lean_box(0); +} +if (lean_is_scalar(x_353)) { + x_363 = lean_alloc_ctor(1, 1, 0); +} else { + x_363 = x_353; +} +lean_ctor_set(x_363, 0, x_361); +x_364 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_364, 0, x_31); +lean_ctor_set(x_364, 1, x_32); +lean_ctor_set(x_364, 2, x_38); +lean_ctor_set(x_364, 3, x_38); +lean_ctor_set(x_364, 4, x_34); +lean_ctor_set(x_364, 5, x_343); +lean_ctor_set(x_364, 6, x_351); +lean_ctor_set(x_364, 7, x_363); +if (lean_is_scalar(x_362)) { + x_365 = lean_alloc_ctor(1, 1, 0); +} else { + x_365 = x_362; +} +lean_ctor_set(x_365, 0, x_364); +if (lean_is_scalar(x_360)) { + x_366 = lean_alloc_ctor(0, 2, 0); +} else { + x_366 = x_360; +} +lean_ctor_set(x_366, 0, x_365); +lean_ctor_set(x_366, 1, x_359); +x_11 = x_366; +goto block_29; +} +} +} +} +} +else +{ +lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; +x_398 = lean_ctor_get(x_34, 0); +lean_inc(x_398); +lean_dec(x_34); +x_399 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_399, 0, x_398); +x_400 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_401 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_400, x_35, x_4); +x_402 = lean_ctor_get(x_401, 0); +lean_inc(x_402); +if (lean_obj_tag(x_402) == 0) +{ +lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; +lean_dec(x_399); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_32); +lean_dec(x_31); +x_403 = lean_ctor_get(x_401, 1); +lean_inc(x_403); +if (lean_is_exclusive(x_401)) { + lean_ctor_release(x_401, 0); + lean_ctor_release(x_401, 1); + x_404 = x_401; +} else { + lean_dec_ref(x_401); + x_404 = lean_box(0); +} +x_405 = lean_ctor_get(x_402, 0); +lean_inc(x_405); +if (lean_is_exclusive(x_402)) { + lean_ctor_release(x_402, 0); + x_406 = x_402; +} else { + lean_dec_ref(x_402); + x_406 = lean_box(0); +} +if (lean_is_scalar(x_406)) { + x_407 = lean_alloc_ctor(0, 1, 0); +} else { + x_407 = x_406; +} +lean_ctor_set(x_407, 0, x_405); +if (lean_is_scalar(x_404)) { + x_408 = lean_alloc_ctor(0, 2, 0); +} else { + x_408 = x_404; +} +lean_ctor_set(x_408, 0, x_407); +lean_ctor_set(x_408, 1, x_403); +x_11 = x_408; +goto block_29; +} +else +{ +lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; +x_409 = lean_ctor_get(x_401, 1); +lean_inc(x_409); +if (lean_is_exclusive(x_401)) { + lean_ctor_release(x_401, 0); + lean_ctor_release(x_401, 1); + x_410 = x_401; +} else { + lean_dec_ref(x_401); + x_410 = lean_box(0); +} +x_411 = lean_ctor_get(x_402, 0); +lean_inc(x_411); +if (lean_is_exclusive(x_402)) { + lean_ctor_release(x_402, 0); + x_412 = x_402; +} else { + lean_dec_ref(x_402); + x_412 = lean_box(0); +} +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_410); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_437; lean_object* x_438; lean_object* x_439; +x_437 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_437, 0, x_31); +lean_ctor_set(x_437, 1, x_32); +lean_ctor_set(x_437, 2, x_38); +lean_ctor_set(x_437, 3, x_38); +lean_ctor_set(x_437, 4, x_399); +lean_ctor_set(x_437, 5, x_411); +lean_ctor_set(x_437, 6, x_38); +lean_ctor_set(x_437, 7, x_38); +if (lean_is_scalar(x_412)) { + x_438 = lean_alloc_ctor(1, 1, 0); +} else { + x_438 = x_412; +} +lean_ctor_set(x_438, 0, x_437); +x_439 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_439, 0, x_438); +lean_ctor_set(x_439, 1, x_409); +x_11 = x_439; +goto block_29; +} +else +{ +lean_object* x_440; lean_object* x_441; lean_object* x_442; size_t x_443; size_t x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; +lean_dec(x_412); +x_440 = lean_ctor_get(x_37, 0); +lean_inc(x_440); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_441 = x_37; +} else { + lean_dec_ref(x_37); + x_441 = lean_box(0); +} +x_442 = lean_array_get_size(x_440); +x_443 = lean_usize_of_nat(x_442); +lean_dec(x_442); +x_444 = 0; +x_445 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_443, x_444, x_440, x_409); +x_446 = lean_ctor_get(x_445, 0); +lean_inc(x_446); +x_447 = lean_ctor_get(x_445, 1); +lean_inc(x_447); +if (lean_is_exclusive(x_445)) { + lean_ctor_release(x_445, 0); + lean_ctor_release(x_445, 1); + x_448 = x_445; +} else { + lean_dec_ref(x_445); + x_448 = lean_box(0); +} +x_449 = lean_ctor_get(x_446, 0); +lean_inc(x_449); +if (lean_is_exclusive(x_446)) { + lean_ctor_release(x_446, 0); + x_450 = x_446; +} else { + lean_dec_ref(x_446); + x_450 = lean_box(0); +} +if (lean_is_scalar(x_441)) { + x_451 = lean_alloc_ctor(1, 1, 0); +} else { + x_451 = x_441; +} +lean_ctor_set(x_451, 0, x_449); +x_452 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_452, 0, x_31); +lean_ctor_set(x_452, 1, x_32); +lean_ctor_set(x_452, 2, x_38); +lean_ctor_set(x_452, 3, x_38); +lean_ctor_set(x_452, 4, x_399); +lean_ctor_set(x_452, 5, x_411); +lean_ctor_set(x_452, 6, x_38); +lean_ctor_set(x_452, 7, x_451); +if (lean_is_scalar(x_450)) { + x_453 = lean_alloc_ctor(1, 1, 0); +} else { + x_453 = x_450; +} +lean_ctor_set(x_453, 0, x_452); +if (lean_is_scalar(x_448)) { + x_454 = lean_alloc_ctor(0, 2, 0); +} else { + x_454 = x_448; +} +lean_ctor_set(x_454, 0, x_453); +lean_ctor_set(x_454, 1, x_447); +x_11 = x_454; +goto block_29; +} +} +else +{ +lean_object* x_455; lean_object* x_456; lean_object* x_457; size_t x_458; size_t x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; +lean_dec(x_412); +x_455 = lean_ctor_get(x_36, 0); +lean_inc(x_455); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_456 = x_36; +} else { + lean_dec_ref(x_36); + x_456 = lean_box(0); +} +x_457 = lean_array_get_size(x_455); +x_458 = lean_usize_of_nat(x_457); +lean_dec(x_457); +x_459 = 0; +x_460 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_458, x_459, x_455, x_409); +x_461 = lean_ctor_get(x_460, 0); +lean_inc(x_461); +x_462 = lean_ctor_get(x_460, 1); +lean_inc(x_462); +lean_dec(x_460); +x_463 = lean_ctor_get(x_461, 0); +lean_inc(x_463); +if (lean_is_exclusive(x_461)) { + lean_ctor_release(x_461, 0); + x_464 = x_461; +} else { + lean_dec_ref(x_461); + x_464 = lean_box(0); +} +if (lean_is_scalar(x_456)) { + x_465 = lean_alloc_ctor(1, 1, 0); +} else { + x_465 = x_456; +} +lean_ctor_set(x_465, 0, x_463); +if (lean_is_scalar(x_464)) { + x_466 = lean_alloc_ctor(1, 1, 0); +} else { + x_466 = x_464; +} +lean_ctor_set(x_466, 0, x_465); +x_413 = x_466; +x_414 = x_462; +goto block_436; +} +block_436: +{ +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; +x_415 = lean_ctor_get(x_413, 0); +lean_inc(x_415); +if (lean_is_exclusive(x_413)) { + lean_ctor_release(x_413, 0); + x_416 = x_413; +} else { + lean_dec_ref(x_413); + x_416 = lean_box(0); +} +x_417 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_417, 0, x_31); +lean_ctor_set(x_417, 1, x_32); +lean_ctor_set(x_417, 2, x_38); +lean_ctor_set(x_417, 3, x_38); +lean_ctor_set(x_417, 4, x_399); +lean_ctor_set(x_417, 5, x_411); +lean_ctor_set(x_417, 6, x_415); +lean_ctor_set(x_417, 7, x_38); +if (lean_is_scalar(x_416)) { + x_418 = lean_alloc_ctor(1, 1, 0); +} else { + x_418 = x_416; +} +lean_ctor_set(x_418, 0, x_417); +if (lean_is_scalar(x_410)) { + x_419 = lean_alloc_ctor(0, 2, 0); +} else { + x_419 = x_410; +} +lean_ctor_set(x_419, 0, x_418); +lean_ctor_set(x_419, 1, x_414); +x_11 = x_419; +goto block_29; +} +else +{ +lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; size_t x_424; size_t x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; +lean_dec(x_410); +x_420 = lean_ctor_get(x_413, 0); +lean_inc(x_420); +lean_dec(x_413); +x_421 = lean_ctor_get(x_37, 0); +lean_inc(x_421); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_422 = x_37; +} else { + lean_dec_ref(x_37); + x_422 = lean_box(0); +} +x_423 = lean_array_get_size(x_421); +x_424 = lean_usize_of_nat(x_423); +lean_dec(x_423); +x_425 = 0; +x_426 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_424, x_425, x_421, x_414); +x_427 = lean_ctor_get(x_426, 0); +lean_inc(x_427); +x_428 = lean_ctor_get(x_426, 1); +lean_inc(x_428); +if (lean_is_exclusive(x_426)) { + lean_ctor_release(x_426, 0); + lean_ctor_release(x_426, 1); + x_429 = x_426; +} else { + lean_dec_ref(x_426); + x_429 = lean_box(0); +} +x_430 = lean_ctor_get(x_427, 0); +lean_inc(x_430); +if (lean_is_exclusive(x_427)) { + lean_ctor_release(x_427, 0); + x_431 = x_427; +} else { + lean_dec_ref(x_427); + x_431 = lean_box(0); +} +if (lean_is_scalar(x_422)) { + x_432 = lean_alloc_ctor(1, 1, 0); +} else { + x_432 = x_422; +} +lean_ctor_set(x_432, 0, x_430); +x_433 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_433, 0, x_31); +lean_ctor_set(x_433, 1, x_32); +lean_ctor_set(x_433, 2, x_38); +lean_ctor_set(x_433, 3, x_38); +lean_ctor_set(x_433, 4, x_399); +lean_ctor_set(x_433, 5, x_411); +lean_ctor_set(x_433, 6, x_420); +lean_ctor_set(x_433, 7, x_432); +if (lean_is_scalar(x_431)) { + x_434 = lean_alloc_ctor(1, 1, 0); +} else { + x_434 = x_431; +} +lean_ctor_set(x_434, 0, x_433); +if (lean_is_scalar(x_429)) { + x_435 = lean_alloc_ctor(0, 2, 0); +} else { + x_435 = x_429; +} +lean_ctor_set(x_435, 0, x_434); +lean_ctor_set(x_435, 1, x_428); +x_11 = x_435; +goto block_29; +} +} +} +} +} +} +else +{ +uint8_t x_467; +x_467 = !lean_is_exclusive(x_33); +if (x_467 == 0) +{ +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_468; lean_object* x_469; lean_object* x_470; +x_468 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_469 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_468, x_35, x_4); +x_470 = lean_ctor_get(x_469, 0); +lean_inc(x_470); +if (lean_obj_tag(x_470) == 0) +{ +uint8_t x_471; +lean_dec(x_33); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_32); +lean_dec(x_31); +x_471 = !lean_is_exclusive(x_469); +if (x_471 == 0) +{ +lean_object* x_472; uint8_t x_473; +x_472 = lean_ctor_get(x_469, 0); +lean_dec(x_472); +x_473 = !lean_is_exclusive(x_470); +if (x_473 == 0) +{ +x_11 = x_469; +goto block_29; +} +else +{ +lean_object* x_474; lean_object* x_475; +x_474 = lean_ctor_get(x_470, 0); +lean_inc(x_474); +lean_dec(x_470); +x_475 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_475, 0, x_474); +lean_ctor_set(x_469, 0, x_475); +x_11 = x_469; +goto block_29; +} +} +else +{ +lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; +x_476 = lean_ctor_get(x_469, 1); +lean_inc(x_476); +lean_dec(x_469); +x_477 = lean_ctor_get(x_470, 0); +lean_inc(x_477); +if (lean_is_exclusive(x_470)) { + lean_ctor_release(x_470, 0); + x_478 = x_470; +} else { + lean_dec_ref(x_470); + x_478 = lean_box(0); +} +if (lean_is_scalar(x_478)) { + x_479 = lean_alloc_ctor(0, 1, 0); +} else { + x_479 = x_478; +} +lean_ctor_set(x_479, 0, x_477); +x_480 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_480, 0, x_479); +lean_ctor_set(x_480, 1, x_476); +x_11 = x_480; +goto block_29; +} +} +else +{ +lean_object* x_481; lean_object* x_482; uint8_t x_483; +x_481 = lean_ctor_get(x_469, 1); +lean_inc(x_481); +if (lean_is_exclusive(x_469)) { + lean_ctor_release(x_469, 0); + lean_ctor_release(x_469, 1); + x_482 = x_469; +} else { + lean_dec_ref(x_469); + x_482 = lean_box(0); +} +x_483 = !lean_is_exclusive(x_470); +if (x_483 == 0) +{ +lean_object* x_484; lean_object* x_485; lean_object* x_486; +x_484 = lean_ctor_get(x_470, 0); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_482); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_532; lean_object* x_533; +x_532 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_532, 0, x_31); +lean_ctor_set(x_532, 1, x_32); +lean_ctor_set(x_532, 2, x_38); +lean_ctor_set(x_532, 3, x_33); +lean_ctor_set(x_532, 4, x_38); +lean_ctor_set(x_532, 5, x_484); +lean_ctor_set(x_532, 6, x_38); +lean_ctor_set(x_532, 7, x_38); +lean_ctor_set(x_470, 0, x_532); +x_533 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_533, 0, x_470); +lean_ctor_set(x_533, 1, x_481); +x_11 = x_533; +goto block_29; +} +else +{ +uint8_t x_534; +lean_free_object(x_470); +x_534 = !lean_is_exclusive(x_37); +if (x_534 == 0) +{ +lean_object* x_535; lean_object* x_536; size_t x_537; size_t x_538; lean_object* x_539; uint8_t x_540; +x_535 = lean_ctor_get(x_37, 0); +x_536 = lean_array_get_size(x_535); +x_537 = lean_usize_of_nat(x_536); +lean_dec(x_536); +x_538 = 0; +x_539 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_537, x_538, x_535, x_481); +x_540 = !lean_is_exclusive(x_539); +if (x_540 == 0) +{ +lean_object* x_541; uint8_t x_542; +x_541 = lean_ctor_get(x_539, 0); +x_542 = !lean_is_exclusive(x_541); +if (x_542 == 0) +{ +lean_object* x_543; lean_object* x_544; +x_543 = lean_ctor_get(x_541, 0); +lean_ctor_set(x_37, 0, x_543); +x_544 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_544, 0, x_31); +lean_ctor_set(x_544, 1, x_32); +lean_ctor_set(x_544, 2, x_38); +lean_ctor_set(x_544, 3, x_33); +lean_ctor_set(x_544, 4, x_38); +lean_ctor_set(x_544, 5, x_484); +lean_ctor_set(x_544, 6, x_38); +lean_ctor_set(x_544, 7, x_37); +lean_ctor_set(x_541, 0, x_544); +x_11 = x_539; +goto block_29; +} +else +{ +lean_object* x_545; lean_object* x_546; lean_object* x_547; +x_545 = lean_ctor_get(x_541, 0); +lean_inc(x_545); +lean_dec(x_541); +lean_ctor_set(x_37, 0, x_545); +x_546 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_546, 0, x_31); +lean_ctor_set(x_546, 1, x_32); +lean_ctor_set(x_546, 2, x_38); +lean_ctor_set(x_546, 3, x_33); +lean_ctor_set(x_546, 4, x_38); +lean_ctor_set(x_546, 5, x_484); +lean_ctor_set(x_546, 6, x_38); +lean_ctor_set(x_546, 7, x_37); +x_547 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_547, 0, x_546); +lean_ctor_set(x_539, 0, x_547); +x_11 = x_539; +goto block_29; +} +} +else +{ +lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; +x_548 = lean_ctor_get(x_539, 0); +x_549 = lean_ctor_get(x_539, 1); +lean_inc(x_549); +lean_inc(x_548); +lean_dec(x_539); +x_550 = lean_ctor_get(x_548, 0); +lean_inc(x_550); +if (lean_is_exclusive(x_548)) { + lean_ctor_release(x_548, 0); + x_551 = x_548; +} else { + lean_dec_ref(x_548); + x_551 = lean_box(0); +} +lean_ctor_set(x_37, 0, x_550); +x_552 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_552, 0, x_31); +lean_ctor_set(x_552, 1, x_32); +lean_ctor_set(x_552, 2, x_38); +lean_ctor_set(x_552, 3, x_33); +lean_ctor_set(x_552, 4, x_38); +lean_ctor_set(x_552, 5, x_484); +lean_ctor_set(x_552, 6, x_38); +lean_ctor_set(x_552, 7, x_37); +if (lean_is_scalar(x_551)) { + x_553 = lean_alloc_ctor(1, 1, 0); +} else { + x_553 = x_551; +} +lean_ctor_set(x_553, 0, x_552); +x_554 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_554, 0, x_553); +lean_ctor_set(x_554, 1, x_549); +x_11 = x_554; +goto block_29; +} +} +else +{ +lean_object* x_555; lean_object* x_556; size_t x_557; size_t x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; +x_555 = lean_ctor_get(x_37, 0); +lean_inc(x_555); +lean_dec(x_37); +x_556 = lean_array_get_size(x_555); +x_557 = lean_usize_of_nat(x_556); +lean_dec(x_556); +x_558 = 0; +x_559 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_557, x_558, x_555, x_481); +x_560 = lean_ctor_get(x_559, 0); +lean_inc(x_560); +x_561 = lean_ctor_get(x_559, 1); +lean_inc(x_561); +if (lean_is_exclusive(x_559)) { + lean_ctor_release(x_559, 0); + lean_ctor_release(x_559, 1); + x_562 = x_559; +} else { + lean_dec_ref(x_559); + x_562 = lean_box(0); +} +x_563 = lean_ctor_get(x_560, 0); +lean_inc(x_563); +if (lean_is_exclusive(x_560)) { + lean_ctor_release(x_560, 0); + x_564 = x_560; +} else { + lean_dec_ref(x_560); + x_564 = lean_box(0); +} +x_565 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_565, 0, x_563); +x_566 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_566, 0, x_31); +lean_ctor_set(x_566, 1, x_32); +lean_ctor_set(x_566, 2, x_38); +lean_ctor_set(x_566, 3, x_33); +lean_ctor_set(x_566, 4, x_38); +lean_ctor_set(x_566, 5, x_484); +lean_ctor_set(x_566, 6, x_38); +lean_ctor_set(x_566, 7, x_565); +if (lean_is_scalar(x_564)) { + x_567 = lean_alloc_ctor(1, 1, 0); +} else { + x_567 = x_564; +} +lean_ctor_set(x_567, 0, x_566); +if (lean_is_scalar(x_562)) { + x_568 = lean_alloc_ctor(0, 2, 0); +} else { + x_568 = x_562; +} +lean_ctor_set(x_568, 0, x_567); +lean_ctor_set(x_568, 1, x_561); +x_11 = x_568; +goto block_29; +} +} +} +else +{ +uint8_t x_569; +lean_free_object(x_470); +x_569 = !lean_is_exclusive(x_36); +if (x_569 == 0) +{ +lean_object* x_570; lean_object* x_571; size_t x_572; size_t x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; uint8_t x_577; +x_570 = lean_ctor_get(x_36, 0); +x_571 = lean_array_get_size(x_570); +x_572 = lean_usize_of_nat(x_571); +lean_dec(x_571); +x_573 = 0; +x_574 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_572, x_573, x_570, x_481); +x_575 = lean_ctor_get(x_574, 0); +lean_inc(x_575); +x_576 = lean_ctor_get(x_574, 1); +lean_inc(x_576); +lean_dec(x_574); +x_577 = !lean_is_exclusive(x_575); +if (x_577 == 0) +{ +lean_object* x_578; +x_578 = lean_ctor_get(x_575, 0); +lean_ctor_set(x_36, 0, x_578); +lean_ctor_set(x_575, 0, x_36); +x_485 = x_575; +x_486 = x_576; +goto block_531; +} +else +{ +lean_object* x_579; lean_object* x_580; +x_579 = lean_ctor_get(x_575, 0); +lean_inc(x_579); +lean_dec(x_575); +lean_ctor_set(x_36, 0, x_579); +x_580 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_580, 0, x_36); +x_485 = x_580; +x_486 = x_576; +goto block_531; +} +} +else +{ +lean_object* x_581; lean_object* x_582; size_t x_583; size_t x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; +x_581 = lean_ctor_get(x_36, 0); +lean_inc(x_581); +lean_dec(x_36); +x_582 = lean_array_get_size(x_581); +x_583 = lean_usize_of_nat(x_582); +lean_dec(x_582); +x_584 = 0; +x_585 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_583, x_584, x_581, x_481); +x_586 = lean_ctor_get(x_585, 0); +lean_inc(x_586); +x_587 = lean_ctor_get(x_585, 1); +lean_inc(x_587); +lean_dec(x_585); +x_588 = lean_ctor_get(x_586, 0); +lean_inc(x_588); +if (lean_is_exclusive(x_586)) { + lean_ctor_release(x_586, 0); + x_589 = x_586; +} else { + lean_dec_ref(x_586); + x_589 = lean_box(0); +} +x_590 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_590, 0, x_588); +if (lean_is_scalar(x_589)) { + x_591 = lean_alloc_ctor(1, 1, 0); +} else { + x_591 = x_589; +} +lean_ctor_set(x_591, 0, x_590); +x_485 = x_591; +x_486 = x_587; +goto block_531; +} +} +block_531: +{ +if (lean_obj_tag(x_37) == 0) +{ +uint8_t x_487; +x_487 = !lean_is_exclusive(x_485); +if (x_487 == 0) +{ +lean_object* x_488; lean_object* x_489; lean_object* x_490; +x_488 = lean_ctor_get(x_485, 0); +x_489 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_489, 0, x_31); +lean_ctor_set(x_489, 1, x_32); +lean_ctor_set(x_489, 2, x_38); +lean_ctor_set(x_489, 3, x_33); +lean_ctor_set(x_489, 4, x_38); +lean_ctor_set(x_489, 5, x_484); +lean_ctor_set(x_489, 6, x_488); +lean_ctor_set(x_489, 7, x_38); +lean_ctor_set(x_485, 0, x_489); +if (lean_is_scalar(x_482)) { + x_490 = lean_alloc_ctor(0, 2, 0); +} else { + x_490 = x_482; +} +lean_ctor_set(x_490, 0, x_485); +lean_ctor_set(x_490, 1, x_486); +x_11 = x_490; +goto block_29; +} +else +{ +lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; +x_491 = lean_ctor_get(x_485, 0); +lean_inc(x_491); +lean_dec(x_485); +x_492 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_492, 0, x_31); +lean_ctor_set(x_492, 1, x_32); +lean_ctor_set(x_492, 2, x_38); +lean_ctor_set(x_492, 3, x_33); +lean_ctor_set(x_492, 4, x_38); +lean_ctor_set(x_492, 5, x_484); +lean_ctor_set(x_492, 6, x_491); +lean_ctor_set(x_492, 7, x_38); +x_493 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_493, 0, x_492); +if (lean_is_scalar(x_482)) { + x_494 = lean_alloc_ctor(0, 2, 0); +} else { + x_494 = x_482; +} +lean_ctor_set(x_494, 0, x_493); +lean_ctor_set(x_494, 1, x_486); +x_11 = x_494; +goto block_29; +} +} +else +{ +lean_object* x_495; uint8_t x_496; +lean_dec(x_482); +x_495 = lean_ctor_get(x_485, 0); +lean_inc(x_495); +lean_dec(x_485); +x_496 = !lean_is_exclusive(x_37); +if (x_496 == 0) +{ +lean_object* x_497; lean_object* x_498; size_t x_499; size_t x_500; lean_object* x_501; uint8_t x_502; +x_497 = lean_ctor_get(x_37, 0); +x_498 = lean_array_get_size(x_497); +x_499 = lean_usize_of_nat(x_498); +lean_dec(x_498); +x_500 = 0; +x_501 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_499, x_500, x_497, x_486); +x_502 = !lean_is_exclusive(x_501); +if (x_502 == 0) +{ +lean_object* x_503; uint8_t x_504; +x_503 = lean_ctor_get(x_501, 0); +x_504 = !lean_is_exclusive(x_503); +if (x_504 == 0) +{ +lean_object* x_505; lean_object* x_506; +x_505 = lean_ctor_get(x_503, 0); +lean_ctor_set(x_37, 0, x_505); +x_506 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_506, 0, x_31); +lean_ctor_set(x_506, 1, x_32); +lean_ctor_set(x_506, 2, x_38); +lean_ctor_set(x_506, 3, x_33); +lean_ctor_set(x_506, 4, x_38); +lean_ctor_set(x_506, 5, x_484); +lean_ctor_set(x_506, 6, x_495); +lean_ctor_set(x_506, 7, x_37); +lean_ctor_set(x_503, 0, x_506); +x_11 = x_501; +goto block_29; +} +else +{ +lean_object* x_507; lean_object* x_508; lean_object* x_509; +x_507 = lean_ctor_get(x_503, 0); +lean_inc(x_507); +lean_dec(x_503); +lean_ctor_set(x_37, 0, x_507); +x_508 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_508, 0, x_31); +lean_ctor_set(x_508, 1, x_32); +lean_ctor_set(x_508, 2, x_38); +lean_ctor_set(x_508, 3, x_33); +lean_ctor_set(x_508, 4, x_38); +lean_ctor_set(x_508, 5, x_484); +lean_ctor_set(x_508, 6, x_495); +lean_ctor_set(x_508, 7, x_37); +x_509 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_509, 0, x_508); +lean_ctor_set(x_501, 0, x_509); +x_11 = x_501; +goto block_29; +} +} +else +{ +lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; +x_510 = lean_ctor_get(x_501, 0); +x_511 = lean_ctor_get(x_501, 1); +lean_inc(x_511); +lean_inc(x_510); +lean_dec(x_501); +x_512 = lean_ctor_get(x_510, 0); +lean_inc(x_512); +if (lean_is_exclusive(x_510)) { + lean_ctor_release(x_510, 0); + x_513 = x_510; +} else { + lean_dec_ref(x_510); + x_513 = lean_box(0); +} +lean_ctor_set(x_37, 0, x_512); +x_514 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_514, 0, x_31); +lean_ctor_set(x_514, 1, x_32); +lean_ctor_set(x_514, 2, x_38); +lean_ctor_set(x_514, 3, x_33); +lean_ctor_set(x_514, 4, x_38); +lean_ctor_set(x_514, 5, x_484); +lean_ctor_set(x_514, 6, x_495); +lean_ctor_set(x_514, 7, x_37); +if (lean_is_scalar(x_513)) { + x_515 = lean_alloc_ctor(1, 1, 0); +} else { + x_515 = x_513; +} +lean_ctor_set(x_515, 0, x_514); +x_516 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_516, 0, x_515); +lean_ctor_set(x_516, 1, x_511); +x_11 = x_516; +goto block_29; +} +} +else +{ +lean_object* x_517; lean_object* x_518; size_t x_519; size_t x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; +x_517 = lean_ctor_get(x_37, 0); +lean_inc(x_517); +lean_dec(x_37); +x_518 = lean_array_get_size(x_517); +x_519 = lean_usize_of_nat(x_518); +lean_dec(x_518); +x_520 = 0; +x_521 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_519, x_520, x_517, x_486); +x_522 = lean_ctor_get(x_521, 0); +lean_inc(x_522); +x_523 = lean_ctor_get(x_521, 1); +lean_inc(x_523); +if (lean_is_exclusive(x_521)) { + lean_ctor_release(x_521, 0); + lean_ctor_release(x_521, 1); + x_524 = x_521; +} else { + lean_dec_ref(x_521); + x_524 = lean_box(0); +} +x_525 = lean_ctor_get(x_522, 0); +lean_inc(x_525); +if (lean_is_exclusive(x_522)) { + lean_ctor_release(x_522, 0); + x_526 = x_522; +} else { + lean_dec_ref(x_522); + x_526 = lean_box(0); +} +x_527 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_527, 0, x_525); +x_528 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_528, 0, x_31); +lean_ctor_set(x_528, 1, x_32); +lean_ctor_set(x_528, 2, x_38); +lean_ctor_set(x_528, 3, x_33); +lean_ctor_set(x_528, 4, x_38); +lean_ctor_set(x_528, 5, x_484); +lean_ctor_set(x_528, 6, x_495); +lean_ctor_set(x_528, 7, x_527); +if (lean_is_scalar(x_526)) { + x_529 = lean_alloc_ctor(1, 1, 0); +} else { + x_529 = x_526; +} +lean_ctor_set(x_529, 0, x_528); +if (lean_is_scalar(x_524)) { + x_530 = lean_alloc_ctor(0, 2, 0); +} else { + x_530 = x_524; +} +lean_ctor_set(x_530, 0, x_529); +lean_ctor_set(x_530, 1, x_523); +x_11 = x_530; +goto block_29; +} +} +} +} +else +{ +lean_object* x_592; lean_object* x_593; lean_object* x_594; +x_592 = lean_ctor_get(x_470, 0); +lean_inc(x_592); +lean_dec(x_470); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_482); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_617; lean_object* x_618; lean_object* x_619; +x_617 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_617, 0, x_31); +lean_ctor_set(x_617, 1, x_32); +lean_ctor_set(x_617, 2, x_38); +lean_ctor_set(x_617, 3, x_33); +lean_ctor_set(x_617, 4, x_38); +lean_ctor_set(x_617, 5, x_592); +lean_ctor_set(x_617, 6, x_38); +lean_ctor_set(x_617, 7, x_38); +x_618 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_618, 0, x_617); +x_619 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_619, 0, x_618); +lean_ctor_set(x_619, 1, x_481); +x_11 = x_619; +goto block_29; +} +else +{ +lean_object* x_620; lean_object* x_621; lean_object* x_622; size_t x_623; size_t x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; +x_620 = lean_ctor_get(x_37, 0); +lean_inc(x_620); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_621 = x_37; +} else { + lean_dec_ref(x_37); + x_621 = lean_box(0); +} +x_622 = lean_array_get_size(x_620); +x_623 = lean_usize_of_nat(x_622); +lean_dec(x_622); +x_624 = 0; +x_625 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_623, x_624, x_620, x_481); +x_626 = lean_ctor_get(x_625, 0); +lean_inc(x_626); +x_627 = lean_ctor_get(x_625, 1); +lean_inc(x_627); +if (lean_is_exclusive(x_625)) { + lean_ctor_release(x_625, 0); + lean_ctor_release(x_625, 1); + x_628 = x_625; +} else { + lean_dec_ref(x_625); + x_628 = lean_box(0); +} +x_629 = lean_ctor_get(x_626, 0); +lean_inc(x_629); +if (lean_is_exclusive(x_626)) { + lean_ctor_release(x_626, 0); + x_630 = x_626; +} else { + lean_dec_ref(x_626); + x_630 = lean_box(0); +} +if (lean_is_scalar(x_621)) { + x_631 = lean_alloc_ctor(1, 1, 0); +} else { + x_631 = x_621; +} +lean_ctor_set(x_631, 0, x_629); +x_632 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_632, 0, x_31); +lean_ctor_set(x_632, 1, x_32); +lean_ctor_set(x_632, 2, x_38); +lean_ctor_set(x_632, 3, x_33); +lean_ctor_set(x_632, 4, x_38); +lean_ctor_set(x_632, 5, x_592); +lean_ctor_set(x_632, 6, x_38); +lean_ctor_set(x_632, 7, x_631); +if (lean_is_scalar(x_630)) { + x_633 = lean_alloc_ctor(1, 1, 0); +} else { + x_633 = x_630; +} +lean_ctor_set(x_633, 0, x_632); +if (lean_is_scalar(x_628)) { + x_634 = lean_alloc_ctor(0, 2, 0); +} else { + x_634 = x_628; +} +lean_ctor_set(x_634, 0, x_633); +lean_ctor_set(x_634, 1, x_627); +x_11 = x_634; +goto block_29; +} +} +else +{ +lean_object* x_635; lean_object* x_636; lean_object* x_637; size_t x_638; size_t x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; +x_635 = lean_ctor_get(x_36, 0); +lean_inc(x_635); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_636 = x_36; +} else { + lean_dec_ref(x_36); + x_636 = lean_box(0); +} +x_637 = lean_array_get_size(x_635); +x_638 = lean_usize_of_nat(x_637); +lean_dec(x_637); +x_639 = 0; +x_640 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_638, x_639, x_635, x_481); +x_641 = lean_ctor_get(x_640, 0); +lean_inc(x_641); +x_642 = lean_ctor_get(x_640, 1); +lean_inc(x_642); +lean_dec(x_640); +x_643 = lean_ctor_get(x_641, 0); +lean_inc(x_643); +if (lean_is_exclusive(x_641)) { + lean_ctor_release(x_641, 0); + x_644 = x_641; +} else { + lean_dec_ref(x_641); + x_644 = lean_box(0); +} +if (lean_is_scalar(x_636)) { + x_645 = lean_alloc_ctor(1, 1, 0); +} else { + x_645 = x_636; +} +lean_ctor_set(x_645, 0, x_643); +if (lean_is_scalar(x_644)) { + x_646 = lean_alloc_ctor(1, 1, 0); +} else { + x_646 = x_644; +} +lean_ctor_set(x_646, 0, x_645); +x_593 = x_646; +x_594 = x_642; +goto block_616; +} +block_616: +{ +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; +x_595 = lean_ctor_get(x_593, 0); +lean_inc(x_595); +if (lean_is_exclusive(x_593)) { + lean_ctor_release(x_593, 0); + x_596 = x_593; +} else { + lean_dec_ref(x_593); + x_596 = lean_box(0); +} +x_597 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_597, 0, x_31); +lean_ctor_set(x_597, 1, x_32); +lean_ctor_set(x_597, 2, x_38); +lean_ctor_set(x_597, 3, x_33); +lean_ctor_set(x_597, 4, x_38); +lean_ctor_set(x_597, 5, x_592); +lean_ctor_set(x_597, 6, x_595); +lean_ctor_set(x_597, 7, x_38); +if (lean_is_scalar(x_596)) { + x_598 = lean_alloc_ctor(1, 1, 0); +} else { + x_598 = x_596; +} +lean_ctor_set(x_598, 0, x_597); +if (lean_is_scalar(x_482)) { + x_599 = lean_alloc_ctor(0, 2, 0); +} else { + x_599 = x_482; +} +lean_ctor_set(x_599, 0, x_598); +lean_ctor_set(x_599, 1, x_594); +x_11 = x_599; +goto block_29; +} +else +{ +lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; size_t x_604; size_t x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; lean_object* x_615; +lean_dec(x_482); +x_600 = lean_ctor_get(x_593, 0); +lean_inc(x_600); +lean_dec(x_593); +x_601 = lean_ctor_get(x_37, 0); +lean_inc(x_601); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_602 = x_37; +} else { + lean_dec_ref(x_37); + x_602 = lean_box(0); +} +x_603 = lean_array_get_size(x_601); +x_604 = lean_usize_of_nat(x_603); +lean_dec(x_603); +x_605 = 0; +x_606 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_604, x_605, x_601, x_594); +x_607 = lean_ctor_get(x_606, 0); +lean_inc(x_607); +x_608 = lean_ctor_get(x_606, 1); +lean_inc(x_608); +if (lean_is_exclusive(x_606)) { + lean_ctor_release(x_606, 0); + lean_ctor_release(x_606, 1); + x_609 = x_606; +} else { + lean_dec_ref(x_606); + x_609 = lean_box(0); +} +x_610 = lean_ctor_get(x_607, 0); +lean_inc(x_610); +if (lean_is_exclusive(x_607)) { + lean_ctor_release(x_607, 0); + x_611 = x_607; +} else { + lean_dec_ref(x_607); + x_611 = lean_box(0); +} +if (lean_is_scalar(x_602)) { + x_612 = lean_alloc_ctor(1, 1, 0); +} else { + x_612 = x_602; +} +lean_ctor_set(x_612, 0, x_610); +x_613 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_613, 0, x_31); +lean_ctor_set(x_613, 1, x_32); +lean_ctor_set(x_613, 2, x_38); +lean_ctor_set(x_613, 3, x_33); +lean_ctor_set(x_613, 4, x_38); +lean_ctor_set(x_613, 5, x_592); +lean_ctor_set(x_613, 6, x_600); +lean_ctor_set(x_613, 7, x_612); +if (lean_is_scalar(x_611)) { + x_614 = lean_alloc_ctor(1, 1, 0); +} else { + x_614 = x_611; +} +lean_ctor_set(x_614, 0, x_613); +if (lean_is_scalar(x_609)) { + x_615 = lean_alloc_ctor(0, 2, 0); +} else { + x_615 = x_609; +} +lean_ctor_set(x_615, 0, x_614); +lean_ctor_set(x_615, 1, x_608); +x_11 = x_615; +goto block_29; +} +} +} +} +} +else +{ +uint8_t x_647; +x_647 = !lean_is_exclusive(x_34); +if (x_647 == 0) +{ +lean_object* x_648; lean_object* x_649; lean_object* x_650; +x_648 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_649 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_648, x_35, x_4); +x_650 = lean_ctor_get(x_649, 0); +lean_inc(x_650); +if (lean_obj_tag(x_650) == 0) +{ +uint8_t x_651; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_32); +lean_dec(x_31); +x_651 = !lean_is_exclusive(x_649); +if (x_651 == 0) +{ +lean_object* x_652; uint8_t x_653; +x_652 = lean_ctor_get(x_649, 0); +lean_dec(x_652); +x_653 = !lean_is_exclusive(x_650); +if (x_653 == 0) +{ +x_11 = x_649; +goto block_29; +} +else +{ +lean_object* x_654; lean_object* x_655; +x_654 = lean_ctor_get(x_650, 0); +lean_inc(x_654); +lean_dec(x_650); +x_655 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_655, 0, x_654); +lean_ctor_set(x_649, 0, x_655); +x_11 = x_649; +goto block_29; +} +} +else +{ +lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; +x_656 = lean_ctor_get(x_649, 1); +lean_inc(x_656); +lean_dec(x_649); +x_657 = lean_ctor_get(x_650, 0); +lean_inc(x_657); +if (lean_is_exclusive(x_650)) { + lean_ctor_release(x_650, 0); + x_658 = x_650; +} else { + lean_dec_ref(x_650); + x_658 = lean_box(0); +} +if (lean_is_scalar(x_658)) { + x_659 = lean_alloc_ctor(0, 1, 0); +} else { + x_659 = x_658; +} +lean_ctor_set(x_659, 0, x_657); +x_660 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_660, 0, x_659); +lean_ctor_set(x_660, 1, x_656); +x_11 = x_660; +goto block_29; +} +} +else +{ +lean_object* x_661; lean_object* x_662; uint8_t x_663; +x_661 = lean_ctor_get(x_649, 1); +lean_inc(x_661); +if (lean_is_exclusive(x_649)) { + lean_ctor_release(x_649, 0); + lean_ctor_release(x_649, 1); + x_662 = x_649; +} else { + lean_dec_ref(x_649); + x_662 = lean_box(0); +} +x_663 = !lean_is_exclusive(x_650); +if (x_663 == 0) +{ +lean_object* x_664; lean_object* x_665; lean_object* x_666; +x_664 = lean_ctor_get(x_650, 0); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_662); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_712; lean_object* x_713; +x_712 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_712, 0, x_31); +lean_ctor_set(x_712, 1, x_32); +lean_ctor_set(x_712, 2, x_38); +lean_ctor_set(x_712, 3, x_33); +lean_ctor_set(x_712, 4, x_34); +lean_ctor_set(x_712, 5, x_664); +lean_ctor_set(x_712, 6, x_38); +lean_ctor_set(x_712, 7, x_38); +lean_ctor_set(x_650, 0, x_712); +x_713 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_713, 0, x_650); +lean_ctor_set(x_713, 1, x_661); +x_11 = x_713; +goto block_29; +} +else +{ +uint8_t x_714; +lean_free_object(x_650); +x_714 = !lean_is_exclusive(x_37); +if (x_714 == 0) +{ +lean_object* x_715; lean_object* x_716; size_t x_717; size_t x_718; lean_object* x_719; uint8_t x_720; +x_715 = lean_ctor_get(x_37, 0); +x_716 = lean_array_get_size(x_715); +x_717 = lean_usize_of_nat(x_716); +lean_dec(x_716); +x_718 = 0; +x_719 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_717, x_718, x_715, x_661); +x_720 = !lean_is_exclusive(x_719); +if (x_720 == 0) +{ +lean_object* x_721; uint8_t x_722; +x_721 = lean_ctor_get(x_719, 0); +x_722 = !lean_is_exclusive(x_721); +if (x_722 == 0) +{ +lean_object* x_723; lean_object* x_724; +x_723 = lean_ctor_get(x_721, 0); +lean_ctor_set(x_37, 0, x_723); +x_724 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_724, 0, x_31); +lean_ctor_set(x_724, 1, x_32); +lean_ctor_set(x_724, 2, x_38); +lean_ctor_set(x_724, 3, x_33); +lean_ctor_set(x_724, 4, x_34); +lean_ctor_set(x_724, 5, x_664); +lean_ctor_set(x_724, 6, x_38); +lean_ctor_set(x_724, 7, x_37); +lean_ctor_set(x_721, 0, x_724); +x_11 = x_719; +goto block_29; +} +else +{ +lean_object* x_725; lean_object* x_726; lean_object* x_727; +x_725 = lean_ctor_get(x_721, 0); +lean_inc(x_725); +lean_dec(x_721); +lean_ctor_set(x_37, 0, x_725); +x_726 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_726, 0, x_31); +lean_ctor_set(x_726, 1, x_32); +lean_ctor_set(x_726, 2, x_38); +lean_ctor_set(x_726, 3, x_33); +lean_ctor_set(x_726, 4, x_34); +lean_ctor_set(x_726, 5, x_664); +lean_ctor_set(x_726, 6, x_38); +lean_ctor_set(x_726, 7, x_37); +x_727 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_727, 0, x_726); +lean_ctor_set(x_719, 0, x_727); +x_11 = x_719; +goto block_29; +} +} +else +{ +lean_object* x_728; lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; +x_728 = lean_ctor_get(x_719, 0); +x_729 = lean_ctor_get(x_719, 1); +lean_inc(x_729); +lean_inc(x_728); +lean_dec(x_719); +x_730 = lean_ctor_get(x_728, 0); +lean_inc(x_730); +if (lean_is_exclusive(x_728)) { + lean_ctor_release(x_728, 0); + x_731 = x_728; +} else { + lean_dec_ref(x_728); + x_731 = lean_box(0); +} +lean_ctor_set(x_37, 0, x_730); +x_732 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_732, 0, x_31); +lean_ctor_set(x_732, 1, x_32); +lean_ctor_set(x_732, 2, x_38); +lean_ctor_set(x_732, 3, x_33); +lean_ctor_set(x_732, 4, x_34); +lean_ctor_set(x_732, 5, x_664); +lean_ctor_set(x_732, 6, x_38); +lean_ctor_set(x_732, 7, x_37); +if (lean_is_scalar(x_731)) { + x_733 = lean_alloc_ctor(1, 1, 0); +} else { + x_733 = x_731; +} +lean_ctor_set(x_733, 0, x_732); +x_734 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_734, 0, x_733); +lean_ctor_set(x_734, 1, x_729); +x_11 = x_734; +goto block_29; +} +} +else +{ +lean_object* x_735; lean_object* x_736; size_t x_737; size_t x_738; lean_object* x_739; lean_object* x_740; lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; lean_object* x_747; lean_object* x_748; +x_735 = lean_ctor_get(x_37, 0); +lean_inc(x_735); +lean_dec(x_37); +x_736 = lean_array_get_size(x_735); +x_737 = lean_usize_of_nat(x_736); +lean_dec(x_736); +x_738 = 0; +x_739 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_737, x_738, x_735, x_661); +x_740 = lean_ctor_get(x_739, 0); +lean_inc(x_740); +x_741 = lean_ctor_get(x_739, 1); +lean_inc(x_741); +if (lean_is_exclusive(x_739)) { + lean_ctor_release(x_739, 0); + lean_ctor_release(x_739, 1); + x_742 = x_739; +} else { + lean_dec_ref(x_739); + x_742 = lean_box(0); +} +x_743 = lean_ctor_get(x_740, 0); +lean_inc(x_743); +if (lean_is_exclusive(x_740)) { + lean_ctor_release(x_740, 0); + x_744 = x_740; +} else { + lean_dec_ref(x_740); + x_744 = lean_box(0); +} +x_745 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_745, 0, x_743); +x_746 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_746, 0, x_31); +lean_ctor_set(x_746, 1, x_32); +lean_ctor_set(x_746, 2, x_38); +lean_ctor_set(x_746, 3, x_33); +lean_ctor_set(x_746, 4, x_34); +lean_ctor_set(x_746, 5, x_664); +lean_ctor_set(x_746, 6, x_38); +lean_ctor_set(x_746, 7, x_745); +if (lean_is_scalar(x_744)) { + x_747 = lean_alloc_ctor(1, 1, 0); +} else { + x_747 = x_744; +} +lean_ctor_set(x_747, 0, x_746); +if (lean_is_scalar(x_742)) { + x_748 = lean_alloc_ctor(0, 2, 0); +} else { + x_748 = x_742; +} +lean_ctor_set(x_748, 0, x_747); +lean_ctor_set(x_748, 1, x_741); +x_11 = x_748; +goto block_29; +} +} +} +else +{ +uint8_t x_749; +lean_free_object(x_650); +x_749 = !lean_is_exclusive(x_36); +if (x_749 == 0) +{ +lean_object* x_750; lean_object* x_751; size_t x_752; size_t x_753; lean_object* x_754; lean_object* x_755; lean_object* x_756; uint8_t x_757; +x_750 = lean_ctor_get(x_36, 0); +x_751 = lean_array_get_size(x_750); +x_752 = lean_usize_of_nat(x_751); +lean_dec(x_751); +x_753 = 0; +x_754 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_752, x_753, x_750, x_661); +x_755 = lean_ctor_get(x_754, 0); +lean_inc(x_755); +x_756 = lean_ctor_get(x_754, 1); +lean_inc(x_756); +lean_dec(x_754); +x_757 = !lean_is_exclusive(x_755); +if (x_757 == 0) +{ +lean_object* x_758; +x_758 = lean_ctor_get(x_755, 0); +lean_ctor_set(x_36, 0, x_758); +lean_ctor_set(x_755, 0, x_36); +x_665 = x_755; +x_666 = x_756; +goto block_711; +} +else +{ +lean_object* x_759; lean_object* x_760; +x_759 = lean_ctor_get(x_755, 0); +lean_inc(x_759); +lean_dec(x_755); +lean_ctor_set(x_36, 0, x_759); +x_760 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_760, 0, x_36); +x_665 = x_760; +x_666 = x_756; +goto block_711; +} +} +else +{ +lean_object* x_761; lean_object* x_762; size_t x_763; size_t x_764; lean_object* x_765; lean_object* x_766; lean_object* x_767; lean_object* x_768; lean_object* x_769; lean_object* x_770; lean_object* x_771; +x_761 = lean_ctor_get(x_36, 0); +lean_inc(x_761); +lean_dec(x_36); +x_762 = lean_array_get_size(x_761); +x_763 = lean_usize_of_nat(x_762); +lean_dec(x_762); +x_764 = 0; +x_765 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_763, x_764, x_761, x_661); +x_766 = lean_ctor_get(x_765, 0); +lean_inc(x_766); +x_767 = lean_ctor_get(x_765, 1); +lean_inc(x_767); +lean_dec(x_765); +x_768 = lean_ctor_get(x_766, 0); +lean_inc(x_768); +if (lean_is_exclusive(x_766)) { + lean_ctor_release(x_766, 0); + x_769 = x_766; +} else { + lean_dec_ref(x_766); + x_769 = lean_box(0); +} +x_770 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_770, 0, x_768); +if (lean_is_scalar(x_769)) { + x_771 = lean_alloc_ctor(1, 1, 0); +} else { + x_771 = x_769; +} +lean_ctor_set(x_771, 0, x_770); +x_665 = x_771; +x_666 = x_767; +goto block_711; +} +} +block_711: +{ +if (lean_obj_tag(x_37) == 0) +{ +uint8_t x_667; +x_667 = !lean_is_exclusive(x_665); +if (x_667 == 0) +{ +lean_object* x_668; lean_object* x_669; lean_object* x_670; +x_668 = lean_ctor_get(x_665, 0); +x_669 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_669, 0, x_31); +lean_ctor_set(x_669, 1, x_32); +lean_ctor_set(x_669, 2, x_38); +lean_ctor_set(x_669, 3, x_33); +lean_ctor_set(x_669, 4, x_34); +lean_ctor_set(x_669, 5, x_664); +lean_ctor_set(x_669, 6, x_668); +lean_ctor_set(x_669, 7, x_38); +lean_ctor_set(x_665, 0, x_669); +if (lean_is_scalar(x_662)) { + x_670 = lean_alloc_ctor(0, 2, 0); +} else { + x_670 = x_662; +} +lean_ctor_set(x_670, 0, x_665); +lean_ctor_set(x_670, 1, x_666); +x_11 = x_670; +goto block_29; +} +else +{ +lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; +x_671 = lean_ctor_get(x_665, 0); +lean_inc(x_671); +lean_dec(x_665); +x_672 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_672, 0, x_31); +lean_ctor_set(x_672, 1, x_32); +lean_ctor_set(x_672, 2, x_38); +lean_ctor_set(x_672, 3, x_33); +lean_ctor_set(x_672, 4, x_34); +lean_ctor_set(x_672, 5, x_664); +lean_ctor_set(x_672, 6, x_671); +lean_ctor_set(x_672, 7, x_38); +x_673 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_673, 0, x_672); +if (lean_is_scalar(x_662)) { + x_674 = lean_alloc_ctor(0, 2, 0); +} else { + x_674 = x_662; +} +lean_ctor_set(x_674, 0, x_673); +lean_ctor_set(x_674, 1, x_666); +x_11 = x_674; +goto block_29; +} +} +else +{ +lean_object* x_675; uint8_t x_676; +lean_dec(x_662); +x_675 = lean_ctor_get(x_665, 0); +lean_inc(x_675); +lean_dec(x_665); +x_676 = !lean_is_exclusive(x_37); +if (x_676 == 0) +{ +lean_object* x_677; lean_object* x_678; size_t x_679; size_t x_680; lean_object* x_681; uint8_t x_682; +x_677 = lean_ctor_get(x_37, 0); +x_678 = lean_array_get_size(x_677); +x_679 = lean_usize_of_nat(x_678); +lean_dec(x_678); +x_680 = 0; +x_681 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_679, x_680, x_677, x_666); +x_682 = !lean_is_exclusive(x_681); +if (x_682 == 0) +{ +lean_object* x_683; uint8_t x_684; +x_683 = lean_ctor_get(x_681, 0); +x_684 = !lean_is_exclusive(x_683); +if (x_684 == 0) +{ +lean_object* x_685; lean_object* x_686; +x_685 = lean_ctor_get(x_683, 0); +lean_ctor_set(x_37, 0, x_685); +x_686 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_686, 0, x_31); +lean_ctor_set(x_686, 1, x_32); +lean_ctor_set(x_686, 2, x_38); +lean_ctor_set(x_686, 3, x_33); +lean_ctor_set(x_686, 4, x_34); +lean_ctor_set(x_686, 5, x_664); +lean_ctor_set(x_686, 6, x_675); +lean_ctor_set(x_686, 7, x_37); +lean_ctor_set(x_683, 0, x_686); +x_11 = x_681; +goto block_29; +} +else +{ +lean_object* x_687; lean_object* x_688; lean_object* x_689; +x_687 = lean_ctor_get(x_683, 0); +lean_inc(x_687); +lean_dec(x_683); +lean_ctor_set(x_37, 0, x_687); +x_688 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_688, 0, x_31); +lean_ctor_set(x_688, 1, x_32); +lean_ctor_set(x_688, 2, x_38); +lean_ctor_set(x_688, 3, x_33); +lean_ctor_set(x_688, 4, x_34); +lean_ctor_set(x_688, 5, x_664); +lean_ctor_set(x_688, 6, x_675); +lean_ctor_set(x_688, 7, x_37); +x_689 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_689, 0, x_688); +lean_ctor_set(x_681, 0, x_689); +x_11 = x_681; +goto block_29; +} +} +else +{ +lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; +x_690 = lean_ctor_get(x_681, 0); +x_691 = lean_ctor_get(x_681, 1); +lean_inc(x_691); +lean_inc(x_690); +lean_dec(x_681); +x_692 = lean_ctor_get(x_690, 0); +lean_inc(x_692); +if (lean_is_exclusive(x_690)) { + lean_ctor_release(x_690, 0); + x_693 = x_690; +} else { + lean_dec_ref(x_690); + x_693 = lean_box(0); +} +lean_ctor_set(x_37, 0, x_692); +x_694 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_694, 0, x_31); +lean_ctor_set(x_694, 1, x_32); +lean_ctor_set(x_694, 2, x_38); +lean_ctor_set(x_694, 3, x_33); +lean_ctor_set(x_694, 4, x_34); +lean_ctor_set(x_694, 5, x_664); +lean_ctor_set(x_694, 6, x_675); +lean_ctor_set(x_694, 7, x_37); +if (lean_is_scalar(x_693)) { + x_695 = lean_alloc_ctor(1, 1, 0); +} else { + x_695 = x_693; +} +lean_ctor_set(x_695, 0, x_694); +x_696 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_696, 0, x_695); +lean_ctor_set(x_696, 1, x_691); +x_11 = x_696; +goto block_29; +} +} +else +{ +lean_object* x_697; lean_object* x_698; size_t x_699; size_t x_700; lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; +x_697 = lean_ctor_get(x_37, 0); +lean_inc(x_697); +lean_dec(x_37); +x_698 = lean_array_get_size(x_697); +x_699 = lean_usize_of_nat(x_698); +lean_dec(x_698); +x_700 = 0; +x_701 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_699, x_700, x_697, x_666); +x_702 = lean_ctor_get(x_701, 0); +lean_inc(x_702); +x_703 = lean_ctor_get(x_701, 1); +lean_inc(x_703); +if (lean_is_exclusive(x_701)) { + lean_ctor_release(x_701, 0); + lean_ctor_release(x_701, 1); + x_704 = x_701; +} else { + lean_dec_ref(x_701); + x_704 = lean_box(0); +} +x_705 = lean_ctor_get(x_702, 0); +lean_inc(x_705); +if (lean_is_exclusive(x_702)) { + lean_ctor_release(x_702, 0); + x_706 = x_702; +} else { + lean_dec_ref(x_702); + x_706 = lean_box(0); +} +x_707 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_707, 0, x_705); +x_708 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_708, 0, x_31); +lean_ctor_set(x_708, 1, x_32); +lean_ctor_set(x_708, 2, x_38); +lean_ctor_set(x_708, 3, x_33); +lean_ctor_set(x_708, 4, x_34); +lean_ctor_set(x_708, 5, x_664); +lean_ctor_set(x_708, 6, x_675); +lean_ctor_set(x_708, 7, x_707); +if (lean_is_scalar(x_706)) { + x_709 = lean_alloc_ctor(1, 1, 0); +} else { + x_709 = x_706; +} +lean_ctor_set(x_709, 0, x_708); +if (lean_is_scalar(x_704)) { + x_710 = lean_alloc_ctor(0, 2, 0); +} else { + x_710 = x_704; +} +lean_ctor_set(x_710, 0, x_709); +lean_ctor_set(x_710, 1, x_703); +x_11 = x_710; +goto block_29; +} +} +} +} +else +{ +lean_object* x_772; lean_object* x_773; lean_object* x_774; +x_772 = lean_ctor_get(x_650, 0); +lean_inc(x_772); +lean_dec(x_650); +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_662); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_797; lean_object* x_798; lean_object* x_799; +x_797 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_797, 0, x_31); +lean_ctor_set(x_797, 1, x_32); +lean_ctor_set(x_797, 2, x_38); +lean_ctor_set(x_797, 3, x_33); +lean_ctor_set(x_797, 4, x_34); +lean_ctor_set(x_797, 5, x_772); +lean_ctor_set(x_797, 6, x_38); +lean_ctor_set(x_797, 7, x_38); +x_798 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_798, 0, x_797); +x_799 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_799, 0, x_798); +lean_ctor_set(x_799, 1, x_661); +x_11 = x_799; +goto block_29; +} +else +{ +lean_object* x_800; lean_object* x_801; lean_object* x_802; size_t x_803; size_t x_804; lean_object* x_805; lean_object* x_806; lean_object* x_807; lean_object* x_808; lean_object* x_809; lean_object* x_810; lean_object* x_811; lean_object* x_812; lean_object* x_813; lean_object* x_814; +x_800 = lean_ctor_get(x_37, 0); +lean_inc(x_800); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_801 = x_37; +} else { + lean_dec_ref(x_37); + x_801 = lean_box(0); +} +x_802 = lean_array_get_size(x_800); +x_803 = lean_usize_of_nat(x_802); +lean_dec(x_802); +x_804 = 0; +x_805 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_803, x_804, x_800, x_661); +x_806 = lean_ctor_get(x_805, 0); +lean_inc(x_806); +x_807 = lean_ctor_get(x_805, 1); +lean_inc(x_807); +if (lean_is_exclusive(x_805)) { + lean_ctor_release(x_805, 0); + lean_ctor_release(x_805, 1); + x_808 = x_805; +} else { + lean_dec_ref(x_805); + x_808 = lean_box(0); +} +x_809 = lean_ctor_get(x_806, 0); +lean_inc(x_809); +if (lean_is_exclusive(x_806)) { + lean_ctor_release(x_806, 0); + x_810 = x_806; +} else { + lean_dec_ref(x_806); + x_810 = lean_box(0); +} +if (lean_is_scalar(x_801)) { + x_811 = lean_alloc_ctor(1, 1, 0); +} else { + x_811 = x_801; +} +lean_ctor_set(x_811, 0, x_809); +x_812 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_812, 0, x_31); +lean_ctor_set(x_812, 1, x_32); +lean_ctor_set(x_812, 2, x_38); +lean_ctor_set(x_812, 3, x_33); +lean_ctor_set(x_812, 4, x_34); +lean_ctor_set(x_812, 5, x_772); +lean_ctor_set(x_812, 6, x_38); +lean_ctor_set(x_812, 7, x_811); +if (lean_is_scalar(x_810)) { + x_813 = lean_alloc_ctor(1, 1, 0); +} else { + x_813 = x_810; +} +lean_ctor_set(x_813, 0, x_812); +if (lean_is_scalar(x_808)) { + x_814 = lean_alloc_ctor(0, 2, 0); +} else { + x_814 = x_808; +} +lean_ctor_set(x_814, 0, x_813); +lean_ctor_set(x_814, 1, x_807); +x_11 = x_814; +goto block_29; +} +} +else +{ +lean_object* x_815; lean_object* x_816; lean_object* x_817; size_t x_818; size_t x_819; lean_object* x_820; lean_object* x_821; lean_object* x_822; lean_object* x_823; lean_object* x_824; lean_object* x_825; lean_object* x_826; +x_815 = lean_ctor_get(x_36, 0); +lean_inc(x_815); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_816 = x_36; +} else { + lean_dec_ref(x_36); + x_816 = lean_box(0); +} +x_817 = lean_array_get_size(x_815); +x_818 = lean_usize_of_nat(x_817); +lean_dec(x_817); +x_819 = 0; +x_820 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_818, x_819, x_815, x_661); +x_821 = lean_ctor_get(x_820, 0); +lean_inc(x_821); +x_822 = lean_ctor_get(x_820, 1); +lean_inc(x_822); +lean_dec(x_820); +x_823 = lean_ctor_get(x_821, 0); +lean_inc(x_823); +if (lean_is_exclusive(x_821)) { + lean_ctor_release(x_821, 0); + x_824 = x_821; +} else { + lean_dec_ref(x_821); + x_824 = lean_box(0); +} +if (lean_is_scalar(x_816)) { + x_825 = lean_alloc_ctor(1, 1, 0); +} else { + x_825 = x_816; +} +lean_ctor_set(x_825, 0, x_823); +if (lean_is_scalar(x_824)) { + x_826 = lean_alloc_ctor(1, 1, 0); +} else { + x_826 = x_824; +} +lean_ctor_set(x_826, 0, x_825); +x_773 = x_826; +x_774 = x_822; +goto block_796; +} +block_796: +{ +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; +x_775 = lean_ctor_get(x_773, 0); +lean_inc(x_775); +if (lean_is_exclusive(x_773)) { + lean_ctor_release(x_773, 0); + x_776 = x_773; +} else { + lean_dec_ref(x_773); + x_776 = lean_box(0); +} +x_777 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_777, 0, x_31); +lean_ctor_set(x_777, 1, x_32); +lean_ctor_set(x_777, 2, x_38); +lean_ctor_set(x_777, 3, x_33); +lean_ctor_set(x_777, 4, x_34); +lean_ctor_set(x_777, 5, x_772); +lean_ctor_set(x_777, 6, x_775); +lean_ctor_set(x_777, 7, x_38); +if (lean_is_scalar(x_776)) { + x_778 = lean_alloc_ctor(1, 1, 0); +} else { + x_778 = x_776; +} +lean_ctor_set(x_778, 0, x_777); +if (lean_is_scalar(x_662)) { + x_779 = lean_alloc_ctor(0, 2, 0); +} else { + x_779 = x_662; +} +lean_ctor_set(x_779, 0, x_778); +lean_ctor_set(x_779, 1, x_774); +x_11 = x_779; +goto block_29; +} +else +{ +lean_object* x_780; lean_object* x_781; lean_object* x_782; lean_object* x_783; size_t x_784; size_t x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; +lean_dec(x_662); +x_780 = lean_ctor_get(x_773, 0); +lean_inc(x_780); +lean_dec(x_773); +x_781 = lean_ctor_get(x_37, 0); +lean_inc(x_781); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_782 = x_37; +} else { + lean_dec_ref(x_37); + x_782 = lean_box(0); +} +x_783 = lean_array_get_size(x_781); +x_784 = lean_usize_of_nat(x_783); +lean_dec(x_783); +x_785 = 0; +x_786 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_784, x_785, x_781, x_774); +x_787 = lean_ctor_get(x_786, 0); +lean_inc(x_787); +x_788 = lean_ctor_get(x_786, 1); +lean_inc(x_788); +if (lean_is_exclusive(x_786)) { + lean_ctor_release(x_786, 0); + lean_ctor_release(x_786, 1); + x_789 = x_786; +} else { + lean_dec_ref(x_786); + x_789 = lean_box(0); +} +x_790 = lean_ctor_get(x_787, 0); +lean_inc(x_790); +if (lean_is_exclusive(x_787)) { + lean_ctor_release(x_787, 0); + x_791 = x_787; +} else { + lean_dec_ref(x_787); + x_791 = lean_box(0); +} +if (lean_is_scalar(x_782)) { + x_792 = lean_alloc_ctor(1, 1, 0); +} else { + x_792 = x_782; +} +lean_ctor_set(x_792, 0, x_790); +x_793 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_793, 0, x_31); +lean_ctor_set(x_793, 1, x_32); +lean_ctor_set(x_793, 2, x_38); +lean_ctor_set(x_793, 3, x_33); +lean_ctor_set(x_793, 4, x_34); +lean_ctor_set(x_793, 5, x_772); +lean_ctor_set(x_793, 6, x_780); +lean_ctor_set(x_793, 7, x_792); +if (lean_is_scalar(x_791)) { + x_794 = lean_alloc_ctor(1, 1, 0); +} else { + x_794 = x_791; +} +lean_ctor_set(x_794, 0, x_793); +if (lean_is_scalar(x_789)) { + x_795 = lean_alloc_ctor(0, 2, 0); +} else { + x_795 = x_789; +} +lean_ctor_set(x_795, 0, x_794); +lean_ctor_set(x_795, 1, x_788); +x_11 = x_795; +goto block_29; +} +} +} +} +} +else +{ +lean_object* x_827; lean_object* x_828; lean_object* x_829; lean_object* x_830; lean_object* x_831; +x_827 = lean_ctor_get(x_34, 0); +lean_inc(x_827); +lean_dec(x_34); +x_828 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_828, 0, x_827); +x_829 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_830 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_829, x_35, x_4); +x_831 = lean_ctor_get(x_830, 0); +lean_inc(x_831); +if (lean_obj_tag(x_831) == 0) +{ +lean_object* x_832; lean_object* x_833; lean_object* x_834; lean_object* x_835; lean_object* x_836; lean_object* x_837; +lean_dec(x_828); +lean_dec(x_33); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_32); +lean_dec(x_31); +x_832 = lean_ctor_get(x_830, 1); +lean_inc(x_832); +if (lean_is_exclusive(x_830)) { + lean_ctor_release(x_830, 0); + lean_ctor_release(x_830, 1); + x_833 = x_830; +} else { + lean_dec_ref(x_830); + x_833 = lean_box(0); +} +x_834 = lean_ctor_get(x_831, 0); +lean_inc(x_834); +if (lean_is_exclusive(x_831)) { + lean_ctor_release(x_831, 0); + x_835 = x_831; +} else { + lean_dec_ref(x_831); + x_835 = lean_box(0); +} +if (lean_is_scalar(x_835)) { + x_836 = lean_alloc_ctor(0, 1, 0); +} else { + x_836 = x_835; +} +lean_ctor_set(x_836, 0, x_834); +if (lean_is_scalar(x_833)) { + x_837 = lean_alloc_ctor(0, 2, 0); +} else { + x_837 = x_833; +} +lean_ctor_set(x_837, 0, x_836); +lean_ctor_set(x_837, 1, x_832); +x_11 = x_837; +goto block_29; +} +else +{ +lean_object* x_838; lean_object* x_839; lean_object* x_840; lean_object* x_841; lean_object* x_842; lean_object* x_843; +x_838 = lean_ctor_get(x_830, 1); +lean_inc(x_838); +if (lean_is_exclusive(x_830)) { + lean_ctor_release(x_830, 0); + lean_ctor_release(x_830, 1); + x_839 = x_830; +} else { + lean_dec_ref(x_830); + x_839 = lean_box(0); +} +x_840 = lean_ctor_get(x_831, 0); +lean_inc(x_840); +if (lean_is_exclusive(x_831)) { + lean_ctor_release(x_831, 0); + x_841 = x_831; +} else { + lean_dec_ref(x_831); + x_841 = lean_box(0); +} +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_839); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_866; lean_object* x_867; lean_object* x_868; +x_866 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_866, 0, x_31); +lean_ctor_set(x_866, 1, x_32); +lean_ctor_set(x_866, 2, x_38); +lean_ctor_set(x_866, 3, x_33); +lean_ctor_set(x_866, 4, x_828); +lean_ctor_set(x_866, 5, x_840); +lean_ctor_set(x_866, 6, x_38); +lean_ctor_set(x_866, 7, x_38); +if (lean_is_scalar(x_841)) { + x_867 = lean_alloc_ctor(1, 1, 0); +} else { + x_867 = x_841; +} +lean_ctor_set(x_867, 0, x_866); +x_868 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_868, 0, x_867); +lean_ctor_set(x_868, 1, x_838); +x_11 = x_868; +goto block_29; +} +else +{ +lean_object* x_869; lean_object* x_870; lean_object* x_871; size_t x_872; size_t x_873; lean_object* x_874; lean_object* x_875; lean_object* x_876; lean_object* x_877; lean_object* x_878; lean_object* x_879; lean_object* x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; +lean_dec(x_841); +x_869 = lean_ctor_get(x_37, 0); +lean_inc(x_869); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_870 = x_37; +} else { + lean_dec_ref(x_37); + x_870 = lean_box(0); +} +x_871 = lean_array_get_size(x_869); +x_872 = lean_usize_of_nat(x_871); +lean_dec(x_871); +x_873 = 0; +x_874 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_872, x_873, x_869, x_838); +x_875 = lean_ctor_get(x_874, 0); +lean_inc(x_875); +x_876 = lean_ctor_get(x_874, 1); +lean_inc(x_876); +if (lean_is_exclusive(x_874)) { + lean_ctor_release(x_874, 0); + lean_ctor_release(x_874, 1); + x_877 = x_874; +} else { + lean_dec_ref(x_874); + x_877 = lean_box(0); +} +x_878 = lean_ctor_get(x_875, 0); +lean_inc(x_878); +if (lean_is_exclusive(x_875)) { + lean_ctor_release(x_875, 0); + x_879 = x_875; +} else { + lean_dec_ref(x_875); + x_879 = lean_box(0); +} +if (lean_is_scalar(x_870)) { + x_880 = lean_alloc_ctor(1, 1, 0); +} else { + x_880 = x_870; +} +lean_ctor_set(x_880, 0, x_878); +x_881 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_881, 0, x_31); +lean_ctor_set(x_881, 1, x_32); +lean_ctor_set(x_881, 2, x_38); +lean_ctor_set(x_881, 3, x_33); +lean_ctor_set(x_881, 4, x_828); +lean_ctor_set(x_881, 5, x_840); +lean_ctor_set(x_881, 6, x_38); +lean_ctor_set(x_881, 7, x_880); +if (lean_is_scalar(x_879)) { + x_882 = lean_alloc_ctor(1, 1, 0); +} else { + x_882 = x_879; +} +lean_ctor_set(x_882, 0, x_881); +if (lean_is_scalar(x_877)) { + x_883 = lean_alloc_ctor(0, 2, 0); +} else { + x_883 = x_877; +} +lean_ctor_set(x_883, 0, x_882); +lean_ctor_set(x_883, 1, x_876); +x_11 = x_883; +goto block_29; +} +} +else +{ +lean_object* x_884; lean_object* x_885; lean_object* x_886; size_t x_887; size_t x_888; lean_object* x_889; lean_object* x_890; lean_object* x_891; lean_object* x_892; lean_object* x_893; lean_object* x_894; lean_object* x_895; +lean_dec(x_841); +x_884 = lean_ctor_get(x_36, 0); +lean_inc(x_884); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_885 = x_36; +} else { + lean_dec_ref(x_36); + x_885 = lean_box(0); +} +x_886 = lean_array_get_size(x_884); +x_887 = lean_usize_of_nat(x_886); +lean_dec(x_886); +x_888 = 0; +x_889 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_887, x_888, x_884, x_838); +x_890 = lean_ctor_get(x_889, 0); +lean_inc(x_890); +x_891 = lean_ctor_get(x_889, 1); +lean_inc(x_891); +lean_dec(x_889); +x_892 = lean_ctor_get(x_890, 0); +lean_inc(x_892); +if (lean_is_exclusive(x_890)) { + lean_ctor_release(x_890, 0); + x_893 = x_890; +} else { + lean_dec_ref(x_890); + x_893 = lean_box(0); +} +if (lean_is_scalar(x_885)) { + x_894 = lean_alloc_ctor(1, 1, 0); +} else { + x_894 = x_885; +} +lean_ctor_set(x_894, 0, x_892); +if (lean_is_scalar(x_893)) { + x_895 = lean_alloc_ctor(1, 1, 0); +} else { + x_895 = x_893; +} +lean_ctor_set(x_895, 0, x_894); +x_842 = x_895; +x_843 = x_891; +goto block_865; +} +block_865: +{ +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_844; lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; +x_844 = lean_ctor_get(x_842, 0); +lean_inc(x_844); +if (lean_is_exclusive(x_842)) { + lean_ctor_release(x_842, 0); + x_845 = x_842; +} else { + lean_dec_ref(x_842); + x_845 = lean_box(0); +} +x_846 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_846, 0, x_31); +lean_ctor_set(x_846, 1, x_32); +lean_ctor_set(x_846, 2, x_38); +lean_ctor_set(x_846, 3, x_33); +lean_ctor_set(x_846, 4, x_828); +lean_ctor_set(x_846, 5, x_840); +lean_ctor_set(x_846, 6, x_844); +lean_ctor_set(x_846, 7, x_38); +if (lean_is_scalar(x_845)) { + x_847 = lean_alloc_ctor(1, 1, 0); +} else { + x_847 = x_845; +} +lean_ctor_set(x_847, 0, x_846); +if (lean_is_scalar(x_839)) { + x_848 = lean_alloc_ctor(0, 2, 0); +} else { + x_848 = x_839; +} +lean_ctor_set(x_848, 0, x_847); +lean_ctor_set(x_848, 1, x_843); +x_11 = x_848; +goto block_29; +} +else +{ +lean_object* x_849; lean_object* x_850; lean_object* x_851; lean_object* x_852; size_t x_853; size_t x_854; lean_object* x_855; lean_object* x_856; lean_object* x_857; lean_object* x_858; lean_object* x_859; lean_object* x_860; lean_object* x_861; lean_object* x_862; lean_object* x_863; lean_object* x_864; +lean_dec(x_839); +x_849 = lean_ctor_get(x_842, 0); +lean_inc(x_849); +lean_dec(x_842); +x_850 = lean_ctor_get(x_37, 0); +lean_inc(x_850); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_851 = x_37; +} else { + lean_dec_ref(x_37); + x_851 = lean_box(0); +} +x_852 = lean_array_get_size(x_850); +x_853 = lean_usize_of_nat(x_852); +lean_dec(x_852); +x_854 = 0; +x_855 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_853, x_854, x_850, x_843); +x_856 = lean_ctor_get(x_855, 0); +lean_inc(x_856); +x_857 = lean_ctor_get(x_855, 1); +lean_inc(x_857); +if (lean_is_exclusive(x_855)) { + lean_ctor_release(x_855, 0); + lean_ctor_release(x_855, 1); + x_858 = x_855; +} else { + lean_dec_ref(x_855); + x_858 = lean_box(0); +} +x_859 = lean_ctor_get(x_856, 0); +lean_inc(x_859); +if (lean_is_exclusive(x_856)) { + lean_ctor_release(x_856, 0); + x_860 = x_856; +} else { + lean_dec_ref(x_856); + x_860 = lean_box(0); +} +if (lean_is_scalar(x_851)) { + x_861 = lean_alloc_ctor(1, 1, 0); +} else { + x_861 = x_851; +} +lean_ctor_set(x_861, 0, x_859); +x_862 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_862, 0, x_31); +lean_ctor_set(x_862, 1, x_32); +lean_ctor_set(x_862, 2, x_38); +lean_ctor_set(x_862, 3, x_33); +lean_ctor_set(x_862, 4, x_828); +lean_ctor_set(x_862, 5, x_840); +lean_ctor_set(x_862, 6, x_849); +lean_ctor_set(x_862, 7, x_861); +if (lean_is_scalar(x_860)) { + x_863 = lean_alloc_ctor(1, 1, 0); +} else { + x_863 = x_860; +} +lean_ctor_set(x_863, 0, x_862); +if (lean_is_scalar(x_858)) { + x_864 = lean_alloc_ctor(0, 2, 0); +} else { + x_864 = x_858; +} +lean_ctor_set(x_864, 0, x_863); +lean_ctor_set(x_864, 1, x_857); +x_11 = x_864; +goto block_29; +} +} +} +} +} +} +else +{ +lean_object* x_896; lean_object* x_897; +x_896 = lean_ctor_get(x_33, 0); +lean_inc(x_896); +lean_dec(x_33); +x_897 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_897, 0, x_896); +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_898; lean_object* x_899; lean_object* x_900; +x_898 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_899 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_898, x_35, x_4); +x_900 = lean_ctor_get(x_899, 0); +lean_inc(x_900); +if (lean_obj_tag(x_900) == 0) +{ +lean_object* x_901; lean_object* x_902; lean_object* x_903; lean_object* x_904; lean_object* x_905; lean_object* x_906; +lean_dec(x_897); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_32); +lean_dec(x_31); +x_901 = lean_ctor_get(x_899, 1); +lean_inc(x_901); +if (lean_is_exclusive(x_899)) { + lean_ctor_release(x_899, 0); + lean_ctor_release(x_899, 1); + x_902 = x_899; +} else { + lean_dec_ref(x_899); + x_902 = lean_box(0); +} +x_903 = lean_ctor_get(x_900, 0); +lean_inc(x_903); +if (lean_is_exclusive(x_900)) { + lean_ctor_release(x_900, 0); + x_904 = x_900; +} else { + lean_dec_ref(x_900); + x_904 = lean_box(0); +} +if (lean_is_scalar(x_904)) { + x_905 = lean_alloc_ctor(0, 1, 0); +} else { + x_905 = x_904; +} +lean_ctor_set(x_905, 0, x_903); +if (lean_is_scalar(x_902)) { + x_906 = lean_alloc_ctor(0, 2, 0); +} else { + x_906 = x_902; +} +lean_ctor_set(x_906, 0, x_905); +lean_ctor_set(x_906, 1, x_901); +x_11 = x_906; +goto block_29; +} +else +{ +lean_object* x_907; lean_object* x_908; lean_object* x_909; lean_object* x_910; lean_object* x_911; lean_object* x_912; +x_907 = lean_ctor_get(x_899, 1); +lean_inc(x_907); +if (lean_is_exclusive(x_899)) { + lean_ctor_release(x_899, 0); + lean_ctor_release(x_899, 1); + x_908 = x_899; +} else { + lean_dec_ref(x_899); + x_908 = lean_box(0); +} +x_909 = lean_ctor_get(x_900, 0); +lean_inc(x_909); +if (lean_is_exclusive(x_900)) { + lean_ctor_release(x_900, 0); + x_910 = x_900; +} else { + lean_dec_ref(x_900); + x_910 = lean_box(0); +} +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_908); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_935; lean_object* x_936; lean_object* x_937; +x_935 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_935, 0, x_31); +lean_ctor_set(x_935, 1, x_32); +lean_ctor_set(x_935, 2, x_38); +lean_ctor_set(x_935, 3, x_897); +lean_ctor_set(x_935, 4, x_38); +lean_ctor_set(x_935, 5, x_909); +lean_ctor_set(x_935, 6, x_38); +lean_ctor_set(x_935, 7, x_38); +if (lean_is_scalar(x_910)) { + x_936 = lean_alloc_ctor(1, 1, 0); +} else { + x_936 = x_910; +} +lean_ctor_set(x_936, 0, x_935); +x_937 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_937, 0, x_936); +lean_ctor_set(x_937, 1, x_907); +x_11 = x_937; +goto block_29; +} +else +{ +lean_object* x_938; lean_object* x_939; lean_object* x_940; size_t x_941; size_t x_942; lean_object* x_943; lean_object* x_944; lean_object* x_945; lean_object* x_946; lean_object* x_947; lean_object* x_948; lean_object* x_949; lean_object* x_950; lean_object* x_951; lean_object* x_952; +lean_dec(x_910); +x_938 = lean_ctor_get(x_37, 0); +lean_inc(x_938); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_939 = x_37; +} else { + lean_dec_ref(x_37); + x_939 = lean_box(0); +} +x_940 = lean_array_get_size(x_938); +x_941 = lean_usize_of_nat(x_940); +lean_dec(x_940); +x_942 = 0; +x_943 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_941, x_942, x_938, x_907); +x_944 = lean_ctor_get(x_943, 0); +lean_inc(x_944); +x_945 = lean_ctor_get(x_943, 1); +lean_inc(x_945); +if (lean_is_exclusive(x_943)) { + lean_ctor_release(x_943, 0); + lean_ctor_release(x_943, 1); + x_946 = x_943; +} else { + lean_dec_ref(x_943); + x_946 = lean_box(0); +} +x_947 = lean_ctor_get(x_944, 0); +lean_inc(x_947); +if (lean_is_exclusive(x_944)) { + lean_ctor_release(x_944, 0); + x_948 = x_944; +} else { + lean_dec_ref(x_944); + x_948 = lean_box(0); +} +if (lean_is_scalar(x_939)) { + x_949 = lean_alloc_ctor(1, 1, 0); +} else { + x_949 = x_939; +} +lean_ctor_set(x_949, 0, x_947); +x_950 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_950, 0, x_31); +lean_ctor_set(x_950, 1, x_32); +lean_ctor_set(x_950, 2, x_38); +lean_ctor_set(x_950, 3, x_897); +lean_ctor_set(x_950, 4, x_38); +lean_ctor_set(x_950, 5, x_909); +lean_ctor_set(x_950, 6, x_38); +lean_ctor_set(x_950, 7, x_949); +if (lean_is_scalar(x_948)) { + x_951 = lean_alloc_ctor(1, 1, 0); +} else { + x_951 = x_948; +} +lean_ctor_set(x_951, 0, x_950); +if (lean_is_scalar(x_946)) { + x_952 = lean_alloc_ctor(0, 2, 0); +} else { + x_952 = x_946; +} +lean_ctor_set(x_952, 0, x_951); +lean_ctor_set(x_952, 1, x_945); +x_11 = x_952; +goto block_29; +} +} +else +{ +lean_object* x_953; lean_object* x_954; lean_object* x_955; size_t x_956; size_t x_957; lean_object* x_958; lean_object* x_959; lean_object* x_960; lean_object* x_961; lean_object* x_962; lean_object* x_963; lean_object* x_964; +lean_dec(x_910); +x_953 = lean_ctor_get(x_36, 0); +lean_inc(x_953); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_954 = x_36; +} else { + lean_dec_ref(x_36); + x_954 = lean_box(0); +} +x_955 = lean_array_get_size(x_953); +x_956 = lean_usize_of_nat(x_955); +lean_dec(x_955); +x_957 = 0; +x_958 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_956, x_957, x_953, x_907); +x_959 = lean_ctor_get(x_958, 0); +lean_inc(x_959); +x_960 = lean_ctor_get(x_958, 1); +lean_inc(x_960); +lean_dec(x_958); +x_961 = lean_ctor_get(x_959, 0); +lean_inc(x_961); +if (lean_is_exclusive(x_959)) { + lean_ctor_release(x_959, 0); + x_962 = x_959; +} else { + lean_dec_ref(x_959); + x_962 = lean_box(0); +} +if (lean_is_scalar(x_954)) { + x_963 = lean_alloc_ctor(1, 1, 0); +} else { + x_963 = x_954; +} +lean_ctor_set(x_963, 0, x_961); +if (lean_is_scalar(x_962)) { + x_964 = lean_alloc_ctor(1, 1, 0); +} else { + x_964 = x_962; +} +lean_ctor_set(x_964, 0, x_963); +x_911 = x_964; +x_912 = x_960; +goto block_934; +} +block_934: +{ +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_913; lean_object* x_914; lean_object* x_915; lean_object* x_916; lean_object* x_917; +x_913 = lean_ctor_get(x_911, 0); +lean_inc(x_913); +if (lean_is_exclusive(x_911)) { + lean_ctor_release(x_911, 0); + x_914 = x_911; +} else { + lean_dec_ref(x_911); + x_914 = lean_box(0); +} +x_915 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_915, 0, x_31); +lean_ctor_set(x_915, 1, x_32); +lean_ctor_set(x_915, 2, x_38); +lean_ctor_set(x_915, 3, x_897); +lean_ctor_set(x_915, 4, x_38); +lean_ctor_set(x_915, 5, x_909); +lean_ctor_set(x_915, 6, x_913); +lean_ctor_set(x_915, 7, x_38); +if (lean_is_scalar(x_914)) { + x_916 = lean_alloc_ctor(1, 1, 0); +} else { + x_916 = x_914; +} +lean_ctor_set(x_916, 0, x_915); +if (lean_is_scalar(x_908)) { + x_917 = lean_alloc_ctor(0, 2, 0); +} else { + x_917 = x_908; +} +lean_ctor_set(x_917, 0, x_916); +lean_ctor_set(x_917, 1, x_912); +x_11 = x_917; +goto block_29; +} +else +{ +lean_object* x_918; lean_object* x_919; lean_object* x_920; lean_object* x_921; size_t x_922; size_t x_923; lean_object* x_924; lean_object* x_925; lean_object* x_926; lean_object* x_927; lean_object* x_928; lean_object* x_929; lean_object* x_930; lean_object* x_931; lean_object* x_932; lean_object* x_933; +lean_dec(x_908); +x_918 = lean_ctor_get(x_911, 0); +lean_inc(x_918); +lean_dec(x_911); +x_919 = lean_ctor_get(x_37, 0); +lean_inc(x_919); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_920 = x_37; +} else { + lean_dec_ref(x_37); + x_920 = lean_box(0); +} +x_921 = lean_array_get_size(x_919); +x_922 = lean_usize_of_nat(x_921); +lean_dec(x_921); +x_923 = 0; +x_924 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_922, x_923, x_919, x_912); +x_925 = lean_ctor_get(x_924, 0); +lean_inc(x_925); +x_926 = lean_ctor_get(x_924, 1); +lean_inc(x_926); +if (lean_is_exclusive(x_924)) { + lean_ctor_release(x_924, 0); + lean_ctor_release(x_924, 1); + x_927 = x_924; +} else { + lean_dec_ref(x_924); + x_927 = lean_box(0); +} +x_928 = lean_ctor_get(x_925, 0); +lean_inc(x_928); +if (lean_is_exclusive(x_925)) { + lean_ctor_release(x_925, 0); + x_929 = x_925; +} else { + lean_dec_ref(x_925); + x_929 = lean_box(0); +} +if (lean_is_scalar(x_920)) { + x_930 = lean_alloc_ctor(1, 1, 0); +} else { + x_930 = x_920; +} +lean_ctor_set(x_930, 0, x_928); +x_931 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_931, 0, x_31); +lean_ctor_set(x_931, 1, x_32); +lean_ctor_set(x_931, 2, x_38); +lean_ctor_set(x_931, 3, x_897); +lean_ctor_set(x_931, 4, x_38); +lean_ctor_set(x_931, 5, x_909); +lean_ctor_set(x_931, 6, x_918); +lean_ctor_set(x_931, 7, x_930); +if (lean_is_scalar(x_929)) { + x_932 = lean_alloc_ctor(1, 1, 0); +} else { + x_932 = x_929; +} +lean_ctor_set(x_932, 0, x_931); +if (lean_is_scalar(x_927)) { + x_933 = lean_alloc_ctor(0, 2, 0); +} else { + x_933 = x_927; +} +lean_ctor_set(x_933, 0, x_932); +lean_ctor_set(x_933, 1, x_926); +x_11 = x_933; +goto block_29; +} +} +} +} +else +{ +lean_object* x_965; lean_object* x_966; lean_object* x_967; lean_object* x_968; lean_object* x_969; lean_object* x_970; +x_965 = lean_ctor_get(x_34, 0); +lean_inc(x_965); +if (lean_is_exclusive(x_34)) { + lean_ctor_release(x_34, 0); + x_966 = x_34; +} else { + lean_dec_ref(x_34); + x_966 = lean_box(0); +} +if (lean_is_scalar(x_966)) { + x_967 = lean_alloc_ctor(1, 1, 0); +} else { + x_967 = x_966; +} +lean_ctor_set(x_967, 0, x_965); +x_968 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_969 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_968, x_35, x_4); +x_970 = lean_ctor_get(x_969, 0); +lean_inc(x_970); +if (lean_obj_tag(x_970) == 0) +{ +lean_object* x_971; lean_object* x_972; lean_object* x_973; lean_object* x_974; lean_object* x_975; lean_object* x_976; +lean_dec(x_967); +lean_dec(x_897); +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_32); +lean_dec(x_31); +x_971 = lean_ctor_get(x_969, 1); +lean_inc(x_971); +if (lean_is_exclusive(x_969)) { + lean_ctor_release(x_969, 0); + lean_ctor_release(x_969, 1); + x_972 = x_969; +} else { + lean_dec_ref(x_969); + x_972 = lean_box(0); +} +x_973 = lean_ctor_get(x_970, 0); +lean_inc(x_973); +if (lean_is_exclusive(x_970)) { + lean_ctor_release(x_970, 0); + x_974 = x_970; +} else { + lean_dec_ref(x_970); + x_974 = lean_box(0); +} +if (lean_is_scalar(x_974)) { + x_975 = lean_alloc_ctor(0, 1, 0); +} else { + x_975 = x_974; +} +lean_ctor_set(x_975, 0, x_973); +if (lean_is_scalar(x_972)) { + x_976 = lean_alloc_ctor(0, 2, 0); +} else { + x_976 = x_972; +} +lean_ctor_set(x_976, 0, x_975); +lean_ctor_set(x_976, 1, x_971); +x_11 = x_976; +goto block_29; +} +else +{ +lean_object* x_977; lean_object* x_978; lean_object* x_979; lean_object* x_980; lean_object* x_981; lean_object* x_982; +x_977 = lean_ctor_get(x_969, 1); +lean_inc(x_977); +if (lean_is_exclusive(x_969)) { + lean_ctor_release(x_969, 0); + lean_ctor_release(x_969, 1); + x_978 = x_969; +} else { + lean_dec_ref(x_969); + x_978 = lean_box(0); +} +x_979 = lean_ctor_get(x_970, 0); +lean_inc(x_979); +if (lean_is_exclusive(x_970)) { + lean_ctor_release(x_970, 0); + x_980 = x_970; +} else { + lean_dec_ref(x_970); + x_980 = lean_box(0); +} +if (lean_obj_tag(x_36) == 0) +{ +lean_dec(x_978); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_1005; lean_object* x_1006; lean_object* x_1007; +x_1005 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1005, 0, x_31); +lean_ctor_set(x_1005, 1, x_32); +lean_ctor_set(x_1005, 2, x_38); +lean_ctor_set(x_1005, 3, x_897); +lean_ctor_set(x_1005, 4, x_967); +lean_ctor_set(x_1005, 5, x_979); +lean_ctor_set(x_1005, 6, x_38); +lean_ctor_set(x_1005, 7, x_38); +if (lean_is_scalar(x_980)) { + x_1006 = lean_alloc_ctor(1, 1, 0); +} else { + x_1006 = x_980; +} +lean_ctor_set(x_1006, 0, x_1005); +x_1007 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1007, 0, x_1006); +lean_ctor_set(x_1007, 1, x_977); +x_11 = x_1007; +goto block_29; +} +else +{ +lean_object* x_1008; lean_object* x_1009; lean_object* x_1010; size_t x_1011; size_t x_1012; lean_object* x_1013; lean_object* x_1014; lean_object* x_1015; lean_object* x_1016; lean_object* x_1017; lean_object* x_1018; lean_object* x_1019; lean_object* x_1020; lean_object* x_1021; lean_object* x_1022; +lean_dec(x_980); +x_1008 = lean_ctor_get(x_37, 0); +lean_inc(x_1008); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_1009 = x_37; +} else { + lean_dec_ref(x_37); + x_1009 = lean_box(0); +} +x_1010 = lean_array_get_size(x_1008); +x_1011 = lean_usize_of_nat(x_1010); +lean_dec(x_1010); +x_1012 = 0; +x_1013 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1011, x_1012, x_1008, x_977); +x_1014 = lean_ctor_get(x_1013, 0); +lean_inc(x_1014); +x_1015 = lean_ctor_get(x_1013, 1); +lean_inc(x_1015); +if (lean_is_exclusive(x_1013)) { + lean_ctor_release(x_1013, 0); + lean_ctor_release(x_1013, 1); + x_1016 = x_1013; +} else { + lean_dec_ref(x_1013); + x_1016 = lean_box(0); +} +x_1017 = lean_ctor_get(x_1014, 0); +lean_inc(x_1017); +if (lean_is_exclusive(x_1014)) { + lean_ctor_release(x_1014, 0); + x_1018 = x_1014; +} else { + lean_dec_ref(x_1014); + x_1018 = lean_box(0); +} +if (lean_is_scalar(x_1009)) { + x_1019 = lean_alloc_ctor(1, 1, 0); +} else { + x_1019 = x_1009; +} +lean_ctor_set(x_1019, 0, x_1017); +x_1020 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1020, 0, x_31); +lean_ctor_set(x_1020, 1, x_32); +lean_ctor_set(x_1020, 2, x_38); +lean_ctor_set(x_1020, 3, x_897); +lean_ctor_set(x_1020, 4, x_967); +lean_ctor_set(x_1020, 5, x_979); +lean_ctor_set(x_1020, 6, x_38); +lean_ctor_set(x_1020, 7, x_1019); +if (lean_is_scalar(x_1018)) { + x_1021 = lean_alloc_ctor(1, 1, 0); +} else { + x_1021 = x_1018; +} +lean_ctor_set(x_1021, 0, x_1020); +if (lean_is_scalar(x_1016)) { + x_1022 = lean_alloc_ctor(0, 2, 0); +} else { + x_1022 = x_1016; +} +lean_ctor_set(x_1022, 0, x_1021); +lean_ctor_set(x_1022, 1, x_1015); +x_11 = x_1022; +goto block_29; +} +} +else +{ +lean_object* x_1023; lean_object* x_1024; lean_object* x_1025; size_t x_1026; size_t x_1027; lean_object* x_1028; lean_object* x_1029; lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; lean_object* x_1033; lean_object* x_1034; +lean_dec(x_980); +x_1023 = lean_ctor_get(x_36, 0); +lean_inc(x_1023); +if (lean_is_exclusive(x_36)) { + lean_ctor_release(x_36, 0); + x_1024 = x_36; +} else { + lean_dec_ref(x_36); + x_1024 = lean_box(0); +} +x_1025 = lean_array_get_size(x_1023); +x_1026 = lean_usize_of_nat(x_1025); +lean_dec(x_1025); +x_1027 = 0; +x_1028 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1026, x_1027, x_1023, x_977); +x_1029 = lean_ctor_get(x_1028, 0); +lean_inc(x_1029); +x_1030 = lean_ctor_get(x_1028, 1); +lean_inc(x_1030); +lean_dec(x_1028); +x_1031 = lean_ctor_get(x_1029, 0); +lean_inc(x_1031); +if (lean_is_exclusive(x_1029)) { + lean_ctor_release(x_1029, 0); + x_1032 = x_1029; +} else { + lean_dec_ref(x_1029); + x_1032 = lean_box(0); +} +if (lean_is_scalar(x_1024)) { + x_1033 = lean_alloc_ctor(1, 1, 0); +} else { + x_1033 = x_1024; +} +lean_ctor_set(x_1033, 0, x_1031); +if (lean_is_scalar(x_1032)) { + x_1034 = lean_alloc_ctor(1, 1, 0); +} else { + x_1034 = x_1032; +} +lean_ctor_set(x_1034, 0, x_1033); +x_981 = x_1034; +x_982 = x_1030; +goto block_1004; +} +block_1004: +{ +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_983; lean_object* x_984; lean_object* x_985; lean_object* x_986; lean_object* x_987; +x_983 = lean_ctor_get(x_981, 0); +lean_inc(x_983); +if (lean_is_exclusive(x_981)) { + lean_ctor_release(x_981, 0); + x_984 = x_981; +} else { + lean_dec_ref(x_981); + x_984 = lean_box(0); +} +x_985 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_985, 0, x_31); +lean_ctor_set(x_985, 1, x_32); +lean_ctor_set(x_985, 2, x_38); +lean_ctor_set(x_985, 3, x_897); +lean_ctor_set(x_985, 4, x_967); +lean_ctor_set(x_985, 5, x_979); +lean_ctor_set(x_985, 6, x_983); +lean_ctor_set(x_985, 7, x_38); +if (lean_is_scalar(x_984)) { + x_986 = lean_alloc_ctor(1, 1, 0); +} else { + x_986 = x_984; +} +lean_ctor_set(x_986, 0, x_985); +if (lean_is_scalar(x_978)) { + x_987 = lean_alloc_ctor(0, 2, 0); +} else { + x_987 = x_978; +} +lean_ctor_set(x_987, 0, x_986); +lean_ctor_set(x_987, 1, x_982); +x_11 = x_987; +goto block_29; +} +else +{ +lean_object* x_988; lean_object* x_989; lean_object* x_990; lean_object* x_991; size_t x_992; size_t x_993; lean_object* x_994; lean_object* x_995; lean_object* x_996; lean_object* x_997; lean_object* x_998; lean_object* x_999; lean_object* x_1000; lean_object* x_1001; lean_object* x_1002; lean_object* x_1003; +lean_dec(x_978); +x_988 = lean_ctor_get(x_981, 0); +lean_inc(x_988); +lean_dec(x_981); +x_989 = lean_ctor_get(x_37, 0); +lean_inc(x_989); +if (lean_is_exclusive(x_37)) { + lean_ctor_release(x_37, 0); + x_990 = x_37; +} else { + lean_dec_ref(x_37); + x_990 = lean_box(0); +} +x_991 = lean_array_get_size(x_989); +x_992 = lean_usize_of_nat(x_991); +lean_dec(x_991); +x_993 = 0; +x_994 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_992, x_993, x_989, x_982); +x_995 = lean_ctor_get(x_994, 0); +lean_inc(x_995); +x_996 = lean_ctor_get(x_994, 1); +lean_inc(x_996); +if (lean_is_exclusive(x_994)) { + lean_ctor_release(x_994, 0); + lean_ctor_release(x_994, 1); + x_997 = x_994; +} else { + lean_dec_ref(x_994); + x_997 = lean_box(0); +} +x_998 = lean_ctor_get(x_995, 0); +lean_inc(x_998); +if (lean_is_exclusive(x_995)) { + lean_ctor_release(x_995, 0); + x_999 = x_995; +} else { + lean_dec_ref(x_995); + x_999 = lean_box(0); +} +if (lean_is_scalar(x_990)) { + x_1000 = lean_alloc_ctor(1, 1, 0); +} else { + x_1000 = x_990; +} +lean_ctor_set(x_1000, 0, x_998); +x_1001 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1001, 0, x_31); +lean_ctor_set(x_1001, 1, x_32); +lean_ctor_set(x_1001, 2, x_38); +lean_ctor_set(x_1001, 3, x_897); +lean_ctor_set(x_1001, 4, x_967); +lean_ctor_set(x_1001, 5, x_979); +lean_ctor_set(x_1001, 6, x_988); +lean_ctor_set(x_1001, 7, x_1000); +if (lean_is_scalar(x_999)) { + x_1002 = lean_alloc_ctor(1, 1, 0); +} else { + x_1002 = x_999; +} +lean_ctor_set(x_1002, 0, x_1001); +if (lean_is_scalar(x_997)) { + x_1003 = lean_alloc_ctor(0, 2, 0); +} else { + x_1003 = x_997; +} +lean_ctor_set(x_1003, 0, x_1002); +lean_ctor_set(x_1003, 1, x_996); +x_11 = x_1003; +goto block_29; +} +} +} +} +} +} +} +else +{ +lean_object* x_1035; lean_object* x_1036; lean_object* x_1037; lean_object* x_1038; lean_object* x_1039; lean_object* x_1040; lean_object* x_1041; uint8_t x_1042; +x_1035 = lean_ctor_get(x_8, 0); +lean_inc(x_1035); +x_1036 = lean_ctor_get(x_8, 1); +lean_inc(x_1036); +x_1037 = lean_ctor_get(x_8, 3); +lean_inc(x_1037); +x_1038 = lean_ctor_get(x_8, 4); +lean_inc(x_1038); +x_1039 = lean_ctor_get(x_8, 5); +lean_inc(x_1039); +x_1040 = lean_ctor_get(x_8, 6); +lean_inc(x_1040); +x_1041 = lean_ctor_get(x_8, 7); +lean_inc(x_1041); +lean_dec(x_8); +x_1042 = !lean_is_exclusive(x_30); +if (x_1042 == 0) +{ +if (lean_obj_tag(x_1037) == 0) +{ +lean_object* x_1043; +x_1043 = lean_box(0); +if (lean_obj_tag(x_1038) == 0) +{ +lean_object* x_1044; lean_object* x_1045; lean_object* x_1046; +x_1044 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_1045 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1044, x_1039, x_4); +x_1046 = lean_ctor_get(x_1045, 0); +lean_inc(x_1046); +if (lean_obj_tag(x_1046) == 0) +{ +uint8_t x_1047; +lean_dec(x_30); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_1047 = !lean_is_exclusive(x_1045); +if (x_1047 == 0) +{ +lean_object* x_1048; uint8_t x_1049; +x_1048 = lean_ctor_get(x_1045, 0); +lean_dec(x_1048); +x_1049 = !lean_is_exclusive(x_1046); +if (x_1049 == 0) +{ +x_11 = x_1045; +goto block_29; +} +else +{ +lean_object* x_1050; lean_object* x_1051; +x_1050 = lean_ctor_get(x_1046, 0); +lean_inc(x_1050); +lean_dec(x_1046); +x_1051 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_1051, 0, x_1050); +lean_ctor_set(x_1045, 0, x_1051); +x_11 = x_1045; +goto block_29; +} +} +else +{ +lean_object* x_1052; lean_object* x_1053; lean_object* x_1054; lean_object* x_1055; lean_object* x_1056; +x_1052 = lean_ctor_get(x_1045, 1); +lean_inc(x_1052); +lean_dec(x_1045); +x_1053 = lean_ctor_get(x_1046, 0); +lean_inc(x_1053); +if (lean_is_exclusive(x_1046)) { + lean_ctor_release(x_1046, 0); + x_1054 = x_1046; +} else { + lean_dec_ref(x_1046); + x_1054 = lean_box(0); +} +if (lean_is_scalar(x_1054)) { + x_1055 = lean_alloc_ctor(0, 1, 0); +} else { + x_1055 = x_1054; +} +lean_ctor_set(x_1055, 0, x_1053); +x_1056 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1056, 0, x_1055); +lean_ctor_set(x_1056, 1, x_1052); +x_11 = x_1056; +goto block_29; +} +} +else +{ +lean_object* x_1057; lean_object* x_1058; uint8_t x_1059; +x_1057 = lean_ctor_get(x_1045, 1); +lean_inc(x_1057); +if (lean_is_exclusive(x_1045)) { + lean_ctor_release(x_1045, 0); + lean_ctor_release(x_1045, 1); + x_1058 = x_1045; +} else { + lean_dec_ref(x_1045); + x_1058 = lean_box(0); +} +x_1059 = !lean_is_exclusive(x_1046); +if (x_1059 == 0) +{ +lean_object* x_1060; lean_object* x_1061; lean_object* x_1062; +x_1060 = lean_ctor_get(x_1046, 0); +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_1058); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1108; lean_object* x_1109; +x_1108 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1108, 0, x_1035); +lean_ctor_set(x_1108, 1, x_1036); +lean_ctor_set(x_1108, 2, x_30); +lean_ctor_set(x_1108, 3, x_1043); +lean_ctor_set(x_1108, 4, x_1043); +lean_ctor_set(x_1108, 5, x_1060); +lean_ctor_set(x_1108, 6, x_1043); +lean_ctor_set(x_1108, 7, x_1043); +lean_ctor_set(x_1046, 0, x_1108); +x_1109 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1109, 0, x_1046); +lean_ctor_set(x_1109, 1, x_1057); +x_11 = x_1109; +goto block_29; +} +else +{ +uint8_t x_1110; +lean_free_object(x_1046); +x_1110 = !lean_is_exclusive(x_1041); +if (x_1110 == 0) +{ +lean_object* x_1111; lean_object* x_1112; size_t x_1113; size_t x_1114; lean_object* x_1115; uint8_t x_1116; +x_1111 = lean_ctor_get(x_1041, 0); +x_1112 = lean_array_get_size(x_1111); +x_1113 = lean_usize_of_nat(x_1112); +lean_dec(x_1112); +x_1114 = 0; +x_1115 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1113, x_1114, x_1111, x_1057); +x_1116 = !lean_is_exclusive(x_1115); +if (x_1116 == 0) +{ +lean_object* x_1117; uint8_t x_1118; +x_1117 = lean_ctor_get(x_1115, 0); +x_1118 = !lean_is_exclusive(x_1117); +if (x_1118 == 0) +{ +lean_object* x_1119; lean_object* x_1120; +x_1119 = lean_ctor_get(x_1117, 0); +lean_ctor_set(x_1041, 0, x_1119); +x_1120 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1120, 0, x_1035); +lean_ctor_set(x_1120, 1, x_1036); +lean_ctor_set(x_1120, 2, x_30); +lean_ctor_set(x_1120, 3, x_1043); +lean_ctor_set(x_1120, 4, x_1043); +lean_ctor_set(x_1120, 5, x_1060); +lean_ctor_set(x_1120, 6, x_1043); +lean_ctor_set(x_1120, 7, x_1041); +lean_ctor_set(x_1117, 0, x_1120); +x_11 = x_1115; +goto block_29; +} +else +{ +lean_object* x_1121; lean_object* x_1122; lean_object* x_1123; +x_1121 = lean_ctor_get(x_1117, 0); +lean_inc(x_1121); +lean_dec(x_1117); +lean_ctor_set(x_1041, 0, x_1121); +x_1122 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1122, 0, x_1035); +lean_ctor_set(x_1122, 1, x_1036); +lean_ctor_set(x_1122, 2, x_30); +lean_ctor_set(x_1122, 3, x_1043); +lean_ctor_set(x_1122, 4, x_1043); +lean_ctor_set(x_1122, 5, x_1060); +lean_ctor_set(x_1122, 6, x_1043); +lean_ctor_set(x_1122, 7, x_1041); +x_1123 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1123, 0, x_1122); +lean_ctor_set(x_1115, 0, x_1123); +x_11 = x_1115; +goto block_29; +} +} +else +{ +lean_object* x_1124; lean_object* x_1125; lean_object* x_1126; lean_object* x_1127; lean_object* x_1128; lean_object* x_1129; lean_object* x_1130; +x_1124 = lean_ctor_get(x_1115, 0); +x_1125 = lean_ctor_get(x_1115, 1); +lean_inc(x_1125); +lean_inc(x_1124); +lean_dec(x_1115); +x_1126 = lean_ctor_get(x_1124, 0); +lean_inc(x_1126); +if (lean_is_exclusive(x_1124)) { + lean_ctor_release(x_1124, 0); + x_1127 = x_1124; +} else { + lean_dec_ref(x_1124); + x_1127 = lean_box(0); +} +lean_ctor_set(x_1041, 0, x_1126); +x_1128 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1128, 0, x_1035); +lean_ctor_set(x_1128, 1, x_1036); +lean_ctor_set(x_1128, 2, x_30); +lean_ctor_set(x_1128, 3, x_1043); +lean_ctor_set(x_1128, 4, x_1043); +lean_ctor_set(x_1128, 5, x_1060); +lean_ctor_set(x_1128, 6, x_1043); +lean_ctor_set(x_1128, 7, x_1041); +if (lean_is_scalar(x_1127)) { + x_1129 = lean_alloc_ctor(1, 1, 0); +} else { + x_1129 = x_1127; +} +lean_ctor_set(x_1129, 0, x_1128); +x_1130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1130, 0, x_1129); +lean_ctor_set(x_1130, 1, x_1125); +x_11 = x_1130; +goto block_29; +} +} +else +{ +lean_object* x_1131; lean_object* x_1132; size_t x_1133; size_t x_1134; lean_object* x_1135; lean_object* x_1136; lean_object* x_1137; lean_object* x_1138; lean_object* x_1139; lean_object* x_1140; lean_object* x_1141; lean_object* x_1142; lean_object* x_1143; lean_object* x_1144; +x_1131 = lean_ctor_get(x_1041, 0); +lean_inc(x_1131); +lean_dec(x_1041); +x_1132 = lean_array_get_size(x_1131); +x_1133 = lean_usize_of_nat(x_1132); +lean_dec(x_1132); +x_1134 = 0; +x_1135 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1133, x_1134, x_1131, x_1057); +x_1136 = lean_ctor_get(x_1135, 0); +lean_inc(x_1136); +x_1137 = lean_ctor_get(x_1135, 1); +lean_inc(x_1137); +if (lean_is_exclusive(x_1135)) { + lean_ctor_release(x_1135, 0); + lean_ctor_release(x_1135, 1); + x_1138 = x_1135; +} else { + lean_dec_ref(x_1135); + x_1138 = lean_box(0); +} +x_1139 = lean_ctor_get(x_1136, 0); +lean_inc(x_1139); +if (lean_is_exclusive(x_1136)) { + lean_ctor_release(x_1136, 0); + x_1140 = x_1136; +} else { + lean_dec_ref(x_1136); + x_1140 = lean_box(0); +} +x_1141 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1141, 0, x_1139); +x_1142 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1142, 0, x_1035); +lean_ctor_set(x_1142, 1, x_1036); +lean_ctor_set(x_1142, 2, x_30); +lean_ctor_set(x_1142, 3, x_1043); +lean_ctor_set(x_1142, 4, x_1043); +lean_ctor_set(x_1142, 5, x_1060); +lean_ctor_set(x_1142, 6, x_1043); +lean_ctor_set(x_1142, 7, x_1141); +if (lean_is_scalar(x_1140)) { + x_1143 = lean_alloc_ctor(1, 1, 0); +} else { + x_1143 = x_1140; +} +lean_ctor_set(x_1143, 0, x_1142); +if (lean_is_scalar(x_1138)) { + x_1144 = lean_alloc_ctor(0, 2, 0); +} else { + x_1144 = x_1138; +} +lean_ctor_set(x_1144, 0, x_1143); +lean_ctor_set(x_1144, 1, x_1137); +x_11 = x_1144; +goto block_29; +} +} +} +else +{ +uint8_t x_1145; +lean_free_object(x_1046); +x_1145 = !lean_is_exclusive(x_1040); +if (x_1145 == 0) +{ +lean_object* x_1146; lean_object* x_1147; size_t x_1148; size_t x_1149; lean_object* x_1150; lean_object* x_1151; lean_object* x_1152; uint8_t x_1153; +x_1146 = lean_ctor_get(x_1040, 0); +x_1147 = lean_array_get_size(x_1146); +x_1148 = lean_usize_of_nat(x_1147); +lean_dec(x_1147); +x_1149 = 0; +x_1150 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1148, x_1149, x_1146, x_1057); +x_1151 = lean_ctor_get(x_1150, 0); +lean_inc(x_1151); +x_1152 = lean_ctor_get(x_1150, 1); +lean_inc(x_1152); +lean_dec(x_1150); +x_1153 = !lean_is_exclusive(x_1151); +if (x_1153 == 0) +{ +lean_object* x_1154; +x_1154 = lean_ctor_get(x_1151, 0); +lean_ctor_set(x_1040, 0, x_1154); +lean_ctor_set(x_1151, 0, x_1040); +x_1061 = x_1151; +x_1062 = x_1152; +goto block_1107; +} +else +{ +lean_object* x_1155; lean_object* x_1156; +x_1155 = lean_ctor_get(x_1151, 0); +lean_inc(x_1155); +lean_dec(x_1151); +lean_ctor_set(x_1040, 0, x_1155); +x_1156 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1156, 0, x_1040); +x_1061 = x_1156; +x_1062 = x_1152; +goto block_1107; +} +} +else +{ +lean_object* x_1157; lean_object* x_1158; size_t x_1159; size_t x_1160; lean_object* x_1161; lean_object* x_1162; lean_object* x_1163; lean_object* x_1164; lean_object* x_1165; lean_object* x_1166; lean_object* x_1167; +x_1157 = lean_ctor_get(x_1040, 0); +lean_inc(x_1157); +lean_dec(x_1040); +x_1158 = lean_array_get_size(x_1157); +x_1159 = lean_usize_of_nat(x_1158); +lean_dec(x_1158); +x_1160 = 0; +x_1161 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1159, x_1160, x_1157, x_1057); +x_1162 = lean_ctor_get(x_1161, 0); +lean_inc(x_1162); +x_1163 = lean_ctor_get(x_1161, 1); +lean_inc(x_1163); +lean_dec(x_1161); +x_1164 = lean_ctor_get(x_1162, 0); +lean_inc(x_1164); +if (lean_is_exclusive(x_1162)) { + lean_ctor_release(x_1162, 0); + x_1165 = x_1162; +} else { + lean_dec_ref(x_1162); + x_1165 = lean_box(0); } +x_1166 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1166, 0, x_1164); +if (lean_is_scalar(x_1165)) { + x_1167 = lean_alloc_ctor(1, 1, 0); +} else { + x_1167 = x_1165; +} +lean_ctor_set(x_1167, 0, x_1166); +x_1061 = x_1167; +x_1062 = x_1163; +goto block_1107; +} +} +block_1107: +{ +if (lean_obj_tag(x_1041) == 0) +{ +uint8_t x_1063; +x_1063 = !lean_is_exclusive(x_1061); +if (x_1063 == 0) +{ +lean_object* x_1064; lean_object* x_1065; lean_object* x_1066; +x_1064 = lean_ctor_get(x_1061, 0); +x_1065 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1065, 0, x_1035); +lean_ctor_set(x_1065, 1, x_1036); +lean_ctor_set(x_1065, 2, x_30); +lean_ctor_set(x_1065, 3, x_1043); +lean_ctor_set(x_1065, 4, x_1043); +lean_ctor_set(x_1065, 5, x_1060); +lean_ctor_set(x_1065, 6, x_1064); +lean_ctor_set(x_1065, 7, x_1043); +lean_ctor_set(x_1061, 0, x_1065); +if (lean_is_scalar(x_1058)) { + x_1066 = lean_alloc_ctor(0, 2, 0); +} else { + x_1066 = x_1058; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +lean_ctor_set(x_1066, 0, x_1061); +lean_ctor_set(x_1066, 1, x_1062); +x_11 = x_1066; +goto block_29; +} +else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -lean_inc(x_3); -lean_inc(x_1); -x_4 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__4), 6, 2); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_3); -x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg___lambda__8), 6, 2); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_3); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_4); -lean_ctor_set(x_6, 1, x_5); -return x_6; +lean_object* x_1067; lean_object* x_1068; lean_object* x_1069; lean_object* x_1070; +x_1067 = lean_ctor_get(x_1061, 0); +lean_inc(x_1067); +lean_dec(x_1061); +x_1068 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1068, 0, x_1035); +lean_ctor_set(x_1068, 1, x_1036); +lean_ctor_set(x_1068, 2, x_30); +lean_ctor_set(x_1068, 3, x_1043); +lean_ctor_set(x_1068, 4, x_1043); +lean_ctor_set(x_1068, 5, x_1060); +lean_ctor_set(x_1068, 6, x_1067); +lean_ctor_set(x_1068, 7, x_1043); +x_1069 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1069, 0, x_1068); +if (lean_is_scalar(x_1058)) { + x_1070 = lean_alloc_ctor(0, 2, 0); +} else { + x_1070 = x_1058; } +lean_ctor_set(x_1070, 0, x_1069); +lean_ctor_set(x_1070, 1, x_1062); +x_11 = x_1070; +goto block_29; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket(lean_object* x_1) { -_start: +} +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg), 3, 0); -return x_2; +lean_object* x_1071; uint8_t x_1072; +lean_dec(x_1058); +x_1071 = lean_ctor_get(x_1061, 0); +lean_inc(x_1071); +lean_dec(x_1061); +x_1072 = !lean_is_exclusive(x_1041); +if (x_1072 == 0) +{ +lean_object* x_1073; lean_object* x_1074; size_t x_1075; size_t x_1076; lean_object* x_1077; uint8_t x_1078; +x_1073 = lean_ctor_get(x_1041, 0); +x_1074 = lean_array_get_size(x_1073); +x_1075 = lean_usize_of_nat(x_1074); +lean_dec(x_1074); +x_1076 = 0; +x_1077 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1075, x_1076, x_1073, x_1062); +x_1078 = !lean_is_exclusive(x_1077); +if (x_1078 == 0) +{ +lean_object* x_1079; uint8_t x_1080; +x_1079 = lean_ctor_get(x_1077, 0); +x_1080 = !lean_is_exclusive(x_1079); +if (x_1080 == 0) +{ +lean_object* x_1081; lean_object* x_1082; +x_1081 = lean_ctor_get(x_1079, 0); +lean_ctor_set(x_1041, 0, x_1081); +x_1082 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1082, 0, x_1035); +lean_ctor_set(x_1082, 1, x_1036); +lean_ctor_set(x_1082, 2, x_30); +lean_ctor_set(x_1082, 3, x_1043); +lean_ctor_set(x_1082, 4, x_1043); +lean_ctor_set(x_1082, 5, x_1060); +lean_ctor_set(x_1082, 6, x_1071); +lean_ctor_set(x_1082, 7, x_1041); +lean_ctor_set(x_1079, 0, x_1082); +x_11 = x_1077; +goto block_29; +} +else +{ +lean_object* x_1083; lean_object* x_1084; lean_object* x_1085; +x_1083 = lean_ctor_get(x_1079, 0); +lean_inc(x_1083); +lean_dec(x_1079); +lean_ctor_set(x_1041, 0, x_1083); +x_1084 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1084, 0, x_1035); +lean_ctor_set(x_1084, 1, x_1036); +lean_ctor_set(x_1084, 2, x_30); +lean_ctor_set(x_1084, 3, x_1043); +lean_ctor_set(x_1084, 4, x_1043); +lean_ctor_set(x_1084, 5, x_1060); +lean_ctor_set(x_1084, 6, x_1071); +lean_ctor_set(x_1084, 7, x_1041); +x_1085 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1085, 0, x_1084); +lean_ctor_set(x_1077, 0, x_1085); +x_11 = x_1077; +goto block_29; } } -LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; -x_9 = l_Lean_Elab_Info_docString_x3f(x_1, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) +lean_object* x_1086; lean_object* x_1087; lean_object* x_1088; lean_object* x_1089; lean_object* x_1090; lean_object* x_1091; lean_object* x_1092; +x_1086 = lean_ctor_get(x_1077, 0); +x_1087 = lean_ctor_get(x_1077, 1); +lean_inc(x_1087); +lean_inc(x_1086); +lean_dec(x_1077); +x_1088 = lean_ctor_get(x_1086, 0); +lean_inc(x_1088); +if (lean_is_exclusive(x_1086)) { + lean_ctor_release(x_1086, 0); + x_1089 = x_1086; +} else { + lean_dec_ref(x_1086); + x_1089 = lean_box(0); +} +lean_ctor_set(x_1041, 0, x_1088); +x_1090 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1090, 0, x_1035); +lean_ctor_set(x_1090, 1, x_1036); +lean_ctor_set(x_1090, 2, x_30); +lean_ctor_set(x_1090, 3, x_1043); +lean_ctor_set(x_1090, 4, x_1043); +lean_ctor_set(x_1090, 5, x_1060); +lean_ctor_set(x_1090, 6, x_1071); +lean_ctor_set(x_1090, 7, x_1041); +if (lean_is_scalar(x_1089)) { + x_1091 = lean_alloc_ctor(1, 1, 0); +} else { + x_1091 = x_1089; +} +lean_ctor_set(x_1091, 0, x_1090); +x_1092 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1092, 0, x_1091); +lean_ctor_set(x_1092, 1, x_1087); +x_11 = x_1092; +goto block_29; +} +} +else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) +lean_object* x_1093; lean_object* x_1094; size_t x_1095; size_t x_1096; lean_object* x_1097; lean_object* x_1098; lean_object* x_1099; lean_object* x_1100; lean_object* x_1101; lean_object* x_1102; lean_object* x_1103; lean_object* x_1104; lean_object* x_1105; lean_object* x_1106; +x_1093 = lean_ctor_get(x_1041, 0); +lean_inc(x_1093); +lean_dec(x_1041); +x_1094 = lean_array_get_size(x_1093); +x_1095 = lean_usize_of_nat(x_1094); +lean_dec(x_1094); +x_1096 = 0; +x_1097 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1095, x_1096, x_1093, x_1062); +x_1098 = lean_ctor_get(x_1097, 0); +lean_inc(x_1098); +x_1099 = lean_ctor_get(x_1097, 1); +lean_inc(x_1099); +if (lean_is_exclusive(x_1097)) { + lean_ctor_release(x_1097, 0); + lean_ctor_release(x_1097, 1); + x_1100 = x_1097; +} else { + lean_dec_ref(x_1097); + x_1100 = lean_box(0); +} +x_1101 = lean_ctor_get(x_1098, 0); +lean_inc(x_1101); +if (lean_is_exclusive(x_1098)) { + lean_ctor_release(x_1098, 0); + x_1102 = x_1098; +} else { + lean_dec_ref(x_1098); + x_1102 = lean_box(0); +} +x_1103 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1103, 0, x_1101); +x_1104 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1104, 0, x_1035); +lean_ctor_set(x_1104, 1, x_1036); +lean_ctor_set(x_1104, 2, x_30); +lean_ctor_set(x_1104, 3, x_1043); +lean_ctor_set(x_1104, 4, x_1043); +lean_ctor_set(x_1104, 5, x_1060); +lean_ctor_set(x_1104, 6, x_1071); +lean_ctor_set(x_1104, 7, x_1103); +if (lean_is_scalar(x_1102)) { + x_1105 = lean_alloc_ctor(1, 1, 0); +} else { + x_1105 = x_1102; +} +lean_ctor_set(x_1105, 0, x_1104); +if (lean_is_scalar(x_1100)) { + x_1106 = lean_alloc_ctor(0, 2, 0); +} else { + x_1106 = x_1100; +} +lean_ctor_set(x_1106, 0, x_1105); +lean_ctor_set(x_1106, 1, x_1099); +x_11 = x_1106; +goto block_29; +} +} +} +} +else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_12, 0, x_2); -lean_ctor_set(x_12, 1, x_3); -lean_ctor_set(x_12, 2, x_11); -lean_ctor_set(x_9, 0, x_12); -return x_9; +lean_object* x_1168; lean_object* x_1169; lean_object* x_1170; +x_1168 = lean_ctor_get(x_1046, 0); +lean_inc(x_1168); +lean_dec(x_1046); +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_1058); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1193; lean_object* x_1194; lean_object* x_1195; +x_1193 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1193, 0, x_1035); +lean_ctor_set(x_1193, 1, x_1036); +lean_ctor_set(x_1193, 2, x_30); +lean_ctor_set(x_1193, 3, x_1043); +lean_ctor_set(x_1193, 4, x_1043); +lean_ctor_set(x_1193, 5, x_1168); +lean_ctor_set(x_1193, 6, x_1043); +lean_ctor_set(x_1193, 7, x_1043); +x_1194 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1194, 0, x_1193); +x_1195 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1195, 0, x_1194); +lean_ctor_set(x_1195, 1, x_1057); +x_11 = x_1195; +goto block_29; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_9, 0); -x_14 = lean_ctor_get(x_9, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_9); -x_15 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_15, 0, x_2); -lean_ctor_set(x_15, 1, x_3); -lean_ctor_set(x_15, 2, x_13); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -return x_16; +lean_object* x_1196; lean_object* x_1197; lean_object* x_1198; size_t x_1199; size_t x_1200; lean_object* x_1201; lean_object* x_1202; lean_object* x_1203; lean_object* x_1204; lean_object* x_1205; lean_object* x_1206; lean_object* x_1207; lean_object* x_1208; lean_object* x_1209; lean_object* x_1210; +x_1196 = lean_ctor_get(x_1041, 0); +lean_inc(x_1196); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1197 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1197 = lean_box(0); +} +x_1198 = lean_array_get_size(x_1196); +x_1199 = lean_usize_of_nat(x_1198); +lean_dec(x_1198); +x_1200 = 0; +x_1201 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1199, x_1200, x_1196, x_1057); +x_1202 = lean_ctor_get(x_1201, 0); +lean_inc(x_1202); +x_1203 = lean_ctor_get(x_1201, 1); +lean_inc(x_1203); +if (lean_is_exclusive(x_1201)) { + lean_ctor_release(x_1201, 0); + lean_ctor_release(x_1201, 1); + x_1204 = x_1201; +} else { + lean_dec_ref(x_1201); + x_1204 = lean_box(0); +} +x_1205 = lean_ctor_get(x_1202, 0); +lean_inc(x_1205); +if (lean_is_exclusive(x_1202)) { + lean_ctor_release(x_1202, 0); + x_1206 = x_1202; +} else { + lean_dec_ref(x_1202); + x_1206 = lean_box(0); +} +if (lean_is_scalar(x_1197)) { + x_1207 = lean_alloc_ctor(1, 1, 0); +} else { + x_1207 = x_1197; +} +lean_ctor_set(x_1207, 0, x_1205); +x_1208 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1208, 0, x_1035); +lean_ctor_set(x_1208, 1, x_1036); +lean_ctor_set(x_1208, 2, x_30); +lean_ctor_set(x_1208, 3, x_1043); +lean_ctor_set(x_1208, 4, x_1043); +lean_ctor_set(x_1208, 5, x_1168); +lean_ctor_set(x_1208, 6, x_1043); +lean_ctor_set(x_1208, 7, x_1207); +if (lean_is_scalar(x_1206)) { + x_1209 = lean_alloc_ctor(1, 1, 0); +} else { + x_1209 = x_1206; +} +lean_ctor_set(x_1209, 0, x_1208); +if (lean_is_scalar(x_1204)) { + x_1210 = lean_alloc_ctor(0, 2, 0); +} else { + x_1210 = x_1204; +} +lean_ctor_set(x_1210, 0, x_1209); +lean_ctor_set(x_1210, 1, x_1203); +x_11 = x_1210; +goto block_29; } } else { -uint8_t x_17; -lean_dec(x_3); -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_9); -if (x_17 == 0) +lean_object* x_1211; lean_object* x_1212; lean_object* x_1213; size_t x_1214; size_t x_1215; lean_object* x_1216; lean_object* x_1217; lean_object* x_1218; lean_object* x_1219; lean_object* x_1220; lean_object* x_1221; lean_object* x_1222; +x_1211 = lean_ctor_get(x_1040, 0); +lean_inc(x_1211); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_1212 = x_1040; +} else { + lean_dec_ref(x_1040); + x_1212 = lean_box(0); +} +x_1213 = lean_array_get_size(x_1211); +x_1214 = lean_usize_of_nat(x_1213); +lean_dec(x_1213); +x_1215 = 0; +x_1216 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1214, x_1215, x_1211, x_1057); +x_1217 = lean_ctor_get(x_1216, 0); +lean_inc(x_1217); +x_1218 = lean_ctor_get(x_1216, 1); +lean_inc(x_1218); +lean_dec(x_1216); +x_1219 = lean_ctor_get(x_1217, 0); +lean_inc(x_1219); +if (lean_is_exclusive(x_1217)) { + lean_ctor_release(x_1217, 0); + x_1220 = x_1217; +} else { + lean_dec_ref(x_1217); + x_1220 = lean_box(0); +} +if (lean_is_scalar(x_1212)) { + x_1221 = lean_alloc_ctor(1, 1, 0); +} else { + x_1221 = x_1212; +} +lean_ctor_set(x_1221, 0, x_1219); +if (lean_is_scalar(x_1220)) { + x_1222 = lean_alloc_ctor(1, 1, 0); +} else { + x_1222 = x_1220; +} +lean_ctor_set(x_1222, 0, x_1221); +x_1169 = x_1222; +x_1170 = x_1218; +goto block_1192; +} +block_1192: { -return x_9; +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1171; lean_object* x_1172; lean_object* x_1173; lean_object* x_1174; lean_object* x_1175; +x_1171 = lean_ctor_get(x_1169, 0); +lean_inc(x_1171); +if (lean_is_exclusive(x_1169)) { + lean_ctor_release(x_1169, 0); + x_1172 = x_1169; +} else { + lean_dec_ref(x_1169); + x_1172 = lean_box(0); +} +x_1173 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1173, 0, x_1035); +lean_ctor_set(x_1173, 1, x_1036); +lean_ctor_set(x_1173, 2, x_30); +lean_ctor_set(x_1173, 3, x_1043); +lean_ctor_set(x_1173, 4, x_1043); +lean_ctor_set(x_1173, 5, x_1168); +lean_ctor_set(x_1173, 6, x_1171); +lean_ctor_set(x_1173, 7, x_1043); +if (lean_is_scalar(x_1172)) { + x_1174 = lean_alloc_ctor(1, 1, 0); +} else { + x_1174 = x_1172; +} +lean_ctor_set(x_1174, 0, x_1173); +if (lean_is_scalar(x_1058)) { + x_1175 = lean_alloc_ctor(0, 2, 0); +} else { + x_1175 = x_1058; +} +lean_ctor_set(x_1175, 0, x_1174); +lean_ctor_set(x_1175, 1, x_1170); +x_11 = x_1175; +goto block_29; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_9, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_9); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; +lean_object* x_1176; lean_object* x_1177; lean_object* x_1178; lean_object* x_1179; size_t x_1180; size_t x_1181; lean_object* x_1182; lean_object* x_1183; lean_object* x_1184; lean_object* x_1185; lean_object* x_1186; lean_object* x_1187; lean_object* x_1188; lean_object* x_1189; lean_object* x_1190; lean_object* x_1191; +lean_dec(x_1058); +x_1176 = lean_ctor_get(x_1169, 0); +lean_inc(x_1176); +lean_dec(x_1169); +x_1177 = lean_ctor_get(x_1041, 0); +lean_inc(x_1177); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1178 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1178 = lean_box(0); +} +x_1179 = lean_array_get_size(x_1177); +x_1180 = lean_usize_of_nat(x_1179); +lean_dec(x_1179); +x_1181 = 0; +x_1182 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1180, x_1181, x_1177, x_1170); +x_1183 = lean_ctor_get(x_1182, 0); +lean_inc(x_1183); +x_1184 = lean_ctor_get(x_1182, 1); +lean_inc(x_1184); +if (lean_is_exclusive(x_1182)) { + lean_ctor_release(x_1182, 0); + lean_ctor_release(x_1182, 1); + x_1185 = x_1182; +} else { + lean_dec_ref(x_1182); + x_1185 = lean_box(0); +} +x_1186 = lean_ctor_get(x_1183, 0); +lean_inc(x_1186); +if (lean_is_exclusive(x_1183)) { + lean_ctor_release(x_1183, 0); + x_1187 = x_1183; +} else { + lean_dec_ref(x_1183); + x_1187 = lean_box(0); } +if (lean_is_scalar(x_1178)) { + x_1188 = lean_alloc_ctor(1, 1, 0); +} else { + x_1188 = x_1178; +} +lean_ctor_set(x_1188, 0, x_1186); +x_1189 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1189, 0, x_1035); +lean_ctor_set(x_1189, 1, x_1036); +lean_ctor_set(x_1189, 2, x_30); +lean_ctor_set(x_1189, 3, x_1043); +lean_ctor_set(x_1189, 4, x_1043); +lean_ctor_set(x_1189, 5, x_1168); +lean_ctor_set(x_1189, 6, x_1176); +lean_ctor_set(x_1189, 7, x_1188); +if (lean_is_scalar(x_1187)) { + x_1190 = lean_alloc_ctor(1, 1, 0); +} else { + x_1190 = x_1187; } +lean_ctor_set(x_1190, 0, x_1189); +if (lean_is_scalar(x_1185)) { + x_1191 = lean_alloc_ctor(0, 2, 0); +} else { + x_1191 = x_1185; } +lean_ctor_set(x_1191, 0, x_1190); +lean_ctor_set(x_1191, 1, x_1184); +x_11 = x_1191; +goto block_29; } -LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -switch (lean_obj_tag(x_1)) { -case 1: +} +} +} +} +else { -lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_8, 3); -lean_inc(x_9); -lean_dec(x_8); -x_10 = 1; -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_11 = l_Lean_Widget_ppExprTagged(x_9, x_10, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_11) == 0) +uint8_t x_1223; +x_1223 = !lean_is_exclusive(x_1038); +if (x_1223 == 0) { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 2) +lean_object* x_1224; lean_object* x_1225; lean_object* x_1226; +x_1224 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_1225 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1224, x_1039, x_4); +x_1226 = lean_ctor_get(x_1225, 0); +lean_inc(x_1226); +if (lean_obj_tag(x_1226) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -x_16 = l_Lean_Widget_makePopup___lambda__1(x_1, x_2, x_15, x_3, x_4, x_5, x_6, x_13); -return x_16; +uint8_t x_1227; +lean_dec(x_1038); +lean_dec(x_30); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_1227 = !lean_is_exclusive(x_1225); +if (x_1227 == 0) +{ +lean_object* x_1228; uint8_t x_1229; +x_1228 = lean_ctor_get(x_1225, 0); +lean_dec(x_1228); +x_1229 = !lean_is_exclusive(x_1226); +if (x_1229 == 0) +{ +x_11 = x_1225; +goto block_29; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_dec(x_11); -x_18 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_18, 0, x_12); -x_19 = l_Lean_Widget_makePopup___lambda__1(x_1, x_2, x_18, x_3, x_4, x_5, x_6, x_17); -return x_19; +lean_object* x_1230; lean_object* x_1231; +x_1230 = lean_ctor_get(x_1226, 0); +lean_inc(x_1230); +lean_dec(x_1226); +x_1231 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_1231, 0, x_1230); +lean_ctor_set(x_1225, 0, x_1231); +x_11 = x_1225; +goto block_29; } } else { -uint8_t x_20; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_20 = !lean_is_exclusive(x_11); -if (x_20 == 0) +lean_object* x_1232; lean_object* x_1233; lean_object* x_1234; lean_object* x_1235; lean_object* x_1236; +x_1232 = lean_ctor_get(x_1225, 1); +lean_inc(x_1232); +lean_dec(x_1225); +x_1233 = lean_ctor_get(x_1226, 0); +lean_inc(x_1233); +if (lean_is_exclusive(x_1226)) { + lean_ctor_release(x_1226, 0); + x_1234 = x_1226; +} else { + lean_dec_ref(x_1226); + x_1234 = lean_box(0); +} +if (lean_is_scalar(x_1234)) { + x_1235 = lean_alloc_ctor(0, 1, 0); +} else { + x_1235 = x_1234; +} +lean_ctor_set(x_1235, 0, x_1233); +x_1236 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1236, 0, x_1235); +lean_ctor_set(x_1236, 1, x_1232); +x_11 = x_1236; +goto block_29; +} +} +else { -return x_11; +lean_object* x_1237; lean_object* x_1238; uint8_t x_1239; +x_1237 = lean_ctor_get(x_1225, 1); +lean_inc(x_1237); +if (lean_is_exclusive(x_1225)) { + lean_ctor_release(x_1225, 0); + lean_ctor_release(x_1225, 1); + x_1238 = x_1225; +} else { + lean_dec_ref(x_1225); + x_1238 = lean_box(0); +} +x_1239 = !lean_is_exclusive(x_1226); +if (x_1239 == 0) +{ +lean_object* x_1240; lean_object* x_1241; lean_object* x_1242; +x_1240 = lean_ctor_get(x_1226, 0); +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_1238); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1288; lean_object* x_1289; +x_1288 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1288, 0, x_1035); +lean_ctor_set(x_1288, 1, x_1036); +lean_ctor_set(x_1288, 2, x_30); +lean_ctor_set(x_1288, 3, x_1043); +lean_ctor_set(x_1288, 4, x_1038); +lean_ctor_set(x_1288, 5, x_1240); +lean_ctor_set(x_1288, 6, x_1043); +lean_ctor_set(x_1288, 7, x_1043); +lean_ctor_set(x_1226, 0, x_1288); +x_1289 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1289, 0, x_1226); +lean_ctor_set(x_1289, 1, x_1237); +x_11 = x_1289; +goto block_29; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_11, 0); -x_22 = lean_ctor_get(x_11, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_11); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +uint8_t x_1290; +lean_free_object(x_1226); +x_1290 = !lean_is_exclusive(x_1041); +if (x_1290 == 0) +{ +lean_object* x_1291; lean_object* x_1292; size_t x_1293; size_t x_1294; lean_object* x_1295; uint8_t x_1296; +x_1291 = lean_ctor_get(x_1041, 0); +x_1292 = lean_array_get_size(x_1291); +x_1293 = lean_usize_of_nat(x_1292); +lean_dec(x_1292); +x_1294 = 0; +x_1295 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1293, x_1294, x_1291, x_1237); +x_1296 = !lean_is_exclusive(x_1295); +if (x_1296 == 0) +{ +lean_object* x_1297; uint8_t x_1298; +x_1297 = lean_ctor_get(x_1295, 0); +x_1298 = !lean_is_exclusive(x_1297); +if (x_1298 == 0) +{ +lean_object* x_1299; lean_object* x_1300; +x_1299 = lean_ctor_get(x_1297, 0); +lean_ctor_set(x_1041, 0, x_1299); +x_1300 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1300, 0, x_1035); +lean_ctor_set(x_1300, 1, x_1036); +lean_ctor_set(x_1300, 2, x_30); +lean_ctor_set(x_1300, 3, x_1043); +lean_ctor_set(x_1300, 4, x_1038); +lean_ctor_set(x_1300, 5, x_1240); +lean_ctor_set(x_1300, 6, x_1043); +lean_ctor_set(x_1300, 7, x_1041); +lean_ctor_set(x_1297, 0, x_1300); +x_11 = x_1295; +goto block_29; } +else +{ +lean_object* x_1301; lean_object* x_1302; lean_object* x_1303; +x_1301 = lean_ctor_get(x_1297, 0); +lean_inc(x_1301); +lean_dec(x_1297); +lean_ctor_set(x_1041, 0, x_1301); +x_1302 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1302, 0, x_1035); +lean_ctor_set(x_1302, 1, x_1036); +lean_ctor_set(x_1302, 2, x_30); +lean_ctor_set(x_1302, 3, x_1043); +lean_ctor_set(x_1302, 4, x_1038); +lean_ctor_set(x_1302, 5, x_1240); +lean_ctor_set(x_1302, 6, x_1043); +lean_ctor_set(x_1302, 7, x_1041); +x_1303 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1303, 0, x_1302); +lean_ctor_set(x_1295, 0, x_1303); +x_11 = x_1295; +goto block_29; } } -case 4: +else { -lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_24 = lean_ctor_get(x_1, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = 1; -x_27 = l_Lean_Name_toString(x_25, x_26); -x_28 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_28); -x_30 = l_Lean_Widget_makePopup___lambda__1(x_1, x_2, x_29, x_3, x_4, x_5, x_6, x_7); -return x_30; +lean_object* x_1304; lean_object* x_1305; lean_object* x_1306; lean_object* x_1307; lean_object* x_1308; lean_object* x_1309; lean_object* x_1310; +x_1304 = lean_ctor_get(x_1295, 0); +x_1305 = lean_ctor_get(x_1295, 1); +lean_inc(x_1305); +lean_inc(x_1304); +lean_dec(x_1295); +x_1306 = lean_ctor_get(x_1304, 0); +lean_inc(x_1306); +if (lean_is_exclusive(x_1304)) { + lean_ctor_release(x_1304, 0); + x_1307 = x_1304; +} else { + lean_dec_ref(x_1304); + x_1307 = lean_box(0); +} +lean_ctor_set(x_1041, 0, x_1306); +x_1308 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1308, 0, x_1035); +lean_ctor_set(x_1308, 1, x_1036); +lean_ctor_set(x_1308, 2, x_30); +lean_ctor_set(x_1308, 3, x_1043); +lean_ctor_set(x_1308, 4, x_1038); +lean_ctor_set(x_1308, 5, x_1240); +lean_ctor_set(x_1308, 6, x_1043); +lean_ctor_set(x_1308, 7, x_1041); +if (lean_is_scalar(x_1307)) { + x_1309 = lean_alloc_ctor(1, 1, 0); +} else { + x_1309 = x_1307; } -default: +lean_ctor_set(x_1309, 0, x_1308); +x_1310 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1310, 0, x_1309); +lean_ctor_set(x_1310, 1, x_1305); +x_11 = x_1310; +goto block_29; +} +} +else { -lean_object* x_31; lean_object* x_32; -x_31 = lean_box(0); -x_32 = l_Lean_Widget_makePopup___lambda__1(x_1, x_2, x_31, x_3, x_4, x_5, x_6, x_7); -return x_32; +lean_object* x_1311; lean_object* x_1312; size_t x_1313; size_t x_1314; lean_object* x_1315; lean_object* x_1316; lean_object* x_1317; lean_object* x_1318; lean_object* x_1319; lean_object* x_1320; lean_object* x_1321; lean_object* x_1322; lean_object* x_1323; lean_object* x_1324; +x_1311 = lean_ctor_get(x_1041, 0); +lean_inc(x_1311); +lean_dec(x_1041); +x_1312 = lean_array_get_size(x_1311); +x_1313 = lean_usize_of_nat(x_1312); +lean_dec(x_1312); +x_1314 = 0; +x_1315 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1313, x_1314, x_1311, x_1237); +x_1316 = lean_ctor_get(x_1315, 0); +lean_inc(x_1316); +x_1317 = lean_ctor_get(x_1315, 1); +lean_inc(x_1317); +if (lean_is_exclusive(x_1315)) { + lean_ctor_release(x_1315, 0); + lean_ctor_release(x_1315, 1); + x_1318 = x_1315; +} else { + lean_dec_ref(x_1315); + x_1318 = lean_box(0); +} +x_1319 = lean_ctor_get(x_1316, 0); +lean_inc(x_1319); +if (lean_is_exclusive(x_1316)) { + lean_ctor_release(x_1316, 0); + x_1320 = x_1316; +} else { + lean_dec_ref(x_1316); + x_1320 = lean_box(0); +} +x_1321 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1321, 0, x_1319); +x_1322 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1322, 0, x_1035); +lean_ctor_set(x_1322, 1, x_1036); +lean_ctor_set(x_1322, 2, x_30); +lean_ctor_set(x_1322, 3, x_1043); +lean_ctor_set(x_1322, 4, x_1038); +lean_ctor_set(x_1322, 5, x_1240); +lean_ctor_set(x_1322, 6, x_1043); +lean_ctor_set(x_1322, 7, x_1321); +if (lean_is_scalar(x_1320)) { + x_1323 = lean_alloc_ctor(1, 1, 0); +} else { + x_1323 = x_1320; } +lean_ctor_set(x_1323, 0, x_1322); +if (lean_is_scalar(x_1318)) { + x_1324 = lean_alloc_ctor(0, 2, 0); +} else { + x_1324 = x_1318; } +lean_ctor_set(x_1324, 0, x_1323); +lean_ctor_set(x_1324, 1, x_1317); +x_11 = x_1324; +goto block_29; } } -LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +} +else { -lean_object* x_7; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_7 = l_Lean_Elab_Info_type_x3f(x_1, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_7) == 0) +uint8_t x_1325; +lean_free_object(x_1226); +x_1325 = !lean_is_exclusive(x_1040); +if (x_1325 == 0) +{ +lean_object* x_1326; lean_object* x_1327; size_t x_1328; size_t x_1329; lean_object* x_1330; lean_object* x_1331; lean_object* x_1332; uint8_t x_1333; +x_1326 = lean_ctor_get(x_1040, 0); +x_1327 = lean_array_get_size(x_1326); +x_1328 = lean_usize_of_nat(x_1327); +lean_dec(x_1327); +x_1329 = 0; +x_1330 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1328, x_1329, x_1326, x_1237); +x_1331 = lean_ctor_get(x_1330, 0); +lean_inc(x_1331); +x_1332 = lean_ctor_get(x_1330, 1); +lean_inc(x_1332); +lean_dec(x_1330); +x_1333 = !lean_is_exclusive(x_1331); +if (x_1333 == 0) +{ +lean_object* x_1334; +x_1334 = lean_ctor_get(x_1331, 0); +lean_ctor_set(x_1040, 0, x_1334); +lean_ctor_set(x_1331, 0, x_1040); +x_1241 = x_1331; +x_1242 = x_1332; +goto block_1287; +} +else { -lean_object* x_8; -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -if (lean_obj_tag(x_8) == 0) +lean_object* x_1335; lean_object* x_1336; +x_1335 = lean_ctor_get(x_1331, 0); +lean_inc(x_1335); +lean_dec(x_1331); +lean_ctor_set(x_1040, 0, x_1335); +x_1336 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1336, 0, x_1040); +x_1241 = x_1336; +x_1242 = x_1332; +goto block_1287; +} +} +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = lean_box(0); -x_11 = l_Lean_Widget_makePopup___lambda__2(x_1, x_10, x_2, x_3, x_4, x_5, x_9); -return x_11; +lean_object* x_1337; lean_object* x_1338; size_t x_1339; size_t x_1340; lean_object* x_1341; lean_object* x_1342; lean_object* x_1343; lean_object* x_1344; lean_object* x_1345; lean_object* x_1346; lean_object* x_1347; +x_1337 = lean_ctor_get(x_1040, 0); +lean_inc(x_1337); +lean_dec(x_1040); +x_1338 = lean_array_get_size(x_1337); +x_1339 = lean_usize_of_nat(x_1338); +lean_dec(x_1338); +x_1340 = 0; +x_1341 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1339, x_1340, x_1337, x_1237); +x_1342 = lean_ctor_get(x_1341, 0); +lean_inc(x_1342); +x_1343 = lean_ctor_get(x_1341, 1); +lean_inc(x_1343); +lean_dec(x_1341); +x_1344 = lean_ctor_get(x_1342, 0); +lean_inc(x_1344); +if (lean_is_exclusive(x_1342)) { + lean_ctor_release(x_1342, 0); + x_1345 = x_1342; +} else { + lean_dec_ref(x_1342); + x_1345 = lean_box(0); +} +x_1346 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1346, 0, x_1344); +if (lean_is_scalar(x_1345)) { + x_1347 = lean_alloc_ctor(1, 1, 0); +} else { + x_1347 = x_1345; +} +lean_ctor_set(x_1347, 0, x_1346); +x_1241 = x_1347; +x_1242 = x_1343; +goto block_1287; +} +} +block_1287: +{ +if (lean_obj_tag(x_1041) == 0) +{ +uint8_t x_1243; +x_1243 = !lean_is_exclusive(x_1241); +if (x_1243 == 0) +{ +lean_object* x_1244; lean_object* x_1245; lean_object* x_1246; +x_1244 = lean_ctor_get(x_1241, 0); +x_1245 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1245, 0, x_1035); +lean_ctor_set(x_1245, 1, x_1036); +lean_ctor_set(x_1245, 2, x_30); +lean_ctor_set(x_1245, 3, x_1043); +lean_ctor_set(x_1245, 4, x_1038); +lean_ctor_set(x_1245, 5, x_1240); +lean_ctor_set(x_1245, 6, x_1244); +lean_ctor_set(x_1245, 7, x_1043); +lean_ctor_set(x_1241, 0, x_1245); +if (lean_is_scalar(x_1238)) { + x_1246 = lean_alloc_ctor(0, 2, 0); +} else { + x_1246 = x_1238; +} +lean_ctor_set(x_1246, 0, x_1241); +lean_ctor_set(x_1246, 1, x_1242); +x_11 = x_1246; +goto block_29; +} +else +{ +lean_object* x_1247; lean_object* x_1248; lean_object* x_1249; lean_object* x_1250; +x_1247 = lean_ctor_get(x_1241, 0); +lean_inc(x_1247); +lean_dec(x_1241); +x_1248 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1248, 0, x_1035); +lean_ctor_set(x_1248, 1, x_1036); +lean_ctor_set(x_1248, 2, x_30); +lean_ctor_set(x_1248, 3, x_1043); +lean_ctor_set(x_1248, 4, x_1038); +lean_ctor_set(x_1248, 5, x_1240); +lean_ctor_set(x_1248, 6, x_1247); +lean_ctor_set(x_1248, 7, x_1043); +x_1249 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1249, 0, x_1248); +if (lean_is_scalar(x_1238)) { + x_1250 = lean_alloc_ctor(0, 2, 0); +} else { + x_1250 = x_1238; +} +lean_ctor_set(x_1250, 0, x_1249); +lean_ctor_set(x_1250, 1, x_1242); +x_11 = x_1250; +goto block_29; +} } else { -lean_object* x_12; uint8_t x_13; -x_12 = lean_ctor_get(x_7, 1); -lean_inc(x_12); -lean_dec(x_7); -x_13 = !lean_is_exclusive(x_8); -if (x_13 == 0) +lean_object* x_1251; uint8_t x_1252; +lean_dec(x_1238); +x_1251 = lean_ctor_get(x_1241, 0); +lean_inc(x_1251); +lean_dec(x_1241); +x_1252 = !lean_is_exclusive(x_1041); +if (x_1252 == 0) +{ +lean_object* x_1253; lean_object* x_1254; size_t x_1255; size_t x_1256; lean_object* x_1257; uint8_t x_1258; +x_1253 = lean_ctor_get(x_1041, 0); +x_1254 = lean_array_get_size(x_1253); +x_1255 = lean_usize_of_nat(x_1254); +lean_dec(x_1254); +x_1256 = 0; +x_1257 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1255, x_1256, x_1253, x_1242); +x_1258 = !lean_is_exclusive(x_1257); +if (x_1258 == 0) +{ +lean_object* x_1259; uint8_t x_1260; +x_1259 = lean_ctor_get(x_1257, 0); +x_1260 = !lean_is_exclusive(x_1259); +if (x_1260 == 0) +{ +lean_object* x_1261; lean_object* x_1262; +x_1261 = lean_ctor_get(x_1259, 0); +lean_ctor_set(x_1041, 0, x_1261); +x_1262 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1262, 0, x_1035); +lean_ctor_set(x_1262, 1, x_1036); +lean_ctor_set(x_1262, 2, x_30); +lean_ctor_set(x_1262, 3, x_1043); +lean_ctor_set(x_1262, 4, x_1038); +lean_ctor_set(x_1262, 5, x_1240); +lean_ctor_set(x_1262, 6, x_1251); +lean_ctor_set(x_1262, 7, x_1041); +lean_ctor_set(x_1259, 0, x_1262); +x_11 = x_1257; +goto block_29; +} +else { -lean_object* x_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_8, 0); -x_15 = 0; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_16 = l_Lean_Widget_ppExprTagged(x_14, x_15, x_2, x_3, x_4, x_5, x_12); -if (lean_obj_tag(x_16) == 0) +lean_object* x_1263; lean_object* x_1264; lean_object* x_1265; +x_1263 = lean_ctor_get(x_1259, 0); +lean_inc(x_1263); +lean_dec(x_1259); +lean_ctor_set(x_1041, 0, x_1263); +x_1264 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1264, 0, x_1035); +lean_ctor_set(x_1264, 1, x_1036); +lean_ctor_set(x_1264, 2, x_30); +lean_ctor_set(x_1264, 3, x_1043); +lean_ctor_set(x_1264, 4, x_1038); +lean_ctor_set(x_1264, 5, x_1240); +lean_ctor_set(x_1264, 6, x_1251); +lean_ctor_set(x_1264, 7, x_1041); +x_1265 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1265, 0, x_1264); +lean_ctor_set(x_1257, 0, x_1265); +x_11 = x_1257; +goto block_29; +} +} +else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -lean_ctor_set(x_8, 0, x_17); -x_19 = l_Lean_Widget_makePopup___lambda__2(x_1, x_8, x_2, x_3, x_4, x_5, x_18); -return x_19; +lean_object* x_1266; lean_object* x_1267; lean_object* x_1268; lean_object* x_1269; lean_object* x_1270; lean_object* x_1271; lean_object* x_1272; +x_1266 = lean_ctor_get(x_1257, 0); +x_1267 = lean_ctor_get(x_1257, 1); +lean_inc(x_1267); +lean_inc(x_1266); +lean_dec(x_1257); +x_1268 = lean_ctor_get(x_1266, 0); +lean_inc(x_1268); +if (lean_is_exclusive(x_1266)) { + lean_ctor_release(x_1266, 0); + x_1269 = x_1266; +} else { + lean_dec_ref(x_1266); + x_1269 = lean_box(0); +} +lean_ctor_set(x_1041, 0, x_1268); +x_1270 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1270, 0, x_1035); +lean_ctor_set(x_1270, 1, x_1036); +lean_ctor_set(x_1270, 2, x_30); +lean_ctor_set(x_1270, 3, x_1043); +lean_ctor_set(x_1270, 4, x_1038); +lean_ctor_set(x_1270, 5, x_1240); +lean_ctor_set(x_1270, 6, x_1251); +lean_ctor_set(x_1270, 7, x_1041); +if (lean_is_scalar(x_1269)) { + x_1271 = lean_alloc_ctor(1, 1, 0); +} else { + x_1271 = x_1269; +} +lean_ctor_set(x_1271, 0, x_1270); +x_1272 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1272, 0, x_1271); +lean_ctor_set(x_1272, 1, x_1267); +x_11 = x_1272; +goto block_29; +} } else { -uint8_t x_20; -lean_free_object(x_8); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_20 = !lean_is_exclusive(x_16); -if (x_20 == 0) +lean_object* x_1273; lean_object* x_1274; size_t x_1275; size_t x_1276; lean_object* x_1277; lean_object* x_1278; lean_object* x_1279; lean_object* x_1280; lean_object* x_1281; lean_object* x_1282; lean_object* x_1283; lean_object* x_1284; lean_object* x_1285; lean_object* x_1286; +x_1273 = lean_ctor_get(x_1041, 0); +lean_inc(x_1273); +lean_dec(x_1041); +x_1274 = lean_array_get_size(x_1273); +x_1275 = lean_usize_of_nat(x_1274); +lean_dec(x_1274); +x_1276 = 0; +x_1277 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1275, x_1276, x_1273, x_1242); +x_1278 = lean_ctor_get(x_1277, 0); +lean_inc(x_1278); +x_1279 = lean_ctor_get(x_1277, 1); +lean_inc(x_1279); +if (lean_is_exclusive(x_1277)) { + lean_ctor_release(x_1277, 0); + lean_ctor_release(x_1277, 1); + x_1280 = x_1277; +} else { + lean_dec_ref(x_1277); + x_1280 = lean_box(0); +} +x_1281 = lean_ctor_get(x_1278, 0); +lean_inc(x_1281); +if (lean_is_exclusive(x_1278)) { + lean_ctor_release(x_1278, 0); + x_1282 = x_1278; +} else { + lean_dec_ref(x_1278); + x_1282 = lean_box(0); +} +x_1283 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1283, 0, x_1281); +x_1284 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1284, 0, x_1035); +lean_ctor_set(x_1284, 1, x_1036); +lean_ctor_set(x_1284, 2, x_30); +lean_ctor_set(x_1284, 3, x_1043); +lean_ctor_set(x_1284, 4, x_1038); +lean_ctor_set(x_1284, 5, x_1240); +lean_ctor_set(x_1284, 6, x_1251); +lean_ctor_set(x_1284, 7, x_1283); +if (lean_is_scalar(x_1282)) { + x_1285 = lean_alloc_ctor(1, 1, 0); +} else { + x_1285 = x_1282; +} +lean_ctor_set(x_1285, 0, x_1284); +if (lean_is_scalar(x_1280)) { + x_1286 = lean_alloc_ctor(0, 2, 0); +} else { + x_1286 = x_1280; +} +lean_ctor_set(x_1286, 0, x_1285); +lean_ctor_set(x_1286, 1, x_1279); +x_11 = x_1286; +goto block_29; +} +} +} +} +else { -return x_16; +lean_object* x_1348; lean_object* x_1349; lean_object* x_1350; +x_1348 = lean_ctor_get(x_1226, 0); +lean_inc(x_1348); +lean_dec(x_1226); +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_1238); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1373; lean_object* x_1374; lean_object* x_1375; +x_1373 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1373, 0, x_1035); +lean_ctor_set(x_1373, 1, x_1036); +lean_ctor_set(x_1373, 2, x_30); +lean_ctor_set(x_1373, 3, x_1043); +lean_ctor_set(x_1373, 4, x_1038); +lean_ctor_set(x_1373, 5, x_1348); +lean_ctor_set(x_1373, 6, x_1043); +lean_ctor_set(x_1373, 7, x_1043); +x_1374 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1374, 0, x_1373); +x_1375 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1375, 0, x_1374); +lean_ctor_set(x_1375, 1, x_1237); +x_11 = x_1375; +goto block_29; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_16, 0); -x_22 = lean_ctor_get(x_16, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_16); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +lean_object* x_1376; lean_object* x_1377; lean_object* x_1378; size_t x_1379; size_t x_1380; lean_object* x_1381; lean_object* x_1382; lean_object* x_1383; lean_object* x_1384; lean_object* x_1385; lean_object* x_1386; lean_object* x_1387; lean_object* x_1388; lean_object* x_1389; lean_object* x_1390; +x_1376 = lean_ctor_get(x_1041, 0); +lean_inc(x_1376); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1377 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1377 = lean_box(0); +} +x_1378 = lean_array_get_size(x_1376); +x_1379 = lean_usize_of_nat(x_1378); +lean_dec(x_1378); +x_1380 = 0; +x_1381 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1379, x_1380, x_1376, x_1237); +x_1382 = lean_ctor_get(x_1381, 0); +lean_inc(x_1382); +x_1383 = lean_ctor_get(x_1381, 1); +lean_inc(x_1383); +if (lean_is_exclusive(x_1381)) { + lean_ctor_release(x_1381, 0); + lean_ctor_release(x_1381, 1); + x_1384 = x_1381; +} else { + lean_dec_ref(x_1381); + x_1384 = lean_box(0); +} +x_1385 = lean_ctor_get(x_1382, 0); +lean_inc(x_1385); +if (lean_is_exclusive(x_1382)) { + lean_ctor_release(x_1382, 0); + x_1386 = x_1382; +} else { + lean_dec_ref(x_1382); + x_1386 = lean_box(0); } +if (lean_is_scalar(x_1377)) { + x_1387 = lean_alloc_ctor(1, 1, 0); +} else { + x_1387 = x_1377; +} +lean_ctor_set(x_1387, 0, x_1385); +x_1388 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1388, 0, x_1035); +lean_ctor_set(x_1388, 1, x_1036); +lean_ctor_set(x_1388, 2, x_30); +lean_ctor_set(x_1388, 3, x_1043); +lean_ctor_set(x_1388, 4, x_1038); +lean_ctor_set(x_1388, 5, x_1348); +lean_ctor_set(x_1388, 6, x_1043); +lean_ctor_set(x_1388, 7, x_1387); +if (lean_is_scalar(x_1386)) { + x_1389 = lean_alloc_ctor(1, 1, 0); +} else { + x_1389 = x_1386; +} +lean_ctor_set(x_1389, 0, x_1388); +if (lean_is_scalar(x_1384)) { + x_1390 = lean_alloc_ctor(0, 2, 0); +} else { + x_1390 = x_1384; +} +lean_ctor_set(x_1390, 0, x_1389); +lean_ctor_set(x_1390, 1, x_1383); +x_11 = x_1390; +goto block_29; } } else { -lean_object* x_24; uint8_t x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_8, 0); -lean_inc(x_24); -lean_dec(x_8); -x_25 = 0; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_26 = l_Lean_Widget_ppExprTagged(x_24, x_25, x_2, x_3, x_4, x_5, x_12); -if (lean_obj_tag(x_26) == 0) +lean_object* x_1391; lean_object* x_1392; lean_object* x_1393; size_t x_1394; size_t x_1395; lean_object* x_1396; lean_object* x_1397; lean_object* x_1398; lean_object* x_1399; lean_object* x_1400; lean_object* x_1401; lean_object* x_1402; +x_1391 = lean_ctor_get(x_1040, 0); +lean_inc(x_1391); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_1392 = x_1040; +} else { + lean_dec_ref(x_1040); + x_1392 = lean_box(0); +} +x_1393 = lean_array_get_size(x_1391); +x_1394 = lean_usize_of_nat(x_1393); +lean_dec(x_1393); +x_1395 = 0; +x_1396 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1394, x_1395, x_1391, x_1237); +x_1397 = lean_ctor_get(x_1396, 0); +lean_inc(x_1397); +x_1398 = lean_ctor_get(x_1396, 1); +lean_inc(x_1398); +lean_dec(x_1396); +x_1399 = lean_ctor_get(x_1397, 0); +lean_inc(x_1399); +if (lean_is_exclusive(x_1397)) { + lean_ctor_release(x_1397, 0); + x_1400 = x_1397; +} else { + lean_dec_ref(x_1397); + x_1400 = lean_box(0); +} +if (lean_is_scalar(x_1392)) { + x_1401 = lean_alloc_ctor(1, 1, 0); +} else { + x_1401 = x_1392; +} +lean_ctor_set(x_1401, 0, x_1399); +if (lean_is_scalar(x_1400)) { + x_1402 = lean_alloc_ctor(1, 1, 0); +} else { + x_1402 = x_1400; +} +lean_ctor_set(x_1402, 0, x_1401); +x_1349 = x_1402; +x_1350 = x_1398; +goto block_1372; +} +block_1372: { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_27); -x_30 = l_Lean_Widget_makePopup___lambda__2(x_1, x_29, x_2, x_3, x_4, x_5, x_28); -return x_30; +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1351; lean_object* x_1352; lean_object* x_1353; lean_object* x_1354; lean_object* x_1355; +x_1351 = lean_ctor_get(x_1349, 0); +lean_inc(x_1351); +if (lean_is_exclusive(x_1349)) { + lean_ctor_release(x_1349, 0); + x_1352 = x_1349; +} else { + lean_dec_ref(x_1349); + x_1352 = lean_box(0); +} +x_1353 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1353, 0, x_1035); +lean_ctor_set(x_1353, 1, x_1036); +lean_ctor_set(x_1353, 2, x_30); +lean_ctor_set(x_1353, 3, x_1043); +lean_ctor_set(x_1353, 4, x_1038); +lean_ctor_set(x_1353, 5, x_1348); +lean_ctor_set(x_1353, 6, x_1351); +lean_ctor_set(x_1353, 7, x_1043); +if (lean_is_scalar(x_1352)) { + x_1354 = lean_alloc_ctor(1, 1, 0); +} else { + x_1354 = x_1352; +} +lean_ctor_set(x_1354, 0, x_1353); +if (lean_is_scalar(x_1238)) { + x_1355 = lean_alloc_ctor(0, 2, 0); +} else { + x_1355 = x_1238; +} +lean_ctor_set(x_1355, 0, x_1354); +lean_ctor_set(x_1355, 1, x_1350); +x_11 = x_1355; +goto block_29; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_31 = lean_ctor_get(x_26, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_26, 1); -lean_inc(x_32); -if (lean_is_exclusive(x_26)) { - lean_ctor_release(x_26, 0); - lean_ctor_release(x_26, 1); - x_33 = x_26; +lean_object* x_1356; lean_object* x_1357; lean_object* x_1358; lean_object* x_1359; size_t x_1360; size_t x_1361; lean_object* x_1362; lean_object* x_1363; lean_object* x_1364; lean_object* x_1365; lean_object* x_1366; lean_object* x_1367; lean_object* x_1368; lean_object* x_1369; lean_object* x_1370; lean_object* x_1371; +lean_dec(x_1238); +x_1356 = lean_ctor_get(x_1349, 0); +lean_inc(x_1356); +lean_dec(x_1349); +x_1357 = lean_ctor_get(x_1041, 0); +lean_inc(x_1357); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1358 = x_1041; } else { - lean_dec_ref(x_26); - x_33 = lean_box(0); + lean_dec_ref(x_1041); + x_1358 = lean_box(0); +} +x_1359 = lean_array_get_size(x_1357); +x_1360 = lean_usize_of_nat(x_1359); +lean_dec(x_1359); +x_1361 = 0; +x_1362 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1360, x_1361, x_1357, x_1350); +x_1363 = lean_ctor_get(x_1362, 0); +lean_inc(x_1363); +x_1364 = lean_ctor_get(x_1362, 1); +lean_inc(x_1364); +if (lean_is_exclusive(x_1362)) { + lean_ctor_release(x_1362, 0); + lean_ctor_release(x_1362, 1); + x_1365 = x_1362; +} else { + lean_dec_ref(x_1362); + x_1365 = lean_box(0); +} +x_1366 = lean_ctor_get(x_1363, 0); +lean_inc(x_1366); +if (lean_is_exclusive(x_1363)) { + lean_ctor_release(x_1363, 0); + x_1367 = x_1363; +} else { + lean_dec_ref(x_1363); + x_1367 = lean_box(0); } -if (lean_is_scalar(x_33)) { - x_34 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_1358)) { + x_1368 = lean_alloc_ctor(1, 1, 0); } else { - x_34 = x_33; + x_1368 = x_1358; +} +lean_ctor_set(x_1368, 0, x_1366); +x_1369 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1369, 0, x_1035); +lean_ctor_set(x_1369, 1, x_1036); +lean_ctor_set(x_1369, 2, x_30); +lean_ctor_set(x_1369, 3, x_1043); +lean_ctor_set(x_1369, 4, x_1038); +lean_ctor_set(x_1369, 5, x_1348); +lean_ctor_set(x_1369, 6, x_1356); +lean_ctor_set(x_1369, 7, x_1368); +if (lean_is_scalar(x_1367)) { + x_1370 = lean_alloc_ctor(1, 1, 0); +} else { + x_1370 = x_1367; +} +lean_ctor_set(x_1370, 0, x_1369); +if (lean_is_scalar(x_1365)) { + x_1371 = lean_alloc_ctor(0, 2, 0); +} else { + x_1371 = x_1365; +} +lean_ctor_set(x_1371, 0, x_1370); +lean_ctor_set(x_1371, 1, x_1364); +x_11 = x_1371; +goto block_29; } -lean_ctor_set(x_34, 0, x_31); -lean_ctor_set(x_34, 1, x_32); -return x_34; } } } } else { -uint8_t x_35; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_35 = !lean_is_exclusive(x_7); -if (x_35 == 0) +lean_object* x_1403; lean_object* x_1404; lean_object* x_1405; lean_object* x_1406; lean_object* x_1407; +x_1403 = lean_ctor_get(x_1038, 0); +lean_inc(x_1403); +lean_dec(x_1038); +x_1404 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1404, 0, x_1403); +x_1405 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_1406 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1405, x_1039, x_4); +x_1407 = lean_ctor_get(x_1406, 0); +lean_inc(x_1407); +if (lean_obj_tag(x_1407) == 0) +{ +lean_object* x_1408; lean_object* x_1409; lean_object* x_1410; lean_object* x_1411; lean_object* x_1412; lean_object* x_1413; +lean_dec(x_1404); +lean_dec(x_30); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_1408 = lean_ctor_get(x_1406, 1); +lean_inc(x_1408); +if (lean_is_exclusive(x_1406)) { + lean_ctor_release(x_1406, 0); + lean_ctor_release(x_1406, 1); + x_1409 = x_1406; +} else { + lean_dec_ref(x_1406); + x_1409 = lean_box(0); +} +x_1410 = lean_ctor_get(x_1407, 0); +lean_inc(x_1410); +if (lean_is_exclusive(x_1407)) { + lean_ctor_release(x_1407, 0); + x_1411 = x_1407; +} else { + lean_dec_ref(x_1407); + x_1411 = lean_box(0); +} +if (lean_is_scalar(x_1411)) { + x_1412 = lean_alloc_ctor(0, 1, 0); +} else { + x_1412 = x_1411; +} +lean_ctor_set(x_1412, 0, x_1410); +if (lean_is_scalar(x_1409)) { + x_1413 = lean_alloc_ctor(0, 2, 0); +} else { + x_1413 = x_1409; +} +lean_ctor_set(x_1413, 0, x_1412); +lean_ctor_set(x_1413, 1, x_1408); +x_11 = x_1413; +goto block_29; +} +else { -return x_7; +lean_object* x_1414; lean_object* x_1415; lean_object* x_1416; lean_object* x_1417; lean_object* x_1418; lean_object* x_1419; +x_1414 = lean_ctor_get(x_1406, 1); +lean_inc(x_1414); +if (lean_is_exclusive(x_1406)) { + lean_ctor_release(x_1406, 0); + lean_ctor_release(x_1406, 1); + x_1415 = x_1406; +} else { + lean_dec_ref(x_1406); + x_1415 = lean_box(0); +} +x_1416 = lean_ctor_get(x_1407, 0); +lean_inc(x_1416); +if (lean_is_exclusive(x_1407)) { + lean_ctor_release(x_1407, 0); + x_1417 = x_1407; +} else { + lean_dec_ref(x_1407); + x_1417 = lean_box(0); +} +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_1415); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1442; lean_object* x_1443; lean_object* x_1444; +x_1442 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1442, 0, x_1035); +lean_ctor_set(x_1442, 1, x_1036); +lean_ctor_set(x_1442, 2, x_30); +lean_ctor_set(x_1442, 3, x_1043); +lean_ctor_set(x_1442, 4, x_1404); +lean_ctor_set(x_1442, 5, x_1416); +lean_ctor_set(x_1442, 6, x_1043); +lean_ctor_set(x_1442, 7, x_1043); +if (lean_is_scalar(x_1417)) { + x_1443 = lean_alloc_ctor(1, 1, 0); +} else { + x_1443 = x_1417; +} +lean_ctor_set(x_1443, 0, x_1442); +x_1444 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1444, 0, x_1443); +lean_ctor_set(x_1444, 1, x_1414); +x_11 = x_1444; +goto block_29; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_7, 0); -x_37 = lean_ctor_get(x_7, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_7); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_object* x_1445; lean_object* x_1446; lean_object* x_1447; size_t x_1448; size_t x_1449; lean_object* x_1450; lean_object* x_1451; lean_object* x_1452; lean_object* x_1453; lean_object* x_1454; lean_object* x_1455; lean_object* x_1456; lean_object* x_1457; lean_object* x_1458; lean_object* x_1459; +lean_dec(x_1417); +x_1445 = lean_ctor_get(x_1041, 0); +lean_inc(x_1445); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1446 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1446 = lean_box(0); +} +x_1447 = lean_array_get_size(x_1445); +x_1448 = lean_usize_of_nat(x_1447); +lean_dec(x_1447); +x_1449 = 0; +x_1450 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1448, x_1449, x_1445, x_1414); +x_1451 = lean_ctor_get(x_1450, 0); +lean_inc(x_1451); +x_1452 = lean_ctor_get(x_1450, 1); +lean_inc(x_1452); +if (lean_is_exclusive(x_1450)) { + lean_ctor_release(x_1450, 0); + lean_ctor_release(x_1450, 1); + x_1453 = x_1450; +} else { + lean_dec_ref(x_1450); + x_1453 = lean_box(0); +} +x_1454 = lean_ctor_get(x_1451, 0); +lean_inc(x_1454); +if (lean_is_exclusive(x_1451)) { + lean_ctor_release(x_1451, 0); + x_1455 = x_1451; +} else { + lean_dec_ref(x_1451); + x_1455 = lean_box(0); } +if (lean_is_scalar(x_1446)) { + x_1456 = lean_alloc_ctor(1, 1, 0); +} else { + x_1456 = x_1446; +} +lean_ctor_set(x_1456, 0, x_1454); +x_1457 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1457, 0, x_1035); +lean_ctor_set(x_1457, 1, x_1036); +lean_ctor_set(x_1457, 2, x_30); +lean_ctor_set(x_1457, 3, x_1043); +lean_ctor_set(x_1457, 4, x_1404); +lean_ctor_set(x_1457, 5, x_1416); +lean_ctor_set(x_1457, 6, x_1043); +lean_ctor_set(x_1457, 7, x_1456); +if (lean_is_scalar(x_1455)) { + x_1458 = lean_alloc_ctor(1, 1, 0); +} else { + x_1458 = x_1455; } +lean_ctor_set(x_1458, 0, x_1457); +if (lean_is_scalar(x_1453)) { + x_1459 = lean_alloc_ctor(0, 2, 0); +} else { + x_1459 = x_1453; } +lean_ctor_set(x_1459, 0, x_1458); +lean_ctor_set(x_1459, 1, x_1452); +x_11 = x_1459; +goto block_29; } -LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +} +else { -lean_object* x_6; -x_6 = l_Lean_Elab_ContextInfo_runMetaM___rarg(x_1, x_2, x_3, x_5); -if (lean_obj_tag(x_6) == 0) +lean_object* x_1460; lean_object* x_1461; lean_object* x_1462; size_t x_1463; size_t x_1464; lean_object* x_1465; lean_object* x_1466; lean_object* x_1467; lean_object* x_1468; lean_object* x_1469; lean_object* x_1470; lean_object* x_1471; +lean_dec(x_1417); +x_1460 = lean_ctor_get(x_1040, 0); +lean_inc(x_1460); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_1461 = x_1040; +} else { + lean_dec_ref(x_1040); + x_1461 = lean_box(0); +} +x_1462 = lean_array_get_size(x_1460); +x_1463 = lean_usize_of_nat(x_1462); +lean_dec(x_1462); +x_1464 = 0; +x_1465 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1463, x_1464, x_1460, x_1414); +x_1466 = lean_ctor_get(x_1465, 0); +lean_inc(x_1466); +x_1467 = lean_ctor_get(x_1465, 1); +lean_inc(x_1467); +lean_dec(x_1465); +x_1468 = lean_ctor_get(x_1466, 0); +lean_inc(x_1468); +if (lean_is_exclusive(x_1466)) { + lean_ctor_release(x_1466, 0); + x_1469 = x_1466; +} else { + lean_dec_ref(x_1466); + x_1469 = lean_box(0); +} +if (lean_is_scalar(x_1461)) { + x_1470 = lean_alloc_ctor(1, 1, 0); +} else { + x_1470 = x_1461; +} +lean_ctor_set(x_1470, 0, x_1468); +if (lean_is_scalar(x_1469)) { + x_1471 = lean_alloc_ctor(1, 1, 0); +} else { + x_1471 = x_1469; +} +lean_ctor_set(x_1471, 0, x_1470); +x_1418 = x_1471; +x_1419 = x_1467; +goto block_1441; +} +block_1441: { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +if (lean_obj_tag(x_1041) == 0) { -return x_6; +lean_object* x_1420; lean_object* x_1421; lean_object* x_1422; lean_object* x_1423; lean_object* x_1424; +x_1420 = lean_ctor_get(x_1418, 0); +lean_inc(x_1420); +if (lean_is_exclusive(x_1418)) { + lean_ctor_release(x_1418, 0); + x_1421 = x_1418; +} else { + lean_dec_ref(x_1418); + x_1421 = lean_box(0); +} +x_1422 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1422, 0, x_1035); +lean_ctor_set(x_1422, 1, x_1036); +lean_ctor_set(x_1422, 2, x_30); +lean_ctor_set(x_1422, 3, x_1043); +lean_ctor_set(x_1422, 4, x_1404); +lean_ctor_set(x_1422, 5, x_1416); +lean_ctor_set(x_1422, 6, x_1420); +lean_ctor_set(x_1422, 7, x_1043); +if (lean_is_scalar(x_1421)) { + x_1423 = lean_alloc_ctor(1, 1, 0); +} else { + x_1423 = x_1421; +} +lean_ctor_set(x_1423, 0, x_1422); +if (lean_is_scalar(x_1415)) { + x_1424 = lean_alloc_ctor(0, 2, 0); +} else { + x_1424 = x_1415; +} +lean_ctor_set(x_1424, 0, x_1423); +lean_ctor_set(x_1424, 1, x_1419); +x_11 = x_1424; +goto block_29; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_inc(x_8); -lean_dec(x_6); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -return x_10; +lean_object* x_1425; lean_object* x_1426; lean_object* x_1427; lean_object* x_1428; size_t x_1429; size_t x_1430; lean_object* x_1431; lean_object* x_1432; lean_object* x_1433; lean_object* x_1434; lean_object* x_1435; lean_object* x_1436; lean_object* x_1437; lean_object* x_1438; lean_object* x_1439; lean_object* x_1440; +lean_dec(x_1415); +x_1425 = lean_ctor_get(x_1418, 0); +lean_inc(x_1425); +lean_dec(x_1418); +x_1426 = lean_ctor_get(x_1041, 0); +lean_inc(x_1426); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1427 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1427 = lean_box(0); +} +x_1428 = lean_array_get_size(x_1426); +x_1429 = lean_usize_of_nat(x_1428); +lean_dec(x_1428); +x_1430 = 0; +x_1431 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1429, x_1430, x_1426, x_1419); +x_1432 = lean_ctor_get(x_1431, 0); +lean_inc(x_1432); +x_1433 = lean_ctor_get(x_1431, 1); +lean_inc(x_1433); +if (lean_is_exclusive(x_1431)) { + lean_ctor_release(x_1431, 0); + lean_ctor_release(x_1431, 1); + x_1434 = x_1431; +} else { + lean_dec_ref(x_1431); + x_1434 = lean_box(0); +} +x_1435 = lean_ctor_get(x_1432, 0); +lean_inc(x_1435); +if (lean_is_exclusive(x_1432)) { + lean_ctor_release(x_1432, 0); + x_1436 = x_1432; +} else { + lean_dec_ref(x_1432); + x_1436 = lean_box(0); +} +if (lean_is_scalar(x_1427)) { + x_1437 = lean_alloc_ctor(1, 1, 0); +} else { + x_1437 = x_1427; +} +lean_ctor_set(x_1437, 0, x_1435); +x_1438 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1438, 0, x_1035); +lean_ctor_set(x_1438, 1, x_1036); +lean_ctor_set(x_1438, 2, x_30); +lean_ctor_set(x_1438, 3, x_1043); +lean_ctor_set(x_1438, 4, x_1404); +lean_ctor_set(x_1438, 5, x_1416); +lean_ctor_set(x_1438, 6, x_1425); +lean_ctor_set(x_1438, 7, x_1437); +if (lean_is_scalar(x_1436)) { + x_1439 = lean_alloc_ctor(1, 1, 0); +} else { + x_1439 = x_1436; +} +lean_ctor_set(x_1439, 0, x_1438); +if (lean_is_scalar(x_1434)) { + x_1440 = lean_alloc_ctor(0, 2, 0); +} else { + x_1440 = x_1434; +} +lean_ctor_set(x_1440, 0, x_1439); +lean_ctor_set(x_1440, 1, x_1433); +x_11 = x_1440; +goto block_29; +} +} +} +} } } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_6); -if (x_11 == 0) +uint8_t x_1472; +x_1472 = !lean_is_exclusive(x_1037); +if (x_1472 == 0) { -lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_6, 0); -x_13 = lean_io_error_to_string(x_12); -x_14 = 4; -x_15 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set_uint8(x_15, sizeof(void*)*1, x_14); -lean_ctor_set(x_6, 0, x_15); -return x_6; +if (lean_obj_tag(x_1038) == 0) +{ +lean_object* x_1473; lean_object* x_1474; lean_object* x_1475; lean_object* x_1476; +x_1473 = lean_box(0); +x_1474 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_1475 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1474, x_1039, x_4); +x_1476 = lean_ctor_get(x_1475, 0); +lean_inc(x_1476); +if (lean_obj_tag(x_1476) == 0) +{ +uint8_t x_1477; +lean_dec(x_1037); +lean_dec(x_30); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_1477 = !lean_is_exclusive(x_1475); +if (x_1477 == 0) +{ +lean_object* x_1478; uint8_t x_1479; +x_1478 = lean_ctor_get(x_1475, 0); +lean_dec(x_1478); +x_1479 = !lean_is_exclusive(x_1476); +if (x_1479 == 0) +{ +x_11 = x_1475; +goto block_29; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; -x_16 = lean_ctor_get(x_6, 0); -x_17 = lean_ctor_get(x_6, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_6); -x_18 = lean_io_error_to_string(x_16); -x_19 = 4; -x_20 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set_uint8(x_20, sizeof(void*)*1, x_19); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_17); -return x_21; +lean_object* x_1480; lean_object* x_1481; +x_1480 = lean_ctor_get(x_1476, 0); +lean_inc(x_1480); +lean_dec(x_1476); +x_1481 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_1481, 0, x_1480); +lean_ctor_set(x_1475, 0, x_1481); +x_11 = x_1475; +goto block_29; } } +else +{ +lean_object* x_1482; lean_object* x_1483; lean_object* x_1484; lean_object* x_1485; lean_object* x_1486; +x_1482 = lean_ctor_get(x_1475, 1); +lean_inc(x_1482); +lean_dec(x_1475); +x_1483 = lean_ctor_get(x_1476, 0); +lean_inc(x_1483); +if (lean_is_exclusive(x_1476)) { + lean_ctor_release(x_1476, 0); + x_1484 = x_1476; +} else { + lean_dec_ref(x_1476); + x_1484 = lean_box(0); } +if (lean_is_scalar(x_1484)) { + x_1485 = lean_alloc_ctor(0, 1, 0); +} else { + x_1485 = x_1484; } -LEAN_EXPORT lean_object* l_Lean_Widget_makePopup(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_1, 1); -lean_inc(x_5); -lean_dec(x_1); -x_6 = l_Lean_Elab_Info_lctx(x_5); -x_7 = lean_alloc_closure((void*)(l_Lean_Widget_makePopup___lambda__3), 6, 1); -lean_closure_set(x_7, 0, x_5); -x_8 = lean_alloc_closure((void*)(l_Lean_Widget_makePopup___lambda__4___boxed), 5, 3); -lean_closure_set(x_8, 0, x_4); -lean_closure_set(x_8, 1, x_6); -lean_closure_set(x_8, 2, x_7); -x_9 = l_Lean_Server_RequestM_asTask___rarg(x_8, x_2, x_3); -return x_9; +lean_ctor_set(x_1485, 0, x_1483); +x_1486 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1486, 0, x_1485); +lean_ctor_set(x_1486, 1, x_1482); +x_11 = x_1486; +goto block_29; } } -LEAN_EXPORT lean_object* l_Lean_Widget_makePopup___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; -x_6 = l_Lean_Widget_makePopup___lambda__4(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_6; +lean_object* x_1487; lean_object* x_1488; uint8_t x_1489; +x_1487 = lean_ctor_get(x_1475, 1); +lean_inc(x_1487); +if (lean_is_exclusive(x_1475)) { + lean_ctor_release(x_1475, 0); + lean_ctor_release(x_1475, 1); + x_1488 = x_1475; +} else { + lean_dec_ref(x_1475); + x_1488 = lean_box(0); +} +x_1489 = !lean_is_exclusive(x_1476); +if (x_1489 == 0) +{ +lean_object* x_1490; lean_object* x_1491; lean_object* x_1492; +x_1490 = lean_ctor_get(x_1476, 0); +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_1488); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1538; lean_object* x_1539; +x_1538 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1538, 0, x_1035); +lean_ctor_set(x_1538, 1, x_1036); +lean_ctor_set(x_1538, 2, x_30); +lean_ctor_set(x_1538, 3, x_1037); +lean_ctor_set(x_1538, 4, x_1473); +lean_ctor_set(x_1538, 5, x_1490); +lean_ctor_set(x_1538, 6, x_1473); +lean_ctor_set(x_1538, 7, x_1473); +lean_ctor_set(x_1476, 0, x_1538); +x_1539 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1539, 0, x_1476); +lean_ctor_set(x_1539, 1, x_1487); +x_11 = x_1539; +goto block_29; } +else +{ +uint8_t x_1540; +lean_free_object(x_1476); +x_1540 = !lean_is_exclusive(x_1041); +if (x_1540 == 0) +{ +lean_object* x_1541; lean_object* x_1542; size_t x_1543; size_t x_1544; lean_object* x_1545; uint8_t x_1546; +x_1541 = lean_ctor_get(x_1041, 0); +x_1542 = lean_array_get_size(x_1541); +x_1543 = lean_usize_of_nat(x_1542); +lean_dec(x_1542); +x_1544 = 0; +x_1545 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1543, x_1544, x_1541, x_1487); +x_1546 = !lean_is_exclusive(x_1545); +if (x_1546 == 0) +{ +lean_object* x_1547; uint8_t x_1548; +x_1547 = lean_ctor_get(x_1545, 0); +x_1548 = !lean_is_exclusive(x_1547); +if (x_1548 == 0) +{ +lean_object* x_1549; lean_object* x_1550; +x_1549 = lean_ctor_get(x_1547, 0); +lean_ctor_set(x_1041, 0, x_1549); +x_1550 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1550, 0, x_1035); +lean_ctor_set(x_1550, 1, x_1036); +lean_ctor_set(x_1550, 2, x_30); +lean_ctor_set(x_1550, 3, x_1037); +lean_ctor_set(x_1550, 4, x_1473); +lean_ctor_set(x_1550, 5, x_1490); +lean_ctor_set(x_1550, 6, x_1473); +lean_ctor_set(x_1550, 7, x_1041); +lean_ctor_set(x_1547, 0, x_1550); +x_11 = x_1545; +goto block_29; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__1() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7; -x_2 = l_Lean_Server_instRpcEncodingOption___rarg(x_1); -return x_2; +lean_object* x_1551; lean_object* x_1552; lean_object* x_1553; +x_1551 = lean_ctor_get(x_1547, 0); +lean_inc(x_1551); +lean_dec(x_1547); +lean_ctor_set(x_1041, 0, x_1551); +x_1552 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1552, 0, x_1035); +lean_ctor_set(x_1552, 1, x_1036); +lean_ctor_set(x_1552, 2, x_30); +lean_ctor_set(x_1552, 3, x_1037); +lean_ctor_set(x_1552, 4, x_1473); +lean_ctor_set(x_1552, 5, x_1490); +lean_ctor_set(x_1552, 6, x_1473); +lean_ctor_set(x_1552, 7, x_1041); +x_1553 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1553, 0, x_1552); +lean_ctor_set(x_1545, 0, x_1553); +x_11 = x_1545; +goto block_29; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_2 = l_Lean_Server_instRpcEncodingOption___rarg(x_1); -return x_2; +lean_object* x_1554; lean_object* x_1555; lean_object* x_1556; lean_object* x_1557; lean_object* x_1558; lean_object* x_1559; lean_object* x_1560; +x_1554 = lean_ctor_get(x_1545, 0); +x_1555 = lean_ctor_get(x_1545, 1); +lean_inc(x_1555); +lean_inc(x_1554); +lean_dec(x_1545); +x_1556 = lean_ctor_get(x_1554, 0); +lean_inc(x_1556); +if (lean_is_exclusive(x_1554)) { + lean_ctor_release(x_1554, 0); + x_1557 = x_1554; +} else { + lean_dec_ref(x_1554); + x_1557 = lean_box(0); +} +lean_ctor_set(x_1041, 0, x_1556); +x_1558 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1558, 0, x_1035); +lean_ctor_set(x_1558, 1, x_1036); +lean_ctor_set(x_1558, 2, x_30); +lean_ctor_set(x_1558, 3, x_1037); +lean_ctor_set(x_1558, 4, x_1473); +lean_ctor_set(x_1558, 5, x_1490); +lean_ctor_set(x_1558, 6, x_1473); +lean_ctor_set(x_1558, 7, x_1041); +if (lean_is_scalar(x_1557)) { + x_1559 = lean_alloc_ctor(1, 1, 0); +} else { + x_1559 = x_1557; } +lean_ctor_set(x_1559, 0, x_1558); +x_1560 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1560, 0, x_1559); +lean_ctor_set(x_1560, 1, x_1555); +x_11 = x_1560; +goto block_29; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__3() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__1; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__2; -x_3 = l_Lean_Widget_instRpcEncodingInfoPopupRpcEncodingPacket___rarg(x_1, lean_box(0), x_2); -return x_3; +lean_object* x_1561; lean_object* x_1562; size_t x_1563; size_t x_1564; lean_object* x_1565; lean_object* x_1566; lean_object* x_1567; lean_object* x_1568; lean_object* x_1569; lean_object* x_1570; lean_object* x_1571; lean_object* x_1572; lean_object* x_1573; lean_object* x_1574; +x_1561 = lean_ctor_get(x_1041, 0); +lean_inc(x_1561); +lean_dec(x_1041); +x_1562 = lean_array_get_size(x_1561); +x_1563 = lean_usize_of_nat(x_1562); +lean_dec(x_1562); +x_1564 = 0; +x_1565 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1563, x_1564, x_1561, x_1487); +x_1566 = lean_ctor_get(x_1565, 0); +lean_inc(x_1566); +x_1567 = lean_ctor_get(x_1565, 1); +lean_inc(x_1567); +if (lean_is_exclusive(x_1565)) { + lean_ctor_release(x_1565, 0); + lean_ctor_release(x_1565, 1); + x_1568 = x_1565; +} else { + lean_dec_ref(x_1565); + x_1568 = lean_box(0); +} +x_1569 = lean_ctor_get(x_1566, 0); +lean_inc(x_1569); +if (lean_is_exclusive(x_1566)) { + lean_ctor_release(x_1566, 0); + x_1570 = x_1566; +} else { + lean_dec_ref(x_1566); + x_1570 = lean_box(0); +} +x_1571 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1571, 0, x_1569); +x_1572 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1572, 0, x_1035); +lean_ctor_set(x_1572, 1, x_1036); +lean_ctor_set(x_1572, 2, x_30); +lean_ctor_set(x_1572, 3, x_1037); +lean_ctor_set(x_1572, 4, x_1473); +lean_ctor_set(x_1572, 5, x_1490); +lean_ctor_set(x_1572, 6, x_1473); +lean_ctor_set(x_1572, 7, x_1571); +if (lean_is_scalar(x_1570)) { + x_1573 = lean_alloc_ctor(1, 1, 0); +} else { + x_1573 = x_1570; } +lean_ctor_set(x_1573, 0, x_1572); +if (lean_is_scalar(x_1568)) { + x_1574 = lean_alloc_ctor(0, 2, 0); +} else { + x_1574 = x_1568; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonOption___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_ctor_set(x_1574, 0, x_1573); +lean_ctor_set(x_1574, 1, x_1567); +x_11 = x_1574; +goto block_29; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonOption___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; } +else +{ +uint8_t x_1575; +lean_free_object(x_1476); +x_1575 = !lean_is_exclusive(x_1040); +if (x_1575 == 0) +{ +lean_object* x_1576; lean_object* x_1577; size_t x_1578; size_t x_1579; lean_object* x_1580; lean_object* x_1581; lean_object* x_1582; uint8_t x_1583; +x_1576 = lean_ctor_get(x_1040, 0); +x_1577 = lean_array_get_size(x_1576); +x_1578 = lean_usize_of_nat(x_1577); +lean_dec(x_1577); +x_1579 = 0; +x_1580 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1578, x_1579, x_1576, x_1487); +x_1581 = lean_ctor_get(x_1580, 0); +lean_inc(x_1581); +x_1582 = lean_ctor_get(x_1580, 1); +lean_inc(x_1582); +lean_dec(x_1580); +x_1583 = !lean_is_exclusive(x_1581); +if (x_1583 == 0) +{ +lean_object* x_1584; +x_1584 = lean_ctor_get(x_1581, 0); +lean_ctor_set(x_1040, 0, x_1584); +lean_ctor_set(x_1581, 0, x_1040); +x_1491 = x_1581; +x_1492 = x_1582; +goto block_1537; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__6() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__4; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__5; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_689____rarg), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; +lean_object* x_1585; lean_object* x_1586; +x_1585 = lean_ctor_get(x_1581, 0); +lean_inc(x_1585); +lean_dec(x_1581); +lean_ctor_set(x_1040, 0, x_1585); +x_1586 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1586, 0, x_1040); +x_1491 = x_1586; +x_1492 = x_1582; +goto block_1537; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; -x_4 = l_Lean_Lsp_instFromJsonRpcRef; -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__3; -x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__6; -x_7 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___boxed), 14, 10); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, lean_box(0)); -lean_closure_set(x_7, 2, lean_box(0)); -lean_closure_set(x_7, 3, lean_box(0)); -lean_closure_set(x_7, 4, x_3); -lean_closure_set(x_7, 5, x_4); -lean_closure_set(x_7, 6, lean_box(0)); -lean_closure_set(x_7, 7, x_5); -lean_closure_set(x_7, 8, x_6); -lean_closure_set(x_7, 9, x_2); -return x_7; +lean_object* x_1587; lean_object* x_1588; size_t x_1589; size_t x_1590; lean_object* x_1591; lean_object* x_1592; lean_object* x_1593; lean_object* x_1594; lean_object* x_1595; lean_object* x_1596; lean_object* x_1597; +x_1587 = lean_ctor_get(x_1040, 0); +lean_inc(x_1587); +lean_dec(x_1040); +x_1588 = lean_array_get_size(x_1587); +x_1589 = lean_usize_of_nat(x_1588); +lean_dec(x_1588); +x_1590 = 0; +x_1591 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1589, x_1590, x_1587, x_1487); +x_1592 = lean_ctor_get(x_1591, 0); +lean_inc(x_1592); +x_1593 = lean_ctor_get(x_1591, 1); +lean_inc(x_1593); +lean_dec(x_1591); +x_1594 = lean_ctor_get(x_1592, 0); +lean_inc(x_1594); +if (lean_is_exclusive(x_1592)) { + lean_ctor_release(x_1592, 0); + x_1595 = x_1592; +} else { + lean_dec_ref(x_1592); + x_1595 = lean_box(0); } +x_1596 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1596, 0, x_1594); +if (lean_is_scalar(x_1595)) { + x_1597 = lean_alloc_ctor(1, 1, 0); +} else { + x_1597 = x_1595; +} +lean_ctor_set(x_1597, 0, x_1596); +x_1491 = x_1597; +x_1492 = x_1593; +goto block_1537; +} +} +block_1537: +{ +if (lean_obj_tag(x_1041) == 0) +{ +uint8_t x_1493; +x_1493 = !lean_is_exclusive(x_1491); +if (x_1493 == 0) +{ +lean_object* x_1494; lean_object* x_1495; lean_object* x_1496; +x_1494 = lean_ctor_get(x_1491, 0); +x_1495 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1495, 0, x_1035); +lean_ctor_set(x_1495, 1, x_1036); +lean_ctor_set(x_1495, 2, x_30); +lean_ctor_set(x_1495, 3, x_1037); +lean_ctor_set(x_1495, 4, x_1473); +lean_ctor_set(x_1495, 5, x_1490); +lean_ctor_set(x_1495, 6, x_1494); +lean_ctor_set(x_1495, 7, x_1473); +lean_ctor_set(x_1491, 0, x_1495); +if (lean_is_scalar(x_1488)) { + x_1496 = lean_alloc_ctor(0, 2, 0); +} else { + x_1496 = x_1488; } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -lean_inc(x_1); -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2(x_1, x_2); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; -x_7 = lean_st_ref_take(x_6, x_4); -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_8, x_1, x_5); -x_11 = lean_st_ref_set(x_6, x_10, x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -return x_11; +lean_ctor_set(x_1496, 0, x_1491); +lean_ctor_set(x_1496, 1, x_1492); +x_11 = x_1496; +goto block_29; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -return x_15; +lean_object* x_1497; lean_object* x_1498; lean_object* x_1499; lean_object* x_1500; +x_1497 = lean_ctor_get(x_1491, 0); +lean_inc(x_1497); +lean_dec(x_1491); +x_1498 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1498, 0, x_1035); +lean_ctor_set(x_1498, 1, x_1036); +lean_ctor_set(x_1498, 2, x_30); +lean_ctor_set(x_1498, 3, x_1037); +lean_ctor_set(x_1498, 4, x_1473); +lean_ctor_set(x_1498, 5, x_1490); +lean_ctor_set(x_1498, 6, x_1497); +lean_ctor_set(x_1498, 7, x_1473); +x_1499 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1499, 0, x_1498); +if (lean_is_scalar(x_1488)) { + x_1500 = lean_alloc_ctor(0, 2, 0); +} else { + x_1500 = x_1488; } +lean_ctor_set(x_1500, 0, x_1499); +lean_ctor_set(x_1500, 1, x_1492); +x_11 = x_1500; +goto block_29; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -lean_dec(x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; -x_7 = lean_st_ref_get(x_6, x_5); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) +else { -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_7, 1); -lean_inc(x_1); -x_11 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_9, x_1); -if (x_11 == 0) +lean_object* x_1501; uint8_t x_1502; +lean_dec(x_1488); +x_1501 = lean_ctor_get(x_1491, 0); +lean_inc(x_1501); +lean_dec(x_1491); +x_1502 = !lean_is_exclusive(x_1041); +if (x_1502 == 0) +{ +lean_object* x_1503; lean_object* x_1504; size_t x_1505; size_t x_1506; lean_object* x_1507; uint8_t x_1508; +x_1503 = lean_ctor_get(x_1041, 0); +x_1504 = lean_array_get_size(x_1503); +x_1505 = lean_usize_of_nat(x_1504); +lean_dec(x_1504); +x_1506 = 0; +x_1507 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1505, x_1506, x_1503, x_1492); +x_1508 = !lean_is_exclusive(x_1507); +if (x_1508 == 0) +{ +lean_object* x_1509; uint8_t x_1510; +x_1509 = lean_ctor_get(x_1507, 0); +x_1510 = !lean_is_exclusive(x_1509); +if (x_1510 == 0) +{ +lean_object* x_1511; lean_object* x_1512; +x_1511 = lean_ctor_get(x_1509, 0); +lean_ctor_set(x_1041, 0, x_1511); +x_1512 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1512, 0, x_1035); +lean_ctor_set(x_1512, 1, x_1036); +lean_ctor_set(x_1512, 2, x_30); +lean_ctor_set(x_1512, 3, x_1037); +lean_ctor_set(x_1512, 4, x_1473); +lean_ctor_set(x_1512, 5, x_1490); +lean_ctor_set(x_1512, 6, x_1501); +lean_ctor_set(x_1512, 7, x_1041); +lean_ctor_set(x_1509, 0, x_1512); +x_11 = x_1507; +goto block_29; +} +else { -lean_object* x_12; lean_object* x_13; -lean_free_object(x_7); -lean_dec(x_3); -x_12 = lean_box(0); -x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__1(x_1, x_2, x_12, x_10); -return x_13; +lean_object* x_1513; lean_object* x_1514; lean_object* x_1515; +x_1513 = lean_ctor_get(x_1509, 0); +lean_inc(x_1513); +lean_dec(x_1509); +lean_ctor_set(x_1041, 0, x_1513); +x_1514 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1514, 0, x_1035); +lean_ctor_set(x_1514, 1, x_1036); +lean_ctor_set(x_1514, 2, x_30); +lean_ctor_set(x_1514, 3, x_1037); +lean_ctor_set(x_1514, 4, x_1473); +lean_ctor_set(x_1514, 5, x_1490); +lean_ctor_set(x_1514, 6, x_1501); +lean_ctor_set(x_1514, 7, x_1041); +x_1515 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1515, 0, x_1514); +lean_ctor_set(x_1507, 0, x_1515); +x_11 = x_1507; +goto block_29; +} } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -lean_dec(x_2); -lean_dec(x_1); -x_14 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_15 = lean_string_append(x_14, x_3); -lean_dec(x_3); -x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -x_17 = lean_string_append(x_15, x_16); -x_18 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set_tag(x_7, 1); -lean_ctor_set(x_7, 0, x_18); -return x_7; +lean_object* x_1516; lean_object* x_1517; lean_object* x_1518; lean_object* x_1519; lean_object* x_1520; lean_object* x_1521; lean_object* x_1522; +x_1516 = lean_ctor_get(x_1507, 0); +x_1517 = lean_ctor_get(x_1507, 1); +lean_inc(x_1517); +lean_inc(x_1516); +lean_dec(x_1507); +x_1518 = lean_ctor_get(x_1516, 0); +lean_inc(x_1518); +if (lean_is_exclusive(x_1516)) { + lean_ctor_release(x_1516, 0); + x_1519 = x_1516; +} else { + lean_dec_ref(x_1516); + x_1519 = lean_box(0); +} +lean_ctor_set(x_1041, 0, x_1518); +x_1520 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1520, 0, x_1035); +lean_ctor_set(x_1520, 1, x_1036); +lean_ctor_set(x_1520, 2, x_30); +lean_ctor_set(x_1520, 3, x_1037); +lean_ctor_set(x_1520, 4, x_1473); +lean_ctor_set(x_1520, 5, x_1490); +lean_ctor_set(x_1520, 6, x_1501); +lean_ctor_set(x_1520, 7, x_1041); +if (lean_is_scalar(x_1519)) { + x_1521 = lean_alloc_ctor(1, 1, 0); +} else { + x_1521 = x_1519; +} +lean_ctor_set(x_1521, 0, x_1520); +x_1522 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1522, 0, x_1521); +lean_ctor_set(x_1522, 1, x_1517); +x_11 = x_1522; +goto block_29; } } else { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_7, 0); -x_20 = lean_ctor_get(x_7, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_7); -lean_inc(x_1); -x_21 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_19, x_1); -if (x_21 == 0) +lean_object* x_1523; lean_object* x_1524; size_t x_1525; size_t x_1526; lean_object* x_1527; lean_object* x_1528; lean_object* x_1529; lean_object* x_1530; lean_object* x_1531; lean_object* x_1532; lean_object* x_1533; lean_object* x_1534; lean_object* x_1535; lean_object* x_1536; +x_1523 = lean_ctor_get(x_1041, 0); +lean_inc(x_1523); +lean_dec(x_1041); +x_1524 = lean_array_get_size(x_1523); +x_1525 = lean_usize_of_nat(x_1524); +lean_dec(x_1524); +x_1526 = 0; +x_1527 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1525, x_1526, x_1523, x_1492); +x_1528 = lean_ctor_get(x_1527, 0); +lean_inc(x_1528); +x_1529 = lean_ctor_get(x_1527, 1); +lean_inc(x_1529); +if (lean_is_exclusive(x_1527)) { + lean_ctor_release(x_1527, 0); + lean_ctor_release(x_1527, 1); + x_1530 = x_1527; +} else { + lean_dec_ref(x_1527); + x_1530 = lean_box(0); +} +x_1531 = lean_ctor_get(x_1528, 0); +lean_inc(x_1531); +if (lean_is_exclusive(x_1528)) { + lean_ctor_release(x_1528, 0); + x_1532 = x_1528; +} else { + lean_dec_ref(x_1528); + x_1532 = lean_box(0); +} +x_1533 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1533, 0, x_1531); +x_1534 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1534, 0, x_1035); +lean_ctor_set(x_1534, 1, x_1036); +lean_ctor_set(x_1534, 2, x_30); +lean_ctor_set(x_1534, 3, x_1037); +lean_ctor_set(x_1534, 4, x_1473); +lean_ctor_set(x_1534, 5, x_1490); +lean_ctor_set(x_1534, 6, x_1501); +lean_ctor_set(x_1534, 7, x_1533); +if (lean_is_scalar(x_1532)) { + x_1535 = lean_alloc_ctor(1, 1, 0); +} else { + x_1535 = x_1532; +} +lean_ctor_set(x_1535, 0, x_1534); +if (lean_is_scalar(x_1530)) { + x_1536 = lean_alloc_ctor(0, 2, 0); +} else { + x_1536 = x_1530; +} +lean_ctor_set(x_1536, 0, x_1535); +lean_ctor_set(x_1536, 1, x_1529); +x_11 = x_1536; +goto block_29; +} +} +} +} +else { -lean_object* x_22; lean_object* x_23; -lean_dec(x_3); -x_22 = lean_box(0); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__1(x_1, x_2, x_22, x_20); -return x_23; +lean_object* x_1598; lean_object* x_1599; lean_object* x_1600; +x_1598 = lean_ctor_get(x_1476, 0); +lean_inc(x_1598); +lean_dec(x_1476); +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_1488); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1623; lean_object* x_1624; lean_object* x_1625; +x_1623 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1623, 0, x_1035); +lean_ctor_set(x_1623, 1, x_1036); +lean_ctor_set(x_1623, 2, x_30); +lean_ctor_set(x_1623, 3, x_1037); +lean_ctor_set(x_1623, 4, x_1473); +lean_ctor_set(x_1623, 5, x_1598); +lean_ctor_set(x_1623, 6, x_1473); +lean_ctor_set(x_1623, 7, x_1473); +x_1624 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1624, 0, x_1623); +x_1625 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1625, 0, x_1624); +lean_ctor_set(x_1625, 1, x_1487); +x_11 = x_1625; +goto block_29; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_2); -lean_dec(x_1); -x_24 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_25 = lean_string_append(x_24, x_3); -lean_dec(x_3); -x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -x_27 = lean_string_append(x_25, x_26); -x_28 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_20); -return x_29; +lean_object* x_1626; lean_object* x_1627; lean_object* x_1628; size_t x_1629; size_t x_1630; lean_object* x_1631; lean_object* x_1632; lean_object* x_1633; lean_object* x_1634; lean_object* x_1635; lean_object* x_1636; lean_object* x_1637; lean_object* x_1638; lean_object* x_1639; lean_object* x_1640; +x_1626 = lean_ctor_get(x_1041, 0); +lean_inc(x_1626); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1627 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1627 = lean_box(0); +} +x_1628 = lean_array_get_size(x_1626); +x_1629 = lean_usize_of_nat(x_1628); +lean_dec(x_1628); +x_1630 = 0; +x_1631 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1629, x_1630, x_1626, x_1487); +x_1632 = lean_ctor_get(x_1631, 0); +lean_inc(x_1632); +x_1633 = lean_ctor_get(x_1631, 1); +lean_inc(x_1633); +if (lean_is_exclusive(x_1631)) { + lean_ctor_release(x_1631, 0); + lean_ctor_release(x_1631, 1); + x_1634 = x_1631; +} else { + lean_dec_ref(x_1631); + x_1634 = lean_box(0); +} +x_1635 = lean_ctor_get(x_1632, 0); +lean_inc(x_1635); +if (lean_is_exclusive(x_1632)) { + lean_ctor_release(x_1632, 0); + x_1636 = x_1632; +} else { + lean_dec_ref(x_1632); + x_1636 = lean_box(0); +} +if (lean_is_scalar(x_1627)) { + x_1637 = lean_alloc_ctor(1, 1, 0); +} else { + x_1637 = x_1627; +} +lean_ctor_set(x_1637, 0, x_1635); +x_1638 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1638, 0, x_1035); +lean_ctor_set(x_1638, 1, x_1036); +lean_ctor_set(x_1638, 2, x_30); +lean_ctor_set(x_1638, 3, x_1037); +lean_ctor_set(x_1638, 4, x_1473); +lean_ctor_set(x_1638, 5, x_1598); +lean_ctor_set(x_1638, 6, x_1473); +lean_ctor_set(x_1638, 7, x_1637); +if (lean_is_scalar(x_1636)) { + x_1639 = lean_alloc_ctor(1, 1, 0); +} else { + x_1639 = x_1636; } +lean_ctor_set(x_1639, 0, x_1638); +if (lean_is_scalar(x_1634)) { + x_1640 = lean_alloc_ctor(0, 2, 0); +} else { + x_1640 = x_1634; } +lean_ctor_set(x_1640, 0, x_1639); +lean_ctor_set(x_1640, 1, x_1633); +x_11 = x_1640; +goto block_29; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_4 = 1; -lean_inc(x_1); -x_5 = l_Lean_Name_toString(x_1, x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1; -x_7 = lean_string_append(x_6, x_5); -lean_dec(x_5); -x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2; -x_9 = lean_string_append(x_7, x_8); -x_10 = lean_io_initializing(x_3); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_unbox(x_11); -lean_dec(x_11); -if (x_12 == 0) +lean_object* x_1641; lean_object* x_1642; lean_object* x_1643; size_t x_1644; size_t x_1645; lean_object* x_1646; lean_object* x_1647; lean_object* x_1648; lean_object* x_1649; lean_object* x_1650; lean_object* x_1651; lean_object* x_1652; +x_1641 = lean_ctor_get(x_1040, 0); +lean_inc(x_1641); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_1642 = x_1040; +} else { + lean_dec_ref(x_1040); + x_1642 = lean_box(0); +} +x_1643 = lean_array_get_size(x_1641); +x_1644 = lean_usize_of_nat(x_1643); +lean_dec(x_1643); +x_1645 = 0; +x_1646 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1644, x_1645, x_1641, x_1487); +x_1647 = lean_ctor_get(x_1646, 0); +lean_inc(x_1647); +x_1648 = lean_ctor_get(x_1646, 1); +lean_inc(x_1648); +lean_dec(x_1646); +x_1649 = lean_ctor_get(x_1647, 0); +lean_inc(x_1649); +if (lean_is_exclusive(x_1647)) { + lean_ctor_release(x_1647, 0); + x_1650 = x_1647; +} else { + lean_dec_ref(x_1647); + x_1650 = lean_box(0); +} +if (lean_is_scalar(x_1642)) { + x_1651 = lean_alloc_ctor(1, 1, 0); +} else { + x_1651 = x_1642; +} +lean_ctor_set(x_1651, 0, x_1649); +if (lean_is_scalar(x_1650)) { + x_1652 = lean_alloc_ctor(1, 1, 0); +} else { + x_1652 = x_1650; +} +lean_ctor_set(x_1652, 0, x_1651); +x_1599 = x_1652; +x_1600 = x_1648; +goto block_1622; +} +block_1622: { -uint8_t x_13; -lean_dec(x_2); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_10); -if (x_13 == 0) +if (lean_obj_tag(x_1041) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_ctor_get(x_10, 0); -lean_dec(x_14); -x_15 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_16 = lean_string_append(x_15, x_9); -lean_dec(x_9); -x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -x_18 = lean_string_append(x_16, x_17); -x_19 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set_tag(x_10, 1); -lean_ctor_set(x_10, 0, x_19); -return x_10; +lean_object* x_1601; lean_object* x_1602; lean_object* x_1603; lean_object* x_1604; lean_object* x_1605; +x_1601 = lean_ctor_get(x_1599, 0); +lean_inc(x_1601); +if (lean_is_exclusive(x_1599)) { + lean_ctor_release(x_1599, 0); + x_1602 = x_1599; +} else { + lean_dec_ref(x_1599); + x_1602 = lean_box(0); +} +x_1603 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1603, 0, x_1035); +lean_ctor_set(x_1603, 1, x_1036); +lean_ctor_set(x_1603, 2, x_30); +lean_ctor_set(x_1603, 3, x_1037); +lean_ctor_set(x_1603, 4, x_1473); +lean_ctor_set(x_1603, 5, x_1598); +lean_ctor_set(x_1603, 6, x_1601); +lean_ctor_set(x_1603, 7, x_1473); +if (lean_is_scalar(x_1602)) { + x_1604 = lean_alloc_ctor(1, 1, 0); +} else { + x_1604 = x_1602; } -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_20 = lean_ctor_get(x_10, 1); -lean_inc(x_20); -lean_dec(x_10); -x_21 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_22 = lean_string_append(x_21, x_9); -lean_dec(x_9); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -x_24 = lean_string_append(x_22, x_23); -x_25 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_20); -return x_26; +lean_ctor_set(x_1604, 0, x_1603); +if (lean_is_scalar(x_1488)) { + x_1605 = lean_alloc_ctor(0, 2, 0); +} else { + x_1605 = x_1488; } +lean_ctor_set(x_1605, 0, x_1604); +lean_ctor_set(x_1605, 1, x_1600); +x_11 = x_1605; +goto block_29; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_10, 1); -lean_inc(x_27); -lean_dec(x_10); -x_28 = lean_box(0); -x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); -return x_29; +lean_object* x_1606; lean_object* x_1607; lean_object* x_1608; lean_object* x_1609; size_t x_1610; size_t x_1611; lean_object* x_1612; lean_object* x_1613; lean_object* x_1614; lean_object* x_1615; lean_object* x_1616; lean_object* x_1617; lean_object* x_1618; lean_object* x_1619; lean_object* x_1620; lean_object* x_1621; +lean_dec(x_1488); +x_1606 = lean_ctor_get(x_1599, 0); +lean_inc(x_1606); +lean_dec(x_1599); +x_1607 = lean_ctor_get(x_1041, 0); +lean_inc(x_1607); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1608 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1608 = lean_box(0); +} +x_1609 = lean_array_get_size(x_1607); +x_1610 = lean_usize_of_nat(x_1609); +lean_dec(x_1609); +x_1611 = 0; +x_1612 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1610, x_1611, x_1607, x_1600); +x_1613 = lean_ctor_get(x_1612, 0); +lean_inc(x_1613); +x_1614 = lean_ctor_get(x_1612, 1); +lean_inc(x_1614); +if (lean_is_exclusive(x_1612)) { + lean_ctor_release(x_1612, 0); + lean_ctor_release(x_1612, 1); + x_1615 = x_1612; +} else { + lean_dec_ref(x_1612); + x_1615 = lean_box(0); +} +x_1616 = lean_ctor_get(x_1613, 0); +lean_inc(x_1616); +if (lean_is_exclusive(x_1613)) { + lean_ctor_release(x_1613, 0); + x_1617 = x_1613; +} else { + lean_dec_ref(x_1613); + x_1617 = lean_box(0); +} +if (lean_is_scalar(x_1608)) { + x_1618 = lean_alloc_ctor(1, 1, 0); +} else { + x_1618 = x_1608; +} +lean_ctor_set(x_1618, 0, x_1616); +x_1619 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1619, 0, x_1035); +lean_ctor_set(x_1619, 1, x_1036); +lean_ctor_set(x_1619, 2, x_30); +lean_ctor_set(x_1619, 3, x_1037); +lean_ctor_set(x_1619, 4, x_1473); +lean_ctor_set(x_1619, 5, x_1598); +lean_ctor_set(x_1619, 6, x_1606); +lean_ctor_set(x_1619, 7, x_1618); +if (lean_is_scalar(x_1617)) { + x_1620 = lean_alloc_ctor(1, 1, 0); +} else { + x_1620 = x_1617; } +lean_ctor_set(x_1620, 0, x_1619); +if (lean_is_scalar(x_1615)) { + x_1621 = lean_alloc_ctor(0, 2, 0); +} else { + x_1621 = x_1615; } +lean_ctor_set(x_1621, 0, x_1620); +lean_ctor_set(x_1621, 1, x_1614); +x_11 = x_1621; +goto block_29; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("infoToInteractive", 17); -return x_1; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__6; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_makePopup), 3, 0); -return x_1; -} +uint8_t x_1653; +x_1653 = !lean_is_exclusive(x_1038); +if (x_1653 == 0) +{ +lean_object* x_1654; lean_object* x_1655; lean_object* x_1656; +x_1654 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_1655 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1654, x_1039, x_4); +x_1656 = lean_ctor_get(x_1655, 0); +lean_inc(x_1656); +if (lean_obj_tag(x_1656) == 0) +{ +uint8_t x_1657; +lean_dec(x_1038); +lean_dec(x_1037); +lean_dec(x_30); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_1657 = !lean_is_exclusive(x_1655); +if (x_1657 == 0) +{ +lean_object* x_1658; uint8_t x_1659; +x_1658 = lean_ctor_get(x_1655, 0); +lean_dec(x_1658); +x_1659 = !lean_is_exclusive(x_1656); +if (x_1659 == 0) +{ +x_11 = x_1655; +goto block_29; } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234_(lean_object* x_1) { -_start: +else { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__2; -x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__3; -x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1(x_2, x_3, x_1); -return x_4; +lean_object* x_1660; lean_object* x_1661; +x_1660 = lean_ctor_get(x_1656, 0); +lean_inc(x_1660); +lean_dec(x_1656); +x_1661 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_1661, 0, x_1660); +lean_ctor_set(x_1655, 0, x_1661); +x_11 = x_1655; +goto block_29; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -lean_object* x_5; -x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__1___lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_object* x_1662; lean_object* x_1663; lean_object* x_1664; lean_object* x_1665; lean_object* x_1666; +x_1662 = lean_ctor_get(x_1655, 1); +lean_inc(x_1662); +lean_dec(x_1655); +x_1663 = lean_ctor_get(x_1656, 0); +lean_inc(x_1663); +if (lean_is_exclusive(x_1656)) { + lean_ctor_release(x_1656, 0); + x_1664 = x_1656; +} else { + lean_dec_ref(x_1656); + x_1664 = lean_box(0); } +if (lean_is_scalar(x_1664)) { + x_1665 = lean_alloc_ctor(0, 1, 0); +} else { + x_1665 = x_1664; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg(x_1, lean_box(0), x_1, lean_box(0), x_2, lean_box(0), x_3); -return x_4; +lean_ctor_set(x_1665, 0, x_1663); +x_1666 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1666, 0, x_1665); +lean_ctor_set(x_1666, 1, x_1662); +x_11 = x_1666; +goto block_29; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__1; -x_2 = l_Lean_Server_instRpcEncodingArray___rarg(x_1); -return x_2; +lean_object* x_1667; lean_object* x_1668; uint8_t x_1669; +x_1667 = lean_ctor_get(x_1655, 1); +lean_inc(x_1667); +if (lean_is_exclusive(x_1655)) { + lean_ctor_release(x_1655, 0); + lean_ctor_release(x_1655, 1); + x_1668 = x_1655; +} else { + lean_dec_ref(x_1655); + x_1668 = lean_box(0); +} +x_1669 = !lean_is_exclusive(x_1656); +if (x_1669 == 0) +{ +lean_object* x_1670; lean_object* x_1671; lean_object* x_1672; +x_1670 = lean_ctor_get(x_1656, 0); +if (lean_obj_tag(x_1040) == 0) +{ +lean_object* x_1720; +lean_dec(x_1668); +x_1720 = lean_box(0); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1721; lean_object* x_1722; +x_1721 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1721, 0, x_1035); +lean_ctor_set(x_1721, 1, x_1036); +lean_ctor_set(x_1721, 2, x_30); +lean_ctor_set(x_1721, 3, x_1037); +lean_ctor_set(x_1721, 4, x_1038); +lean_ctor_set(x_1721, 5, x_1670); +lean_ctor_set(x_1721, 6, x_1720); +lean_ctor_set(x_1721, 7, x_1720); +lean_ctor_set(x_1656, 0, x_1721); +x_1722 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1722, 0, x_1656); +lean_ctor_set(x_1722, 1, x_1667); +x_11 = x_1722; +goto block_29; } +else +{ +uint8_t x_1723; +lean_free_object(x_1656); +x_1723 = !lean_is_exclusive(x_1041); +if (x_1723 == 0) +{ +lean_object* x_1724; lean_object* x_1725; size_t x_1726; size_t x_1727; lean_object* x_1728; uint8_t x_1729; +x_1724 = lean_ctor_get(x_1041, 0); +x_1725 = lean_array_get_size(x_1724); +x_1726 = lean_usize_of_nat(x_1725); +lean_dec(x_1725); +x_1727 = 0; +x_1728 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1726, x_1727, x_1724, x_1667); +x_1729 = !lean_is_exclusive(x_1728); +if (x_1729 == 0) +{ +lean_object* x_1730; uint8_t x_1731; +x_1730 = lean_ctor_get(x_1728, 0); +x_1731 = !lean_is_exclusive(x_1730); +if (x_1731 == 0) +{ +lean_object* x_1732; lean_object* x_1733; +x_1732 = lean_ctor_get(x_1730, 0); +lean_ctor_set(x_1041, 0, x_1732); +x_1733 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1733, 0, x_1035); +lean_ctor_set(x_1733, 1, x_1036); +lean_ctor_set(x_1733, 2, x_30); +lean_ctor_set(x_1733, 3, x_1037); +lean_ctor_set(x_1733, 4, x_1038); +lean_ctor_set(x_1733, 5, x_1670); +lean_ctor_set(x_1733, 6, x_1720); +lean_ctor_set(x_1733, 7, x_1041); +lean_ctor_set(x_1730, 0, x_1733); +x_11 = x_1728; +goto block_29; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__3() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__2; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg(x_1, lean_box(0), x_2, lean_box(0), x_3, lean_box(0), x_3); -return x_4; +lean_object* x_1734; lean_object* x_1735; lean_object* x_1736; +x_1734 = lean_ctor_get(x_1730, 0); +lean_inc(x_1734); +lean_dec(x_1730); +lean_ctor_set(x_1041, 0, x_1734); +x_1735 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1735, 0, x_1035); +lean_ctor_set(x_1735, 1, x_1036); +lean_ctor_set(x_1735, 2, x_30); +lean_ctor_set(x_1735, 3, x_1037); +lean_ctor_set(x_1735, 4, x_1038); +lean_ctor_set(x_1735, 5, x_1670); +lean_ctor_set(x_1735, 6, x_1720); +lean_ctor_set(x_1735, 7, x_1041); +x_1736 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1736, 0, x_1735); +lean_ctor_set(x_1728, 0, x_1736); +x_11 = x_1728; +goto block_29; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__3; -x_2 = l_Lean_Server_instRpcEncodingArray___rarg(x_1); -return x_2; +lean_object* x_1737; lean_object* x_1738; lean_object* x_1739; lean_object* x_1740; lean_object* x_1741; lean_object* x_1742; lean_object* x_1743; +x_1737 = lean_ctor_get(x_1728, 0); +x_1738 = lean_ctor_get(x_1728, 1); +lean_inc(x_1738); +lean_inc(x_1737); +lean_dec(x_1728); +x_1739 = lean_ctor_get(x_1737, 0); +lean_inc(x_1739); +if (lean_is_exclusive(x_1737)) { + lean_ctor_release(x_1737, 0); + x_1740 = x_1737; +} else { + lean_dec_ref(x_1737); + x_1740 = lean_box(0); +} +lean_ctor_set(x_1041, 0, x_1739); +x_1741 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1741, 0, x_1035); +lean_ctor_set(x_1741, 1, x_1036); +lean_ctor_set(x_1741, 2, x_30); +lean_ctor_set(x_1741, 3, x_1037); +lean_ctor_set(x_1741, 4, x_1038); +lean_ctor_set(x_1741, 5, x_1670); +lean_ctor_set(x_1741, 6, x_1720); +lean_ctor_set(x_1741, 7, x_1041); +if (lean_is_scalar(x_1740)) { + x_1742 = lean_alloc_ctor(1, 1, 0); +} else { + x_1742 = x_1740; } +lean_ctor_set(x_1742, 0, x_1741); +x_1743 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1743, 0, x_1742); +lean_ctor_set(x_1743, 1, x_1738); +x_11 = x_1743; +goto block_29; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__5() { -_start: +} +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__4; -x_2 = l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg(x_1); -return x_2; +lean_object* x_1744; lean_object* x_1745; size_t x_1746; size_t x_1747; lean_object* x_1748; lean_object* x_1749; lean_object* x_1750; lean_object* x_1751; lean_object* x_1752; lean_object* x_1753; lean_object* x_1754; lean_object* x_1755; lean_object* x_1756; lean_object* x_1757; +x_1744 = lean_ctor_get(x_1041, 0); +lean_inc(x_1744); +lean_dec(x_1041); +x_1745 = lean_array_get_size(x_1744); +x_1746 = lean_usize_of_nat(x_1745); +lean_dec(x_1745); +x_1747 = 0; +x_1748 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1746, x_1747, x_1744, x_1667); +x_1749 = lean_ctor_get(x_1748, 0); +lean_inc(x_1749); +x_1750 = lean_ctor_get(x_1748, 1); +lean_inc(x_1750); +if (lean_is_exclusive(x_1748)) { + lean_ctor_release(x_1748, 0); + lean_ctor_release(x_1748, 1); + x_1751 = x_1748; +} else { + lean_dec_ref(x_1748); + x_1751 = lean_box(0); +} +x_1752 = lean_ctor_get(x_1749, 0); +lean_inc(x_1752); +if (lean_is_exclusive(x_1749)) { + lean_ctor_release(x_1749, 0); + x_1753 = x_1749; +} else { + lean_dec_ref(x_1749); + x_1753 = lean_box(0); +} +x_1754 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1754, 0, x_1752); +x_1755 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1755, 0, x_1035); +lean_ctor_set(x_1755, 1, x_1036); +lean_ctor_set(x_1755, 2, x_30); +lean_ctor_set(x_1755, 3, x_1037); +lean_ctor_set(x_1755, 4, x_1038); +lean_ctor_set(x_1755, 5, x_1670); +lean_ctor_set(x_1755, 6, x_1720); +lean_ctor_set(x_1755, 7, x_1754); +if (lean_is_scalar(x_1753)) { + x_1756 = lean_alloc_ctor(1, 1, 0); +} else { + x_1756 = x_1753; } +lean_ctor_set(x_1756, 0, x_1755); +if (lean_is_scalar(x_1751)) { + x_1757 = lean_alloc_ctor(0, 2, 0); +} else { + x_1757 = x_1751; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__5; -x_2 = l_Lean_Server_instRpcEncodingOption___rarg(x_1); -return x_2; +lean_ctor_set(x_1757, 0, x_1756); +lean_ctor_set(x_1757, 1, x_1750); +x_11 = x_1757; +goto block_29; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__17; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__19; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15; -x_4 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__20; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414____rarg), 5, 4); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_2); -lean_closure_set(x_5, 2, x_3); -lean_closure_set(x_5, 3, x_4); -return x_5; } +else +{ +uint8_t x_1758; +lean_free_object(x_1656); +x_1758 = !lean_is_exclusive(x_1040); +if (x_1758 == 0) +{ +lean_object* x_1759; lean_object* x_1760; size_t x_1761; size_t x_1762; lean_object* x_1763; lean_object* x_1764; lean_object* x_1765; uint8_t x_1766; +x_1759 = lean_ctor_get(x_1040, 0); +x_1760 = lean_array_get_size(x_1759); +x_1761 = lean_usize_of_nat(x_1760); +lean_dec(x_1760); +x_1762 = 0; +x_1763 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1761, x_1762, x_1759, x_1667); +x_1764 = lean_ctor_get(x_1763, 0); +lean_inc(x_1764); +x_1765 = lean_ctor_get(x_1763, 1); +lean_inc(x_1765); +lean_dec(x_1763); +x_1766 = !lean_is_exclusive(x_1764); +if (x_1766 == 0) +{ +lean_object* x_1767; +x_1767 = lean_ctor_get(x_1764, 0); +lean_ctor_set(x_1040, 0, x_1767); +lean_ctor_set(x_1764, 0, x_1040); +x_1671 = x_1764; +x_1672 = x_1765; +goto block_1719; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__8() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__7; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_1768; lean_object* x_1769; +x_1768 = lean_ctor_get(x_1764, 0); +lean_inc(x_1768); +lean_dec(x_1764); +lean_ctor_set(x_1040, 0, x_1768); +x_1769 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1769, 0, x_1040); +x_1671 = x_1769; +x_1672 = x_1765; +goto block_1719; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__9() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__8; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23; -x_4 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__24; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237____rarg), 5, 4); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_2); -lean_closure_set(x_5, 2, x_3); -lean_closure_set(x_5, 3, x_4); -return x_5; +lean_object* x_1770; lean_object* x_1771; size_t x_1772; size_t x_1773; lean_object* x_1774; lean_object* x_1775; lean_object* x_1776; lean_object* x_1777; lean_object* x_1778; lean_object* x_1779; lean_object* x_1780; +x_1770 = lean_ctor_get(x_1040, 0); +lean_inc(x_1770); +lean_dec(x_1040); +x_1771 = lean_array_get_size(x_1770); +x_1772 = lean_usize_of_nat(x_1771); +lean_dec(x_1771); +x_1773 = 0; +x_1774 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1772, x_1773, x_1770, x_1667); +x_1775 = lean_ctor_get(x_1774, 0); +lean_inc(x_1775); +x_1776 = lean_ctor_get(x_1774, 1); +lean_inc(x_1776); +lean_dec(x_1774); +x_1777 = lean_ctor_get(x_1775, 0); +lean_inc(x_1777); +if (lean_is_exclusive(x_1775)) { + lean_ctor_release(x_1775, 0); + x_1778 = x_1775; +} else { + lean_dec_ref(x_1775); + x_1778 = lean_box(0); +} +x_1779 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1779, 0, x_1777); +if (lean_is_scalar(x_1778)) { + x_1780 = lean_alloc_ctor(1, 1, 0); +} else { + x_1780 = x_1778; +} +lean_ctor_set(x_1780, 0, x_1779); +x_1671 = x_1780; +x_1672 = x_1776; +goto block_1719; +} +} +block_1719: +{ +if (lean_obj_tag(x_1041) == 0) +{ +uint8_t x_1673; +x_1673 = !lean_is_exclusive(x_1671); +if (x_1673 == 0) +{ +lean_object* x_1674; lean_object* x_1675; lean_object* x_1676; lean_object* x_1677; +x_1674 = lean_ctor_get(x_1671, 0); +x_1675 = lean_box(0); +x_1676 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1676, 0, x_1035); +lean_ctor_set(x_1676, 1, x_1036); +lean_ctor_set(x_1676, 2, x_30); +lean_ctor_set(x_1676, 3, x_1037); +lean_ctor_set(x_1676, 4, x_1038); +lean_ctor_set(x_1676, 5, x_1670); +lean_ctor_set(x_1676, 6, x_1674); +lean_ctor_set(x_1676, 7, x_1675); +lean_ctor_set(x_1671, 0, x_1676); +if (lean_is_scalar(x_1668)) { + x_1677 = lean_alloc_ctor(0, 2, 0); +} else { + x_1677 = x_1668; } +lean_ctor_set(x_1677, 0, x_1671); +lean_ctor_set(x_1677, 1, x_1672); +x_11 = x_1677; +goto block_29; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__10() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__9; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_1678; lean_object* x_1679; lean_object* x_1680; lean_object* x_1681; lean_object* x_1682; +x_1678 = lean_ctor_get(x_1671, 0); +lean_inc(x_1678); +lean_dec(x_1671); +x_1679 = lean_box(0); +x_1680 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1680, 0, x_1035); +lean_ctor_set(x_1680, 1, x_1036); +lean_ctor_set(x_1680, 2, x_30); +lean_ctor_set(x_1680, 3, x_1037); +lean_ctor_set(x_1680, 4, x_1038); +lean_ctor_set(x_1680, 5, x_1670); +lean_ctor_set(x_1680, 6, x_1678); +lean_ctor_set(x_1680, 7, x_1679); +x_1681 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1681, 0, x_1680); +if (lean_is_scalar(x_1668)) { + x_1682 = lean_alloc_ctor(0, 2, 0); +} else { + x_1682 = x_1668; } +lean_ctor_set(x_1682, 0, x_1681); +lean_ctor_set(x_1682, 1, x_1672); +x_11 = x_1682; +goto block_29; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__10; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2648____rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; } +else +{ +lean_object* x_1683; uint8_t x_1684; +lean_dec(x_1668); +x_1683 = lean_ctor_get(x_1671, 0); +lean_inc(x_1683); +lean_dec(x_1671); +x_1684 = !lean_is_exclusive(x_1041); +if (x_1684 == 0) +{ +lean_object* x_1685; lean_object* x_1686; size_t x_1687; size_t x_1688; lean_object* x_1689; uint8_t x_1690; +x_1685 = lean_ctor_get(x_1041, 0); +x_1686 = lean_array_get_size(x_1685); +x_1687 = lean_usize_of_nat(x_1686); +lean_dec(x_1686); +x_1688 = 0; +x_1689 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1687, x_1688, x_1685, x_1672); +x_1690 = !lean_is_exclusive(x_1689); +if (x_1690 == 0) +{ +lean_object* x_1691; uint8_t x_1692; +x_1691 = lean_ctor_get(x_1689, 0); +x_1692 = !lean_is_exclusive(x_1691); +if (x_1692 == 0) +{ +lean_object* x_1693; lean_object* x_1694; +x_1693 = lean_ctor_get(x_1691, 0); +lean_ctor_set(x_1041, 0, x_1693); +x_1694 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1694, 0, x_1035); +lean_ctor_set(x_1694, 1, x_1036); +lean_ctor_set(x_1694, 2, x_30); +lean_ctor_set(x_1694, 3, x_1037); +lean_ctor_set(x_1694, 4, x_1038); +lean_ctor_set(x_1694, 5, x_1670); +lean_ctor_set(x_1694, 6, x_1683); +lean_ctor_set(x_1694, 7, x_1041); +lean_ctor_set(x_1691, 0, x_1694); +x_11 = x_1689; +goto block_29; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__12() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__11; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonOption___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_1695; lean_object* x_1696; lean_object* x_1697; +x_1695 = lean_ctor_get(x_1691, 0); +lean_inc(x_1695); +lean_dec(x_1691); +lean_ctor_set(x_1041, 0, x_1695); +x_1696 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1696, 0, x_1035); +lean_ctor_set(x_1696, 1, x_1036); +lean_ctor_set(x_1696, 2, x_30); +lean_ctor_set(x_1696, 3, x_1037); +lean_ctor_set(x_1696, 4, x_1038); +lean_ctor_set(x_1696, 5, x_1670); +lean_ctor_set(x_1696, 6, x_1683); +lean_ctor_set(x_1696, 7, x_1041); +x_1697 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1697, 0, x_1696); +lean_ctor_set(x_1689, 0, x_1697); +x_11 = x_1689; +goto block_29; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Lsp_instFromJsonPlainGoalParams; -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__6; -x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__12; -x_7 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___boxed), 14, 10); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, lean_box(0)); -lean_closure_set(x_7, 2, lean_box(0)); -lean_closure_set(x_7, 3, lean_box(0)); -lean_closure_set(x_7, 4, x_3); -lean_closure_set(x_7, 5, x_4); -lean_closure_set(x_7, 6, lean_box(0)); -lean_closure_set(x_7, 7, x_5); -lean_closure_set(x_7, 8, x_6); -lean_closure_set(x_7, 9, x_2); -return x_7; +lean_object* x_1698; lean_object* x_1699; lean_object* x_1700; lean_object* x_1701; lean_object* x_1702; lean_object* x_1703; lean_object* x_1704; +x_1698 = lean_ctor_get(x_1689, 0); +x_1699 = lean_ctor_get(x_1689, 1); +lean_inc(x_1699); +lean_inc(x_1698); +lean_dec(x_1689); +x_1700 = lean_ctor_get(x_1698, 0); +lean_inc(x_1700); +if (lean_is_exclusive(x_1698)) { + lean_ctor_release(x_1698, 0); + x_1701 = x_1698; +} else { + lean_dec_ref(x_1698); + x_1701 = lean_box(0); +} +lean_ctor_set(x_1041, 0, x_1700); +x_1702 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1702, 0, x_1035); +lean_ctor_set(x_1702, 1, x_1036); +lean_ctor_set(x_1702, 2, x_30); +lean_ctor_set(x_1702, 3, x_1037); +lean_ctor_set(x_1702, 4, x_1038); +lean_ctor_set(x_1702, 5, x_1670); +lean_ctor_set(x_1702, 6, x_1683); +lean_ctor_set(x_1702, 7, x_1041); +if (lean_is_scalar(x_1701)) { + x_1703 = lean_alloc_ctor(1, 1, 0); +} else { + x_1703 = x_1701; } +lean_ctor_set(x_1703, 0, x_1702); +x_1704 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1704, 0, x_1703); +lean_ctor_set(x_1704, 1, x_1699); +x_11 = x_1704; +goto block_29; } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -lean_inc(x_1); -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2(x_1, x_2); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; -x_7 = lean_st_ref_take(x_6, x_4); -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_8, x_1, x_5); -x_11 = lean_st_ref_set(x_6, x_10, x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -return x_11; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -return x_15; +lean_object* x_1705; lean_object* x_1706; size_t x_1707; size_t x_1708; lean_object* x_1709; lean_object* x_1710; lean_object* x_1711; lean_object* x_1712; lean_object* x_1713; lean_object* x_1714; lean_object* x_1715; lean_object* x_1716; lean_object* x_1717; lean_object* x_1718; +x_1705 = lean_ctor_get(x_1041, 0); +lean_inc(x_1705); +lean_dec(x_1041); +x_1706 = lean_array_get_size(x_1705); +x_1707 = lean_usize_of_nat(x_1706); +lean_dec(x_1706); +x_1708 = 0; +x_1709 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1707, x_1708, x_1705, x_1672); +x_1710 = lean_ctor_get(x_1709, 0); +lean_inc(x_1710); +x_1711 = lean_ctor_get(x_1709, 1); +lean_inc(x_1711); +if (lean_is_exclusive(x_1709)) { + lean_ctor_release(x_1709, 0); + lean_ctor_release(x_1709, 1); + x_1712 = x_1709; +} else { + lean_dec_ref(x_1709); + x_1712 = lean_box(0); +} +x_1713 = lean_ctor_get(x_1710, 0); +lean_inc(x_1713); +if (lean_is_exclusive(x_1710)) { + lean_ctor_release(x_1710, 0); + x_1714 = x_1710; +} else { + lean_dec_ref(x_1710); + x_1714 = lean_box(0); +} +x_1715 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1715, 0, x_1713); +x_1716 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1716, 0, x_1035); +lean_ctor_set(x_1716, 1, x_1036); +lean_ctor_set(x_1716, 2, x_30); +lean_ctor_set(x_1716, 3, x_1037); +lean_ctor_set(x_1716, 4, x_1038); +lean_ctor_set(x_1716, 5, x_1670); +lean_ctor_set(x_1716, 6, x_1683); +lean_ctor_set(x_1716, 7, x_1715); +if (lean_is_scalar(x_1714)) { + x_1717 = lean_alloc_ctor(1, 1, 0); +} else { + x_1717 = x_1714; +} +lean_ctor_set(x_1717, 0, x_1716); +if (lean_is_scalar(x_1712)) { + x_1718 = lean_alloc_ctor(0, 2, 0); +} else { + x_1718 = x_1712; +} +lean_ctor_set(x_1718, 0, x_1717); +lean_ctor_set(x_1718, 1, x_1711); +x_11 = x_1718; +goto block_29; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -lean_dec(x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; -x_7 = lean_st_ref_get(x_6, x_5); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_7, 1); -lean_inc(x_1); -x_11 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_9, x_1); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; -lean_free_object(x_7); -lean_dec(x_3); -x_12 = lean_box(0); -x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__1(x_1, x_2, x_12, x_10); -return x_13; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -lean_dec(x_2); -lean_dec(x_1); -x_14 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_15 = lean_string_append(x_14, x_3); -lean_dec(x_3); -x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -x_17 = lean_string_append(x_15, x_16); -x_18 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set_tag(x_7, 1); -lean_ctor_set(x_7, 0, x_18); -return x_7; -} +lean_object* x_1781; lean_object* x_1782; lean_object* x_1783; +x_1781 = lean_ctor_get(x_1656, 0); +lean_inc(x_1781); +lean_dec(x_1656); +if (lean_obj_tag(x_1040) == 0) +{ +lean_object* x_1807; +lean_dec(x_1668); +x_1807 = lean_box(0); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1808; lean_object* x_1809; lean_object* x_1810; +x_1808 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1808, 0, x_1035); +lean_ctor_set(x_1808, 1, x_1036); +lean_ctor_set(x_1808, 2, x_30); +lean_ctor_set(x_1808, 3, x_1037); +lean_ctor_set(x_1808, 4, x_1038); +lean_ctor_set(x_1808, 5, x_1781); +lean_ctor_set(x_1808, 6, x_1807); +lean_ctor_set(x_1808, 7, x_1807); +x_1809 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1809, 0, x_1808); +x_1810 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1810, 0, x_1809); +lean_ctor_set(x_1810, 1, x_1667); +x_11 = x_1810; +goto block_29; } else { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_7, 0); -x_20 = lean_ctor_get(x_7, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_7); -lean_inc(x_1); -x_21 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_19, x_1); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -lean_dec(x_3); -x_22 = lean_box(0); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__1(x_1, x_2, x_22, x_20); -return x_23; +lean_object* x_1811; lean_object* x_1812; lean_object* x_1813; size_t x_1814; size_t x_1815; lean_object* x_1816; lean_object* x_1817; lean_object* x_1818; lean_object* x_1819; lean_object* x_1820; lean_object* x_1821; lean_object* x_1822; lean_object* x_1823; lean_object* x_1824; lean_object* x_1825; +x_1811 = lean_ctor_get(x_1041, 0); +lean_inc(x_1811); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1812 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1812 = lean_box(0); +} +x_1813 = lean_array_get_size(x_1811); +x_1814 = lean_usize_of_nat(x_1813); +lean_dec(x_1813); +x_1815 = 0; +x_1816 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1814, x_1815, x_1811, x_1667); +x_1817 = lean_ctor_get(x_1816, 0); +lean_inc(x_1817); +x_1818 = lean_ctor_get(x_1816, 1); +lean_inc(x_1818); +if (lean_is_exclusive(x_1816)) { + lean_ctor_release(x_1816, 0); + lean_ctor_release(x_1816, 1); + x_1819 = x_1816; +} else { + lean_dec_ref(x_1816); + x_1819 = lean_box(0); +} +x_1820 = lean_ctor_get(x_1817, 0); +lean_inc(x_1820); +if (lean_is_exclusive(x_1817)) { + lean_ctor_release(x_1817, 0); + x_1821 = x_1817; +} else { + lean_dec_ref(x_1817); + x_1821 = lean_box(0); +} +if (lean_is_scalar(x_1812)) { + x_1822 = lean_alloc_ctor(1, 1, 0); +} else { + x_1822 = x_1812; +} +lean_ctor_set(x_1822, 0, x_1820); +x_1823 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1823, 0, x_1035); +lean_ctor_set(x_1823, 1, x_1036); +lean_ctor_set(x_1823, 2, x_30); +lean_ctor_set(x_1823, 3, x_1037); +lean_ctor_set(x_1823, 4, x_1038); +lean_ctor_set(x_1823, 5, x_1781); +lean_ctor_set(x_1823, 6, x_1807); +lean_ctor_set(x_1823, 7, x_1822); +if (lean_is_scalar(x_1821)) { + x_1824 = lean_alloc_ctor(1, 1, 0); +} else { + x_1824 = x_1821; +} +lean_ctor_set(x_1824, 0, x_1823); +if (lean_is_scalar(x_1819)) { + x_1825 = lean_alloc_ctor(0, 2, 0); +} else { + x_1825 = x_1819; +} +lean_ctor_set(x_1825, 0, x_1824); +lean_ctor_set(x_1825, 1, x_1818); +x_11 = x_1825; +goto block_29; +} } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_2); -lean_dec(x_1); -x_24 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_25 = lean_string_append(x_24, x_3); -lean_dec(x_3); -x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -x_27 = lean_string_append(x_25, x_26); -x_28 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_20); -return x_29; +lean_object* x_1826; lean_object* x_1827; lean_object* x_1828; size_t x_1829; size_t x_1830; lean_object* x_1831; lean_object* x_1832; lean_object* x_1833; lean_object* x_1834; lean_object* x_1835; lean_object* x_1836; lean_object* x_1837; +x_1826 = lean_ctor_get(x_1040, 0); +lean_inc(x_1826); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_1827 = x_1040; +} else { + lean_dec_ref(x_1040); + x_1827 = lean_box(0); +} +x_1828 = lean_array_get_size(x_1826); +x_1829 = lean_usize_of_nat(x_1828); +lean_dec(x_1828); +x_1830 = 0; +x_1831 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1829, x_1830, x_1826, x_1667); +x_1832 = lean_ctor_get(x_1831, 0); +lean_inc(x_1832); +x_1833 = lean_ctor_get(x_1831, 1); +lean_inc(x_1833); +lean_dec(x_1831); +x_1834 = lean_ctor_get(x_1832, 0); +lean_inc(x_1834); +if (lean_is_exclusive(x_1832)) { + lean_ctor_release(x_1832, 0); + x_1835 = x_1832; +} else { + lean_dec_ref(x_1832); + x_1835 = lean_box(0); } +if (lean_is_scalar(x_1827)) { + x_1836 = lean_alloc_ctor(1, 1, 0); +} else { + x_1836 = x_1827; } +lean_ctor_set(x_1836, 0, x_1834); +if (lean_is_scalar(x_1835)) { + x_1837 = lean_alloc_ctor(1, 1, 0); +} else { + x_1837 = x_1835; } +lean_ctor_set(x_1837, 0, x_1836); +x_1782 = x_1837; +x_1783 = x_1833; +goto block_1806; } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_4 = 1; -lean_inc(x_1); -x_5 = l_Lean_Name_toString(x_1, x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1; -x_7 = lean_string_append(x_6, x_5); -lean_dec(x_5); -x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2; -x_9 = lean_string_append(x_7, x_8); -x_10 = lean_io_initializing(x_3); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_unbox(x_11); -lean_dec(x_11); -if (x_12 == 0) +block_1806: { -uint8_t x_13; -lean_dec(x_2); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_10); -if (x_13 == 0) +if (lean_obj_tag(x_1041) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_ctor_get(x_10, 0); -lean_dec(x_14); -x_15 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_16 = lean_string_append(x_15, x_9); -lean_dec(x_9); -x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -x_18 = lean_string_append(x_16, x_17); -x_19 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set_tag(x_10, 1); -lean_ctor_set(x_10, 0, x_19); -return x_10; +lean_object* x_1784; lean_object* x_1785; lean_object* x_1786; lean_object* x_1787; lean_object* x_1788; lean_object* x_1789; +x_1784 = lean_ctor_get(x_1782, 0); +lean_inc(x_1784); +if (lean_is_exclusive(x_1782)) { + lean_ctor_release(x_1782, 0); + x_1785 = x_1782; +} else { + lean_dec_ref(x_1782); + x_1785 = lean_box(0); +} +x_1786 = lean_box(0); +x_1787 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1787, 0, x_1035); +lean_ctor_set(x_1787, 1, x_1036); +lean_ctor_set(x_1787, 2, x_30); +lean_ctor_set(x_1787, 3, x_1037); +lean_ctor_set(x_1787, 4, x_1038); +lean_ctor_set(x_1787, 5, x_1781); +lean_ctor_set(x_1787, 6, x_1784); +lean_ctor_set(x_1787, 7, x_1786); +if (lean_is_scalar(x_1785)) { + x_1788 = lean_alloc_ctor(1, 1, 0); +} else { + x_1788 = x_1785; +} +lean_ctor_set(x_1788, 0, x_1787); +if (lean_is_scalar(x_1668)) { + x_1789 = lean_alloc_ctor(0, 2, 0); +} else { + x_1789 = x_1668; +} +lean_ctor_set(x_1789, 0, x_1788); +lean_ctor_set(x_1789, 1, x_1783); +x_11 = x_1789; +goto block_29; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_20 = lean_ctor_get(x_10, 1); -lean_inc(x_20); -lean_dec(x_10); -x_21 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_22 = lean_string_append(x_21, x_9); -lean_dec(x_9); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -x_24 = lean_string_append(x_22, x_23); -x_25 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_20); -return x_26; +lean_object* x_1790; lean_object* x_1791; lean_object* x_1792; lean_object* x_1793; size_t x_1794; size_t x_1795; lean_object* x_1796; lean_object* x_1797; lean_object* x_1798; lean_object* x_1799; lean_object* x_1800; lean_object* x_1801; lean_object* x_1802; lean_object* x_1803; lean_object* x_1804; lean_object* x_1805; +lean_dec(x_1668); +x_1790 = lean_ctor_get(x_1782, 0); +lean_inc(x_1790); +lean_dec(x_1782); +x_1791 = lean_ctor_get(x_1041, 0); +lean_inc(x_1791); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1792 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1792 = lean_box(0); +} +x_1793 = lean_array_get_size(x_1791); +x_1794 = lean_usize_of_nat(x_1793); +lean_dec(x_1793); +x_1795 = 0; +x_1796 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1794, x_1795, x_1791, x_1783); +x_1797 = lean_ctor_get(x_1796, 0); +lean_inc(x_1797); +x_1798 = lean_ctor_get(x_1796, 1); +lean_inc(x_1798); +if (lean_is_exclusive(x_1796)) { + lean_ctor_release(x_1796, 0); + lean_ctor_release(x_1796, 1); + x_1799 = x_1796; +} else { + lean_dec_ref(x_1796); + x_1799 = lean_box(0); +} +x_1800 = lean_ctor_get(x_1797, 0); +lean_inc(x_1800); +if (lean_is_exclusive(x_1797)) { + lean_ctor_release(x_1797, 0); + x_1801 = x_1797; +} else { + lean_dec_ref(x_1797); + x_1801 = lean_box(0); +} +if (lean_is_scalar(x_1792)) { + x_1802 = lean_alloc_ctor(1, 1, 0); +} else { + x_1802 = x_1792; +} +lean_ctor_set(x_1802, 0, x_1800); +x_1803 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1803, 0, x_1035); +lean_ctor_set(x_1803, 1, x_1036); +lean_ctor_set(x_1803, 2, x_30); +lean_ctor_set(x_1803, 3, x_1037); +lean_ctor_set(x_1803, 4, x_1038); +lean_ctor_set(x_1803, 5, x_1781); +lean_ctor_set(x_1803, 6, x_1790); +lean_ctor_set(x_1803, 7, x_1802); +if (lean_is_scalar(x_1801)) { + x_1804 = lean_alloc_ctor(1, 1, 0); +} else { + x_1804 = x_1801; +} +lean_ctor_set(x_1804, 0, x_1803); +if (lean_is_scalar(x_1799)) { + x_1805 = lean_alloc_ctor(0, 2, 0); +} else { + x_1805 = x_1799; +} +lean_ctor_set(x_1805, 0, x_1804); +lean_ctor_set(x_1805, 1, x_1798); +x_11 = x_1805; +goto block_29; +} +} +} } } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_10, 1); -lean_inc(x_27); -lean_dec(x_10); -x_28 = lean_box(0); -x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); -return x_29; +lean_object* x_1838; lean_object* x_1839; lean_object* x_1840; lean_object* x_1841; lean_object* x_1842; +x_1838 = lean_ctor_get(x_1038, 0); +lean_inc(x_1838); +lean_dec(x_1038); +x_1839 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1839, 0, x_1838); +x_1840 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_1841 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1840, x_1039, x_4); +x_1842 = lean_ctor_get(x_1841, 0); +lean_inc(x_1842); +if (lean_obj_tag(x_1842) == 0) +{ +lean_object* x_1843; lean_object* x_1844; lean_object* x_1845; lean_object* x_1846; lean_object* x_1847; lean_object* x_1848; +lean_dec(x_1839); +lean_dec(x_1037); +lean_dec(x_30); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_1843 = lean_ctor_get(x_1841, 1); +lean_inc(x_1843); +if (lean_is_exclusive(x_1841)) { + lean_ctor_release(x_1841, 0); + lean_ctor_release(x_1841, 1); + x_1844 = x_1841; +} else { + lean_dec_ref(x_1841); + x_1844 = lean_box(0); +} +x_1845 = lean_ctor_get(x_1842, 0); +lean_inc(x_1845); +if (lean_is_exclusive(x_1842)) { + lean_ctor_release(x_1842, 0); + x_1846 = x_1842; +} else { + lean_dec_ref(x_1842); + x_1846 = lean_box(0); } +if (lean_is_scalar(x_1846)) { + x_1847 = lean_alloc_ctor(0, 1, 0); +} else { + x_1847 = x_1846; +} +lean_ctor_set(x_1847, 0, x_1845); +if (lean_is_scalar(x_1844)) { + x_1848 = lean_alloc_ctor(0, 2, 0); +} else { + x_1848 = x_1844; } +lean_ctor_set(x_1848, 0, x_1847); +lean_ctor_set(x_1848, 1, x_1843); +x_11 = x_1848; +goto block_29; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("getInteractiveGoals", 19); -return x_1; +lean_object* x_1849; lean_object* x_1850; lean_object* x_1851; lean_object* x_1852; lean_object* x_1853; lean_object* x_1854; +x_1849 = lean_ctor_get(x_1841, 1); +lean_inc(x_1849); +if (lean_is_exclusive(x_1841)) { + lean_ctor_release(x_1841, 0); + lean_ctor_release(x_1841, 1); + x_1850 = x_1841; +} else { + lean_dec_ref(x_1841); + x_1850 = lean_box(0); +} +x_1851 = lean_ctor_get(x_1842, 0); +lean_inc(x_1851); +if (lean_is_exclusive(x_1842)) { + lean_ctor_release(x_1842, 0); + x_1852 = x_1842; +} else { + lean_dec_ref(x_1842); + x_1852 = lean_box(0); +} +if (lean_obj_tag(x_1040) == 0) +{ +lean_object* x_1878; +lean_dec(x_1850); +x_1878 = lean_box(0); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1879; lean_object* x_1880; lean_object* x_1881; +x_1879 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1879, 0, x_1035); +lean_ctor_set(x_1879, 1, x_1036); +lean_ctor_set(x_1879, 2, x_30); +lean_ctor_set(x_1879, 3, x_1037); +lean_ctor_set(x_1879, 4, x_1839); +lean_ctor_set(x_1879, 5, x_1851); +lean_ctor_set(x_1879, 6, x_1878); +lean_ctor_set(x_1879, 7, x_1878); +if (lean_is_scalar(x_1852)) { + x_1880 = lean_alloc_ctor(1, 1, 0); +} else { + x_1880 = x_1852; } +lean_ctor_set(x_1880, 0, x_1879); +x_1881 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1881, 0, x_1880); +lean_ctor_set(x_1881, 1, x_1849); +x_11 = x_1881; +goto block_29; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1882; lean_object* x_1883; lean_object* x_1884; size_t x_1885; size_t x_1886; lean_object* x_1887; lean_object* x_1888; lean_object* x_1889; lean_object* x_1890; lean_object* x_1891; lean_object* x_1892; lean_object* x_1893; lean_object* x_1894; lean_object* x_1895; lean_object* x_1896; +lean_dec(x_1852); +x_1882 = lean_ctor_get(x_1041, 0); +lean_inc(x_1882); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1883 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1883 = lean_box(0); +} +x_1884 = lean_array_get_size(x_1882); +x_1885 = lean_usize_of_nat(x_1884); +lean_dec(x_1884); +x_1886 = 0; +x_1887 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1885, x_1886, x_1882, x_1849); +x_1888 = lean_ctor_get(x_1887, 0); +lean_inc(x_1888); +x_1889 = lean_ctor_get(x_1887, 1); +lean_inc(x_1889); +if (lean_is_exclusive(x_1887)) { + lean_ctor_release(x_1887, 0); + lean_ctor_release(x_1887, 1); + x_1890 = x_1887; +} else { + lean_dec_ref(x_1887); + x_1890 = lean_box(0); +} +x_1891 = lean_ctor_get(x_1888, 0); +lean_inc(x_1891); +if (lean_is_exclusive(x_1888)) { + lean_ctor_release(x_1888, 0); + x_1892 = x_1888; +} else { + lean_dec_ref(x_1888); + x_1892 = lean_box(0); } +if (lean_is_scalar(x_1883)) { + x_1893 = lean_alloc_ctor(1, 1, 0); +} else { + x_1893 = x_1883; +} +lean_ctor_set(x_1893, 0, x_1891); +x_1894 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1894, 0, x_1035); +lean_ctor_set(x_1894, 1, x_1036); +lean_ctor_set(x_1894, 2, x_30); +lean_ctor_set(x_1894, 3, x_1037); +lean_ctor_set(x_1894, 4, x_1839); +lean_ctor_set(x_1894, 5, x_1851); +lean_ctor_set(x_1894, 6, x_1878); +lean_ctor_set(x_1894, 7, x_1893); +if (lean_is_scalar(x_1892)) { + x_1895 = lean_alloc_ctor(1, 1, 0); +} else { + x_1895 = x_1892; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_getInteractiveGoals), 3, 0); -return x_1; +lean_ctor_set(x_1895, 0, x_1894); +if (lean_is_scalar(x_1890)) { + x_1896 = lean_alloc_ctor(0, 2, 0); +} else { + x_1896 = x_1890; } +lean_ctor_set(x_1896, 0, x_1895); +lean_ctor_set(x_1896, 1, x_1889); +x_11 = x_1896; +goto block_29; } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253_(lean_object* x_1) { -_start: +} +else { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__2; -x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__3; -x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1(x_2, x_3, x_1); -return x_4; +lean_object* x_1897; lean_object* x_1898; lean_object* x_1899; size_t x_1900; size_t x_1901; lean_object* x_1902; lean_object* x_1903; lean_object* x_1904; lean_object* x_1905; lean_object* x_1906; lean_object* x_1907; lean_object* x_1908; +lean_dec(x_1852); +x_1897 = lean_ctor_get(x_1040, 0); +lean_inc(x_1897); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_1898 = x_1040; +} else { + lean_dec_ref(x_1040); + x_1898 = lean_box(0); +} +x_1899 = lean_array_get_size(x_1897); +x_1900 = lean_usize_of_nat(x_1899); +lean_dec(x_1899); +x_1901 = 0; +x_1902 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1900, x_1901, x_1897, x_1849); +x_1903 = lean_ctor_get(x_1902, 0); +lean_inc(x_1903); +x_1904 = lean_ctor_get(x_1902, 1); +lean_inc(x_1904); +lean_dec(x_1902); +x_1905 = lean_ctor_get(x_1903, 0); +lean_inc(x_1905); +if (lean_is_exclusive(x_1903)) { + lean_ctor_release(x_1903, 0); + x_1906 = x_1903; +} else { + lean_dec_ref(x_1903); + x_1906 = lean_box(0); } +if (lean_is_scalar(x_1898)) { + x_1907 = lean_alloc_ctor(1, 1, 0); +} else { + x_1907 = x_1898; } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__1___lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_ctor_set(x_1907, 0, x_1905); +if (lean_is_scalar(x_1906)) { + x_1908 = lean_alloc_ctor(1, 1, 0); +} else { + x_1908 = x_1906; } +lean_ctor_set(x_1908, 0, x_1907); +x_1853 = x_1908; +x_1854 = x_1904; +goto block_1877; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__1() { -_start: +block_1877: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__2; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg(x_1, lean_box(0), x_2, lean_box(0), x_3); -return x_4; +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1855; lean_object* x_1856; lean_object* x_1857; lean_object* x_1858; lean_object* x_1859; lean_object* x_1860; +x_1855 = lean_ctor_get(x_1853, 0); +lean_inc(x_1855); +if (lean_is_exclusive(x_1853)) { + lean_ctor_release(x_1853, 0); + x_1856 = x_1853; +} else { + lean_dec_ref(x_1853); + x_1856 = lean_box(0); +} +x_1857 = lean_box(0); +x_1858 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1858, 0, x_1035); +lean_ctor_set(x_1858, 1, x_1036); +lean_ctor_set(x_1858, 2, x_30); +lean_ctor_set(x_1858, 3, x_1037); +lean_ctor_set(x_1858, 4, x_1839); +lean_ctor_set(x_1858, 5, x_1851); +lean_ctor_set(x_1858, 6, x_1855); +lean_ctor_set(x_1858, 7, x_1857); +if (lean_is_scalar(x_1856)) { + x_1859 = lean_alloc_ctor(1, 1, 0); +} else { + x_1859 = x_1856; } +lean_ctor_set(x_1859, 0, x_1858); +if (lean_is_scalar(x_1850)) { + x_1860 = lean_alloc_ctor(0, 2, 0); +} else { + x_1860 = x_1850; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__2() { -_start: +lean_ctor_set(x_1860, 0, x_1859); +lean_ctor_set(x_1860, 1, x_1854); +x_11 = x_1860; +goto block_29; +} +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__1; -x_2 = l_Lean_Server_instRpcEncodingOption___rarg(x_1); -return x_2; +lean_object* x_1861; lean_object* x_1862; lean_object* x_1863; lean_object* x_1864; size_t x_1865; size_t x_1866; lean_object* x_1867; lean_object* x_1868; lean_object* x_1869; lean_object* x_1870; lean_object* x_1871; lean_object* x_1872; lean_object* x_1873; lean_object* x_1874; lean_object* x_1875; lean_object* x_1876; +lean_dec(x_1850); +x_1861 = lean_ctor_get(x_1853, 0); +lean_inc(x_1861); +lean_dec(x_1853); +x_1862 = lean_ctor_get(x_1041, 0); +lean_inc(x_1862); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1863 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1863 = lean_box(0); +} +x_1864 = lean_array_get_size(x_1862); +x_1865 = lean_usize_of_nat(x_1864); +lean_dec(x_1864); +x_1866 = 0; +x_1867 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1865, x_1866, x_1862, x_1854); +x_1868 = lean_ctor_get(x_1867, 0); +lean_inc(x_1868); +x_1869 = lean_ctor_get(x_1867, 1); +lean_inc(x_1869); +if (lean_is_exclusive(x_1867)) { + lean_ctor_release(x_1867, 0); + lean_ctor_release(x_1867, 1); + x_1870 = x_1867; +} else { + lean_dec_ref(x_1867); + x_1870 = lean_box(0); +} +x_1871 = lean_ctor_get(x_1868, 0); +lean_inc(x_1871); +if (lean_is_exclusive(x_1868)) { + lean_ctor_release(x_1868, 0); + x_1872 = x_1868; +} else { + lean_dec_ref(x_1868); + x_1872 = lean_box(0); } +if (lean_is_scalar(x_1863)) { + x_1873 = lean_alloc_ctor(1, 1, 0); +} else { + x_1873 = x_1863; +} +lean_ctor_set(x_1873, 0, x_1871); +x_1874 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1874, 0, x_1035); +lean_ctor_set(x_1874, 1, x_1036); +lean_ctor_set(x_1874, 2, x_30); +lean_ctor_set(x_1874, 3, x_1037); +lean_ctor_set(x_1874, 4, x_1839); +lean_ctor_set(x_1874, 5, x_1851); +lean_ctor_set(x_1874, 6, x_1861); +lean_ctor_set(x_1874, 7, x_1873); +if (lean_is_scalar(x_1872)) { + x_1875 = lean_alloc_ctor(1, 1, 0); +} else { + x_1875 = x_1872; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__8; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15; -x_3 = l_Lean_Lsp_instToJsonRange; -x_4 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2236____rarg), 4, 3); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_2); -lean_closure_set(x_4, 2, x_3); -return x_4; +lean_ctor_set(x_1875, 0, x_1874); +if (lean_is_scalar(x_1870)) { + x_1876 = lean_alloc_ctor(0, 2, 0); +} else { + x_1876 = x_1870; } +lean_ctor_set(x_1876, 0, x_1875); +lean_ctor_set(x_1876, 1, x_1869); +x_11 = x_1876; +goto block_29; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__3; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonOption___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Lsp_instFromJsonPlainTermGoalParams; -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__2; -x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__4; -x_7 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___boxed), 14, 10); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, lean_box(0)); -lean_closure_set(x_7, 2, lean_box(0)); -lean_closure_set(x_7, 3, lean_box(0)); -lean_closure_set(x_7, 4, x_3); -lean_closure_set(x_7, 5, x_4); -lean_closure_set(x_7, 6, lean_box(0)); -lean_closure_set(x_7, 7, x_5); -lean_closure_set(x_7, 8, x_6); -lean_closure_set(x_7, 9, x_2); -return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -lean_inc(x_1); -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2(x_1, x_2); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; -x_7 = lean_st_ref_take(x_6, x_4); -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_8, x_1, x_5); -x_11 = lean_st_ref_set(x_6, x_10, x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -return x_11; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -return x_15; +lean_object* x_1909; lean_object* x_1910; +x_1909 = lean_ctor_get(x_1037, 0); +lean_inc(x_1909); +lean_dec(x_1037); +x_1910 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1910, 0, x_1909); +if (lean_obj_tag(x_1038) == 0) +{ +lean_object* x_1911; lean_object* x_1912; lean_object* x_1913; lean_object* x_1914; +x_1911 = lean_box(0); +x_1912 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_1913 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1912, x_1039, x_4); +x_1914 = lean_ctor_get(x_1913, 0); +lean_inc(x_1914); +if (lean_obj_tag(x_1914) == 0) +{ +lean_object* x_1915; lean_object* x_1916; lean_object* x_1917; lean_object* x_1918; lean_object* x_1919; lean_object* x_1920; +lean_dec(x_1910); +lean_dec(x_30); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_1915 = lean_ctor_get(x_1913, 1); +lean_inc(x_1915); +if (lean_is_exclusive(x_1913)) { + lean_ctor_release(x_1913, 0); + lean_ctor_release(x_1913, 1); + x_1916 = x_1913; +} else { + lean_dec_ref(x_1913); + x_1916 = lean_box(0); +} +x_1917 = lean_ctor_get(x_1914, 0); +lean_inc(x_1917); +if (lean_is_exclusive(x_1914)) { + lean_ctor_release(x_1914, 0); + x_1918 = x_1914; +} else { + lean_dec_ref(x_1914); + x_1918 = lean_box(0); } +if (lean_is_scalar(x_1918)) { + x_1919 = lean_alloc_ctor(0, 1, 0); +} else { + x_1919 = x_1918; } +lean_ctor_set(x_1919, 0, x_1917); +if (lean_is_scalar(x_1916)) { + x_1920 = lean_alloc_ctor(0, 2, 0); +} else { + x_1920 = x_1916; } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -lean_dec(x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; -x_7 = lean_st_ref_get(x_6, x_5); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_7, 1); -lean_inc(x_1); -x_11 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_9, x_1); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; -lean_free_object(x_7); -lean_dec(x_3); -x_12 = lean_box(0); -x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(x_1, x_2, x_12, x_10); -return x_13; +lean_ctor_set(x_1920, 0, x_1919); +lean_ctor_set(x_1920, 1, x_1915); +x_11 = x_1920; +goto block_29; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -lean_dec(x_2); -lean_dec(x_1); -x_14 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_15 = lean_string_append(x_14, x_3); -lean_dec(x_3); -x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -x_17 = lean_string_append(x_15, x_16); -x_18 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set_tag(x_7, 1); -lean_ctor_set(x_7, 0, x_18); -return x_7; +lean_object* x_1921; lean_object* x_1922; lean_object* x_1923; lean_object* x_1924; lean_object* x_1925; lean_object* x_1926; +x_1921 = lean_ctor_get(x_1913, 1); +lean_inc(x_1921); +if (lean_is_exclusive(x_1913)) { + lean_ctor_release(x_1913, 0); + lean_ctor_release(x_1913, 1); + x_1922 = x_1913; +} else { + lean_dec_ref(x_1913); + x_1922 = lean_box(0); +} +x_1923 = lean_ctor_get(x_1914, 0); +lean_inc(x_1923); +if (lean_is_exclusive(x_1914)) { + lean_ctor_release(x_1914, 0); + x_1924 = x_1914; +} else { + lean_dec_ref(x_1914); + x_1924 = lean_box(0); +} +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_1922); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_1949; lean_object* x_1950; lean_object* x_1951; +x_1949 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1949, 0, x_1035); +lean_ctor_set(x_1949, 1, x_1036); +lean_ctor_set(x_1949, 2, x_30); +lean_ctor_set(x_1949, 3, x_1910); +lean_ctor_set(x_1949, 4, x_1911); +lean_ctor_set(x_1949, 5, x_1923); +lean_ctor_set(x_1949, 6, x_1911); +lean_ctor_set(x_1949, 7, x_1911); +if (lean_is_scalar(x_1924)) { + x_1950 = lean_alloc_ctor(1, 1, 0); +} else { + x_1950 = x_1924; } +lean_ctor_set(x_1950, 0, x_1949); +x_1951 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1951, 0, x_1950); +lean_ctor_set(x_1951, 1, x_1921); +x_11 = x_1951; +goto block_29; } else { -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_7, 0); -x_20 = lean_ctor_get(x_7, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_7); -lean_inc(x_1); -x_21 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_19, x_1); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -lean_dec(x_3); -x_22 = lean_box(0); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(x_1, x_2, x_22, x_20); -return x_23; +lean_object* x_1952; lean_object* x_1953; lean_object* x_1954; size_t x_1955; size_t x_1956; lean_object* x_1957; lean_object* x_1958; lean_object* x_1959; lean_object* x_1960; lean_object* x_1961; lean_object* x_1962; lean_object* x_1963; lean_object* x_1964; lean_object* x_1965; lean_object* x_1966; +lean_dec(x_1924); +x_1952 = lean_ctor_get(x_1041, 0); +lean_inc(x_1952); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1953 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1953 = lean_box(0); +} +x_1954 = lean_array_get_size(x_1952); +x_1955 = lean_usize_of_nat(x_1954); +lean_dec(x_1954); +x_1956 = 0; +x_1957 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1955, x_1956, x_1952, x_1921); +x_1958 = lean_ctor_get(x_1957, 0); +lean_inc(x_1958); +x_1959 = lean_ctor_get(x_1957, 1); +lean_inc(x_1959); +if (lean_is_exclusive(x_1957)) { + lean_ctor_release(x_1957, 0); + lean_ctor_release(x_1957, 1); + x_1960 = x_1957; +} else { + lean_dec_ref(x_1957); + x_1960 = lean_box(0); +} +x_1961 = lean_ctor_get(x_1958, 0); +lean_inc(x_1961); +if (lean_is_exclusive(x_1958)) { + lean_ctor_release(x_1958, 0); + x_1962 = x_1958; +} else { + lean_dec_ref(x_1958); + x_1962 = lean_box(0); +} +if (lean_is_scalar(x_1953)) { + x_1963 = lean_alloc_ctor(1, 1, 0); +} else { + x_1963 = x_1953; +} +lean_ctor_set(x_1963, 0, x_1961); +x_1964 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1964, 0, x_1035); +lean_ctor_set(x_1964, 1, x_1036); +lean_ctor_set(x_1964, 2, x_30); +lean_ctor_set(x_1964, 3, x_1910); +lean_ctor_set(x_1964, 4, x_1911); +lean_ctor_set(x_1964, 5, x_1923); +lean_ctor_set(x_1964, 6, x_1911); +lean_ctor_set(x_1964, 7, x_1963); +if (lean_is_scalar(x_1962)) { + x_1965 = lean_alloc_ctor(1, 1, 0); +} else { + x_1965 = x_1962; +} +lean_ctor_set(x_1965, 0, x_1964); +if (lean_is_scalar(x_1960)) { + x_1966 = lean_alloc_ctor(0, 2, 0); +} else { + x_1966 = x_1960; +} +lean_ctor_set(x_1966, 0, x_1965); +lean_ctor_set(x_1966, 1, x_1959); +x_11 = x_1966; +goto block_29; +} } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_2); -lean_dec(x_1); -x_24 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_25 = lean_string_append(x_24, x_3); -lean_dec(x_3); -x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; -x_27 = lean_string_append(x_25, x_26); -x_28 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_20); -return x_29; +lean_object* x_1967; lean_object* x_1968; lean_object* x_1969; size_t x_1970; size_t x_1971; lean_object* x_1972; lean_object* x_1973; lean_object* x_1974; lean_object* x_1975; lean_object* x_1976; lean_object* x_1977; lean_object* x_1978; +lean_dec(x_1924); +x_1967 = lean_ctor_get(x_1040, 0); +lean_inc(x_1967); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_1968 = x_1040; +} else { + lean_dec_ref(x_1040); + x_1968 = lean_box(0); +} +x_1969 = lean_array_get_size(x_1967); +x_1970 = lean_usize_of_nat(x_1969); +lean_dec(x_1969); +x_1971 = 0; +x_1972 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_1970, x_1971, x_1967, x_1921); +x_1973 = lean_ctor_get(x_1972, 0); +lean_inc(x_1973); +x_1974 = lean_ctor_get(x_1972, 1); +lean_inc(x_1974); +lean_dec(x_1972); +x_1975 = lean_ctor_get(x_1973, 0); +lean_inc(x_1975); +if (lean_is_exclusive(x_1973)) { + lean_ctor_release(x_1973, 0); + x_1976 = x_1973; +} else { + lean_dec_ref(x_1973); + x_1976 = lean_box(0); } +if (lean_is_scalar(x_1968)) { + x_1977 = lean_alloc_ctor(1, 1, 0); +} else { + x_1977 = x_1968; } +lean_ctor_set(x_1977, 0, x_1975); +if (lean_is_scalar(x_1976)) { + x_1978 = lean_alloc_ctor(1, 1, 0); +} else { + x_1978 = x_1976; } +lean_ctor_set(x_1978, 0, x_1977); +x_1925 = x_1978; +x_1926 = x_1974; +goto block_1948; } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_4 = 1; -lean_inc(x_1); -x_5 = l_Lean_Name_toString(x_1, x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1; -x_7 = lean_string_append(x_6, x_5); -lean_dec(x_5); -x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2; -x_9 = lean_string_append(x_7, x_8); -x_10 = lean_io_initializing(x_3); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_unbox(x_11); -lean_dec(x_11); -if (x_12 == 0) +block_1948: { -uint8_t x_13; -lean_dec(x_2); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_10); -if (x_13 == 0) +if (lean_obj_tag(x_1041) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_ctor_get(x_10, 0); -lean_dec(x_14); -x_15 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_16 = lean_string_append(x_15, x_9); -lean_dec(x_9); -x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -x_18 = lean_string_append(x_16, x_17); -x_19 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set_tag(x_10, 1); -lean_ctor_set(x_10, 0, x_19); -return x_10; +lean_object* x_1927; lean_object* x_1928; lean_object* x_1929; lean_object* x_1930; lean_object* x_1931; +x_1927 = lean_ctor_get(x_1925, 0); +lean_inc(x_1927); +if (lean_is_exclusive(x_1925)) { + lean_ctor_release(x_1925, 0); + x_1928 = x_1925; +} else { + lean_dec_ref(x_1925); + x_1928 = lean_box(0); +} +x_1929 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1929, 0, x_1035); +lean_ctor_set(x_1929, 1, x_1036); +lean_ctor_set(x_1929, 2, x_30); +lean_ctor_set(x_1929, 3, x_1910); +lean_ctor_set(x_1929, 4, x_1911); +lean_ctor_set(x_1929, 5, x_1923); +lean_ctor_set(x_1929, 6, x_1927); +lean_ctor_set(x_1929, 7, x_1911); +if (lean_is_scalar(x_1928)) { + x_1930 = lean_alloc_ctor(1, 1, 0); +} else { + x_1930 = x_1928; } -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_20 = lean_ctor_get(x_10, 1); -lean_inc(x_20); -lean_dec(x_10); -x_21 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; -x_22 = lean_string_append(x_21, x_9); -lean_dec(x_9); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; -x_24 = lean_string_append(x_22, x_23); -x_25 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_20); -return x_26; +lean_ctor_set(x_1930, 0, x_1929); +if (lean_is_scalar(x_1922)) { + x_1931 = lean_alloc_ctor(0, 2, 0); +} else { + x_1931 = x_1922; } +lean_ctor_set(x_1931, 0, x_1930); +lean_ctor_set(x_1931, 1, x_1926); +x_11 = x_1931; +goto block_29; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_10, 1); -lean_inc(x_27); -lean_dec(x_10); -x_28 = lean_box(0); -x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); -return x_29; +lean_object* x_1932; lean_object* x_1933; lean_object* x_1934; lean_object* x_1935; size_t x_1936; size_t x_1937; lean_object* x_1938; lean_object* x_1939; lean_object* x_1940; lean_object* x_1941; lean_object* x_1942; lean_object* x_1943; lean_object* x_1944; lean_object* x_1945; lean_object* x_1946; lean_object* x_1947; +lean_dec(x_1922); +x_1932 = lean_ctor_get(x_1925, 0); +lean_inc(x_1932); +lean_dec(x_1925); +x_1933 = lean_ctor_get(x_1041, 0); +lean_inc(x_1933); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_1934 = x_1041; +} else { + lean_dec_ref(x_1041); + x_1934 = lean_box(0); +} +x_1935 = lean_array_get_size(x_1933); +x_1936 = lean_usize_of_nat(x_1935); +lean_dec(x_1935); +x_1937 = 0; +x_1938 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_1936, x_1937, x_1933, x_1926); +x_1939 = lean_ctor_get(x_1938, 0); +lean_inc(x_1939); +x_1940 = lean_ctor_get(x_1938, 1); +lean_inc(x_1940); +if (lean_is_exclusive(x_1938)) { + lean_ctor_release(x_1938, 0); + lean_ctor_release(x_1938, 1); + x_1941 = x_1938; +} else { + lean_dec_ref(x_1938); + x_1941 = lean_box(0); +} +x_1942 = lean_ctor_get(x_1939, 0); +lean_inc(x_1942); +if (lean_is_exclusive(x_1939)) { + lean_ctor_release(x_1939, 0); + x_1943 = x_1939; +} else { + lean_dec_ref(x_1939); + x_1943 = lean_box(0); } +if (lean_is_scalar(x_1934)) { + x_1944 = lean_alloc_ctor(1, 1, 0); +} else { + x_1944 = x_1934; +} +lean_ctor_set(x_1944, 0, x_1942); +x_1945 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_1945, 0, x_1035); +lean_ctor_set(x_1945, 1, x_1036); +lean_ctor_set(x_1945, 2, x_30); +lean_ctor_set(x_1945, 3, x_1910); +lean_ctor_set(x_1945, 4, x_1911); +lean_ctor_set(x_1945, 5, x_1923); +lean_ctor_set(x_1945, 6, x_1932); +lean_ctor_set(x_1945, 7, x_1944); +if (lean_is_scalar(x_1943)) { + x_1946 = lean_alloc_ctor(1, 1, 0); +} else { + x_1946 = x_1943; } +lean_ctor_set(x_1946, 0, x_1945); +if (lean_is_scalar(x_1941)) { + x_1947 = lean_alloc_ctor(0, 2, 0); +} else { + x_1947 = x_1941; } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("getInteractiveTermGoal", 22); -return x_1; +lean_ctor_set(x_1947, 0, x_1946); +lean_ctor_set(x_1947, 1, x_1940); +x_11 = x_1947; +goto block_29; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_FileWorker_getInteractiveTermGoal), 3, 0); -return x_1; +lean_object* x_1979; lean_object* x_1980; lean_object* x_1981; lean_object* x_1982; lean_object* x_1983; lean_object* x_1984; +x_1979 = lean_ctor_get(x_1038, 0); +lean_inc(x_1979); +if (lean_is_exclusive(x_1038)) { + lean_ctor_release(x_1038, 0); + x_1980 = x_1038; +} else { + lean_dec_ref(x_1038); + x_1980 = lean_box(0); } +if (lean_is_scalar(x_1980)) { + x_1981 = lean_alloc_ctor(1, 1, 0); +} else { + x_1981 = x_1980; +} +lean_ctor_set(x_1981, 0, x_1979); +x_1982 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_1983 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_1982, x_1039, x_4); +x_1984 = lean_ctor_get(x_1983, 0); +lean_inc(x_1984); +if (lean_obj_tag(x_1984) == 0) +{ +lean_object* x_1985; lean_object* x_1986; lean_object* x_1987; lean_object* x_1988; lean_object* x_1989; lean_object* x_1990; +lean_dec(x_1981); +lean_dec(x_1910); +lean_dec(x_30); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_1985 = lean_ctor_get(x_1983, 1); +lean_inc(x_1985); +if (lean_is_exclusive(x_1983)) { + lean_ctor_release(x_1983, 0); + lean_ctor_release(x_1983, 1); + x_1986 = x_1983; +} else { + lean_dec_ref(x_1983); + x_1986 = lean_box(0); +} +x_1987 = lean_ctor_get(x_1984, 0); +lean_inc(x_1987); +if (lean_is_exclusive(x_1984)) { + lean_ctor_release(x_1984, 0); + x_1988 = x_1984; +} else { + lean_dec_ref(x_1984); + x_1988 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2; -x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3; -x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1(x_2, x_3, x_1); -return x_4; +if (lean_is_scalar(x_1988)) { + x_1989 = lean_alloc_ctor(0, 1, 0); +} else { + x_1989 = x_1988; +} +lean_ctor_set(x_1989, 0, x_1987); +if (lean_is_scalar(x_1986)) { + x_1990 = lean_alloc_ctor(0, 2, 0); +} else { + x_1990 = x_1986; } +lean_ctor_set(x_1990, 0, x_1989); +lean_ctor_set(x_1990, 1, x_1985); +x_11 = x_1990; +goto block_29; } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -lean_object* x_5; -x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; +lean_object* x_1991; lean_object* x_1992; lean_object* x_1993; lean_object* x_1994; lean_object* x_1995; lean_object* x_1996; +x_1991 = lean_ctor_get(x_1983, 1); +lean_inc(x_1991); +if (lean_is_exclusive(x_1983)) { + lean_ctor_release(x_1983, 0); + lean_ctor_release(x_1983, 1); + x_1992 = x_1983; +} else { + lean_dec_ref(x_1983); + x_1992 = lean_box(0); +} +x_1993 = lean_ctor_get(x_1984, 0); +lean_inc(x_1993); +if (lean_is_exclusive(x_1984)) { + lean_ctor_release(x_1984, 0); + x_1994 = x_1984; +} else { + lean_dec_ref(x_1984); + x_1994 = lean_box(0); +} +if (lean_obj_tag(x_1040) == 0) +{ +lean_object* x_2020; +lean_dec(x_1992); +x_2020 = lean_box(0); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_2021; lean_object* x_2022; lean_object* x_2023; +x_2021 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2021, 0, x_1035); +lean_ctor_set(x_2021, 1, x_1036); +lean_ctor_set(x_2021, 2, x_30); +lean_ctor_set(x_2021, 3, x_1910); +lean_ctor_set(x_2021, 4, x_1981); +lean_ctor_set(x_2021, 5, x_1993); +lean_ctor_set(x_2021, 6, x_2020); +lean_ctor_set(x_2021, 7, x_2020); +if (lean_is_scalar(x_1994)) { + x_2022 = lean_alloc_ctor(1, 1, 0); +} else { + x_2022 = x_1994; } +lean_ctor_set(x_2022, 0, x_2021); +x_2023 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2023, 0, x_2022); +lean_ctor_set(x_2023, 1, x_1991); +x_11 = x_2023; +goto block_29; } -static lean_object* _init_l_Lean_Widget_instInhabitedGetInteractiveDiagnosticsParams() { -_start: +else { -lean_object* x_1; -x_1 = lean_box(0); -return x_1; +lean_object* x_2024; lean_object* x_2025; lean_object* x_2026; size_t x_2027; size_t x_2028; lean_object* x_2029; lean_object* x_2030; lean_object* x_2031; lean_object* x_2032; lean_object* x_2033; lean_object* x_2034; lean_object* x_2035; lean_object* x_2036; lean_object* x_2037; lean_object* x_2038; +lean_dec(x_1994); +x_2024 = lean_ctor_get(x_1041, 0); +lean_inc(x_2024); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2025 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2025 = lean_box(0); +} +x_2026 = lean_array_get_size(x_2024); +x_2027 = lean_usize_of_nat(x_2026); +lean_dec(x_2026); +x_2028 = 0; +x_2029 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2027, x_2028, x_2024, x_1991); +x_2030 = lean_ctor_get(x_2029, 0); +lean_inc(x_2030); +x_2031 = lean_ctor_get(x_2029, 1); +lean_inc(x_2031); +if (lean_is_exclusive(x_2029)) { + lean_ctor_release(x_2029, 0); + lean_ctor_release(x_2029, 1); + x_2032 = x_2029; +} else { + lean_dec_ref(x_2029); + x_2032 = lean_box(0); +} +x_2033 = lean_ctor_get(x_2030, 0); +lean_inc(x_2033); +if (lean_is_exclusive(x_2030)) { + lean_ctor_release(x_2030, 0); + x_2034 = x_2030; +} else { + lean_dec_ref(x_2030); + x_2034 = lean_box(0); } +if (lean_is_scalar(x_2025)) { + x_2035 = lean_alloc_ctor(1, 1, 0); +} else { + x_2035 = x_2025; +} +lean_ctor_set(x_2035, 0, x_2033); +x_2036 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2036, 0, x_1035); +lean_ctor_set(x_2036, 1, x_1036); +lean_ctor_set(x_2036, 2, x_30); +lean_ctor_set(x_2036, 3, x_1910); +lean_ctor_set(x_2036, 4, x_1981); +lean_ctor_set(x_2036, 5, x_1993); +lean_ctor_set(x_2036, 6, x_2020); +lean_ctor_set(x_2036, 7, x_2035); +if (lean_is_scalar(x_2034)) { + x_2037 = lean_alloc_ctor(1, 1, 0); +} else { + x_2037 = x_2034; } -static lean_object* _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_ctor_set(x_2037, 0, x_2036); +if (lean_is_scalar(x_2032)) { + x_2038 = lean_alloc_ctor(0, 2, 0); +} else { + x_2038 = x_2032; } +lean_ctor_set(x_2038, 0, x_2037); +lean_ctor_set(x_2038, 1, x_2031); +x_11 = x_2038; +goto block_29; } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Lean_Json_getObjValD(x_1, x_2); -if (lean_obj_tag(x_3) == 0) -{ -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1___closed__1; -return x_4; } else { -lean_object* x_5; -x_5 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonLineRange____x40_Lean_Data_Lsp_Extra___hyg_1810_(x_3); -lean_dec(x_3); -if (lean_obj_tag(x_5) == 0) -{ -uint8_t x_6; -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) -{ -return x_5; +lean_object* x_2039; lean_object* x_2040; lean_object* x_2041; size_t x_2042; size_t x_2043; lean_object* x_2044; lean_object* x_2045; lean_object* x_2046; lean_object* x_2047; lean_object* x_2048; lean_object* x_2049; lean_object* x_2050; +lean_dec(x_1994); +x_2039 = lean_ctor_get(x_1040, 0); +lean_inc(x_2039); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_2040 = x_1040; +} else { + lean_dec_ref(x_1040); + x_2040 = lean_box(0); +} +x_2041 = lean_array_get_size(x_2039); +x_2042 = lean_usize_of_nat(x_2041); +lean_dec(x_2041); +x_2043 = 0; +x_2044 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_2042, x_2043, x_2039, x_1991); +x_2045 = lean_ctor_get(x_2044, 0); +lean_inc(x_2045); +x_2046 = lean_ctor_get(x_2044, 1); +lean_inc(x_2046); +lean_dec(x_2044); +x_2047 = lean_ctor_get(x_2045, 0); +lean_inc(x_2047); +if (lean_is_exclusive(x_2045)) { + lean_ctor_release(x_2045, 0); + x_2048 = x_2045; +} else { + lean_dec_ref(x_2045); + x_2048 = lean_box(0); } -else -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; +if (lean_is_scalar(x_2040)) { + x_2049 = lean_alloc_ctor(1, 1, 0); +} else { + x_2049 = x_2040; } +lean_ctor_set(x_2049, 0, x_2047); +if (lean_is_scalar(x_2048)) { + x_2050 = lean_alloc_ctor(1, 1, 0); +} else { + x_2050 = x_2048; } -else +lean_ctor_set(x_2050, 0, x_2049); +x_1995 = x_2050; +x_1996 = x_2046; +goto block_2019; +} +block_2019: { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_5); -if (x_9 == 0) +if (lean_obj_tag(x_1041) == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_5, 0); -x_11 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_5, 0, x_11); -return x_5; +lean_object* x_1997; lean_object* x_1998; lean_object* x_1999; lean_object* x_2000; lean_object* x_2001; lean_object* x_2002; +x_1997 = lean_ctor_get(x_1995, 0); +lean_inc(x_1997); +if (lean_is_exclusive(x_1995)) { + lean_ctor_release(x_1995, 0); + x_1998 = x_1995; +} else { + lean_dec_ref(x_1995); + x_1998 = lean_box(0); +} +x_1999 = lean_box(0); +x_2000 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2000, 0, x_1035); +lean_ctor_set(x_2000, 1, x_1036); +lean_ctor_set(x_2000, 2, x_30); +lean_ctor_set(x_2000, 3, x_1910); +lean_ctor_set(x_2000, 4, x_1981); +lean_ctor_set(x_2000, 5, x_1993); +lean_ctor_set(x_2000, 6, x_1997); +lean_ctor_set(x_2000, 7, x_1999); +if (lean_is_scalar(x_1998)) { + x_2001 = lean_alloc_ctor(1, 1, 0); +} else { + x_2001 = x_1998; +} +lean_ctor_set(x_2001, 0, x_2000); +if (lean_is_scalar(x_1992)) { + x_2002 = lean_alloc_ctor(0, 2, 0); +} else { + x_2002 = x_1992; +} +lean_ctor_set(x_2002, 0, x_2001); +lean_ctor_set(x_2002, 1, x_1996); +x_11 = x_2002; +goto block_29; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_5, 0); -lean_inc(x_12); -lean_dec(x_5); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +lean_object* x_2003; lean_object* x_2004; lean_object* x_2005; lean_object* x_2006; size_t x_2007; size_t x_2008; lean_object* x_2009; lean_object* x_2010; lean_object* x_2011; lean_object* x_2012; lean_object* x_2013; lean_object* x_2014; lean_object* x_2015; lean_object* x_2016; lean_object* x_2017; lean_object* x_2018; +lean_dec(x_1992); +x_2003 = lean_ctor_get(x_1995, 0); +lean_inc(x_2003); +lean_dec(x_1995); +x_2004 = lean_ctor_get(x_1041, 0); +lean_inc(x_2004); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2005 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2005 = lean_box(0); +} +x_2006 = lean_array_get_size(x_2004); +x_2007 = lean_usize_of_nat(x_2006); +lean_dec(x_2006); +x_2008 = 0; +x_2009 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2007, x_2008, x_2004, x_1996); +x_2010 = lean_ctor_get(x_2009, 0); +lean_inc(x_2010); +x_2011 = lean_ctor_get(x_2009, 1); +lean_inc(x_2011); +if (lean_is_exclusive(x_2009)) { + lean_ctor_release(x_2009, 0); + lean_ctor_release(x_2009, 1); + x_2012 = x_2009; +} else { + lean_dec_ref(x_2009); + x_2012 = lean_box(0); +} +x_2013 = lean_ctor_get(x_2010, 0); +lean_inc(x_2013); +if (lean_is_exclusive(x_2010)) { + lean_ctor_release(x_2010, 0); + x_2014 = x_2010; +} else { + lean_dec_ref(x_2010); + x_2014 = lean_box(0); +} +if (lean_is_scalar(x_2005)) { + x_2015 = lean_alloc_ctor(1, 1, 0); +} else { + x_2015 = x_2005; +} +lean_ctor_set(x_2015, 0, x_2013); +x_2016 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2016, 0, x_1035); +lean_ctor_set(x_2016, 1, x_1036); +lean_ctor_set(x_2016, 2, x_30); +lean_ctor_set(x_2016, 3, x_1910); +lean_ctor_set(x_2016, 4, x_1981); +lean_ctor_set(x_2016, 5, x_1993); +lean_ctor_set(x_2016, 6, x_2003); +lean_ctor_set(x_2016, 7, x_2015); +if (lean_is_scalar(x_2014)) { + x_2017 = lean_alloc_ctor(1, 1, 0); +} else { + x_2017 = x_2014; } +lean_ctor_set(x_2017, 0, x_2016); +if (lean_is_scalar(x_2012)) { + x_2018 = lean_alloc_ctor(0, 2, 0); +} else { + x_2018 = x_2012; +} +lean_ctor_set(x_2018, 0, x_2017); +lean_ctor_set(x_2018, 1, x_2011); +x_11 = x_2018; +goto block_29; } } } } -static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("lineRange", 9); -return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; -x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____closed__1; -x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1(x_1, x_2); -if (lean_obj_tag(x_3) == 0) -{ -uint8_t x_4; -x_4 = !lean_is_exclusive(x_3); -if (x_4 == 0) -{ -return x_3; } else { -lean_object* x_5; lean_object* x_6; -x_5 = lean_ctor_get(x_3, 0); -lean_inc(x_5); -lean_dec(x_3); -x_6 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_6, 0, x_5); -return x_6; +lean_object* x_2051; lean_object* x_2052; +x_2051 = lean_ctor_get(x_30, 0); +lean_inc(x_2051); +lean_dec(x_30); +x_2052 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2052, 0, x_2051); +if (lean_obj_tag(x_1037) == 0) +{ +lean_object* x_2053; +x_2053 = lean_box(0); +if (lean_obj_tag(x_1038) == 0) +{ +lean_object* x_2054; lean_object* x_2055; lean_object* x_2056; +x_2054 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_2055 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_2054, x_1039, x_4); +x_2056 = lean_ctor_get(x_2055, 0); +lean_inc(x_2056); +if (lean_obj_tag(x_2056) == 0) +{ +lean_object* x_2057; lean_object* x_2058; lean_object* x_2059; lean_object* x_2060; lean_object* x_2061; lean_object* x_2062; +lean_dec(x_2052); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_2057 = lean_ctor_get(x_2055, 1); +lean_inc(x_2057); +if (lean_is_exclusive(x_2055)) { + lean_ctor_release(x_2055, 0); + lean_ctor_release(x_2055, 1); + x_2058 = x_2055; +} else { + lean_dec_ref(x_2055); + x_2058 = lean_box(0); +} +x_2059 = lean_ctor_get(x_2056, 0); +lean_inc(x_2059); +if (lean_is_exclusive(x_2056)) { + lean_ctor_release(x_2056, 0); + x_2060 = x_2056; +} else { + lean_dec_ref(x_2056); + x_2060 = lean_box(0); +} +if (lean_is_scalar(x_2060)) { + x_2061 = lean_alloc_ctor(0, 1, 0); +} else { + x_2061 = x_2060; +} +lean_ctor_set(x_2061, 0, x_2059); +if (lean_is_scalar(x_2058)) { + x_2062 = lean_alloc_ctor(0, 2, 0); +} else { + x_2062 = x_2058; } +lean_ctor_set(x_2062, 0, x_2061); +lean_ctor_set(x_2062, 1, x_2057); +x_11 = x_2062; +goto block_29; } else { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_3); -if (x_7 == 0) -{ -return x_3; +lean_object* x_2063; lean_object* x_2064; lean_object* x_2065; lean_object* x_2066; lean_object* x_2067; lean_object* x_2068; +x_2063 = lean_ctor_get(x_2055, 1); +lean_inc(x_2063); +if (lean_is_exclusive(x_2055)) { + lean_ctor_release(x_2055, 0); + lean_ctor_release(x_2055, 1); + x_2064 = x_2055; +} else { + lean_dec_ref(x_2055); + x_2064 = lean_box(0); +} +x_2065 = lean_ctor_get(x_2056, 0); +lean_inc(x_2065); +if (lean_is_exclusive(x_2056)) { + lean_ctor_release(x_2056, 0); + x_2066 = x_2056; +} else { + lean_dec_ref(x_2056); + x_2066 = lean_box(0); +} +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_2064); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_2091; lean_object* x_2092; lean_object* x_2093; +x_2091 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2091, 0, x_1035); +lean_ctor_set(x_2091, 1, x_1036); +lean_ctor_set(x_2091, 2, x_2052); +lean_ctor_set(x_2091, 3, x_2053); +lean_ctor_set(x_2091, 4, x_2053); +lean_ctor_set(x_2091, 5, x_2065); +lean_ctor_set(x_2091, 6, x_2053); +lean_ctor_set(x_2091, 7, x_2053); +if (lean_is_scalar(x_2066)) { + x_2092 = lean_alloc_ctor(1, 1, 0); +} else { + x_2092 = x_2066; +} +lean_ctor_set(x_2092, 0, x_2091); +x_2093 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2093, 0, x_2092); +lean_ctor_set(x_2093, 1, x_2063); +x_11 = x_2093; +goto block_29; } else { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_3, 0); -lean_inc(x_8); -lean_dec(x_3); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_8); -return x_9; -} +lean_object* x_2094; lean_object* x_2095; lean_object* x_2096; size_t x_2097; size_t x_2098; lean_object* x_2099; lean_object* x_2100; lean_object* x_2101; lean_object* x_2102; lean_object* x_2103; lean_object* x_2104; lean_object* x_2105; lean_object* x_2106; lean_object* x_2107; lean_object* x_2108; +lean_dec(x_2066); +x_2094 = lean_ctor_get(x_1041, 0); +lean_inc(x_2094); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2095 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2095 = lean_box(0); +} +x_2096 = lean_array_get_size(x_2094); +x_2097 = lean_usize_of_nat(x_2096); +lean_dec(x_2096); +x_2098 = 0; +x_2099 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2097, x_2098, x_2094, x_2063); +x_2100 = lean_ctor_get(x_2099, 0); +lean_inc(x_2100); +x_2101 = lean_ctor_get(x_2099, 1); +lean_inc(x_2101); +if (lean_is_exclusive(x_2099)) { + lean_ctor_release(x_2099, 0); + lean_ctor_release(x_2099, 1); + x_2102 = x_2099; +} else { + lean_dec_ref(x_2099); + x_2102 = lean_box(0); +} +x_2103 = lean_ctor_get(x_2100, 0); +lean_inc(x_2103); +if (lean_is_exclusive(x_2100)) { + lean_ctor_release(x_2100, 0); + x_2104 = x_2100; +} else { + lean_dec_ref(x_2100); + x_2104 = lean_box(0); } +if (lean_is_scalar(x_2095)) { + x_2105 = lean_alloc_ctor(1, 1, 0); +} else { + x_2105 = x_2095; +} +lean_ctor_set(x_2105, 0, x_2103); +x_2106 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2106, 0, x_1035); +lean_ctor_set(x_2106, 1, x_1036); +lean_ctor_set(x_2106, 2, x_2052); +lean_ctor_set(x_2106, 3, x_2053); +lean_ctor_set(x_2106, 4, x_2053); +lean_ctor_set(x_2106, 5, x_2065); +lean_ctor_set(x_2106, 6, x_2053); +lean_ctor_set(x_2106, 7, x_2105); +if (lean_is_scalar(x_2104)) { + x_2107 = lean_alloc_ctor(1, 1, 0); +} else { + x_2107 = x_2104; } +lean_ctor_set(x_2107, 0, x_2106); +if (lean_is_scalar(x_2102)) { + x_2108 = lean_alloc_ctor(0, 2, 0); +} else { + x_2108 = x_2102; } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; +lean_ctor_set(x_2108, 0, x_2107); +lean_ctor_set(x_2108, 1, x_2101); +x_11 = x_2108; +goto block_29; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____boxed(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311_(x_1); -lean_dec(x_1); -return x_2; +lean_object* x_2109; lean_object* x_2110; lean_object* x_2111; size_t x_2112; size_t x_2113; lean_object* x_2114; lean_object* x_2115; lean_object* x_2116; lean_object* x_2117; lean_object* x_2118; lean_object* x_2119; lean_object* x_2120; +lean_dec(x_2066); +x_2109 = lean_ctor_get(x_1040, 0); +lean_inc(x_2109); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_2110 = x_1040; +} else { + lean_dec_ref(x_1040); + x_2110 = lean_box(0); +} +x_2111 = lean_array_get_size(x_2109); +x_2112 = lean_usize_of_nat(x_2111); +lean_dec(x_2111); +x_2113 = 0; +x_2114 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_2112, x_2113, x_2109, x_2063); +x_2115 = lean_ctor_get(x_2114, 0); +lean_inc(x_2115); +x_2116 = lean_ctor_get(x_2114, 1); +lean_inc(x_2116); +lean_dec(x_2114); +x_2117 = lean_ctor_get(x_2115, 0); +lean_inc(x_2117); +if (lean_is_exclusive(x_2115)) { + lean_ctor_release(x_2115, 0); + x_2118 = x_2115; +} else { + lean_dec_ref(x_2115); + x_2118 = lean_box(0); } +if (lean_is_scalar(x_2110)) { + x_2119 = lean_alloc_ctor(1, 1, 0); +} else { + x_2119 = x_2110; } -static lean_object* _init_l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____boxed), 1, 0); -return x_1; +lean_ctor_set(x_2119, 0, x_2117); +if (lean_is_scalar(x_2118)) { + x_2120 = lean_alloc_ctor(1, 1, 0); +} else { + x_2120 = x_2118; } +lean_ctor_set(x_2120, 0, x_2119); +x_2067 = x_2120; +x_2068 = x_2116; +goto block_2090; } -static lean_object* _init_l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams() { -_start: +block_2090: { -lean_object* x_1; -x_1 = l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams___closed__1; -return x_1; +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_2069; lean_object* x_2070; lean_object* x_2071; lean_object* x_2072; lean_object* x_2073; +x_2069 = lean_ctor_get(x_2067, 0); +lean_inc(x_2069); +if (lean_is_exclusive(x_2067)) { + lean_ctor_release(x_2067, 0); + x_2070 = x_2067; +} else { + lean_dec_ref(x_2067); + x_2070 = lean_box(0); +} +x_2071 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2071, 0, x_1035); +lean_ctor_set(x_2071, 1, x_1036); +lean_ctor_set(x_2071, 2, x_2052); +lean_ctor_set(x_2071, 3, x_2053); +lean_ctor_set(x_2071, 4, x_2053); +lean_ctor_set(x_2071, 5, x_2065); +lean_ctor_set(x_2071, 6, x_2069); +lean_ctor_set(x_2071, 7, x_2053); +if (lean_is_scalar(x_2070)) { + x_2072 = lean_alloc_ctor(1, 1, 0); +} else { + x_2072 = x_2070; } +lean_ctor_set(x_2072, 0, x_2071); +if (lean_is_scalar(x_2064)) { + x_2073 = lean_alloc_ctor(0, 2, 0); +} else { + x_2073 = x_2064; } -LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1349____spec__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -lean_dec(x_1); -x_3 = lean_box(0); -return x_3; +lean_ctor_set(x_2073, 0, x_2072); +lean_ctor_set(x_2073, 1, x_2068); +x_11 = x_2073; +goto block_29; } else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -lean_dec(x_2); -x_5 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonLineRange____x40_Lean_Data_Lsp_Extra___hyg_1865_(x_4); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -x_7 = lean_box(0); -x_8 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_8, 0, x_6); -lean_ctor_set(x_8, 1, x_7); -return x_8; +lean_object* x_2074; lean_object* x_2075; lean_object* x_2076; lean_object* x_2077; size_t x_2078; size_t x_2079; lean_object* x_2080; lean_object* x_2081; lean_object* x_2082; lean_object* x_2083; lean_object* x_2084; lean_object* x_2085; lean_object* x_2086; lean_object* x_2087; lean_object* x_2088; lean_object* x_2089; +lean_dec(x_2064); +x_2074 = lean_ctor_get(x_2067, 0); +lean_inc(x_2074); +lean_dec(x_2067); +x_2075 = lean_ctor_get(x_1041, 0); +lean_inc(x_2075); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2076 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2076 = lean_box(0); +} +x_2077 = lean_array_get_size(x_2075); +x_2078 = lean_usize_of_nat(x_2077); +lean_dec(x_2077); +x_2079 = 0; +x_2080 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2078, x_2079, x_2075, x_2068); +x_2081 = lean_ctor_get(x_2080, 0); +lean_inc(x_2081); +x_2082 = lean_ctor_get(x_2080, 1); +lean_inc(x_2082); +if (lean_is_exclusive(x_2080)) { + lean_ctor_release(x_2080, 0); + lean_ctor_release(x_2080, 1); + x_2083 = x_2080; +} else { + lean_dec_ref(x_2080); + x_2083 = lean_box(0); +} +x_2084 = lean_ctor_get(x_2081, 0); +lean_inc(x_2084); +if (lean_is_exclusive(x_2081)) { + lean_ctor_release(x_2081, 0); + x_2085 = x_2081; +} else { + lean_dec_ref(x_2081); + x_2085 = lean_box(0); +} +if (lean_is_scalar(x_2076)) { + x_2086 = lean_alloc_ctor(1, 1, 0); +} else { + x_2086 = x_2076; +} +lean_ctor_set(x_2086, 0, x_2084); +x_2087 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2087, 0, x_1035); +lean_ctor_set(x_2087, 1, x_1036); +lean_ctor_set(x_2087, 2, x_2052); +lean_ctor_set(x_2087, 3, x_2053); +lean_ctor_set(x_2087, 4, x_2053); +lean_ctor_set(x_2087, 5, x_2065); +lean_ctor_set(x_2087, 6, x_2074); +lean_ctor_set(x_2087, 7, x_2086); +if (lean_is_scalar(x_2085)) { + x_2088 = lean_alloc_ctor(1, 1, 0); +} else { + x_2088 = x_2085; } +lean_ctor_set(x_2088, 0, x_2087); +if (lean_is_scalar(x_2083)) { + x_2089 = lean_alloc_ctor(0, 2, 0); +} else { + x_2089 = x_2083; } +lean_ctor_set(x_2089, 0, x_2088); +lean_ctor_set(x_2089, 1, x_2082); +x_11 = x_2089; +goto block_29; } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1349_(lean_object* x_1) { -_start: +} +} +} +else { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____closed__1; -x_3 = l_Lean_Json_opt___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1349____spec__1(x_2, x_1); -x_4 = lean_box(0); -x_5 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_5, 0, x_3); -lean_ctor_set(x_5, 1, x_4); -x_6 = l_List_join___rarg(x_5); -x_7 = l_Lean_Json_mkObj(x_6); -return x_7; +lean_object* x_2121; lean_object* x_2122; lean_object* x_2123; lean_object* x_2124; lean_object* x_2125; lean_object* x_2126; +x_2121 = lean_ctor_get(x_1038, 0); +lean_inc(x_2121); +if (lean_is_exclusive(x_1038)) { + lean_ctor_release(x_1038, 0); + x_2122 = x_1038; +} else { + lean_dec_ref(x_1038); + x_2122 = lean_box(0); +} +if (lean_is_scalar(x_2122)) { + x_2123 = lean_alloc_ctor(1, 1, 0); +} else { + x_2123 = x_2122; +} +lean_ctor_set(x_2123, 0, x_2121); +x_2124 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_2125 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_2124, x_1039, x_4); +x_2126 = lean_ctor_get(x_2125, 0); +lean_inc(x_2126); +if (lean_obj_tag(x_2126) == 0) +{ +lean_object* x_2127; lean_object* x_2128; lean_object* x_2129; lean_object* x_2130; lean_object* x_2131; lean_object* x_2132; +lean_dec(x_2123); +lean_dec(x_2052); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_2127 = lean_ctor_get(x_2125, 1); +lean_inc(x_2127); +if (lean_is_exclusive(x_2125)) { + lean_ctor_release(x_2125, 0); + lean_ctor_release(x_2125, 1); + x_2128 = x_2125; +} else { + lean_dec_ref(x_2125); + x_2128 = lean_box(0); +} +x_2129 = lean_ctor_get(x_2126, 0); +lean_inc(x_2129); +if (lean_is_exclusive(x_2126)) { + lean_ctor_release(x_2126, 0); + x_2130 = x_2126; +} else { + lean_dec_ref(x_2126); + x_2130 = lean_box(0); } +if (lean_is_scalar(x_2130)) { + x_2131 = lean_alloc_ctor(0, 1, 0); +} else { + x_2131 = x_2130; } -static lean_object* _init_l_Lean_Widget_instToJsonGetInteractiveDiagnosticsParams___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1349_), 1, 0); -return x_1; +lean_ctor_set(x_2131, 0, x_2129); +if (lean_is_scalar(x_2128)) { + x_2132 = lean_alloc_ctor(0, 2, 0); +} else { + x_2132 = x_2128; } +lean_ctor_set(x_2132, 0, x_2131); +lean_ctor_set(x_2132, 1, x_2127); +x_11 = x_2132; +goto block_29; } -static lean_object* _init_l_Lean_Widget_instToJsonGetInteractiveDiagnosticsParams() { -_start: +else { -lean_object* x_1; -x_1 = l_Lean_Widget_instToJsonGetInteractiveDiagnosticsParams___closed__1; -return x_1; +lean_object* x_2133; lean_object* x_2134; lean_object* x_2135; lean_object* x_2136; lean_object* x_2137; lean_object* x_2138; +x_2133 = lean_ctor_get(x_2125, 1); +lean_inc(x_2133); +if (lean_is_exclusive(x_2125)) { + lean_ctor_release(x_2125, 0); + lean_ctor_release(x_2125, 1); + x_2134 = x_2125; +} else { + lean_dec_ref(x_2125); + x_2134 = lean_box(0); +} +x_2135 = lean_ctor_get(x_2126, 0); +lean_inc(x_2135); +if (lean_is_exclusive(x_2126)) { + lean_ctor_release(x_2126, 0); + x_2136 = x_2126; +} else { + lean_dec_ref(x_2126); + x_2136 = lean_box(0); +} +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_2134); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_2161; lean_object* x_2162; lean_object* x_2163; +x_2161 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2161, 0, x_1035); +lean_ctor_set(x_2161, 1, x_1036); +lean_ctor_set(x_2161, 2, x_2052); +lean_ctor_set(x_2161, 3, x_2053); +lean_ctor_set(x_2161, 4, x_2123); +lean_ctor_set(x_2161, 5, x_2135); +lean_ctor_set(x_2161, 6, x_2053); +lean_ctor_set(x_2161, 7, x_2053); +if (lean_is_scalar(x_2136)) { + x_2162 = lean_alloc_ctor(1, 1, 0); +} else { + x_2162 = x_2136; } +lean_ctor_set(x_2162, 0, x_2161); +x_2163 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2163, 0, x_2162); +lean_ctor_set(x_2163, 1, x_2133); +x_11 = x_2163; +goto block_29; } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; -x_6 = lean_usize_dec_eq(x_3, x_4); -if (x_6 == 0) -{ -lean_object* x_7; size_t x_8; size_t x_9; -x_7 = lean_array_uget(x_2, x_3); -x_8 = 1; -x_9 = lean_usize_add(x_3, x_8); -if (lean_obj_tag(x_1) == 0) +else { -lean_object* x_10; -x_10 = lean_array_push(x_5, x_7); -x_3 = x_9; -x_5 = x_10; -goto _start; +lean_object* x_2164; lean_object* x_2165; lean_object* x_2166; size_t x_2167; size_t x_2168; lean_object* x_2169; lean_object* x_2170; lean_object* x_2171; lean_object* x_2172; lean_object* x_2173; lean_object* x_2174; lean_object* x_2175; lean_object* x_2176; lean_object* x_2177; lean_object* x_2178; +lean_dec(x_2136); +x_2164 = lean_ctor_get(x_1041, 0); +lean_inc(x_2164); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2165 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2165 = lean_box(0); +} +x_2166 = lean_array_get_size(x_2164); +x_2167 = lean_usize_of_nat(x_2166); +lean_dec(x_2166); +x_2168 = 0; +x_2169 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2167, x_2168, x_2164, x_2133); +x_2170 = lean_ctor_get(x_2169, 0); +lean_inc(x_2170); +x_2171 = lean_ctor_get(x_2169, 1); +lean_inc(x_2171); +if (lean_is_exclusive(x_2169)) { + lean_ctor_release(x_2169, 0); + lean_ctor_release(x_2169, 1); + x_2172 = x_2169; +} else { + lean_dec_ref(x_2169); + x_2172 = lean_box(0); +} +x_2173 = lean_ctor_get(x_2170, 0); +lean_inc(x_2173); +if (lean_is_exclusive(x_2170)) { + lean_ctor_release(x_2170, 0); + x_2174 = x_2170; +} else { + lean_dec_ref(x_2170); + x_2174 = lean_box(0); +} +if (lean_is_scalar(x_2165)) { + x_2175 = lean_alloc_ctor(1, 1, 0); +} else { + x_2175 = x_2165; +} +lean_ctor_set(x_2175, 0, x_2173); +x_2176 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2176, 0, x_1035); +lean_ctor_set(x_2176, 1, x_1036); +lean_ctor_set(x_2176, 2, x_2052); +lean_ctor_set(x_2176, 3, x_2053); +lean_ctor_set(x_2176, 4, x_2123); +lean_ctor_set(x_2176, 5, x_2135); +lean_ctor_set(x_2176, 6, x_2053); +lean_ctor_set(x_2176, 7, x_2175); +if (lean_is_scalar(x_2174)) { + x_2177 = lean_alloc_ctor(1, 1, 0); +} else { + x_2177 = x_2174; +} +lean_ctor_set(x_2177, 0, x_2176); +if (lean_is_scalar(x_2172)) { + x_2178 = lean_alloc_ctor(0, 2, 0); +} else { + x_2178 = x_2172; +} +lean_ctor_set(x_2178, 0, x_2177); +lean_ctor_set(x_2178, 1, x_2171); +x_11 = x_2178; +goto block_29; +} } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_12 = lean_ctor_get(x_1, 0); -x_13 = lean_ctor_get(x_12, 0); -x_14 = lean_ctor_get(x_12, 1); -x_15 = lean_ctor_get(x_7, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -lean_dec(x_16); -x_18 = lean_nat_dec_le(x_13, x_17); -if (x_18 == 0) -{ -uint8_t x_19; -x_19 = lean_nat_dec_le(x_17, x_13); -lean_dec(x_17); -if (x_19 == 0) -{ -lean_dec(x_15); -lean_dec(x_7); -x_3 = x_9; -goto _start; +lean_object* x_2179; lean_object* x_2180; lean_object* x_2181; size_t x_2182; size_t x_2183; lean_object* x_2184; lean_object* x_2185; lean_object* x_2186; lean_object* x_2187; lean_object* x_2188; lean_object* x_2189; lean_object* x_2190; +lean_dec(x_2136); +x_2179 = lean_ctor_get(x_1040, 0); +lean_inc(x_2179); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_2180 = x_1040; +} else { + lean_dec_ref(x_1040); + x_2180 = lean_box(0); +} +x_2181 = lean_array_get_size(x_2179); +x_2182 = lean_usize_of_nat(x_2181); +lean_dec(x_2181); +x_2183 = 0; +x_2184 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_2182, x_2183, x_2179, x_2133); +x_2185 = lean_ctor_get(x_2184, 0); +lean_inc(x_2185); +x_2186 = lean_ctor_get(x_2184, 1); +lean_inc(x_2186); +lean_dec(x_2184); +x_2187 = lean_ctor_get(x_2185, 0); +lean_inc(x_2187); +if (lean_is_exclusive(x_2185)) { + lean_ctor_release(x_2185, 0); + x_2188 = x_2185; +} else { + lean_dec_ref(x_2185); + x_2188 = lean_box(0); } -else +if (lean_is_scalar(x_2180)) { + x_2189 = lean_alloc_ctor(1, 1, 0); +} else { + x_2189 = x_2180; +} +lean_ctor_set(x_2189, 0, x_2187); +if (lean_is_scalar(x_2188)) { + x_2190 = lean_alloc_ctor(1, 1, 0); +} else { + x_2190 = x_2188; +} +lean_ctor_set(x_2190, 0, x_2189); +x_2137 = x_2190; +x_2138 = x_2186; +goto block_2160; +} +block_2160: { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = lean_ctor_get(x_15, 1); -lean_inc(x_21); -lean_dec(x_15); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_nat_dec_lt(x_13, x_22); -lean_dec(x_22); -if (x_23 == 0) +if (lean_obj_tag(x_1041) == 0) { -lean_dec(x_7); -x_3 = x_9; -goto _start; +lean_object* x_2139; lean_object* x_2140; lean_object* x_2141; lean_object* x_2142; lean_object* x_2143; +x_2139 = lean_ctor_get(x_2137, 0); +lean_inc(x_2139); +if (lean_is_exclusive(x_2137)) { + lean_ctor_release(x_2137, 0); + x_2140 = x_2137; +} else { + lean_dec_ref(x_2137); + x_2140 = lean_box(0); +} +x_2141 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2141, 0, x_1035); +lean_ctor_set(x_2141, 1, x_1036); +lean_ctor_set(x_2141, 2, x_2052); +lean_ctor_set(x_2141, 3, x_2053); +lean_ctor_set(x_2141, 4, x_2123); +lean_ctor_set(x_2141, 5, x_2135); +lean_ctor_set(x_2141, 6, x_2139); +lean_ctor_set(x_2141, 7, x_2053); +if (lean_is_scalar(x_2140)) { + x_2142 = lean_alloc_ctor(1, 1, 0); +} else { + x_2142 = x_2140; +} +lean_ctor_set(x_2142, 0, x_2141); +if (lean_is_scalar(x_2134)) { + x_2143 = lean_alloc_ctor(0, 2, 0); +} else { + x_2143 = x_2134; +} +lean_ctor_set(x_2143, 0, x_2142); +lean_ctor_set(x_2143, 1, x_2138); +x_11 = x_2143; +goto block_29; } else { -lean_object* x_25; -x_25 = lean_array_push(x_5, x_7); -x_3 = x_9; -x_5 = x_25; -goto _start; +lean_object* x_2144; lean_object* x_2145; lean_object* x_2146; lean_object* x_2147; size_t x_2148; size_t x_2149; lean_object* x_2150; lean_object* x_2151; lean_object* x_2152; lean_object* x_2153; lean_object* x_2154; lean_object* x_2155; lean_object* x_2156; lean_object* x_2157; lean_object* x_2158; lean_object* x_2159; +lean_dec(x_2134); +x_2144 = lean_ctor_get(x_2137, 0); +lean_inc(x_2144); +lean_dec(x_2137); +x_2145 = lean_ctor_get(x_1041, 0); +lean_inc(x_2145); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2146 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2146 = lean_box(0); +} +x_2147 = lean_array_get_size(x_2145); +x_2148 = lean_usize_of_nat(x_2147); +lean_dec(x_2147); +x_2149 = 0; +x_2150 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2148, x_2149, x_2145, x_2138); +x_2151 = lean_ctor_get(x_2150, 0); +lean_inc(x_2151); +x_2152 = lean_ctor_get(x_2150, 1); +lean_inc(x_2152); +if (lean_is_exclusive(x_2150)) { + lean_ctor_release(x_2150, 0); + lean_ctor_release(x_2150, 1); + x_2153 = x_2150; +} else { + lean_dec_ref(x_2150); + x_2153 = lean_box(0); +} +x_2154 = lean_ctor_get(x_2151, 0); +lean_inc(x_2154); +if (lean_is_exclusive(x_2151)) { + lean_ctor_release(x_2151, 0); + x_2155 = x_2151; +} else { + lean_dec_ref(x_2151); + x_2155 = lean_box(0); +} +if (lean_is_scalar(x_2146)) { + x_2156 = lean_alloc_ctor(1, 1, 0); +} else { + x_2156 = x_2146; +} +lean_ctor_set(x_2156, 0, x_2154); +x_2157 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2157, 0, x_1035); +lean_ctor_set(x_2157, 1, x_1036); +lean_ctor_set(x_2157, 2, x_2052); +lean_ctor_set(x_2157, 3, x_2053); +lean_ctor_set(x_2157, 4, x_2123); +lean_ctor_set(x_2157, 5, x_2135); +lean_ctor_set(x_2157, 6, x_2144); +lean_ctor_set(x_2157, 7, x_2156); +if (lean_is_scalar(x_2155)) { + x_2158 = lean_alloc_ctor(1, 1, 0); +} else { + x_2158 = x_2155; +} +lean_ctor_set(x_2158, 0, x_2157); +if (lean_is_scalar(x_2153)) { + x_2159 = lean_alloc_ctor(0, 2, 0); +} else { + x_2159 = x_2153; +} +lean_ctor_set(x_2159, 0, x_2158); +lean_ctor_set(x_2159, 1, x_2152); +x_11 = x_2159; +goto block_29; +} +} } } } else { -uint8_t x_27; -x_27 = lean_nat_dec_lt(x_17, x_14); -if (x_27 == 0) -{ -uint8_t x_28; -x_28 = lean_nat_dec_le(x_17, x_13); -lean_dec(x_17); -if (x_28 == 0) -{ -lean_dec(x_15); -lean_dec(x_7); -x_3 = x_9; -goto _start; +lean_object* x_2191; lean_object* x_2192; lean_object* x_2193; +x_2191 = lean_ctor_get(x_1037, 0); +lean_inc(x_2191); +if (lean_is_exclusive(x_1037)) { + lean_ctor_release(x_1037, 0); + x_2192 = x_1037; +} else { + lean_dec_ref(x_1037); + x_2192 = lean_box(0); +} +if (lean_is_scalar(x_2192)) { + x_2193 = lean_alloc_ctor(1, 1, 0); +} else { + x_2193 = x_2192; +} +lean_ctor_set(x_2193, 0, x_2191); +if (lean_obj_tag(x_1038) == 0) +{ +lean_object* x_2194; lean_object* x_2195; lean_object* x_2196; lean_object* x_2197; +x_2194 = lean_box(0); +x_2195 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_2196 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_2195, x_1039, x_4); +x_2197 = lean_ctor_get(x_2196, 0); +lean_inc(x_2197); +if (lean_obj_tag(x_2197) == 0) +{ +lean_object* x_2198; lean_object* x_2199; lean_object* x_2200; lean_object* x_2201; lean_object* x_2202; lean_object* x_2203; +lean_dec(x_2193); +lean_dec(x_2052); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_2198 = lean_ctor_get(x_2196, 1); +lean_inc(x_2198); +if (lean_is_exclusive(x_2196)) { + lean_ctor_release(x_2196, 0); + lean_ctor_release(x_2196, 1); + x_2199 = x_2196; +} else { + lean_dec_ref(x_2196); + x_2199 = lean_box(0); +} +x_2200 = lean_ctor_get(x_2197, 0); +lean_inc(x_2200); +if (lean_is_exclusive(x_2197)) { + lean_ctor_release(x_2197, 0); + x_2201 = x_2197; +} else { + lean_dec_ref(x_2197); + x_2201 = lean_box(0); +} +if (lean_is_scalar(x_2201)) { + x_2202 = lean_alloc_ctor(0, 1, 0); +} else { + x_2202 = x_2201; +} +lean_ctor_set(x_2202, 0, x_2200); +if (lean_is_scalar(x_2199)) { + x_2203 = lean_alloc_ctor(0, 2, 0); +} else { + x_2203 = x_2199; +} +lean_ctor_set(x_2203, 0, x_2202); +lean_ctor_set(x_2203, 1, x_2198); +x_11 = x_2203; +goto block_29; } else { -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = lean_ctor_get(x_15, 1); -lean_inc(x_30); -lean_dec(x_15); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -lean_dec(x_30); -x_32 = lean_nat_dec_lt(x_13, x_31); -lean_dec(x_31); -if (x_32 == 0) -{ -lean_dec(x_7); -x_3 = x_9; -goto _start; +lean_object* x_2204; lean_object* x_2205; lean_object* x_2206; lean_object* x_2207; lean_object* x_2208; lean_object* x_2209; +x_2204 = lean_ctor_get(x_2196, 1); +lean_inc(x_2204); +if (lean_is_exclusive(x_2196)) { + lean_ctor_release(x_2196, 0); + lean_ctor_release(x_2196, 1); + x_2205 = x_2196; +} else { + lean_dec_ref(x_2196); + x_2205 = lean_box(0); +} +x_2206 = lean_ctor_get(x_2197, 0); +lean_inc(x_2206); +if (lean_is_exclusive(x_2197)) { + lean_ctor_release(x_2197, 0); + x_2207 = x_2197; +} else { + lean_dec_ref(x_2197); + x_2207 = lean_box(0); +} +if (lean_obj_tag(x_1040) == 0) +{ +lean_dec(x_2205); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_2232; lean_object* x_2233; lean_object* x_2234; +x_2232 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2232, 0, x_1035); +lean_ctor_set(x_2232, 1, x_1036); +lean_ctor_set(x_2232, 2, x_2052); +lean_ctor_set(x_2232, 3, x_2193); +lean_ctor_set(x_2232, 4, x_2194); +lean_ctor_set(x_2232, 5, x_2206); +lean_ctor_set(x_2232, 6, x_2194); +lean_ctor_set(x_2232, 7, x_2194); +if (lean_is_scalar(x_2207)) { + x_2233 = lean_alloc_ctor(1, 1, 0); +} else { + x_2233 = x_2207; +} +lean_ctor_set(x_2233, 0, x_2232); +x_2234 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2234, 0, x_2233); +lean_ctor_set(x_2234, 1, x_2204); +x_11 = x_2234; +goto block_29; } else { -lean_object* x_34; -x_34 = lean_array_push(x_5, x_7); -x_3 = x_9; -x_5 = x_34; -goto _start; +lean_object* x_2235; lean_object* x_2236; lean_object* x_2237; size_t x_2238; size_t x_2239; lean_object* x_2240; lean_object* x_2241; lean_object* x_2242; lean_object* x_2243; lean_object* x_2244; lean_object* x_2245; lean_object* x_2246; lean_object* x_2247; lean_object* x_2248; lean_object* x_2249; +lean_dec(x_2207); +x_2235 = lean_ctor_get(x_1041, 0); +lean_inc(x_2235); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2236 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2236 = lean_box(0); +} +x_2237 = lean_array_get_size(x_2235); +x_2238 = lean_usize_of_nat(x_2237); +lean_dec(x_2237); +x_2239 = 0; +x_2240 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2238, x_2239, x_2235, x_2204); +x_2241 = lean_ctor_get(x_2240, 0); +lean_inc(x_2241); +x_2242 = lean_ctor_get(x_2240, 1); +lean_inc(x_2242); +if (lean_is_exclusive(x_2240)) { + lean_ctor_release(x_2240, 0); + lean_ctor_release(x_2240, 1); + x_2243 = x_2240; +} else { + lean_dec_ref(x_2240); + x_2243 = lean_box(0); +} +x_2244 = lean_ctor_get(x_2241, 0); +lean_inc(x_2244); +if (lean_is_exclusive(x_2241)) { + lean_ctor_release(x_2241, 0); + x_2245 = x_2241; +} else { + lean_dec_ref(x_2241); + x_2245 = lean_box(0); +} +if (lean_is_scalar(x_2236)) { + x_2246 = lean_alloc_ctor(1, 1, 0); +} else { + x_2246 = x_2236; +} +lean_ctor_set(x_2246, 0, x_2244); +x_2247 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2247, 0, x_1035); +lean_ctor_set(x_2247, 1, x_1036); +lean_ctor_set(x_2247, 2, x_2052); +lean_ctor_set(x_2247, 3, x_2193); +lean_ctor_set(x_2247, 4, x_2194); +lean_ctor_set(x_2247, 5, x_2206); +lean_ctor_set(x_2247, 6, x_2194); +lean_ctor_set(x_2247, 7, x_2246); +if (lean_is_scalar(x_2245)) { + x_2248 = lean_alloc_ctor(1, 1, 0); +} else { + x_2248 = x_2245; +} +lean_ctor_set(x_2248, 0, x_2247); +if (lean_is_scalar(x_2243)) { + x_2249 = lean_alloc_ctor(0, 2, 0); +} else { + x_2249 = x_2243; } +lean_ctor_set(x_2249, 0, x_2248); +lean_ctor_set(x_2249, 1, x_2242); +x_11 = x_2249; +goto block_29; } } else { -lean_object* x_36; -lean_dec(x_17); -lean_dec(x_15); -x_36 = lean_array_push(x_5, x_7); -x_3 = x_9; -x_5 = x_36; -goto _start; +lean_object* x_2250; lean_object* x_2251; lean_object* x_2252; size_t x_2253; size_t x_2254; lean_object* x_2255; lean_object* x_2256; lean_object* x_2257; lean_object* x_2258; lean_object* x_2259; lean_object* x_2260; lean_object* x_2261; +lean_dec(x_2207); +x_2250 = lean_ctor_get(x_1040, 0); +lean_inc(x_2250); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_2251 = x_1040; +} else { + lean_dec_ref(x_1040); + x_2251 = lean_box(0); +} +x_2252 = lean_array_get_size(x_2250); +x_2253 = lean_usize_of_nat(x_2252); +lean_dec(x_2252); +x_2254 = 0; +x_2255 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_2253, x_2254, x_2250, x_2204); +x_2256 = lean_ctor_get(x_2255, 0); +lean_inc(x_2256); +x_2257 = lean_ctor_get(x_2255, 1); +lean_inc(x_2257); +lean_dec(x_2255); +x_2258 = lean_ctor_get(x_2256, 0); +lean_inc(x_2258); +if (lean_is_exclusive(x_2256)) { + lean_ctor_release(x_2256, 0); + x_2259 = x_2256; +} else { + lean_dec_ref(x_2256); + x_2259 = lean_box(0); } +if (lean_is_scalar(x_2251)) { + x_2260 = lean_alloc_ctor(1, 1, 0); +} else { + x_2260 = x_2251; } +lean_ctor_set(x_2260, 0, x_2258); +if (lean_is_scalar(x_2259)) { + x_2261 = lean_alloc_ctor(1, 1, 0); +} else { + x_2261 = x_2259; } +lean_ctor_set(x_2261, 0, x_2260); +x_2208 = x_2261; +x_2209 = x_2257; +goto block_2231; } -else +block_2231: { -return x_5; +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_2210; lean_object* x_2211; lean_object* x_2212; lean_object* x_2213; lean_object* x_2214; +x_2210 = lean_ctor_get(x_2208, 0); +lean_inc(x_2210); +if (lean_is_exclusive(x_2208)) { + lean_ctor_release(x_2208, 0); + x_2211 = x_2208; +} else { + lean_dec_ref(x_2208); + x_2211 = lean_box(0); +} +x_2212 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2212, 0, x_1035); +lean_ctor_set(x_2212, 1, x_1036); +lean_ctor_set(x_2212, 2, x_2052); +lean_ctor_set(x_2212, 3, x_2193); +lean_ctor_set(x_2212, 4, x_2194); +lean_ctor_set(x_2212, 5, x_2206); +lean_ctor_set(x_2212, 6, x_2210); +lean_ctor_set(x_2212, 7, x_2194); +if (lean_is_scalar(x_2211)) { + x_2213 = lean_alloc_ctor(1, 1, 0); +} else { + x_2213 = x_2211; } +lean_ctor_set(x_2213, 0, x_2212); +if (lean_is_scalar(x_2205)) { + x_2214 = lean_alloc_ctor(0, 2, 0); +} else { + x_2214 = x_2205; } +lean_ctor_set(x_2214, 0, x_2213); +lean_ctor_set(x_2214, 1, x_2209); +x_11 = x_2214; +goto block_29; } -static lean_object* _init_l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__1() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(0u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; +lean_object* x_2215; lean_object* x_2216; lean_object* x_2217; lean_object* x_2218; size_t x_2219; size_t x_2220; lean_object* x_2221; lean_object* x_2222; lean_object* x_2223; lean_object* x_2224; lean_object* x_2225; lean_object* x_2226; lean_object* x_2227; lean_object* x_2228; lean_object* x_2229; lean_object* x_2230; +lean_dec(x_2205); +x_2215 = lean_ctor_get(x_2208, 0); +lean_inc(x_2215); +lean_dec(x_2208); +x_2216 = lean_ctor_get(x_1041, 0); +lean_inc(x_2216); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2217 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2217 = lean_box(0); +} +x_2218 = lean_array_get_size(x_2216); +x_2219 = lean_usize_of_nat(x_2218); +lean_dec(x_2218); +x_2220 = 0; +x_2221 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2219, x_2220, x_2216, x_2209); +x_2222 = lean_ctor_get(x_2221, 0); +lean_inc(x_2222); +x_2223 = lean_ctor_get(x_2221, 1); +lean_inc(x_2223); +if (lean_is_exclusive(x_2221)) { + lean_ctor_release(x_2221, 0); + lean_ctor_release(x_2221, 1); + x_2224 = x_2221; +} else { + lean_dec_ref(x_2221); + x_2224 = lean_box(0); +} +x_2225 = lean_ctor_get(x_2222, 0); +lean_inc(x_2225); +if (lean_is_exclusive(x_2222)) { + lean_ctor_release(x_2222, 0); + x_2226 = x_2222; +} else { + lean_dec_ref(x_2222); + x_2226 = lean_box(0); +} +if (lean_is_scalar(x_2217)) { + x_2227 = lean_alloc_ctor(1, 1, 0); +} else { + x_2227 = x_2217; +} +lean_ctor_set(x_2227, 0, x_2225); +x_2228 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2228, 0, x_1035); +lean_ctor_set(x_2228, 1, x_1036); +lean_ctor_set(x_2228, 2, x_2052); +lean_ctor_set(x_2228, 3, x_2193); +lean_ctor_set(x_2228, 4, x_2194); +lean_ctor_set(x_2228, 5, x_2206); +lean_ctor_set(x_2228, 6, x_2215); +lean_ctor_set(x_2228, 7, x_2227); +if (lean_is_scalar(x_2226)) { + x_2229 = lean_alloc_ctor(1, 1, 0); +} else { + x_2229 = x_2226; } +lean_ctor_set(x_2229, 0, x_2228); +if (lean_is_scalar(x_2224)) { + x_2230 = lean_alloc_ctor(0, 2, 0); +} else { + x_2230 = x_2224; +} +lean_ctor_set(x_2230, 0, x_2229); +lean_ctor_set(x_2230, 1, x_2223); +x_11 = x_2230; +goto block_29; } -static lean_object* _init_l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__1; -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; -x_3 = lean_ctor_get(x_2, 0); -lean_inc(x_3); -lean_dec(x_2); -x_4 = l_List_getLast_x3f___rarg(x_3); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; -x_5 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2; -return x_5; } else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_6 = lean_ctor_get(x_4, 0); -lean_inc(x_6); -lean_dec(x_4); -x_7 = lean_ctor_get(x_6, 4); -lean_inc(x_7); -lean_dec(x_6); -x_8 = l_Std_PersistentArray_toArray___rarg(x_7); -x_9 = lean_array_get_size(x_8); -x_10 = lean_unsigned_to_nat(0u); -x_11 = lean_nat_dec_lt(x_10, x_9); -if (x_11 == 0) -{ -lean_object* x_12; -lean_dec(x_9); -lean_dec(x_8); -x_12 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2; -return x_12; +lean_object* x_2262; lean_object* x_2263; lean_object* x_2264; lean_object* x_2265; lean_object* x_2266; lean_object* x_2267; +x_2262 = lean_ctor_get(x_1038, 0); +lean_inc(x_2262); +if (lean_is_exclusive(x_1038)) { + lean_ctor_release(x_1038, 0); + x_2263 = x_1038; +} else { + lean_dec_ref(x_1038); + x_2263 = lean_box(0); +} +if (lean_is_scalar(x_2263)) { + x_2264 = lean_alloc_ctor(1, 1, 0); +} else { + x_2264 = x_2263; +} +lean_ctor_set(x_2264, 0, x_2262); +x_2265 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3; +x_2266 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__14(x_2265, x_1039, x_4); +x_2267 = lean_ctor_get(x_2266, 0); +lean_inc(x_2267); +if (lean_obj_tag(x_2267) == 0) +{ +lean_object* x_2268; lean_object* x_2269; lean_object* x_2270; lean_object* x_2271; lean_object* x_2272; lean_object* x_2273; +lean_dec(x_2264); +lean_dec(x_2193); +lean_dec(x_2052); +lean_dec(x_1041); +lean_dec(x_1040); +lean_dec(x_1036); +lean_dec(x_1035); +x_2268 = lean_ctor_get(x_2266, 1); +lean_inc(x_2268); +if (lean_is_exclusive(x_2266)) { + lean_ctor_release(x_2266, 0); + lean_ctor_release(x_2266, 1); + x_2269 = x_2266; +} else { + lean_dec_ref(x_2266); + x_2269 = lean_box(0); +} +x_2270 = lean_ctor_get(x_2267, 0); +lean_inc(x_2270); +if (lean_is_exclusive(x_2267)) { + lean_ctor_release(x_2267, 0); + x_2271 = x_2267; +} else { + lean_dec_ref(x_2267); + x_2271 = lean_box(0); +} +if (lean_is_scalar(x_2271)) { + x_2272 = lean_alloc_ctor(0, 1, 0); +} else { + x_2272 = x_2271; +} +lean_ctor_set(x_2272, 0, x_2270); +if (lean_is_scalar(x_2269)) { + x_2273 = lean_alloc_ctor(0, 2, 0); +} else { + x_2273 = x_2269; +} +lean_ctor_set(x_2273, 0, x_2272); +lean_ctor_set(x_2273, 1, x_2268); +x_11 = x_2273; +goto block_29; } else { -uint8_t x_13; -x_13 = lean_nat_dec_le(x_9, x_9); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_9); -lean_dec(x_8); -x_14 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2; -return x_14; +lean_object* x_2274; lean_object* x_2275; lean_object* x_2276; lean_object* x_2277; lean_object* x_2278; lean_object* x_2279; +x_2274 = lean_ctor_get(x_2266, 1); +lean_inc(x_2274); +if (lean_is_exclusive(x_2266)) { + lean_ctor_release(x_2266, 0); + lean_ctor_release(x_2266, 1); + x_2275 = x_2266; +} else { + lean_dec_ref(x_2266); + x_2275 = lean_box(0); +} +x_2276 = lean_ctor_get(x_2267, 0); +lean_inc(x_2276); +if (lean_is_exclusive(x_2267)) { + lean_ctor_release(x_2267, 0); + x_2277 = x_2267; +} else { + lean_dec_ref(x_2267); + x_2277 = lean_box(0); +} +if (lean_obj_tag(x_1040) == 0) +{ +lean_object* x_2303; +lean_dec(x_2275); +x_2303 = lean_box(0); +if (lean_obj_tag(x_1041) == 0) +{ +lean_object* x_2304; lean_object* x_2305; lean_object* x_2306; +x_2304 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2304, 0, x_1035); +lean_ctor_set(x_2304, 1, x_1036); +lean_ctor_set(x_2304, 2, x_2052); +lean_ctor_set(x_2304, 3, x_2193); +lean_ctor_set(x_2304, 4, x_2264); +lean_ctor_set(x_2304, 5, x_2276); +lean_ctor_set(x_2304, 6, x_2303); +lean_ctor_set(x_2304, 7, x_2303); +if (lean_is_scalar(x_2277)) { + x_2305 = lean_alloc_ctor(1, 1, 0); +} else { + x_2305 = x_2277; +} +lean_ctor_set(x_2305, 0, x_2304); +x_2306 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2306, 0, x_2305); +lean_ctor_set(x_2306, 1, x_2274); +x_11 = x_2306; +goto block_29; } else { -size_t x_15; size_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_15 = 0; -x_16 = lean_usize_of_nat(x_9); -lean_dec(x_9); -x_17 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__1; -x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1(x_1, x_8, x_15, x_16, x_17); -lean_dec(x_8); -x_19 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +lean_object* x_2307; lean_object* x_2308; lean_object* x_2309; size_t x_2310; size_t x_2311; lean_object* x_2312; lean_object* x_2313; lean_object* x_2314; lean_object* x_2315; lean_object* x_2316; lean_object* x_2317; lean_object* x_2318; lean_object* x_2319; lean_object* x_2320; lean_object* x_2321; +lean_dec(x_2277); +x_2307 = lean_ctor_get(x_1041, 0); +lean_inc(x_2307); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2308 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2308 = lean_box(0); +} +x_2309 = lean_array_get_size(x_2307); +x_2310 = lean_usize_of_nat(x_2309); +lean_dec(x_2309); +x_2311 = 0; +x_2312 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2310, x_2311, x_2307, x_2274); +x_2313 = lean_ctor_get(x_2312, 0); +lean_inc(x_2313); +x_2314 = lean_ctor_get(x_2312, 1); +lean_inc(x_2314); +if (lean_is_exclusive(x_2312)) { + lean_ctor_release(x_2312, 0); + lean_ctor_release(x_2312, 1); + x_2315 = x_2312; +} else { + lean_dec_ref(x_2312); + x_2315 = lean_box(0); +} +x_2316 = lean_ctor_get(x_2313, 0); +lean_inc(x_2316); +if (lean_is_exclusive(x_2313)) { + lean_ctor_release(x_2313, 0); + x_2317 = x_2313; +} else { + lean_dec_ref(x_2313); + x_2317 = lean_box(0); } +if (lean_is_scalar(x_2308)) { + x_2318 = lean_alloc_ctor(1, 1, 0); +} else { + x_2318 = x_2308; +} +lean_ctor_set(x_2318, 0, x_2316); +x_2319 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2319, 0, x_1035); +lean_ctor_set(x_2319, 1, x_1036); +lean_ctor_set(x_2319, 2, x_2052); +lean_ctor_set(x_2319, 3, x_2193); +lean_ctor_set(x_2319, 4, x_2264); +lean_ctor_set(x_2319, 5, x_2276); +lean_ctor_set(x_2319, 6, x_2303); +lean_ctor_set(x_2319, 7, x_2318); +if (lean_is_scalar(x_2317)) { + x_2320 = lean_alloc_ctor(1, 1, 0); +} else { + x_2320 = x_2317; } +lean_ctor_set(x_2320, 0, x_2319); +if (lean_is_scalar(x_2315)) { + x_2321 = lean_alloc_ctor(0, 2, 0); +} else { + x_2321 = x_2315; } +lean_ctor_set(x_2321, 0, x_2320); +lean_ctor_set(x_2321, 1, x_2314); +x_11 = x_2321; +goto block_29; } } -LEAN_EXPORT uint8_t l_Lean_Widget_getInteractiveDiagnostics___lambda__2(lean_object* x_1) { -_start: +else { -uint8_t x_2; -x_2 = 1; -return x_2; +lean_object* x_2322; lean_object* x_2323; lean_object* x_2324; size_t x_2325; size_t x_2326; lean_object* x_2327; lean_object* x_2328; lean_object* x_2329; lean_object* x_2330; lean_object* x_2331; lean_object* x_2332; lean_object* x_2333; +lean_dec(x_2277); +x_2322 = lean_ctor_get(x_1040, 0); +lean_inc(x_2322); +if (lean_is_exclusive(x_1040)) { + lean_ctor_release(x_1040, 0); + x_2323 = x_1040; +} else { + lean_dec_ref(x_1040); + x_2323 = lean_box(0); +} +x_2324 = lean_array_get_size(x_2322); +x_2325 = lean_usize_of_nat(x_2324); +lean_dec(x_2324); +x_2326 = 0; +x_2327 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_2325, x_2326, x_2322, x_2274); +x_2328 = lean_ctor_get(x_2327, 0); +lean_inc(x_2328); +x_2329 = lean_ctor_get(x_2327, 1); +lean_inc(x_2329); +lean_dec(x_2327); +x_2330 = lean_ctor_get(x_2328, 0); +lean_inc(x_2330); +if (lean_is_exclusive(x_2328)) { + lean_ctor_release(x_2328, 0); + x_2331 = x_2328; +} else { + lean_dec_ref(x_2328); + x_2331 = lean_box(0); } +if (lean_is_scalar(x_2323)) { + x_2332 = lean_alloc_ctor(1, 1, 0); +} else { + x_2332 = x_2323; } -LEAN_EXPORT uint8_t l_Lean_Widget_getInteractiveDiagnostics___lambda__3(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; uint8_t x_4; -x_3 = lean_ctor_get(x_2, 0); -x_4 = lean_nat_dec_lt(x_3, x_1); -return x_4; +lean_ctor_set(x_2332, 0, x_2330); +if (lean_is_scalar(x_2331)) { + x_2333 = lean_alloc_ctor(1, 1, 0); +} else { + x_2333 = x_2331; } +lean_ctor_set(x_2333, 0, x_2332); +x_2278 = x_2333; +x_2279 = x_2329; +goto block_2302; } -static lean_object* _init_l_Lean_Widget_getInteractiveDiagnostics___closed__1() { -_start: +block_2302: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_getInteractiveDiagnostics___lambda__2___boxed), 1, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +if (lean_obj_tag(x_1041) == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_4 = l_Lean_Server_RequestM_readDoc(x_2, x_3); -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(x_4, 1); -lean_inc(x_6); -if (lean_is_exclusive(x_4)) { - lean_ctor_release(x_4, 0); - lean_ctor_release(x_4, 1); - x_7 = x_4; +lean_object* x_2280; lean_object* x_2281; lean_object* x_2282; lean_object* x_2283; lean_object* x_2284; lean_object* x_2285; +x_2280 = lean_ctor_get(x_2278, 0); +lean_inc(x_2280); +if (lean_is_exclusive(x_2278)) { + lean_ctor_release(x_2278, 0); + x_2281 = x_2278; } else { - lean_dec_ref(x_4); - x_7 = lean_box(0); + lean_dec_ref(x_2278); + x_2281 = lean_box(0); +} +x_2282 = lean_box(0); +x_2283 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2283, 0, x_1035); +lean_ctor_set(x_2283, 1, x_1036); +lean_ctor_set(x_2283, 2, x_2052); +lean_ctor_set(x_2283, 3, x_2193); +lean_ctor_set(x_2283, 4, x_2264); +lean_ctor_set(x_2283, 5, x_2276); +lean_ctor_set(x_2283, 6, x_2280); +lean_ctor_set(x_2283, 7, x_2282); +if (lean_is_scalar(x_2281)) { + x_2284 = lean_alloc_ctor(1, 1, 0); +} else { + x_2284 = x_2281; } -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_15 = lean_ctor_get(x_5, 1); -lean_inc(x_15); -lean_dec(x_5); -x_16 = l_Lean_Widget_getInteractiveDiagnostics___closed__1; -x_17 = l_IO_AsyncList_waitAll___rarg(x_16, x_15, x_6); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_8 = x_18; -x_9 = x_19; -goto block_14; +lean_ctor_set(x_2284, 0, x_2283); +if (lean_is_scalar(x_2275)) { + x_2285 = lean_alloc_ctor(0, 2, 0); +} else { + x_2285 = x_2275; +} +lean_ctor_set(x_2285, 0, x_2284); +lean_ctor_set(x_2285, 1, x_2279); +x_11 = x_2285; +goto block_29; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_20 = lean_ctor_get(x_5, 1); -lean_inc(x_20); -x_21 = lean_ctor_get(x_1, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_5, 0); -lean_inc(x_22); -lean_dec(x_5); -x_23 = lean_ctor_get(x_22, 2); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -x_25 = lean_unsigned_to_nat(0u); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -x_27 = l_Lean_FileMap_lspPosToUtf8Pos(x_23, x_26); -lean_dec(x_23); -x_28 = lean_alloc_closure((void*)(l_Lean_Widget_getInteractiveDiagnostics___lambda__3___boxed), 2, 1); -lean_closure_set(x_28, 0, x_27); -x_29 = l_IO_AsyncList_waitAll___rarg(x_28, x_20, x_6); -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_8 = x_30; -x_9 = x_31; -goto block_14; +lean_object* x_2286; lean_object* x_2287; lean_object* x_2288; lean_object* x_2289; size_t x_2290; size_t x_2291; lean_object* x_2292; lean_object* x_2293; lean_object* x_2294; lean_object* x_2295; lean_object* x_2296; lean_object* x_2297; lean_object* x_2298; lean_object* x_2299; lean_object* x_2300; lean_object* x_2301; +lean_dec(x_2275); +x_2286 = lean_ctor_get(x_2278, 0); +lean_inc(x_2286); +lean_dec(x_2278); +x_2287 = lean_ctor_get(x_1041, 0); +lean_inc(x_2287); +if (lean_is_exclusive(x_1041)) { + lean_ctor_release(x_1041, 0); + x_2288 = x_1041; +} else { + lean_dec_ref(x_1041); + x_2288 = lean_box(0); +} +x_2289 = lean_array_get_size(x_2287); +x_2290 = lean_usize_of_nat(x_2289); +lean_dec(x_2289); +x_2291 = 0; +x_2292 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_2290, x_2291, x_2287, x_2279); +x_2293 = lean_ctor_get(x_2292, 0); +lean_inc(x_2293); +x_2294 = lean_ctor_get(x_2292, 1); +lean_inc(x_2294); +if (lean_is_exclusive(x_2292)) { + lean_ctor_release(x_2292, 0); + lean_ctor_release(x_2292, 1); + x_2295 = x_2292; +} else { + lean_dec_ref(x_2292); + x_2295 = lean_box(0); +} +x_2296 = lean_ctor_get(x_2293, 0); +lean_inc(x_2296); +if (lean_is_exclusive(x_2293)) { + lean_ctor_release(x_2293, 0); + x_2297 = x_2293; +} else { + lean_dec_ref(x_2293); + x_2297 = lean_box(0); } -block_14: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_getInteractiveDiagnostics___lambda__1___boxed), 2, 1); -lean_closure_set(x_10, 0, x_1); -x_11 = l_Task_Priority_default; -x_12 = lean_task_map(x_10, x_8, x_11); -if (lean_is_scalar(x_7)) { - x_13 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_2288)) { + x_2298 = lean_alloc_ctor(1, 1, 0); } else { - x_13 = x_7; + x_2298 = x_2288; +} +lean_ctor_set(x_2298, 0, x_2296); +x_2299 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_2299, 0, x_1035); +lean_ctor_set(x_2299, 1, x_1036); +lean_ctor_set(x_2299, 2, x_2052); +lean_ctor_set(x_2299, 3, x_2193); +lean_ctor_set(x_2299, 4, x_2264); +lean_ctor_set(x_2299, 5, x_2276); +lean_ctor_set(x_2299, 6, x_2286); +lean_ctor_set(x_2299, 7, x_2298); +if (lean_is_scalar(x_2297)) { + x_2300 = lean_alloc_ctor(1, 1, 0); +} else { + x_2300 = x_2297; } -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_9); -return x_13; +lean_ctor_set(x_2300, 0, x_2299); +if (lean_is_scalar(x_2295)) { + x_2301 = lean_alloc_ctor(0, 2, 0); +} else { + x_2301 = x_2295; } +lean_ctor_set(x_2301, 0, x_2300); +lean_ctor_set(x_2301, 1, x_2294); +x_11 = x_2301; +goto block_29; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_8 = l_Array_foldlMUnsafe_fold___at_Lean_Widget_getInteractiveDiagnostics___spec__1(x_1, x_2, x_6, x_7, x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Lean_Widget_getInteractiveDiagnostics___lambda__1(x_1, x_2); -lean_dec(x_1); -return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__2___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Widget_getInteractiveDiagnostics___lambda__2(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; } +block_29: +{ +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_10); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = !lean_is_exclusive(x_12); +if (x_15 == 0) +{ +return x_11; } -LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___lambda__3___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Widget_getInteractiveDiagnostics___lambda__3(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_12, 0); +lean_inc(x_16); +lean_dec(x_12); +x_17 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_11, 0, x_17); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Widget_getInteractiveDiagnostics___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = l_Lean_Widget_getInteractiveDiagnostics(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_ctor_get(x_11, 1); +lean_inc(x_18); +lean_dec(x_11); +x_19 = lean_ctor_get(x_12, 0); +lean_inc(x_19); +if (lean_is_exclusive(x_12)) { + lean_ctor_release(x_12, 0); + x_20 = x_12; +} else { + lean_dec_ref(x_12); + x_20 = lean_box(0); } +if (lean_is_scalar(x_20)) { + x_21 = lean_alloc_ctor(0, 1, 0); +} else { + x_21 = x_20; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__13; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8; -x_4 = l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg(x_1, lean_box(0), x_1, lean_box(0), x_1, lean_box(0), x_1, lean_box(0), x_2, lean_box(0), x_3, lean_box(0), x_3); -return x_4; +lean_ctor_set(x_21, 0, x_19); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_18); +return x_22; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__1; -x_2 = l_Lean_Server_instRpcEncodingArray___rarg(x_1); -return x_2; +lean_object* x_23; lean_object* x_24; size_t x_25; size_t x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_11, 1); +lean_inc(x_23); +lean_dec(x_11); +x_24 = lean_ctor_get(x_12, 0); +lean_inc(x_24); +lean_dec(x_12); +x_25 = 1; +x_26 = lean_usize_add(x_2, x_25); +x_27 = lean_array_uset(x_10, x_2, x_24); +x_2 = x_26; +x_3 = x_27; +x_4 = x_23; +goto _start; +} } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Lsp_instToJsonDiagnosticTag___boxed), 1, 0); -return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__4() { +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__3; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_6; lean_object* x_7; +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_2); +x_29 = lean_ctor_get(x_3, 0); +lean_inc(x_29); +lean_dec(x_3); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_5); +return x_30; } +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_39; +x_31 = lean_ctor_get(x_3, 0); +lean_inc(x_31); +lean_dec(x_3); +x_32 = lean_st_ref_take(x_1, x_5); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = lean_array_get_size(x_31); +x_36 = lean_usize_of_nat(x_35); +lean_dec(x_35); +x_37 = 0; +lean_inc(x_33); +x_38 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__9(x_36, x_37, x_31, x_33); +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +if (lean_obj_tag(x_39) == 0) +{ +uint8_t x_40; +lean_dec(x_38); +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +x_41 = lean_st_ref_set(x_1, x_33, x_34); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_6 = x_39; +x_7 = x_42; +goto block_28; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__5() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Lsp_instToJsonDiagnosticRelatedInformation; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_43 = lean_ctor_get(x_39, 0); +lean_inc(x_43); +lean_dec(x_39); +x_44 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_44, 0, x_43); +x_45 = lean_st_ref_set(x_1, x_33, x_34); +x_46 = lean_ctor_get(x_45, 1); +lean_inc(x_46); +lean_dec(x_45); +x_6 = x_44; +x_7 = x_46; +goto block_28; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__6() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Lsp_instToJsonDiagnosticSeverity___boxed), 1, 0); -return x_1; -} +lean_object* x_47; uint8_t x_48; +lean_dec(x_33); +x_47 = lean_ctor_get(x_38, 1); +lean_inc(x_47); +lean_dec(x_38); +x_48 = !lean_is_exclusive(x_39); +if (x_48 == 0) +{ +lean_object* x_49; lean_object* x_50; +x_49 = lean_st_ref_set(x_1, x_47, x_34); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +lean_dec(x_49); +x_6 = x_39; +x_7 = x_50; +goto block_28; } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__7() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Lsp_instToJsonDiagnosticCode___boxed), 1, 0); -return x_1; +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_51 = lean_ctor_get(x_39, 0); +lean_inc(x_51); +lean_dec(x_39); +x_52 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_52, 0, x_51); +x_53 = lean_st_ref_set(x_1, x_47, x_34); +x_54 = lean_ctor_get(x_53, 1); +lean_inc(x_54); +lean_dec(x_53); +x_6 = x_52; +x_7 = x_54; +goto block_28; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__8() { -_start: +} +block_28: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l_Lean_Lsp_instToJsonRange; -x_2 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__6; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__7; -x_4 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23; -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__28; -x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__4; -x_7 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__5; -x_8 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1642____rarg), 8, 7); -lean_closure_set(x_8, 0, x_1); -lean_closure_set(x_8, 1, x_2); -lean_closure_set(x_8, 2, x_3); -lean_closure_set(x_8, 3, x_4); -lean_closure_set(x_8, 4, x_5); -lean_closure_set(x_8, 5, x_6); -lean_closure_set(x_8, 6, x_7); -return x_8; +if (lean_obj_tag(x_6) == 0) +{ +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; uint8_t x_18; lean_object* x_19; lean_object* x_20; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +x_9 = 1; +x_10 = l_Lean_Name_toString(x_2, x_9); +x_11 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_string_append(x_14, x_8); +lean_dec(x_8); +x_16 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_17 = lean_string_append(x_15, x_16); +x_18 = 3; +x_19 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set_uint8(x_19, sizeof(void*)*1, x_18); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_7); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +lean_dec(x_2); +x_21 = lean_ctor_get(x_6, 0); +lean_inc(x_21); +lean_dec(x_6); +x_22 = lean_array_get_size(x_21); +x_23 = lean_usize_of_nat(x_22); +lean_dec(x_22); +x_24 = 0; +x_25 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__4(x_23, x_24, x_21); +x_26 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_7); +return x_27; +} } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__9() { +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__2(lean_object* x_1, lean_object* x_2, uint64_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__8; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +x_8 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_7, x_3); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2; +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_11 = lean_ctor_get(x_8, 0); +lean_inc(x_11); +lean_dec(x_8); +x_12 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__5(x_4); +x_13 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__6___boxed), 3, 1); +lean_closure_set(x_13, 0, x_12); +lean_inc(x_11); +x_14 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____spec__2___lambda__1___boxed), 4, 1); +lean_closure_set(x_14, 0, x_11); +x_15 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 2); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_14); +lean_inc(x_5); +x_16 = l_Lean_Server_RequestM_asTask___rarg(x_15, x_5, x_6); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__2), 4, 1); +lean_closure_set(x_19, 0, x_1); +lean_inc(x_5); +x_20 = l_Lean_Server_RequestM_bindTask___rarg(x_17, x_19, x_5, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__1___boxed), 5, 2); +lean_closure_set(x_23, 0, x_11); +lean_closure_set(x_23, 1, x_2); +x_24 = l_Lean_Server_RequestM_mapTask___rarg(x_21, x_23, x_5, x_22); +return x_24; +} } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_4 = l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams; -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__2; -x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__9; -x_7 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___boxed), 14, 10); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, lean_box(0)); -lean_closure_set(x_7, 2, lean_box(0)); -lean_closure_set(x_7, 3, lean_box(0)); -lean_closure_set(x_7, 4, x_3); -lean_closure_set(x_7, 5, x_4); -lean_closure_set(x_7, 6, lean_box(0)); -lean_closure_set(x_7, 7, x_5); -lean_closure_set(x_7, 8, x_6); -lean_closure_set(x_7, 9, x_2); -return x_7; +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__2___boxed), 6, 2); +lean_closure_set(x_3, 0, x_2); +lean_closure_set(x_3, 1, x_1); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_inc(x_1); -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2(x_1, x_2); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; +x_5 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__2___boxed), 6, 2); +lean_closure_set(x_5, 0, x_2); +lean_closure_set(x_5, 1, x_1); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); @@ -4447,12 +26639,12 @@ return x_15; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_dec(x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; x_7 = lean_st_ref_get(x_6, x_5); x_8 = !lean_is_exclusive(x_7); if (x_8 == 0) @@ -4468,7 +26660,7 @@ lean_object* x_12; lean_object* x_13; lean_free_object(x_7); lean_dec(x_3); x_12 = lean_box(0); -x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__1(x_1, x_2, x_12, x_10); +x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(x_1, x_2, x_12, x_10); return x_13; } else @@ -4476,10 +26668,10 @@ else lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_dec(x_2); lean_dec(x_1); -x_14 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; +x_14 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; x_15 = lean_string_append(x_14, x_3); lean_dec(x_3); -x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; +x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; x_17 = lean_string_append(x_15, x_16); x_18 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_18, 0, x_17); @@ -4503,7 +26695,7 @@ if (x_21 == 0) lean_object* x_22; lean_object* x_23; lean_dec(x_3); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__1(x_1, x_2, x_22, x_20); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(x_1, x_2, x_22, x_20); return x_23; } else @@ -4511,10 +26703,10 @@ else lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_dec(x_2); lean_dec(x_1); -x_24 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; +x_24 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; x_25 = lean_string_append(x_24, x_3); lean_dec(x_3); -x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; +x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; x_27 = lean_string_append(x_25, x_26); x_28 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_28, 0, x_27); @@ -4526,17 +26718,17 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; x_4 = 1; lean_inc(x_1); x_5 = l_Lean_Name_toString(x_1, x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1; +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2; +x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_io_initializing(x_3); x_11 = lean_ctor_get(x_10, 0); @@ -4554,10 +26746,10 @@ if (x_13 == 0) lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_14 = lean_ctor_get(x_10, 0); lean_dec(x_14); -x_15 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; +x_15 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; x_16 = lean_string_append(x_15, x_9); lean_dec(x_9); -x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; +x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -4571,10 +26763,10 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean x_20 = lean_ctor_get(x_10, 1); lean_inc(x_20); lean_dec(x_10); -x_21 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; +x_21 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; x_22 = lean_string_append(x_21, x_9); lean_dec(x_9); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; x_24 = lean_string_append(x_22, x_23); x_25 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_25, 0, x_24); @@ -4591,12 +26783,12 @@ x_27 = lean_ctor_get(x_10, 1); lean_inc(x_27); lean_dec(x_10); x_28 = lean_box(0); -x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); +x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__2(x_1, x_2, x_9, x_28, x_27); return x_29; } } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__1() { +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1() { _start: { lean_object* x_1; @@ -4604,17 +26796,17 @@ x_1 = lean_mk_string_from_bytes("getInteractiveDiagnostics", 25); return x_1; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__2() { +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__1; +x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__3() { +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3() { _start: { lean_object* x_1; @@ -4622,26 +26814,113 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Widget_getInteractiveDiagnostics___boxed return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__2; -x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__3; -x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1(x_2, x_3, x_1); +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2; +x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3; +x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__4(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__6(x_1, x_2, x_3); +lean_dec(x_2); +lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__7(x_5, x_6, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__8(x_5, x_6, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__9(x_5, x_6, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint64_t x_7; lean_object* x_8; +x_7 = lean_unbox_uint64(x_3); +lean_dec(x_3); +x_8 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__1___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__1___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +x_4 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49_(x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__1() { _start: { lean_object* x_1; @@ -4649,7 +26928,7 @@ x_1 = lean_mk_string_from_bytes("kind", 4); return x_1; } } -static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__2() { +static lean_object* _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__2() { _start: { lean_object* x_1; @@ -4657,190 +26936,300 @@ x_1 = lean_mk_string_from_bytes("info", 4); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335_(lean_object* x_1) { _start: { -lean_object* x_4; lean_object* x_5; -x_4 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__1; -x_5 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_1, x_4); -if (lean_obj_tag(x_5) == 0) +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____spec__1(x_1, x_2); +if (lean_obj_tag(x_3) == 0) { -uint8_t x_6; -lean_dec(x_2); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) { -return x_5; +return x_3; } else { -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -lean_dec(x_5); -x_10 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__2; -x_11 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_2, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +x_8 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__2; +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1(x_1, x_8); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_12; +uint8_t x_10; +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); lean_dec(x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; +} +} +else { -return x_11; +uint8_t x_13; +x_13 = !lean_is_exclusive(x_9); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_9, 0); +x_15 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_15, 0, x_14); +x_16 = lean_unbox(x_7); +lean_dec(x_7); +lean_ctor_set_uint8(x_15, sizeof(void*)*1, x_16); +lean_ctor_set(x_9, 0, x_15); +return x_9; } else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_alloc_ctor(0, 1, 0); +lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_9, 0); +lean_inc(x_17); +lean_dec(x_9); +x_18 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_18, 0, x_17); +x_19 = lean_unbox(x_7); +lean_dec(x_7); +lean_ctor_set_uint8(x_18, sizeof(void*)*1, x_19); +x_20 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_20, 0, x_18); +return x_20; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335_(x_1); +lean_dec(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__9___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__9() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket__9___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1390_(lean_object* x_1) { +_start: +{ +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; size_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_2 = lean_ctor_get_uint8(x_1, sizeof(void*)*1); +x_3 = l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24_(x_2); +x_4 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__1; +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_box(0); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_6); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_unbox_usize(x_8); +lean_dec(x_8); +x_10 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1065_(x_9); +x_11 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__2; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_6); +x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_13); -return x_14; +lean_ctor_set(x_14, 1, x_6); +x_15 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_15, 0, x_7); +lean_ctor_set(x_15, 1, x_14); +x_16 = l_List_join___rarg(x_15); +x_17 = l_Lean_Json_mkObj(x_16); +return x_17; } } -else +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__9___closed__1() { +_start: { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_11); -if (x_15 == 0) +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1390_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__9() { +_start: { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_11, 0); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_9); -lean_ctor_set(x_17, 1, x_16); -lean_ctor_set(x_11, 0, x_17); -return x_11; +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket__9___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_11, 0); -lean_inc(x_18); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); lean_dec(x_11); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_9); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_20, 0, x_19); -return x_20; +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__1(lean_object* x_1) { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___boxed), 3, 0); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__1___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_4; -x_4 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__9___rarg(lean_object* x_1, lean_object* x_2) { -_start: +if (lean_obj_tag(x_5) == 0) { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___boxed), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__9(lean_object* x_1, lean_object* x_2) { -_start: +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__9___rarg), 2, 0); -return x_3; -} +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1744____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); -x_5 = lean_apply_1(x_1, x_4); -x_6 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__1; -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_9, 0, x_7); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_ctor_get(x_3, 1); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); lean_inc(x_10); -lean_dec(x_3); -x_11 = lean_apply_1(x_2, x_10); -x_12 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__2; -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_8); -x_15 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_8); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_9); -lean_ctor_set(x_16, 1, x_15); -x_17 = l_List_join___rarg(x_16); -x_18 = l_Lean_Json_mkObj(x_17); -return x_18; +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1744_(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1744____rarg), 3, 0); -return x_3; -} +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__9___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1744____rarg), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__9(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__2(lean_object* x_1) { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__9___rarg), 2, 0); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__2___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -4890,15 +27279,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__1___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__3___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -4948,198 +27337,238 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__4(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__2___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__4___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__1(uint8_t x_1, lean_object* x_2, size_t x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_2); -lean_ctor_set(x_6, 1, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); +x_4 = lean_box_usize(x_3); +x_5 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set_uint8(x_5, sizeof(void*)*1, x_1); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_2, lean_box(0), x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_ctor_get(x_1, 0); +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_7 = lean_ctor_get(x_6, 0); lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_2, 0); +x_8 = lean_ctor_get(x_1, 0); lean_inc(x_8); -lean_dec(x_2); -lean_inc(x_3); -x_9 = lean_apply_4(x_7, lean_box(0), x_3, x_4, x_8); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__1), 3, 2); -lean_closure_set(x_10, 0, x_3); -lean_closure_set(x_10, 1, x_6); -x_11 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_9, x_10); -return x_11; +lean_dec(x_1); +lean_inc(x_2); +x_9 = lean_apply_4(x_7, lean_box(0), x_2, x_3, x_8); +x_10 = lean_box(x_5); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__1___boxed), 3, 2); +lean_closure_set(x_11, 0, x_10); +lean_closure_set(x_11, 1, x_4); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__1___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_9, x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_4, 1); +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; +x_5 = lean_ctor_get_uint8(x_4, sizeof(void*)*1); +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get_uint8(x_6, sizeof(void*)*1); -x_10 = lean_box(x_9); -lean_inc(x_5); -lean_inc(x_4); -x_11 = lean_apply_4(x_8, lean_box(0), x_4, x_5, x_10); +lean_dec(x_6); +x_8 = lean_box(x_5); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); lean_inc(x_7); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__2), 6, 5); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_6); -lean_closure_set(x_12, 2, x_4); -lean_closure_set(x_12, 3, x_5); -lean_closure_set(x_12, 4, x_7); -x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_11, x_12); -return x_13; +x_10 = lean_apply_2(x_7, lean_box(0), x_9); +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__2___boxed), 5, 4); +lean_closure_set(x_11, 0, x_4); +lean_closure_set(x_11, 1, x_2); +lean_closure_set(x_11, 2, x_3); +lean_closure_set(x_11, 3, x_7); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__2___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__4(uint8_t x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__4(uint8_t x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_4, 0, x_3); lean_ctor_set_uint8(x_4, sizeof(void*)*1, x_1); -x_5 = lean_ctor_get(x_2, 0); -lean_inc(x_5); -lean_dec(x_2); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_7, 0, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +x_6 = lean_apply_2(x_2, lean_box(0), x_5); +return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -lean_dec(x_1); -x_7 = lean_ctor_get(x_2, 1); +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); -lean_dec(x_2); -lean_inc(x_3); -x_8 = lean_apply_4(x_6, lean_box(0), x_3, x_4, x_7); -x_9 = lean_box(x_5); -lean_inc(x_3); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__4___boxed), 3, 2); -lean_closure_set(x_10, 0, x_9); -lean_closure_set(x_10, 1, x_3); -x_11 = lean_ctor_get(x_3, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_12, 0, x_3); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); -return x_13; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +lean_inc(x_2); +x_9 = lean_apply_4(x_7, lean_box(0), x_2, x_3, x_8); +x_10 = lean_box(x_5); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__4___boxed), 3, 2); +lean_closure_set(x_11, 0, x_10); +lean_closure_set(x_11, 1, x_4); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__3___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_9, x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_1, 1); +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; +x_5 = lean_ctor_get_uint8(x_4, sizeof(void*)*1); +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_inc(x_5); -lean_inc(x_4); -x_9 = lean_apply_4(x_7, lean_box(0), x_4, x_5, x_8); -lean_inc(x_4); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__5___boxed), 5, 4); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_6); -lean_closure_set(x_10, 2, x_4); -lean_closure_set(x_10, 3, x_5); -x_11 = lean_ctor_get(x_4, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_12, 0, x_4); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); -return x_13; +lean_dec(x_6); +x_8 = lean_box(x_5); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +lean_inc(x_7); +x_10 = lean_apply_2(x_7, lean_box(0), x_9); +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__5___boxed), 5, 4); +lean_closure_set(x_11, 0, x_4); +lean_closure_set(x_11, 1, x_2); +lean_closure_set(x_11, 2, x_3); +lean_closure_set(x_11, 3, x_7); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingGetGoToLocationParams___spec__4___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__1() { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -lean_inc(x_3); -lean_inc(x_1); -x_4 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__3), 6, 2); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_3); -x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__6), 6, 2); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_3); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_4); -lean_ctor_set(x_6, 1, x_5); +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__3), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__6), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingGetGoToLocationParams() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__3; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_6 = l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__1(x_4, x_2, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg), 3, 0); -return x_2; +uint8_t x_6; lean_object* x_7; +x_6 = lean_unbox(x_5); +lean_dec(x_5); +x_7 = l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__2(x_1, x_2, x_3, x_4, x_6); +return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; x_4 = lean_unbox(x_1); lean_dec(x_1); -x_5 = l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__4(x_4, x_2, x_3); +x_5 = l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__4(x_4, x_2, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { uint8_t x_6; lean_object* x_7; x_6 = lean_unbox(x_5); lean_dec(x_5); -x_7 = l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg___lambda__5(x_1, x_2, x_3, x_4, x_6); +x_7 = l_Lean_Widget_instRpcEncodingGetGoToLocationParams___lambda__5(x_1, x_2, x_3, x_4, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_ReaderT_read___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_ReaderT_read___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; @@ -5149,67 +27578,445 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__4(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3; -x_2 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; -x_3 = l_Lean_Widget_instRpcEncodingGetGoToLocationParamsRpcEncodingPacket___rarg(x_1, lean_box(0), x_2); -return x_3; +lean_object* x_2; +x_2 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335_(x_1); +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; +x_4 = lean_ctor_get(x_2, 0); +x_5 = l_Lean_Json_compress(x_1); +x_6 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +x_7 = lean_string_append(x_6, x_5); +lean_dec(x_5); +x_8 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; +x_9 = lean_string_append(x_7, x_8); +x_10 = lean_string_append(x_9, x_4); +lean_dec(x_4); +x_11 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_12 = lean_string_append(x_10, x_11); +x_13 = 0; +x_14 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set_uint8(x_14, sizeof(void*)*1, x_13); +lean_ctor_set(x_2, 0, x_14); +return x_2; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = l_Lean_Json_compress(x_1); +x_17 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1; +x_18 = lean_string_append(x_17, x_16); +lean_dec(x_16); +x_19 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2; +x_20 = lean_string_append(x_18, x_19); +x_21 = lean_string_append(x_20, x_15); +lean_dec(x_15); +x_22 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_23 = lean_string_append(x_21, x_22); +x_24 = 0; +x_25 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set_uint8(x_25, sizeof(void*)*1, x_24); +x_26 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_26, 0, x_25); +return x_26; +} +} +else +{ +uint8_t x_27; +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_2); +if (x_27 == 0) +{ +return x_2; +} +else +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_2, 0); +lean_inc(x_28); +lean_dec(x_2); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +return x_29; +} } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__2() { +} +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Server_instFromJsonGoToKind; -x_2 = l_Lean_Lsp_instFromJsonRpcRef; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___boxed), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__3() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__6(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Lsp_instToJsonLocationLink; -x_2 = lean_alloc_closure((void*)(l_Lean_instToJsonArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_2, x_1); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_4); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_8 = lean_array_uget(x_3, x_2); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_array_uset(x_3, x_2, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_2, x_11); +x_13 = lean_array_uset(x_10, x_2, x_8); +x_2 = x_12; +x_3 = x_13; +goto _start; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3(lean_object* x_1, lean_object* x_2) { +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__1; -x_4 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__2; -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8; -x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__3; -x_7 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___boxed), 14, 10); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, lean_box(0)); -lean_closure_set(x_7, 2, lean_box(0)); -lean_closure_set(x_7, 3, lean_box(0)); -lean_closure_set(x_7, 4, x_3); -lean_closure_set(x_7, 5, x_4); -lean_closure_set(x_7, 6, lean_box(0)); -lean_closure_set(x_7, 7, x_5); -lean_closure_set(x_7, 8, x_6); -lean_closure_set(x_7, 9, x_2); +lean_object* x_7; uint8_t x_8; +x_7 = lean_st_ref_get(x_1, x_6); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; 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; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get_uint8(x_4, sizeof(void*)*1); +x_11 = lean_ctor_get(x_4, 0); +lean_inc(x_11); +lean_dec(x_4); +x_12 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +x_14 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_15 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_16 = lean_apply_5(x_13, lean_box(0), x_14, x_15, x_11, x_9); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +lean_dec(x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +lean_dec(x_17); +x_19 = 1; +x_20 = l_Lean_Name_toString(x_2, x_19); +x_21 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1; +x_22 = lean_string_append(x_21, x_20); +lean_dec(x_20); +x_23 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2; +x_24 = lean_string_append(x_22, x_23); +x_25 = l_Lean_Json_compress(x_3); +x_26 = lean_string_append(x_24, x_25); +lean_dec(x_25); +x_27 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3; +x_28 = lean_string_append(x_26, x_27); +x_29 = lean_string_append(x_28, x_18); +lean_dec(x_18); +x_30 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_31 = lean_string_append(x_29, x_30); +x_32 = 3; +x_33 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); +lean_ctor_set_tag(x_7, 1); +lean_ctor_set(x_7, 0, x_33); +return x_7; +} +else +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_3); +lean_dec(x_2); +x_34 = lean_ctor_get(x_17, 0); +lean_inc(x_34); +lean_dec(x_17); +x_35 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set_uint8(x_35, sizeof(void*)*1, x_10); +lean_ctor_set(x_7, 0, x_35); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +else +{ +lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_36 = lean_ctor_get(x_7, 0); +x_37 = lean_ctor_get(x_7, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_7); +x_38 = lean_ctor_get_uint8(x_4, sizeof(void*)*1); +x_39 = lean_ctor_get(x_4, 0); +lean_inc(x_39); +lean_dec(x_4); +x_40 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +x_42 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1; +x_43 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3; +x_44 = lean_apply_5(x_41, lean_box(0), x_42, x_43, x_39, x_36); +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +lean_dec(x_44); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; uint8_t 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; uint8_t x_60; lean_object* x_61; lean_object* x_62; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +lean_dec(x_45); +x_47 = 1; +x_48 = l_Lean_Name_toString(x_2, x_47); +x_49 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1; +x_50 = lean_string_append(x_49, x_48); +lean_dec(x_48); +x_51 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2; +x_52 = lean_string_append(x_50, x_51); +x_53 = l_Lean_Json_compress(x_3); +x_54 = lean_string_append(x_52, x_53); +lean_dec(x_53); +x_55 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3; +x_56 = lean_string_append(x_54, x_55); +x_57 = lean_string_append(x_56, x_46); +lean_dec(x_46); +x_58 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; +x_59 = lean_string_append(x_57, x_58); +x_60 = 3; +x_61 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set_uint8(x_61, sizeof(void*)*1, x_60); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_37); +return x_62; +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_3); +lean_dec(x_2); +x_63 = lean_ctor_get(x_45, 0); +lean_inc(x_63); +lean_dec(x_45); +x_64 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set_uint8(x_64, sizeof(void*)*1, x_38); +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_37); +return x_65; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_3, 0); +lean_inc(x_16); +lean_dec(x_3); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_5); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; size_t x_23; size_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_18 = lean_ctor_get(x_3, 0); +lean_inc(x_18); +lean_dec(x_3); +x_19 = lean_st_ref_take(x_1, x_5); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_array_get_size(x_18); +x_23 = lean_usize_of_nat(x_22); +lean_dec(x_22); +x_24 = 0; +x_25 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__6(x_23, x_24, x_18, x_20); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = !lean_is_exclusive(x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_st_ref_set(x_1, x_27, x_21); +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +x_6 = x_26; +x_7 = x_30; +goto block_15; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_26, 0); +lean_inc(x_31); +lean_dec(x_26); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +x_33 = lean_st_ref_set(x_1, x_27, x_21); +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_6 = x_32; +x_7 = x_34; +goto block_15; +} +} +block_15: +{ +lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +x_9 = lean_array_get_size(x_8); +x_10 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_11 = 0; +x_12 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_9629____spec__13(x_10, x_11, x_8); +x_13 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_7); +return x_14; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__3(lean_object* x_1, lean_object* x_2, uint64_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +x_8 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_7, x_3); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_9 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2; +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_6); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_11 = lean_ctor_get(x_8, 0); +lean_inc(x_11); +lean_dec(x_8); +lean_inc(x_4); +x_12 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__4(x_4); +x_13 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__5___boxed), 3, 1); +lean_closure_set(x_13, 0, x_12); +lean_inc(x_1); +lean_inc(x_11); +x_14 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__1___boxed), 6, 3); +lean_closure_set(x_14, 0, x_11); +lean_closure_set(x_14, 1, x_1); +lean_closure_set(x_14, 2, x_4); +x_15 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 2); +lean_closure_set(x_15, 0, x_13); +lean_closure_set(x_15, 1, x_14); +lean_inc(x_5); +x_16 = l_Lean_Server_RequestM_asTask___rarg(x_15, x_5, x_6); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__2), 4, 1); +lean_closure_set(x_19, 0, x_2); +lean_inc(x_5); +x_20 = l_Lean_Server_RequestM_bindTask___rarg(x_17, x_19, x_5, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__2___boxed), 5, 2); +lean_closure_set(x_23, 0, x_11); +lean_closure_set(x_23, 1, x_1); +x_24 = l_Lean_Server_RequestM_mapTask___rarg(x_21, x_23, x_5, x_22); +return x_24; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__3___boxed), 6, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___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; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_inc(x_1); -x_5 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3(x_1, x_2); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; +x_5 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__3___boxed), 6, 2); +lean_closure_set(x_5, 0, x_1); +lean_closure_set(x_5, 1, x_2); +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; x_7 = lean_st_ref_take(x_6, x_4); x_8 = lean_ctor_get(x_7, 0); lean_inc(x_8); @@ -5238,12 +28045,12 @@ return x_15; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_dec(x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1; +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1; x_7 = lean_st_ref_get(x_6, x_5); x_8 = !lean_is_exclusive(x_7); if (x_8 == 0) @@ -5259,7 +28066,7 @@ lean_object* x_12; lean_object* x_13; lean_free_object(x_7); lean_dec(x_3); x_12 = lean_box(0); -x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__1(x_1, x_2, x_12, x_10); +x_13 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___lambda__1(x_1, x_2, x_12, x_10); return x_13; } else @@ -5267,10 +28074,10 @@ else lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_dec(x_2); lean_dec(x_1); -x_14 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; +x_14 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; x_15 = lean_string_append(x_14, x_3); lean_dec(x_3); -x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; +x_16 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; x_17 = lean_string_append(x_15, x_16); x_18 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_18, 0, x_17); @@ -5294,7 +28101,7 @@ if (x_21 == 0) lean_object* x_22; lean_object* x_23; lean_dec(x_3); x_22 = lean_box(0); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__1(x_1, x_2, x_22, x_20); +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___lambda__1(x_1, x_2, x_22, x_20); return x_23; } else @@ -5302,10 +28109,10 @@ else lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_dec(x_2); lean_dec(x_1); -x_24 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; +x_24 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; x_25 = lean_string_append(x_24, x_3); lean_dec(x_3); -x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2; +x_26 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1; x_27 = lean_string_append(x_25, x_26); x_28 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_28, 0, x_27); @@ -5317,17 +28124,17 @@ return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; x_4 = 1; lean_inc(x_1); x_5 = l_Lean_Name_toString(x_1, x_4); -x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1; +x_6 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1; x_7 = lean_string_append(x_6, x_5); lean_dec(x_5); -x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2; +x_8 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2; x_9 = lean_string_append(x_7, x_8); x_10 = lean_io_initializing(x_3); x_11 = lean_ctor_get(x_10, 0); @@ -5345,10 +28152,10 @@ if (x_13 == 0) lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_14 = lean_ctor_get(x_10, 0); lean_dec(x_14); -x_15 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; +x_15 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; x_16 = lean_string_append(x_15, x_9); lean_dec(x_9); -x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; +x_17 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; x_18 = lean_string_append(x_16, x_17); x_19 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_19, 0, x_18); @@ -5362,10 +28169,10 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean x_20 = lean_ctor_get(x_10, 1); lean_inc(x_20); lean_dec(x_10); -x_21 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1; +x_21 = l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3; x_22 = lean_string_append(x_21, x_9); lean_dec(x_9); -x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3; +x_23 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3; x_24 = lean_string_append(x_22, x_23); x_25 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_25, 0, x_24); @@ -5382,12 +28189,12 @@ x_27 = lean_ctor_get(x_10, 1); lean_inc(x_27); lean_dec(x_10); x_28 = lean_box(0); -x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__2(x_1, x_2, x_9, x_28, x_27); +x_29 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___lambda__2(x_1, x_2, x_9, x_28, x_27); return x_29; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { if (lean_obj_tag(x_1) == 1) @@ -5530,7 +28337,7 @@ return x_40; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; @@ -5568,7 +28375,7 @@ lean_object* x_14; lean_object* x_15; lean_free_object(x_9); lean_dec(x_11); x_14 = lean_box(0); -x_15 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__1(x_7, x_3, x_8, x_6, x_14, x_4, x_12); +x_15 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__1(x_7, x_3, x_8, x_6, x_14, x_4, x_12); lean_dec(x_4); lean_dec(x_6); return x_15; @@ -5600,7 +28407,7 @@ else lean_object* x_20; lean_object* x_21; lean_dec(x_16); x_20 = lean_box(0); -x_21 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__1(x_7, x_3, x_8, x_6, x_20, x_4, x_17); +x_21 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__1(x_7, x_3, x_8, x_6, x_20, x_4, x_17); lean_dec(x_4); lean_dec(x_6); return x_21; @@ -5635,15 +28442,15 @@ return x_25; } } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3___closed__1() { +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_ReaderT_read___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__1), 2, 0); +x_1 = lean_alloc_closure((void*)(l_ReaderT_read___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__1), 2, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; @@ -5652,18 +28459,18 @@ x_5 = lean_ctor_get(x_1, 0); lean_inc(x_5); lean_dec(x_1); x_6 = lean_box(x_4); -x_7 = lean_alloc_closure((void*)(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__2___boxed), 5, 2); +x_7 = lean_alloc_closure((void*)(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__2___boxed), 5, 2); lean_closure_set(x_7, 0, x_5); lean_closure_set(x_7, 1, x_6); -x_8 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3___closed__1; -x_9 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__3___rarg), 4, 2); +x_8 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3___closed__1; +x_9 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 2); lean_closure_set(x_9, 0, x_8); lean_closure_set(x_9, 1, x_7); x_10 = l_Lean_Server_RequestM_asTask___rarg(x_9, x_2, x_3); return x_10; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__1() { +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__1() { _start: { lean_object* x_1; @@ -5671,61 +28478,114 @@ x_1 = lean_mk_string_from_bytes("getGoToLocation", 15); return x_1; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__2() { +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__1; +x_1 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4; +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__3() { +static lean_object* _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__3() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3), 3, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3), 3, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__2; -x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__3; -x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2(x_2, x_3, x_1); +x_2 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__2; +x_3 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__3; +x_4 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2(x_2, x_3, x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_liftExcept___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__5(x_1, x_2, x_3); +lean_dec(x_2); +lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__6(x_5, x_6, x_3, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__2(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint64_t x_7; lean_object* x_8; +x_7 = lean_unbox_uint64(x_3); +lean_dec(x_3); +x_8 = l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__3___lambda__3(x_1, x_2, x_7, x_4, x_5, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___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_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__2___lambda__1(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____spec__2___lambda__1(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { uint8_t x_6; lean_object* x_7; x_6 = lean_unbox(x_2); lean_dec(x_2); -x_7 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__2(x_1, x_6, x_3, x_4, x_5); +x_7 = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__2(x_1, x_6, x_3, x_4, x_5); return x_7; } } @@ -5768,186 +28628,170 @@ l_Lean_Widget_instInhabitedMsgToInteractive___closed__2 = _init_l_Lean_Widget_in lean_mark_persistent(l_Lean_Widget_instInhabitedMsgToInteractive___closed__2); l_Lean_Widget_instInhabitedMsgToInteractive = _init_l_Lean_Widget_instInhabitedMsgToInteractive(); lean_mark_persistent(l_Lean_Widget_instInhabitedMsgToInteractive); -l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__1); -l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__2 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__2(); -lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_93____rarg___closed__2); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__1(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__1); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__2(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__2); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__3); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__4 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__4(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__4); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__5 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__5(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__5); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__6 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__6(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__6); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__7); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__8); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__9 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__9(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__9); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__10 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__10(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__10); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__11 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__11(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__11); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__12 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__12(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__12); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__13 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__13(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__13); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__14 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__14(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__14); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__15); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__16 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__16(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__16); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__17 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__17(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__17); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__18 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__18(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__18); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__19 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__19(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__19); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__20 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__20(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__20); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__21 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__21(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__21); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__22 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__22(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__22); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__23); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__24 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__24(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__24); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__25 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__25(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__25); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__26 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__26(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__26); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__27 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__27(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__27); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__28 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__28(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__2___closed__28); -l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__1___closed__1); -l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__1); -l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___lambda__2___closed__2); -l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1(); -lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__1); -l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2(); -lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__2); -l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3(); -lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____spec__1___closed__3); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__1(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__1); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__2(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__2); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__3(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__3); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__4); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__5 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__5(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__5); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__6 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__6(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__6); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__7 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__7(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__7); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__8 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__8(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__8); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__9 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__9(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411____closed__9); -res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_411_(lean_io_mk_world()); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__1(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__1); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__2 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__2(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_60____closed__2); +l_Lean_Widget_instFromJsonRpcEncodingPacket__7___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__7___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__7___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__7 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__7(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__7); +l_Lean_Widget_instToJsonRpcEncodingPacket__7___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__7___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__7___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__7 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__7(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__7); +l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__1 = _init_l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__1); +l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__2 = _init_l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__2); +l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__3 = _init_l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgToInteractive___closed__3); +l_Lean_Widget_instRpcEncodingMsgToInteractive = _init_l_Lean_Widget_instRpcEncodingMsgToInteractive(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgToInteractive); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__1 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__1); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__2 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__2(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__2); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__3 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__3(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__3); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__4 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__4(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__3___closed__4); +l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1 = _init_l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1(); +lean_mark_persistent(l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__1); +l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2 = _init_l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2(); +lean_mark_persistent(l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__2); +l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3 = _init_l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3(); +lean_mark_persistent(l_Lean_Server_parseRequestParams___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__5___closed__3); +l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1 = _init_l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__1); +l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__2 = _init_l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__2); +l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3 = _init_l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__7___closed__3); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__1); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__2); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__1___closed__3); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__1); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__2); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__3___closed__3); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__1); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__2___lambda__4___closed__2); +l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__1___closed__1); +l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___lambda__2___closed__1); +l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1(); +lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__1); +l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2(); +lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__2); +l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3 = _init_l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3(); +lean_mark_persistent(l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____spec__1___closed__3); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__1(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__1); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__2(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__2); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__3(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__3); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__4); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__5 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__5(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__5); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__6 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__6(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__6); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__7 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__7(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__7); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__8 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__8(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__8); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__9 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__9(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275____closed__9); +res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_275_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Widget_instInhabitedInfoPopup___closed__1 = _init_l_Lean_Widget_instInhabitedInfoPopup___closed__1(); lean_mark_persistent(l_Lean_Widget_instInhabitedInfoPopup___closed__1); l_Lean_Widget_instInhabitedInfoPopup = _init_l_Lean_Widget_instInhabitedInfoPopup(); lean_mark_persistent(l_Lean_Widget_instInhabitedInfoPopup); -l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__1); -l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__2 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__2(); -lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__2); -l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__3 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__3(); -lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_569____rarg___closed__3); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__1(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__1); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__2(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__2); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__3(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__3); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__4 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__4(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__4); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__5 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__5(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__5); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__6 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__6(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____spec__2___closed__6); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__1(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__1); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__2(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__2); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__3(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234____closed__3); -res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1234_(lean_io_mk_world()); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__1(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__1); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__2 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__2(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__2); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_403____closed__3); +l_Lean_Widget_instFromJsonRpcEncodingPacket__8___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__8___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__8___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__8 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__8(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__8); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__1(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__1); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__2 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__2(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__2); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__3 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__3(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__3); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__4 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__4(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__4); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__5 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__5(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__5); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__6 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__6(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_475____closed__6); +l_Lean_Widget_instToJsonRpcEncodingPacket__8___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__8___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__8___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__8 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__8(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__8); +l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1 = _init_l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInfoPopup___lambda__3___closed__1); +l_Lean_Widget_instRpcEncodingInfoPopup___closed__1 = _init_l_Lean_Widget_instRpcEncodingInfoPopup___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInfoPopup___closed__1); +l_Lean_Widget_instRpcEncodingInfoPopup___closed__2 = _init_l_Lean_Widget_instRpcEncodingInfoPopup___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInfoPopup___closed__2); +l_Lean_Widget_instRpcEncodingInfoPopup___closed__3 = _init_l_Lean_Widget_instRpcEncodingInfoPopup___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInfoPopup___closed__3); +l_Lean_Widget_instRpcEncodingInfoPopup = _init_l_Lean_Widget_instRpcEncodingInfoPopup(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInfoPopup); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__1); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__2); +l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____spec__2___lambda__2___closed__3); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__1(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__1); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__2(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__2); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__3(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959____closed__3); +res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_959_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__1(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__1); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__2(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__2); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__3(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__3); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__4 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__4(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__4); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__5 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__5(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__5); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__6 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__6(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__6); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__7 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__7(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__7); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__8 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__8(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__8); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__9 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__9(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__9); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__10 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__10(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__10); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__11 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__11(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__11); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__12 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__12(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____spec__2___closed__12); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__1(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__1); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__2(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__2); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__3(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253____closed__3); -res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1253_(lean_io_mk_world()); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__1(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__1); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__2(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__2); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__3(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978____closed__3); +res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_978_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__1(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__1); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__2(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__2); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__3(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__3); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__4 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__4(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__2___closed__4); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3); -res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272_(lean_io_mk_world()); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__1(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__1); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__2(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__2); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__3(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997____closed__3); +res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_997_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Widget_instInhabitedGetInteractiveDiagnosticsParams = _init_l_Lean_Widget_instInhabitedGetInteractiveDiagnosticsParams(); lean_mark_persistent(l_Lean_Widget_instInhabitedGetInteractiveDiagnosticsParams); -l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1___closed__1 = _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1___closed__1(); -lean_mark_persistent(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____spec__1___closed__1); -l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____closed__1(); -lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1311____closed__1); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____closed__1(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonGetInteractiveDiagnosticsParams____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1036____closed__1); l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams___closed__1 = _init_l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams___closed__1(); lean_mark_persistent(l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams___closed__1); l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams = _init_l_Lean_Widget_instFromJsonGetInteractiveDiagnosticsParams(); @@ -5962,52 +28806,60 @@ l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2 = _init_l_Lean_W lean_mark_persistent(l_Lean_Widget_getInteractiveDiagnostics___lambda__1___closed__2); l_Lean_Widget_getInteractiveDiagnostics___closed__1 = _init_l_Lean_Widget_getInteractiveDiagnostics___closed__1(); lean_mark_persistent(l_Lean_Widget_getInteractiveDiagnostics___closed__1); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__1(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__1); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__2(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__2); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__3(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__3); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__4 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__4(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__4); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__5 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__5(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__5); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__6 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__6(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__6); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__7 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__7(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__7); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__8 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__8(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__8); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__9 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__9(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____spec__2___closed__9); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__1(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__1); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__2(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__2); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__3(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547____closed__3); -res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1547_(lean_io_mk_world()); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__1); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__2 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__2(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__2); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__3 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__3(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__3); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__4 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__4(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__4); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__5 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__5(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__5); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__6 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__6(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__6); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__7 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__7(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__7); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__8 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__8(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____spec__3___closed__8); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__1); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__2); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272____closed__3); +res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1272_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__1); -l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__2 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__2(); -lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1643____rarg___closed__2); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__1(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__1); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__2(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__2); -l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__3(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____spec__3___closed__3); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3___closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____lambda__3___closed__1); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__1(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__1); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__2(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__2); -l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__3(); -lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961____closed__3); -res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1961_(lean_io_mk_world()); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__1 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__1(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__1); +l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__2 = _init_l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__2(); +lean_mark_persistent(l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1335____closed__2); +l_Lean_Widget_instFromJsonRpcEncodingPacket__9___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__9___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__9___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__9 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__9(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__9); +l_Lean_Widget_instToJsonRpcEncodingPacket__9___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__9___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__9___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__9 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__9(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__9); +l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__1 = _init_l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__1); +l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__2 = _init_l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__2); +l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__3 = _init_l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingGetGoToLocationParams___closed__3); +l_Lean_Widget_instRpcEncodingGetGoToLocationParams = _init_l_Lean_Widget_instRpcEncodingGetGoToLocationParams(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingGetGoToLocationParams); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3___closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____lambda__3___closed__1); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__1 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__1(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__1); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__2 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__2(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__2); +l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__3 = _init_l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__3(); +lean_mark_persistent(l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550____closed__3); +res = l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1550_(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/Server/GoTo.c b/stage0/stdlib/Lean/Server/GoTo.c index a666f2b45030..c5fb9b1d6fda 100644 --- a/stage0/stdlib/Lean/Server/GoTo.c +++ b/stage0/stdlib/Lean/Server/GoTo.c @@ -13,9 +13,7 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__2; static lean_object* l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksFromDecl___spec__1___closed__2; -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__1; lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksFromDecl___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_locationLinksFromDecl___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -24,19 +22,21 @@ static lean_object* l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksFromDe static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24____closed__2; lean_object* lean_io_error_to_string(lean_object*); static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24____closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_findDeclarationRanges_x3f___at_Lean_Server_locationLinksFromDecl___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_noConfusionExt; LEAN_EXPORT lean_object* l_Lean_Server_instFromJsonGoToKind; +static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Except_orElseLazy___rarg(lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__2; lean_object* lean_st_ref_get(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___boxed(lean_object*); extern lean_object* l_Lean_declRangeExt; -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_locationLinksFromDecl___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___closed__1; static lean_object* l_Lean_Server_instToJsonGoToKind___closed__1; LEAN_EXPORT lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Server_locationLinksFromDecl___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Server_locationLinksFromDecl___spec__3___closed__1; @@ -45,41 +45,39 @@ static lean_object* l_Lean_Server_documentUriFromModule___closed__1; static lean_object* l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksFromDecl___spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Server_locationLinksFromDecl___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_locationLinksFromDecl___lambda__2___closed__1; +static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_locationLinksFromDecl___lambda__1(lean_object*, lean_object*, lean_object*, 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___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__2; LEAN_EXPORT lean_object* l_Lean_Server_instBEqGoToKind; lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Json_parseTagged(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instToJsonGoToKind; -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__3; lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* lean_io_realpath(lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__2; LEAN_EXPORT lean_object* l_Lean_findDeclarationRangesCore_x3f___at_Lean_Server_locationLinksFromDecl___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_documentUriFromModule(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__3; static lean_object* l_Lean_Server_instBEqGoToKind___closed__1; -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_Server_GoToKind_toCtorIdx(uint8_t); -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1(lean_object*); lean_object* l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_GoToKind_noConfusion___rarg___closed__1; -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__1; -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__1; static lean_object* l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksFromDecl___spec__1___closed__3; -static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__2; static lean_object* l_Lean_Server_instFromJsonGoToKind___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_GoToKind_noConfusion(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24_(uint8_t); LEAN_EXPORT lean_object* l_Lean_Server_GoToKind_toCtorIdx___boxed(lean_object*); lean_object* l_Lean_isRec___at___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_getKeyArgs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3(lean_object*, lean_object*, lean_object*); lean_object* l_Std_RBNode_find___at_Lean_findDeclarationRanges_x3f___spec__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__1; LEAN_EXPORT lean_object* l_Lean_findDeclarationRanges_x3f___at_Lean_Server_locationLinksFromDecl___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_findDeclarationRanges_x3f___at_Lean_Server_locationLinksFromDecl___spec__2___lambda__1___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_locationLinksFromDecl___lambda__2___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1(lean_object*); +static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__3; uint8_t lean_is_aux_recursor(lean_object*, lean_object*); static lean_object* l_Lean_findDeclarationRanges_x3f___at_Lean_Server_locationLinksFromDecl___spec__2___closed__1; extern lean_object* l_Lean_instInhabitedDeclarationRanges; @@ -96,14 +94,16 @@ LEAN_EXPORT lean_object* l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksF uint8_t l_Lean_TagDeclarationExtension_isTagged(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_locationLinksFromDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_GoToKind_noConfusion___rarg___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49_(lean_object*); static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24____closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_GoToKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SearchPath_findModuleWithExt(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24____closed__5; LEAN_EXPORT lean_object* l_Lean_Server_GoToKind_noConfusion___rarg___lambda__1___boxed(lean_object*); extern lean_object* l_Lean_builtinDeclRanges; lean_object* l_Lean_Lsp_DocumentUri_ofPath(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_GoToKind_toCtorIdx(uint8_t x_1) { _start: @@ -338,7 +338,7 @@ x_1 = l_Lean_Server_instToJsonGoToKind___closed__1; return x_1; } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__1() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -346,33 +346,33 @@ x_1 = lean_mk_string_from_bytes("no inductive constructor matched", 32); return x_1; } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__2() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__1; +x_1 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__1; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__2; +x_2 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__2; return x_2; } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__1() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___boxed), 1, 0); return x_1; } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__2() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__2() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; @@ -383,17 +383,17 @@ lean_ctor_set(x_3, 0, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__3() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__2; -x_2 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__1; +x_1 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__2; +x_2 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__1; x_3 = l_Except_orElseLazy___rarg(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -407,7 +407,7 @@ x_7 = !lean_is_exclusive(x_6); if (x_7 == 0) { lean_object* x_8; lean_object* x_9; -x_8 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__1; +x_8 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__1; x_9 = l_Except_orElseLazy___rarg(x_6, x_8); return x_9; } @@ -419,7 +419,7 @@ lean_inc(x_10); lean_dec(x_6); x_11 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_11, 0, x_10); -x_12 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__1; +x_12 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__1; x_13 = l_Except_orElseLazy___rarg(x_11, x_12); return x_13; } @@ -428,12 +428,12 @@ else { lean_object* x_14; lean_dec(x_6); -x_14 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__3; +x_14 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__3; return x_14; } } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___closed__1() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___closed__1() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; @@ -444,14 +444,14 @@ lean_ctor_set(x_3, 0, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24____closed__1; x_5 = lean_unsigned_to_nat(0u); x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); -x_7 = lean_alloc_closure((void*)(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___boxed), 3, 2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___boxed), 3, 2); lean_closure_set(x_7, 0, x_1); lean_closure_set(x_7, 1, x_2); if (lean_obj_tag(x_6) == 0) @@ -480,13 +480,13 @@ else { lean_object* x_13; lean_object* x_14; lean_dec(x_6); -x_13 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___closed__1; +x_13 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___closed__1; x_14 = l_Except_orElseLazy___rarg(x_13, x_7); return x_14; } } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__1() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -495,17 +495,17 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__2() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__1; +x_1 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__1; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__3() { +static lean_object* _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__3() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; @@ -516,15 +516,15 @@ lean_ctor_set(x_3, 0, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_2 = l___private_Lean_Server_GoTo_0__Lean_Server_toJsonGoToKind____x40_Lean_Server_GoTo___hyg_24____closed__5; x_3 = lean_unsigned_to_nat(0u); -x_4 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__2; +x_4 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__2; x_5 = l_Lean_Json_parseTagged(x_1, x_2, x_3, x_4); -x_6 = lean_alloc_closure((void*)(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___boxed), 3, 2); +x_6 = lean_alloc_closure((void*)(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___boxed), 3, 2); lean_closure_set(x_6, 0, x_1); lean_closure_set(x_6, 1, x_4); if (lean_obj_tag(x_5) == 0) @@ -553,37 +553,37 @@ else { lean_object* x_12; lean_object* x_13; lean_dec(x_5); -x_12 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__3; +x_12 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__3; x_13 = l_Except_orElseLazy___rarg(x_12, x_6); return x_13; } } } -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1(x_1); +x_2 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2(x_1, x_2, x_3); +x_4 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2(x_1, x_2, x_3); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3(x_1, x_2, x_3); +x_4 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3(x_1, x_2, x_3); lean_dec(x_3); return x_4; } @@ -592,7 +592,7 @@ static lean_object* _init_l_Lean_Server_instFromJsonGoToKind___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51_), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49_), 1, 0); return x_1; } } @@ -829,7 +829,7 @@ static lean_object* _init_l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinks lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksFromDecl___spec__1___closed__1; x_2 = l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksFromDecl___spec__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_findModuleOf_x3f___at_Lean_Server_locationLinksFromDecl___spec__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1373,7 +1373,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_locationLinksFromDecl___lambda__1(lean_ob _start: { lean_object* x_7; lean_object* x_8; -x_7 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__1; +x_7 = l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__1; x_8 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_8, 0, x_7); lean_ctor_set(x_8, 1, x_6); @@ -1875,24 +1875,24 @@ l_Lean_Server_instToJsonGoToKind___closed__1 = _init_l_Lean_Server_instToJsonGoT lean_mark_persistent(l_Lean_Server_instToJsonGoToKind___closed__1); l_Lean_Server_instToJsonGoToKind = _init_l_Lean_Server_instToJsonGoToKind(); lean_mark_persistent(l_Lean_Server_instToJsonGoToKind); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__1 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__1(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__1); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__2 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__2(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__1___closed__2); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__1 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__1(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__1); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__2 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__2(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__2); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__3 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__3(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__2___closed__3); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___closed__1 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___closed__1(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____lambda__3___closed__1); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__1 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__1(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__1); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__2 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__2(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__2); -l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__3 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__3(); -lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_51____closed__3); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__1 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__1); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__2 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__1___closed__2); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__1 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__1); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__2 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__2); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__3 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__2___closed__3); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___closed__1 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___closed__1(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____lambda__3___closed__1); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__1 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__1(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__1); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__2 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__2(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__2); +l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__3 = _init_l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__3(); +lean_mark_persistent(l___private_Lean_Server_GoTo_0__Lean_Server_fromJsonGoToKind____x40_Lean_Server_GoTo___hyg_49____closed__3); l_Lean_Server_instFromJsonGoToKind___closed__1 = _init_l_Lean_Server_instFromJsonGoToKind___closed__1(); lean_mark_persistent(l_Lean_Server_instFromJsonGoToKind___closed__1); l_Lean_Server_instFromJsonGoToKind = _init_l_Lean_Server_instFromJsonGoToKind(); diff --git a/stage0/stdlib/Lean/Server/InfoUtils.c b/stage0/stdlib/Lean/Server/InfoUtils.c index 21091993aacd..1dcab37e6220 100644 --- a/stage0/stdlib/Lean/Server/InfoUtils.c +++ b/stage0/stdlib/Lean/Server/InfoUtils.c @@ -106,6 +106,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_visitM_go___rarg(lean_object*, lea LEAN_EXPORT lean_object* l_String_Range_contains___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_String_instBEqRange; LEAN_EXPORT lean_object* l_Lean_Elab_Info_fmtHover_x3f_fmtTerm_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_InfoTree_foldInfo_go___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Elab_InfoTree_hasSorry_go___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_Format_joinSep___at_instReprProd___spec__1(lean_object*, lean_object*); @@ -257,7 +258,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_InfoTree_goalsAt_x3f___lambda__1___boxed(le LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_InfoTree_hoverableInfoAt_x3f___lambda__2___closed__6; size_t lean_usize_of_nat(lean_object*); -uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Info_docString_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PrettyPrinter_ppConst___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_getMax_x3f___at_Lean_Elab_InfoTree_smallestInfo_x3f___spec__2___boxed(lean_object*); @@ -5782,7 +5782,7 @@ x_3 = lean_ctor_get(x_2, 0); lean_inc(x_3); x_4 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_4, 0, x_3); -x_5 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_4, x_1); +x_5 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_4, x_1); lean_dec(x_4); return x_5; } @@ -8707,7 +8707,7 @@ x_8 = lean_ctor_get(x_6, 2); lean_inc(x_8); x_9 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_9, 0, x_8); -x_10 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_9, x_1); +x_10 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_9, x_1); lean_dec(x_9); if (x_10 == 0) { @@ -8740,7 +8740,7 @@ x_15 = lean_ctor_get(x_13, 2); lean_inc(x_15); x_16 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_16, 0, x_15); -x_17 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_344____spec__1(x_16, x_1); +x_17 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_364____spec__1(x_16, x_1); lean_dec(x_16); if (x_17 == 0) { diff --git a/stage0/stdlib/Lean/Server/References.c b/stage0/stdlib/Lean/Server/References.c index 94522b6ee981..160120574730 100644 --- a/stage0/stdlib/Lean/Server/References.c +++ b/stage0/stdlib/Lean/Server/References.c @@ -34,6 +34,7 @@ LEAN_EXPORT uint8_t l_Std_HashMapImp_contains___at_Lean_Server_combineFvars___sp LEAN_EXPORT lean_object* l_Lean_Server_References_definitionOf_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_updateWorkerRefs___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instFromJsonIlean; +static lean_object* l_Lean_Server_dedupReferences___closed__7; lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_Server_References_updateWorkerRefs___spec__3(lean_object*, lean_object*); @@ -42,7 +43,7 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_References_re LEAN_EXPORT lean_object* l_Std_AssocList_contains___at_Lean_Server_dedupReferences___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_erase___at_Lean_Server_References_removeWorkerRefs___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_dedupReferences___spec__14(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_referringTo___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT uint8_t l_Std_AssocList_contains___at_Lean_Server_ModuleRefs_addRef___spec__4(lean_object*, lean_object*); @@ -84,6 +85,7 @@ LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_References_allRefs___s uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Server_References_referringTo___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_References_0__Lean_Server_fromJsonIlean____x40_Lean_Server_References___hyg_804____boxed(lean_object*); +static lean_object* l_Lean_Server_dedupReferences___closed__11; LEAN_EXPORT lean_object* l_Lean_Server_References_referringTo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_erase___at_Lean_Server_References_removeIlean___spec__6(lean_object*, lean_object*); static lean_object* l_Lean_Server_instInhabitedReference___closed__1; @@ -91,7 +93,7 @@ static lean_object* l_Lean_Server_Reference_aliases___default___closed__1; lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Server_RefInfo_instCoeRefInfoRefInfo(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_contains___lambda__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_References_empty___spec__2___boxed(lean_object*); @@ -142,7 +144,7 @@ LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at_Lean_Server_ModuleRefs_add LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_combineFvars___spec__1___boxed(lean_object*); static lean_object* l_Lean_Server_instInhabitedReference___closed__14; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_RefInfo_instCoeRefInfoRefInfo___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11(uint8_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Server_dedupReferences___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_findModuleRefs___spec__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Server_References_findAt___spec__2___boxed(lean_object*, lean_object*); @@ -176,6 +178,7 @@ lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_Server_combineFvars___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Server_References_allRefs___spec__8(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Server_dedupReferences___lambda__1(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Server_combineFvars___spec__12(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Ilean_load(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Server_ModuleRefs_addRef___spec__3(lean_object*, lean_object*, lean_object*); @@ -185,6 +188,7 @@ static lean_object* l_Lean_Server_dedupReferences___closed__4; LEAN_EXPORT uint8_t l_Lean_Lsp_RefInfo_contains___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_referringTo___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_moveEntries___at_Lean_Server_dedupReferences___spec__7(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_dedupReferences___closed__8; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_referringTo___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_allRefs(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -194,6 +198,7 @@ static lean_object* l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__ LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_Server_ModuleRefs_addRef___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Server_References_updateWorkerRefs___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_Server_References_updateWorkerRefs___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_referringTo___spec__4(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Server_dedupReferences___closed__1; LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at_Lean_Server_References_addIlean___spec__3(lean_object*, lean_object*); @@ -211,6 +216,7 @@ LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Server_References_remo size_t lean_usize_modn(size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instHashableRange; +static uint64_t l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__1; lean_object* l_Lean_Elab_Info_stx(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Lsp_RefInfo_contains___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_findModuleRefs___spec__3(lean_object*, size_t, size_t, lean_object*); @@ -220,10 +226,11 @@ LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_References_empty___spe LEAN_EXPORT lean_object* l_Lean_Server_findReferences___boxed(lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Lsp_RefInfo_contains___spec__1___closed__2; static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__1___lambda__2___closed__2; +static lean_object* l_Lean_Server_dedupReferences___closed__9; LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Server_References_updateWorkerRefs___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_contains___at_Lean_Server_combineFvars___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Server_combineFvars___spec__11___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at_Lean_Server_dedupReferences___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_ModuleRefs_addRef(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -263,11 +270,13 @@ LEAN_EXPORT lean_object* l_Std_HashMap_toList___at_Lean_Server_References_referr lean_object* l_List_redLength___rarg(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Server_combineFvars___spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_References_allRefs___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_instHashableOption___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_ofList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_moveEntries___at_Lean_Server_References_updateWorkerRefs___spec__9(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_JsonNumber_fromNat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs(lean_object*, lean_object*, uint8_t, uint8_t); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__1___lambda__2___closed__1; +static lean_object* l_Lean_Server_dedupReferences___closed__5; static lean_object* l_Lean_Server_instInhabitedReference___closed__19; static lean_object* l_Lean_Server_Ilean_load___closed__2; LEAN_EXPORT lean_object* l_Std_HashMapImp_erase___at_Lean_Server_References_removeWorkerRefs___spec__1___boxed(lean_object*, lean_object*); @@ -292,6 +301,7 @@ static lean_object* l_Lean_Server_instInhabitedReference___closed__20; LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__8___at_Lean_Server_dedupReferences___spec__9(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_definitionsMatching___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Server_combineFvars_findCanonicalBinder___spec__2___boxed(lean_object*, lean_object*); +static uint64_t l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__2; LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_beqRefIdent____x40_Lean_Data_Lsp_Internal___hyg_28_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs___lambda__1(lean_object*, lean_object*); @@ -305,13 +315,17 @@ LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars_ lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_referringTo___spec__5(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_contains___at_Lean_Server_References_updateWorkerRefs___spec__7___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences___lambda__1___boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RefInfo_addRef(lean_object*, lean_object*); lean_object* l_List_toArrayAux___rarg(lean_object*, lean_object*); +lean_object* l_instBEq___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_instToJsonIlean___closed__1; LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_dedupReferences___spec__1___boxed(lean_object*); +static lean_object* l_Lean_Server_dedupReferences___closed__6; lean_object* l_Std_HashMap_toList___at_Lean_Lsp_instToJsonModuleRefs___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at_Lean_Server_combineFvars___spec__14(lean_object*, lean_object*); +uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_PrettyPrinter_delabCore___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_toList___at_Lean_Server_ModuleRefs_instCoeModuleRefsModuleRefs___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Server_dedupReferences___spec__8(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_References_definitionsMatching___rarg___closed__1; @@ -346,11 +360,13 @@ LEAN_EXPORT lean_object* l_Std_HashMapImp_moveEntries___at_Lean_Server_Reference LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_findModuleRefs___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_dedupReferences___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_contains___lambda__2___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_dedupReferences___closed__10; LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_Server_ModuleRefs_addRef___spec__7(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__1___lambda__1___boxed(lean_object*); static lean_object* l_Lean_Lsp_RefInfo_contains___lambda__2___closed__1; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_References_referringTo___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_Server_References_addIlean___spec__6(lean_object*, lean_object*, lean_object*); +lean_object* l_instHashableBool___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Lsp_RefInfo_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMapImp_erase___at_Lean_Server_References_removeIlean___spec__6___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_References_findAt___lambda__1(lean_object*); @@ -369,6 +385,7 @@ lean_object* l_Lean_Lsp_DocumentUri_ofPath(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instToJsonIlean; LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_Server_combineFvars___spec__11(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Ilean_version___default; +lean_object* l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_instInhabitedReference___closed__12; LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_combineFvars___spec__1(lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); @@ -4329,168 +4346,90 @@ goto _start; } else { -uint8_t x_13; -x_13 = lean_ctor_get_uint8(x_7, sizeof(void*)*6); -if (x_13 == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_7); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; size_t x_18; size_t x_19; -x_15 = lean_ctor_get(x_7, 0); -lean_dec(x_15); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; uint8_t x_19; +x_13 = lean_ctor_get(x_7, 2); +lean_inc(x_13); +x_14 = lean_ctor_get(x_7, 3); +lean_inc(x_14); +x_15 = lean_ctor_get(x_7, 4); +lean_inc(x_15); +x_16 = lean_ctor_get(x_7, 5); +lean_inc(x_16); +x_17 = lean_ctor_get_uint8(x_7, sizeof(void*)*6); +x_18 = lean_ctor_get(x_8, 0); +lean_inc(x_18); lean_inc(x_1); -x_16 = l_Lean_Server_combineFvars_applyIdMap(x_1, x_8); -lean_ctor_set(x_7, 0, x_16); -x_17 = lean_array_push(x_5, x_7); -x_18 = 1; -x_19 = lean_usize_add(x_4, x_18); -x_4 = x_19; -x_5 = x_17; -goto _start; -} -else +x_19 = l_Std_HashMapImp_contains___at_Lean_Server_combineFvars___spec__19(x_1, x_18); +if (x_19 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; size_t x_29; size_t x_30; -x_21 = lean_ctor_get(x_7, 1); -x_22 = lean_ctor_get(x_7, 2); -x_23 = lean_ctor_get(x_7, 3); -x_24 = lean_ctor_get(x_7, 4); -x_25 = lean_ctor_get(x_7, 5); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_7); -lean_inc(x_1); -x_26 = l_Lean_Server_combineFvars_applyIdMap(x_1, x_8); -x_27 = lean_alloc_ctor(0, 6, 1); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_21); -lean_ctor_set(x_27, 2, x_22); -lean_ctor_set(x_27, 3, x_23); -lean_ctor_set(x_27, 4, x_24); -lean_ctor_set(x_27, 5, x_25); -lean_ctor_set_uint8(x_27, sizeof(void*)*6, x_13); -x_28 = lean_array_push(x_5, x_27); -x_29 = 1; -x_30 = lean_usize_add(x_4, x_29); -x_4 = x_30; -x_5 = x_28; +lean_object* x_20; size_t x_21; size_t x_22; +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_8); +x_20 = lean_array_push(x_5, x_7); +x_21 = 1; +x_22 = lean_usize_add(x_4, x_21); +x_4 = x_22; +x_5 = x_20; goto _start; } -} else { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_7); -if (x_32 == 0) -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_33 = lean_ctor_get(x_7, 1); -x_34 = lean_ctor_get(x_7, 0); -lean_dec(x_34); -x_35 = lean_ctor_get(x_8, 0); -lean_inc(x_35); -lean_inc(x_1); -x_36 = l_Std_HashMapImp_contains___at_Lean_Server_combineFvars___spec__19(x_1, x_35); -if (x_36 == 0) -{ -lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; -lean_inc(x_1); -x_37 = l_Lean_Server_combineFvars_applyIdMap(x_1, x_8); -lean_ctor_set(x_7, 0, x_37); -x_38 = lean_array_push(x_5, x_7); -x_39 = 1; -x_40 = lean_usize_add(x_4, x_39); -x_4 = x_40; -x_5 = x_38; -goto _start; -} -else +uint8_t x_24; +x_24 = !lean_is_exclusive(x_7); +if (x_24 == 0) { -lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; size_t x_47; size_t x_48; -lean_dec(x_33); +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; size_t x_35; size_t x_36; +x_25 = lean_ctor_get(x_7, 5); +lean_dec(x_25); +x_26 = lean_ctor_get(x_7, 4); +lean_dec(x_26); +x_27 = lean_ctor_get(x_7, 3); +lean_dec(x_27); +x_28 = lean_ctor_get(x_7, 2); +lean_dec(x_28); +x_29 = lean_ctor_get(x_7, 1); +lean_dec(x_29); +x_30 = lean_ctor_get(x_7, 0); +lean_dec(x_30); lean_inc(x_8); lean_inc(x_1); -x_42 = l_Lean_Server_combineFvars_applyIdMap(x_1, x_8); -x_43 = l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__20___closed__1; -x_44 = lean_array_push(x_43, x_8); -x_45 = 0; -lean_ctor_set(x_7, 1, x_44); -lean_ctor_set(x_7, 0, x_42); -lean_ctor_set_uint8(x_7, sizeof(void*)*6, x_45); -x_46 = lean_array_push(x_5, x_7); -x_47 = 1; -x_48 = lean_usize_add(x_4, x_47); -x_4 = x_48; -x_5 = x_46; +x_31 = l_Lean_Server_combineFvars_applyIdMap(x_1, x_8); +x_32 = l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__20___closed__1; +x_33 = lean_array_push(x_32, x_8); +lean_ctor_set(x_7, 1, x_33); +lean_ctor_set(x_7, 0, x_31); +x_34 = lean_array_push(x_5, x_7); +x_35 = 1; +x_36 = lean_usize_add(x_4, x_35); +x_4 = x_36; +x_5 = x_34; goto _start; } -} else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; -x_50 = lean_ctor_get(x_7, 1); -x_51 = lean_ctor_get(x_7, 2); -x_52 = lean_ctor_get(x_7, 3); -x_53 = lean_ctor_get(x_7, 4); -x_54 = lean_ctor_get(x_7, 5); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -lean_inc(x_50); +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_dec(x_7); -x_55 = lean_ctor_get(x_8, 0); -lean_inc(x_55); -lean_inc(x_1); -x_56 = l_Std_HashMapImp_contains___at_Lean_Server_combineFvars___spec__19(x_1, x_55); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; -lean_inc(x_1); -x_57 = l_Lean_Server_combineFvars_applyIdMap(x_1, x_8); -x_58 = lean_alloc_ctor(0, 6, 1); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_50); -lean_ctor_set(x_58, 2, x_51); -lean_ctor_set(x_58, 3, x_52); -lean_ctor_set(x_58, 4, x_53); -lean_ctor_set(x_58, 5, x_54); -lean_ctor_set_uint8(x_58, sizeof(void*)*6, x_13); -x_59 = lean_array_push(x_5, x_58); -x_60 = 1; -x_61 = lean_usize_add(x_4, x_60); -x_4 = x_61; -x_5 = x_59; -goto _start; -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; size_t x_69; size_t x_70; -lean_dec(x_50); lean_inc(x_8); lean_inc(x_1); -x_63 = l_Lean_Server_combineFvars_applyIdMap(x_1, x_8); -x_64 = l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__20___closed__1; -x_65 = lean_array_push(x_64, x_8); -x_66 = 0; -x_67 = lean_alloc_ctor(0, 6, 1); -lean_ctor_set(x_67, 0, x_63); -lean_ctor_set(x_67, 1, x_65); -lean_ctor_set(x_67, 2, x_51); -lean_ctor_set(x_67, 3, x_52); -lean_ctor_set(x_67, 4, x_53); -lean_ctor_set(x_67, 5, x_54); -lean_ctor_set_uint8(x_67, sizeof(void*)*6, x_66); -x_68 = lean_array_push(x_5, x_67); -x_69 = 1; -x_70 = lean_usize_add(x_4, x_69); -x_4 = x_70; -x_5 = x_68; +x_38 = l_Lean_Server_combineFvars_applyIdMap(x_1, x_8); +x_39 = l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__20___closed__1; +x_40 = lean_array_push(x_39, x_8); +x_41 = lean_alloc_ctor(0, 6, 1); +lean_ctor_set(x_41, 0, x_38); +lean_ctor_set(x_41, 1, x_40); +lean_ctor_set(x_41, 2, x_13); +lean_ctor_set(x_41, 3, x_14); +lean_ctor_set(x_41, 4, x_15); +lean_ctor_set(x_41, 5, x_16); +lean_ctor_set_uint8(x_41, sizeof(void*)*6, x_17); +x_42 = lean_array_push(x_5, x_41); +x_43 = 1; +x_44 = lean_usize_add(x_4, x_43); +x_4 = x_44; +x_5 = x_42; goto _start; } } @@ -4498,7 +4437,6 @@ goto _start; } } } -} LEAN_EXPORT lean_object* l_Lean_Server_combineFvars(lean_object* x_1) { _start: { @@ -4651,29 +4589,62 @@ goto _start; } else { -uint8_t x_13; -x_13 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_515_(x_8, x_10); -if (x_13 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_8, 0); +x_14 = lean_ctor_get(x_8, 1); +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +x_17 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_PrettyPrinter_delabCore___spec__3(x_13, x_15); +if (x_17 == 0) { x_2 = x_6; goto _start; } else { -lean_object* x_15; +uint8_t x_19; +x_19 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_515_(x_14, x_16); +if (x_19 == 0) +{ +x_2 = x_6; +goto _start; +} +else +{ +lean_object* x_21; lean_inc(x_5); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_5); -return x_15; +x_21 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_21, 0, x_5); +return x_21; +} } } } } } +static uint64_t _init_l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__1() { +_start: +{ +uint64_t x_1; uint64_t x_2; +x_1 = 13; +x_2 = lean_uint64_mix_hash(x_1, x_1); +return x_2; +} +} +static uint64_t _init_l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__2() { +_start: +{ +uint64_t x_1; uint64_t x_2; uint64_t x_3; +x_1 = 13; +x_2 = 11; +x_3 = lean_uint64_mix_hash(x_2, x_1); +return x_3; +} +} LEAN_EXPORT lean_object* l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2(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; uint64_t x_7; uint64_t x_8; uint64_t x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint64_t x_7; lean_object* x_8; lean_object* x_9; uint64_t x_10; x_3 = lean_ctor_get(x_1, 1); lean_inc(x_3); lean_dec(x_1); @@ -4684,18 +4655,70 @@ x_6 = lean_ctor_get(x_2, 1); lean_inc(x_6); x_7 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean_Data_Lsp_Internal___hyg_106_(x_5); lean_dec(x_5); -x_8 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_6); +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_6, 1); +lean_inc(x_9); lean_dec(x_6); -x_9 = lean_uint64_mix_hash(x_7, x_8); -x_10 = lean_uint64_to_usize(x_9); -x_11 = lean_usize_modn(x_10, x_4); +x_10 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_9); +lean_dec(x_9); +if (lean_obj_tag(x_8) == 0) +{ +uint64_t x_11; uint64_t x_12; uint64_t x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; +x_11 = 11; +x_12 = lean_uint64_mix_hash(x_11, x_10); +x_13 = lean_uint64_mix_hash(x_7, x_12); +x_14 = lean_uint64_to_usize(x_13); +x_15 = lean_usize_modn(x_14, x_4); lean_dec(x_4); -x_12 = lean_array_uget(x_3, x_11); +x_16 = lean_array_uget(x_3, x_15); lean_dec(x_3); -x_13 = l_Std_AssocList_find_x3f___at_Lean_Server_dedupReferences___spec__3(x_2, x_12); -lean_dec(x_12); +x_17 = l_Std_AssocList_find_x3f___at_Lean_Server_dedupReferences___spec__3(x_2, x_16); +lean_dec(x_16); lean_dec(x_2); -return x_13; +return x_17; +} +else +{ +lean_object* x_18; uint8_t x_19; +x_18 = lean_ctor_get(x_8, 0); +lean_inc(x_18); +lean_dec(x_8); +x_19 = lean_unbox(x_18); +lean_dec(x_18); +if (x_19 == 0) +{ +uint64_t x_20; uint64_t x_21; uint64_t x_22; size_t x_23; size_t x_24; lean_object* x_25; lean_object* x_26; +x_20 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__1; +x_21 = lean_uint64_mix_hash(x_20, x_10); +x_22 = lean_uint64_mix_hash(x_7, x_21); +x_23 = lean_uint64_to_usize(x_22); +x_24 = lean_usize_modn(x_23, x_4); +lean_dec(x_4); +x_25 = lean_array_uget(x_3, x_24); +lean_dec(x_3); +x_26 = l_Std_AssocList_find_x3f___at_Lean_Server_dedupReferences___spec__3(x_2, x_25); +lean_dec(x_25); +lean_dec(x_2); +return x_26; +} +else +{ +uint64_t x_27; uint64_t x_28; uint64_t x_29; size_t x_30; size_t x_31; lean_object* x_32; lean_object* x_33; +x_27 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__2; +x_28 = lean_uint64_mix_hash(x_27, x_10); +x_29 = lean_uint64_mix_hash(x_7, x_28); +x_30 = lean_uint64_to_usize(x_29); +x_31 = lean_usize_modn(x_30, x_4); +lean_dec(x_4); +x_32 = lean_array_uget(x_3, x_31); +lean_dec(x_3); +x_33 = l_Std_AssocList_find_x3f___at_Lean_Server_dedupReferences___spec__3(x_2, x_32); +lean_dec(x_32); +lean_dec(x_2); +return x_33; +} +} } } LEAN_EXPORT uint8_t l_Std_AssocList_contains___at_Lean_Server_dedupReferences___spec__5(lean_object* x_1, lean_object* x_2) { @@ -4724,18 +4747,32 @@ goto _start; } else { -uint8_t x_12; -x_12 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_515_(x_7, x_9); -if (x_12 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_12 = lean_ctor_get(x_7, 0); +x_13 = lean_ctor_get(x_7, 1); +x_14 = lean_ctor_get(x_9, 0); +x_15 = lean_ctor_get(x_9, 1); +x_16 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_PrettyPrinter_delabCore___spec__3(x_12, x_14); +if (x_16 == 0) { x_2 = x_5; goto _start; } else { -uint8_t x_14; -x_14 = 1; -return x_14; +uint8_t x_18; +x_18 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_515_(x_13, x_15); +if (x_18 == 0) +{ +x_2 = x_5; +goto _start; +} +else +{ +uint8_t x_20; +x_20 = 1; +return x_20; +} } } } @@ -4819,7 +4856,7 @@ uint8_t x_3; x_3 = !lean_is_exclusive(x_2); if (x_3 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint64_t x_9; uint64_t x_10; uint64_t x_11; size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint64_t x_9; lean_object* x_10; lean_object* x_11; uint64_t x_12; x_4 = lean_ctor_get(x_2, 0); x_5 = lean_ctor_get(x_2, 2); x_6 = lean_array_get_size(x_1); @@ -4829,52 +4866,162 @@ x_8 = lean_ctor_get(x_4, 1); lean_inc(x_8); x_9 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean_Data_Lsp_Internal___hyg_106_(x_7); lean_dec(x_7); -x_10 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_8); +x_10 = lean_ctor_get(x_8, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_8, 1); +lean_inc(x_11); lean_dec(x_8); -x_11 = lean_uint64_mix_hash(x_9, x_10); -x_12 = lean_uint64_to_usize(x_11); -x_13 = lean_usize_modn(x_12, x_6); +x_12 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_11); +lean_dec(x_11); +if (lean_obj_tag(x_10) == 0) +{ +uint64_t x_13; uint64_t x_14; uint64_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; +x_13 = 11; +x_14 = lean_uint64_mix_hash(x_13, x_12); +x_15 = lean_uint64_mix_hash(x_9, x_14); +x_16 = lean_uint64_to_usize(x_15); +x_17 = lean_usize_modn(x_16, x_6); lean_dec(x_6); -x_14 = lean_array_uget(x_1, x_13); -lean_ctor_set(x_2, 2, x_14); -x_15 = lean_array_uset(x_1, x_13, x_2); -x_1 = x_15; +x_18 = lean_array_uget(x_1, x_17); +lean_ctor_set(x_2, 2, x_18); +x_19 = lean_array_uset(x_1, x_17, x_2); +x_1 = x_19; x_2 = x_5; goto _start; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint64_t x_23; uint64_t x_24; uint64_t x_25; size_t x_26; size_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_17 = lean_ctor_get(x_2, 0); -x_18 = lean_ctor_get(x_2, 1); -x_19 = lean_ctor_get(x_2, 2); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_2); -x_20 = lean_array_get_size(x_1); -x_21 = lean_ctor_get(x_17, 0); +lean_object* x_21; uint8_t x_22; +x_21 = lean_ctor_get(x_10, 0); lean_inc(x_21); -x_22 = lean_ctor_get(x_17, 1); -lean_inc(x_22); -x_23 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean_Data_Lsp_Internal___hyg_106_(x_21); +lean_dec(x_10); +x_22 = lean_unbox(x_21); lean_dec(x_21); -x_24 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_22); -lean_dec(x_22); -x_25 = lean_uint64_mix_hash(x_23, x_24); +if (x_22 == 0) +{ +uint64_t x_23; uint64_t x_24; uint64_t x_25; size_t x_26; size_t x_27; lean_object* x_28; lean_object* x_29; +x_23 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__1; +x_24 = lean_uint64_mix_hash(x_23, x_12); +x_25 = lean_uint64_mix_hash(x_9, x_24); x_26 = lean_uint64_to_usize(x_25); -x_27 = lean_usize_modn(x_26, x_20); -lean_dec(x_20); +x_27 = lean_usize_modn(x_26, x_6); +lean_dec(x_6); x_28 = lean_array_uget(x_1, x_27); -x_29 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_29, 0, x_17); -lean_ctor_set(x_29, 1, x_18); -lean_ctor_set(x_29, 2, x_28); -x_30 = lean_array_uset(x_1, x_27, x_29); -x_1 = x_30; -x_2 = x_19; +lean_ctor_set(x_2, 2, x_28); +x_29 = lean_array_uset(x_1, x_27, x_2); +x_1 = x_29; +x_2 = x_5; goto _start; } +else +{ +uint64_t x_31; uint64_t x_32; uint64_t x_33; size_t x_34; size_t x_35; lean_object* x_36; lean_object* x_37; +x_31 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__2; +x_32 = lean_uint64_mix_hash(x_31, x_12); +x_33 = lean_uint64_mix_hash(x_9, x_32); +x_34 = lean_uint64_to_usize(x_33); +x_35 = lean_usize_modn(x_34, x_6); +lean_dec(x_6); +x_36 = lean_array_uget(x_1, x_35); +lean_ctor_set(x_2, 2, x_36); +x_37 = lean_array_uset(x_1, x_35, x_2); +x_1 = x_37; +x_2 = x_5; +goto _start; +} +} +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint64_t x_45; lean_object* x_46; lean_object* x_47; uint64_t x_48; +x_39 = lean_ctor_get(x_2, 0); +x_40 = lean_ctor_get(x_2, 1); +x_41 = lean_ctor_get(x_2, 2); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_2); +x_42 = lean_array_get_size(x_1); +x_43 = lean_ctor_get(x_39, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_39, 1); +lean_inc(x_44); +x_45 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean_Data_Lsp_Internal___hyg_106_(x_43); +lean_dec(x_43); +x_46 = lean_ctor_get(x_44, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_44, 1); +lean_inc(x_47); +lean_dec(x_44); +x_48 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_47); +lean_dec(x_47); +if (lean_obj_tag(x_46) == 0) +{ +uint64_t x_49; uint64_t x_50; uint64_t x_51; size_t x_52; size_t x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_49 = 11; +x_50 = lean_uint64_mix_hash(x_49, x_48); +x_51 = lean_uint64_mix_hash(x_45, x_50); +x_52 = lean_uint64_to_usize(x_51); +x_53 = lean_usize_modn(x_52, x_42); +lean_dec(x_42); +x_54 = lean_array_uget(x_1, x_53); +x_55 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_55, 0, x_39); +lean_ctor_set(x_55, 1, x_40); +lean_ctor_set(x_55, 2, x_54); +x_56 = lean_array_uset(x_1, x_53, x_55); +x_1 = x_56; +x_2 = x_41; +goto _start; +} +else +{ +lean_object* x_58; uint8_t x_59; +x_58 = lean_ctor_get(x_46, 0); +lean_inc(x_58); +lean_dec(x_46); +x_59 = lean_unbox(x_58); +lean_dec(x_58); +if (x_59 == 0) +{ +uint64_t x_60; uint64_t x_61; uint64_t x_62; size_t x_63; size_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_60 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__1; +x_61 = lean_uint64_mix_hash(x_60, x_48); +x_62 = lean_uint64_mix_hash(x_45, x_61); +x_63 = lean_uint64_to_usize(x_62); +x_64 = lean_usize_modn(x_63, x_42); +lean_dec(x_42); +x_65 = lean_array_uget(x_1, x_64); +x_66 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_66, 0, x_39); +lean_ctor_set(x_66, 1, x_40); +lean_ctor_set(x_66, 2, x_65); +x_67 = lean_array_uset(x_1, x_64, x_66); +x_1 = x_67; +x_2 = x_41; +goto _start; +} +else +{ +uint64_t x_69; uint64_t x_70; uint64_t x_71; size_t x_72; size_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_69 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__2; +x_70 = lean_uint64_mix_hash(x_69, x_48); +x_71 = lean_uint64_mix_hash(x_45, x_70); +x_72 = lean_uint64_to_usize(x_71); +x_73 = lean_usize_modn(x_72, x_42); +lean_dec(x_42); +x_74 = lean_array_uget(x_1, x_73); +x_75 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_75, 0, x_39); +lean_ctor_set(x_75, 1, x_40); +lean_ctor_set(x_75, 2, x_74); +x_76 = lean_array_uset(x_1, x_73, x_75); +x_1 = x_76; +x_2 = x_41; +goto _start; +} +} +} } } } @@ -4969,15 +5116,40 @@ return x_3; } else { -uint8_t x_15; -x_15 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_515_(x_10, x_12); -lean_dec(x_12); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_15 = lean_ctor_get(x_10, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); lean_dec(x_10); -if (x_15 == 0) +x_17 = lean_ctor_get(x_12, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_12, 1); +lean_inc(x_18); +lean_dec(x_12); +x_19 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_PrettyPrinter_delabCore___spec__3(x_15, x_17); +lean_dec(x_17); +lean_dec(x_15); +if (x_19 == 0) { -lean_object* x_16; -x_16 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_16); +lean_object* x_20; +lean_dec(x_18); +lean_dec(x_16); +x_20 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_1, x_2, x_8); +lean_ctor_set(x_3, 2, x_20); +return x_3; +} +else +{ +uint8_t x_21; +x_21 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_515_(x_16, x_18); +lean_dec(x_18); +lean_dec(x_16); +if (x_21 == 0) +{ +lean_object* x_22; +x_22 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_1, x_2, x_8); +lean_ctor_set(x_3, 2, x_22); return x_3; } else @@ -4990,65 +5162,95 @@ return x_3; } } } +} else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_17 = lean_ctor_get(x_3, 0); -x_18 = lean_ctor_get(x_3, 1); -x_19 = lean_ctor_get(x_3, 2); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_3); -x_20 = lean_ctor_get(x_17, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_17, 1); -lean_inc(x_21); -x_22 = lean_ctor_get(x_1, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_1, 1); +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; uint8_t x_30; +x_23 = lean_ctor_get(x_3, 0); +x_24 = lean_ctor_get(x_3, 1); +x_25 = lean_ctor_get(x_3, 2); +lean_inc(x_25); +lean_inc(x_24); lean_inc(x_23); -x_24 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_beqRefIdent____x40_Lean_Data_Lsp_Internal___hyg_28_(x_20, x_22); -lean_dec(x_22); -lean_dec(x_20); -if (x_24 == 0) +lean_dec(x_3); +x_26 = lean_ctor_get(x_23, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_23, 1); +lean_inc(x_27); +x_28 = lean_ctor_get(x_1, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_1, 1); +lean_inc(x_29); +x_30 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_beqRefIdent____x40_Lean_Data_Lsp_Internal___hyg_28_(x_26, x_28); +lean_dec(x_28); +lean_dec(x_26); +if (x_30 == 0) { -lean_object* x_25; lean_object* x_26; -lean_dec(x_23); -lean_dec(x_21); -x_25 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_1, x_2, x_19); -x_26 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_26, 0, x_17); -lean_ctor_set(x_26, 1, x_18); -lean_ctor_set(x_26, 2, x_25); -return x_26; +lean_object* x_31; lean_object* x_32; +lean_dec(x_29); +lean_dec(x_27); +x_31 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_1, x_2, x_25); +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_23); +lean_ctor_set(x_32, 1, x_24); +lean_ctor_set(x_32, 2, x_31); +return x_32; } else { -uint8_t x_27; -x_27 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_515_(x_21, x_23); -lean_dec(x_23); -lean_dec(x_21); -if (x_27 == 0) +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_33 = lean_ctor_get(x_27, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_27, 1); +lean_inc(x_34); +lean_dec(x_27); +x_35 = lean_ctor_get(x_29, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_29, 1); +lean_inc(x_36); +lean_dec(x_29); +x_37 = l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_PrettyPrinter_delabCore___spec__3(x_33, x_35); +lean_dec(x_35); +lean_dec(x_33); +if (x_37 == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_1, x_2, x_19); -x_29 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_29, 0, x_17); -lean_ctor_set(x_29, 1, x_18); -lean_ctor_set(x_29, 2, x_28); -return x_29; +lean_object* x_38; lean_object* x_39; +lean_dec(x_36); +lean_dec(x_34); +x_38 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_1, x_2, x_25); +x_39 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_39, 0, x_23); +lean_ctor_set(x_39, 1, x_24); +lean_ctor_set(x_39, 2, x_38); +return x_39; } else { -lean_object* x_30; -lean_dec(x_18); -lean_dec(x_17); -x_30 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_30, 0, x_1); -lean_ctor_set(x_30, 1, x_2); -lean_ctor_set(x_30, 2, x_19); -return x_30; +uint8_t x_40; +x_40 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqRange____x40_Lean_Data_Lsp_Basic___hyg_515_(x_34, x_36); +lean_dec(x_36); +lean_dec(x_34); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +x_41 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_1, x_2, x_25); +x_42 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_42, 0, x_23); +lean_ctor_set(x_42, 1, x_24); +lean_ctor_set(x_42, 2, x_41); +return x_42; +} +else +{ +lean_object* x_43; +lean_dec(x_24); +lean_dec(x_23); +x_43 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_43, 0, x_1); +lean_ctor_set(x_43, 1, x_2); +lean_ctor_set(x_43, 2, x_25); +return x_43; +} } } } @@ -5058,262 +5260,313 @@ return x_30; LEAN_EXPORT lean_object* l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_1); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; size_t x_13; size_t x_14; lean_object* x_15; uint8_t x_16; -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_1, 1); -x_7 = lean_array_get_size(x_6); -x_8 = lean_ctor_get(x_2, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_2, 1); -lean_inc(x_9); -x_10 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean_Data_Lsp_Internal___hyg_106_(x_8); -lean_dec(x_8); -x_11 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_9); -lean_dec(x_9); -x_12 = lean_uint64_mix_hash(x_10, x_11); -x_13 = lean_uint64_to_usize(x_12); -x_14 = lean_usize_modn(x_13, x_7); -x_15 = lean_array_uget(x_6, x_14); -x_16 = l_Std_AssocList_contains___at_Lean_Server_dedupReferences___spec__5(x_2, x_15); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_nat_add(x_5, x_17); -lean_dec(x_5); -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_2); -lean_ctor_set(x_19, 1, x_3); -lean_ctor_set(x_19, 2, x_15); -x_20 = lean_array_uset(x_6, x_14, x_19); -x_21 = l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(x_18); -x_22 = lean_nat_dec_le(x_21, x_7); -lean_dec(x_7); -lean_dec(x_21); -if (x_22 == 0) +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint64_t x_8; lean_object* x_25; lean_object* x_26; uint64_t x_27; lean_object* x_28; lean_object* x_29; uint64_t x_30; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +if (lean_is_exclusive(x_1)) { + lean_ctor_release(x_1, 0); + lean_ctor_release(x_1, 1); + x_6 = x_1; +} else { + lean_dec_ref(x_1); + x_6 = lean_box(0); +} +x_7 = lean_array_get_size(x_5); +x_25 = lean_ctor_get(x_2, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_2, 1); +lean_inc(x_26); +x_27 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean_Data_Lsp_Internal___hyg_106_(x_25); +lean_dec(x_25); +x_28 = lean_ctor_get(x_26, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_26, 1); +lean_inc(x_29); +lean_dec(x_26); +x_30 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_29); +lean_dec(x_29); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_23; -lean_free_object(x_1); -x_23 = l_Std_HashMapImp_expand___at_Lean_Server_dedupReferences___spec__6(x_18, x_20); -return x_23; +uint64_t x_31; uint64_t x_32; uint64_t x_33; +x_31 = 11; +x_32 = lean_uint64_mix_hash(x_31, x_30); +x_33 = lean_uint64_mix_hash(x_27, x_32); +x_8 = x_33; +goto block_24; } else { -lean_ctor_set(x_1, 1, x_20); -lean_ctor_set(x_1, 0, x_18); -return x_1; -} +lean_object* x_34; uint8_t x_35; +x_34 = lean_ctor_get(x_28, 0); +lean_inc(x_34); +lean_dec(x_28); +x_35 = lean_unbox(x_34); +lean_dec(x_34); +if (x_35 == 0) +{ +uint64_t x_36; uint64_t x_37; uint64_t x_38; +x_36 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__1; +x_37 = lean_uint64_mix_hash(x_36, x_30); +x_38 = lean_uint64_mix_hash(x_27, x_37); +x_8 = x_38; +goto block_24; } else { -lean_object* x_24; lean_object* x_25; -lean_dec(x_7); -x_24 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_2, x_3, x_15); -x_25 = lean_array_uset(x_6, x_14, x_24); -lean_ctor_set(x_1, 1, x_25); -return x_1; +uint64_t x_39; uint64_t x_40; uint64_t x_41; +x_39 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__2; +x_40 = lean_uint64_mix_hash(x_39, x_30); +x_41 = lean_uint64_mix_hash(x_27, x_40); +x_8 = x_41; +goto block_24; } } -else +block_24: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint64_t x_31; uint64_t x_32; uint64_t x_33; size_t x_34; size_t x_35; lean_object* x_36; uint8_t x_37; -x_26 = lean_ctor_get(x_1, 0); -x_27 = lean_ctor_get(x_1, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_1); -x_28 = lean_array_get_size(x_27); -x_29 = lean_ctor_get(x_2, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_2, 1); -lean_inc(x_30); -x_31 = l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean_Data_Lsp_Internal___hyg_106_(x_29); -lean_dec(x_29); -x_32 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashRange____x40_Lean_Data_Lsp_Basic___hyg_586_(x_30); -lean_dec(x_30); -x_33 = lean_uint64_mix_hash(x_31, x_32); -x_34 = lean_uint64_to_usize(x_33); -x_35 = lean_usize_modn(x_34, x_28); -x_36 = lean_array_uget(x_27, x_35); -x_37 = l_Std_AssocList_contains___at_Lean_Server_dedupReferences___spec__5(x_2, x_36); -if (x_37 == 0) +size_t x_9; size_t x_10; lean_object* x_11; uint8_t x_12; +x_9 = lean_uint64_to_usize(x_8); +x_10 = lean_usize_modn(x_9, x_7); +x_11 = lean_array_uget(x_5, x_10); +x_12 = l_Std_AssocList_contains___at_Lean_Server_dedupReferences___spec__5(x_2, x_11); +if (x_12 == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_nat_add(x_26, x_38); -lean_dec(x_26); -x_40 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_40, 0, x_2); -lean_ctor_set(x_40, 1, x_3); -lean_ctor_set(x_40, 2, x_36); -x_41 = lean_array_uset(x_27, x_35, x_40); -x_42 = l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(x_39); -x_43 = lean_nat_dec_le(x_42, x_28); -lean_dec(x_28); -lean_dec(x_42); -if (x_43 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_13 = lean_unsigned_to_nat(1u); +x_14 = lean_nat_add(x_4, x_13); +lean_dec(x_4); +x_15 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_3); +lean_ctor_set(x_15, 2, x_11); +x_16 = lean_array_uset(x_5, x_10, x_15); +x_17 = l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(x_14); +x_18 = lean_nat_dec_le(x_17, x_7); +lean_dec(x_7); +lean_dec(x_17); +if (x_18 == 0) { -lean_object* x_44; -x_44 = l_Std_HashMapImp_expand___at_Lean_Server_dedupReferences___spec__6(x_39, x_41); -return x_44; +lean_object* x_19; +lean_dec(x_6); +x_19 = l_Std_HashMapImp_expand___at_Lean_Server_dedupReferences___spec__6(x_14, x_16); +return x_19; } else { -lean_object* x_45; -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_39); -lean_ctor_set(x_45, 1, x_41); -return x_45; +lean_object* x_20; +if (lean_is_scalar(x_6)) { + x_20 = lean_alloc_ctor(0, 2, 0); +} else { + x_20 = x_6; +} +lean_ctor_set(x_20, 0, x_14); +lean_ctor_set(x_20, 1, x_16); +return x_20; } } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -lean_dec(x_28); -x_46 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_2, x_3, x_36); -x_47 = lean_array_uset(x_27, x_35, x_46); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_26); -lean_ctor_set(x_48, 1, x_47); -return x_48; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_7); +x_21 = l_Std_AssocList_replace___at_Lean_Server_dedupReferences___spec__10(x_2, x_3, x_11); +x_22 = lean_array_uset(x_5, x_10, x_21); +if (lean_is_scalar(x_6)) { + x_23 = lean_alloc_ctor(0, 2, 0); +} else { + x_23 = x_6; +} +lean_ctor_set(x_23, 0, x_4); +lean_ctor_set(x_23, 1, x_22); +return x_23; } } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7) { _start: { -uint8_t x_7; -x_7 = lean_usize_dec_lt(x_5, x_4); -if (x_7 == 0) +uint8_t x_8; +x_8 = lean_usize_dec_lt(x_6, x_5); +if (x_8 == 0) { -return x_6; +return x_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_8 = lean_array_uget(x_3, x_5); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 1); +lean_object* x_9; +x_9 = lean_array_uget(x_4, x_6); +if (x_1 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); -x_11 = lean_ctor_get(x_8, 2); +x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); -x_12 = lean_ctor_get_uint8(x_8, sizeof(void*)*6); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_9); -lean_ctor_set(x_13, 1, x_11); -lean_inc(x_13); -lean_inc(x_6); -x_14 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2(x_6, x_13); -if (lean_obj_tag(x_14) == 0) +x_12 = lean_ctor_get(x_9, 2); +lean_inc(x_12); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_10); +lean_ctor_set(x_15, 1, x_14); +lean_inc(x_15); +lean_inc(x_7); +x_16 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2(x_7, x_15); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_15; size_t x_16; size_t x_17; -lean_dec(x_10); -x_15 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_6, x_13, x_8); -x_16 = 1; -x_17 = lean_usize_add(x_5, x_16); -x_5 = x_17; -x_6 = x_15; +lean_object* x_17; size_t x_18; size_t x_19; +lean_dec(x_11); +x_17 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_7, x_15, x_9); +x_18 = 1; +x_19 = lean_usize_add(x_6, x_18); +x_6 = x_19; +x_7 = x_17; goto _start; } else { -lean_object* x_19; uint8_t x_20; -lean_dec(x_8); -x_19 = lean_ctor_get(x_14, 0); -lean_inc(x_19); -lean_dec(x_14); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) -{ -lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_19, 1); -x_22 = lean_ctor_get_uint8(x_19, sizeof(void*)*6); -x_23 = l_Array_append___rarg(x_21, x_10); +lean_object* x_21; uint8_t x_22; +lean_dec(x_9); +x_21 = lean_ctor_get(x_16, 0); +lean_inc(x_21); +lean_dec(x_16); +x_22 = !lean_is_exclusive(x_21); if (x_22 == 0) { -lean_object* x_24; size_t x_25; size_t x_26; -lean_ctor_set(x_19, 1, x_23); -lean_ctor_set_uint8(x_19, sizeof(void*)*6, x_12); -x_24 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_6, x_13, x_19); -x_25 = 1; -x_26 = lean_usize_add(x_5, x_25); -x_5 = x_26; -x_6 = x_24; +lean_object* x_23; lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; +x_23 = lean_ctor_get(x_21, 1); +x_24 = l_Array_append___rarg(x_23, x_11); +lean_ctor_set(x_21, 1, x_24); +x_25 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_7, x_15, x_21); +x_26 = 1; +x_27 = lean_usize_add(x_6, x_26); +x_6 = x_27; +x_7 = x_25; goto _start; } else { -uint8_t x_28; lean_object* x_29; size_t x_30; size_t x_31; -x_28 = 1; -lean_ctor_set(x_19, 1, x_23); -lean_ctor_set_uint8(x_19, sizeof(void*)*6, x_28); -x_29 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_6, x_13, x_19); -x_30 = 1; -x_31 = lean_usize_add(x_5, x_30); -x_5 = x_31; -x_6 = x_29; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; size_t x_39; size_t x_40; +x_29 = lean_ctor_get(x_21, 0); +x_30 = lean_ctor_get(x_21, 1); +x_31 = lean_ctor_get(x_21, 2); +x_32 = lean_ctor_get(x_21, 3); +x_33 = lean_ctor_get(x_21, 4); +x_34 = lean_ctor_get(x_21, 5); +x_35 = lean_ctor_get_uint8(x_21, sizeof(void*)*6); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_21); +x_36 = l_Array_append___rarg(x_30, x_11); +x_37 = lean_alloc_ctor(0, 6, 1); +lean_ctor_set(x_37, 0, x_29); +lean_ctor_set(x_37, 1, x_36); +lean_ctor_set(x_37, 2, x_31); +lean_ctor_set(x_37, 3, x_32); +lean_ctor_set(x_37, 4, x_33); +lean_ctor_set(x_37, 5, x_34); +lean_ctor_set_uint8(x_37, sizeof(void*)*6, x_35); +x_38 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_7, x_15, x_37); +x_39 = 1; +x_40 = lean_usize_add(x_6, x_39); +x_6 = x_40; +x_7 = x_38; goto _start; } } +} else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; -x_33 = lean_ctor_get(x_19, 0); -x_34 = lean_ctor_get(x_19, 1); -x_35 = lean_ctor_get(x_19, 2); -x_36 = lean_ctor_get(x_19, 3); -x_37 = lean_ctor_get(x_19, 4); -x_38 = lean_ctor_get(x_19, 5); -x_39 = lean_ctor_get_uint8(x_19, sizeof(void*)*6); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_19); -x_40 = l_Array_append___rarg(x_34, x_10); -if (x_39 == 0) +lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_42 = lean_ctor_get(x_9, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_9, 1); +lean_inc(x_43); +x_44 = lean_ctor_get(x_9, 2); +lean_inc(x_44); +x_45 = lean_ctor_get_uint8(x_9, sizeof(void*)*6); +x_46 = lean_box(x_45); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_44); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_42); +lean_ctor_set(x_49, 1, x_48); +lean_inc(x_49); +lean_inc(x_7); +x_50 = l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2(x_7, x_49); +if (lean_obj_tag(x_50) == 0) { -lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; -x_41 = lean_alloc_ctor(0, 6, 1); -lean_ctor_set(x_41, 0, x_33); -lean_ctor_set(x_41, 1, x_40); -lean_ctor_set(x_41, 2, x_35); -lean_ctor_set(x_41, 3, x_36); -lean_ctor_set(x_41, 4, x_37); -lean_ctor_set(x_41, 5, x_38); -lean_ctor_set_uint8(x_41, sizeof(void*)*6, x_12); -x_42 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_6, x_13, x_41); -x_43 = 1; -x_44 = lean_usize_add(x_5, x_43); -x_5 = x_44; -x_6 = x_42; +lean_object* x_51; size_t x_52; size_t x_53; +lean_dec(x_43); +x_51 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_7, x_49, x_9); +x_52 = 1; +x_53 = lean_usize_add(x_6, x_52); +x_6 = x_53; +x_7 = x_51; +goto _start; +} +else +{ +lean_object* x_55; uint8_t x_56; +lean_dec(x_9); +x_55 = lean_ctor_get(x_50, 0); +lean_inc(x_55); +lean_dec(x_50); +x_56 = !lean_is_exclusive(x_55); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; +x_57 = lean_ctor_get(x_55, 1); +x_58 = l_Array_append___rarg(x_57, x_43); +lean_ctor_set(x_55, 1, x_58); +x_59 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_7, x_49, x_55); +x_60 = 1; +x_61 = lean_usize_add(x_6, x_60); +x_6 = x_61; +x_7 = x_59; goto _start; } else { -uint8_t x_46; lean_object* x_47; lean_object* x_48; size_t x_49; size_t x_50; -x_46 = 1; -x_47 = lean_alloc_ctor(0, 6, 1); -lean_ctor_set(x_47, 0, x_33); -lean_ctor_set(x_47, 1, x_40); -lean_ctor_set(x_47, 2, x_35); -lean_ctor_set(x_47, 3, x_36); -lean_ctor_set(x_47, 4, x_37); -lean_ctor_set(x_47, 5, x_38); -lean_ctor_set_uint8(x_47, sizeof(void*)*6, x_46); -x_48 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_6, x_13, x_47); -x_49 = 1; -x_50 = lean_usize_add(x_5, x_49); -x_5 = x_50; -x_6 = x_48; +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; size_t x_73; size_t x_74; +x_63 = lean_ctor_get(x_55, 0); +x_64 = lean_ctor_get(x_55, 1); +x_65 = lean_ctor_get(x_55, 2); +x_66 = lean_ctor_get(x_55, 3); +x_67 = lean_ctor_get(x_55, 4); +x_68 = lean_ctor_get(x_55, 5); +x_69 = lean_ctor_get_uint8(x_55, sizeof(void*)*6); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +lean_inc(x_65); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_55); +x_70 = l_Array_append___rarg(x_64, x_43); +x_71 = lean_alloc_ctor(0, 6, 1); +lean_ctor_set(x_71, 0, x_63); +lean_ctor_set(x_71, 1, x_70); +lean_ctor_set(x_71, 2, x_65); +lean_ctor_set(x_71, 3, x_66); +lean_ctor_set(x_71, 4, x_67); +lean_ctor_set(x_71, 5, x_68); +lean_ctor_set_uint8(x_71, sizeof(void*)*6, x_69); +x_72 = l_Std_HashMap_insert___at_Lean_Server_dedupReferences___spec__4(x_7, x_49, x_71); +x_73 = 1; +x_74 = lean_usize_add(x_6, x_73); +x_6 = x_74; +x_7 = x_72; goto _start; } } @@ -5557,11 +5810,63 @@ return x_4; } } } +LEAN_EXPORT uint8_t l_Lean_Server_dedupReferences___lambda__1(uint8_t x_1, uint8_t x_2) { +_start: +{ +if (x_1 == 0) +{ +if (x_2 == 0) +{ +uint8_t x_3; +x_3 = 1; +return x_3; +} +else +{ +uint8_t x_4; +x_4 = 0; +return x_4; +} +} +else +{ +return x_2; +} +} +} static lean_object* _init_l_Lean_Server_dedupReferences___closed__1() { _start: { +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Server_dedupReferences___lambda__1___boxed), 2, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_dedupReferences___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Server_dedupReferences___closed__1; +x_2 = lean_alloc_closure((void*)(l_instBEq___rarg), 3, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Server_dedupReferences___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Server_dedupReferences___closed__2; +x_2 = lean_alloc_closure((void*)(l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____rarg), 3, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Server_dedupReferences___closed__4() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Lsp_instBEqRefIdent; +x_1 = l_Lean_Server_dedupReferences___closed__3; x_2 = l_Lean_Lsp_instBEqRange; x_3 = lean_alloc_closure((void*)(l_instBEqProd___rarg), 4, 2); lean_closure_set(x_3, 0, x_1); @@ -5569,11 +5874,41 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_dedupReferences___closed__2() { +static lean_object* _init_l_Lean_Server_dedupReferences___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Lsp_instHashableRefIdent; +x_1 = l_Lean_Lsp_instBEqRefIdent; +x_2 = l_Lean_Server_dedupReferences___closed__4; +x_3 = lean_alloc_closure((void*)(l_instBEqProd___rarg), 4, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Server_dedupReferences___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_instHashableBool___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_dedupReferences___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Server_dedupReferences___closed__6; +x_2 = lean_alloc_closure((void*)(l_instHashableOption___rarg___boxed), 2, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Server_dedupReferences___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Server_dedupReferences___closed__7; x_2 = l_Lean_Lsp_instHashableRange; x_3 = lean_alloc_closure((void*)(l_instHashableProd___rarg___boxed), 3, 2); lean_closure_set(x_3, 0, x_1); @@ -5581,7 +5916,19 @@ lean_closure_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_dedupReferences___closed__3() { +static lean_object* _init_l_Lean_Server_dedupReferences___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Lsp_instHashableRefIdent; +x_2 = l_Lean_Server_dedupReferences___closed__8; +x_3 = lean_alloc_closure((void*)(l_instHashableProd___rarg___boxed), 3, 2); +lean_closure_set(x_3, 0, x_1); +lean_closure_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Server_dedupReferences___closed__10() { _start: { lean_object* x_1; lean_object* x_2; @@ -5590,77 +5937,77 @@ x_2 = lean_array_get_size(x_1); return x_2; } } -static lean_object* _init_l_Lean_Server_dedupReferences___closed__4() { +static lean_object* _init_l_Lean_Server_dedupReferences___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Server_dedupReferences___closed__3; +x_1 = l_Lean_Server_dedupReferences___closed__10; x_2 = lean_unsigned_to_nat(1u); x_3 = lean_nat_sub(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences(lean_object* x_1, uint8_t x_2) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Std_mkHashMapImp___rarg(x_2); -x_4 = lean_array_get_size(x_1); -x_5 = lean_usize_of_nat(x_4); -lean_dec(x_4); -x_6 = 0; -x_7 = l_Lean_Server_dedupReferences___closed__1; -x_8 = l_Lean_Server_dedupReferences___closed__2; -x_9 = l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11(x_7, x_8, x_1, x_5, x_6, x_3); +lean_object* x_3; lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Std_mkHashMapImp___rarg(x_3); +x_5 = lean_array_get_size(x_1); +x_6 = lean_usize_of_nat(x_5); +lean_dec(x_5); +x_7 = 0; +x_8 = l_Lean_Server_dedupReferences___closed__5; +x_9 = l_Lean_Server_dedupReferences___closed__9; +x_10 = l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11(x_2, x_8, x_9, x_1, x_6, x_7, x_4); lean_dec(x_1); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_array_get_size(x_10); -x_12 = lean_nat_dec_lt(x_2, x_11); -if (x_12 == 0) +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_array_get_size(x_11); +x_13 = lean_nat_dec_lt(x_3, x_12); +if (x_13 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); -x_13 = l_Lean_Server_instInhabitedReference; -x_14 = l_Lean_Server_Reference_aliases___default___closed__1; -x_15 = l_Lean_Server_dedupReferences___closed__4; -x_16 = l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13(x_13, x_14, x_2, x_15); -return x_16; +x_14 = l_Lean_Server_instInhabitedReference; +x_15 = l_Lean_Server_Reference_aliases___default___closed__1; +x_16 = l_Lean_Server_dedupReferences___closed__11; +x_17 = l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13(x_14, x_15, x_3, x_16); +return x_17; } else { -uint8_t x_17; -x_17 = lean_nat_dec_le(x_11, x_11); -if (x_17 == 0) +uint8_t x_18; +x_18 = lean_nat_dec_le(x_12, x_12); +if (x_18 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); -x_18 = l_Lean_Server_instInhabitedReference; -x_19 = l_Lean_Server_Reference_aliases___default___closed__1; -x_20 = l_Lean_Server_dedupReferences___closed__4; -x_21 = l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13(x_18, x_19, x_2, x_20); -return x_21; +x_19 = l_Lean_Server_instInhabitedReference; +x_20 = l_Lean_Server_Reference_aliases___default___closed__1; +x_21 = l_Lean_Server_dedupReferences___closed__11; +x_22 = l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13(x_19, x_20, x_3, x_21); +return x_22; } else { -size_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_22 = lean_usize_of_nat(x_11); +size_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_23 = lean_usize_of_nat(x_12); +lean_dec(x_12); +x_24 = l_Lean_Server_Reference_aliases___default___closed__1; +x_25 = l_Array_foldlMUnsafe_fold___at_Lean_Server_dedupReferences___spec__14(x_11, x_7, x_23, x_24); lean_dec(x_11); -x_23 = l_Lean_Server_Reference_aliases___default___closed__1; -x_24 = l_Array_foldlMUnsafe_fold___at_Lean_Server_dedupReferences___spec__14(x_10, x_6, x_22, x_23); -lean_dec(x_10); -x_25 = lean_array_get_size(x_24); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_nat_sub(x_25, x_26); -lean_dec(x_25); -x_28 = l_Lean_Server_instInhabitedReference; -x_29 = l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13(x_28, x_24, x_2, x_27); -lean_dec(x_27); -return x_29; +x_26 = lean_array_get_size(x_25); +x_27 = lean_unsigned_to_nat(1u); +x_28 = lean_nat_sub(x_26, x_27); +lean_dec(x_26); +x_29 = l_Lean_Server_instInhabitedReference; +x_30 = l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13(x_29, x_25, x_3, x_28); +lean_dec(x_28); +return x_30; } } } @@ -5695,19 +6042,21 @@ x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -size_t x_7; size_t x_8; lean_object* x_9; -x_7 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_8 = lean_unbox_usize(x_5); +uint8_t x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_8 = lean_unbox(x_1); +lean_dec(x_1); +x_9 = lean_unbox_usize(x_5); lean_dec(x_5); -x_9 = l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11(x_1, x_2, x_3, x_7, x_8, x_6); +x_10 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_dedupReferences___spec__11(x_8, x_2, x_3, x_4, x_9, x_10, x_7); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -return x_9; +return x_11; } } LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { @@ -5741,6 +6090,29 @@ lean_dec(x_1); return x_7; } } +LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; +x_3 = lean_unbox(x_1); +lean_dec(x_1); +x_4 = lean_unbox(x_2); +lean_dec(x_2); +x_5 = l_Lean_Server_dedupReferences___lambda__1(x_3, x_4); +x_6 = lean_box(x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_dedupReferences___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = lean_unbox(x_2); +lean_dec(x_2); +x_4 = l_Lean_Server_dedupReferences(x_1, x_3); +return x_4; +} +} LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_findModuleRefs___spec__1(lean_object* x_1) { _start: { @@ -5861,61 +6233,61 @@ x_4 = lean_apply_2(x_1, x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs(lean_object* x_1, lean_object* x_2, uint8_t x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = l_Lean_Server_findReferences(x_1, x_2); -x_5 = l_Lean_Server_combineFvars(x_4); -x_6 = l_Lean_Server_dedupReferences(x_5); -x_7 = l_Lean_Server_findModuleRefs___closed__1; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = l_Lean_Server_findReferences(x_1, x_2); +x_6 = l_Lean_Server_combineFvars(x_5); +x_7 = l_Lean_Server_dedupReferences(x_6, x_4); +x_8 = l_Lean_Server_findModuleRefs___closed__1; if (x_3 == 0) { -lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_array_get_size(x_6); -x_9 = lean_unsigned_to_nat(0u); -x_10 = lean_nat_dec_lt(x_9, x_8); -if (x_10 == 0) +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_array_get_size(x_7); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_lt(x_10, x_9); +if (x_11 == 0) { -lean_object* x_11; -lean_dec(x_8); -lean_dec(x_6); -x_11 = l_Lean_Server_findModuleRefs___closed__2; -return x_11; +lean_object* x_12; +lean_dec(x_9); +lean_dec(x_7); +x_12 = l_Lean_Server_findModuleRefs___closed__2; +return x_12; } else { -uint8_t x_12; -x_12 = lean_nat_dec_le(x_8, x_8); -if (x_12 == 0) +uint8_t x_13; +x_13 = lean_nat_dec_le(x_9, x_9); +if (x_13 == 0) { -lean_object* x_13; -lean_dec(x_8); -lean_dec(x_6); -x_13 = l_Lean_Server_findModuleRefs___closed__2; -return x_13; +lean_object* x_14; +lean_dec(x_9); +lean_dec(x_7); +x_14 = l_Lean_Server_findModuleRefs___closed__2; +return x_14; } else { -size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = 0; -x_15 = lean_usize_of_nat(x_8); -lean_dec(x_8); -x_16 = l_Lean_Server_Reference_aliases___default___closed__1; -x_17 = l_Array_foldlMUnsafe_fold___at_Lean_Server_findModuleRefs___spec__3(x_6, x_14, x_15, x_16); -lean_dec(x_6); -x_18 = lean_box(0); -x_19 = lean_apply_2(x_7, x_17, x_18); -return x_19; +size_t x_15; size_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = 0; +x_16 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_17 = l_Lean_Server_Reference_aliases___default___closed__1; +x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Server_findModuleRefs___spec__3(x_7, x_15, x_16, x_17); +lean_dec(x_7); +x_19 = lean_box(0); +x_20 = lean_apply_2(x_8, x_18, x_19); +return x_20; } } } else { -lean_object* x_20; lean_object* x_21; -x_20 = lean_box(0); -x_21 = lean_apply_2(x_7, x_6, x_20); -return x_21; +lean_object* x_21; lean_object* x_22; +x_21 = lean_box(0); +x_22 = lean_apply_2(x_8, x_7, x_21); +return x_22; } } } @@ -5963,15 +6335,17 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_findModuleRefs___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 = lean_unbox(x_3); +uint8_t x_5; uint8_t x_6; lean_object* x_7; +x_5 = lean_unbox(x_3); lean_dec(x_3); -x_5 = l_Lean_Server_findModuleRefs(x_1, x_2, x_4); +x_6 = lean_unbox(x_4); +lean_dec(x_4); +x_7 = l_Lean_Server_findModuleRefs(x_1, x_2, x_5, x_6); lean_dec(x_2); -return x_5; +return x_7; } } LEAN_EXPORT lean_object* l_Std_mkHashMap___at_Lean_Server_References_empty___spec__1(lean_object* x_1) { @@ -11443,6 +11817,8 @@ l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__1___lambda__2__ lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Server_findReferences___spec__1___lambda__2___closed__2); l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__20___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__20___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Server_combineFvars___spec__20___closed__1); +l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__1 = _init_l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__1(); +l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__2 = _init_l_Std_HashMapImp_find_x3f___at_Lean_Server_dedupReferences___spec__2___closed__2(); l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13___closed__1 = _init_l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13___closed__1(); lean_mark_persistent(l_Array_qsort_sort___at_Lean_Server_dedupReferences___spec__13___closed__1); l_Lean_Server_dedupReferences___closed__1 = _init_l_Lean_Server_dedupReferences___closed__1(); @@ -11453,6 +11829,20 @@ l_Lean_Server_dedupReferences___closed__3 = _init_l_Lean_Server_dedupReferences_ lean_mark_persistent(l_Lean_Server_dedupReferences___closed__3); l_Lean_Server_dedupReferences___closed__4 = _init_l_Lean_Server_dedupReferences___closed__4(); lean_mark_persistent(l_Lean_Server_dedupReferences___closed__4); +l_Lean_Server_dedupReferences___closed__5 = _init_l_Lean_Server_dedupReferences___closed__5(); +lean_mark_persistent(l_Lean_Server_dedupReferences___closed__5); +l_Lean_Server_dedupReferences___closed__6 = _init_l_Lean_Server_dedupReferences___closed__6(); +lean_mark_persistent(l_Lean_Server_dedupReferences___closed__6); +l_Lean_Server_dedupReferences___closed__7 = _init_l_Lean_Server_dedupReferences___closed__7(); +lean_mark_persistent(l_Lean_Server_dedupReferences___closed__7); +l_Lean_Server_dedupReferences___closed__8 = _init_l_Lean_Server_dedupReferences___closed__8(); +lean_mark_persistent(l_Lean_Server_dedupReferences___closed__8); +l_Lean_Server_dedupReferences___closed__9 = _init_l_Lean_Server_dedupReferences___closed__9(); +lean_mark_persistent(l_Lean_Server_dedupReferences___closed__9); +l_Lean_Server_dedupReferences___closed__10 = _init_l_Lean_Server_dedupReferences___closed__10(); +lean_mark_persistent(l_Lean_Server_dedupReferences___closed__10); +l_Lean_Server_dedupReferences___closed__11 = _init_l_Lean_Server_dedupReferences___closed__11(); +lean_mark_persistent(l_Lean_Server_dedupReferences___closed__11); l_Lean_Server_findModuleRefs___closed__1 = _init_l_Lean_Server_findModuleRefs___closed__1(); lean_mark_persistent(l_Lean_Server_findModuleRefs___closed__1); l_Lean_Server_findModuleRefs___closed__2 = _init_l_Lean_Server_findModuleRefs___closed__2(); diff --git a/stage0/stdlib/Lean/Server/Requests.c b/stage0/stdlib/Lean/Server/Requests.c index d5e5f25a45c5..67c4fa71962a 100644 --- a/stage0/stdlib/Lean/Server/Requests.c +++ b/stage0/stdlib/Lean/Server/Requests.c @@ -13,6 +13,7 @@ #ifdef __cplusplus extern "C" { #endif +lean_object* l_Lean_initializing(lean_object*); static lean_object* l_Lean_Server_handleLspRequest___closed__1; size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -124,7 +125,6 @@ lean_object* l_instBEq___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RequestM_withWaitFindSnap___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RequestM_readDoc___boxed(lean_object*, lean_object*); -lean_object* lean_io_initializing(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RequestM_bindWaitFindSnap(lean_object*); static lean_object* l_Lean_Server_parseRequestParams___rarg___closed__3; static lean_object* l_Lean_Server_chainLspRequestHandler___lambda__1___closed__2; @@ -2122,7 +2122,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler(lean_object* x_ _start: { lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_io_initializing(x_8); +x_9 = l_Lean_initializing(x_8); x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); x_11 = lean_unbox(x_10); @@ -2905,7 +2905,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_chainLspRequestHandler(lean_object* x_1, _start: { lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_9 = lean_io_initializing(x_8); +x_9 = l_Lean_initializing(x_8); x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); x_11 = lean_unbox(x_10); diff --git a/stage0/stdlib/Lean/Server/Rpc/Basic.c b/stage0/stdlib/Lean/Server/Rpc/Basic.c index 931ff1e89c28..ba6e7234a698 100644 --- a/stage0/stdlib/Lean/Server/Rpc/Basic.c +++ b/stage0/stdlib/Lean/Server/Rpc/Basic.c @@ -16,6 +16,7 @@ extern "C" { LEAN_EXPORT lean_object* l_Lean_Server_instInhabitedWithRpcRef___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instInhabitedWithRpcRef(lean_object*); size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingArray___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe(lean_object*); @@ -27,17 +28,16 @@ lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingArray___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instMonadRpcSession___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__4(lean_object*); lean_object* lean_array_get_size(lean_object*); -static lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__4___closed__1; lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instMonadRpcSession___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_instRpcEncoding___closed__3; LEAN_EXPORT lean_object* l_Lean_Server_instMonadRpcSession___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instInhabitedWithRpcRef___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingArray(lean_object*, lean_object*); static lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3___closed__5; @@ -45,12 +45,12 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncoding LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__1(lean_object*); static lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__3(lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingArray___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingArray___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_WithRpcRef_decodeUnsafeAs___spec__3(lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_WithRpcRef_decodeUnsafeAs___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t); @@ -58,45 +58,49 @@ LEAN_EXPORT lean_object* l_Lean_Server_instMonadRpcSession___rarg___lambda__2(le lean_object* l_Nat_repr(lean_object*); static lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instMonadRpcSession___rarg___lambda__3(lean_object*, lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3___closed__7; LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_WithRpcRef_decodeUnsafeAs___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instMonadRpcSession___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Array_mapMUnsafe_map___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___closed__1; LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_WithRpcRef_decodeUnsafeAs___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3___closed__3; LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg(lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instMonadRpcSession(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingArray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingArray___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingArray___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__1___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT uint8_t l_Lean_Server_RpcEncoding_DerivingParams_withRef___default; LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_WithRpcRef_decodeUnsafeAs___spec__1(lean_object*); static lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3___closed__6; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_WithRpcRef_decodeUnsafeAs___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_instRpcEncoding___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption(lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__4(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___boxed(lean_object*, lean_object*, lean_object*); @@ -194,20 +198,6 @@ return x_5; LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___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; -x_5 = lean_ctor_get(x_2, 0); -lean_inc(x_5); -lean_dec(x_2); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_apply_2(x_6, lean_box(0), x_4); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_5 = lean_ctor_get(x_2, 0); lean_inc(x_5); @@ -232,28 +222,19 @@ return x_1; static lean_object* _init_l_Lean_Server_instRpcEncoding___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncoding___lambda__2___boxed), 4, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Server_instRpcEncoding___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; +lean_object* x_1; lean_object* x_2; x_1 = l_Lean_Server_instRpcEncoding___closed__1; -x_2 = l_Lean_Server_instRpcEncoding___closed__2; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; } } LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_Lean_Server_instRpcEncoding___closed__3; +x_4 = l_Lean_Server_instRpcEncoding___closed__2; return x_4; } } @@ -266,15 +247,6 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Server_instRpcEncoding___lambda__2(x_1, x_2, x_3, x_4); -lean_dec(x_3); -return x_5; -} -} LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncoding___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { @@ -285,66 +257,7 @@ lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__1(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingOption___rarg___lambda__1), 1, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -if (lean_obj_tag(x_5) == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -lean_dec(x_4); -lean_dec(x_1); -x_6 = lean_ctor_get(x_3, 0); -lean_inc(x_6); -lean_dec(x_3); -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_box(0); -x_9 = lean_apply_2(x_7, lean_box(0), x_8); -return x_9; -} -else -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_3, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -lean_dec(x_12); -x_14 = lean_ctor_get(x_1, 0); -lean_inc(x_14); -lean_dec(x_1); -x_15 = lean_apply_4(x_14, lean_box(0), x_3, x_4, x_10); -x_16 = l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1; -x_17 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_16, x_15); -return x_17; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -423,7 +336,7 @@ return x_23; } } } -static lean_object* _init_l_Lean_Server_instRpcEncodingOption___rarg___lambda__4___closed__1() { +static lean_object* _init_l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -433,7 +346,45 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_dec(x_4); +lean_dec(x_1); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_dec(x_3); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1; +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +lean_inc(x_3); +x_12 = lean_apply_4(x_11, lean_box(0), x_3, x_4, x_10); +x_13 = lean_ctor_get(x_3, 1); +lean_inc(x_13); +x_14 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingOption___rarg___lambda__1), 2, 1); +lean_closure_set(x_14, 0, x_3); +x_15 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_12, x_14); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingOption___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -447,7 +398,7 @@ lean_dec(x_3); x_7 = lean_ctor_get(x_6, 1); lean_inc(x_7); lean_dec(x_6); -x_8 = l_Lean_Server_instRpcEncodingOption___rarg___lambda__4___closed__1; +x_8 = l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1; x_9 = lean_apply_2(x_7, lean_box(0), x_8); return x_9; } @@ -464,7 +415,7 @@ lean_inc(x_3); x_12 = lean_apply_4(x_11, lean_box(0), x_3, x_4, x_10); x_13 = lean_ctor_get(x_3, 1); lean_inc(x_13); -x_14 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingOption___rarg___lambda__3), 2, 1); +x_14 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingOption___rarg___lambda__1), 2, 1); lean_closure_set(x_14, 0, x_3); x_15 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_12, x_14); return x_15; @@ -478,7 +429,7 @@ lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_inc(x_1); x_2 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingOption___rarg___lambda__2), 5, 1); lean_closure_set(x_2, 0, x_1); -x_3 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingOption___rarg___lambda__4), 5, 1); +x_3 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingOption___rarg___lambda__3), 5, 1); lean_closure_set(x_3, 0, x_1); x_4 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_4, 0, x_2); @@ -624,21 +575,149 @@ x_4 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Server_instRpc return x_4; } } +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingArray___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingArray___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingArray___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; +x_8 = 1; +x_9 = lean_usize_add(x_1, x_8); +x_10 = lean_array_uset(x_2, x_1, x_7); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg(x_3, x_4, x_5, x_6, x_9, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_5, x_4); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_dec(x_3); +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_6); +x_11 = lean_apply_2(x_9, lean_box(0), x_10); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_12 = lean_array_uget(x_6, x_5); +x_13 = lean_unsigned_to_nat(0u); +x_14 = lean_array_uset(x_6, x_5, x_13); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_15 = lean_apply_4(x_3, lean_box(0), x_1, x_2, x_12); +x_16 = lean_box_usize(x_5); +x_17 = lean_box_usize(x_4); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___lambda__1___boxed), 7, 6); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_14); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_3); +lean_closure_set(x_18, 5, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingArray___spec__4___rarg), 5, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_15, x_20); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___boxed), 6, 0); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingArray___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; x_6 = lean_ctor_get(x_1, 0); lean_inc(x_6); lean_dec(x_1); -lean_inc(x_3); -x_7 = lean_apply_3(x_6, lean_box(0), x_3, x_4); -x_8 = lean_array_get_size(x_5); -x_9 = lean_usize_of_nat(x_8); -lean_dec(x_8); -x_10 = 0; -x_11 = l_Array_mapMUnsafe_map___rarg(x_3, x_7, x_9, x_10, x_5); -return x_11; +x_7 = lean_array_get_size(x_5); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +x_9 = 0; +x_10 = l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__1___rarg(x_3, x_4, x_6, x_8, x_9, x_5); +return x_10; } } LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingArray___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { @@ -652,7 +731,7 @@ x_7 = lean_array_get_size(x_5); x_8 = lean_usize_of_nat(x_7); lean_dec(x_7); x_9 = 0; -x_10 = l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__1___rarg(x_3, x_4, x_6, x_8, x_9, x_5); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg(x_3, x_4, x_6, x_8, x_9, x_5); return x_10; } } @@ -703,6 +782,30 @@ x_9 = l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__1___r return x_9; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; +x_8 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_9 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___lambda__1(x_8, x_2, x_3, x_4, x_5, x_9, x_7); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodingArray___spec__3___rarg(x_1, x_2, x_3, x_7, x_8, x_6); +return x_9; +} +} LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -819,68 +922,123 @@ x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Server_instRpcEnco return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; lean_dec(x_4); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_2); -lean_ctor_set(x_6, 1, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_1, 0); lean_inc(x_7); lean_dec(x_1); -lean_inc(x_2); -x_8 = lean_apply_4(x_7, lean_box(0), x_2, x_3, x_4); -x_9 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__1), 3, 2); -lean_closure_set(x_9, 0, x_2); -lean_closure_set(x_9, 1, x_6); -x_10 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_8, x_9); -return x_10; +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__3(lean_object* x_1) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_6, 0); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__3___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); lean_inc(x_7); -x_8 = lean_ctor_get(x_6, 1); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_ctor_get(x_4, 1); -lean_inc(x_9); -x_10 = lean_ctor_get(x_1, 0); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -lean_inc(x_5); -lean_inc(x_4); -x_11 = lean_apply_4(x_10, lean_box(0), x_4, x_5, x_7); -lean_inc(x_9); -x_12 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__2), 6, 5); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_4); -lean_closure_set(x_12, 2, x_5); -lean_closure_set(x_12, 3, x_8); -lean_closure_set(x_12, 4, x_9); -x_13 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_11, x_12); -return x_13; +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -899,17 +1057,17 @@ x_8 = lean_apply_2(x_6, lean_box(0), x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_6 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_1, 0); lean_inc(x_6); lean_dec(x_1); lean_inc(x_2); x_7 = lean_apply_4(x_6, lean_box(0), x_2, x_3, x_4); lean_inc(x_2); -x_8 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__4), 3, 2); +x_8 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__1), 3, 2); lean_closure_set(x_8, 0, x_5); lean_closure_set(x_8, 1, x_2); x_9 = lean_ctor_get(x_2, 1); @@ -923,7 +1081,7 @@ x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; @@ -932,14 +1090,14 @@ lean_inc(x_7); x_8 = lean_ctor_get(x_6, 1); lean_inc(x_8); lean_dec(x_6); -x_9 = lean_ctor_get(x_1, 1); +x_9 = lean_ctor_get(x_1, 0); lean_inc(x_9); lean_dec(x_1); lean_inc(x_5); lean_inc(x_4); x_10 = lean_apply_4(x_9, lean_box(0), x_4, x_5, x_7); lean_inc(x_4); -x_11 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__5), 5, 4); +x_11 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__2), 5, 4); lean_closure_set(x_11, 0, x_2); lean_closure_set(x_11, 1, x_4); lean_closure_set(x_11, 2, x_5); @@ -955,6 +1113,62 @@ x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); return x_14; } } +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +lean_dec(x_1); +lean_inc(x_2); +x_7 = lean_apply_4(x_6, lean_box(0), x_2, x_3, x_4); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__1), 3, 2); +lean_closure_set(x_8, 0, x_5); +lean_closure_set(x_8, 1, x_2); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__3___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +lean_dec(x_1); +lean_inc(x_5); +lean_inc(x_4); +x_10 = lean_apply_4(x_9, lean_box(0), x_4, x_5, x_7); +lean_inc(x_4); +x_11 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__4), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, x_4); +lean_closure_set(x_11, 2, x_5); +lean_closure_set(x_11, 3, x_8); +x_12 = lean_ctor_get(x_4, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Server_instRpcEncodingProd___spec__4___rarg), 5, 4); +lean_closure_set(x_13, 0, x_4); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} LEAN_EXPORT lean_object* l_Lean_Server_instRpcEncodingProd___rarg(lean_object* x_1, lean_object* x_2) { _start: { @@ -964,7 +1178,7 @@ lean_inc(x_1); x_3 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__3), 6, 2); lean_closure_set(x_3, 0, x_1); lean_closure_set(x_3, 1, x_2); -x_4 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__6), 6, 2); +x_4 = lean_alloc_closure((void*)(l_Lean_Server_instRpcEncodingProd___rarg___lambda__5), 6, 2); lean_closure_set(x_4, 0, x_1); lean_closure_set(x_4, 1, x_2); x_5 = lean_alloc_ctor(0, 2, 0); @@ -1492,12 +1706,8 @@ l_Lean_Server_instRpcEncoding___closed__1 = _init_l_Lean_Server_instRpcEncoding_ lean_mark_persistent(l_Lean_Server_instRpcEncoding___closed__1); l_Lean_Server_instRpcEncoding___closed__2 = _init_l_Lean_Server_instRpcEncoding___closed__2(); lean_mark_persistent(l_Lean_Server_instRpcEncoding___closed__2); -l_Lean_Server_instRpcEncoding___closed__3 = _init_l_Lean_Server_instRpcEncoding___closed__3(); -lean_mark_persistent(l_Lean_Server_instRpcEncoding___closed__3); l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1 = _init_l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Server_instRpcEncodingOption___rarg___lambda__2___closed__1); -l_Lean_Server_instRpcEncodingOption___rarg___lambda__4___closed__1 = _init_l_Lean_Server_instRpcEncodingOption___rarg___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Server_instRpcEncodingOption___rarg___lambda__4___closed__1); l_Lean_Server_RpcEncoding_DerivingParams_withRef___default = _init_l_Lean_Server_RpcEncoding_DerivingParams_withRef___default(); l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3___closed__1 = _init_l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg___lambda__3___closed__1); diff --git a/stage0/stdlib/Lean/Server/Rpc/Deriving.c b/stage0/stdlib/Lean/Server/Rpc/Deriving.c index 3ed01f73ccaa..28d0e1625c63 100644 --- a/stage0/stdlib/Lean/Server/Rpc/Deriving.c +++ b/stage0/stdlib/Lean/Server/Rpc/Deriving.c @@ -13,104 +13,70 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__3; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__8; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__17; -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__17; +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9(lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__11; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__69; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__237; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__21(lean_object*, lean_object*, size_t, size_t); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__20(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53; -lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_shouldVisit(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__151; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4; -lean_object* l_panic___at_Lean_Meta_DiscrTree_insertCore___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11(lean_object*); lean_object* l_Lean_registerTraceClass(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__55; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__4; lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__27(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__37; lean_object* l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207; -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__18(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__101; -lean_object* lean_nat_div(lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__9; -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__34___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Elab_elabDeriving___spec__14(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__20; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238; -lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__3; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__10; +lean_object* l_Lean_addDecl___at_Lean_Elab_Term_declareTacticSyntax___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__36(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__172; lean_object* l_Lean_Elab_Command_liftTermElabM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__169; -uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__19(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__22(lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__20; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__6; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__124; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__2; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__32; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__10; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_decodes___default; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__148; -static lean_object* l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__43; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__1; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__22; +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__244; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__46(lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__138; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__1; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__79; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__3; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__2; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___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*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__37; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__65; -static lean_object* l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944____closed__1; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); @@ -118,749 +84,531 @@ static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncod LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__140; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__18; -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__17___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__15; -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206; -uint8_t l_Lean_Syntax_structEq(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4(size_t, size_t, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__15; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__204; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__13(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*); -size_t lean_usize_sub(size_t, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__18; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__156; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__10; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__77; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__56; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__102; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__6; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__90; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__2; lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Command_mkDefViewOfInstance___spec__11(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; lean_object* lean_st_ref_get(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__3; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__39(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__85; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__128; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__38(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231; -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__192; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__71; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__7; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__126; -uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__73; static lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___closed__2; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__5; -LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__20(lean_object*, lean_object*); -lean_object* l_Lean_Meta_DiscrTree_instInhabitedDiscrTree(lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___boxed(lean_object*, lean_object*, lean_object*); -static size_t l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__1; +lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__2; LEAN_EXPORT lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__246; -LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__19(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__37; lean_object* lean_array_get_size(lean_object*); -lean_object* l_Std_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__240; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__6; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__81; +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__23(lean_object*, lean_object*, size_t, size_t); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__7; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; lean_object* l_Lean_MessageData_ofList(lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__3___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__120; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__32; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__10; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__174; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__2; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__1; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__215; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__98; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__7; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__165; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__5; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__29(lean_object*, lean_object*, size_t, size_t); -lean_object* l_Std_mkHashSetImp___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); -size_t lean_usize_shift_right(size_t, size_t); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__5; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__212; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__81; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__73; lean_object* lean_string_utf8_byte_size(lean_object*); -lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__26(lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__219; -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_instInhabitedCtorState; -lean_object* l_Lean_Elab_Term_instInhabitedTermElabM(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__136; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__196; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__37___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__75; lean_object* l_Lean_Meta_inferType___boxed(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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__114; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -lean_object* l_Array_back_x3f___rarg(lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__161; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__127; -lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__88; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__41; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__34; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__25; +lean_object* l_Lean_setEnv___at_Lean_Elab_Term_expandDeclId___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72; lean_object* l_Array_zip___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__167; -LEAN_EXPORT uint8_t l_Array_contains___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__133; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAppN(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__29(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241; -size_t lean_uint64_to_usize(uint64_t); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__1; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__12; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__48; -uint8_t l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__121; -LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__20___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__28; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___closed__1; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__22(lean_object*, lean_object*, size_t, size_t); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__22; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__1; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__3; lean_object* l_Lean_Syntax_mkApp(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__54; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__2; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__132; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__103; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__137; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__84; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTRAux___at_Lean_MessageData_instCoeListExprMessageData___spec__1(lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__10; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__32; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__76; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__108; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__63; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__20; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__78; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__7; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__242; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__55; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_contains___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12___boxed(lean_object*, lean_object*); uint8_t l_instDecidableNot___rarg(uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__30; lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__2; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__208; -lean_object* lean_st_ref_take(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__42(lean_object*, lean_object*, size_t, size_t, lean_object*); -lean_object* l_Lean_Core_mkFreshUserName___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2(lean_object*, lean_object*, lean_object*); -lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__134; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__160; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__243; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__21; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__11; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__38; -lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___closed__4; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__214; -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__2; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__13; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__29; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__186; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; lean_object* l_Lean_getStructureFieldsFlattened(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__234; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__8; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__16; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__52; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6___boxed__const__1; lean_object* l_Lean_Elab_Term_elabTerm(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_mkFreshBinderName___at___private_Lean_Elab_Binders_0__Lean_Elab_Term_expandBinderIdent___spec__2___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__177; +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__4; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__24; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__202; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__164; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__43(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__36___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__158; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__13; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__106; -lean_object* l_Lean_Name_toString(lean_object*, uint8_t); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__21(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__78; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__40(lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__91; -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__49; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__123; -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__9; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; -LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__27___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__26(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__2; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__40; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1(lean_object*); -lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__6; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__1; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__54; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__84; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__22; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__110; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__5; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__5; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8; static lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__33___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__36; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__91; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__154; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(lean_object*, size_t, size_t, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__28(lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__1; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__153; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__6; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2(lean_object*); -static lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__7; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__71; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__63; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__6; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__2; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__2; lean_object* l_Lean_Meta_evalExpr_x27___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__62; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__166; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__16; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1; +lean_object* l_Lean_Syntax_getId(lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_String_endsWith(lean_object*, lean_object*); -static lean_object* l_Lean_Server_RpcEncoding_instInhabitedCtorState___closed__1; -lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; lean_object* l_Array_back___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__77; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__185; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__149; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___rarg___lambda__1(lean_object*, lean_object*); lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__66; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56; lean_object* l_Lean_addMessageContextPartial___at_Lean_Elab_Command_instAddMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__25; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2; -size_t lean_usize_shift_left(size_t, size_t); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__4; lean_object* lean_array_to_list(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__86; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__105; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__4; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__27; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2(lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__181; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__125; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__30(lean_object*, lean_object*, size_t, size_t); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35(size_t, size_t, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__4; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__19; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__51; -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__210; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__217; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__65; -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__30; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___closed__2; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__10; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__155; lean_object* l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__182; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__200; static lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__130; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Array_reverse___rarg(lean_object*); -uint8_t l_Array_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__37(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__28; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__76; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__176; -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__5; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__5; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__14; lean_object* l_Lean_mkSepArray(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35; lean_object* l_Lean_Elab_Command_elabCommand(lean_object*, lean_object*, lean_object*, lean_object*); -size_t lean_usize_mul(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__41___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__6; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__1; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__7; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__36; -LEAN_EXPORT uint8_t l_Lean_Server_RpcEncoding_isOptField(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__171; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__89; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__3; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__30; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__33; +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__157; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__4; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__2; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__2; -lean_object* l_Lean_Elab_Command_liftCoreM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__44(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__2; size_t lean_usize_of_nat(lean_object*); -lean_object* l_Lean_getExprMVarAssignment_x3f___at_Lean_exprDependsOn___spec__4(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__34(lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__162; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__3; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__39; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__239; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__111; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__48; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__193; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__31; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -size_t lean_usize_land(size_t, size_t); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__15; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(lean_object*, size_t, size_t, lean_object*, lean_object*); -lean_object* l_Lean_LocalDecl_fvarId(lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__3; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__191; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__141; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__226; -lean_object* l_Lean_Meta_DiscrTree_mkPath(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__5; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__3; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__3; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__163; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__35; lean_object* l_Lean_Meta_mkProjection(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__53; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__3; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17(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_PrettyPrinter_delab(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__142; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__5; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__213; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__2; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__1; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__184; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__229; +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__29; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__152; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17; -uint8_t l_Array_contains___at___private_Lean_Meta_Match_Value_0__Lean_Meta_isUIntTypeName___spec__1(lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__5; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__2; lean_object* l_Lean_Name_getString_x21(lean_object*); lean_object* l_String_intercalate(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__3; uint8_t l_Lean_Expr_isType(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__44; +lean_object* l_Lean_Meta_synthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__19; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__57; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__46; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -extern lean_object* l_Lean_Meta_DiscrTree_instInhabitedKey; +lean_object* lean_name_append_after(lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__1; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__236; -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__6; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__178; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Term_matchAlt(lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__11; lean_object* lean_environment_main_module(lean_object*); -uint8_t lean_expr_eqv(lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__173; -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3; -uint8_t l_Lean_Expr_isMVar(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__1; +static lean_object* l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985____closed__1; lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Command_instAddErrorMessageContextCommandElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t lean_nat_dec_le(lean_object*, lean_object*); -uint8_t lean_usize_dec_le(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__64; lean_object* l_Lean_Elab_Command_getCurrMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; lean_object* l_Lean_Parser_categoryParser(lean_object*, lean_object*); -uint8_t l_Lean_Expr_hasMVar(lean_object*); static lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___closed__1; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__74; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5(lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__74; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__46___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__2; +lean_object* l_Lean_Name_append(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; static lean_object* l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___closed__3; lean_object* l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__197; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__64; lean_object* l_Lean_quoteNameMk(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23___closed__1; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__235; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__29; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__144; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_uniqEncArgTypes___default; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__6; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__4; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__80; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5(lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__41; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__97; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45(size_t, size_t, lean_object*); lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__150; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__9; -LEAN_EXPORT lean_object* l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__4; -static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__19___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__18___boxed(lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_Meta_DiscrTree_Key_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_getMainModule___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__198; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__8; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__8; -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__220; +lean_object* l_Array_ofSubarray___rarg(lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__26; lean_object* l_Lean_Elab_Command_getRef(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__195; lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__40___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__96; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__216; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__72; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__227; -lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__27(lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__28___boxed(lean_object*, lean_object*); -uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__12; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors(lean_object*); -static size_t l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(lean_object*, size_t, lean_object*); -extern lean_object* l_Lean_instInhabitedName; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_binders___default; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__188; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__168; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__179; -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__15(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___boxed(lean_object**); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__44___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__21; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__222; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__170; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__199; -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_isOptField___boxed(lean_object*); +lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__107; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__82; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; -lean_object* lean_panic_fn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__87; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; -static lean_object* l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__209; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_ctors___default; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__17(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__203; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__68; -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__33(lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__4; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__145; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__45; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__31; -lean_object* l_Lean_Meta_DiscrTree_getMatch___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___boxed(lean_object**); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__11; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__104; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2; lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Elab_Deriving_mkInductArgNames___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__183; +lean_object* l_Lean_Elab_Term_elabBinders___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__59; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__61; -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__5(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___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*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__82; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__70; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__41(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__94; -lean_object* l_Lean_indentD(lean_object*); -static lean_object* l_Lean_Server_RpcEncoding_isOptField___closed__1; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__1; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___rarg(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__36; lean_object* l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__3; lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__245; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3(lean_object*); lean_object* lean_mk_syntax_ident(lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__233; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(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_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__34; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__88; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__218; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__180; +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_name_append_before(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__14; -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___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___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_getAppFn(lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__139; +lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__26; -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5; -lean_object* l_Lean_instantiateMVars___at_Lean_exprDependsOn___spec__11(lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__201; -lean_object* l_Lean_MetavarContext_getDecl(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__38; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__21; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__57; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__129; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__4; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__131; -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__1; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__189; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__67; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__75; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__175; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__3; -static lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__1; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__7; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__23; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__113; -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__31(lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encArgTypes___default; -lean_object* lean_usize_to_nat(size_t); lean_object* l_Lean_Elab_registerBuiltinDerivingHandlerWithArgs(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__13; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__27; +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10___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*); extern lean_object* l_Lean_levelOne; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__43___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__24; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__143; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__42___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__11; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__87; -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(lean_object*, lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_Expr_hasFVar(lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__27; -static lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2; +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -lean_object* l_Array_insertAt___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__2; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__187; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__159; -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__26___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__6; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__45; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__70; -static lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encodes___default; -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205; -lean_object* l_Std_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); +static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__83; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__112; -uint64_t l_Lean_Meta_DiscrTree_Key_hash(lean_object*); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__19; -static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__12; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__146; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__9; lean_object* l_Lean_Meta_forallTelescopeReducing___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__25___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_DiscrTree_instInhabitedTrie(lean_object*); -static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__194; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__40; static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__24(lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__25(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985_(lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__4; +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5; uint8_t l_Lean_isStructure(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___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*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__122; -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; -lean_object* l_Std_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened(lean_object*); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__9; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__39___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); lean_object* l_Lean_Meta_getFVarLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3; LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4___boxed(lean_object*, lean_object*, lean_object*); static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__1() { _start: { @@ -937,7 +685,7 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("section", 7); +x_1 = lean_mk_string_from_bytes("declaration", 11); return x_1; } } @@ -954,19 +702,37 @@ return x_3; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("declModifiers", 13); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13() { +_start: +{ lean_object* x_1; lean_object* x_2; x_1 = lean_unsigned_to_nat(0u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -974,114 +740,96 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(2u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("variable", 8); +x_1 = lean_mk_string_from_bytes("unsafe", 6); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__16() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Term", 4); -return x_1; -} -} static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__6; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__16; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("implicitBinder", 14); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(6u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_3 = lean_array_push(x_1, x_2); return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__20() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("{", 1); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__19; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__21() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("m", 1); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__20; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__22() { _start: { -lean_object* x_1; lean_object* x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__21; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__21; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__22; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("def", 3); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__21; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -1089,52 +837,58 @@ return x_3; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("declId", 6); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(":", 1); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__27() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("arrow", 5); +x_1 = lean_mk_string_from_bytes("unsafeInst", 10); return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__28() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__27; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__27; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__29() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("type", 4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__27; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__28; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__30() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__29; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__27; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -1142,50 +896,53 @@ return x_3; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Type", 4); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(2u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__32() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("→", 3); +x_1 = lean_mk_string_from_bytes("optDeclSig", 10); return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(3u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__32; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("}", 1); +x_1 = lean_mk_string_from_bytes("Term", 4); return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(4u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__6; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__36() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declaration", 11); +x_1 = lean_mk_string_from_bytes("typeSpec", 8); return x_1; } } @@ -1193,7 +950,7 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__36; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -1203,147 +960,171 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declModifiers", 13); +x_1 = lean_mk_string_from_bytes(":", 1); return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("app", 3); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("unsafe", 6); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__41() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("RpcEncoding", 11); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(6u); -x_2 = lean_mk_empty_array_with_capacity(x_1); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__41; +x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__41; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_3 = lean_array_push(x_1, x_2); +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__41; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__45() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_3 = lean_array_push(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Server", 6); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__46() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__45; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_3 = lean_array_push(x_1, x_2); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__45; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("def", 3); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__46; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__41; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__48() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_1 = lean_box(0); x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__49() { _start: { +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__48; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50() { +_start: +{ lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declId", 6); +x_1 = lean_mk_string_from_bytes("paren", 5); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__49; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("encodeUnsafe", 12); +x_1 = lean_mk_string_from_bytes("(", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__53() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("WithRpcRef", 10); +return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__53() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__54() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__53; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__55() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__53; x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__54; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -1351,83 +1132,72 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__54() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__53; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__55() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("optDeclSig", 10); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__57() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__55; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__46; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__53; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__57() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("instBinder", 10); -return x_1; -} -} static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_1 = lean_box(0); x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__57; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("[", 1); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("app", 3); +x_1 = lean_mk_string_from_bytes(")", 1); return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(3u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__62() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Monad", 5); +x_1 = lean_mk_string_from_bytes("Lsp.RpcRef", 10); return x_1; } } @@ -1457,11 +1227,9 @@ return x_4; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__65() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__62; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Lsp", 3); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__66() { @@ -1470,61 +1238,58 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__65; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__67() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__66; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("RpcRef", 6); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("]", 1); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__66; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__67; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__69() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("MonadRpcSession", 15); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__65; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__70() { _start: { -lean_object* x_1; lean_object* x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__69; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__67; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__71() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__69; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__70; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__70; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__72() { @@ -1532,35 +1297,37 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__69; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__71; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__73() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Server", 6); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__74() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__73; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("whereStructInst", 15); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__75() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__74; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__69; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__74; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -1568,118 +1335,89 @@ return x_3; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__76() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__75; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("where", 5); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__77() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__76; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__78() { -_start: -{ lean_object* x_1; -x_1 = lean_mk_string_from_bytes("explicitBinder", 14); +x_1 = lean_mk_string_from_bytes("whereStructField", 16); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__78() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__78; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__77; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("(", 1); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__81() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("r", 1); +x_1 = lean_mk_string_from_bytes("letDecl", 7); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__82() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__81; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__81() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__81; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__82; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("letIdDecl", 9); +return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__84() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__82() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__81; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("WithRpcRef", 10); +x_1 = lean_mk_string_from_bytes("rpcEncode", 9); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__84() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__87() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__84; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -1687,109 +1425,82 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__88() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__89() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__87() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__74; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__88() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__89; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__87; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__91() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__89() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__88; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(")", 1); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(5u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__94() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("typeSpec", 8); +x_1 = lean_mk_string_from_bytes(":=", 2); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__94; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__96() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__91() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lsp.RpcRef", 10); +x_1 = lean_mk_string_from_bytes("WithRpcRef.encodeUnsafe", 23); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__97() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__96; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__91; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__98() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__96; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__91; x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__97; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -1797,48 +1508,104 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__94() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lsp", 3); +x_1 = lean_mk_string_from_bytes("encodeUnsafe", 12); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__94; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__101() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__96() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__57; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__94; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__97() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__96; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__98() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__97; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(5u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("RpcRef", 6); +x_1 = lean_mk_string_from_bytes("rpcDecode", 9); return x_1; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__101() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__102() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__101; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__101; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__103() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -1847,8 +1614,8 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__103; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__101; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -1881,52 +1648,26 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("declValSimple", 13); +x_1 = lean_mk_string_from_bytes("WithRpcRef.decodeUnsafeAs", 25); return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__108() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__107; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(":=", 2); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__110() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("WithRpcRef.encodeUnsafe", 23); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__111() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__110; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__107; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__112() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__110; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__107; x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__111; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__108; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -1934,51 +1675,68 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__113() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__110() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("decodeUnsafeAs", 14); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__111() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__88; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__110; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__114() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__112() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__89; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__57; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__110; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__113() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__114; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__112; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__114() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__113; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(4u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116() { _start: { lean_object* x_1; lean_object* x_2; @@ -1987,7 +1745,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__118() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117() { _start: { lean_object* x_1; @@ -1995,17 +1753,17 @@ x_1 = lean_mk_string_from_bytes("attributes", 10); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__118() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__118; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__120() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119() { _start: { lean_object* x_1; @@ -2013,7 +1771,7 @@ x_1 = lean_mk_string_from_bytes("@[", 2); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__121() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__120() { _start: { lean_object* x_1; @@ -2021,17 +1779,17 @@ x_1 = lean_mk_string_from_bytes("attrInstance", 12); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__122() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__121() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__121; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__120; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__123() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__122() { _start: { lean_object* x_1; @@ -2039,33 +1797,33 @@ x_1 = lean_mk_string_from_bytes("attrKind", 8); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__124() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__123() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__123; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__122; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__125() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__124() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__126() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__125() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__124; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__125; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__123; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__124; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -2073,7 +1831,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__127() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__126() { _start: { lean_object* x_1; @@ -2081,17 +1839,17 @@ x_1 = lean_mk_string_from_bytes("Attr", 4); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__128() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__127() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__6; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__127; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__126; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__129() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__128() { _start: { lean_object* x_1; @@ -2099,17 +1857,17 @@ x_1 = lean_mk_string_from_bytes("simple", 6); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__130() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__129() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__128; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__129; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__127; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__128; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__131() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__130() { _start: { lean_object* x_1; @@ -2117,22 +1875,22 @@ x_1 = lean_mk_string_from_bytes("implementedBy", 13); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__132() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__131() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__131; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__130; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__133() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__132() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__131; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__130; x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__132; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__131; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -2140,26 +1898,34 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__134() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__133() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__131; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__130; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__134() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__126; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__125; x_3 = lean_array_push(x_1, x_2); return x_3; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("]", 1); +return x_1; +} +} static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__136() { _start: { @@ -2182,7 +1948,7 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("encode", 6); +x_1 = lean_mk_string_from_bytes("inst", 4); return x_1; } } @@ -2240,28 +2006,31 @@ return x_3; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__144() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("pure", 4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__22; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__145() { _start: { -lean_object* x_1; lean_object* x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__144; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__146() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__144; -x_2 = lean_unsigned_to_nat(0u); +x_1 = lean_box(2); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__145; -x_4 = lean_alloc_ctor(0, 3, 0); +x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); lean_ctor_set(x_4, 2, x_3); @@ -2271,37 +2040,35 @@ return x_4; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__144; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("instance", 8); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__148() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Pure", 4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__149() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__148; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("declValSimple", 13); +return x_1; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__150() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__149; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__144; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__149; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -2309,13556 +2076,5948 @@ return x_3; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__151() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__150; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(8u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__152() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__151; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__151; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__125; +x_3 = lean_array_push(x_1, x_2); return x_3; } } static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__153() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("anonymousCtor", 13); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__154() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__153; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__146; +x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__155() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("⟨", 3); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__156() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__154() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("num", 3); +x_1 = lean_mk_string_from_bytes("quotedName", 10); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__157() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__155() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__156; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__154; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__158() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__156() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("0", 1); +x_1 = lean_mk_string_from_bytes(".", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__159() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__157() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("⟩", 3); +x_1 = lean_mk_string_from_bytes("`", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__160() { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("decodeUnsafe", 12); -return x_1; -} +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; 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; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; +lean_inc(x_1); +x_5 = lean_mk_syntax_ident(x_1); +x_6 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Command_mkDefViewOfInstance___spec__11(x_2, x_3, x_4); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = l_Lean_Elab_Command_getCurrMacroScope(x_2, x_3, x_8); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = l_Lean_Elab_Command_getMainModule___rarg(x_3, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; +lean_inc(x_7); +x_16 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_16, 0, x_7); +lean_ctor_set(x_16, 1, x_15); +x_17 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_18 = lean_array_push(x_17, x_16); +x_19 = lean_box(2); +x_20 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__16; +x_21 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +lean_ctor_set(x_21, 2, x_18); +x_22 = lean_array_push(x_17, x_21); +x_23 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_24 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_24, 0, x_19); +lean_ctor_set(x_24, 1, x_23); +lean_ctor_set(x_24, 2, x_22); +x_25 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__22; +x_26 = lean_array_push(x_25, x_24); +x_27 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_28 = lean_array_push(x_26, x_27); +x_29 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; +x_30 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_30, 0, x_19); +lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_30, 2, x_28); +x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23; +lean_inc(x_7); +x_32 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_32, 0, x_7); +lean_ctor_set(x_32, 1, x_31); +x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__30; +lean_inc(x_10); +lean_inc(x_13); +x_34 = l_Lean_addMacroScope(x_13, x_33, x_10); +x_35 = lean_box(0); +x_36 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__29; +lean_inc(x_7); +x_37 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_37, 0, x_7); +lean_ctor_set(x_37, 1, x_36); +lean_ctor_set(x_37, 2, x_34); +lean_ctor_set(x_37, 3, x_35); +x_38 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +lean_inc(x_37); +x_39 = lean_array_push(x_38, x_37); +x_40 = lean_array_push(x_39, x_27); +x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; +x_42 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_42, 0, x_19); +lean_ctor_set(x_42, 1, x_41); +lean_ctor_set(x_42, 2, x_40); +x_43 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; +lean_inc(x_7); +x_44 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_44, 0, x_7); +lean_ctor_set(x_44, 1, x_43); +x_45 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; +lean_inc(x_10); +lean_inc(x_13); +x_46 = l_Lean_addMacroScope(x_13, x_45, x_10); +x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; +x_48 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__49; +lean_inc(x_7); +x_49 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_49, 0, x_7); +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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +lean_inc(x_7); +x_51 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_51, 0, x_7); +lean_ctor_set(x_51, 1, x_50); +x_52 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56; +lean_inc(x_10); +lean_inc(x_13); +x_53 = l_Lean_addMacroScope(x_13, x_52, x_10); +x_54 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__55; +x_55 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; +lean_inc(x_7); +x_56 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_56, 0, x_7); +lean_ctor_set(x_56, 1, x_54); +lean_ctor_set(x_56, 2, x_53); +lean_ctor_set(x_56, 3, x_55); +lean_inc(x_5); +x_57 = lean_array_push(x_17, x_5); +x_58 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_58, 0, x_19); +lean_ctor_set(x_58, 1, x_23); +lean_ctor_set(x_58, 2, x_57); +x_59 = lean_array_push(x_38, x_56); +x_60 = lean_array_push(x_59, x_58); +x_61 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; +x_62 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_62, 0, x_19); +lean_ctor_set(x_62, 1, x_61); +lean_ctor_set(x_62, 2, x_60); +x_63 = lean_array_push(x_38, x_62); +x_64 = lean_array_push(x_63, x_27); +x_65 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_65, 0, x_19); +lean_ctor_set(x_65, 1, x_23); +lean_ctor_set(x_65, 2, x_64); +x_66 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +lean_inc(x_7); +x_67 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_67, 0, x_7); +lean_ctor_set(x_67, 1, x_66); +x_68 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +x_69 = lean_array_push(x_68, x_51); +x_70 = lean_array_push(x_69, x_65); +x_71 = lean_array_push(x_70, x_67); +x_72 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; +x_73 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_73, 0, x_19); +lean_ctor_set(x_73, 1, x_72); +lean_ctor_set(x_73, 2, x_71); +x_74 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; +lean_inc(x_10); +lean_inc(x_13); +x_75 = l_Lean_addMacroScope(x_13, x_74, x_10); +x_76 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__64; +x_77 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__72; +lean_inc(x_7); +x_78 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_78, 0, x_7); +lean_ctor_set(x_78, 1, x_76); +lean_ctor_set(x_78, 2, x_75); +lean_ctor_set(x_78, 3, x_77); +x_79 = lean_array_push(x_38, x_73); +x_80 = lean_array_push(x_79, x_78); +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_19); +lean_ctor_set(x_81, 1, x_23); +lean_ctor_set(x_81, 2, x_80); +x_82 = lean_array_push(x_38, x_49); +x_83 = lean_array_push(x_82, x_81); +x_84 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_84, 0, x_19); +lean_ctor_set(x_84, 1, x_61); +lean_ctor_set(x_84, 2, x_83); +x_85 = lean_array_push(x_38, x_44); +x_86 = lean_array_push(x_85, x_84); +x_87 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__37; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_19); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +lean_inc(x_88); +x_89 = lean_array_push(x_17, x_88); +x_90 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_90, 0, x_19); +lean_ctor_set(x_90, 1, x_23); +lean_ctor_set(x_90, 2, x_89); +x_91 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__73; +x_92 = lean_array_push(x_91, x_90); +x_93 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; +x_94 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_94, 0, x_19); +lean_ctor_set(x_94, 1, x_93); +lean_ctor_set(x_94, 2, x_92); +x_95 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__76; +lean_inc(x_7); +x_96 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_96, 0, x_7); +lean_ctor_set(x_96, 1, x_95); +x_97 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86; +lean_inc(x_10); +lean_inc(x_13); +x_98 = l_Lean_addMacroScope(x_13, x_97, x_10); +x_99 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +x_100 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__89; +lean_inc(x_7); +x_101 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_101, 0, x_7); +lean_ctor_set(x_101, 1, x_99); +lean_ctor_set(x_101, 2, x_98); +lean_ctor_set(x_101, 3, x_100); +x_102 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; +lean_inc(x_7); +x_103 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_103, 0, x_7); +lean_ctor_set(x_103, 1, x_102); +x_104 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95; +lean_inc(x_10); +lean_inc(x_13); +x_105 = l_Lean_addMacroScope(x_13, x_104, x_10); +x_106 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; +x_107 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__98; +lean_inc(x_7); +x_108 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_108, 0, x_7); +lean_ctor_set(x_108, 1, x_106); +lean_ctor_set(x_108, 2, x_105); +lean_ctor_set(x_108, 3, x_107); +lean_inc(x_1); +x_109 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_35, x_1); +x_110 = lean_array_push(x_38, x_108); +x_111 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; +x_112 = lean_array_push(x_111, x_101); +x_113 = lean_array_push(x_112, x_27); +x_114 = lean_array_push(x_113, x_27); +lean_inc(x_103); +x_115 = lean_array_push(x_114, x_103); +x_116 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__103; +lean_inc(x_10); +lean_inc(x_13); +x_117 = l_Lean_addMacroScope(x_13, x_116, x_10); +x_118 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__102; +x_119 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__106; +lean_inc(x_7); +x_120 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_120, 0, x_7); +lean_ctor_set(x_120, 1, x_118); +lean_ctor_set(x_120, 2, x_117); +lean_ctor_set(x_120, 3, x_119); +x_121 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__111; +lean_inc(x_10); +lean_inc(x_13); +x_122 = l_Lean_addMacroScope(x_13, x_121, x_10); +x_123 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; +x_124 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__114; +lean_inc(x_7); +x_125 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_125, 0, x_7); +lean_ctor_set(x_125, 1, x_123); +lean_ctor_set(x_125, 2, x_122); +lean_ctor_set(x_125, 3, x_124); +x_126 = lean_array_push(x_38, x_5); +x_127 = lean_array_push(x_38, x_125); +x_128 = lean_array_push(x_111, x_120); +x_129 = lean_array_push(x_128, x_27); +x_130 = lean_array_push(x_129, x_27); +lean_inc(x_103); +x_131 = lean_array_push(x_130, x_103); +x_132 = lean_array_push(x_68, x_96); +x_133 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116; +x_134 = lean_array_push(x_133, x_32); +x_135 = lean_array_push(x_134, x_42); +x_136 = lean_array_push(x_135, x_94); +x_137 = lean_array_push(x_38, x_30); +x_138 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119; +lean_inc(x_7); +x_139 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_139, 0, x_7); +lean_ctor_set(x_139, 1, x_138); +x_140 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__133; +lean_inc(x_10); +lean_inc(x_13); +x_141 = l_Lean_addMacroScope(x_13, x_140, x_10); +x_142 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__132; +lean_inc(x_7); +x_143 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_143, 0, x_7); +lean_ctor_set(x_143, 1, x_142); +lean_ctor_set(x_143, 2, x_141); +lean_ctor_set(x_143, 3, x_35); +x_144 = lean_array_push(x_17, x_37); +x_145 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_145, 0, x_19); +lean_ctor_set(x_145, 1, x_23); +lean_ctor_set(x_145, 2, x_144); +x_146 = lean_array_push(x_38, x_143); +x_147 = lean_array_push(x_146, x_145); +x_148 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__129; +x_149 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_149, 0, x_19); +lean_ctor_set(x_149, 1, x_148); +lean_ctor_set(x_149, 2, x_147); +x_150 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__134; +x_151 = lean_array_push(x_150, x_149); +x_152 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__121; +x_153 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_153, 0, x_19); +lean_ctor_set(x_153, 1, x_152); +lean_ctor_set(x_153, 2, x_151); +x_154 = lean_array_push(x_17, x_153); +x_155 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_155, 0, x_19); +lean_ctor_set(x_155, 1, x_23); +lean_ctor_set(x_155, 2, x_154); +x_156 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; +lean_inc(x_7); +x_157 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_157, 0, x_7); +lean_ctor_set(x_157, 1, x_156); +x_158 = lean_array_push(x_68, x_139); +x_159 = lean_array_push(x_158, x_155); +x_160 = lean_array_push(x_159, x_157); +x_161 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__118; +x_162 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_162, 0, x_19); +lean_ctor_set(x_162, 1, x_161); +lean_ctor_set(x_162, 2, x_160); +x_163 = lean_array_push(x_17, x_162); +x_164 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_164, 0, x_19); +lean_ctor_set(x_164, 1, x_23); +lean_ctor_set(x_164, 2, x_163); +x_165 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__19; +x_166 = lean_array_push(x_165, x_164); +x_167 = lean_array_push(x_166, x_27); +x_168 = lean_array_push(x_167, x_27); +x_169 = lean_array_push(x_168, x_27); +x_170 = lean_array_push(x_169, x_27); +x_171 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_171, 0, x_19); +lean_ctor_set(x_171, 1, x_29); +lean_ctor_set(x_171, 2, x_170); +x_172 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__136; +lean_inc(x_7); +x_173 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_173, 0, x_7); +lean_ctor_set(x_173, 1, x_172); +x_174 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__141; +x_175 = l_Lean_addMacroScope(x_13, x_174, x_10); +x_176 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__140; +lean_inc(x_7); +x_177 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_177, 0, x_7); +lean_ctor_set(x_177, 1, x_176); +lean_ctor_set(x_177, 2, x_175); +lean_ctor_set(x_177, 3, x_35); +lean_inc(x_177); +x_178 = lean_array_push(x_38, x_177); +x_179 = lean_array_push(x_178, x_27); +x_180 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_180, 0, x_19); +lean_ctor_set(x_180, 1, x_41); +lean_ctor_set(x_180, 2, x_179); +x_181 = lean_array_push(x_91, x_88); +x_182 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__143; +x_183 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_183, 0, x_19); +lean_ctor_set(x_183, 1, x_182); +lean_ctor_set(x_183, 2, x_181); +x_184 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_185 = lean_array_push(x_184, x_173); +x_186 = lean_array_push(x_185, x_180); +lean_inc(x_183); +x_187 = lean_array_push(x_186, x_183); +x_188 = lean_array_push(x_187, x_27); +x_189 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__137; +x_190 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_190, 0, x_19); +lean_ctor_set(x_190, 1, x_189); +lean_ctor_set(x_190, 2, x_188); +x_191 = lean_array_push(x_38, x_171); +x_192 = lean_array_push(x_191, x_190); +x_193 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__10; +x_194 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_194, 0, x_19); +lean_ctor_set(x_194, 1, x_193); +lean_ctor_set(x_194, 2, x_192); +x_195 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; +x_196 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_196, 0, x_7); +lean_ctor_set(x_196, 1, x_195); +x_197 = lean_array_push(x_68, x_103); +x_198 = lean_array_push(x_197, x_177); +x_199 = lean_array_push(x_198, x_27); +x_200 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__150; +x_201 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_201, 0, x_19); +lean_ctor_set(x_201, 1, x_200); +lean_ctor_set(x_201, 2, x_199); +x_202 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__152; +x_203 = lean_array_push(x_202, x_196); +x_204 = lean_array_push(x_203, x_27); +x_205 = lean_array_push(x_204, x_27); +x_206 = lean_array_push(x_205, x_183); +x_207 = lean_array_push(x_206, x_201); +x_208 = lean_array_push(x_207, x_27); +x_209 = lean_array_push(x_208, x_27); +x_210 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__148; +x_211 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_211, 0, x_19); +lean_ctor_set(x_211, 1, x_210); +lean_ctor_set(x_211, 2, x_209); +x_212 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__153; +x_213 = lean_array_push(x_212, x_211); +x_214 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_214, 0, x_19); +lean_ctor_set(x_214, 1, x_193); +lean_ctor_set(x_214, 2, x_213); +if (lean_obj_tag(x_109) == 0) +{ +lean_object* x_274; +x_274 = l_Lean_quoteNameMk(x_1); +x_215 = x_274; +goto block_273; +} +else +{ +lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; +lean_dec(x_1); +x_275 = lean_ctor_get(x_109, 0); +lean_inc(x_275); +lean_dec(x_109); +x_276 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__156; +x_277 = l_String_intercalate(x_276, x_275); +x_278 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__157; +x_279 = lean_string_append(x_278, x_277); +lean_dec(x_277); +x_280 = l_Lean_Syntax_mkNameLit(x_279, x_19); +x_281 = lean_array_push(x_17, x_280); +x_282 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__155; +x_283 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_283, 0, x_19); +lean_ctor_set(x_283, 1, x_282); +lean_ctor_set(x_283, 2, x_281); +x_215 = x_283; +goto block_273; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__161() { -_start: +block_273: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__160; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__162() { -_start: +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; +lean_inc(x_215); +x_216 = lean_array_push(x_17, x_215); +x_217 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_217, 0, x_19); +lean_ctor_set(x_217, 1, x_23); +lean_ctor_set(x_217, 2, x_216); +x_218 = lean_array_push(x_110, x_217); +x_219 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_219, 0, x_19); +lean_ctor_set(x_219, 1, x_61); +lean_ctor_set(x_219, 2, x_218); +x_220 = lean_array_push(x_115, x_219); +x_221 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__82; +x_222 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_222, 0, x_19); +lean_ctor_set(x_222, 1, x_221); +lean_ctor_set(x_222, 2, x_220); +x_223 = lean_array_push(x_17, x_222); +x_224 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; +x_225 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_225, 0, x_19); +lean_ctor_set(x_225, 1, x_224); +lean_ctor_set(x_225, 2, x_223); +x_226 = lean_array_push(x_17, x_225); +x_227 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__78; +x_228 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_228, 0, x_19); +lean_ctor_set(x_228, 1, x_227); +lean_ctor_set(x_228, 2, x_226); +x_229 = lean_array_push(x_126, x_215); +x_230 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_230, 0, x_19); +lean_ctor_set(x_230, 1, x_23); +lean_ctor_set(x_230, 2, x_229); +x_231 = lean_array_push(x_127, x_230); +x_232 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_232, 0, x_19); +lean_ctor_set(x_232, 1, x_61); +lean_ctor_set(x_232, 2, x_231); +x_233 = lean_array_push(x_131, x_232); +x_234 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_234, 0, x_19); +lean_ctor_set(x_234, 1, x_221); +lean_ctor_set(x_234, 2, x_233); +x_235 = lean_array_push(x_17, x_234); +x_236 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_236, 0, x_19); +lean_ctor_set(x_236, 1, x_224); +lean_ctor_set(x_236, 2, x_235); +x_237 = lean_array_push(x_17, x_236); +x_238 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_238, 0, x_19); +lean_ctor_set(x_238, 1, x_227); +lean_ctor_set(x_238, 2, x_237); +x_239 = lean_array_push(x_184, x_228); +x_240 = lean_array_push(x_239, x_27); +x_241 = lean_array_push(x_240, x_238); +x_242 = lean_array_push(x_241, x_27); +x_243 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_243, 0, x_19); +lean_ctor_set(x_243, 1, x_23); +lean_ctor_set(x_243, 2, x_242); +x_244 = lean_array_push(x_132, x_243); +x_245 = lean_array_push(x_244, x_27); +x_246 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__75; +x_247 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_247, 0, x_19); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_245); +x_248 = lean_array_push(x_136, x_247); +x_249 = lean_array_push(x_248, x_27); +x_250 = lean_array_push(x_249, x_27); +x_251 = lean_array_push(x_250, x_27); +x_252 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__24; +x_253 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_253, 0, x_19); +lean_ctor_set(x_253, 1, x_252); +lean_ctor_set(x_253, 2, x_251); +x_254 = lean_array_push(x_137, x_253); +x_255 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_255, 0, x_19); +lean_ctor_set(x_255, 1, x_193); +lean_ctor_set(x_255, 2, x_254); +x_256 = lean_array_push(x_68, x_255); +x_257 = lean_array_push(x_256, x_194); +x_258 = lean_array_push(x_257, x_214); +x_259 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_259, 0, x_19); +lean_ctor_set(x_259, 1, x_23); +lean_ctor_set(x_259, 2, x_258); +x_260 = l_Lean_Elab_Command_elabCommand(x_259, x_2, x_3, x_14); +if (lean_obj_tag(x_260) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__160; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__161; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__163() { -_start: +uint8_t x_261; +x_261 = !lean_is_exclusive(x_260); +if (x_261 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__160; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_262; uint8_t x_263; lean_object* x_264; +x_262 = lean_ctor_get(x_260, 0); +lean_dec(x_262); +x_263 = 1; +x_264 = lean_box(x_263); +lean_ctor_set(x_260, 0, x_264); +return x_260; } -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__164() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("ExceptT", 7); -return x_1; +lean_object* x_265; uint8_t x_266; lean_object* x_267; lean_object* x_268; +x_265 = lean_ctor_get(x_260, 1); +lean_inc(x_265); +lean_dec(x_260); +x_266 = 1; +x_267 = lean_box(x_266); +x_268 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_265); +return x_268; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__165() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__164; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__166() { -_start: +uint8_t x_269; +x_269 = !lean_is_exclusive(x_260); +if (x_269 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__164; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__165; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} +return x_260; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__167() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__164; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_270; lean_object* x_271; lean_object* x_272; +x_270 = lean_ctor_get(x_260, 0); +x_271 = lean_ctor_get(x_260, 1); +lean_inc(x_271); +lean_inc(x_270); +lean_dec(x_260); +x_272 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_272, 0, x_270); +lean_ctor_set(x_272, 1, x_271); +return x_272; +} } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__168() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__167; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__169() { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__168; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_4; lean_object* x_5; +x_4 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_4, 0, x_1); +x_5 = lean_apply_2(x_2, lean_box(0), x_4); +return x_5; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__170() { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("String", 6); -return x_1; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_box(0); +lean_inc(x_5); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +x_8 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_5); +x_9 = lean_apply_4(x_2, lean_box(0), lean_box(0), x_7, x_8); +return x_9; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__171() { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__170; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_apply_2(x_1, x_2, x_3); +lean_inc(x_5); +x_9 = l_Lean_Meta_forallTelescopeReducing___rarg(x_4, x_5, lean_box(0), x_7, x_8); +lean_inc(x_6); +x_10 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__2), 3, 2); +lean_closure_set(x_10, 0, x_5); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_9, x_10); +return x_11; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__172() { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__170; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__171; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__173() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__170; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Expr_const___override(x_12, x_1); +x_14 = l_Lean_mkAppN(x_13, x_2); +x_15 = lean_alloc_closure((void*)(l_Lean_Meta_inferType___boxed), 6, 1); +lean_closure_set(x_15, 0, x_14); +x_16 = lean_apply_2(x_3, lean_box(0), x_15); +lean_inc(x_9); +x_17 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__3), 7, 6); +lean_closure_set(x_17, 0, x_4); +lean_closure_set(x_17, 1, x_5); +lean_closure_set(x_17, 2, x_6); +lean_closure_set(x_17, 3, x_7); +lean_closure_set(x_17, 4, x_8); +lean_closure_set(x_17, 5, x_9); +x_18 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_16, x_17); +return x_18; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__174() { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__173; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__175() { -_start: +if (lean_obj_tag(x_9) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__174; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +lean_dec(x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_apply_2(x_12, lean_box(0), x_10); +return x_13; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__176() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("paren", 5); -return x_1; +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_9, 0); +lean_inc(x_14); +lean_dec(x_9); +x_15 = l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg(x_1, x_2, x_3, lean_box(0), x_4, x_5, x_6, x_7, x_8, x_14); +return x_15; +} } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__177() { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__176; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_apply_2(x_12, lean_box(0), x_10); +return x_13; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__178() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("WithRpcRef.decodeUnsafeAs", 25); -return x_1; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_14 = lean_ctor_get(x_9, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_9, 1); +lean_inc(x_15); +lean_dec(x_9); +x_16 = lean_ctor_get(x_1, 1); +lean_inc(x_16); +lean_inc(x_14); +x_17 = lean_alloc_closure((void*)(l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1___boxed), 6, 1); +lean_closure_set(x_17, 0, x_14); +lean_inc(x_3); +x_18 = lean_apply_2(x_3, lean_box(0), x_17); +lean_inc(x_8); +lean_inc(x_1); +lean_inc(x_2); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_5); +lean_inc(x_7); +x_19 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__4), 10, 9); +lean_closure_set(x_19, 0, x_7); +lean_closure_set(x_19, 1, x_5); +lean_closure_set(x_19, 2, x_3); +lean_closure_set(x_19, 3, x_6); +lean_closure_set(x_19, 4, x_10); +lean_closure_set(x_19, 5, x_14); +lean_closure_set(x_19, 6, x_2); +lean_closure_set(x_19, 7, x_1); +lean_closure_set(x_19, 8, x_8); +lean_inc(x_8); +x_20 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__5), 9, 8); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_2); +lean_closure_set(x_21, 2, x_3); +lean_closure_set(x_21, 3, x_5); +lean_closure_set(x_21, 4, x_6); +lean_closure_set(x_21, 5, x_7); +lean_closure_set(x_21, 6, x_8); +lean_closure_set(x_21, 7, x_15); +x_22 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_20, x_21); +return x_22; +} } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__179() { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__178; -x_2 = lean_string_utf8_byte_size(x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg), 10, 0); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__180() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__178; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__179; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +lean_dec(x_1); +x_4 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_apply_2(x_4, lean_box(0), x_2); +return x_5; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__181() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("decodeUnsafeAs", 14); -return x_1; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_9 = lean_ctor_get(x_5, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = lean_box(0); +x_12 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_10, x_11); +x_13 = lean_ctor_get(x_1, 1); +lean_inc(x_13); +x_14 = lean_ctor_get(x_5, 4); +lean_inc(x_14); +lean_dec(x_5); +lean_inc(x_13); +lean_inc(x_1); +x_15 = l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg(x_1, x_2, x_3, lean_box(0), x_6, x_7, x_12, x_13, x_14, x_8); +x_16 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_foldWithConstructors___rarg___lambda__1), 2, 1); +lean_closure_set(x_16, 0, x_1); +x_17 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_15, x_16); +return x_17; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__182() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__88; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__181; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_foldWithConstructors___rarg), 8, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__183() { +LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__89; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__181; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_4; +x_4 = l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__184() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__183; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_1); +lean_ctor_set(x_6, 1, x_5); +x_7 = lean_array_push(x_2, x_6); +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +lean_dec(x_3); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(0); +lean_inc(x_9); +x_11 = lean_apply_2(x_9, lean_box(0), x_10); +x_12 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_12, 0, x_7); +lean_closure_set(x_12, 1, x_9); +x_13 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_11, x_12); +return x_13; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__185() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__184; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_alloc_closure((void*)(l_Lean_Meta_inferType___boxed), 6, 1); +lean_closure_set(x_7, 0, x_6); +x_8 = lean_apply_2(x_1, lean_box(0), x_7); +lean_inc(x_5); +x_9 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__1), 5, 4); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +x_10 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_8, x_9); +return x_10; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__186() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, lean_object* x_8) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("decode", 6); -return x_1; +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +lean_dec(x_1); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_apply_2(x_11, lean_box(0), x_9); +return x_12; +} +else +{ +lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_8, 0); +lean_inc(x_13); +lean_dec(x_8); +x_14 = 1; +x_15 = lean_usize_add(x_2, x_14); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_15, x_13); +return x_16; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__187() { +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__186; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_7, x_6); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +lean_dec(x_1); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_apply_2(x_11, lean_box(0), x_8); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_13 = lean_array_uget(x_5, x_7); +x_14 = lean_ctor_get(x_1, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_3); +x_15 = lean_alloc_closure((void*)(l_Lean_Meta_mkProjection), 7, 2); +lean_closure_set(x_15, 0, x_3); +lean_closure_set(x_15, 1, x_13); +lean_inc(x_2); +x_16 = lean_apply_2(x_2, lean_box(0), x_15); +lean_inc(x_4); +lean_inc(x_1); +lean_inc(x_2); +x_17 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2), 6, 5); +lean_closure_set(x_17, 0, x_2); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_8); +lean_closure_set(x_17, 3, x_1); +lean_closure_set(x_17, 4, x_4); +lean_inc(x_4); +x_18 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_16, x_17); +x_19 = lean_box_usize(x_7); +x_20 = lean_box_usize(x_6); +x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_19); +lean_closure_set(x_21, 2, x_2); +lean_closure_set(x_21, 3, x_3); +lean_closure_set(x_21, 4, x_4); +lean_closure_set(x_21, 5, x_5); +lean_closure_set(x_21, 6, x_20); +x_22 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_18, x_21); +return x_22; +} } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__188() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__186; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__187; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___boxed), 8, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__189() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__186; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_9; lean_object* x_10; +x_9 = lean_apply_1(x_1, x_3); +x_10 = lean_apply_7(x_2, lean_box(0), x_9, x_4, x_5, x_6, x_7, x_8); +return x_10; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("throw", 5); -return x_1; +lean_object* x_11; lean_object* x_12; +x_11 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__1), 8, 2); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_5); +x_12 = l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); +return x_12; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__191() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +lean_object* x_8; lean_object* x_9; 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_1, 1); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_box(x_5); +x_10 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed), 10, 4); +lean_closure_set(x_10, 0, x_7); +lean_closure_set(x_10, 1, x_4); +lean_closure_set(x_10, 2, x_9); +lean_closure_set(x_10, 3, x_6); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +x_12 = lean_apply_2(x_11, lean_box(0), x_10); +x_13 = lean_ctor_get(x_2, 1); +lean_inc(x_13); +lean_dec(x_2); +x_14 = lean_apply_1(x_13, lean_box(0)); +x_15 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_12, x_14); +return x_15; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__192() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__191; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___boxed), 7, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__193() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_box(0); +x_8 = lean_apply_1(x_2, x_7); +x_9 = lean_array_get_size(x_8); +x_10 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_11 = 0; +x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +lean_inc(x_6); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(x_1, x_3, x_5, x_6, x_8, x_10, x_11, x_12); +x_14 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_13, x_4); +return x_14; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__194() { +static lean_object* _init_l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("MonadExcept", 11); +x_1 = lean_mk_string_from_bytes("s", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__195() { +static lean_object* _init_l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__194; +x_2 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__196() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__195; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; +x_9 = lean_ctor_get(x_5, 0); +lean_inc(x_9); +lean_dec(x_5); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +x_11 = lean_box(0); +x_12 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_10, x_11); +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = l_Lean_Expr_const___override(x_13, x_12); +x_15 = l_Lean_mkAppN(x_14, x_6); +lean_inc(x_1); +x_16 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___rarg___lambda__1), 5, 4); +lean_closure_set(x_16, 0, x_1); +lean_closure_set(x_16, 1, x_8); +lean_closure_set(x_16, 2, x_3); +lean_closure_set(x_16, 3, x_7); +x_17 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; +x_18 = 0; +x_19 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg(x_1, x_2, lean_box(0), x_17, x_18, x_15, x_16); +return x_19; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__197() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__196; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___rarg), 8, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__198() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__197; -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; +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_10 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3(x_1, x_9, x_3, x_4, x_5, x_6, x_10, x_8); +return x_11; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__199() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("str", 3); -return x_1; +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_10 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); +return x_11; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__200() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__199; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_3); +lean_dec(x_3); +x_12 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__201() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("\"unreachable\"", 13); -return x_1; +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +return x_9; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__202() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__46; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__203() { -_start: +if (lean_obj_tag(x_8) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__202; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +lean_dec(x_1); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_apply_2(x_11, lean_box(0), x_9); +return x_12; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__204() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__203; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} +lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_8, 0); +lean_inc(x_13); +lean_dec(x_8); +x_14 = 1; +x_15 = lean_usize_add(x_2, x_14); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_15, x_13); +return x_16; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("instance", 8); -return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_7, x_6); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +lean_dec(x_1); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_apply_2(x_11, lean_box(0), x_8); +return x_12; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("RpcEncoding", 11); -return x_1; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_13 = lean_array_uget(x_5, x_7); +x_14 = lean_ctor_get(x_1, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_3); +x_15 = lean_alloc_closure((void*)(l_Lean_Meta_mkProjection), 7, 2); +lean_closure_set(x_15, 0, x_3); +lean_closure_set(x_15, 1, x_13); +lean_inc(x_2); +x_16 = lean_apply_2(x_2, lean_box(0), x_15); +lean_inc(x_4); +lean_inc(x_1); +lean_inc(x_2); +x_17 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2), 6, 5); +lean_closure_set(x_17, 0, x_2); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_8); +lean_closure_set(x_17, 3, x_1); +lean_closure_set(x_17, 4, x_4); +lean_inc(x_4); +x_18 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_16, x_17); +x_19 = lean_box_usize(x_7); +x_20 = lean_box_usize(x_6); +x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1___boxed), 8, 7); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_19); +lean_closure_set(x_21, 2, x_2); +lean_closure_set(x_21, 3, x_3); +lean_closure_set(x_21, 4, x_4); +lean_closure_set(x_21, 5, x_5); +lean_closure_set(x_21, 6, x_20); +x_22 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_18, x_21); +return x_22; +} } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__208() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207; -x_2 = lean_string_utf8_byte_size(x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___boxed), 8, 0); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__209() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__208; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_8; lean_object* x_9; 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_1, 1); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_box(x_5); +x_10 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed), 10, 4); +lean_closure_set(x_10, 0, x_7); +lean_closure_set(x_10, 1, x_4); +lean_closure_set(x_10, 2, x_9); +lean_closure_set(x_10, 3, x_6); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +x_12 = lean_apply_2(x_11, lean_box(0), x_10); +x_13 = lean_ctor_get(x_2, 1); +lean_inc(x_13); +lean_dec(x_2); +x_14 = lean_apply_1(x_13, lean_box(0)); +x_15 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_12, x_14); +return x_15; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__210() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg___boxed), 7, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__74; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_box(0); +x_8 = lean_apply_1(x_2, x_7); +x_9 = lean_array_get_size(x_8); +x_10 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_11 = 0; +x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +lean_inc(x_6); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(x_1, x_3, x_5, x_6, x_8, x_10, x_11, x_12); +x_14 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_13, x_4); +return x_14; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__212() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; +x_9 = lean_ctor_get(x_5, 0); +lean_inc(x_9); +lean_dec(x_5); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +x_11 = lean_box(0); +x_12 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_10, x_11); +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = l_Lean_Expr_const___override(x_13, x_12); +x_15 = l_Lean_mkAppN(x_14, x_6); +lean_inc(x_1); +x_16 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg___lambda__1), 5, 4); +lean_closure_set(x_16, 0, x_1); +lean_closure_set(x_16, 1, x_8); +lean_closure_set(x_16, 2, x_3); +lean_closure_set(x_16, 3, x_7); +x_17 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; +x_18 = 0; +x_19 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg(x_1, x_2, lean_box(0), x_17, x_18, x_15, x_16); +return x_19; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__213() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__212; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg), 8, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__214() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} +lean_object* x_6; uint8_t x_7; +x_6 = lean_st_ref_get(x_4, x_5); +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +lean_dec(x_8); +lean_ctor_set(x_6, 0, x_9); +return x_6; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__215() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("structInst", 10); -return x_1; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +lean_inc(x_11); +lean_inc(x_10); +lean_dec(x_6); +x_12 = lean_ctor_get(x_10, 0); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__216() { +} +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__215; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__217() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("structInstField", 15); -return x_1; +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +lean_dec(x_4); +x_6 = l_Lean_getStructureFields(x_2, x_5); +return x_6; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__218() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__217; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2___boxed), 3, 2); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_7); +x_9 = l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg(x_2, x_3, x_4, lean_box(0), x_1, x_5, x_6, x_8); +return x_9; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__219() { +static lean_object* _init_l_Lean_Server_RpcEncoding_withFields___rarg___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("structInstLVal", 14); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1___boxed), 5, 0); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__220() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__219; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); +x_9 = l_Lean_Server_RpcEncoding_withFields___rarg___closed__1; +lean_inc(x_3); +x_10 = lean_apply_2(x_3, lean_box(0), x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg___lambda__3), 7, 6); +lean_closure_set(x_11, 0, x_5); +lean_closure_set(x_11, 1, x_1); +lean_closure_set(x_11, 2, x_2); +lean_closure_set(x_11, 3, x_3); +lean_closure_set(x_11, 4, x_6); +lean_closure_set(x_11, 5, x_7); +x_12 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_10, x_11); +return x_12; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("rpcEncode", 9); -return x_1; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg), 7, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__222() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_10 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1(x_1, x_9, x_3, x_4, x_5, x_6, x_10, x_8); +return x_11; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__222; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_10 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); +return x_11; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +return x_9; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_6; +x_6 = l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_6; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__226() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_4; +x_4 = l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__227() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__226; -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; +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +lean_dec(x_1); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_apply_2(x_11, lean_box(0), x_9); +return x_12; +} +else +{ +lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_8, 0); +lean_inc(x_13); +lean_dec(x_8); +x_14 = 1; +x_15 = lean_usize_add(x_2, x_14); +x_16 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_15, x_13); +return x_16; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228() { +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("rpcDecode", 9); -return x_1; +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_7, x_6); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_10 = lean_ctor_get(x_1, 0); +lean_inc(x_10); +lean_dec(x_1); +x_11 = lean_ctor_get(x_10, 1); +lean_inc(x_11); +lean_dec(x_10); +x_12 = lean_apply_2(x_11, lean_box(0), x_8); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_13 = lean_array_uget(x_5, x_7); +x_14 = lean_ctor_get(x_1, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_3); +x_15 = lean_alloc_closure((void*)(l_Lean_Meta_mkProjection), 7, 2); +lean_closure_set(x_15, 0, x_3); +lean_closure_set(x_15, 1, x_13); +lean_inc(x_2); +x_16 = lean_apply_2(x_2, lean_box(0), x_15); +lean_inc(x_4); +lean_inc(x_1); +lean_inc(x_2); +x_17 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2), 6, 5); +lean_closure_set(x_17, 0, x_2); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_8); +lean_closure_set(x_17, 3, x_1); +lean_closure_set(x_17, 4, x_4); +lean_inc(x_4); +x_18 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_16, x_17); +x_19 = lean_box_usize(x_7); +x_20 = lean_box_usize(x_6); +x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1___boxed), 8, 7); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, x_19); +lean_closure_set(x_21, 2, x_2); +lean_closure_set(x_21, 3, x_3); +lean_closure_set(x_21, 4, x_4); +lean_closure_set(x_21, 5, x_5); +lean_closure_set(x_21, 6, x_20); +x_22 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_18, x_21); +return x_22; +} } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__229() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228; -x_2 = lean_string_utf8_byte_size(x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___boxed), 8, 0); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__229; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_8; lean_object* x_9; 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_1, 1); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_box(x_5); +x_10 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed), 10, 4); +lean_closure_set(x_10, 0, x_7); +lean_closure_set(x_10, 1, x_4); +lean_closure_set(x_10, 2, x_9); +lean_closure_set(x_10, 3, x_6); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +x_12 = lean_apply_2(x_11, lean_box(0), x_10); +x_13 = lean_ctor_get(x_2, 1); +lean_inc(x_13); +lean_dec(x_2); +x_14 = lean_apply_1(x_13, lean_box(0)); +x_15 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_12, x_14); +return x_15; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg___boxed), 7, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_box(0); +x_8 = lean_apply_1(x_2, x_7); +x_9 = lean_array_get_size(x_8); +x_10 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_11 = 0; +x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +lean_inc(x_6); +x_13 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(x_1, x_3, x_5, x_6, x_8, x_10, x_11, x_12); +x_14 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_13, x_4); +return x_14; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__233() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; +x_9 = lean_ctor_get(x_5, 0); +lean_inc(x_9); +lean_dec(x_5); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +x_11 = lean_box(0); +x_12 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_10, x_11); +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = l_Lean_Expr_const___override(x_13, x_12); +x_15 = l_Lean_mkAppN(x_14, x_6); +lean_inc(x_1); +x_16 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg___lambda__1), 5, 4); +lean_closure_set(x_16, 0, x_1); +lean_closure_set(x_16, 1, x_8); +lean_closure_set(x_16, 2, x_3); +lean_closure_set(x_16, 3, x_7); +x_17 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; +x_18 = 0; +x_19 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg(x_1, x_2, lean_box(0), x_17, x_18, x_15, x_16); +return x_19; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__234() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__233; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg), 8, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__235() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("optEllipsis", 11); -return x_1; +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +lean_dec(x_5); +x_7 = l_Lean_getStructureFieldsFlattened(x_2, x_6, x_3); +return x_7; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__236() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___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) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__235; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_box(x_2); +lean_inc(x_1); +x_10 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1___boxed), 4, 3); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_8); +lean_closure_set(x_10, 2, x_9); +x_11 = l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg(x_3, x_4, x_5, lean_box(0), x_1, x_6, x_7, x_10); +return x_11; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__237() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__236; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__125; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = l_Lean_Server_RpcEncoding_withFields___rarg___closed__1; +lean_inc(x_3); +x_11 = lean_apply_2(x_3, lean_box(0), x_10); +x_12 = lean_box(x_8); +x_13 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__2___boxed), 8, 7); +lean_closure_set(x_13, 0, x_5); +lean_closure_set(x_13, 1, x_12); +lean_closure_set(x_13, 2, x_1); +lean_closure_set(x_13, 3, x_2); +lean_closure_set(x_13, 4, x_3); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_7); +x_14 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_11, x_13); +return x_14; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(8u); -x_2 = lean_mk_empty_array_with_capacity(x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___boxed), 8, 0); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__239() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__126; -x_3 = lean_array_push(x_1, x_2); -return x_3; +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_10 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1(x_1, x_9, x_3, x_4, x_5, x_6, x_10, x_8); +return x_11; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__240() { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__204; -x_3 = lean_array_push(x_1, x_2); -return x_3; +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_10 = lean_unbox_usize(x_7); +lean_dec(x_7); +x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); +return x_11; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241() { +LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("end", 3); -return x_1; +uint8_t x_8; lean_object* x_9; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg(x_1, x_2, x_3, x_4, x_8, x_6, x_7); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; lean_object* x_6; +x_5 = lean_unbox(x_3); +lean_dec(x_3); +x_6 = l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1(x_1, x_2, x_5, x_4); +lean_dec(x_4); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_2); +lean_dec(x_2); +x_10 = l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__2(x_1, x_9, x_3, x_4, x_5, x_6, x_7, x_8); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +return x_10; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_levelOne; +x_2 = l_Lean_Expr_sort___override(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__1; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__242() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; +x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__243() { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__2; +x_8 = 0; +x_9 = lean_box(0); +lean_inc(x_2); +x_10 = l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarImpl(x_7, x_8, x_9, x_2, x_3, x_4, x_5, x_6); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__3; +lean_inc(x_11); +x_14 = l_Lean_mkAppB(x_13, x_1, x_11); +x_15 = lean_box(0); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_16 = l_Lean_Meta_synthInstance(x_14, x_15, x_2, x_3, x_4, x_5, x_12); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__1(x_11, x_2, x_3, x_4, x_5, x_17); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_18; +} +else +{ +uint8_t x_19; +lean_dec(x_11); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_16); +if (x_19 == 0) +{ +return x_16; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_16, 0); +x_21 = lean_ctor_get(x_16, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_16); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("quotedName", 10); +x_1 = lean_mk_string_from_bytes("instBinder", 10); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__244() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__243; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__245() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes(".", 1); +x_1 = lean_mk_string_from_bytes("[", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__246() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("`", 1); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5() { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; -lean_inc(x_1); -x_5 = lean_mk_syntax_ident(x_1); -x_6 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Command_mkDefViewOfInstance___spec__11(x_2, x_3, x_4); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_6, 1); -lean_inc(x_8); -lean_dec(x_6); -x_9 = l_Lean_Elab_Command_getCurrMacroScope(x_2, x_3, x_8); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__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; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_lt(x_3, x_2); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_10); lean_dec(x_9); -x_12 = l_Lean_Elab_Command_getMainModule___rarg(x_3, x_11); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__9; -lean_inc(x_7); -x_16 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_16, 0, x_7); -lean_ctor_set(x_16, 1, x_15); -x_17 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_18 = lean_array_push(x_17, x_16); -x_19 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_20 = lean_array_push(x_18, x_19); -x_21 = lean_box(2); -x_22 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__10; -x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -lean_ctor_set(x_23, 2, x_20); -x_24 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; -lean_inc(x_7); -x_25 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_25, 0, x_7); -lean_ctor_set(x_25, 1, x_24); -x_26 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__20; -lean_inc(x_7); -x_27 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_27, 0, x_7); -lean_ctor_set(x_27, 1, x_26); -x_28 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__24; +lean_dec(x_8); +lean_dec(x_7); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_4); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_array_uget(x_1, x_3); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_4, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_4, 1); +lean_inc(x_18); +lean_dec(x_4); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); lean_inc(x_10); -lean_inc(x_13); -x_29 = l_Lean_addMacroScope(x_13, x_28, x_10); -x_30 = lean_box(0); -x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23; -lean_inc(x_7); -x_32 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_32, 0, x_7); -lean_ctor_set(x_32, 1, x_31); -lean_ctor_set(x_32, 2, x_29); -lean_ctor_set(x_32, 3, x_30); -x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -lean_inc(x_32); -x_34 = lean_array_push(x_33, x_32); -x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_21); -lean_ctor_set(x_36, 1, x_35); -lean_ctor_set(x_36, 2, x_34); -x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; -lean_inc(x_7); -x_38 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_38, 0, x_7); -lean_ctor_set(x_38, 1, x_37); -x_39 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; -lean_inc(x_7); -x_40 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_40, 0, x_7); -lean_ctor_set(x_40, 1, x_39); -x_41 = lean_array_push(x_17, x_40); -x_42 = lean_array_push(x_41, x_19); -x_43 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__30; -x_44 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_44, 0, x_21); -lean_ctor_set(x_44, 1, x_43); -lean_ctor_set(x_44, 2, x_42); -x_45 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__32; -lean_inc(x_7); -x_46 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_46, 0, x_7); -lean_ctor_set(x_46, 1, x_45); -x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; -lean_inc(x_44); -x_48 = lean_array_push(x_47, x_44); -x_49 = lean_array_push(x_48, x_46); -x_50 = lean_array_push(x_49, x_44); -x_51 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__28; -x_52 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_52, 0, x_21); -lean_ctor_set(x_52, 1, x_51); -lean_ctor_set(x_52, 2, x_50); -x_53 = lean_array_push(x_17, x_38); -lean_inc(x_53); -x_54 = lean_array_push(x_53, x_52); -x_55 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_55, 0, x_21); -lean_ctor_set(x_55, 1, x_35); -lean_ctor_set(x_55, 2, x_54); -x_56 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; -lean_inc(x_7); -x_57 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_57, 0, x_7); -lean_ctor_set(x_57, 1, x_56); -x_58 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -lean_inc(x_27); -x_59 = lean_array_push(x_58, x_27); -lean_inc(x_36); -x_60 = lean_array_push(x_59, x_36); -x_61 = lean_array_push(x_60, x_55); -lean_inc(x_57); -x_62 = lean_array_push(x_61, x_57); -x_63 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__19; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_21); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = lean_array_push(x_33, x_64); -x_66 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_66, 0, x_21); -lean_ctor_set(x_66, 1, x_35); -lean_ctor_set(x_66, 2, x_65); -x_67 = lean_array_push(x_17, x_25); -x_68 = lean_array_push(x_67, x_66); -x_69 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_21); -lean_ctor_set(x_70, 1, x_69); -lean_ctor_set(x_70, 2, x_68); -x_71 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; -lean_inc(x_7); -x_72 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_72, 0, x_7); -lean_ctor_set(x_72, 1, x_71); -x_73 = lean_array_push(x_33, x_72); -x_74 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__41; -x_75 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_75, 0, x_21); -lean_ctor_set(x_75, 1, x_74); -lean_ctor_set(x_75, 2, x_73); -x_76 = lean_array_push(x_33, x_75); -x_77 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_77, 0, x_21); -lean_ctor_set(x_77, 1, x_35); -lean_ctor_set(x_77, 2, x_76); -x_78 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__46; -x_79 = lean_array_push(x_78, x_77); -x_80 = lean_array_push(x_79, x_19); -x_81 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; -x_82 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_82, 0, x_21); -lean_ctor_set(x_82, 1, x_81); -lean_ctor_set(x_82, 2, x_80); -x_83 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); -x_84 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_84, 0, x_7); -lean_ctor_set(x_84, 1, x_83); -x_85 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__54; +lean_inc(x_16); +x_21 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor(x_16, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_box(0); lean_inc(x_10); -lean_inc(x_13); -x_86 = l_Lean_addMacroScope(x_13, x_85, x_10); -x_87 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__53; -lean_inc(x_7); -x_88 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_88, 0, x_7); -lean_ctor_set(x_88, 1, x_87); -lean_ctor_set(x_88, 2, x_86); -lean_ctor_set(x_88, 3, x_30); -lean_inc(x_88); -x_89 = lean_array_push(x_17, x_88); -x_90 = lean_array_push(x_89, x_19); -x_91 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; -x_92 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_92, 0, x_21); -lean_ctor_set(x_92, 1, x_91); -lean_ctor_set(x_92, 2, x_90); -x_93 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); -x_94 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_94, 0, x_7); -lean_ctor_set(x_94, 1, x_93); -x_95 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__65; +x_25 = l_Lean_PrettyPrinter_delab(x_22, x_24, x_7, x_8, x_9, x_10, x_23); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); lean_inc(x_10); -lean_inc(x_13); -x_96 = l_Lean_addMacroScope(x_13, x_95, x_10); -x_97 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__64; -x_98 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__67; +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_7); -x_99 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_99, 0, x_7); -lean_ctor_set(x_99, 1, x_97); -lean_ctor_set(x_99, 2, x_96); -lean_ctor_set(x_99, 3, x_98); -x_100 = lean_array_push(x_17, x_99); +x_28 = l_Lean_PrettyPrinter_delab(x_16, x_24, x_7, x_8, x_9, x_10, x_27); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; 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; size_t x_73; size_t x_74; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_mk_syntax_ident(x_15); +x_32 = lean_array_push(x_20, x_31); +lean_inc(x_26); +x_33 = lean_array_push(x_19, x_26); +lean_inc(x_9); +x_34 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_30); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); lean_inc(x_36); -x_101 = lean_array_push(x_100, x_36); -x_102 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_103 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_103, 0, x_21); -lean_ctor_set(x_103, 1, x_102); -lean_ctor_set(x_103, 2, x_101); -x_104 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; -lean_inc(x_7); -x_105 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_105, 0, x_7); -lean_ctor_set(x_105, 1, x_104); -x_106 = lean_array_push(x_58, x_94); -x_107 = lean_array_push(x_106, x_19); -lean_inc(x_107); -x_108 = lean_array_push(x_107, x_103); -lean_inc(x_105); -x_109 = lean_array_push(x_108, x_105); -x_110 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58; -x_111 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_111, 0, x_21); -lean_ctor_set(x_111, 1, x_110); -lean_ctor_set(x_111, 2, x_109); -x_112 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__72; -lean_inc(x_10); -lean_inc(x_13); -x_113 = l_Lean_addMacroScope(x_13, x_112, x_10); -x_114 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__71; -x_115 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__77; -lean_inc(x_7); -x_116 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_116, 0, x_7); -lean_ctor_set(x_116, 1, x_114); -lean_ctor_set(x_116, 2, x_113); -lean_ctor_set(x_116, 3, x_115); -x_117 = lean_array_push(x_17, x_116); -x_118 = lean_array_push(x_117, x_36); -x_119 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_119, 0, x_21); -lean_ctor_set(x_119, 1, x_102); -lean_ctor_set(x_119, 2, x_118); -x_120 = lean_array_push(x_107, x_119); -lean_inc(x_105); -x_121 = lean_array_push(x_120, x_105); -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_21); -lean_ctor_set(x_122, 1, x_110); -lean_ctor_set(x_122, 2, x_121); -x_123 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; -lean_inc(x_7); -x_124 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_124, 0, x_7); -lean_ctor_set(x_124, 1, x_123); -x_125 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__84; -lean_inc(x_10); -lean_inc(x_13); -x_126 = l_Lean_addMacroScope(x_13, x_125, x_10); -x_127 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; -lean_inc(x_7); -x_128 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_128, 0, x_7); -lean_ctor_set(x_128, 1, x_127); -lean_ctor_set(x_128, 2, x_126); -lean_ctor_set(x_128, 3, x_30); -lean_inc(x_128); -x_129 = lean_array_push(x_33, x_128); -x_130 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_130, 0, x_21); -lean_ctor_set(x_130, 1, x_35); -lean_ctor_set(x_130, 2, x_129); -x_131 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__88; -lean_inc(x_10); -lean_inc(x_13); -x_132 = l_Lean_addMacroScope(x_13, x_131, x_10); -x_133 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__87; -x_134 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__91; -lean_inc(x_7); -x_135 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_135, 0, x_7); -lean_ctor_set(x_135, 1, x_133); -lean_ctor_set(x_135, 2, x_132); -lean_ctor_set(x_135, 3, x_134); -lean_inc(x_5); -x_136 = lean_array_push(x_33, x_5); -x_137 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_137, 0, x_21); -lean_ctor_set(x_137, 1, x_35); -lean_ctor_set(x_137, 2, x_136); -x_138 = lean_array_push(x_17, x_135); -x_139 = lean_array_push(x_138, x_137); -x_140 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_140, 0, x_21); -lean_ctor_set(x_140, 1, x_102); -lean_ctor_set(x_140, 2, x_139); -lean_inc(x_140); -lean_inc(x_53); -x_141 = lean_array_push(x_53, x_140); -x_142 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_142, 0, x_21); -lean_ctor_set(x_142, 1, x_35); -lean_ctor_set(x_142, 2, x_141); -x_143 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -lean_inc(x_7); -x_144 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_144, 0, x_7); -lean_ctor_set(x_144, 1, x_143); -x_145 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -lean_inc(x_124); -x_146 = lean_array_push(x_145, x_124); -x_147 = lean_array_push(x_146, x_130); -lean_inc(x_147); -x_148 = lean_array_push(x_147, x_142); -x_149 = lean_array_push(x_148, x_19); -lean_inc(x_144); -x_150 = lean_array_push(x_149, x_144); -x_151 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; -x_152 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_152, 0, x_21); -lean_ctor_set(x_152, 1, x_151); -lean_ctor_set(x_152, 2, x_150); -x_153 = lean_array_push(x_47, x_111); -x_154 = lean_array_push(x_153, x_122); -lean_inc(x_154); -x_155 = lean_array_push(x_154, x_152); -x_156 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_156, 0, x_21); -lean_ctor_set(x_156, 1, x_35); -lean_ctor_set(x_156, 2, x_155); -x_157 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__102; -lean_inc(x_10); -lean_inc(x_13); -x_158 = l_Lean_addMacroScope(x_13, x_157, x_10); -x_159 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__98; -x_160 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__106; -lean_inc(x_7); -x_161 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_161, 0, x_7); -lean_ctor_set(x_161, 1, x_159); -lean_ctor_set(x_161, 2, x_158); -lean_ctor_set(x_161, 3, x_160); -lean_inc(x_161); -x_162 = lean_array_push(x_33, x_161); -x_163 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_163, 0, x_21); -lean_ctor_set(x_163, 1, x_35); -lean_ctor_set(x_163, 2, x_162); -lean_inc(x_32); -x_164 = lean_array_push(x_17, x_32); -x_165 = lean_array_push(x_164, x_163); -x_166 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_166, 0, x_21); -lean_ctor_set(x_166, 1, x_102); -lean_ctor_set(x_166, 2, x_165); -lean_inc(x_53); -x_167 = lean_array_push(x_53, x_166); -x_168 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95; -x_169 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_169, 0, x_21); -lean_ctor_set(x_169, 1, x_168); -lean_ctor_set(x_169, 2, x_167); -lean_inc(x_169); -x_170 = lean_array_push(x_33, x_169); -x_171 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_171, 0, x_21); -lean_ctor_set(x_171, 1, x_35); -lean_ctor_set(x_171, 2, x_170); -x_172 = lean_array_push(x_17, x_156); -lean_inc(x_172); -x_173 = lean_array_push(x_172, x_171); -x_174 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56; -x_175 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_175, 0, x_21); -lean_ctor_set(x_175, 1, x_174); -lean_ctor_set(x_175, 2, x_173); -x_176 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; -lean_inc(x_7); -x_177 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_177, 0, x_7); -lean_ctor_set(x_177, 1, x_176); -x_178 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__113; -lean_inc(x_10); -lean_inc(x_13); -x_179 = l_Lean_addMacroScope(x_13, x_178, x_10); -x_180 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__112; -x_181 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116; -lean_inc(x_7); -x_182 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_182, 0, x_7); -lean_ctor_set(x_182, 1, x_180); -lean_ctor_set(x_182, 2, x_179); -lean_ctor_set(x_182, 3, x_181); -lean_inc(x_1); -x_183 = l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(x_30, x_1); -x_184 = lean_array_push(x_17, x_182); -lean_inc(x_177); -x_185 = lean_array_push(x_47, x_177); -x_186 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; -x_187 = lean_array_push(x_186, x_84); -lean_inc(x_187); -x_188 = lean_array_push(x_187, x_92); -x_189 = lean_array_push(x_188, x_175); -x_190 = lean_array_push(x_17, x_82); -x_191 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__120; -lean_inc(x_7); -x_192 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_192, 0, x_7); -lean_ctor_set(x_192, 1, x_191); -x_193 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__134; -lean_inc(x_10); -lean_inc(x_13); -x_194 = l_Lean_addMacroScope(x_13, x_193, x_10); -x_195 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__133; -lean_inc(x_7); -x_196 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_196, 0, x_7); -lean_ctor_set(x_196, 1, x_195); -lean_ctor_set(x_196, 2, x_194); -lean_ctor_set(x_196, 3, x_30); -x_197 = lean_array_push(x_33, x_88); -x_198 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_198, 0, x_21); -lean_ctor_set(x_198, 1, x_35); -lean_ctor_set(x_198, 2, x_197); -x_199 = lean_array_push(x_17, x_196); -lean_inc(x_199); -x_200 = lean_array_push(x_199, x_198); -x_201 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__130; -x_202 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_202, 0, x_21); -lean_ctor_set(x_202, 1, x_201); -lean_ctor_set(x_202, 2, x_200); -x_203 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; -x_204 = lean_array_push(x_203, x_202); -x_205 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__122; -x_206 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_206, 0, x_21); -lean_ctor_set(x_206, 1, x_205); -lean_ctor_set(x_206, 2, x_204); -x_207 = lean_array_push(x_33, x_206); -x_208 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_208, 0, x_21); -lean_ctor_set(x_208, 1, x_35); -lean_ctor_set(x_208, 2, x_207); -x_209 = lean_array_push(x_47, x_192); -lean_inc(x_209); -x_210 = lean_array_push(x_209, x_208); -lean_inc(x_105); -x_211 = lean_array_push(x_210, x_105); -x_212 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119; -x_213 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_213, 0, x_21); -lean_ctor_set(x_213, 1, x_212); -lean_ctor_set(x_213, 2, x_211); -x_214 = lean_array_push(x_33, x_213); -x_215 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_215, 0, x_21); -lean_ctor_set(x_215, 1, x_35); -lean_ctor_set(x_215, 2, x_214); -x_216 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; -x_217 = lean_array_push(x_216, x_215); -x_218 = lean_array_push(x_217, x_19); -x_219 = lean_array_push(x_218, x_19); -x_220 = lean_array_push(x_219, x_19); -x_221 = lean_array_push(x_220, x_19); -x_222 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_222, 0, x_21); -lean_ctor_set(x_222, 1, x_81); -lean_ctor_set(x_222, 2, x_221); -x_223 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__136; -lean_inc(x_7); -x_224 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_224, 0, x_7); -lean_ctor_set(x_224, 1, x_223); -x_225 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__141; -lean_inc(x_10); -lean_inc(x_13); -x_226 = l_Lean_addMacroScope(x_13, x_225, x_10); -x_227 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__140; -lean_inc(x_7); -x_228 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_228, 0, x_7); -lean_ctor_set(x_228, 1, x_227); -lean_ctor_set(x_228, 2, x_226); -lean_ctor_set(x_228, 3, x_30); -lean_inc(x_228); -x_229 = lean_array_push(x_17, x_228); -x_230 = lean_array_push(x_229, x_19); -x_231 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_231, 0, x_21); -lean_ctor_set(x_231, 1, x_91); -lean_ctor_set(x_231, 2, x_230); -x_232 = lean_array_push(x_172, x_169); -x_233 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__143; -x_234 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_234, 0, x_21); -lean_ctor_set(x_234, 1, x_233); -lean_ctor_set(x_234, 2, x_232); -x_235 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; -lean_inc(x_10); -lean_inc(x_13); -x_236 = l_Lean_addMacroScope(x_13, x_235, x_10); -x_237 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__146; -x_238 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__152; -lean_inc(x_7); -x_239 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_239, 0, x_7); -lean_ctor_set(x_239, 1, x_237); -lean_ctor_set(x_239, 2, x_236); -lean_ctor_set(x_239, 3, x_238); -x_240 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__155; -lean_inc(x_7); -x_241 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_241, 0, x_7); -lean_ctor_set(x_241, 1, x_240); -x_242 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__158; -lean_inc(x_7); -x_243 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_243, 0, x_7); -lean_ctor_set(x_243, 1, x_242); -x_244 = lean_array_push(x_33, x_243); -x_245 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__157; -x_246 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_246, 0, x_21); -lean_ctor_set(x_246, 1, x_245); -lean_ctor_set(x_246, 2, x_244); -x_247 = lean_array_push(x_33, x_246); -x_248 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_248, 0, x_21); -lean_ctor_set(x_248, 1, x_35); -lean_ctor_set(x_248, 2, x_247); -x_249 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__159; -lean_inc(x_7); -x_250 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_250, 0, x_7); -lean_ctor_set(x_250, 1, x_249); -x_251 = lean_array_push(x_47, x_241); -x_252 = lean_array_push(x_251, x_248); -x_253 = lean_array_push(x_252, x_250); -x_254 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__154; -x_255 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_255, 0, x_21); -lean_ctor_set(x_255, 1, x_254); -lean_ctor_set(x_255, 2, x_253); -x_256 = lean_array_push(x_33, x_255); -x_257 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_257, 0, x_21); -lean_ctor_set(x_257, 1, x_35); -lean_ctor_set(x_257, 2, x_256); -x_258 = lean_array_push(x_17, x_239); -x_259 = lean_array_push(x_258, x_257); -x_260 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_260, 0, x_21); -lean_ctor_set(x_260, 1, x_102); -lean_ctor_set(x_260, 2, x_259); -lean_inc(x_185); -x_261 = lean_array_push(x_185, x_260); -x_262 = lean_array_push(x_261, x_19); -x_263 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__108; -x_264 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_264, 0, x_21); -lean_ctor_set(x_264, 1, x_263); -lean_ctor_set(x_264, 2, x_262); -x_265 = lean_array_push(x_33, x_264); -x_266 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_266, 0, x_21); -lean_ctor_set(x_266, 1, x_35); -lean_ctor_set(x_266, 2, x_265); -x_267 = lean_array_push(x_58, x_224); -lean_inc(x_267); -x_268 = lean_array_push(x_267, x_231); -x_269 = lean_array_push(x_268, x_234); -x_270 = lean_array_push(x_269, x_266); -x_271 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__137; -x_272 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_272, 0, x_21); -lean_ctor_set(x_272, 1, x_271); -lean_ctor_set(x_272, 2, x_270); -x_273 = lean_array_push(x_17, x_222); -x_274 = lean_array_push(x_273, x_272); -x_275 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__37; -x_276 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_276, 0, x_21); -lean_ctor_set(x_276, 1, x_275); -lean_ctor_set(x_276, 2, x_274); -x_277 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__163; -lean_inc(x_10); -lean_inc(x_13); -x_278 = l_Lean_addMacroScope(x_13, x_277, x_10); -x_279 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__162; -lean_inc(x_7); -x_280 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_280, 0, x_7); -lean_ctor_set(x_280, 1, x_279); -lean_ctor_set(x_280, 2, x_278); -lean_ctor_set(x_280, 3, x_30); -lean_inc(x_280); -x_281 = lean_array_push(x_17, x_280); -x_282 = lean_array_push(x_281, x_19); -x_283 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_283, 0, x_21); -lean_ctor_set(x_283, 1, x_91); -lean_ctor_set(x_283, 2, x_282); -lean_inc(x_161); -lean_inc(x_53); -x_284 = lean_array_push(x_53, x_161); -x_285 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_285, 0, x_21); -lean_ctor_set(x_285, 1, x_35); -lean_ctor_set(x_285, 2, x_284); -x_286 = lean_array_push(x_147, x_285); -x_287 = lean_array_push(x_286, x_19); -lean_inc(x_144); -x_288 = lean_array_push(x_287, x_144); -x_289 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_289, 0, x_21); -lean_ctor_set(x_289, 1, x_151); -lean_ctor_set(x_289, 2, x_288); -x_290 = lean_array_push(x_154, x_289); -x_291 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_291, 0, x_21); -lean_ctor_set(x_291, 1, x_35); -lean_ctor_set(x_291, 2, x_290); -x_292 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__167; -lean_inc(x_10); -lean_inc(x_13); -x_293 = l_Lean_addMacroScope(x_13, x_292, x_10); -x_294 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__166; -x_295 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__169; -lean_inc(x_7); -x_296 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_296, 0, x_7); -lean_ctor_set(x_296, 1, x_294); -lean_ctor_set(x_296, 2, x_293); -lean_ctor_set(x_296, 3, x_295); -x_297 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__173; -lean_inc(x_10); -lean_inc(x_13); -x_298 = l_Lean_addMacroScope(x_13, x_297, x_10); -x_299 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__172; -x_300 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__175; -lean_inc(x_7); -x_301 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_301, 0, x_7); -lean_ctor_set(x_301, 1, x_299); -lean_ctor_set(x_301, 2, x_298); -lean_ctor_set(x_301, 3, x_300); -x_302 = lean_array_push(x_17, x_140); -x_303 = lean_array_push(x_302, x_19); -x_304 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_304, 0, x_21); -lean_ctor_set(x_304, 1, x_35); -lean_ctor_set(x_304, 2, x_303); -x_305 = lean_array_push(x_47, x_124); -x_306 = lean_array_push(x_305, x_304); -x_307 = lean_array_push(x_306, x_144); -x_308 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__177; -x_309 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_309, 0, x_21); -lean_ctor_set(x_309, 1, x_308); -lean_ctor_set(x_309, 2, x_307); -x_310 = lean_array_push(x_47, x_301); -x_311 = lean_array_push(x_310, x_32); -lean_inc(x_309); -x_312 = lean_array_push(x_311, x_309); -x_313 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_313, 0, x_21); -lean_ctor_set(x_313, 1, x_35); -lean_ctor_set(x_313, 2, x_312); -x_314 = lean_array_push(x_17, x_296); -x_315 = lean_array_push(x_314, x_313); -x_316 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_316, 0, x_21); -lean_ctor_set(x_316, 1, x_102); -lean_ctor_set(x_316, 2, x_315); -lean_inc(x_53); -x_317 = lean_array_push(x_53, x_316); -x_318 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_318, 0, x_21); -lean_ctor_set(x_318, 1, x_168); -lean_ctor_set(x_318, 2, x_317); -lean_inc(x_318); -x_319 = lean_array_push(x_33, x_318); -x_320 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_320, 0, x_21); -lean_ctor_set(x_320, 1, x_35); -lean_ctor_set(x_320, 2, x_319); -x_321 = lean_array_push(x_17, x_291); -lean_inc(x_321); -x_322 = lean_array_push(x_321, x_320); -x_323 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_323, 0, x_21); -lean_ctor_set(x_323, 1, x_174); -lean_ctor_set(x_323, 2, x_322); -x_324 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__182; -lean_inc(x_10); -lean_inc(x_13); -x_325 = l_Lean_addMacroScope(x_13, x_324, x_10); -x_326 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__180; -x_327 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__185; -lean_inc(x_7); -x_328 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_328, 0, x_7); -lean_ctor_set(x_328, 1, x_326); -lean_ctor_set(x_328, 2, x_325); -lean_ctor_set(x_328, 3, x_327); -x_329 = lean_array_push(x_47, x_5); -x_330 = lean_array_push(x_17, x_328); -x_331 = lean_array_push(x_187, x_283); -x_332 = lean_array_push(x_331, x_323); -x_333 = lean_array_push(x_33, x_280); -x_334 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_334, 0, x_21); -lean_ctor_set(x_334, 1, x_35); -lean_ctor_set(x_334, 2, x_333); -x_335 = lean_array_push(x_199, x_334); -x_336 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_336, 0, x_21); -lean_ctor_set(x_336, 1, x_201); -lean_ctor_set(x_336, 2, x_335); -x_337 = lean_array_push(x_203, x_336); -x_338 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_338, 0, x_21); -lean_ctor_set(x_338, 1, x_205); -lean_ctor_set(x_338, 2, x_337); -x_339 = lean_array_push(x_33, x_338); -x_340 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_340, 0, x_21); -lean_ctor_set(x_340, 1, x_35); -lean_ctor_set(x_340, 2, x_339); -x_341 = lean_array_push(x_209, x_340); -x_342 = lean_array_push(x_341, x_105); -x_343 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_343, 0, x_21); -lean_ctor_set(x_343, 1, x_212); -lean_ctor_set(x_343, 2, x_342); -x_344 = lean_array_push(x_33, x_343); -x_345 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_345, 0, x_21); -lean_ctor_set(x_345, 1, x_35); -lean_ctor_set(x_345, 2, x_344); -x_346 = lean_array_push(x_216, x_345); -x_347 = lean_array_push(x_346, x_19); -x_348 = lean_array_push(x_347, x_19); -x_349 = lean_array_push(x_348, x_19); -x_350 = lean_array_push(x_349, x_19); -x_351 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_351, 0, x_21); -lean_ctor_set(x_351, 1, x_81); -lean_ctor_set(x_351, 2, x_350); -x_352 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__189; -lean_inc(x_10); -lean_inc(x_13); -x_353 = l_Lean_addMacroScope(x_13, x_352, x_10); -x_354 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__188; -lean_inc(x_7); -x_355 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_355, 0, x_7); -lean_ctor_set(x_355, 1, x_354); -lean_ctor_set(x_355, 2, x_353); -lean_ctor_set(x_355, 3, x_30); -lean_inc(x_355); -x_356 = lean_array_push(x_17, x_355); -x_357 = lean_array_push(x_356, x_19); -x_358 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_358, 0, x_21); -lean_ctor_set(x_358, 1, x_91); -lean_ctor_set(x_358, 2, x_357); -x_359 = lean_array_push(x_321, x_318); -x_360 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_360, 0, x_21); -lean_ctor_set(x_360, 1, x_233); -lean_ctor_set(x_360, 2, x_359); -x_361 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__193; -lean_inc(x_10); -lean_inc(x_13); -x_362 = l_Lean_addMacroScope(x_13, x_361, x_10); -x_363 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__192; -x_364 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__198; -lean_inc(x_7); -x_365 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_365, 0, x_7); -lean_ctor_set(x_365, 1, x_363); -lean_ctor_set(x_365, 2, x_362); -lean_ctor_set(x_365, 3, x_364); -x_366 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__201; -lean_inc(x_7); -x_367 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_367, 0, x_7); -lean_ctor_set(x_367, 1, x_366); -x_368 = lean_array_push(x_33, x_367); -x_369 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__200; -x_370 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_370, 0, x_21); -lean_ctor_set(x_370, 1, x_369); -lean_ctor_set(x_370, 2, x_368); -x_371 = lean_array_push(x_33, x_370); -x_372 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_372, 0, x_21); -lean_ctor_set(x_372, 1, x_35); -lean_ctor_set(x_372, 2, x_371); -x_373 = lean_array_push(x_17, x_365); -x_374 = lean_array_push(x_373, x_372); -x_375 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_375, 0, x_21); -lean_ctor_set(x_375, 1, x_102); -lean_ctor_set(x_375, 2, x_374); -lean_inc(x_185); -x_376 = lean_array_push(x_185, x_375); -x_377 = lean_array_push(x_376, x_19); -x_378 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_378, 0, x_21); -lean_ctor_set(x_378, 1, x_263); -lean_ctor_set(x_378, 2, x_377); -x_379 = lean_array_push(x_33, x_378); -x_380 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_380, 0, x_21); -lean_ctor_set(x_380, 1, x_35); -lean_ctor_set(x_380, 2, x_379); -x_381 = lean_array_push(x_267, x_358); -x_382 = lean_array_push(x_381, x_360); -x_383 = lean_array_push(x_382, x_380); -x_384 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_384, 0, x_21); -lean_ctor_set(x_384, 1, x_271); -lean_ctor_set(x_384, 2, x_383); -x_385 = lean_array_push(x_17, x_351); -x_386 = lean_array_push(x_385, x_384); -x_387 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_387, 0, x_21); -lean_ctor_set(x_387, 1, x_275); -lean_ctor_set(x_387, 2, x_386); -x_388 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205; -lean_inc(x_7); -x_389 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_389, 0, x_7); -lean_ctor_set(x_389, 1, x_388); -x_390 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__210; -lean_inc(x_10); -lean_inc(x_13); -x_391 = l_Lean_addMacroScope(x_13, x_390, x_10); -x_392 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__209; -x_393 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__213; -lean_inc(x_7); -x_394 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_394, 0, x_7); -lean_ctor_set(x_394, 1, x_392); -lean_ctor_set(x_394, 2, x_391); -lean_ctor_set(x_394, 3, x_393); -x_395 = lean_array_push(x_17, x_309); -x_396 = lean_array_push(x_395, x_161); -x_397 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_397, 0, x_21); -lean_ctor_set(x_397, 1, x_35); -lean_ctor_set(x_397, 2, x_396); -x_398 = lean_array_push(x_17, x_394); -x_399 = lean_array_push(x_398, x_397); -x_400 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_400, 0, x_21); -lean_ctor_set(x_400, 1, x_102); -lean_ctor_set(x_400, 2, x_399); -x_401 = lean_array_push(x_53, x_400); -x_402 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_402, 0, x_21); -lean_ctor_set(x_402, 1, x_168); -lean_ctor_set(x_402, 2, x_401); -x_403 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__214; -x_404 = lean_array_push(x_403, x_402); -x_405 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_405, 0, x_21); -lean_ctor_set(x_405, 1, x_233); -lean_ctor_set(x_405, 2, x_404); -x_406 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224; -lean_inc(x_10); -lean_inc(x_13); -x_407 = l_Lean_addMacroScope(x_13, x_406, x_10); -x_408 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223; -x_409 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__227; -lean_inc(x_7); -x_410 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_410, 0, x_7); -lean_ctor_set(x_410, 1, x_408); -lean_ctor_set(x_410, 2, x_407); -lean_ctor_set(x_410, 3, x_409); -x_411 = lean_array_push(x_17, x_410); -x_412 = lean_array_push(x_411, x_19); -x_413 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__220; -x_414 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_414, 0, x_21); -lean_ctor_set(x_414, 1, x_413); -lean_ctor_set(x_414, 2, x_412); -x_415 = lean_array_push(x_47, x_414); -lean_inc(x_177); -x_416 = lean_array_push(x_415, x_177); -x_417 = lean_array_push(x_416, x_228); -x_418 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__218; -x_419 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_419, 0, x_21); -lean_ctor_set(x_419, 1, x_418); -lean_ctor_set(x_419, 2, x_417); -x_420 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231; -x_421 = l_Lean_addMacroScope(x_13, x_420, x_10); -x_422 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230; -x_423 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__234; -lean_inc(x_7); -x_424 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_424, 0, x_7); -lean_ctor_set(x_424, 1, x_422); -lean_ctor_set(x_424, 2, x_421); -lean_ctor_set(x_424, 3, x_423); -x_425 = lean_array_push(x_17, x_424); -x_426 = lean_array_push(x_425, x_19); -x_427 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_427, 0, x_21); -lean_ctor_set(x_427, 1, x_413); -lean_ctor_set(x_427, 2, x_426); -x_428 = lean_array_push(x_47, x_427); -x_429 = lean_array_push(x_428, x_177); -x_430 = lean_array_push(x_429, x_355); -x_431 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_431, 0, x_21); -lean_ctor_set(x_431, 1, x_418); -lean_ctor_set(x_431, 2, x_430); -x_432 = lean_array_push(x_47, x_419); -x_433 = lean_array_push(x_432, x_19); -x_434 = lean_array_push(x_433, x_431); -x_435 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_435, 0, x_21); -lean_ctor_set(x_435, 1, x_35); -lean_ctor_set(x_435, 2, x_434); -x_436 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -x_437 = lean_array_push(x_436, x_27); -x_438 = lean_array_push(x_437, x_19); -x_439 = lean_array_push(x_438, x_435); -x_440 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__237; -x_441 = lean_array_push(x_439, x_440); -x_442 = lean_array_push(x_441, x_19); -x_443 = lean_array_push(x_442, x_57); -x_444 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__216; -x_445 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_445, 0, x_21); -lean_ctor_set(x_445, 1, x_444); -lean_ctor_set(x_445, 2, x_443); -lean_inc(x_185); -x_446 = lean_array_push(x_185, x_445); -x_447 = lean_array_push(x_446, x_19); -x_448 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_448, 0, x_21); -lean_ctor_set(x_448, 1, x_263); -lean_ctor_set(x_448, 2, x_447); -x_449 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__239; -x_450 = lean_array_push(x_449, x_389); -x_451 = lean_array_push(x_450, x_19); -x_452 = lean_array_push(x_451, x_19); -x_453 = lean_array_push(x_452, x_405); -x_454 = lean_array_push(x_453, x_448); -x_455 = lean_array_push(x_454, x_19); -x_456 = lean_array_push(x_455, x_19); -x_457 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206; -x_458 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_458, 0, x_21); -lean_ctor_set(x_458, 1, x_457); -lean_ctor_set(x_458, 2, x_456); -x_459 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__240; -x_460 = lean_array_push(x_459, x_458); -x_461 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_461, 0, x_21); -lean_ctor_set(x_461, 1, x_275); -lean_ctor_set(x_461, 2, x_460); -x_462 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241; -x_463 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_463, 0, x_7); -lean_ctor_set(x_463, 1, x_462); -x_464 = lean_array_push(x_17, x_463); -x_465 = lean_array_push(x_464, x_19); -x_466 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__242; -x_467 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_467, 0, x_21); -lean_ctor_set(x_467, 1, x_466); -lean_ctor_set(x_467, 2, x_465); -x_468 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238; -x_469 = lean_array_push(x_468, x_23); -x_470 = lean_array_push(x_469, x_70); -if (lean_obj_tag(x_183) == 0) -{ -lean_object* x_524; -x_524 = l_Lean_quoteNameMk(x_1); -x_471 = x_524; -goto block_523; +lean_dec(x_34); +x_37 = lean_ctor_get(x_9, 10); +lean_inc(x_37); +x_38 = lean_st_ref_get(x_10, x_36); +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = lean_ctor_get(x_39, 0); +lean_inc(x_41); +lean_dec(x_39); +x_42 = lean_environment_main_module(x_41); +x_43 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3; +lean_inc(x_35); +x_44 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_44, 0, x_35); +lean_ctor_set(x_44, 1, x_43); +x_45 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; +x_46 = l_Lean_addMacroScope(x_42, x_45, x_37); +x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; +x_48 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5; +lean_inc(x_35); +x_49 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_49, 0, x_35); +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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_51 = lean_array_push(x_50, x_29); +x_52 = lean_array_push(x_51, x_26); +x_53 = lean_box(2); +x_54 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_55 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +lean_ctor_set(x_55, 2, x_52); +x_56 = lean_array_push(x_50, x_49); +x_57 = lean_array_push(x_56, x_55); +x_58 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; +x_59 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_59, 0, x_53); +lean_ctor_set(x_59, 1, x_58); +lean_ctor_set(x_59, 2, x_57); +x_60 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; +x_61 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_61, 0, x_35); +lean_ctor_set(x_61, 1, x_60); +x_62 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_63 = lean_array_push(x_62, x_44); +x_64 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_65 = lean_array_push(x_63, x_64); +x_66 = lean_array_push(x_65, x_59); +x_67 = lean_array_push(x_66, x_61); +x_68 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__2; +x_69 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_69, 0, x_53); +lean_ctor_set(x_69, 1, x_68); +lean_ctor_set(x_69, 2, x_67); +x_70 = lean_array_push(x_17, x_69); +x_71 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_71, 0, x_33); +lean_ctor_set(x_71, 1, x_32); +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +x_73 = 1; +x_74 = lean_usize_add(x_3, x_73); +x_3 = x_74; +x_4 = x_72; +x_11 = x_40; +goto _start; } else { -lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; -lean_dec(x_1); -x_525 = lean_ctor_get(x_183, 0); -lean_inc(x_525); -lean_dec(x_183); -x_526 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__245; -x_527 = l_String_intercalate(x_526, x_525); -x_528 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__246; -x_529 = lean_string_append(x_528, x_527); -lean_dec(x_527); -x_530 = l_Lean_Syntax_mkNameLit(x_529, x_21); -x_531 = lean_array_push(x_33, x_530); -x_532 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__244; -x_533 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_533, 0, x_21); -lean_ctor_set(x_533, 1, x_532); -lean_ctor_set(x_533, 2, x_531); -x_471 = x_533; -goto block_523; -} -block_523: -{ -lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; -lean_inc(x_471); -x_472 = lean_array_push(x_17, x_471); -lean_inc(x_128); -x_473 = lean_array_push(x_472, x_128); -x_474 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_474, 0, x_21); -lean_ctor_set(x_474, 1, x_35); -lean_ctor_set(x_474, 2, x_473); -x_475 = lean_array_push(x_184, x_474); -x_476 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_476, 0, x_21); -lean_ctor_set(x_476, 1, x_102); -lean_ctor_set(x_476, 2, x_475); -lean_inc(x_185); -x_477 = lean_array_push(x_185, x_476); -x_478 = lean_array_push(x_477, x_19); -x_479 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_479, 0, x_21); -lean_ctor_set(x_479, 1, x_263); -lean_ctor_set(x_479, 2, x_478); -x_480 = lean_array_push(x_189, x_479); -x_481 = lean_array_push(x_480, x_19); -x_482 = lean_array_push(x_481, x_19); -x_483 = lean_array_push(x_482, x_19); -x_484 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__48; -x_485 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_485, 0, x_21); -lean_ctor_set(x_485, 1, x_484); -lean_ctor_set(x_485, 2, x_483); -lean_inc(x_190); -x_486 = lean_array_push(x_190, x_485); -x_487 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_487, 0, x_21); -lean_ctor_set(x_487, 1, x_275); -lean_ctor_set(x_487, 2, x_486); -x_488 = lean_array_push(x_329, x_471); -x_489 = lean_array_push(x_488, x_128); -x_490 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_490, 0, x_21); -lean_ctor_set(x_490, 1, x_35); -lean_ctor_set(x_490, 2, x_489); -x_491 = lean_array_push(x_330, x_490); -x_492 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_492, 0, x_21); -lean_ctor_set(x_492, 1, x_102); -lean_ctor_set(x_492, 2, x_491); -x_493 = lean_array_push(x_185, x_492); -x_494 = lean_array_push(x_493, x_19); -x_495 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_495, 0, x_21); -lean_ctor_set(x_495, 1, x_263); -lean_ctor_set(x_495, 2, x_494); -x_496 = lean_array_push(x_332, x_495); -x_497 = lean_array_push(x_496, x_19); -x_498 = lean_array_push(x_497, x_19); -x_499 = lean_array_push(x_498, x_19); -x_500 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_500, 0, x_21); -lean_ctor_set(x_500, 1, x_484); -lean_ctor_set(x_500, 2, x_499); -x_501 = lean_array_push(x_190, x_500); -x_502 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_502, 0, x_21); -lean_ctor_set(x_502, 1, x_275); -lean_ctor_set(x_502, 2, x_501); -x_503 = lean_array_push(x_470, x_487); -x_504 = lean_array_push(x_503, x_276); -x_505 = lean_array_push(x_504, x_502); -x_506 = lean_array_push(x_505, x_387); -x_507 = lean_array_push(x_506, x_461); -x_508 = lean_array_push(x_507, x_467); -x_509 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_509, 0, x_21); -lean_ctor_set(x_509, 1, x_35); -lean_ctor_set(x_509, 2, x_508); -x_510 = l_Lean_Elab_Command_elabCommand(x_509, x_2, x_3, x_14); -if (lean_obj_tag(x_510) == 0) +uint8_t x_76; +lean_dec(x_26); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_76 = !lean_is_exclusive(x_28); +if (x_76 == 0) +{ +return x_28; +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_28, 0); +x_78 = lean_ctor_get(x_28, 1); +lean_inc(x_78); +lean_inc(x_77); +lean_dec(x_28); +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; +} +} +} +else { -uint8_t x_511; -x_511 = !lean_is_exclusive(x_510); -if (x_511 == 0) +uint8_t x_80; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_80 = !lean_is_exclusive(x_25); +if (x_80 == 0) { -lean_object* x_512; uint8_t x_513; lean_object* x_514; -x_512 = lean_ctor_get(x_510, 0); -lean_dec(x_512); -x_513 = 1; -x_514 = lean_box(x_513); -lean_ctor_set(x_510, 0, x_514); -return x_510; +return x_25; } else { -lean_object* x_515; uint8_t x_516; lean_object* x_517; lean_object* x_518; -x_515 = lean_ctor_get(x_510, 1); -lean_inc(x_515); -lean_dec(x_510); -x_516 = 1; -x_517 = lean_box(x_516); -x_518 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_518, 0, x_517); -lean_ctor_set(x_518, 1, x_515); -return x_518; +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_25, 0); +x_82 = lean_ctor_get(x_25, 1); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_25); +x_83 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_83, 0, x_81); +lean_ctor_set(x_83, 1, x_82); +return x_83; +} } } else { -uint8_t x_519; -x_519 = !lean_is_exclusive(x_510); -if (x_519 == 0) +uint8_t x_84; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_84 = !lean_is_exclusive(x_21); +if (x_84 == 0) { -return x_510; +return x_21; } else { -lean_object* x_520; lean_object* x_521; lean_object* x_522; -x_520 = lean_ctor_get(x_510, 0); -x_521 = lean_ctor_get(x_510, 1); -lean_inc(x_521); -lean_inc(x_520); -lean_dec(x_510); -x_522 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_522, 0, x_520); -lean_ctor_set(x_522, 1, x_521); -return x_522; +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_21, 0); +x_86 = lean_ctor_get(x_21, 1); +lean_inc(x_86); +lean_inc(x_85); +lean_dec(x_21); +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +return x_87; } } } } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1() { _start: { -lean_object* x_4; lean_object* x_5; -x_4 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_4, 0, x_1); -x_5 = lean_apply_2(x_2, lean_box(0), x_4); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("structInstField", 15); +return x_1; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2() { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_box(0); -lean_inc(x_5); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -x_8 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1___boxed), 3, 2); -lean_closure_set(x_8, 0, x_3); -lean_closure_set(x_8, 1, x_5); -x_9 = lean_apply_4(x_2, lean_box(0), lean_box(0), x_7, x_8); -return x_9; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("structInstLVal", 14); +return x_1; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3() { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_apply_2(x_1, x_2, x_3); -lean_inc(x_5); -x_9 = l_Lean_Meta_forallTelescopeReducing___rarg(x_4, x_5, lean_box(0), x_7, x_8); -lean_inc(x_6); -x_10 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__2), 3, 2); -lean_closure_set(x_10, 0, x_5); -lean_closure_set(x_10, 1, x_6); -x_11 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_9, x_10); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("liftMethod", 10); +return x_1; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4() { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -lean_dec(x_11); -x_13 = l_Lean_Expr_const___override(x_12, x_1); -x_14 = l_Lean_mkAppN(x_13, x_2); -x_15 = lean_alloc_closure((void*)(l_Lean_Meta_inferType___boxed), 6, 1); -lean_closure_set(x_15, 0, x_14); -x_16 = lean_apply_2(x_3, lean_box(0), x_15); -lean_inc(x_9); -x_17 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__3), 7, 6); -lean_closure_set(x_17, 0, x_4); -lean_closure_set(x_17, 1, x_5); -lean_closure_set(x_17, 2, x_6); -lean_closure_set(x_17, 3, x_7); -lean_closure_set(x_17, 4, x_8); -lean_closure_set(x_17, 5, x_9); -x_18 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_16, x_17); -return x_18; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("←", 3); +return x_1; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5() { _start: { -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_apply_2(x_12, lean_box(0), x_10); -return x_13; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("proj", 4); +return x_1; } -else -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_9, 0); -lean_inc(x_14); -lean_dec(x_9); -x_15 = l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg(x_1, x_2, x_3, lean_box(0), x_4, x_5, x_6, x_7, x_8, x_14); -return x_15; } +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("a", 1); +return x_1; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7() { _start: { -if (lean_obj_tag(x_9) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8() { +_start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_apply_2(x_12, lean_box(0), x_10); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_14 = lean_ctor_get(x_9, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_9, 1); -lean_inc(x_15); -lean_dec(x_9); -x_16 = lean_ctor_get(x_1, 1); -lean_inc(x_16); -lean_inc(x_14); -x_17 = lean_alloc_closure((void*)(l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1___boxed), 6, 1); -lean_closure_set(x_17, 0, x_14); -lean_inc(x_3); -x_18 = lean_apply_2(x_3, lean_box(0), x_17); -lean_inc(x_8); -lean_inc(x_1); -lean_inc(x_2); -lean_inc(x_6); -lean_inc(x_3); -lean_inc(x_5); -lean_inc(x_7); -x_19 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__4), 10, 9); -lean_closure_set(x_19, 0, x_7); -lean_closure_set(x_19, 1, x_5); -lean_closure_set(x_19, 2, x_3); -lean_closure_set(x_19, 3, x_6); -lean_closure_set(x_19, 4, x_10); -lean_closure_set(x_19, 5, x_14); -lean_closure_set(x_19, 6, x_2); -lean_closure_set(x_19, 7, x_1); -lean_closure_set(x_19, 8, x_8); -lean_inc(x_8); -x_20 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_18, x_19); -x_21 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__5), 9, 8); -lean_closure_set(x_21, 0, x_1); -lean_closure_set(x_21, 1, x_2); -lean_closure_set(x_21, 2, x_3); -lean_closure_set(x_21, 3, x_5); -lean_closure_set(x_21, 4, x_6); -lean_closure_set(x_21, 5, x_7); -lean_closure_set(x_21, 6, x_8); -lean_closure_set(x_21, 7, x_15); -x_22 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_20, x_21); -return x_22; -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1(lean_object* x_1) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg), 10, 0); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_4, x_3); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_10); +lean_dec(x_2); lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_apply_2(x_4, lean_box(0), x_2); -return x_5; -} +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_5); +lean_ctor_set(x_14, 1, x_12); +return x_14; } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_9, 1); +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; size_t x_78; size_t x_79; lean_object* x_80; +x_15 = lean_array_uget(x_5, x_4); +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_array_uset(x_5, x_4, x_16); lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_box(0); -x_12 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_10, x_11); -x_13 = lean_ctor_get(x_1, 1); -lean_inc(x_13); -x_14 = lean_ctor_get(x_5, 4); -lean_inc(x_14); -lean_dec(x_5); -lean_inc(x_13); +x_18 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_10, x_11, x_12); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_ctor_get(x_10, 10); +lean_inc(x_21); +x_22 = lean_st_ref_get(x_11, x_20); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_environment_main_module(x_25); +x_27 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__5; lean_inc(x_1); -x_15 = l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg(x_1, x_2, x_3, lean_box(0), x_6, x_7, x_12, x_13, x_14, x_8); -x_16 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_foldWithConstructors___rarg___lambda__1), 2, 1); -lean_closure_set(x_16, 0, x_1); -x_17 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_15, x_16); -return x_17; -} +x_28 = l_Lean_Name_str___override(x_1, x_27); +x_29 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; +x_30 = l_Lean_Name_str___override(x_28, x_29); +x_31 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1; +lean_inc(x_30); +x_32 = l_Lean_Name_str___override(x_30, x_31); +x_33 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2; +lean_inc(x_30); +x_34 = l_Lean_Name_str___override(x_30, x_33); +x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +lean_inc(x_15); +x_36 = lean_array_push(x_35, x_15); +x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_38 = lean_array_push(x_36, x_37); +x_39 = lean_box(2); +x_40 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_34); +lean_ctor_set(x_40, 2, x_38); +x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; +lean_inc(x_19); +x_42 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_42, 0, x_19); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3; +lean_inc(x_30); +x_44 = l_Lean_Name_str___override(x_30, x_43); +x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; +lean_inc(x_19); +x_46 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_46, 0, x_19); +lean_ctor_set(x_46, 1, x_45); +x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; +lean_inc(x_30); +x_48 = l_Lean_Name_str___override(x_30, x_47); +lean_inc(x_2); +x_49 = lean_mk_syntax_ident(x_2); +x_50 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5; +x_51 = l_Lean_Name_str___override(x_30, x_50); +x_52 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9; +x_53 = l_Lean_addMacroScope(x_26, x_52, x_21); +x_54 = lean_box(0); +x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8; +lean_inc(x_19); +x_56 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_56, 0, x_19); +lean_ctor_set(x_56, 1, x_55); +lean_ctor_set(x_56, 2, x_53); +lean_ctor_set(x_56, 3, x_54); +x_57 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__156; +x_58 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_58, 0, x_19); +lean_ctor_set(x_58, 1, x_57); +x_59 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +x_60 = lean_array_push(x_59, x_56); +x_61 = lean_array_push(x_60, x_58); +x_62 = lean_array_push(x_61, x_15); +x_63 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_63, 0, x_39); +lean_ctor_set(x_63, 1, x_51); +lean_ctor_set(x_63, 2, x_62); +x_64 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_65 = lean_array_push(x_64, x_63); +x_66 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_67 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_67, 0, x_39); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set(x_67, 2, x_65); +x_68 = lean_array_push(x_35, x_49); +x_69 = lean_array_push(x_68, x_67); +x_70 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_70, 0, x_39); +lean_ctor_set(x_70, 1, x_48); +lean_ctor_set(x_70, 2, x_69); +x_71 = lean_array_push(x_35, x_46); +x_72 = lean_array_push(x_71, x_70); +x_73 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_73, 0, x_39); +lean_ctor_set(x_73, 1, x_44); +lean_ctor_set(x_73, 2, x_72); +x_74 = lean_array_push(x_59, x_40); +x_75 = lean_array_push(x_74, x_42); +x_76 = lean_array_push(x_75, x_73); +x_77 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_77, 0, x_39); +lean_ctor_set(x_77, 1, x_32); +lean_ctor_set(x_77, 2, x_76); +x_78 = 1; +x_79 = lean_usize_add(x_4, x_78); +x_80 = lean_array_uset(x_17, x_4, x_77); +x_4 = x_79; +x_5 = x_80; +x_12 = x_24; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_foldWithConstructors___rarg), 8, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_4; -x_4 = l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; -} +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_4, x_3); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_10); +lean_dec(x_2); +lean_dec(x_1); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_5); +lean_ctor_set(x_14, 1, x_12); +return x_14; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_5); -x_7 = lean_array_push(x_2, x_6); -x_8 = lean_ctor_get(x_3, 0); -lean_inc(x_8); -lean_dec(x_3); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = lean_box(0); -lean_inc(x_9); -x_11 = lean_apply_2(x_9, lean_box(0), x_10); -x_12 = lean_alloc_closure((void*)(l_List_forIn_loop___at_Lean_Server_RpcEncoding_foldWithConstructors___spec__1___rarg___lambda__1___boxed), 3, 2); -lean_closure_set(x_12, 0, x_7); -lean_closure_set(x_12, 1, x_9); -x_13 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_11, x_12); -return x_13; -} +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; 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; size_t x_78; size_t x_79; lean_object* x_80; +x_15 = lean_array_uget(x_5, x_4); +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_array_uset(x_5, x_4, x_16); +lean_inc(x_10); +x_18 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_10, x_11, x_12); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_ctor_get(x_10, 10); +lean_inc(x_21); +x_22 = lean_st_ref_get(x_11, x_20); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_environment_main_module(x_25); +x_27 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__5; +lean_inc(x_1); +x_28 = l_Lean_Name_str___override(x_1, x_27); +x_29 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; +x_30 = l_Lean_Name_str___override(x_28, x_29); +x_31 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1; +lean_inc(x_30); +x_32 = l_Lean_Name_str___override(x_30, x_31); +x_33 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2; +lean_inc(x_30); +x_34 = l_Lean_Name_str___override(x_30, x_33); +x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +lean_inc(x_15); +x_36 = lean_array_push(x_35, x_15); +x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_38 = lean_array_push(x_36, x_37); +x_39 = lean_box(2); +x_40 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_34); +lean_ctor_set(x_40, 2, x_38); +x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; +lean_inc(x_19); +x_42 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_42, 0, x_19); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3; +lean_inc(x_30); +x_44 = l_Lean_Name_str___override(x_30, x_43); +x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; +lean_inc(x_19); +x_46 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_46, 0, x_19); +lean_ctor_set(x_46, 1, x_45); +x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; +lean_inc(x_30); +x_48 = l_Lean_Name_str___override(x_30, x_47); +lean_inc(x_2); +x_49 = lean_mk_syntax_ident(x_2); +x_50 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5; +x_51 = l_Lean_Name_str___override(x_30, x_50); +x_52 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9; +x_53 = l_Lean_addMacroScope(x_26, x_52, x_21); +x_54 = lean_box(0); +x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8; +lean_inc(x_19); +x_56 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_56, 0, x_19); +lean_ctor_set(x_56, 1, x_55); +lean_ctor_set(x_56, 2, x_53); +lean_ctor_set(x_56, 3, x_54); +x_57 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__156; +x_58 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_58, 0, x_19); +lean_ctor_set(x_58, 1, x_57); +x_59 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +x_60 = lean_array_push(x_59, x_56); +x_61 = lean_array_push(x_60, x_58); +x_62 = lean_array_push(x_61, x_15); +x_63 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_63, 0, x_39); +lean_ctor_set(x_63, 1, x_51); +lean_ctor_set(x_63, 2, x_62); +x_64 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_65 = lean_array_push(x_64, x_63); +x_66 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_67 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_67, 0, x_39); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set(x_67, 2, x_65); +x_68 = lean_array_push(x_35, x_49); +x_69 = lean_array_push(x_68, x_67); +x_70 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_70, 0, x_39); +lean_ctor_set(x_70, 1, x_48); +lean_ctor_set(x_70, 2, x_69); +x_71 = lean_array_push(x_35, x_46); +x_72 = lean_array_push(x_71, x_70); +x_73 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_73, 0, x_39); +lean_ctor_set(x_73, 1, x_44); +lean_ctor_set(x_73, 2, x_72); +x_74 = lean_array_push(x_59, x_40); +x_75 = lean_array_push(x_74, x_42); +x_76 = lean_array_push(x_75, x_73); +x_77 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_77, 0, x_39); +lean_ctor_set(x_77, 1, x_32); +lean_ctor_set(x_77, 2, x_76); +x_78 = 1; +x_79 = lean_usize_add(x_4, x_78); +x_80 = lean_array_uset(x_17, x_4, x_77); +x_4 = x_79; +x_5 = x_80; +x_12 = x_24; +goto _start; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_7 = lean_alloc_closure((void*)(l_Lean_Meta_inferType___boxed), 6, 1); -lean_closure_set(x_7, 0, x_6); -x_8 = lean_apply_2(x_1, lean_box(0), x_7); -lean_inc(x_5); -x_9 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__1), 5, 4); -lean_closure_set(x_9, 0, x_2); -lean_closure_set(x_9, 1, x_3); -lean_closure_set(x_9, 2, x_4); -lean_closure_set(x_9, 3, x_5); -x_10 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_8, x_9); -return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -if (lean_obj_tag(x_8) == 0) +uint8_t x_11; +x_11 = lean_usize_dec_lt(x_2, x_1); +if (x_11 == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_12; lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -lean_dec(x_8); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_apply_2(x_11, lean_box(0), x_9); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_3); +lean_ctor_set(x_12, 1, x_10); return x_12; } else { -lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_8, 0); -lean_inc(x_13); -lean_dec(x_8); -x_14 = 1; -x_15 = lean_usize_add(x_2, x_14); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_15, x_13); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_array_uget(x_3, x_2); +x_14 = lean_unsigned_to_nat(0u); +x_15 = lean_array_uset(x_3, x_2, x_14); +lean_inc(x_6); +x_16 = l_Lean_Meta_getFVarLocalDecl(x_13, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Lean_LocalDecl_userName(x_17); +lean_dec(x_17); +x_20 = lean_mk_syntax_ident(x_19); +x_21 = 1; +x_22 = lean_usize_add(x_2, x_21); +x_23 = lean_array_uset(x_15, x_2, x_20); +x_2 = x_22; +x_3 = x_23; +x_10 = x_18; +goto _start; +} +else +{ +uint8_t x_25; +lean_dec(x_15); +lean_dec(x_6); +x_25 = !lean_is_exclusive(x_16); +if (x_25 == 0) +{ return x_16; } +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_16, 0); +x_27 = lean_ctor_get(x_16, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_16); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -uint8_t x_9; -x_9 = lean_usize_dec_lt(x_7, x_6); -if (x_9 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; +return x_4; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_6 = lean_array_uget(x_4, x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_4, x_3, x_7); +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_11 = lean_array_uset(x_8, x_3, x_6); +x_3 = x_10; +x_4 = x_11; +goto _start; +} +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("structExplicitBinder", 20); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, size_t x_10, size_t x_11, lean_object* x_12) { +_start: +{ +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_11, x_10); +if (x_13 == 0) +{ +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_apply_2(x_11, lean_box(0), x_8); return x_12; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_13 = lean_array_uget(x_5, x_7); -x_14 = lean_ctor_get(x_1, 1); -lean_inc(x_14); -lean_inc(x_13); +lean_object* x_14; lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_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; +x_14 = lean_array_uget(x_12, x_11); +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_array_uset(x_12, x_11, x_15); +x_17 = 1; +x_18 = lean_usize_add(x_11, x_17); +x_19 = lean_ctor_get(x_14, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_14, 1); +lean_inc(x_20); +lean_dec(x_14); +x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6___closed__1; +lean_inc(x_5); +x_22 = l_Lean_Name_str___override(x_5, x_21); +x_23 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; lean_inc(x_3); -x_15 = lean_alloc_closure((void*)(l_Lean_Meta_mkProjection), 7, 2); -lean_closure_set(x_15, 0, x_3); -lean_closure_set(x_15, 1, x_13); -lean_inc(x_2); -x_16 = lean_apply_2(x_2, lean_box(0), x_15); +x_24 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_24, 0, x_3); +lean_ctor_set(x_24, 1, x_23); +lean_inc(x_9); +x_25 = lean_array_push(x_9, x_19); +x_26 = lean_box(2); lean_inc(x_4); +x_27 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_4); +lean_ctor_set(x_27, 2, x_25); +x_28 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__32; +lean_inc(x_5); +x_29 = l_Lean_Name_str___override(x_5, x_28); +x_30 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__36; lean_inc(x_1); +x_31 = l_Lean_Name_str___override(x_1, x_30); +x_32 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; +lean_inc(x_3); +x_33 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_33, 0, x_3); +lean_ctor_set(x_33, 1, x_32); lean_inc(x_2); -x_17 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2), 6, 5); -lean_closure_set(x_17, 0, x_2); -lean_closure_set(x_17, 1, x_13); -lean_closure_set(x_17, 2, x_8); -lean_closure_set(x_17, 3, x_1); -lean_closure_set(x_17, 4, x_4); +x_34 = lean_array_push(x_2, x_33); +x_35 = lean_array_push(x_34, x_20); +x_36 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_36, 0, x_26); +lean_ctor_set(x_36, 1, x_31); +lean_ctor_set(x_36, 2, x_35); +lean_inc(x_9); +x_37 = lean_array_push(x_9, x_36); lean_inc(x_4); -x_18 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_16, x_17); -x_19 = lean_box_usize(x_7); -x_20 = lean_box_usize(x_6); -x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3___boxed), 8, 7); -lean_closure_set(x_21, 0, x_1); -lean_closure_set(x_21, 1, x_19); -lean_closure_set(x_21, 2, x_2); -lean_closure_set(x_21, 3, x_3); -lean_closure_set(x_21, 4, x_4); -lean_closure_set(x_21, 5, x_5); -lean_closure_set(x_21, 6, x_20); -x_22 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_18, x_21); -return x_22; +x_38 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_38, 0, x_26); +lean_ctor_set(x_38, 1, x_4); +lean_ctor_set(x_38, 2, x_37); +lean_inc(x_6); +lean_inc(x_2); +x_39 = lean_array_push(x_2, x_6); +x_40 = lean_array_push(x_39, x_38); +x_41 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_41, 0, x_26); +lean_ctor_set(x_41, 1, x_29); +lean_ctor_set(x_41, 2, x_40); +x_42 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +lean_inc(x_3); +x_43 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_43, 0, x_3); +lean_ctor_set(x_43, 1, x_42); +lean_inc(x_8); +lean_inc(x_7); +x_44 = lean_array_push(x_7, x_8); +x_45 = lean_array_push(x_44, x_24); +x_46 = lean_array_push(x_45, x_27); +x_47 = lean_array_push(x_46, x_41); +lean_inc(x_6); +x_48 = lean_array_push(x_47, x_6); +x_49 = lean_array_push(x_48, x_43); +x_50 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_50, 0, x_26); +lean_ctor_set(x_50, 1, x_22); +lean_ctor_set(x_50, 2, x_49); +x_51 = lean_array_uset(x_16, x_11, x_50); +x_11 = x_18; +x_12 = x_51; +goto _start; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___boxed), 8, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_5, x_4); +if (x_7 == 0) { -lean_object* x_9; lean_object* x_10; -x_9 = lean_apply_1(x_1, x_3); -x_10 = lean_apply_7(x_2, lean_box(0), x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} +return x_6; } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__1), 8, 2); -lean_closure_set(x_11, 0, x_1); -lean_closure_set(x_11, 1, x_5); -x_12 = l___private_Lean_Meta_Basic_0__Lean_Meta_withLocalDeclImp___rarg(x_2, x_3, x_4, x_11, x_6, x_7, x_8, x_9, x_10); -return x_12; -} +lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_8 = lean_array_uget(x_6, x_5); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_array_uset(x_6, x_5, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_5, x_11); +x_13 = lean_array_uset(x_10, x_5, x_8); +x_5 = x_12; +x_6 = x_13; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; 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_1, 1); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_box(x_5); -x_10 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed), 10, 4); -lean_closure_set(x_10, 0, x_7); -lean_closure_set(x_10, 1, x_4); -lean_closure_set(x_10, 2, x_9); -lean_closure_set(x_10, 3, x_6); -x_11 = lean_ctor_get(x_2, 0); -lean_inc(x_11); -x_12 = lean_apply_2(x_11, lean_box(0), x_10); -x_13 = lean_ctor_get(x_2, 1); -lean_inc(x_13); -lean_dec(x_2); -x_14 = lean_apply_1(x_13, lean_box(0)); -x_15 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_12, x_14); -return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(size_t x_1, size_t x_2, lean_object* x_3) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___boxed), 7, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -x_7 = lean_box(0); -x_8 = lean_apply_1(x_2, x_7); -x_9 = lean_array_get_size(x_8); -x_10 = lean_usize_of_nat(x_9); -lean_dec(x_9); -x_11 = 0; -x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -lean_inc(x_6); -x_13 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(x_1, x_3, x_5, x_6, x_8, x_10, x_11, x_12); -x_14 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_13, x_4); -return x_14; -} +return x_3; } -static lean_object* _init_l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("s", 1); -return x_1; -} +lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_10 = lean_array_uset(x_7, x_2, x_5); +x_2 = x_9; +x_3 = x_10; +goto _start; } -static lean_object* _init_l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -lean_dec(x_5); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -x_11 = lean_box(0); -x_12 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_10, x_11); -x_13 = lean_ctor_get(x_9, 0); -lean_inc(x_13); -lean_dec(x_9); -x_14 = l_Lean_Expr_const___override(x_13, x_12); -x_15 = l_Lean_mkAppN(x_14, x_6); -lean_inc(x_1); -x_16 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___rarg___lambda__1), 5, 4); -lean_closure_set(x_16, 0, x_1); -lean_closure_set(x_16, 1, x_8); -lean_closure_set(x_16, 2, x_3); -lean_closure_set(x_16, 3, x_7); -x_17 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; -x_18 = 0; -x_19 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg(x_1, x_2, lean_box(0), x_17, x_18, x_15, x_16); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux(lean_object* x_1) { -_start: +uint8_t x_7; +x_7 = lean_usize_dec_lt(x_5, x_4); +if (x_7 == 0) { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___rarg), 8, 0); -return x_2; -} +return x_6; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_10 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__3(x_1, x_9, x_3, x_4, x_5, x_6, x_10, x_8); -return x_11; +lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_8 = lean_array_uget(x_6, x_5); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_array_uset(x_6, x_5, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_5, x_11); +x_13 = lean_array_uset(x_10, x_5, x_8); +x_5 = x_12; +x_6 = x_13; +goto _start; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_10 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_4, x_3); +if (x_13 == 0) { -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_3); -lean_dec(x_3); -x_12 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2(x_1, x_2, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; +lean_object* x_14; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_1); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_5); +lean_ctor_set(x_14, 1, x_12); +return x_14; } +else +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_array_uget(x_2, x_4); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_15); +lean_inc(x_1); +x_16 = l_Lean_Meta_mkProjection(x_1, x_15, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +x_19 = lean_infer_type(x_17, x_8, x_9, x_10, x_11, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; size_t x_24; size_t x_25; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_15); +lean_ctor_set(x_22, 1, x_20); +x_23 = lean_array_push(x_5, x_22); +x_24 = 1; +x_25 = lean_usize_add(x_4, x_24); +x_4 = x_25; +x_5 = x_23; +x_12 = x_21; +goto _start; } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -uint8_t x_8; lean_object* x_9; -x_8 = lean_unbox(x_5); +uint8_t x_27; +lean_dec(x_15); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_5); -x_9 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg(x_1, x_2, x_3, x_4, x_8, x_6, x_7); -return x_9; -} +lean_dec(x_1); +x_27 = !lean_is_exclusive(x_19); +if (x_27 == 0) +{ +return x_19; } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, lean_object* x_8) { -_start: +else { -if (lean_obj_tag(x_8) == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_19, 0); +x_29 = lean_ctor_get(x_19, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_19); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); +uint8_t x_31; +lean_dec(x_15); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +lean_dec(x_5); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_apply_2(x_11, lean_box(0), x_9); -return x_12; +x_31 = !lean_is_exclusive(x_16); +if (x_31 == 0) +{ +return x_16; } else { -lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_8, 0); -lean_inc(x_13); -lean_dec(x_8); -x_14 = 1; -x_15 = lean_usize_add(x_2, x_14); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_15, x_13); -return x_16; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_16, 0); +x_33 = lean_ctor_get(x_16, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_16); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { +} +} +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_9; -x_9 = lean_usize_dec_lt(x_7, x_6); -if (x_9 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; +x_11 = lean_box(0); +x_12 = lean_apply_1(x_1, x_11); +x_13 = lean_array_get_size(x_12); +x_14 = lean_usize_of_nat(x_13); +lean_dec(x_13); +x_15 = 0; +x_16 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12(x_3, x_12, x_14, x_15, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_12); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_apply_8(x_2, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_19); +return x_20; +} +else +{ +uint8_t x_21; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_apply_2(x_11, lean_box(0), x_8); -return x_12; +x_21 = !lean_is_exclusive(x_17); +if (x_21 == 0) +{ +return x_17; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_13 = lean_array_uget(x_5, x_7); -x_14 = lean_ctor_get(x_1, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_3); -x_15 = lean_alloc_closure((void*)(l_Lean_Meta_mkProjection), 7, 2); -lean_closure_set(x_15, 0, x_3); -lean_closure_set(x_15, 1, x_13); -lean_inc(x_2); -x_16 = lean_apply_2(x_2, lean_box(0), x_15); -lean_inc(x_4); -lean_inc(x_1); -lean_inc(x_2); -x_17 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2), 6, 5); -lean_closure_set(x_17, 0, x_2); -lean_closure_set(x_17, 1, x_13); -lean_closure_set(x_17, 2, x_8); -lean_closure_set(x_17, 3, x_1); -lean_closure_set(x_17, 4, x_4); -lean_inc(x_4); -x_18 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_16, x_17); -x_19 = lean_box_usize(x_7); -x_20 = lean_box_usize(x_6); -x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1___boxed), 8, 7); -lean_closure_set(x_21, 0, x_1); -lean_closure_set(x_21, 1, x_19); -lean_closure_set(x_21, 2, x_2); -lean_closure_set(x_21, 3, x_3); -lean_closure_set(x_21, 4, x_4); -lean_closure_set(x_21, 5, x_5); -lean_closure_set(x_21, 6, x_20); -x_22 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_18, x_21); -return x_22; -} +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_17, 0); +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_17); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___boxed), 8, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); lean_dec(x_1); -x_9 = lean_box(x_5); -x_10 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed), 10, 4); -lean_closure_set(x_10, 0, x_7); -lean_closure_set(x_10, 1, x_4); -lean_closure_set(x_10, 2, x_9); -lean_closure_set(x_10, 3, x_6); -x_11 = lean_ctor_get(x_2, 0); -lean_inc(x_11); -x_12 = lean_apply_2(x_11, lean_box(0), x_10); -x_13 = lean_ctor_get(x_2, 1); +x_13 = lean_ctor_get(x_12, 1); lean_inc(x_13); -lean_dec(x_2); -x_14 = lean_apply_1(x_13, lean_box(0)); -x_15 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_12, x_14); -return x_15; +x_14 = lean_box(0); +x_15 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_13, x_14); +x_16 = lean_ctor_get(x_12, 0); +lean_inc(x_16); +lean_dec(x_12); +x_17 = l_Lean_Expr_const___override(x_16, x_15); +x_18 = l_Lean_mkAppN(x_17, x_2); +x_19 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11___rarg___lambda__1), 10, 2); +lean_closure_set(x_19, 0, x_4); +lean_closure_set(x_19, 1, x_3); +x_20 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; +x_21 = 0; +x_22 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__3___rarg(x_20, x_21, x_18, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_22; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg___boxed), 7, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11___rarg), 11, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -x_7 = lean_box(0); -x_8 = lean_apply_1(x_2, x_7); -x_9 = lean_array_get_size(x_8); -x_10 = lean_usize_of_nat(x_9); -lean_dec(x_9); -x_11 = 0; -x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -lean_inc(x_6); -x_13 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(x_1, x_3, x_5, x_6, x_8, x_10, x_11, x_12); -x_14 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_13, x_4); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -lean_dec(x_5); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -x_11 = lean_box(0); -x_12 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_10, x_11); -x_13 = lean_ctor_get(x_9, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_11 = lean_st_ref_get(x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); -lean_dec(x_9); -x_14 = l_Lean_Expr_const___override(x_13, x_12); -x_15 = l_Lean_mkAppN(x_14, x_6); +lean_dec(x_11); +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_14); +lean_dec(x_12); lean_inc(x_1); -x_16 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg___lambda__1), 5, 4); -lean_closure_set(x_16, 0, x_1); -lean_closure_set(x_16, 1, x_8); -lean_closure_set(x_16, 2, x_3); -lean_closure_set(x_16, 3, x_7); -x_17 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; -x_18 = 0; -x_19 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg(x_1, x_2, lean_box(0), x_17, x_18, x_15, x_16); -return x_19; +x_15 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2___boxed), 3, 2); +lean_closure_set(x_15, 0, x_1); +lean_closure_set(x_15, 1, x_14); +x_16 = l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11___rarg(x_1, x_2, x_3, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg), 8, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___rarg), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__1() { _start: { -lean_object* x_6; uint8_t x_7; -x_6 = lean_st_ref_get(x_4, x_5); -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -lean_dec(x_8); -lean_ctor_set(x_6, 0, x_9); -return x_6; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__2() { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_6, 0); -x_11 = lean_ctor_get(x_6, 1); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_6); -x_12 = lean_ctor_get(x_10, 0); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__1; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("term", 4); +return x_1; +} } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__4() { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -lean_dec(x_4); -x_6 = l_Lean_getStructureFields(x_2, x_5); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__5() { _start: { -lean_object* x_8; lean_object* x_9; -lean_inc(x_1); -x_8 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2___boxed), 3, 2); -lean_closure_set(x_8, 0, x_1); -lean_closure_set(x_8, 1, x_7); -x_9 = l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFields___spec__1___rarg(x_2, x_3, x_4, lean_box(0), x_1, x_5, x_6, x_8); -return x_9; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__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_Lean_Server_RpcEncoding_withFields___rarg___closed__1() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1___boxed), 5, 0); +x_1 = lean_mk_string_from_bytes("explicit", 8); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__7() { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); -x_9 = l_Lean_Server_RpcEncoding_withFields___rarg___closed__1; -lean_inc(x_3); -x_10 = lean_apply_2(x_3, lean_box(0), x_9); -x_11 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg___lambda__3), 7, 6); -lean_closure_set(x_11, 0, x_5); -lean_closure_set(x_11, 1, x_1); -lean_closure_set(x_11, 2, x_2); -lean_closure_set(x_11, 3, x_3); -lean_closure_set(x_11, 4, x_6); -lean_closure_set(x_11, 5, x_7); -x_12 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_10, x_11); -return x_12; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__6; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__8() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg), 7, 0); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("@", 1); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__9() { _start: { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_10 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___lambda__1(x_1, x_9, x_3, x_4, x_5, x_6, x_10, x_8); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("_root_", 6); +return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__10() { _start: { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_10 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFields___spec__2___rarg(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); -return x_11; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__9; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__11() { _start: { -uint8_t x_8; lean_object* x_9; -x_8 = lean_unbox(x_5); -lean_dec(x_5); -x_9 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFields___spec__3___rarg(x_1, x_2, x_3, x_4, x_8, x_6, x_7); -return x_9; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("instRpcEncoding", 15); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12() { _start: { -lean_object* x_6; -x_6 = l_Lean_Server_RpcEncoding_withFields___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_6; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("in", 2); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__13() { _start: { -lean_object* x_4; -x_4 = l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14() { _start: { -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -lean_dec(x_8); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_apply_2(x_11, lean_box(0), x_9); -return x_12; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("variable", 8); +return x_1; } -else -{ -lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_8, 0); -lean_inc(x_13); -lean_dec(x_8); -x_14 = 1; -x_15 = lean_usize_add(x_2, x_14); -x_16 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(x_1, x_3, x_4, x_5, x_6, x_7, x_15, x_13); -return x_16; } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16() { _start: { -uint8_t x_9; -x_9 = lean_usize_dec_lt(x_7, x_6); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); -lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_apply_2(x_11, lean_box(0), x_8); -return x_12; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17() { +_start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_13 = lean_array_uget(x_5, x_7); -x_14 = lean_ctor_get(x_1, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_3); -x_15 = lean_alloc_closure((void*)(l_Lean_Meta_mkProjection), 7, 2); -lean_closure_set(x_15, 0, x_3); -lean_closure_set(x_15, 1, x_13); -lean_inc(x_2); -x_16 = lean_apply_2(x_2, lean_box(0), x_15); -lean_inc(x_4); -lean_inc(x_1); -lean_inc(x_2); -x_17 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsAux___spec__1___rarg___lambda__2), 6, 5); -lean_closure_set(x_17, 0, x_2); -lean_closure_set(x_17, 1, x_13); -lean_closure_set(x_17, 2, x_8); -lean_closure_set(x_17, 3, x_1); -lean_closure_set(x_17, 4, x_4); -lean_inc(x_4); -x_18 = lean_apply_4(x_4, lean_box(0), lean_box(0), x_16, x_17); -x_19 = lean_box_usize(x_7); -x_20 = lean_box_usize(x_6); -x_21 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1___boxed), 8, 7); -lean_closure_set(x_21, 0, x_1); -lean_closure_set(x_21, 1, x_19); -lean_closure_set(x_21, 2, x_2); -lean_closure_set(x_21, 3, x_3); -lean_closure_set(x_21, 4, x_4); -lean_closure_set(x_21, 5, x_5); -lean_closure_set(x_21, 6, x_20); -x_22 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_18, x_21); -return x_22; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__19() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___boxed), 8, 0); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__18; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__20() { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_box(x_5); -x_10 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsAux___spec__2___rarg___lambda__2___boxed), 10, 4); -lean_closure_set(x_10, 0, x_7); -lean_closure_set(x_10, 1, x_4); -lean_closure_set(x_10, 2, x_9); -lean_closure_set(x_10, 3, x_6); -x_11 = lean_ctor_get(x_2, 0); -lean_inc(x_11); -x_12 = lean_apply_2(x_11, lean_box(0), x_10); -x_13 = lean_ctor_get(x_2, 1); -lean_inc(x_13); -lean_dec(x_2); -x_14 = lean_apply_1(x_13, lean_box(0)); -x_15 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_12, x_14); -return x_15; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__19; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__21() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg___boxed), 7, 0); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__20; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__22() { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -x_7 = lean_box(0); -x_8 = lean_apply_1(x_2, x_7); -x_9 = lean_array_get_size(x_8); -x_10 = lean_usize_of_nat(x_9); -lean_dec(x_9); -x_11 = 0; -x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -lean_inc(x_6); -x_13 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(x_1, x_3, x_5, x_6, x_8, x_10, x_11, x_12); -x_14 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_13, x_4); -return x_14; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__21; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23() { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -lean_dec(x_5); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -x_11 = lean_box(0); -x_12 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_10, x_11); -x_13 = lean_ctor_get(x_9, 0); -lean_inc(x_13); -lean_dec(x_9); -x_14 = l_Lean_Expr_const___override(x_13, x_12); -x_15 = l_Lean_mkAppN(x_14, x_6); -lean_inc(x_1); -x_16 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg___lambda__1), 5, 4); -lean_closure_set(x_16, 0, x_1); -lean_closure_set(x_16, 1, x_8); -lean_closure_set(x_16, 2, x_3); -lean_closure_set(x_16, 3, x_7); -x_17 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; -x_18 = 0; -x_19 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg(x_1, x_2, lean_box(0), x_17, x_18, x_15, x_16); -return x_19; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__22; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg), 8, 0); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("structure", 9); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__25() { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -lean_dec(x_5); -x_7 = l_Lean_getStructureFieldsFlattened(x_2, x_6, x_3); -return x_7; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___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) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__26() { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_box(x_2); -lean_inc(x_1); -x_10 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1___boxed), 4, 3); -lean_closure_set(x_10, 0, x_1); -lean_closure_set(x_10, 1, x_8); -lean_closure_set(x_10, 2, x_9); -x_11 = l_Lean_Server_RpcEncoding_withFieldsAux___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__1___rarg(x_3, x_4, x_5, lean_box(0), x_1, x_6, x_7, x_10); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("structureTk", 11); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__27() { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); -x_10 = l_Lean_Server_RpcEncoding_withFields___rarg___closed__1; -lean_inc(x_3); -x_11 = lean_apply_2(x_3, lean_box(0), x_10); -x_12 = lean_box(x_8); -x_13 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__2___boxed), 8, 7); -lean_closure_set(x_13, 0, x_5); -lean_closure_set(x_13, 1, x_12); -lean_closure_set(x_13, 2, x_1); -lean_closure_set(x_13, 3, x_2); -lean_closure_set(x_13, 4, x_3); -lean_closure_set(x_13, 5, x_6); -lean_closure_set(x_13, 6, x_7); -x_14 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_11, x_13); -return x_14; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__26; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___boxed), 8, 0); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("RpcEncodingPacket", 17); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__29() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28; +x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__30() { _start: { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_10 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___lambda__1(x_1, x_9, x_3, x_4, x_5, x_6, x_10, x_8); -return x_11; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__29; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__31() { _start: { -size_t x_9; size_t x_10; lean_object* x_11; -x_9 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_10 = lean_unbox_usize(x_7); -lean_dec(x_7); -x_11 = l_Array_forInUnsafe_loop___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__2___rarg(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); -return x_11; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__32() { _start: { -uint8_t x_8; lean_object* x_9; -x_8 = lean_unbox(x_5); -lean_dec(x_5); -x_9 = l_Lean_Meta_withLocalDecl___at_Lean_Server_RpcEncoding_withFieldsFlattened___spec__3___rarg(x_1, x_2, x_3, x_4, x_8, x_6, x_7); -return x_9; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("structFields", 12); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33() { _start: { -uint8_t x_5; lean_object* x_6; -x_5 = lean_unbox(x_3); -lean_dec(x_3); -x_6 = l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__1(x_1, x_2, x_5, x_4); -lean_dec(x_4); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__32; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__34() { _start: { -uint8_t x_9; lean_object* x_10; -x_9 = lean_unbox(x_2); -lean_dec(x_2); -x_10 = l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___lambda__2(x_1, x_9, x_3, x_4, x_5, x_6, x_7, x_8); -return x_10; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("optDeriving", 11); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35() { _start: { -uint8_t x_9; lean_object* x_10; -x_9 = lean_unbox(x_8); -lean_dec(x_8); -x_10 = l_Lean_Server_RpcEncoding_withFieldsFlattened___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); -return x_10; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__34; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Server_RpcEncoding_isOptField___closed__1() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__36() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("?", 1); +x_1 = lean_mk_string_from_bytes("deriving", 8); return x_1; } } -LEAN_EXPORT uint8_t l_Lean_Server_RpcEncoding_isOptField(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__37() { _start: { -uint8_t x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_2 = 1; -x_3 = l_Lean_Name_toString(x_1, x_2); -x_4 = l_Lean_Server_RpcEncoding_isOptField___closed__1; -x_5 = l_String_endsWith(x_3, x_4); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("group", 5); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_isOptField___boxed(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__38() { _start: { -uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Server_RpcEncoding_isOptField(x_1); -x_3 = lean_box(x_2); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__37; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39() { _start: { -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_get_size(x_1); -x_7 = lean_nat_dec_lt(x_4, x_6); -lean_dec(x_6); -if (x_7 == 0) -{ -lean_object* x_8; -lean_dec(x_4); -x_8 = lean_box(0); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("FromJson", 8); +return x_1; } -else -{ -lean_object* x_9; uint8_t x_10; -x_9 = lean_array_fget(x_1, x_4); -x_10 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_5, x_9); -lean_dec(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_nat_add(x_4, x_11); -lean_dec(x_4); -x_3 = lean_box(0); -x_4 = x_12; -goto _start; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__40() { +_start: { -lean_object* x_14; lean_object* x_15; -x_14 = lean_array_fget(x_2, x_4); -lean_dec(x_4); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__41() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__40; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -static size_t _init_l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__1() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42() { _start: { -size_t x_1; size_t x_2; size_t x_3; -x_1 = 1; -x_2 = 5; -x_3 = lean_usize_shift_left(x_1, x_2); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static size_t _init_l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__43() { _start: { -size_t x_1; size_t x_2; size_t x_3; -x_1 = 1; -x_2 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__1; -x_3 = lean_usize_sub(x_2, x_1); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(lean_object* x_1, size_t x_2, lean_object* x_3) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__44() { _start: { -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_4; size_t x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = 5; -x_6 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2; -x_7 = lean_usize_land(x_2, x_6); -x_8 = lean_usize_to_nat(x_7); -x_9 = lean_box(2); -x_10 = lean_array_get(x_9, x_4, x_8); -lean_dec(x_8); -lean_dec(x_4); -switch (lean_obj_tag(x_10)) { -case 0: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_3, x_11); -lean_dec(x_11); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_12); -x_14 = lean_box(0); -return x_14; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__43; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__45() { +_start: { -lean_object* x_15; -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_12); -return x_15; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__44; +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; } } -case 1: +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46() { +_start: { -lean_object* x_16; size_t x_17; -x_16 = lean_ctor_get(x_10, 0); -lean_inc(x_16); -lean_dec(x_10); -x_17 = lean_usize_shift_right(x_2, x_5); -x_1 = x_16; -x_2 = x_17; -goto _start; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(",", 1); +return x_1; } -default: -{ -lean_object* x_19; -x_19 = lean_box(0); -return x_19; } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("ToJson", 6); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__48() { +_start: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_1, 1); -lean_inc(x_21); -lean_dec(x_1); -x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5(x_20, x_21, lean_box(0), x_22, x_3); -lean_dec(x_21); -lean_dec(x_20); -return x_23; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__48; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50() { _start: { -lean_object* x_3; uint64_t x_4; size_t x_5; lean_object* x_6; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -lean_dec(x_1); -x_4 = l_Lean_Meta_DiscrTree_Key_hash(x_2); -x_5 = lean_uint64_to_usize(x_4); -x_6 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(x_3, x_5, x_2); -lean_dec(x_2); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__51() { _start: { -lean_object* x_7; uint8_t x_8; -x_7 = lean_array_get_size(x_2); -x_8 = lean_nat_dec_lt(x_5, x_7); -lean_dec(x_7); -if (x_8 == 0) -{ -lean_dec(x_5); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -else -{ -lean_object* x_9; lean_object* x_10; uint64_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_9 = lean_array_fget(x_2, x_5); -x_10 = lean_array_fget(x_3, x_5); -x_11 = l_Lean_Meta_DiscrTree_Key_hash(x_9); -x_12 = lean_uint64_to_usize(x_11); -x_13 = 1; -x_14 = lean_usize_sub(x_1, x_13); -x_15 = 5; -x_16 = lean_usize_mul(x_15, x_14); -x_17 = lean_usize_shift_right(x_12, x_16); -x_18 = lean_unsigned_to_nat(1u); -x_19 = lean_nat_add(x_5, x_18); -lean_dec(x_5); -x_20 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_6, x_17, x_1, x_9, x_10); -x_4 = lean_box(0); -x_5 = x_19; -x_6 = x_20; -goto _start; } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__52() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__51; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53() { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -x_7 = lean_array_get_size(x_5); -x_8 = lean_nat_dec_lt(x_2, x_7); -lean_dec(x_7); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_2); -x_9 = !lean_is_exclusive(x_1); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_1, 1); -lean_dec(x_10); -x_11 = lean_ctor_get(x_1, 0); -lean_dec(x_11); -x_12 = lean_array_push(x_5, x_3); -x_13 = lean_array_push(x_6, x_4); -lean_ctor_set(x_1, 1, x_13); -lean_ctor_set(x_1, 0, x_12); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__52; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__54() { +_start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_14 = lean_array_push(x_5, x_3); -x_15 = lean_array_push(x_6, x_4); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -return x_16; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__55() { +_start: { -lean_object* x_17; uint8_t x_18; -x_17 = lean_array_fget(x_5, x_2); -x_18 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_3, x_17); -lean_dec(x_17); -if (x_18 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__56() { +_start: { -lean_object* x_19; lean_object* x_20; -lean_dec(x_6); -lean_dec(x_5); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_add(x_2, x_19); -lean_dec(x_2); -x_2 = x_20; -goto _start; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__123; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__55; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__57() { +_start: { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_1); -if (x_22 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__127; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58() { +_start: { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_1, 1); -lean_dec(x_23); -x_24 = lean_ctor_get(x_1, 0); -lean_dec(x_24); -x_25 = lean_array_fset(x_5, x_2, x_3); -x_26 = lean_array_fset(x_6, x_2, x_4); -lean_dec(x_2); -lean_ctor_set(x_1, 1, x_26); -lean_ctor_set(x_1, 0, x_25); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__56; +x_3 = lean_array_push(x_1, x_2); +return x_3; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__59() { +_start: { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_1); -x_27 = lean_array_fset(x_5, x_2, x_3); -x_28 = lean_array_fset(x_6, x_2, x_4); -lean_dec(x_2); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__59; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__61() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -static lean_object* _init_l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62() { _start: { lean_object* x_1; -x_1 = l_Std_PersistentHashMap_mkEmptyEntries(lean_box(0), lean_box(0)); +x_1 = lean_mk_string_from_bytes("show", 4); return x_1; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__63() { _start: { -if (lean_obj_tag(x_1) == 0) -{ -uint8_t x_6; -x_6 = !lean_is_exclusive(x_1); -if (x_6 == 0) -{ -lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_7 = lean_ctor_get(x_1, 0); -x_8 = 1; -x_9 = 5; -x_10 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2; -x_11 = lean_usize_land(x_2, x_10); -x_12 = lean_usize_to_nat(x_11); -x_13 = lean_array_get_size(x_7); -x_14 = lean_nat_dec_lt(x_12, x_13); -lean_dec(x_13); -if (x_14 == 0) -{ -lean_dec(x_12); -lean_dec(x_5); -lean_dec(x_4); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_array_fget(x_7, x_12); -x_16 = lean_box(0); -x_17 = lean_array_fset(x_7, x_12, x_16); -switch (lean_obj_tag(x_15)) { -case 0: -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_15); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_15, 0); -x_20 = lean_ctor_get(x_15, 1); -x_21 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_4, x_19); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_free_object(x_15); -x_22 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_19, x_20, x_4, x_5); -x_23 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_23, 0, x_22); -x_24 = lean_array_fset(x_17, x_12, x_23); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_24); -return x_1; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__64() { +_start: { -lean_object* x_25; -lean_dec(x_20); -lean_dec(x_19); -lean_ctor_set(x_15, 1, x_5); -lean_ctor_set(x_15, 0, x_4); -x_25 = lean_array_fset(x_17, x_12, x_15); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_25); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("ellipsis", 8); return x_1; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__65() { +_start: { -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = lean_ctor_get(x_15, 0); -x_27 = lean_ctor_get(x_15, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_15); -x_28 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_4, x_26); -if (x_28 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__64; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66() { +_start: { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_26, x_27, x_4, x_5); -x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_29); -x_31 = lean_array_fset(x_17, x_12, x_30); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_31); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("..", 2); return x_1; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67() { +_start: { -lean_object* x_32; lean_object* x_33; -lean_dec(x_27); -lean_dec(x_26); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_4); -lean_ctor_set(x_32, 1, x_5); -x_33 = lean_array_fset(x_17, x_12, x_32); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_33); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("fromTerm", 8); return x_1; } } -} -case 1: -{ -uint8_t x_34; -x_34 = !lean_is_exclusive(x_15); -if (x_34 == 0) +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__68() { +_start: { -lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_39; -x_35 = lean_ctor_get(x_15, 0); -x_36 = lean_usize_shift_right(x_2, x_9); -x_37 = lean_usize_add(x_3, x_8); -x_38 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_35, x_36, x_37, x_4, x_5); -lean_ctor_set(x_15, 0, x_38); -x_39 = lean_array_fset(x_17, x_12, x_15); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_39); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69() { +_start: { -lean_object* x_40; size_t x_41; size_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_40 = lean_ctor_get(x_15, 0); -lean_inc(x_40); -lean_dec(x_15); -x_41 = lean_usize_shift_right(x_2, x_9); -x_42 = lean_usize_add(x_3, x_8); -x_43 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_40, x_41, x_42, x_4, x_5); -x_44 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_44, 0, x_43); -x_45 = lean_array_fset(x_17, x_12, x_44); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_45); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("from", 4); return x_1; } } -default: +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__70() { +_start: { -lean_object* x_46; lean_object* x_47; -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_4); -lean_ctor_set(x_46, 1, x_5); -x_47 = lean_array_fset(x_17, x_12, x_46); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_47); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("structInst", 10); return x_1; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__71() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__70; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -else -{ -lean_object* x_48; size_t x_49; size_t x_50; size_t x_51; size_t x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_48 = lean_ctor_get(x_1, 0); -lean_inc(x_48); -lean_dec(x_1); -x_49 = 1; -x_50 = 5; -x_51 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2; -x_52 = lean_usize_land(x_2, x_51); -x_53 = lean_usize_to_nat(x_52); -x_54 = lean_array_get_size(x_48); -x_55 = lean_nat_dec_lt(x_53, x_54); -lean_dec(x_54); -if (x_55 == 0) +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72() { +_start: { -lean_object* x_56; -lean_dec(x_53); -lean_dec(x_5); -lean_dec(x_4); -x_56 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_56, 0, x_48); -return x_56; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("{", 1); +return x_1; } -else -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_array_fget(x_48, x_53); -x_58 = lean_box(0); -x_59 = lean_array_fset(x_48, x_53, x_58); -switch (lean_obj_tag(x_57)) { -case 0: -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; -x_60 = lean_ctor_get(x_57, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_57, 1); -lean_inc(x_61); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_62 = x_57; -} else { - lean_dec_ref(x_57); - x_62 = lean_box(0); -} -x_63 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_4, x_60); -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -lean_dec(x_62); -x_64 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_60, x_61, x_4, x_5); -x_65 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_65, 0, x_64); -x_66 = lean_array_fset(x_59, x_53, x_65); -lean_dec(x_53); -x_67 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_67, 0, x_66); -return x_67; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__73() { +_start: { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -lean_dec(x_61); -lean_dec(x_60); -if (lean_is_scalar(x_62)) { - x_68 = lean_alloc_ctor(0, 2, 0); -} else { - x_68 = x_62; -} -lean_ctor_set(x_68, 0, x_4); -lean_ctor_set(x_68, 1, x_5); -x_69 = lean_array_fset(x_59, x_53, x_68); -lean_dec(x_53); -x_70 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_70, 0, x_69); -return x_70; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -case 1: +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__74() { +_start: { -lean_object* x_71; lean_object* x_72; size_t x_73; size_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_71 = lean_ctor_get(x_57, 0); -lean_inc(x_71); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - x_72 = x_57; -} else { - lean_dec_ref(x_57); - x_72 = lean_box(0); -} -x_73 = lean_usize_shift_right(x_2, x_50); -x_74 = lean_usize_add(x_3, x_49); -x_75 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_71, x_73, x_74, x_4, x_5); -if (lean_is_scalar(x_72)) { - x_76 = lean_alloc_ctor(1, 1, 0); -} else { - x_76 = x_72; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -lean_ctor_set(x_76, 0, x_75); -x_77 = lean_array_fset(x_59, x_53, x_76); -lean_dec(x_53); -x_78 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_78, 0, x_77); -return x_78; } -default: +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__75() { +_start: { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_4); -lean_ctor_set(x_79, 1, x_5); -x_80 = lean_array_fset(x_59, x_53, x_79); -lean_dec(x_53); -x_81 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_81, 0, x_80); -return x_81; -} -} -} -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__87; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } -else -{ -uint8_t x_82; -x_82 = !lean_is_exclusive(x_1); -if (x_82 == 0) -{ -lean_object* x_83; lean_object* x_84; size_t x_85; uint8_t x_86; -x_83 = lean_unsigned_to_nat(0u); -x_84 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(x_1, x_83, x_4, x_5); -x_85 = 7; -x_86 = lean_usize_dec_le(x_85, x_3); -if (x_86 == 0) -{ -lean_object* x_87; lean_object* x_88; uint8_t x_89; -x_87 = l_Std_PersistentHashMap_getCollisionNodeSize___rarg(x_84); -x_88 = lean_unsigned_to_nat(4u); -x_89 = lean_nat_dec_lt(x_87, x_88); -lean_dec(x_87); -if (x_89 == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_90 = lean_ctor_get(x_84, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_84, 1); -lean_inc(x_91); -lean_dec(x_84); -x_92 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1; -x_93 = l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(x_3, x_90, x_91, lean_box(0), x_83, x_92); -lean_dec(x_91); -lean_dec(x_90); -return x_93; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__76() { +_start: { -return x_84; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__75; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__77() { +_start: { -return x_84; -} +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("fun", 3); +return x_1; } -else -{ -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; size_t x_99; uint8_t x_100; -x_94 = lean_ctor_get(x_1, 0); -x_95 = lean_ctor_get(x_1, 1); -lean_inc(x_95); -lean_inc(x_94); -lean_dec(x_1); -x_96 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -x_97 = lean_unsigned_to_nat(0u); -x_98 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(x_96, x_97, x_4, x_5); -x_99 = 7; -x_100 = lean_usize_dec_le(x_99, x_3); -if (x_100 == 0) -{ -lean_object* x_101; lean_object* x_102; uint8_t x_103; -x_101 = l_Std_PersistentHashMap_getCollisionNodeSize___rarg(x_98); -x_102 = lean_unsigned_to_nat(4u); -x_103 = lean_nat_dec_lt(x_101, x_102); -lean_dec(x_101); -if (x_103 == 0) -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_104 = lean_ctor_get(x_98, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_98, 1); -lean_inc(x_105); -lean_dec(x_98); -x_106 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1; -x_107 = l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(x_3, x_104, x_105, lean_box(0), x_97, x_106); -lean_dec(x_105); -lean_dec(x_104); -return x_107; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__78() { +_start: { -return x_98; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__77; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__79() { +_start: { -return x_98; -} +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("basicFun", 8); +return x_1; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__80() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__79; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__81() { _start: { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_1); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; uint64_t x_7; size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_1, 1); -x_7 = l_Lean_Meta_DiscrTree_Key_hash(x_2); -x_8 = lean_uint64_to_usize(x_7); -x_9 = 1; -x_10 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_5, x_8, x_9, x_2, x_3); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_nat_add(x_6, x_11); -lean_dec(x_6); -lean_ctor_set(x_1, 1, x_12); -lean_ctor_set(x_1, 0, x_10); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("=>", 2); return x_1; } -else -{ -lean_object* x_13; lean_object* x_14; uint64_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_13 = lean_ctor_get(x_1, 0); -x_14 = lean_ctor_get(x_1, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_1); -x_15 = l_Lean_Meta_DiscrTree_Key_hash(x_2); -x_16 = lean_uint64_to_usize(x_15); -x_17 = 1; -x_18 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_13, x_16, x_17, x_2, x_3); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_add(x_14, x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_18); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} -} } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__13(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__82() { _start: { -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_uget(x_2, x_3); -lean_inc(x_1); -x_7 = l_Lean_Syntax_structEq(x_1, x_6); -if (x_7 == 0) -{ -size_t x_8; size_t x_9; -x_8 = 1; -x_9 = lean_usize_add(x_3, x_8); -x_3 = x_9; -goto _start; -} -else -{ -uint8_t x_11; -lean_dec(x_1); -x_11 = 1; -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("termReturn", 10); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__83() { +_start: { -uint8_t x_12; -lean_dec(x_1); -x_12 = 0; -return x_12; -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__82; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT uint8_t l_Array_contains___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__84() { _start: { -lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_3 = lean_array_get_size(x_1); -x_4 = lean_unsigned_to_nat(0u); -x_5 = lean_nat_dec_lt(x_4, x_3); -if (x_5 == 0) -{ -uint8_t x_6; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_6 = 0; -return x_6; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("return", 6); +return x_1; } -else -{ -uint8_t x_7; -x_7 = lean_nat_dec_le(x_3, x_3); -if (x_7 == 0) -{ -uint8_t x_8; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_8 = 0; -return x_8; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__85() { +_start: { -size_t x_9; size_t x_10; uint8_t x_11; -x_9 = 0; -x_10 = lean_usize_of_nat(x_3); -lean_dec(x_3); -x_11 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__13(x_2, x_1, x_9, x_10); -lean_dec(x_1); -return x_11; -} -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(2); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; +x_3 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__86() { _start: { -uint8_t x_3; -lean_inc(x_2); -lean_inc(x_1); -x_3 = l_Array_contains___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12(x_1, x_2); -if (x_3 == 0) -{ -lean_object* x_4; -x_4 = lean_array_push(x_1, x_2); -return x_4; -} -else -{ -lean_dec(x_2); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("optEllipsis", 11); return x_1; } } -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__87() { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_10 = lean_nat_add(x_8, x_9); -x_11 = lean_unsigned_to_nat(2u); -x_12 = lean_nat_div(x_10, x_11); -lean_dec(x_10); -lean_inc(x_5); -x_13 = lean_array_get(x_5, x_6, x_12); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_ctor_get(x_7, 0); -x_16 = l_Lean_Meta_DiscrTree_Key_lt(x_14, x_15); -if (x_16 == 0) -{ -uint8_t x_17; -lean_dec(x_9); -x_17 = l_Lean_Meta_DiscrTree_Key_lt(x_15, x_14); -lean_dec(x_14); -if (x_17 == 0) -{ -lean_object* x_18; uint8_t x_19; -lean_dec(x_8); -lean_dec(x_5); -x_18 = lean_array_get_size(x_6); -x_19 = lean_nat_dec_lt(x_12, x_18); -lean_dec(x_18); -if (x_19 == 0) -{ -lean_dec(x_12); -lean_dec(x_4); -lean_dec(x_2); -return x_6; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__86; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_20 = lean_array_fget(x_6, x_12); -x_21 = lean_box(0); -x_22 = lean_array_fset(x_6, x_12, x_21); -x_23 = !lean_is_exclusive(x_20); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_24 = lean_ctor_get(x_20, 1); -x_25 = lean_ctor_get(x_20, 0); -lean_dec(x_25); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_nat_add(x_3, x_26); -x_28 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_1, x_2, x_27, x_24); -lean_dec(x_27); -lean_ctor_set(x_20, 1, x_28); -lean_ctor_set(x_20, 0, x_4); -x_29 = lean_array_fset(x_22, x_12, x_20); -lean_dec(x_12); -return x_29; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__88() { +_start: { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_30 = lean_ctor_get(x_20, 1); -lean_inc(x_30); -lean_dec(x_20); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_nat_add(x_3, x_31); -x_33 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_1, x_2, x_32, x_30); -lean_dec(x_32); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_4); -lean_ctor_set(x_34, 1, x_33); -x_35 = lean_array_fset(x_22, x_12, x_34); -lean_dec(x_12); -return x_35; -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__87; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__55; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89() { +_start: { -x_9 = x_12; -goto _start; -} +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("}", 1); +return x_1; } -else -{ -uint8_t x_37; -lean_dec(x_14); -x_37 = lean_nat_dec_eq(x_12, x_8); -if (x_37 == 0) -{ -lean_dec(x_8); -x_8 = x_12; -goto _start; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__90() { +_start: { -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_dec(x_12); -lean_dec(x_9); -lean_dec(x_5); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_nat_add(x_3, x_39); -x_41 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_1, x_2, x_40); -lean_dec(x_40); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_4); -lean_ctor_set(x_42, 1, x_41); -x_43 = lean_nat_add(x_8, x_39); -lean_dec(x_8); -x_44 = l_Array_insertAt___rarg(x_6, x_43, x_42); -lean_dec(x_43); -return x_44; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__104; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__91() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__90; +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_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -uint8_t x_8; -x_8 = l_Array_isEmpty___rarg(x_6); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_9 = lean_unsigned_to_nat(0u); -lean_inc(x_5); -x_10 = lean_array_get(x_5, x_6, x_9); -x_11 = lean_ctor_get(x_7, 0); -x_12 = lean_ctor_get(x_10, 0); +lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_array_get_size(x_1); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +x_18 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__2; +lean_inc(x_13); lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Meta_DiscrTree_Key_lt(x_11, x_12); -if (x_13 == 0) -{ -uint8_t x_14; -x_14 = l_Lean_Meta_DiscrTree_Key_lt(x_12, x_11); -lean_dec(x_12); -if (x_14 == 0) -{ -lean_object* x_15; uint8_t x_16; -lean_dec(x_5); -x_15 = lean_array_get_size(x_6); -x_16 = lean_nat_dec_lt(x_9, x_15); -lean_dec(x_15); -if (x_16 == 0) -{ -lean_dec(x_4); -lean_dec(x_2); -return x_6; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_array_fget(x_6, x_9); -x_18 = lean_box(0); -x_19 = lean_array_fset(x_6, x_9, x_18); -x_20 = !lean_is_exclusive(x_17); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_17, 1); -x_22 = lean_ctor_get(x_17, 0); -lean_dec(x_22); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_nat_add(x_3, x_23); -x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_1, x_2, x_24, x_21); -lean_dec(x_24); -lean_ctor_set(x_17, 1, x_25); -lean_ctor_set(x_17, 0, x_4); -x_26 = lean_array_fset(x_19, x_9, x_17); -return x_26; -} -else +lean_inc(x_11); +lean_inc(x_10); +x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1(x_1, x_16, x_17, x_18, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_27 = lean_ctor_get(x_17, 1); -lean_inc(x_27); -lean_dec(x_17); -x_28 = lean_unsigned_to_nat(1u); -x_29 = lean_nat_add(x_3, x_28); -x_30 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_1, x_2, x_29, x_27); +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; size_t x_26; 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; size_t x_37; lean_object* x_38; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_array_get_size(x_24); +x_26 = lean_usize_of_nat(x_25); +lean_dec(x_25); +x_27 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; +x_28 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__87; +lean_inc(x_12); +lean_inc(x_24); +x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2(x_27, x_28, x_26, x_17, x_24, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); lean_dec(x_29); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_4); -lean_ctor_set(x_31, 1, x_30); -x_32 = lean_array_fset(x_19, x_9, x_31); -return x_32; -} -} -} -else -{ -lean_object* x_33; lean_object* x_34; uint8_t x_35; -lean_inc(x_5); -x_33 = l_Array_back___rarg(x_5, x_6); +x_32 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__104; +lean_inc(x_12); +lean_inc(x_24); +x_33 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3(x_27, x_32, x_26, x_17, x_24, x_8, x_9, x_10, x_11, x_12, x_13, x_31); 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_35 = l_Lean_Meta_DiscrTree_Key_lt(x_34, x_11); -if (x_35 == 0) -{ -uint8_t x_36; -x_36 = l_Lean_Meta_DiscrTree_Key_lt(x_11, x_34); -lean_dec(x_34); -if (x_36 == 0) -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; -lean_dec(x_5); -x_37 = lean_array_get_size(x_6); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_nat_sub(x_37, x_38); -x_40 = lean_nat_dec_lt(x_39, x_37); -lean_dec(x_37); -if (x_40 == 0) -{ -lean_dec(x_39); -lean_dec(x_4); -lean_dec(x_2); -return x_6; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_41 = lean_array_fget(x_6, x_39); -x_42 = lean_box(0); -x_43 = lean_array_fset(x_6, x_39, x_42); -x_44 = !lean_is_exclusive(x_41); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_45 = lean_ctor_get(x_41, 1); -x_46 = lean_ctor_get(x_41, 0); -lean_dec(x_46); -x_47 = lean_nat_add(x_3, x_38); -x_48 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_1, x_2, x_47, x_45); -lean_dec(x_47); -lean_ctor_set(x_41, 1, x_48); -lean_ctor_set(x_41, 0, x_4); -x_49 = lean_array_fset(x_43, x_39, x_41); -lean_dec(x_39); -return x_49; -} -else +x_36 = lean_array_get_size(x_2); +x_37 = lean_usize_of_nat(x_36); +lean_dec(x_36); +x_38 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(x_37, x_17, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_35); +lean_dec(x_11); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_50 = lean_ctor_get(x_41, 1); -lean_inc(x_50); +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; size_t x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; +x_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); +lean_inc(x_12); +x_41 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_12, x_13, x_40); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); lean_dec(x_41); -x_51 = lean_nat_add(x_3, x_38); -x_52 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_1, x_2, x_51, x_50); -lean_dec(x_51); -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_4); -lean_ctor_set(x_53, 1, x_52); -x_54 = lean_array_fset(x_43, x_39, x_53); -lean_dec(x_39); -return x_54; -} -} -} -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_55 = lean_array_get_size(x_6); -x_56 = lean_unsigned_to_nat(1u); -x_57 = lean_nat_sub(x_55, x_56); -lean_dec(x_55); -x_58 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__15(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_57); -return x_58; -} -} -else -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -lean_dec(x_34); -lean_dec(x_5); -x_59 = lean_unsigned_to_nat(1u); -x_60 = lean_nat_add(x_3, x_59); -x_61 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_1, x_2, x_60); -lean_dec(x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_4); -lean_ctor_set(x_62, 1, x_61); -x_63 = lean_array_push(x_6, x_62); -return x_63; -} -} -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_44 = lean_st_ref_get(x_13, x_43); +x_45 = lean_ctor_get(x_44, 1); +lean_inc(x_45); +lean_dec(x_44); +x_46 = lean_box(0); +x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__8; +x_48 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_48, 0, x_42); +lean_ctor_set(x_48, 1, x_47); +x_49 = lean_ctor_get(x_3, 0); +lean_inc(x_49); +lean_dec(x_3); +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +lean_dec(x_49); +lean_inc(x_50); +x_51 = lean_mk_syntax_ident(x_50); +x_52 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_53 = lean_array_push(x_52, x_48); +x_54 = lean_array_push(x_53, x_51); +x_55 = lean_box(2); +x_56 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__7; +x_57 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +lean_ctor_set(x_57, 2, x_54); +x_58 = lean_array_get_size(x_39); +x_59 = lean_usize_of_nat(x_58); +lean_dec(x_58); +x_60 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__5; +x_61 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5(x_60, x_59, x_17, x_39); +x_62 = l_Lean_Syntax_mkApp(x_57, x_61); +x_63 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__11; +x_64 = lean_name_append_before(x_50, x_63); +x_65 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__10; +x_66 = l_Lean_Name_append(x_65, x_64); +x_67 = lean_mk_syntax_ident(x_66); +lean_inc(x_12); +x_68 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_12, x_13, x_45); +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = lean_ctor_get(x_12, 10); +lean_inc(x_71); lean_dec(x_12); -lean_dec(x_5); -x_64 = lean_unsigned_to_nat(1u); -x_65 = lean_nat_add(x_3, x_64); -x_66 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_1, x_2, x_65); -lean_dec(x_65); -x_67 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_67, 0, x_4); -lean_ctor_set(x_67, 1, x_66); -x_68 = l_Array_insertAt___rarg(x_6, x_9, x_67); -return x_68; -} -} -else -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -lean_dec(x_5); -x_69 = lean_unsigned_to_nat(1u); -x_70 = lean_nat_add(x_3, x_69); -x_71 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_1, x_2, x_70); -lean_dec(x_70); -x_72 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_72, 0, x_4); -lean_ctor_set(x_72, 1, x_71); -x_73 = lean_array_push(x_6, x_72); -return x_73; -} -} -} -static lean_object* _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Meta_DiscrTree_instInhabitedTrie(lean_box(0)); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_DiscrTree_instInhabitedKey; -x_2 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__1; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_6 = lean_ctor_get(x_4, 0); -x_7 = lean_ctor_get(x_4, 1); -x_8 = lean_array_get_size(x_1); -x_9 = lean_nat_dec_lt(x_3, x_8); -lean_dec(x_8); -if (x_9 == 0) -{ -lean_object* x_10; -x_10 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11(x_6, x_2); -lean_ctor_set(x_4, 0, x_10); -return x_4; -} -else -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_array_fget(x_1, x_3); -x_12 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3; -lean_inc(x_11); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -x_14 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2; -x_15 = l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__14(x_1, x_2, x_3, x_11, x_14, x_7, x_13); +x_72 = lean_st_ref_get(x_13, x_70); lean_dec(x_13); -lean_ctor_set(x_4, 1, x_15); -return x_4; -} -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = lean_ctor_get(x_4, 0); -x_17 = lean_ctor_get(x_4, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_4); -x_18 = lean_array_get_size(x_1); -x_19 = lean_nat_dec_lt(x_3, x_18); -lean_dec(x_18); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; -x_20 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__11(x_16, x_2); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_17); -return x_21; -} -else +x_73 = !lean_is_exclusive(x_72); +if (x_73 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_22 = lean_array_fget(x_1, x_3); -x_23 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3; -lean_inc(x_22); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2; -x_26 = l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__14(x_1, x_2, x_3, x_22, x_25, x_17, x_24); +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; size_t x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; size_t x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; size_t x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; size_t x_330; lean_object* x_331; lean_object* x_332; size_t x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; +x_74 = lean_ctor_get(x_72, 0); +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +lean_dec(x_74); +x_76 = lean_environment_main_module(x_75); +x_77 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14; +lean_inc(x_69); +x_78 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_78, 0, x_69); +lean_ctor_set(x_78, 1, x_77); +x_79 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +lean_inc(x_4); +x_80 = l_Array_append___rarg(x_79, x_4); +x_81 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_82 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_82, 0, x_55); +lean_ctor_set(x_82, 1, x_81); +lean_ctor_set(x_82, 2, x_80); +x_83 = lean_array_push(x_52, x_78); +lean_inc(x_83); +x_84 = lean_array_push(x_83, x_82); +x_85 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__15; +x_86 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_86, 0, x_55); +lean_ctor_set(x_86, 1, x_85); +lean_ctor_set(x_86, 2, x_84); +x_87 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12; +lean_inc(x_69); +x_88 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_88, 0, x_69); +lean_ctor_set(x_88, 1, x_87); +x_89 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24; +lean_inc(x_69); +x_90 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_90, 0, x_69); +lean_ctor_set(x_90, 1, x_89); +x_91 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_92 = lean_array_push(x_91, x_90); +x_93 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__27; +x_94 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_94, 0, x_55); +lean_ctor_set(x_94, 1, x_93); +lean_ctor_set(x_94, 2, x_92); +x_95 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__31; +lean_inc(x_71); +lean_inc(x_76); +x_96 = l_Lean_addMacroScope(x_76, x_95, x_71); +x_97 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__30; +lean_inc(x_69); +x_98 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_98, 0, x_69); +lean_ctor_set(x_98, 1, x_97); +lean_ctor_set(x_98, 2, x_96); +lean_ctor_set(x_98, 3, x_46); +x_99 = lean_array_push(x_52, x_98); +x_100 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +lean_inc(x_99); +x_101 = lean_array_push(x_99, x_100); +x_102 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; +x_103 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_103, 0, x_55); +lean_ctor_set(x_103, 1, x_102); +lean_ctor_set(x_103, 2, x_101); +x_104 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__76; +lean_inc(x_69); +x_105 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_105, 0, x_69); +lean_ctor_set(x_105, 1, x_104); +x_106 = l_Array_zip___rarg(x_24, x_23); +lean_dec(x_23); lean_dec(x_24); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_16); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} -} -} -} -static lean_object* _init_l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Meta_DiscrTree_instInhabitedDiscrTree(lean_box(0)); -return x_1; -} -} -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16___closed__1; -x_3 = lean_panic_fn(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Init.Util", 9); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("getElem!", 8); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("index out of bounds", 19); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1; -x_2 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2; -x_3 = lean_unsigned_to_nat(62u); -x_4 = lean_unsigned_to_nat(36u); -x_5 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; -} -} -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Meta.DiscrTree", 19); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Meta.DiscrTree.insertCore", 30); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("invalid key sequence", 20); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5; -x_2 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6; -x_3 = lean_unsigned_to_nat(353u); -x_4 = lean_unsigned_to_nat(23u); -x_5 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = l_Array_isEmpty___rarg(x_2); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_array_get_size(x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_nat_dec_lt(x_6, x_5); -lean_dec(x_5); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; -x_9 = l_panic___at_Lean_Meta_DiscrTree_insertCore___spec__1(x_8); -lean_inc(x_9); -lean_inc(x_1); -x_10 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3(x_1, x_9); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_unsigned_to_nat(1u); -x_12 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_2, x_3, x_11); -lean_dec(x_2); -x_13 = l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(x_1, x_9, x_12); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_10, 0); -lean_inc(x_14); -lean_dec(x_10); -x_15 = lean_unsigned_to_nat(1u); -x_16 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_2, x_3, x_15, x_14); -lean_dec(x_2); -x_17 = l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(x_1, x_9, x_16); -return x_17; -} -} -else -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_array_fget(x_2, x_6); -lean_inc(x_18); -lean_inc(x_1); -x_19 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3(x_1, x_18); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_unsigned_to_nat(1u); -x_21 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_2, x_3, x_20); -lean_dec(x_2); -x_22 = l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(x_1, x_18, x_21); -return x_22; -} -else -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_19, 0); -lean_inc(x_23); -lean_dec(x_19); -x_24 = lean_unsigned_to_nat(1u); -x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_2, x_3, x_24, x_23); -lean_dec(x_2); -x_26 = l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(x_1, x_18, x_25); -return x_26; -} -} -} -else -{ -lean_object* x_27; lean_object* x_28; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_27 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8; -x_28 = l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16(x_27); -return x_28; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Meta_DiscrTree_mkPath(x_2, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) -{ -uint8_t x_10; -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2(x_1, x_11, x_3); -lean_ctor_set(x_9, 0, x_12); -return x_9; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_9, 0); -x_14 = lean_ctor_get(x_9, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_9); -x_15 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2(x_1, x_13, x_3); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -return x_16; -} -} -else -{ -uint8_t x_17; -lean_dec(x_3); -lean_dec(x_1); -x_17 = !lean_is_exclusive(x_9); -if (x_17 == 0) -{ -return x_9; -} -else -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_9, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_9); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; -} -} -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Option", 6); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__1; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__1; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__2; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__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; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___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) { -_start: -{ -uint8_t x_16; -x_16 = l_Lean_Server_RpcEncoding_isOptField(x_1); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -lean_dec(x_13); -x_17 = lean_array_push(x_5, x_4); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_2); -lean_ctor_set(x_18, 1, x_7); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_6); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_17); -lean_ctor_set(x_20, 1, x_19); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_3); -lean_ctor_set(x_21, 1, x_20); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_21); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_15); -return x_23; -} -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -lean_inc(x_13); -x_24 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_13, x_14, x_15); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_ctor_get(x_13, 10); -lean_inc(x_27); -lean_dec(x_13); -x_28 = lean_st_ref_get(x_14, x_26); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -lean_dec(x_30); -x_32 = lean_environment_main_module(x_31); -x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4; -x_34 = l_Lean_addMacroScope(x_32, x_33, x_27); -x_35 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__3; -x_36 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__6; -x_37 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_37, 0, x_25); -lean_ctor_set(x_37, 1, x_35); -lean_ctor_set(x_37, 2, x_34); -lean_ctor_set(x_37, 3, x_36); -x_38 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_39 = lean_array_push(x_38, x_4); -x_40 = lean_box(2); -x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_42 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_42, 2, x_39); -x_43 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_44 = lean_array_push(x_43, x_37); -x_45 = lean_array_push(x_44, x_42); -x_46 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_40); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = lean_array_push(x_5, x_47); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_2); -lean_ctor_set(x_49, 1, x_7); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_6); -lean_ctor_set(x_50, 1, x_49); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_48); -lean_ctor_set(x_51, 1, x_50); -x_52 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_52, 0, x_3); -lean_ctor_set(x_52, 1, x_51); -x_53 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_28, 0, x_53); -return x_28; -} -else -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_54 = lean_ctor_get(x_28, 0); -x_55 = lean_ctor_get(x_28, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_28); -x_56 = lean_ctor_get(x_54, 0); -lean_inc(x_56); -lean_dec(x_54); -x_57 = lean_environment_main_module(x_56); -x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4; -x_59 = l_Lean_addMacroScope(x_57, x_58, x_27); -x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__3; -x_61 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__6; -x_62 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_62, 0, x_25); -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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_64 = lean_array_push(x_63, x_4); -x_65 = lean_box(2); -x_66 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_67 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -lean_ctor_set(x_67, 2, x_64); -x_68 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_69 = lean_array_push(x_68, x_62); -x_70 = lean_array_push(x_69, x_67); -x_71 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_72 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_72, 0, x_65); -lean_ctor_set(x_72, 1, x_71); -lean_ctor_set(x_72, 2, x_70); -x_73 = lean_array_push(x_5, x_72); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_2); -lean_ctor_set(x_74, 1, x_7); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_6); -lean_ctor_set(x_75, 1, x_74); -x_76 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_75); -x_77 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_77, 0, x_3); -lean_ctor_set(x_77, 1, x_76); -x_78 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_78, 0, x_77); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_78); -lean_ctor_set(x_79, 1, x_55); -return x_79; -} -} -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211; -x_2 = lean_mk_syntax_ident(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__1; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -lean_dec(x_8); -lean_inc(x_1); -x_16 = lean_mk_syntax_ident(x_1); -x_17 = lean_array_push(x_5, x_16); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_6); -lean_inc(x_4); -x_18 = l_Lean_Meta_DiscrTree_getMatch___rarg(x_4, x_6, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Array_back_x3f___rarg(x_19); -lean_dec(x_19); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; 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_inc(x_1); -x_22 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_1, x_13, x_14, x_20); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_mk_syntax_ident(x_23); -lean_inc(x_13); -x_26 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_13, x_14, 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); -lean_dec(x_26); -x_29 = lean_st_ref_get(x_14, x_28); -x_30 = lean_ctor_get(x_29, 1); -lean_inc(x_30); -lean_dec(x_29); -x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; -lean_inc(x_27); -x_32 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_32, 0, x_27); -lean_ctor_set(x_32, 1, x_31); -x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -lean_inc(x_25); -x_34 = lean_array_push(x_33, x_25); -x_35 = lean_box(2); -x_36 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_37 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -lean_ctor_set(x_37, 2, x_34); -x_38 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -x_39 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_39, 0, x_27); -lean_ctor_set(x_39, 1, x_38); -x_40 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_41 = lean_array_push(x_40, x_32); -x_42 = lean_array_push(x_41, x_37); -x_43 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_44 = lean_array_push(x_42, x_43); -x_45 = lean_array_push(x_44, x_43); -x_46 = lean_array_push(x_45, x_39); -x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; -x_48 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_48, 0, x_35); -lean_ctor_set(x_48, 1, x_47); -lean_ctor_set(x_48, 2, x_46); -x_49 = lean_array_push(x_2, x_48); -x_50 = lean_box(0); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_6); -x_51 = l_Lean_PrettyPrinter_delab(x_6, x_50, x_11, x_12, x_13, x_14, x_30); -if (lean_obj_tag(x_51) == 0) -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -lean_inc(x_13); -x_54 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_13, x_14, 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); -lean_dec(x_54); -x_57 = lean_st_ref_get(x_14, x_56); -x_58 = lean_ctor_get(x_57, 1); -lean_inc(x_58); -lean_dec(x_57); -x_59 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; -lean_inc(x_55); -x_60 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_60, 0, x_55); -lean_ctor_set(x_60, 1, x_59); -x_61 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_62 = lean_array_push(x_61, x_52); -lean_inc(x_25); -x_63 = lean_array_push(x_62, x_25); -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_35); -lean_ctor_set(x_64, 1, x_36); -lean_ctor_set(x_64, 2, x_63); -x_65 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2; -x_66 = lean_array_push(x_65, x_64); -x_67 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_68 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_68, 0, x_35); -lean_ctor_set(x_68, 1, x_67); -lean_ctor_set(x_68, 2, x_66); -x_69 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; -x_70 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_70, 0, x_55); -lean_ctor_set(x_70, 1, x_69); -x_71 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_72 = lean_array_push(x_71, x_60); -x_73 = lean_array_push(x_72, x_43); -x_74 = lean_array_push(x_73, x_68); -x_75 = lean_array_push(x_74, x_70); -x_76 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58; -x_77 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_77, 0, x_35); -lean_ctor_set(x_77, 1, x_76); -lean_ctor_set(x_77, 2, x_75); -x_78 = lean_array_push(x_49, x_77); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_25); -x_79 = l_Lean_Meta_DiscrTree_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1(x_4, x_6, x_25, x_11, x_12, x_13, x_14, x_58); -if (lean_obj_tag(x_79) == 0) -{ -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_80 = lean_ctor_get(x_79, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_79, 1); -lean_inc(x_81); -lean_dec(x_79); -lean_inc(x_25); -x_82 = lean_array_push(x_7, x_25); -x_83 = lean_box(0); -x_84 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1(x_1, x_17, x_78, x_25, x_3, x_80, x_82, x_83, x_9, x_10, x_11, x_12, x_13, x_14, x_81); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -return x_84; -} -else -{ -uint8_t x_85; -lean_dec(x_78); -lean_dec(x_25); -lean_dec(x_17); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_1); -x_85 = !lean_is_exclusive(x_79); -if (x_85 == 0) -{ -return x_79; -} -else -{ -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_79, 0); -x_87 = lean_ctor_get(x_79, 1); -lean_inc(x_87); -lean_inc(x_86); -lean_dec(x_79); -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -return x_88; -} -} -} -else -{ -uint8_t x_89; -lean_dec(x_49); -lean_dec(x_25); -lean_dec(x_17); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_89 = !lean_is_exclusive(x_51); -if (x_89 == 0) -{ -return x_51; -} -else -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; -x_90 = lean_ctor_get(x_51, 0); -x_91 = lean_ctor_get(x_51, 1); -lean_inc(x_91); -lean_inc(x_90); -lean_dec(x_51); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_90); -lean_ctor_set(x_92, 1, x_91); -return x_92; -} -} -} -else -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; -lean_dec(x_6); -x_93 = lean_ctor_get(x_21, 0); -lean_inc(x_93); -lean_dec(x_21); -x_94 = lean_box(0); -x_95 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1(x_1, x_17, x_2, x_93, x_3, x_4, x_7, x_94, x_9, x_10, x_11, x_12, x_13, x_14, x_20); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -return x_95; -} -} -else -{ -uint8_t x_96; -lean_dec(x_17); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_96 = !lean_is_exclusive(x_18); -if (x_96 == 0) -{ -return x_18; -} -else -{ -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_18, 0); -x_98 = lean_ctor_get(x_18, 1); -lean_inc(x_98); -lean_inc(x_97); -lean_dec(x_18); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -return x_99; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_16 = lean_unsigned_to_nat(0u); -x_17 = l_Lean_Expr_getAppNumArgsAux(x_7, x_16); -x_18 = lean_nat_sub(x_17, x_16); -lean_dec(x_17); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_sub(x_18, x_19); -lean_dec(x_18); -x_21 = l_Lean_Expr_getRevArg_x21(x_7, x_20); -x_22 = lean_box(0); -x_23 = lean_apply_14(x_1, x_2, x_3, x_4, x_5, x_21, x_6, x_22, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -return x_23; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("optional field '", 16); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("' has type", 10); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("", 0); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__5; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("\nbut is expected to have type", 29); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__7; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__9() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Option _", 8); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__9; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__10; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__11; -x_2 = l_Lean_indentD(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; -x_12 = lean_usize_dec_lt(x_3, x_2); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_4); -lean_ctor_set(x_13, 1, x_11); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_14 = lean_array_uget(x_1, x_3); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_4, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_4, 1); -lean_inc(x_18); -lean_dec(x_4); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = lean_ctor_get(x_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_15); -x_25 = lean_alloc_closure((void*)(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___boxed), 15, 1); -lean_closure_set(x_25, 0, x_15); -lean_inc(x_15); -x_26 = l_Lean_Server_RpcEncoding_isOptField(x_15); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; -lean_dec(x_25); -x_27 = lean_box(0); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_28 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2(x_15, x_17, x_19, x_21, x_23, x_16, x_24, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -if (lean_obj_tag(x_29) == 0) -{ -uint8_t x_30; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_30 = !lean_is_exclusive(x_28); -if (x_30 == 0) -{ -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_28, 0); -lean_dec(x_31); -x_32 = lean_ctor_get(x_29, 0); -lean_inc(x_32); -lean_dec(x_29); -lean_ctor_set(x_28, 0, x_32); -return x_28; -} -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_28, 1); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_ctor_get(x_29, 0); -lean_inc(x_34); -lean_dec(x_29); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_33); -return x_35; -} -} -else -{ -lean_object* x_36; lean_object* x_37; size_t x_38; size_t x_39; -x_36 = lean_ctor_get(x_28, 1); -lean_inc(x_36); -lean_dec(x_28); -x_37 = lean_ctor_get(x_29, 0); -lean_inc(x_37); -lean_dec(x_29); -x_38 = 1; -x_39 = lean_usize_add(x_3, x_38); -x_3 = x_39; -x_4 = x_37; -x_11 = x_36; -goto _start; -} -} -else -{ -uint8_t x_41; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_41 = !lean_is_exclusive(x_28); -if (x_41 == 0) -{ -return x_28; -} -else -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_28, 0); -x_43 = lean_ctor_get(x_28, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_28); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; -} -} -} -else -{ -lean_object* x_45; uint8_t x_46; -x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4; -x_46 = l_Lean_Expr_isAppOf(x_16, x_45); -if (x_46 == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; -lean_dec(x_25); -lean_dec(x_24); -lean_dec(x_23); -lean_dec(x_21); -lean_dec(x_19); -lean_dec(x_17); -x_47 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_47, 0, x_15); -x_48 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__2; -x_49 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_47); -x_50 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__4; -x_51 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -x_52 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_52, 0, x_16); -x_53 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6; -x_54 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_52); -x_55 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_53); -x_56 = l_Lean_indentD(x_55); -x_57 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_57, 0, x_51); -lean_ctor_set(x_57, 1, x_56); -x_58 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__8; -x_59 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -x_60 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__12; -x_61 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -x_62 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_53); -x_63 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__4(x_62, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -x_64 = !lean_is_exclusive(x_63); -if (x_64 == 0) -{ -return x_63; -} -else -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_63, 0); -x_66 = lean_ctor_get(x_63, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_63); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -return x_67; -} -} -else -{ -lean_object* x_68; lean_object* x_69; -lean_dec(x_15); -x_68 = lean_box(0); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_69 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__3(x_25, x_17, x_19, x_21, x_23, x_24, x_16, x_68, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_69) == 0) -{ -lean_object* x_70; -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -if (lean_obj_tag(x_70) == 0) -{ -uint8_t x_71; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_71 = !lean_is_exclusive(x_69); -if (x_71 == 0) -{ -lean_object* x_72; lean_object* x_73; -x_72 = lean_ctor_get(x_69, 0); -lean_dec(x_72); -x_73 = lean_ctor_get(x_70, 0); -lean_inc(x_73); -lean_dec(x_70); -lean_ctor_set(x_69, 0, x_73); -return x_69; -} -else -{ -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_69, 1); -lean_inc(x_74); -lean_dec(x_69); -x_75 = lean_ctor_get(x_70, 0); -lean_inc(x_75); -lean_dec(x_70); -x_76 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_74); -return x_76; -} -} -else -{ -lean_object* x_77; lean_object* x_78; size_t x_79; size_t x_80; -x_77 = lean_ctor_get(x_69, 1); -lean_inc(x_77); -lean_dec(x_69); -x_78 = lean_ctor_get(x_70, 0); -lean_inc(x_78); -lean_dec(x_70); -x_79 = 1; -x_80 = lean_usize_add(x_3, x_79); -x_3 = x_80; -x_4 = x_78; -x_11 = x_77; -goto _start; -} -} -else -{ -uint8_t x_82; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_82 = !lean_is_exclusive(x_69); -if (x_82 == 0) -{ -return x_69; -} -else -{ -lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_83 = lean_ctor_get(x_69, 0); -x_84 = lean_ctor_get(x_69, 1); -lean_inc(x_84); -lean_inc(x_83); -lean_dec(x_69); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -return x_85; -} -} -} -} -} -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("liftMethod", 10); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("←", 3); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("proj", 4); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("a", 1); -return x_1; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__4; -x_2 = lean_string_utf8_byte_size(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__4; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__5; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__4; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_10); -lean_dec(x_2); -lean_dec(x_1); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_5); -lean_ctor_set(x_14, 1, x_12); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; 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; size_t x_78; size_t x_79; lean_object* x_80; -x_15 = lean_array_uget(x_5, x_4); -x_16 = lean_unsigned_to_nat(0u); -x_17 = lean_array_uset(x_5, x_4, x_16); -lean_inc(x_10); -x_18 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_10, x_11, x_12); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_10, 10); -lean_inc(x_21); -x_22 = lean_st_ref_get(x_11, x_20); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_ctor_get(x_23, 0); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_environment_main_module(x_25); -x_27 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__5; -lean_inc(x_1); -x_28 = l_Lean_Name_str___override(x_1, x_27); -x_29 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__16; -x_30 = l_Lean_Name_str___override(x_28, x_29); -x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__217; -lean_inc(x_30); -x_32 = l_Lean_Name_str___override(x_30, x_31); -x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__219; -lean_inc(x_30); -x_34 = l_Lean_Name_str___override(x_30, x_33); -x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -lean_inc(x_15); -x_36 = lean_array_push(x_35, x_15); -x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_38 = lean_array_push(x_36, x_37); -x_39 = lean_box(2); -x_40 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_34); -lean_ctor_set(x_40, 2, x_38); -x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; -lean_inc(x_19); -x_42 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_42, 0, x_19); -lean_ctor_set(x_42, 1, x_41); -x_43 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1; -lean_inc(x_30); -x_44 = l_Lean_Name_str___override(x_30, x_43); -x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2; -lean_inc(x_19); -x_46 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_46, 0, x_19); -lean_ctor_set(x_46, 1, x_45); -x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; -lean_inc(x_30); -x_48 = l_Lean_Name_str___override(x_30, x_47); -lean_inc(x_2); -x_49 = lean_mk_syntax_ident(x_2); -x_50 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__3; -x_51 = l_Lean_Name_str___override(x_30, x_50); -x_52 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7; -x_53 = l_Lean_addMacroScope(x_26, x_52, x_21); -x_54 = lean_box(0); -x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6; -lean_inc(x_19); -x_56 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_56, 0, x_19); -lean_ctor_set(x_56, 1, x_55); -lean_ctor_set(x_56, 2, x_53); -lean_ctor_set(x_56, 3, x_54); -x_57 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__245; -x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_19); -lean_ctor_set(x_58, 1, x_57); -x_59 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; -x_60 = lean_array_push(x_59, x_56); -x_61 = lean_array_push(x_60, x_58); -x_62 = lean_array_push(x_61, x_15); -x_63 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_63, 0, x_39); -lean_ctor_set(x_63, 1, x_51); -lean_ctor_set(x_63, 2, x_62); -x_64 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_65 = lean_array_push(x_64, x_63); -x_66 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_67 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_67, 0, x_39); -lean_ctor_set(x_67, 1, x_66); -lean_ctor_set(x_67, 2, x_65); -x_68 = lean_array_push(x_35, x_49); -x_69 = lean_array_push(x_68, x_67); -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_39); -lean_ctor_set(x_70, 1, x_48); -lean_ctor_set(x_70, 2, x_69); -x_71 = lean_array_push(x_35, x_46); -x_72 = lean_array_push(x_71, x_70); -x_73 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_73, 0, x_39); -lean_ctor_set(x_73, 1, x_44); -lean_ctor_set(x_73, 2, x_72); -x_74 = lean_array_push(x_59, x_40); -x_75 = lean_array_push(x_74, x_42); -x_76 = lean_array_push(x_75, x_73); -x_77 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_77, 0, x_39); -lean_ctor_set(x_77, 1, x_32); -lean_ctor_set(x_77, 2, x_76); -x_78 = 1; -x_79 = lean_usize_add(x_4, x_78); -x_80 = lean_array_uset(x_17, x_4, x_77); -x_4 = x_79; -x_5 = x_80; -x_12 = x_24; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__19(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_10); -lean_dec(x_2); -lean_dec(x_1); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_5); -lean_ctor_set(x_14, 1, x_12); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; 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; size_t x_78; size_t x_79; lean_object* x_80; -x_15 = lean_array_uget(x_5, x_4); -x_16 = lean_unsigned_to_nat(0u); -x_17 = lean_array_uset(x_5, x_4, x_16); -lean_inc(x_10); -x_18 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_10, x_11, x_12); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_10, 10); -lean_inc(x_21); -x_22 = lean_st_ref_get(x_11, x_20); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_ctor_get(x_23, 0); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_environment_main_module(x_25); -x_27 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__5; -lean_inc(x_1); -x_28 = l_Lean_Name_str___override(x_1, x_27); -x_29 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__16; -x_30 = l_Lean_Name_str___override(x_28, x_29); -x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__217; -lean_inc(x_30); -x_32 = l_Lean_Name_str___override(x_30, x_31); -x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__219; -lean_inc(x_30); -x_34 = l_Lean_Name_str___override(x_30, x_33); -x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -lean_inc(x_15); -x_36 = lean_array_push(x_35, x_15); -x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_38 = lean_array_push(x_36, x_37); -x_39 = lean_box(2); -x_40 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_34); -lean_ctor_set(x_40, 2, x_38); -x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; -lean_inc(x_19); -x_42 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_42, 0, x_19); -lean_ctor_set(x_42, 1, x_41); -x_43 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1; -lean_inc(x_30); -x_44 = l_Lean_Name_str___override(x_30, x_43); -x_45 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2; -lean_inc(x_19); -x_46 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_46, 0, x_19); -lean_ctor_set(x_46, 1, x_45); -x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; -lean_inc(x_30); -x_48 = l_Lean_Name_str___override(x_30, x_47); -lean_inc(x_2); -x_49 = lean_mk_syntax_ident(x_2); -x_50 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__3; -x_51 = l_Lean_Name_str___override(x_30, x_50); -x_52 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7; -x_53 = l_Lean_addMacroScope(x_26, x_52, x_21); -x_54 = lean_box(0); -x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6; -lean_inc(x_19); -x_56 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_56, 0, x_19); -lean_ctor_set(x_56, 1, x_55); -lean_ctor_set(x_56, 2, x_53); -lean_ctor_set(x_56, 3, x_54); -x_57 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__245; -x_58 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_58, 0, x_19); -lean_ctor_set(x_58, 1, x_57); -x_59 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; -x_60 = lean_array_push(x_59, x_56); -x_61 = lean_array_push(x_60, x_58); -x_62 = lean_array_push(x_61, x_15); -x_63 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_63, 0, x_39); -lean_ctor_set(x_63, 1, x_51); -lean_ctor_set(x_63, 2, x_62); -x_64 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_65 = lean_array_push(x_64, x_63); -x_66 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_67 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_67, 0, x_39); -lean_ctor_set(x_67, 1, x_66); -lean_ctor_set(x_67, 2, x_65); -x_68 = lean_array_push(x_35, x_49); -x_69 = lean_array_push(x_68, x_67); -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_39); -lean_ctor_set(x_70, 1, x_48); -lean_ctor_set(x_70, 2, x_69); -x_71 = lean_array_push(x_35, x_46); -x_72 = lean_array_push(x_71, x_70); -x_73 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_73, 0, x_39); -lean_ctor_set(x_73, 1, x_44); -lean_ctor_set(x_73, 2, x_72); -x_74 = lean_array_push(x_59, x_40); -x_75 = lean_array_push(x_74, x_42); -x_76 = lean_array_push(x_75, x_73); -x_77 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_77, 0, x_39); -lean_ctor_set(x_77, 1, x_32); -lean_ctor_set(x_77, 2, x_76); -x_78 = 1; -x_79 = lean_usize_add(x_4, x_78); -x_80 = lean_array_uset(x_17, x_4, x_77); -x_4 = x_79; -x_5 = x_80; -x_12 = x_24; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__20(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; -x_11 = lean_usize_dec_lt(x_2, x_1); -if (x_11 == 0) -{ -lean_object* x_12; -lean_dec(x_6); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_3); -lean_ctor_set(x_12, 1, x_10); -return x_12; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_array_uget(x_3, x_2); -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_array_uset(x_3, x_2, x_14); -lean_inc(x_6); -x_16 = l_Lean_Meta_getFVarLocalDecl(x_13, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Lean_LocalDecl_userName(x_17); -lean_dec(x_17); -x_20 = lean_mk_syntax_ident(x_19); -x_21 = 1; -x_22 = lean_usize_add(x_2, x_21); -x_23 = lean_array_uset(x_15, x_2, x_20); -x_2 = x_22; -x_3 = x_23; -x_10 = x_18; -goto _start; -} -else -{ -uint8_t x_25; -lean_dec(x_15); -lean_dec(x_6); -x_25 = !lean_is_exclusive(x_16); -if (x_25 == 0) -{ -return x_16; -} -else -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_16, 0); -x_27 = lean_ctor_get(x_16, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_16); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__21(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_lt(x_3, x_2); -if (x_5 == 0) -{ -return x_4; -} -else -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; -x_6 = lean_array_uget(x_4, x_3); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_array_uset(x_4, x_3, x_7); -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_11 = lean_array_uset(x_8, x_3, x_6); -x_3 = x_10; -x_4 = x_11; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__22(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_lt(x_3, x_2); -if (x_5 == 0) -{ -return x_4; -} -else -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; -x_6 = lean_array_uget(x_4, x_3); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_array_uset(x_4, x_3, x_7); -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_11 = lean_array_uset(x_8, x_3, x_6); -x_3 = x_10; -x_4 = x_11; -goto _start; -} -} -} -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("structExplicitBinder", 20); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, size_t x_10, size_t x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_11, x_10); -if (x_13 == 0) -{ -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_12; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_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; -x_14 = lean_array_uget(x_12, x_11); -x_15 = lean_unsigned_to_nat(0u); -x_16 = lean_array_uset(x_12, x_11, x_15); -x_17 = 1; -x_18 = lean_usize_add(x_11, x_17); -x_19 = lean_ctor_get(x_14, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); -lean_dec(x_14); -x_21 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23___closed__1; -lean_inc(x_5); -x_22 = l_Lean_Name_str___override(x_5, x_21); -x_23 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; -lean_inc(x_3); -x_24 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_24, 0, x_3); -lean_ctor_set(x_24, 1, x_23); -lean_inc(x_9); -x_25 = lean_array_push(x_9, x_19); -x_26 = lean_box(2); -lean_inc(x_4); -x_27 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_4); -lean_ctor_set(x_27, 2, x_25); -x_28 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__55; -lean_inc(x_5); -x_29 = l_Lean_Name_str___override(x_5, x_28); -x_30 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__94; -lean_inc(x_1); -x_31 = l_Lean_Name_str___override(x_1, x_30); -x_32 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; -lean_inc(x_3); -x_33 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_33, 0, x_3); -lean_ctor_set(x_33, 1, x_32); -lean_inc(x_2); -x_34 = lean_array_push(x_2, x_33); -x_35 = lean_array_push(x_34, x_20); -x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_26); -lean_ctor_set(x_36, 1, x_31); -lean_ctor_set(x_36, 2, x_35); -lean_inc(x_9); -x_37 = lean_array_push(x_9, x_36); -lean_inc(x_4); -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_26); -lean_ctor_set(x_38, 1, x_4); -lean_ctor_set(x_38, 2, x_37); -lean_inc(x_6); -lean_inc(x_2); -x_39 = lean_array_push(x_2, x_6); -x_40 = lean_array_push(x_39, x_38); -x_41 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_41, 0, x_26); -lean_ctor_set(x_41, 1, x_29); -lean_ctor_set(x_41, 2, x_40); -x_42 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -lean_inc(x_3); -x_43 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_43, 0, x_3); -lean_ctor_set(x_43, 1, x_42); -lean_inc(x_8); -lean_inc(x_7); -x_44 = lean_array_push(x_7, x_8); -x_45 = lean_array_push(x_44, x_24); -x_46 = lean_array_push(x_45, x_27); -x_47 = lean_array_push(x_46, x_41); -lean_inc(x_6); -x_48 = lean_array_push(x_47, x_6); -x_49 = lean_array_push(x_48, x_43); -x_50 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_50, 0, x_26); -lean_ctor_set(x_50, 1, x_22); -lean_ctor_set(x_50, 2, x_49); -x_51 = lean_array_uset(x_16, x_11, x_50); -x_11 = x_18; -x_12 = x_51; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__24(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; -x_6 = lean_usize_dec_lt(x_4, x_3); -if (x_6 == 0) -{ -return x_5; -} -else -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; -x_7 = lean_array_uget(x_5, x_4); -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_array_uset(x_5, x_4, x_8); -x_10 = 1; -x_11 = lean_usize_add(x_4, x_10); -x_12 = lean_array_uset(x_9, x_4, x_7); -x_4 = x_11; -x_5 = x_12; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25(size_t x_1, size_t x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) -{ -return x_3; -} -else -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = lean_array_uset(x_7, x_2, x_5); -x_2 = x_9; -x_3 = x_10; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__26(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; -x_6 = lean_usize_dec_lt(x_4, x_3); -if (x_6 == 0) -{ -return x_5; -} -else -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; -x_7 = lean_array_uget(x_5, x_4); -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_array_uset(x_5, x_4, x_8); -x_10 = 1; -x_11 = lean_usize_add(x_4, x_10); -x_12 = lean_array_uset(x_9, x_4, x_7); -x_4 = x_11; -x_5 = x_12; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__29(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_1); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_5); -lean_ctor_set(x_14, 1, x_12); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_array_uget(x_2, x_4); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_15); -lean_inc(x_1); -x_16 = l_Lean_Meta_mkProjection(x_1, x_15, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_19 = lean_infer_type(x_17, x_8, x_9, x_10, x_11, x_18); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; size_t x_24; size_t x_25; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_15); -lean_ctor_set(x_22, 1, x_20); -x_23 = lean_array_push(x_5, x_22); -x_24 = 1; -x_25 = lean_usize_add(x_4, x_24); -x_4 = x_25; -x_5 = x_23; -x_12 = x_21; -goto _start; -} -else -{ -uint8_t x_27; -lean_dec(x_15); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_5); -lean_dec(x_1); -x_27 = !lean_is_exclusive(x_19); -if (x_27 == 0) -{ -return x_19; -} -else -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_19, 0); -x_29 = lean_ctor_get(x_19, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_19); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; -} -} -} -else -{ -uint8_t x_31; -lean_dec(x_15); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_5); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_16); -if (x_31 == 0) -{ -return x_16; -} -else -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_16, 0); -x_33 = lean_ctor_get(x_16, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_16); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; -x_11 = lean_box(0); -x_12 = lean_apply_1(x_1, x_11); -x_13 = lean_array_get_size(x_12); -x_14 = lean_usize_of_nat(x_13); -lean_dec(x_13); -x_15 = 0; -x_16 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__29(x_3, x_12, x_14, x_15, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_12); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_apply_8(x_2, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_19); -return x_20; -} -else -{ -uint8_t x_21; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_21 = !lean_is_exclusive(x_17); -if (x_21 == 0) -{ -return x_17; -} -else -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_17, 0); -x_23 = lean_ctor_get(x_17, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_17); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); -lean_dec(x_1); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -x_14 = lean_box(0); -x_15 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_13, x_14); -x_16 = lean_ctor_get(x_12, 0); -lean_inc(x_16); -lean_dec(x_12); -x_17 = l_Lean_Expr_const___override(x_16, x_15); -x_18 = l_Lean_mkAppN(x_17, x_2); -x_19 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28___rarg___lambda__1), 10, 2); -lean_closure_set(x_19, 0, x_4); -lean_closure_set(x_19, 1, x_3); -x_20 = l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2; -x_21 = 0; -x_22 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__3___rarg(x_20, x_21, x_18, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_22; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28___rarg), 11, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_11 = lean_st_ref_get(x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_ctor_get(x_12, 0); -lean_inc(x_14); -lean_dec(x_12); -lean_inc(x_1); -x_15 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___rarg___lambda__2___boxed), 3, 2); -lean_closure_set(x_15, 0, x_1); -lean_closure_set(x_15, 1, x_14); -x_16 = l_Lean_Server_RpcEncoding_withFieldsAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__28___rarg(x_1, x_2, x_3, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_16; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__27(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__27___rarg), 10, 0); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___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___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__2; -x_2 = lean_unsigned_to_nat(0u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__3; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__4; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__5; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__6; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("term", 4); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__8; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__9; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("explicit", 8); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__11; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__13() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("@", 1); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("RpcEncodingPacket", 17); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__18() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__19() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__18; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__20() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__19; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__21() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__20; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__22() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__21; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__22; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("structure", 9); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__25() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__26() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("structureTk", 11); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__27() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__26; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("where", 5); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__29() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("structFields", 12); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__30() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__29; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__31() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("optDeriving", 11); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__32() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__31; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("deriving", 8); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__34() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("group", 5); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__34; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__36() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("FromJson", 8); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__37() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__36; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__38() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__37; -x_2 = lean_mk_syntax_ident(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__38; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__40() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__41() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__40; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(",", 1); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__43() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("ToJson", 6); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__44() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__43; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__45() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__44; -x_2 = lean_mk_syntax_ident(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__45; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__48() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__41; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__51() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__52() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__124; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__51; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__1; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__54() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__55() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("whereStructInst", 15); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__56() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__55; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__57() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("whereStructField", 16); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__57; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__59() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("letDecl", 7); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__59; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__61() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("letIdDecl", 9); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__61; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__63() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__64() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__63; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__65() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("termReturn", 10); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__65; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("return", 6); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__68() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; -x_3 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = lean_box(2); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__236; -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__51; -x_4 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__70() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__71() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__70; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__52; -x_3 = lean_array_push(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; -x_12 = lean_array_get_size(x_1); -x_13 = lean_usize_of_nat(x_12); -lean_dec(x_12); -x_14 = 0; -x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__7; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17(x_1, x_13, x_14, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; size_t x_27; 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; size_t x_38; lean_object* x_39; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -x_19 = lean_ctor_get(x_18, 1); -lean_inc(x_19); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_ctor_get(x_16, 1); -lean_inc(x_21); -lean_dec(x_16); -x_22 = lean_ctor_get(x_17, 0); -lean_inc(x_22); -lean_dec(x_17); -x_23 = lean_ctor_get(x_18, 0); -lean_inc(x_23); -lean_dec(x_18); -x_24 = lean_ctor_get(x_20, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_20, 1); -lean_inc(x_25); -lean_dec(x_20); -x_26 = lean_array_get_size(x_24); -x_27 = lean_usize_of_nat(x_26); -lean_dec(x_26); -x_28 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; -x_29 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225; -lean_inc(x_9); -lean_inc(x_24); -x_30 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18(x_28, x_29, x_27, x_14, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_21); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); -lean_inc(x_32); -lean_dec(x_30); -x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232; -lean_inc(x_9); -lean_inc(x_24); -x_34 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__19(x_28, x_33, x_27, x_14, x_24, x_5, x_6, x_7, x_8, x_9, x_10, 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 = lean_array_get_size(x_2); -x_38 = lean_usize_of_nat(x_37); -lean_dec(x_37); -x_39 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__20(x_38, x_14, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_36); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -if (lean_obj_tag(x_39) == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; 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; size_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; size_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; uint8_t x_78; -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); -lean_inc(x_41); -lean_dec(x_39); -lean_inc(x_9); -x_42 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_41); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_st_ref_get(x_10, x_44); -x_46 = lean_ctor_get(x_45, 1); -lean_inc(x_46); -lean_dec(x_45); -x_47 = lean_box(0); -x_48 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__13; -x_49 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_49, 0, x_43); -lean_ctor_set(x_49, 1, x_48); -x_50 = lean_ctor_get(x_3, 0); -lean_inc(x_50); -lean_dec(x_3); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -lean_dec(x_50); -x_52 = lean_mk_syntax_ident(x_51); -x_53 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_54 = lean_array_push(x_53, x_49); -x_55 = lean_array_push(x_54, x_52); -x_56 = lean_box(2); -x_57 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12; -x_58 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -lean_ctor_set(x_58, 2, x_55); -x_59 = lean_array_get_size(x_40); -x_60 = lean_usize_of_nat(x_59); -lean_dec(x_59); -x_61 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__10; -x_62 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__21(x_61, x_60, x_14, x_40); -x_63 = l_Lean_Syntax_mkApp(x_58, x_62); -x_64 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__15; -x_65 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_64, x_9, x_10, x_46); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -lean_dec(x_65); -x_68 = lean_mk_syntax_ident(x_66); -x_69 = lean_array_get_size(x_25); -x_70 = lean_usize_of_nat(x_69); -lean_dec(x_69); -x_71 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__22(x_61, x_70, x_14, x_25); -lean_inc(x_68); -x_72 = l_Lean_Syntax_mkApp(x_68, x_71); -lean_inc(x_9); -x_73 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_67); -x_74 = lean_ctor_get(x_73, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_73, 1); -lean_inc(x_75); -lean_dec(x_73); -x_76 = lean_ctor_get(x_9, 10); -lean_inc(x_76); -lean_dec(x_9); -x_77 = lean_st_ref_get(x_10, x_75); -lean_dec(x_10); -x_78 = !lean_is_exclusive(x_77); -if (x_78 == 0) -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; size_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; 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; size_t x_189; lean_object* x_190; lean_object* x_191; size_t x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; size_t x_236; lean_object* x_237; lean_object* x_238; size_t x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; -x_79 = lean_ctor_get(x_77, 0); -x_80 = lean_ctor_get(x_79, 0); -lean_inc(x_80); -lean_dec(x_79); -x_81 = lean_environment_main_module(x_80); -x_82 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; -lean_inc(x_74); -x_83 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_83, 0, x_74); -lean_ctor_set(x_83, 1, x_82); -x_84 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_85 = l_Array_append___rarg(x_84, x_22); -x_86 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_87 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_87, 0, x_56); -lean_ctor_set(x_87, 1, x_86); -lean_ctor_set(x_87, 2, x_85); -x_88 = lean_array_push(x_53, x_83); -x_89 = lean_array_push(x_88, x_87); -x_90 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; -x_91 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_91, 0, x_56); -lean_ctor_set(x_91, 1, x_90); -lean_ctor_set(x_91, 2, x_89); -x_92 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24; -lean_inc(x_74); -x_93 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_93, 0, x_74); -lean_ctor_set(x_93, 1, x_92); -x_94 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_95 = lean_array_push(x_94, x_93); -x_96 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__27; -x_97 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_97, 0, x_56); -lean_ctor_set(x_97, 1, x_96); -lean_ctor_set(x_97, 2, x_95); -x_98 = lean_array_push(x_53, x_68); -x_99 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_100 = lean_array_push(x_98, x_99); -x_101 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; -x_102 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_102, 0, x_56); -lean_ctor_set(x_102, 1, x_101); -lean_ctor_set(x_102, 2, x_100); -x_103 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28; -lean_inc(x_74); -x_104 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_104, 0, x_74); -lean_ctor_set(x_104, 1, x_103); -x_105 = l_Array_zip___rarg(x_24, x_23); -lean_dec(x_23); -lean_dec(x_24); -x_106 = lean_array_get_size(x_105); -x_107 = lean_usize_of_nat(x_106); -lean_dec(x_106); -x_108 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_109 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_110 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -x_111 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23; -lean_inc(x_74); -x_112 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23(x_108, x_53, x_74, x_86, x_109, x_99, x_110, x_111, x_94, x_107, x_14, x_105); -x_113 = l_Array_append___rarg(x_84, x_112); -x_114 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_114, 0, x_56); -lean_ctor_set(x_114, 1, x_86); -lean_ctor_set(x_114, 2, x_113); -x_115 = lean_array_push(x_94, x_114); -x_116 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__30; -x_117 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_117, 0, x_56); -lean_ctor_set(x_117, 1, x_116); -lean_ctor_set(x_117, 2, x_115); -x_118 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; -x_119 = lean_array_push(x_118, x_104); -lean_inc(x_119); -x_120 = lean_array_push(x_119, x_99); -x_121 = lean_array_push(x_120, x_117); -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_56); -lean_ctor_set(x_122, 1, x_86); -lean_ctor_set(x_122, 2, x_121); -x_123 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33; -lean_inc(x_74); -x_124 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_124, 0, x_74); -lean_ctor_set(x_124, 1, x_123); -x_125 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; -lean_inc(x_74); -x_126 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_126, 0, x_74); -lean_ctor_set(x_126, 1, x_125); -x_127 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49; -x_128 = lean_array_push(x_127, x_126); -x_129 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__48; -x_130 = lean_array_push(x_128, x_129); -x_131 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_131, 0, x_56); -lean_ctor_set(x_131, 1, x_86); -lean_ctor_set(x_131, 2, x_130); -x_132 = lean_array_push(x_53, x_124); -x_133 = lean_array_push(x_132, x_131); -x_134 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_134, 0, x_56); -lean_ctor_set(x_134, 1, x_86); -lean_ctor_set(x_134, 2, x_133); -x_135 = lean_array_push(x_94, x_134); -x_136 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__32; -x_137 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_137, 0, x_56); -lean_ctor_set(x_137, 1, x_136); -lean_ctor_set(x_137, 2, x_135); -x_138 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; -x_139 = lean_array_push(x_138, x_97); -x_140 = lean_array_push(x_139, x_102); -x_141 = lean_array_push(x_140, x_99); -x_142 = lean_array_push(x_141, x_99); -x_143 = lean_array_push(x_142, x_99); -x_144 = lean_array_push(x_143, x_122); -x_145 = lean_array_push(x_144, x_137); -x_146 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__25; -x_147 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_147, 0, x_56); -lean_ctor_set(x_147, 1, x_146); -lean_ctor_set(x_147, 2, x_145); -x_148 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50; -x_149 = lean_array_push(x_148, x_147); -x_150 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__37; -x_151 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_151, 0, x_56); -lean_ctor_set(x_151, 1, x_150); -lean_ctor_set(x_151, 2, x_149); -x_152 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205; -lean_inc(x_74); -x_153 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_153, 0, x_74); -lean_ctor_set(x_153, 1, x_152); -x_154 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; -lean_inc(x_74); -x_155 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_155, 0, x_74); -lean_ctor_set(x_155, 1, x_154); -x_156 = lean_array_push(x_53, x_63); -x_157 = lean_array_push(x_156, x_72); -x_158 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_158, 0, x_56); -lean_ctor_set(x_158, 1, x_86); -lean_ctor_set(x_158, 2, x_157); -x_159 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53; -x_160 = lean_array_push(x_159, x_158); -x_161 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_162 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_162, 0, x_56); -lean_ctor_set(x_162, 1, x_161); -lean_ctor_set(x_162, 2, x_160); -x_163 = lean_array_push(x_53, x_155); -x_164 = lean_array_push(x_163, x_162); -x_165 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95; -x_166 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_166, 0, x_56); -lean_ctor_set(x_166, 1, x_165); -lean_ctor_set(x_166, 2, x_164); -x_167 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__54; -x_168 = lean_array_push(x_167, x_166); -x_169 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__143; -x_170 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_170, 0, x_56); -lean_ctor_set(x_170, 1, x_169); -lean_ctor_set(x_170, 2, x_168); -x_171 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224; -lean_inc(x_76); -lean_inc(x_81); -x_172 = l_Lean_addMacroScope(x_81, x_171, x_76); -x_173 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223; -x_174 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__64; -lean_inc(x_74); -x_175 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_175, 0, x_74); -lean_ctor_set(x_175, 1, x_173); -lean_ctor_set(x_175, 2, x_172); -lean_ctor_set(x_175, 3, x_174); -x_176 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7; -lean_inc(x_76); -lean_inc(x_81); -x_177 = l_Lean_addMacroScope(x_81, x_176, x_76); -x_178 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6; -lean_inc(x_74); -x_179 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_179, 0, x_74); -lean_ctor_set(x_179, 1, x_178); -lean_ctor_set(x_179, 2, x_177); -lean_ctor_set(x_179, 3, x_47); -x_180 = lean_array_push(x_94, x_179); -x_181 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_181, 0, x_56); -lean_ctor_set(x_181, 1, x_86); -lean_ctor_set(x_181, 2, x_180); -x_182 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; -lean_inc(x_74); -x_183 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_183, 0, x_74); -lean_ctor_set(x_183, 1, x_182); -x_184 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67; -lean_inc(x_74); -x_185 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_185, 0, x_74); -lean_ctor_set(x_185, 1, x_184); -x_186 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__20; -lean_inc(x_74); -x_187 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_187, 0, x_74); -lean_ctor_set(x_187, 1, x_186); -x_188 = lean_array_get_size(x_31); -x_189 = lean_usize_of_nat(x_188); -lean_dec(x_188); -x_190 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__24(x_47, x_108, x_189, x_14, x_31); -x_191 = lean_array_get_size(x_190); -x_192 = lean_usize_of_nat(x_191); -lean_dec(x_191); -x_193 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25(x_192, x_14, x_190); -x_194 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__68; -x_195 = l_Lean_mkSepArray(x_193, x_194); -lean_dec(x_193); -x_196 = l_Array_append___rarg(x_84, x_195); -x_197 = lean_array_push(x_196, x_99); -x_198 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_198, 0, x_56); -lean_ctor_set(x_198, 1, x_86); -lean_ctor_set(x_198, 2, x_197); -x_199 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; -lean_inc(x_74); -x_200 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_200, 0, x_74); -lean_ctor_set(x_200, 1, x_199); -x_201 = lean_array_push(x_110, x_187); -x_202 = lean_array_push(x_201, x_99); -lean_inc(x_202); -x_203 = lean_array_push(x_202, x_198); -x_204 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69; -x_205 = lean_array_push(x_203, x_204); -x_206 = lean_array_push(x_205, x_99); -lean_inc(x_200); -x_207 = lean_array_push(x_206, x_200); -x_208 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__216; -x_209 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_209, 0, x_56); -lean_ctor_set(x_209, 1, x_208); -lean_ctor_set(x_209, 2, x_207); -x_210 = lean_array_push(x_94, x_209); -x_211 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_211, 0, x_56); -lean_ctor_set(x_211, 1, x_86); -lean_ctor_set(x_211, 2, x_210); -x_212 = lean_array_push(x_53, x_185); -lean_inc(x_212); -x_213 = lean_array_push(x_212, x_211); -x_214 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66; -x_215 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_215, 0, x_56); -lean_ctor_set(x_215, 1, x_214); -lean_ctor_set(x_215, 2, x_213); -x_216 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_217 = lean_array_push(x_216, x_175); -lean_inc(x_181); -x_218 = lean_array_push(x_217, x_181); -x_219 = lean_array_push(x_218, x_99); -lean_inc(x_183); -x_220 = lean_array_push(x_219, x_183); -x_221 = lean_array_push(x_220, x_215); -x_222 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; -x_223 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_223, 0, x_56); -lean_ctor_set(x_223, 1, x_222); -lean_ctor_set(x_223, 2, x_221); -x_224 = lean_array_push(x_94, x_223); -x_225 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60; -x_226 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_226, 0, x_56); -lean_ctor_set(x_226, 1, x_225); -lean_ctor_set(x_226, 2, x_224); -x_227 = lean_array_push(x_94, x_226); -x_228 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58; -x_229 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_229, 0, x_56); -lean_ctor_set(x_229, 1, x_228); -lean_ctor_set(x_229, 2, x_227); -x_230 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231; -x_231 = l_Lean_addMacroScope(x_81, x_230, x_76); -x_232 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230; -x_233 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__71; -x_234 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_234, 0, x_74); -lean_ctor_set(x_234, 1, x_232); -lean_ctor_set(x_234, 2, x_231); -lean_ctor_set(x_234, 3, x_233); -x_235 = lean_array_get_size(x_35); -x_236 = lean_usize_of_nat(x_235); -lean_dec(x_235); -x_237 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__26(x_47, x_108, x_236, x_14, x_35); -x_238 = lean_array_get_size(x_237); -x_239 = lean_usize_of_nat(x_238); -lean_dec(x_238); -x_240 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25(x_239, x_14, x_237); -x_241 = l_Lean_mkSepArray(x_240, x_194); -lean_dec(x_240); -x_242 = l_Array_append___rarg(x_84, x_241); -x_243 = lean_array_push(x_242, x_99); -x_244 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_244, 0, x_56); -lean_ctor_set(x_244, 1, x_86); -lean_ctor_set(x_244, 2, x_243); -x_245 = lean_array_push(x_202, x_244); -x_246 = lean_array_push(x_245, x_204); -x_247 = lean_array_push(x_246, x_99); -x_248 = lean_array_push(x_247, x_200); -x_249 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_249, 0, x_56); -lean_ctor_set(x_249, 1, x_208); -lean_ctor_set(x_249, 2, x_248); -x_250 = lean_array_push(x_94, x_249); -x_251 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_251, 0, x_56); -lean_ctor_set(x_251, 1, x_86); -lean_ctor_set(x_251, 2, x_250); -x_252 = lean_array_push(x_212, x_251); -x_253 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_253, 0, x_56); -lean_ctor_set(x_253, 1, x_214); -lean_ctor_set(x_253, 2, x_252); -x_254 = lean_array_push(x_216, x_234); -x_255 = lean_array_push(x_254, x_181); -x_256 = lean_array_push(x_255, x_99); -x_257 = lean_array_push(x_256, x_183); -x_258 = lean_array_push(x_257, x_253); -x_259 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_259, 0, x_56); -lean_ctor_set(x_259, 1, x_222); -lean_ctor_set(x_259, 2, x_258); -x_260 = lean_array_push(x_94, x_259); -x_261 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_261, 0, x_56); -lean_ctor_set(x_261, 1, x_225); -lean_ctor_set(x_261, 2, x_260); -x_262 = lean_array_push(x_94, x_261); -x_263 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_263, 0, x_56); -lean_ctor_set(x_263, 1, x_228); -lean_ctor_set(x_263, 2, x_262); -x_264 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_265 = lean_array_push(x_264, x_229); -x_266 = lean_array_push(x_265, x_99); -x_267 = lean_array_push(x_266, x_263); -x_268 = lean_array_push(x_267, x_99); -x_269 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_269, 0, x_56); -lean_ctor_set(x_269, 1, x_86); -lean_ctor_set(x_269, 2, x_268); -x_270 = lean_array_push(x_119, x_269); -x_271 = lean_array_push(x_270, x_99); -x_272 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__56; -x_273 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_273, 0, x_56); -lean_ctor_set(x_273, 1, x_272); -lean_ctor_set(x_273, 2, x_271); -x_274 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72; -x_275 = lean_array_push(x_274, x_153); -x_276 = lean_array_push(x_275, x_99); -x_277 = lean_array_push(x_276, x_99); -x_278 = lean_array_push(x_277, x_170); -x_279 = lean_array_push(x_278, x_273); -x_280 = lean_array_push(x_279, x_99); -x_281 = lean_array_push(x_280, x_99); -x_282 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206; -x_283 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_283, 0, x_56); -lean_ctor_set(x_283, 1, x_282); -lean_ctor_set(x_283, 2, x_281); -x_284 = lean_array_push(x_148, x_283); -x_285 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_285, 0, x_56); -lean_ctor_set(x_285, 1, x_150); -lean_ctor_set(x_285, 2, x_284); -x_286 = lean_array_push(x_118, x_91); -x_287 = lean_array_push(x_286, x_151); -x_288 = lean_array_push(x_287, x_285); -x_289 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_289, 0, x_56); -lean_ctor_set(x_289, 1, x_86); -lean_ctor_set(x_289, 2, x_288); -lean_ctor_set(x_77, 0, x_289); -return x_77; -} -else -{ -lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; size_t x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; size_t x_401; lean_object* x_402; lean_object* x_403; size_t x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; size_t x_448; lean_object* x_449; lean_object* x_450; size_t x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; -x_290 = lean_ctor_get(x_77, 0); -x_291 = lean_ctor_get(x_77, 1); -lean_inc(x_291); -lean_inc(x_290); -lean_dec(x_77); -x_292 = lean_ctor_get(x_290, 0); -lean_inc(x_292); -lean_dec(x_290); -x_293 = lean_environment_main_module(x_292); -x_294 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; -lean_inc(x_74); -x_295 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_295, 0, x_74); -lean_ctor_set(x_295, 1, x_294); -x_296 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_297 = l_Array_append___rarg(x_296, x_22); -x_298 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_299 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_299, 0, x_56); -lean_ctor_set(x_299, 1, x_298); -lean_ctor_set(x_299, 2, x_297); -x_300 = lean_array_push(x_53, x_295); -x_301 = lean_array_push(x_300, x_299); -x_302 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; -x_303 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_303, 0, x_56); -lean_ctor_set(x_303, 1, x_302); -lean_ctor_set(x_303, 2, x_301); -x_304 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24; -lean_inc(x_74); -x_305 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_305, 0, x_74); -lean_ctor_set(x_305, 1, x_304); -x_306 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_307 = lean_array_push(x_306, x_305); -x_308 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__27; -x_309 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_309, 0, x_56); -lean_ctor_set(x_309, 1, x_308); -lean_ctor_set(x_309, 2, x_307); -x_310 = lean_array_push(x_53, x_68); -x_311 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_312 = lean_array_push(x_310, x_311); -x_313 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; -x_314 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_314, 0, x_56); -lean_ctor_set(x_314, 1, x_313); -lean_ctor_set(x_314, 2, x_312); -x_315 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28; -lean_inc(x_74); -x_316 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_316, 0, x_74); -lean_ctor_set(x_316, 1, x_315); -x_317 = l_Array_zip___rarg(x_24, x_23); -lean_dec(x_23); -lean_dec(x_24); -x_318 = lean_array_get_size(x_317); -x_319 = lean_usize_of_nat(x_318); -lean_dec(x_318); -x_320 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_321 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_322 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -x_323 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23; -lean_inc(x_74); -x_324 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23(x_320, x_53, x_74, x_298, x_321, x_311, x_322, x_323, x_306, x_319, x_14, x_317); -x_325 = l_Array_append___rarg(x_296, x_324); -x_326 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_326, 0, x_56); -lean_ctor_set(x_326, 1, x_298); -lean_ctor_set(x_326, 2, x_325); -x_327 = lean_array_push(x_306, x_326); -x_328 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__30; -x_329 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_329, 0, x_56); -lean_ctor_set(x_329, 1, x_328); -lean_ctor_set(x_329, 2, x_327); -x_330 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; -x_331 = lean_array_push(x_330, x_316); -lean_inc(x_331); -x_332 = lean_array_push(x_331, x_311); -x_333 = lean_array_push(x_332, x_329); -x_334 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_334, 0, x_56); -lean_ctor_set(x_334, 1, x_298); -lean_ctor_set(x_334, 2, x_333); -x_335 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33; -lean_inc(x_74); -x_336 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_336, 0, x_74); -lean_ctor_set(x_336, 1, x_335); -x_337 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; -lean_inc(x_74); -x_338 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_338, 0, x_74); -lean_ctor_set(x_338, 1, x_337); -x_339 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49; -x_340 = lean_array_push(x_339, x_338); -x_341 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__48; -x_342 = lean_array_push(x_340, x_341); -x_343 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_343, 0, x_56); -lean_ctor_set(x_343, 1, x_298); -lean_ctor_set(x_343, 2, x_342); -x_344 = lean_array_push(x_53, x_336); -x_345 = lean_array_push(x_344, x_343); -x_346 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_346, 0, x_56); -lean_ctor_set(x_346, 1, x_298); -lean_ctor_set(x_346, 2, x_345); -x_347 = lean_array_push(x_306, x_346); -x_348 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__32; -x_349 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_349, 0, x_56); -lean_ctor_set(x_349, 1, x_348); -lean_ctor_set(x_349, 2, x_347); -x_350 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; -x_351 = lean_array_push(x_350, x_309); -x_352 = lean_array_push(x_351, x_314); -x_353 = lean_array_push(x_352, x_311); -x_354 = lean_array_push(x_353, x_311); -x_355 = lean_array_push(x_354, x_311); -x_356 = lean_array_push(x_355, x_334); -x_357 = lean_array_push(x_356, x_349); -x_358 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__25; -x_359 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_359, 0, x_56); -lean_ctor_set(x_359, 1, x_358); -lean_ctor_set(x_359, 2, x_357); -x_360 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50; -x_361 = lean_array_push(x_360, x_359); -x_362 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__37; -x_363 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_363, 0, x_56); -lean_ctor_set(x_363, 1, x_362); -lean_ctor_set(x_363, 2, x_361); -x_364 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205; -lean_inc(x_74); -x_365 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_365, 0, x_74); -lean_ctor_set(x_365, 1, x_364); -x_366 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; -lean_inc(x_74); -x_367 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_367, 0, x_74); -lean_ctor_set(x_367, 1, x_366); -x_368 = lean_array_push(x_53, x_63); -x_369 = lean_array_push(x_368, x_72); -x_370 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_370, 0, x_56); -lean_ctor_set(x_370, 1, x_298); -lean_ctor_set(x_370, 2, x_369); -x_371 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53; -x_372 = lean_array_push(x_371, x_370); -x_373 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_374 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_374, 0, x_56); -lean_ctor_set(x_374, 1, x_373); -lean_ctor_set(x_374, 2, x_372); -x_375 = lean_array_push(x_53, x_367); -x_376 = lean_array_push(x_375, x_374); -x_377 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95; -x_378 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_378, 0, x_56); -lean_ctor_set(x_378, 1, x_377); -lean_ctor_set(x_378, 2, x_376); -x_379 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__54; -x_380 = lean_array_push(x_379, x_378); -x_381 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__143; -x_382 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_382, 0, x_56); -lean_ctor_set(x_382, 1, x_381); -lean_ctor_set(x_382, 2, x_380); -x_383 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224; -lean_inc(x_76); -lean_inc(x_293); -x_384 = l_Lean_addMacroScope(x_293, x_383, x_76); -x_385 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223; -x_386 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__64; -lean_inc(x_74); -x_387 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_387, 0, x_74); -lean_ctor_set(x_387, 1, x_385); -lean_ctor_set(x_387, 2, x_384); -lean_ctor_set(x_387, 3, x_386); -x_388 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7; -lean_inc(x_76); -lean_inc(x_293); -x_389 = l_Lean_addMacroScope(x_293, x_388, x_76); -x_390 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6; -lean_inc(x_74); -x_391 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_391, 0, x_74); -lean_ctor_set(x_391, 1, x_390); -lean_ctor_set(x_391, 2, x_389); -lean_ctor_set(x_391, 3, x_47); -x_392 = lean_array_push(x_306, x_391); -x_393 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_393, 0, x_56); -lean_ctor_set(x_393, 1, x_298); -lean_ctor_set(x_393, 2, x_392); -x_394 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; -lean_inc(x_74); -x_395 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_395, 0, x_74); -lean_ctor_set(x_395, 1, x_394); -x_396 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67; -lean_inc(x_74); -x_397 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_397, 0, x_74); -lean_ctor_set(x_397, 1, x_396); -x_398 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__20; -lean_inc(x_74); -x_399 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_399, 0, x_74); -lean_ctor_set(x_399, 1, x_398); -x_400 = lean_array_get_size(x_31); -x_401 = lean_usize_of_nat(x_400); -lean_dec(x_400); -x_402 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__24(x_47, x_320, x_401, x_14, x_31); -x_403 = lean_array_get_size(x_402); -x_404 = lean_usize_of_nat(x_403); -lean_dec(x_403); -x_405 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25(x_404, x_14, x_402); -x_406 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__68; -x_407 = l_Lean_mkSepArray(x_405, x_406); -lean_dec(x_405); -x_408 = l_Array_append___rarg(x_296, x_407); -x_409 = lean_array_push(x_408, x_311); -x_410 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_410, 0, x_56); -lean_ctor_set(x_410, 1, x_298); -lean_ctor_set(x_410, 2, x_409); -x_411 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; -lean_inc(x_74); -x_412 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_412, 0, x_74); -lean_ctor_set(x_412, 1, x_411); -x_413 = lean_array_push(x_322, x_399); -x_414 = lean_array_push(x_413, x_311); -lean_inc(x_414); -x_415 = lean_array_push(x_414, x_410); -x_416 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69; -x_417 = lean_array_push(x_415, x_416); -x_418 = lean_array_push(x_417, x_311); -lean_inc(x_412); -x_419 = lean_array_push(x_418, x_412); -x_420 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__216; -x_421 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_421, 0, x_56); -lean_ctor_set(x_421, 1, x_420); -lean_ctor_set(x_421, 2, x_419); -x_422 = lean_array_push(x_306, x_421); -x_423 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_423, 0, x_56); -lean_ctor_set(x_423, 1, x_298); -lean_ctor_set(x_423, 2, x_422); -x_424 = lean_array_push(x_53, x_397); -lean_inc(x_424); -x_425 = lean_array_push(x_424, x_423); -x_426 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66; -x_427 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_427, 0, x_56); -lean_ctor_set(x_427, 1, x_426); -lean_ctor_set(x_427, 2, x_425); -x_428 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_429 = lean_array_push(x_428, x_387); -lean_inc(x_393); -x_430 = lean_array_push(x_429, x_393); -x_431 = lean_array_push(x_430, x_311); -lean_inc(x_395); -x_432 = lean_array_push(x_431, x_395); -x_433 = lean_array_push(x_432, x_427); -x_434 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; -x_435 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_435, 0, x_56); -lean_ctor_set(x_435, 1, x_434); -lean_ctor_set(x_435, 2, x_433); -x_436 = lean_array_push(x_306, x_435); -x_437 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60; -x_438 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_438, 0, x_56); -lean_ctor_set(x_438, 1, x_437); -lean_ctor_set(x_438, 2, x_436); -x_439 = lean_array_push(x_306, x_438); -x_440 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58; -x_441 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_441, 0, x_56); -lean_ctor_set(x_441, 1, x_440); -lean_ctor_set(x_441, 2, x_439); -x_442 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231; -x_443 = l_Lean_addMacroScope(x_293, x_442, x_76); -x_444 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230; -x_445 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__71; -x_446 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_446, 0, x_74); -lean_ctor_set(x_446, 1, x_444); -lean_ctor_set(x_446, 2, x_443); -lean_ctor_set(x_446, 3, x_445); -x_447 = lean_array_get_size(x_35); -x_448 = lean_usize_of_nat(x_447); -lean_dec(x_447); -x_449 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__26(x_47, x_320, x_448, x_14, x_35); -x_450 = lean_array_get_size(x_449); -x_451 = lean_usize_of_nat(x_450); -lean_dec(x_450); -x_452 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25(x_451, x_14, x_449); -x_453 = l_Lean_mkSepArray(x_452, x_406); -lean_dec(x_452); -x_454 = l_Array_append___rarg(x_296, x_453); -x_455 = lean_array_push(x_454, x_311); -x_456 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_456, 0, x_56); -lean_ctor_set(x_456, 1, x_298); -lean_ctor_set(x_456, 2, x_455); -x_457 = lean_array_push(x_414, x_456); -x_458 = lean_array_push(x_457, x_416); -x_459 = lean_array_push(x_458, x_311); -x_460 = lean_array_push(x_459, x_412); -x_461 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_461, 0, x_56); -lean_ctor_set(x_461, 1, x_420); -lean_ctor_set(x_461, 2, x_460); -x_462 = lean_array_push(x_306, x_461); -x_463 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_463, 0, x_56); -lean_ctor_set(x_463, 1, x_298); -lean_ctor_set(x_463, 2, x_462); -x_464 = lean_array_push(x_424, x_463); -x_465 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_465, 0, x_56); -lean_ctor_set(x_465, 1, x_426); -lean_ctor_set(x_465, 2, x_464); -x_466 = lean_array_push(x_428, x_446); -x_467 = lean_array_push(x_466, x_393); -x_468 = lean_array_push(x_467, x_311); -x_469 = lean_array_push(x_468, x_395); -x_470 = lean_array_push(x_469, x_465); -x_471 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_471, 0, x_56); -lean_ctor_set(x_471, 1, x_434); -lean_ctor_set(x_471, 2, x_470); -x_472 = lean_array_push(x_306, x_471); -x_473 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_473, 0, x_56); -lean_ctor_set(x_473, 1, x_437); -lean_ctor_set(x_473, 2, x_472); -x_474 = lean_array_push(x_306, x_473); -x_475 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_475, 0, x_56); -lean_ctor_set(x_475, 1, x_440); -lean_ctor_set(x_475, 2, x_474); -x_476 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_477 = lean_array_push(x_476, x_441); -x_478 = lean_array_push(x_477, x_311); -x_479 = lean_array_push(x_478, x_475); -x_480 = lean_array_push(x_479, x_311); -x_481 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_481, 0, x_56); -lean_ctor_set(x_481, 1, x_298); -lean_ctor_set(x_481, 2, x_480); -x_482 = lean_array_push(x_331, x_481); -x_483 = lean_array_push(x_482, x_311); -x_484 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__56; -x_485 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_485, 0, x_56); -lean_ctor_set(x_485, 1, x_484); -lean_ctor_set(x_485, 2, x_483); -x_486 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72; -x_487 = lean_array_push(x_486, x_365); -x_488 = lean_array_push(x_487, x_311); -x_489 = lean_array_push(x_488, x_311); -x_490 = lean_array_push(x_489, x_382); -x_491 = lean_array_push(x_490, x_485); -x_492 = lean_array_push(x_491, x_311); -x_493 = lean_array_push(x_492, x_311); -x_494 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206; -x_495 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_495, 0, x_56); -lean_ctor_set(x_495, 1, x_494); -lean_ctor_set(x_495, 2, x_493); -x_496 = lean_array_push(x_360, x_495); -x_497 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_497, 0, x_56); -lean_ctor_set(x_497, 1, x_362); -lean_ctor_set(x_497, 2, x_496); -x_498 = lean_array_push(x_330, x_303); -x_499 = lean_array_push(x_498, x_363); -x_500 = lean_array_push(x_499, x_497); -x_501 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_501, 0, x_56); -lean_ctor_set(x_501, 1, x_298); -lean_ctor_set(x_501, 2, x_500); -x_502 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_502, 0, x_501); -lean_ctor_set(x_502, 1, x_291); -return x_502; -} -} -else -{ -uint8_t x_503; -lean_dec(x_35); -lean_dec(x_31); -lean_dec(x_25); -lean_dec(x_24); -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_3); -x_503 = !lean_is_exclusive(x_39); -if (x_503 == 0) -{ -return x_39; -} -else -{ -lean_object* x_504; lean_object* x_505; lean_object* x_506; -x_504 = lean_ctor_get(x_39, 0); -x_505 = lean_ctor_get(x_39, 1); -lean_inc(x_505); -lean_inc(x_504); -lean_dec(x_39); -x_506 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_506, 0, x_504); -lean_ctor_set(x_506, 1, x_505); -return x_506; -} -} -} -else -{ -uint8_t x_507; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -x_507 = !lean_is_exclusive(x_16); -if (x_507 == 0) -{ -return x_16; -} -else -{ -lean_object* x_508; lean_object* x_509; lean_object* x_510; -x_508 = lean_ctor_get(x_16, 0); -x_509 = lean_ctor_get(x_16, 1); -lean_inc(x_509); -lean_inc(x_508); -lean_dec(x_16); -x_510 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_510, 0, x_508); -lean_ctor_set(x_510, 1, x_509); -return x_510; -} -} -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Elab", 4); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Deriving", 8); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__2; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__3; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__4; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("for structure ", 14); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__6; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" with params ", 13); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__8; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_11 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__5; -x_35 = lean_st_ref_get(x_9, x_10); -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_36, 3); -lean_inc(x_37); -lean_dec(x_36); -x_38 = lean_ctor_get_uint8(x_37, sizeof(void*)*1); -lean_dec(x_37); -if (x_38 == 0) -{ -lean_object* x_39; uint8_t x_40; -x_39 = lean_ctor_get(x_35, 1); -lean_inc(x_39); -lean_dec(x_35); -x_40 = 0; -x_12 = x_40; -x_13 = x_39; -goto block_34; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; -x_41 = lean_ctor_get(x_35, 1); -lean_inc(x_41); -lean_dec(x_35); -x_42 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_41); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_unbox(x_43); -lean_dec(x_43); -x_12 = x_45; -x_13 = x_44; -goto block_34; -} -block_34: -{ -if (x_12 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_box(0); -x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(x_3, x_1, x_2, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -lean_dec(x_3); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_16 = lean_ctor_get(x_2, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -lean_dec(x_16); -x_18 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_18, 0, x_17); -x_19 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__7; -x_20 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -x_21 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9; -x_22 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -lean_inc(x_1); -x_23 = lean_array_to_list(lean_box(0), x_1); -x_24 = lean_box(0); -x_25 = l_List_mapTRAux___at_Lean_MessageData_instCoeListExprMessageData___spec__1(x_23, x_24); -x_26 = l_Lean_MessageData_ofList(x_25); -lean_dec(x_25); -x_27 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_27, 0, x_22); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6; -x_29 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_11, x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); -lean_inc(x_32); -lean_dec(x_30); -x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(x_3, x_1, x_2, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_32); -lean_dec(x_31); -lean_dec(x_3); -return x_33; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; -lean_inc(x_1); -lean_inc(x_2); -x_10 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2), 10, 2); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_1); -x_11 = l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__27___rarg(x_1, x_2, x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; lean_object* x_5; -x_4 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_5 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(x_1, x_4, x_3); -lean_dec(x_3); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -size_t x_7; lean_object* x_8; -x_7 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_8 = l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(x_7, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_3); -lean_dec(x_2); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_7 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_8 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_1, x_6, x_7, x_4, x_5); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__13(x_1, x_2, x_5, x_6); -lean_dec(x_2); -x_8 = lean_box(x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Array_contains___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Array_contains___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12(x_1, x_2); -x_4 = lean_box(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__15(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_1); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__14(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_1); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -lean_object* x_16; -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___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); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_16; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -lean_object* x_16; -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_10); -lean_dec(x_9); -return x_16; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -lean_object* x_16; -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_8); -return x_16; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_1); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__19(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_12 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__20(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -size_t x_5; size_t x_6; lean_object* x_7; -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__21(x_1, x_5, x_6, x_4); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -size_t x_5; size_t x_6; lean_object* x_7; -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__22(x_1, x_5, x_6, x_4); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_10); -lean_dec(x_10); -x_14 = lean_unbox_usize(x_11); -lean_dec(x_11); -x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13, x_14, x_12); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__24(x_1, x_2, x_6, x_7, x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; size_t x_5; lean_object* x_6; -x_4 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__25(x_4, x_5, x_3); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__26(x_1, x_2, x_6, x_7, x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__29(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_2); -return x_15; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_4); -lean_dec(x_1); -return x_12; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encArgTypes___default() { -_start: -{ -lean_object* x_1; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__3; -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_uniqEncArgTypes___default() { -_start: -{ -lean_object* x_1; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_binders___default() { -_start: -{ -lean_object* x_1; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_ctors___default() { -_start: -{ -lean_object* x_1; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encodes___default() { -_start: -{ -lean_object* x_1; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_decodes___default() { -_start: -{ -lean_object* x_1; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -return x_1; -} -} -static lean_object* _init_l_Lean_Server_RpcEncoding_instInhabitedCtorState___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__3; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_3 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -lean_ctor_set(x_3, 2, x_2); -lean_ctor_set(x_3, 3, x_2); -lean_ctor_set(x_3, 4, x_2); -lean_ctor_set(x_3, 5, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Server_RpcEncoding_instInhabitedCtorState() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Server_RpcEncoding_instInhabitedCtorState___closed__1; -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__9; -x_2 = lean_unsigned_to_nat(0u); -x_3 = l_Lean_Parser_categoryParser(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__1; -x_2 = l_Lean_Parser_Term_matchAlt(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF() { -_start: -{ -lean_object* x_1; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__2; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; -x_11 = lean_usize_dec_lt(x_2, x_1); -if (x_11 == 0) -{ -lean_object* x_12; -lean_dec(x_6); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_3); -lean_ctor_set(x_12, 1, x_10); -return x_12; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_array_uget(x_3, x_2); -x_14 = lean_unsigned_to_nat(0u); -x_15 = lean_array_uset(x_3, x_2, x_14); -lean_inc(x_6); -x_16 = l_Lean_Meta_getFVarLocalDecl(x_13, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Lean_LocalDecl_fvarId(x_17); -lean_dec(x_17); -x_20 = 1; -x_21 = lean_usize_add(x_2, x_20); -x_22 = lean_array_uset(x_15, x_2, x_19); -x_2 = x_21; -x_3 = x_22; -x_10 = x_18; -goto _start; -} -else -{ -uint8_t x_24; -lean_dec(x_15); -lean_dec(x_6); -x_24 = !lean_is_exclusive(x_16); -if (x_24 == 0) -{ -return x_16; -} -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_16, 0); -x_26 = lean_ctor_get(x_16, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_16); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_get_size(x_1); -x_7 = lean_nat_dec_lt(x_4, x_6); -lean_dec(x_6); -if (x_7 == 0) -{ -lean_object* x_8; -lean_dec(x_4); -x_8 = lean_box(0); -return x_8; -} -else -{ -lean_object* x_9; uint8_t x_10; -x_9 = lean_array_fget(x_1, x_4); -x_10 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_5, x_9); -lean_dec(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_nat_add(x_4, x_11); -lean_dec(x_4); -x_3 = lean_box(0); -x_4 = x_12; -goto _start; -} -else -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_array_fget(x_2, x_4); -lean_dec(x_4); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; -} -} -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5(lean_object* x_1, size_t x_2, lean_object* x_3) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_4; size_t x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = 5; -x_6 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2; -x_7 = lean_usize_land(x_2, x_6); -x_8 = lean_usize_to_nat(x_7); -x_9 = lean_box(2); -x_10 = lean_array_get(x_9, x_4, x_8); -lean_dec(x_8); -lean_dec(x_4); -switch (lean_obj_tag(x_10)) { -case 0: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_3, x_11); -lean_dec(x_11); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_12); -x_14 = lean_box(0); -return x_14; -} -else -{ -lean_object* x_15; -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_12); -return x_15; -} -} -case 1: -{ -lean_object* x_16; size_t x_17; -x_16 = lean_ctor_get(x_10, 0); -lean_inc(x_16); -lean_dec(x_10); -x_17 = lean_usize_shift_right(x_2, x_5); -x_1 = x_16; -x_2 = x_17; -goto _start; -} -default: -{ -lean_object* x_19; -x_19 = lean_box(0); -return x_19; -} -} -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_1, 1); -lean_inc(x_21); -lean_dec(x_1); -x_22 = lean_unsigned_to_nat(0u); -x_23 = l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6(x_20, x_21, lean_box(0), x_22, x_3); -lean_dec(x_21); -lean_dec(x_20); -return x_23; -} -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; uint64_t x_4; size_t x_5; lean_object* x_6; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -lean_dec(x_1); -x_4 = l_Lean_Meta_DiscrTree_Key_hash(x_2); -x_5 = lean_uint64_to_usize(x_4); -x_6 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5(x_3, x_5, x_2); -lean_dec(x_2); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; uint8_t x_8; -x_7 = lean_array_get_size(x_2); -x_8 = lean_nat_dec_lt(x_5, x_7); -lean_dec(x_7); -if (x_8 == 0) -{ -lean_dec(x_5); -return x_6; -} -else -{ -lean_object* x_9; lean_object* x_10; uint64_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_9 = lean_array_fget(x_2, x_5); -x_10 = lean_array_fget(x_3, x_5); -x_11 = l_Lean_Meta_DiscrTree_Key_hash(x_9); -x_12 = lean_uint64_to_usize(x_11); -x_13 = 1; -x_14 = lean_usize_sub(x_1, x_13); -x_15 = 5; -x_16 = lean_usize_mul(x_15, x_14); -x_17 = lean_usize_shift_right(x_12, x_16); -x_18 = lean_unsigned_to_nat(1u); -x_19 = lean_nat_add(x_5, x_18); -lean_dec(x_5); -x_20 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_6, x_17, x_1, x_9, x_10); -x_4 = lean_box(0); -x_5 = x_19; -x_6 = x_20; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); -x_7 = lean_array_get_size(x_5); -x_8 = lean_nat_dec_lt(x_2, x_7); -lean_dec(x_7); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_2); -x_9 = !lean_is_exclusive(x_1); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_1, 1); -lean_dec(x_10); -x_11 = lean_ctor_get(x_1, 0); -lean_dec(x_11); -x_12 = lean_array_push(x_5, x_3); -x_13 = lean_array_push(x_6, x_4); -lean_ctor_set(x_1, 1, x_13); -lean_ctor_set(x_1, 0, x_12); -return x_1; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_14 = lean_array_push(x_5, x_3); -x_15 = lean_array_push(x_6, x_4); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -return x_16; -} -} -else -{ -lean_object* x_17; uint8_t x_18; -x_17 = lean_array_fget(x_5, x_2); -x_18 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_3, x_17); -lean_dec(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_6); -lean_dec(x_5); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_add(x_2, x_19); -lean_dec(x_2); -x_2 = x_20; -goto _start; -} -else -{ -uint8_t x_22; -x_22 = !lean_is_exclusive(x_1); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_1, 1); -lean_dec(x_23); -x_24 = lean_ctor_get(x_1, 0); -lean_dec(x_24); -x_25 = lean_array_fset(x_5, x_2, x_3); -x_26 = lean_array_fset(x_6, x_2, x_4); -lean_dec(x_2); -lean_ctor_set(x_1, 1, x_26); -lean_ctor_set(x_1, 0, x_25); -return x_1; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_1); -x_27 = lean_array_fset(x_5, x_2, x_3); -x_28 = lean_array_fset(x_6, x_2, x_4); -lean_dec(x_2); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -uint8_t x_6; -x_6 = !lean_is_exclusive(x_1); -if (x_6 == 0) -{ -lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_7 = lean_ctor_get(x_1, 0); -x_8 = 1; -x_9 = 5; -x_10 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2; -x_11 = lean_usize_land(x_2, x_10); -x_12 = lean_usize_to_nat(x_11); -x_13 = lean_array_get_size(x_7); -x_14 = lean_nat_dec_lt(x_12, x_13); -lean_dec(x_13); -if (x_14 == 0) -{ -lean_dec(x_12); -lean_dec(x_5); -lean_dec(x_4); -return x_1; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_array_fget(x_7, x_12); -x_16 = lean_box(0); -x_17 = lean_array_fset(x_7, x_12, x_16); -switch (lean_obj_tag(x_15)) { -case 0: -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_15); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_15, 0); -x_20 = lean_ctor_get(x_15, 1); -x_21 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_4, x_19); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_free_object(x_15); -x_22 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_19, x_20, x_4, x_5); -x_23 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_23, 0, x_22); -x_24 = lean_array_fset(x_17, x_12, x_23); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_24); -return x_1; -} -else -{ -lean_object* x_25; -lean_dec(x_20); -lean_dec(x_19); -lean_ctor_set(x_15, 1, x_5); -lean_ctor_set(x_15, 0, x_4); -x_25 = lean_array_fset(x_17, x_12, x_15); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_25); -return x_1; -} -} -else -{ -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = lean_ctor_get(x_15, 0); -x_27 = lean_ctor_get(x_15, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_15); -x_28 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_4, x_26); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_26, x_27, x_4, x_5); -x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_29); -x_31 = lean_array_fset(x_17, x_12, x_30); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_31); -return x_1; -} -else -{ -lean_object* x_32; lean_object* x_33; -lean_dec(x_27); -lean_dec(x_26); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_4); -lean_ctor_set(x_32, 1, x_5); -x_33 = lean_array_fset(x_17, x_12, x_32); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_33); -return x_1; -} -} -} -case 1: -{ -uint8_t x_34; -x_34 = !lean_is_exclusive(x_15); -if (x_34 == 0) -{ -lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_39; -x_35 = lean_ctor_get(x_15, 0); -x_36 = lean_usize_shift_right(x_2, x_9); -x_37 = lean_usize_add(x_3, x_8); -x_38 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_35, x_36, x_37, x_4, x_5); -lean_ctor_set(x_15, 0, x_38); -x_39 = lean_array_fset(x_17, x_12, x_15); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_39); -return x_1; -} -else -{ -lean_object* x_40; size_t x_41; size_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_40 = lean_ctor_get(x_15, 0); -lean_inc(x_40); -lean_dec(x_15); -x_41 = lean_usize_shift_right(x_2, x_9); -x_42 = lean_usize_add(x_3, x_8); -x_43 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_40, x_41, x_42, x_4, x_5); -x_44 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_44, 0, x_43); -x_45 = lean_array_fset(x_17, x_12, x_44); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_45); -return x_1; -} -} -default: -{ -lean_object* x_46; lean_object* x_47; -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_4); -lean_ctor_set(x_46, 1, x_5); -x_47 = lean_array_fset(x_17, x_12, x_46); -lean_dec(x_12); -lean_ctor_set(x_1, 0, x_47); -return x_1; -} -} -} -} -else -{ -lean_object* x_48; size_t x_49; size_t x_50; size_t x_51; size_t x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_48 = lean_ctor_get(x_1, 0); -lean_inc(x_48); -lean_dec(x_1); -x_49 = 1; -x_50 = 5; -x_51 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2; -x_52 = lean_usize_land(x_2, x_51); -x_53 = lean_usize_to_nat(x_52); -x_54 = lean_array_get_size(x_48); -x_55 = lean_nat_dec_lt(x_53, x_54); -lean_dec(x_54); -if (x_55 == 0) -{ -lean_object* x_56; -lean_dec(x_53); -lean_dec(x_5); -lean_dec(x_4); -x_56 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_56, 0, x_48); -return x_56; -} -else -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_array_fget(x_48, x_53); -x_58 = lean_box(0); -x_59 = lean_array_fset(x_48, x_53, x_58); -switch (lean_obj_tag(x_57)) { -case 0: -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; -x_60 = lean_ctor_get(x_57, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_57, 1); -lean_inc(x_61); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_62 = x_57; -} else { - lean_dec_ref(x_57); - x_62 = lean_box(0); -} -x_63 = l___private_Lean_Meta_DiscrTreeTypes_0__Lean_Meta_DiscrTree_beqKey____x40_Lean_Meta_DiscrTreeTypes___hyg_89_(x_4, x_60); -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -lean_dec(x_62); -x_64 = l_Std_PersistentHashMap_mkCollisionNode___rarg(x_60, x_61, x_4, x_5); -x_65 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_65, 0, x_64); -x_66 = lean_array_fset(x_59, x_53, x_65); -lean_dec(x_53); -x_67 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_67, 0, x_66); -return x_67; -} -else -{ -lean_object* x_68; lean_object* x_69; lean_object* x_70; -lean_dec(x_61); -lean_dec(x_60); -if (lean_is_scalar(x_62)) { - x_68 = lean_alloc_ctor(0, 2, 0); -} else { - x_68 = x_62; -} -lean_ctor_set(x_68, 0, x_4); -lean_ctor_set(x_68, 1, x_5); -x_69 = lean_array_fset(x_59, x_53, x_68); -lean_dec(x_53); -x_70 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_70, 0, x_69); -return x_70; -} -} -case 1: -{ -lean_object* x_71; lean_object* x_72; size_t x_73; size_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_71 = lean_ctor_get(x_57, 0); -lean_inc(x_71); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - x_72 = x_57; -} else { - lean_dec_ref(x_57); - x_72 = lean_box(0); -} -x_73 = lean_usize_shift_right(x_2, x_50); -x_74 = lean_usize_add(x_3, x_49); -x_75 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_71, x_73, x_74, x_4, x_5); -if (lean_is_scalar(x_72)) { - x_76 = lean_alloc_ctor(1, 1, 0); -} else { - x_76 = x_72; -} -lean_ctor_set(x_76, 0, x_75); -x_77 = lean_array_fset(x_59, x_53, x_76); -lean_dec(x_53); -x_78 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_78, 0, x_77); -return x_78; -} -default: -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_4); -lean_ctor_set(x_79, 1, x_5); -x_80 = lean_array_fset(x_59, x_53, x_79); -lean_dec(x_53); -x_81 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_81, 0, x_80); -return x_81; -} -} -} -} -} -else -{ -uint8_t x_82; -x_82 = !lean_is_exclusive(x_1); -if (x_82 == 0) -{ -lean_object* x_83; lean_object* x_84; size_t x_85; uint8_t x_86; -x_83 = lean_unsigned_to_nat(0u); -x_84 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10(x_1, x_83, x_4, x_5); -x_85 = 7; -x_86 = lean_usize_dec_le(x_85, x_3); -if (x_86 == 0) -{ -lean_object* x_87; lean_object* x_88; uint8_t x_89; -x_87 = l_Std_PersistentHashMap_getCollisionNodeSize___rarg(x_84); -x_88 = lean_unsigned_to_nat(4u); -x_89 = lean_nat_dec_lt(x_87, x_88); -lean_dec(x_87); -if (x_89 == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_90 = lean_ctor_get(x_84, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_84, 1); -lean_inc(x_91); -lean_dec(x_84); -x_92 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1; -x_93 = l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9(x_3, x_90, x_91, lean_box(0), x_83, x_92); -lean_dec(x_91); -lean_dec(x_90); -return x_93; -} -else -{ -return x_84; -} -} -else -{ -return x_84; -} -} -else -{ -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; size_t x_99; uint8_t x_100; -x_94 = lean_ctor_get(x_1, 0); -x_95 = lean_ctor_get(x_1, 1); -lean_inc(x_95); -lean_inc(x_94); -lean_dec(x_1); -x_96 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -x_97 = lean_unsigned_to_nat(0u); -x_98 = l_Std_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10(x_96, x_97, x_4, x_5); -x_99 = 7; -x_100 = lean_usize_dec_le(x_99, x_3); -if (x_100 == 0) -{ -lean_object* x_101; lean_object* x_102; uint8_t x_103; -x_101 = l_Std_PersistentHashMap_getCollisionNodeSize___rarg(x_98); -x_102 = lean_unsigned_to_nat(4u); -x_103 = lean_nat_dec_lt(x_101, x_102); -lean_dec(x_101); -if (x_103 == 0) -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_104 = lean_ctor_get(x_98, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_98, 1); -lean_inc(x_105); -lean_dec(x_98); -x_106 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1; -x_107 = l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9(x_3, x_104, x_105, lean_box(0), x_97, x_106); -lean_dec(x_105); -lean_dec(x_104); -return x_107; -} -else -{ -return x_98; -} -} -else -{ -return x_98; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = !lean_is_exclusive(x_1); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; uint64_t x_7; size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_1, 1); -x_7 = l_Lean_Meta_DiscrTree_Key_hash(x_2); -x_8 = lean_uint64_to_usize(x_7); -x_9 = 1; -x_10 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_5, x_8, x_9, x_2, x_3); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_nat_add(x_6, x_11); -lean_dec(x_6); -lean_ctor_set(x_1, 1, x_12); -lean_ctor_set(x_1, 0, x_10); -return x_1; -} -else -{ -lean_object* x_13; lean_object* x_14; uint64_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_13 = lean_ctor_get(x_1, 0); -x_14 = lean_ctor_get(x_1, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_1); -x_15 = l_Lean_Meta_DiscrTree_Key_hash(x_2); -x_16 = lean_uint64_to_usize(x_15); -x_17 = 1; -x_18 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_13, x_16, x_17, x_2, x_3); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_add(x_14, x_19); -lean_dec(x_14); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_18); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; -x_3 = l_Array_contains___at___private_Lean_Meta_Match_Value_0__Lean_Meta_isUIntTypeName___spec__1(x_1, x_2); -if (x_3 == 0) -{ -lean_object* x_4; -x_4 = lean_array_push(x_1, x_2); -return x_4; -} -else -{ -lean_dec(x_2); -return x_1; -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_10 = lean_nat_add(x_8, x_9); -x_11 = lean_unsigned_to_nat(2u); -x_12 = lean_nat_div(x_10, x_11); -lean_dec(x_10); -lean_inc(x_5); -x_13 = lean_array_get(x_5, x_6, x_12); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_ctor_get(x_7, 0); -x_16 = l_Lean_Meta_DiscrTree_Key_lt(x_14, x_15); -if (x_16 == 0) -{ -uint8_t x_17; -lean_dec(x_9); -x_17 = l_Lean_Meta_DiscrTree_Key_lt(x_15, x_14); -lean_dec(x_14); -if (x_17 == 0) -{ -lean_object* x_18; uint8_t x_19; -lean_dec(x_8); -lean_dec(x_5); -x_18 = lean_array_get_size(x_6); -x_19 = lean_nat_dec_lt(x_12, x_18); -lean_dec(x_18); -if (x_19 == 0) -{ -lean_dec(x_12); -lean_dec(x_4); -lean_dec(x_2); -return x_6; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_20 = lean_array_fget(x_6, x_12); -x_21 = lean_box(0); -x_22 = lean_array_fset(x_6, x_12, x_21); -x_23 = !lean_is_exclusive(x_20); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_24 = lean_ctor_get(x_20, 1); -x_25 = lean_ctor_get(x_20, 0); -lean_dec(x_25); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_nat_add(x_3, x_26); -x_28 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_1, x_2, x_27, x_24); -lean_dec(x_27); -lean_ctor_set(x_20, 1, x_28); -lean_ctor_set(x_20, 0, x_4); -x_29 = lean_array_fset(x_22, x_12, x_20); -lean_dec(x_12); -return x_29; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_30 = lean_ctor_get(x_20, 1); -lean_inc(x_30); -lean_dec(x_20); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_nat_add(x_3, x_31); -x_33 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_1, x_2, x_32, x_30); -lean_dec(x_32); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_4); -lean_ctor_set(x_34, 1, x_33); -x_35 = lean_array_fset(x_22, x_12, x_34); -lean_dec(x_12); -return x_35; -} -} -} -else -{ -x_9 = x_12; -goto _start; -} -} -else -{ -uint8_t x_37; -lean_dec(x_14); -x_37 = lean_nat_dec_eq(x_12, x_8); -if (x_37 == 0) -{ -lean_dec(x_8); -x_8 = x_12; -goto _start; -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_5); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_nat_add(x_3, x_39); -x_41 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_1, x_2, x_40); -lean_dec(x_40); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_4); -lean_ctor_set(x_42, 1, x_41); -x_43 = lean_nat_add(x_8, x_39); -lean_dec(x_8); -x_44 = l_Array_insertAt___rarg(x_6, x_43, x_42); -lean_dec(x_43); -return x_44; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -uint8_t x_8; -x_8 = l_Array_isEmpty___rarg(x_6); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_9 = lean_unsigned_to_nat(0u); -lean_inc(x_5); -x_10 = lean_array_get(x_5, x_6, x_9); -x_11 = lean_ctor_get(x_7, 0); -x_12 = lean_ctor_get(x_10, 0); -lean_inc(x_12); -lean_dec(x_10); -x_13 = l_Lean_Meta_DiscrTree_Key_lt(x_11, x_12); -if (x_13 == 0) -{ -uint8_t x_14; -x_14 = l_Lean_Meta_DiscrTree_Key_lt(x_12, x_11); -lean_dec(x_12); -if (x_14 == 0) -{ -lean_object* x_15; uint8_t x_16; -lean_dec(x_5); -x_15 = lean_array_get_size(x_6); -x_16 = lean_nat_dec_lt(x_9, x_15); -lean_dec(x_15); -if (x_16 == 0) -{ -lean_dec(x_4); -lean_dec(x_2); -return x_6; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_array_fget(x_6, x_9); -x_18 = lean_box(0); -x_19 = lean_array_fset(x_6, x_9, x_18); -x_20 = !lean_is_exclusive(x_17); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_17, 1); -x_22 = lean_ctor_get(x_17, 0); -lean_dec(x_22); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_nat_add(x_3, x_23); -x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_1, x_2, x_24, x_21); -lean_dec(x_24); -lean_ctor_set(x_17, 1, x_25); -lean_ctor_set(x_17, 0, x_4); -x_26 = lean_array_fset(x_19, x_9, x_17); -return x_26; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_27 = lean_ctor_get(x_17, 1); -lean_inc(x_27); -lean_dec(x_17); -x_28 = lean_unsigned_to_nat(1u); -x_29 = lean_nat_add(x_3, x_28); -x_30 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_1, x_2, x_29, x_27); -lean_dec(x_29); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_4); -lean_ctor_set(x_31, 1, x_30); -x_32 = lean_array_fset(x_19, x_9, x_31); -return x_32; -} -} -} -else -{ -lean_object* x_33; lean_object* x_34; uint8_t x_35; -lean_inc(x_5); -x_33 = l_Array_back___rarg(x_5, x_6); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -lean_dec(x_33); -x_35 = l_Lean_Meta_DiscrTree_Key_lt(x_34, x_11); -if (x_35 == 0) -{ -uint8_t x_36; -x_36 = l_Lean_Meta_DiscrTree_Key_lt(x_11, x_34); -lean_dec(x_34); -if (x_36 == 0) -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; -lean_dec(x_5); -x_37 = lean_array_get_size(x_6); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_nat_sub(x_37, x_38); -x_40 = lean_nat_dec_lt(x_39, x_37); -lean_dec(x_37); -if (x_40 == 0) -{ -lean_dec(x_39); -lean_dec(x_4); -lean_dec(x_2); -return x_6; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_41 = lean_array_fget(x_6, x_39); -x_42 = lean_box(0); -x_43 = lean_array_fset(x_6, x_39, x_42); -x_44 = !lean_is_exclusive(x_41); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_45 = lean_ctor_get(x_41, 1); -x_46 = lean_ctor_get(x_41, 0); -lean_dec(x_46); -x_47 = lean_nat_add(x_3, x_38); -x_48 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_1, x_2, x_47, x_45); -lean_dec(x_47); -lean_ctor_set(x_41, 1, x_48); -lean_ctor_set(x_41, 0, x_4); -x_49 = lean_array_fset(x_43, x_39, x_41); -lean_dec(x_39); -return x_49; -} -else -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_50 = lean_ctor_get(x_41, 1); -lean_inc(x_50); -lean_dec(x_41); -x_51 = lean_nat_add(x_3, x_38); -x_52 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_1, x_2, x_51, x_50); -lean_dec(x_51); -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_4); -lean_ctor_set(x_53, 1, x_52); -x_54 = lean_array_fset(x_43, x_39, x_53); -lean_dec(x_39); -return x_54; -} -} -} -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_55 = lean_array_get_size(x_6); -x_56 = lean_unsigned_to_nat(1u); -x_57 = lean_nat_sub(x_55, x_56); -lean_dec(x_55); -x_58 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__14(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9, x_57); -return x_58; -} -} -else -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -lean_dec(x_34); -lean_dec(x_5); -x_59 = lean_unsigned_to_nat(1u); -x_60 = lean_nat_add(x_3, x_59); -x_61 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_1, x_2, x_60); -lean_dec(x_60); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_4); -lean_ctor_set(x_62, 1, x_61); -x_63 = lean_array_push(x_6, x_62); -return x_63; -} -} -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -lean_dec(x_12); -lean_dec(x_5); -x_64 = lean_unsigned_to_nat(1u); -x_65 = lean_nat_add(x_3, x_64); -x_66 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_1, x_2, x_65); -lean_dec(x_65); -x_67 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_67, 0, x_4); -lean_ctor_set(x_67, 1, x_66); -x_68 = l_Array_insertAt___rarg(x_6, x_9, x_67); -return x_68; -} -} -else -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -lean_dec(x_5); -x_69 = lean_unsigned_to_nat(1u); -x_70 = lean_nat_add(x_3, x_69); -x_71 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_1, x_2, x_70); -lean_dec(x_70); -x_72 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_72, 0, x_4); -lean_ctor_set(x_72, 1, x_71); -x_73 = lean_array_push(x_6, x_72); -return x_73; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_6 = lean_ctor_get(x_4, 0); -x_7 = lean_ctor_get(x_4, 1); -x_8 = lean_array_get_size(x_1); -x_9 = lean_nat_dec_lt(x_3, x_8); -lean_dec(x_8); -if (x_9 == 0) -{ -lean_object* x_10; -x_10 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(x_6, x_2); -lean_ctor_set(x_4, 0, x_10); -return x_4; -} -else -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_array_fget(x_1, x_3); -x_12 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3; -lean_inc(x_11); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -x_14 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2; -x_15 = l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(x_1, x_2, x_3, x_11, x_14, x_7, x_13); -lean_dec(x_13); -lean_ctor_set(x_4, 1, x_15); -return x_4; -} -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = lean_ctor_get(x_4, 0); -x_17 = lean_ctor_get(x_4, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_4); -x_18 = lean_array_get_size(x_1); -x_19 = lean_nat_dec_lt(x_3, x_18); -lean_dec(x_18); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; -x_20 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertVal___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(x_16, x_2); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_17); -return x_21; -} -else -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_22 = lean_array_fget(x_1, x_3); -x_23 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3; -lean_inc(x_22); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2; -x_26 = l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(x_1, x_2, x_3, x_22, x_25, x_17, x_24); -lean_dec(x_24); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_16); -lean_ctor_set(x_27, 1, x_26); -return x_27; -} -} -} -} -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__15(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; -x_2 = l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16___closed__1; -x_3 = lean_panic_fn(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = l_Array_isEmpty___rarg(x_2); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_array_get_size(x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_nat_dec_lt(x_6, x_5); -lean_dec(x_5); -if (x_7 == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; -x_9 = l_panic___at_Lean_Meta_DiscrTree_insertCore___spec__1(x_8); -lean_inc(x_9); -lean_inc(x_1); -x_10 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4(x_1, x_9); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_unsigned_to_nat(1u); -x_12 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_2, x_3, x_11); -lean_dec(x_2); -x_13 = l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(x_1, x_9, x_12); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_10, 0); -lean_inc(x_14); -lean_dec(x_10); -x_15 = lean_unsigned_to_nat(1u); -x_16 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_2, x_3, x_15, x_14); -lean_dec(x_2); -x_17 = l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(x_1, x_9, x_16); -return x_17; -} -} -else -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_array_fget(x_2, x_6); -lean_inc(x_18); -lean_inc(x_1); -x_19 = l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4(x_1, x_18); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_unsigned_to_nat(1u); -x_21 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_createNodes___rarg(x_2, x_3, x_20); -lean_dec(x_2); -x_22 = l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(x_1, x_18, x_21); -return x_22; -} -else -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_19, 0); -lean_inc(x_23); -lean_dec(x_19); -x_24 = lean_unsigned_to_nat(1u); -x_25 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_2, x_3, x_24, x_23); -lean_dec(x_2); -x_26 = l_Std_PersistentHashMap_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(x_1, x_18, x_25); -return x_26; -} -} -} -else -{ -lean_object* x_27; lean_object* x_28; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_27 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8; -x_28 = l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__15(x_27); -return x_28; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_DiscrTree_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Meta_DiscrTree_mkPath(x_2, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) -{ -uint8_t x_10; -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3(x_1, x_11, x_3); -lean_ctor_set(x_9, 0, x_12); -return x_9; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_9, 0); -x_14 = lean_ctor_get(x_9, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_9); -x_15 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3(x_1, x_13, x_3); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -return x_16; -} -} -else -{ -uint8_t x_17; -lean_dec(x_3); -lean_dec(x_1); -x_17 = !lean_is_exclusive(x_9); -if (x_17 == 0) -{ -return x_9; -} -else -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_9, 0); -x_19 = lean_ctor_get(x_9, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_9); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__18(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -if (lean_obj_tag(x_2) == 5) -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -lean_dec(x_2); -x_6 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__18(x_1, x_4, x_3); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -x_8 = lean_unbox(x_7); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; -lean_dec(x_7); -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_5, x_9); -return x_10; -} -else -{ -uint8_t x_11; -lean_dec(x_5); -x_11 = !lean_is_exclusive(x_6); -if (x_11 == 0) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_6, 0); -lean_dec(x_12); -return x_6; -} -else -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_6, 1); -lean_inc(x_13); -lean_dec(x_6); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_7); -lean_ctor_set(x_14, 1, x_13); -return x_14; -} -} -} -else -{ -lean_object* x_15; -x_15 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_2, x_3); -return x_15; -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__21(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_uget(x_2, x_3); -x_7 = l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__20(x_1, x_6); -if (x_7 == 0) -{ -size_t x_8; size_t x_9; -x_8 = 1; -x_9 = lean_usize_add(x_3, x_8); -x_3 = x_9; -goto _start; -} -else -{ -uint8_t x_11; -x_11 = 1; -return x_11; -} -} -else -{ -uint8_t x_12; -x_12 = 0; -return x_12; -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__22(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; -x_6 = lean_array_uget(x_2, x_3); -if (lean_obj_tag(x_6) == 0) -{ -size_t x_7; size_t x_8; -x_7 = 1; -x_8 = lean_usize_add(x_3, x_7); -x_3 = x_8; -goto _start; -} -else -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_6, 0); -lean_inc(x_10); -lean_dec(x_6); -x_11 = l_Lean_LocalDecl_fvarId(x_10); -lean_dec(x_10); -x_12 = l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(x_1, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -size_t x_13; size_t x_14; -x_13 = 1; -x_14 = lean_usize_add(x_3, x_13); -x_3 = x_14; -goto _start; -} -else -{ -uint8_t x_16; -x_16 = 1; -return x_16; -} -} -} -else -{ -uint8_t x_17; -x_17 = 0; -return x_17; -} -} -} -LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__20(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_3 = lean_ctor_get(x_2, 0); -lean_inc(x_3); -lean_dec(x_2); -x_4 = lean_array_get_size(x_3); -x_5 = lean_unsigned_to_nat(0u); -x_6 = lean_nat_dec_lt(x_5, x_4); -if (x_6 == 0) -{ -uint8_t x_7; -lean_dec(x_4); -lean_dec(x_3); -x_7 = 0; -return x_7; -} -else -{ -uint8_t x_8; -x_8 = lean_nat_dec_le(x_4, x_4); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_4); -lean_dec(x_3); -x_9 = 0; -return x_9; -} -else -{ -size_t x_10; size_t x_11; uint8_t x_12; -x_10 = 0; -x_11 = lean_usize_of_nat(x_4); -lean_dec(x_4); -x_12 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__21(x_1, x_3, x_10, x_11); -lean_dec(x_3); -return x_12; -} -} -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = lean_ctor_get(x_2, 0); -lean_inc(x_13); -lean_dec(x_2); -x_14 = lean_array_get_size(x_13); -x_15 = lean_unsigned_to_nat(0u); -x_16 = lean_nat_dec_lt(x_15, x_14); -if (x_16 == 0) -{ -uint8_t x_17; -lean_dec(x_14); -lean_dec(x_13); -x_17 = 0; -return x_17; -} -else -{ -uint8_t x_18; -x_18 = lean_nat_dec_le(x_14, x_14); -if (x_18 == 0) -{ -uint8_t x_19; -lean_dec(x_14); -lean_dec(x_13); -x_19 = 0; -return x_19; -} -else -{ -size_t x_20; size_t x_21; uint8_t x_22; -x_20 = 0; -x_21 = lean_usize_of_nat(x_14); -lean_dec(x_14); -x_22 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__22(x_1, x_13, x_20, x_21); -lean_dec(x_13); -return x_22; -} -} -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__23(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; -x_6 = lean_array_uget(x_2, x_3); -if (lean_obj_tag(x_6) == 0) -{ -size_t x_7; size_t x_8; -x_7 = 1; -x_8 = lean_usize_add(x_3, x_7); -x_3 = x_8; -goto _start; -} -else -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_6, 0); -lean_inc(x_10); -lean_dec(x_6); -x_11 = l_Lean_LocalDecl_fvarId(x_10); -lean_dec(x_10); -x_12 = l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(x_1, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -size_t x_13; size_t x_14; -x_13 = 1; -x_14 = lean_usize_add(x_3, x_13); -x_3 = x_14; -goto _start; -} -else -{ -uint8_t x_16; -x_16 = 1; -return x_16; -} -} -} -else -{ -uint8_t x_17; -x_17 = 0; -return x_17; -} -} -} -LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__19(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; uint8_t x_4; -x_3 = lean_ctor_get(x_2, 0); -lean_inc(x_3); -x_4 = l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__20(x_1, x_3); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -lean_dec(x_2); -x_6 = lean_array_get_size(x_5); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_nat_dec_lt(x_7, x_6); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_6); -lean_dec(x_5); -x_9 = 0; -return x_9; -} -else -{ -uint8_t x_10; -x_10 = lean_nat_dec_le(x_6, x_6); -if (x_10 == 0) -{ -uint8_t x_11; -lean_dec(x_6); -lean_dec(x_5); -x_11 = 0; -return x_11; -} -else -{ -size_t x_12; size_t x_13; uint8_t x_14; -x_12 = 0; -x_13 = lean_usize_of_nat(x_6); -lean_dec(x_6); -x_14 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__23(x_1, x_5, x_12, x_13); -lean_dec(x_5); -return x_14; -} -} -} -else -{ -lean_dec(x_2); -return x_4; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -switch (lean_obj_tag(x_2)) { -case 1: -{ -lean_object* x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -lean_dec(x_2); -x_5 = l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(x_1, x_4); -lean_dec(x_4); -x_6 = lean_box(x_5); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_3); -return x_7; -} -case 2: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_2, 0); -lean_inc(x_8); -lean_dec(x_2); -lean_inc(x_8); -x_9 = l_Lean_getExprMVarAssignment_x3f___at_Lean_exprDependsOn___spec__4(x_8, x_3); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_12 = lean_ctor_get(x_9, 1); -x_13 = lean_ctor_get(x_9, 0); -lean_dec(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -x_15 = l_Lean_MetavarContext_getDecl(x_14, x_8); -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__19(x_1, x_17); -x_19 = lean_box(x_18); -lean_ctor_set(x_9, 0, x_19); -return x_9; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_20 = lean_ctor_get(x_9, 1); -lean_inc(x_20); -lean_dec(x_9); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -x_22 = l_Lean_MetavarContext_getDecl(x_21, x_8); -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_dec(x_23); -x_25 = l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__19(x_1, x_24); -x_26 = lean_box(x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_20); -return x_27; -} -} -else -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -lean_dec(x_8); -x_28 = lean_ctor_get(x_9, 1); -lean_inc(x_28); -lean_dec(x_9); -x_29 = lean_ctor_get(x_10, 0); -lean_inc(x_29); -lean_dec(x_10); -x_30 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_29, x_28); -return x_30; -} -} -case 5: -{ -lean_object* x_31; uint8_t x_32; -x_31 = l_Lean_Expr_getAppFn(x_2); -x_32 = l_Lean_Expr_isMVar(x_31); -if (x_32 == 0) -{ -lean_object* x_33; -lean_dec(x_31); -x_33 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__18(x_1, x_2, x_3); -return x_33; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -lean_inc(x_2); -x_34 = l_Lean_instantiateMVars___at_Lean_exprDependsOn___spec__11(x_2, x_3); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = l_Lean_Expr_getAppFn(x_35); -x_38 = lean_expr_eqv(x_37, x_31); -lean_dec(x_31); -lean_dec(x_37); -if (x_38 == 0) -{ -lean_dec(x_2); -x_2 = x_35; -x_3 = x_36; -goto _start; -} -else -{ -lean_object* x_40; -lean_dec(x_35); -x_40 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__18(x_1, x_2, x_36); -return x_40; -} -} -} -case 6: -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; -x_41 = lean_ctor_get(x_2, 1); -lean_inc(x_41); -x_42 = lean_ctor_get(x_2, 2); -lean_inc(x_42); -lean_dec(x_2); -x_43 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_41, x_3); -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_unbox(x_44); -if (x_45 == 0) -{ -lean_object* x_46; lean_object* x_47; -lean_dec(x_44); -x_46 = lean_ctor_get(x_43, 1); -lean_inc(x_46); -lean_dec(x_43); -x_47 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_42, x_46); -return x_47; -} -else -{ -uint8_t x_48; -lean_dec(x_42); -x_48 = !lean_is_exclusive(x_43); -if (x_48 == 0) -{ -lean_object* x_49; -x_49 = lean_ctor_get(x_43, 0); -lean_dec(x_49); -return x_43; -} -else -{ -lean_object* x_50; lean_object* x_51; -x_50 = lean_ctor_get(x_43, 1); -lean_inc(x_50); -lean_dec(x_43); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_44); -lean_ctor_set(x_51, 1, x_50); -return x_51; -} -} -} -case 7: -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; -x_52 = lean_ctor_get(x_2, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_2, 2); -lean_inc(x_53); -lean_dec(x_2); -x_54 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_52, x_3); -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -x_56 = lean_unbox(x_55); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; -lean_dec(x_55); -x_57 = lean_ctor_get(x_54, 1); -lean_inc(x_57); -lean_dec(x_54); -x_58 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_53, x_57); -return x_58; -} -else -{ -uint8_t x_59; -lean_dec(x_53); -x_59 = !lean_is_exclusive(x_54); -if (x_59 == 0) -{ -lean_object* x_60; -x_60 = lean_ctor_get(x_54, 0); -lean_dec(x_60); -return x_54; -} -else -{ -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_54, 1); -lean_inc(x_61); -lean_dec(x_54); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_55); -lean_ctor_set(x_62, 1, x_61); -return x_62; -} -} -} -case 8: -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; -x_63 = lean_ctor_get(x_2, 1); -lean_inc(x_63); -x_64 = lean_ctor_get(x_2, 2); -lean_inc(x_64); -x_65 = lean_ctor_get(x_2, 3); -lean_inc(x_65); -lean_dec(x_2); -x_66 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_63, x_3); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_unbox(x_67); -if (x_68 == 0) -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -lean_dec(x_67); -x_69 = lean_ctor_get(x_66, 1); -lean_inc(x_69); -lean_dec(x_66); -x_70 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_64, x_69); -x_71 = lean_ctor_get(x_70, 0); -lean_inc(x_71); -x_72 = lean_unbox(x_71); -if (x_72 == 0) -{ -lean_object* x_73; lean_object* x_74; -lean_dec(x_71); -x_73 = lean_ctor_get(x_70, 1); -lean_inc(x_73); -lean_dec(x_70); -x_74 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_65, x_73); -return x_74; -} -else -{ -uint8_t x_75; -lean_dec(x_65); -x_75 = !lean_is_exclusive(x_70); -if (x_75 == 0) -{ -lean_object* x_76; -x_76 = lean_ctor_get(x_70, 0); -lean_dec(x_76); -return x_70; -} -else -{ -lean_object* x_77; lean_object* x_78; -x_77 = lean_ctor_get(x_70, 1); -lean_inc(x_77); -lean_dec(x_70); -x_78 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_78, 0, x_71); -lean_ctor_set(x_78, 1, x_77); -return x_78; -} -} -} -else -{ -uint8_t x_79; -lean_dec(x_65); -lean_dec(x_64); -x_79 = !lean_is_exclusive(x_66); -if (x_79 == 0) -{ -lean_object* x_80; -x_80 = lean_ctor_get(x_66, 0); -lean_dec(x_80); -return x_66; -} -else -{ -lean_object* x_81; lean_object* x_82; -x_81 = lean_ctor_get(x_66, 1); -lean_inc(x_81); -lean_dec(x_66); -x_82 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_82, 0, x_67); -lean_ctor_set(x_82, 1, x_81); -return x_82; -} -} -} -case 10: -{ -lean_object* x_83; lean_object* x_84; -x_83 = lean_ctor_get(x_2, 1); -lean_inc(x_83); -lean_dec(x_2); -x_84 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_83, x_3); -return x_84; -} -case 11: -{ -lean_object* x_85; lean_object* x_86; -x_85 = lean_ctor_get(x_2, 2); -lean_inc(x_85); -lean_dec(x_2); -x_86 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_85, x_3); -return x_86; -} -default: -{ -uint8_t x_87; lean_object* x_88; lean_object* x_89; -lean_dec(x_2); -x_87 = 0; -x_88 = lean_box(x_87); -x_89 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_3); -return x_89; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; uint8_t x_6; -lean_inc(x_2); -x_4 = l___private_Lean_MetavarContext_0__Lean_DependsOn_shouldVisit(x_2, x_3); -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -x_6 = lean_unbox(x_5); -lean_dec(x_5); -if (x_6 == 0) -{ -uint8_t x_7; -lean_dec(x_2); -x_7 = !lean_is_exclusive(x_4); -if (x_7 == 0) -{ -lean_object* x_8; uint8_t x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_4, 0); -lean_dec(x_8); -x_9 = 0; -x_10 = lean_box(x_9); -lean_ctor_set(x_4, 0, x_10); -return x_4; -} -else -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_ctor_get(x_4, 1); -lean_inc(x_11); -lean_dec(x_4); -x_12 = 0; -x_13 = lean_box(x_12); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_11); -return x_14; -} -} -else -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_4, 1); -lean_inc(x_15); -lean_dec(x_4); -x_16 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__17(x_1, x_2, x_15); -return x_16; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__26(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -if (lean_obj_tag(x_2) == 5) -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -lean_dec(x_2); -x_6 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__26(x_1, x_4, x_3); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -x_8 = lean_unbox(x_7); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; -lean_dec(x_7); -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_5, x_9); -return x_10; -} -else -{ -uint8_t x_11; -lean_dec(x_5); -x_11 = !lean_is_exclusive(x_6); -if (x_11 == 0) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_6, 0); -lean_dec(x_12); -return x_6; -} -else -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_6, 1); -lean_inc(x_13); -lean_dec(x_6); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_7); -lean_ctor_set(x_14, 1, x_13); -return x_14; -} -} -} -else -{ -lean_object* x_15; -x_15 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_2, x_3); -return x_15; -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__29(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_uget(x_2, x_3); -x_7 = l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__28(x_1, x_6); -if (x_7 == 0) -{ -size_t x_8; size_t x_9; -x_8 = 1; -x_9 = lean_usize_add(x_3, x_8); -x_3 = x_9; -goto _start; -} -else -{ -uint8_t x_11; -x_11 = 1; -return x_11; -} -} -else -{ -uint8_t x_12; -x_12 = 0; -return x_12; -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__30(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; -x_6 = lean_array_uget(x_2, x_3); -if (lean_obj_tag(x_6) == 0) -{ -size_t x_7; size_t x_8; -x_7 = 1; -x_8 = lean_usize_add(x_3, x_7); -x_3 = x_8; -goto _start; -} -else -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_6, 0); -lean_inc(x_10); -lean_dec(x_6); -x_11 = l_Lean_LocalDecl_fvarId(x_10); -lean_dec(x_10); -x_12 = l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(x_1, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -size_t x_13; size_t x_14; -x_13 = 1; -x_14 = lean_usize_add(x_3, x_13); -x_3 = x_14; -goto _start; -} -else -{ -uint8_t x_16; -x_16 = 1; -return x_16; -} -} -} -else -{ -uint8_t x_17; -x_17 = 0; -return x_17; -} -} -} -LEAN_EXPORT uint8_t l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__28(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_3 = lean_ctor_get(x_2, 0); -lean_inc(x_3); -lean_dec(x_2); -x_4 = lean_array_get_size(x_3); -x_5 = lean_unsigned_to_nat(0u); -x_6 = lean_nat_dec_lt(x_5, x_4); -if (x_6 == 0) -{ -uint8_t x_7; -lean_dec(x_4); -lean_dec(x_3); -x_7 = 0; -return x_7; -} -else -{ -uint8_t x_8; -x_8 = lean_nat_dec_le(x_4, x_4); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_4); -lean_dec(x_3); -x_9 = 0; -return x_9; -} -else -{ -size_t x_10; size_t x_11; uint8_t x_12; -x_10 = 0; -x_11 = lean_usize_of_nat(x_4); -lean_dec(x_4); -x_12 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__29(x_1, x_3, x_10, x_11); -lean_dec(x_3); -return x_12; -} -} -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = lean_ctor_get(x_2, 0); -lean_inc(x_13); -lean_dec(x_2); -x_14 = lean_array_get_size(x_13); -x_15 = lean_unsigned_to_nat(0u); -x_16 = lean_nat_dec_lt(x_15, x_14); -if (x_16 == 0) -{ -uint8_t x_17; -lean_dec(x_14); -lean_dec(x_13); -x_17 = 0; -return x_17; -} -else -{ -uint8_t x_18; -x_18 = lean_nat_dec_le(x_14, x_14); -if (x_18 == 0) -{ -uint8_t x_19; -lean_dec(x_14); -lean_dec(x_13); -x_19 = 0; -return x_19; -} -else -{ -size_t x_20; size_t x_21; uint8_t x_22; -x_20 = 0; -x_21 = lean_usize_of_nat(x_14); -lean_dec(x_14); -x_22 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__30(x_1, x_13, x_20, x_21); -lean_dec(x_13); -return x_22; -} -} -} -} -} -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__31(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_eq(x_3, x_4); -if (x_5 == 0) -{ -lean_object* x_6; -x_6 = lean_array_uget(x_2, x_3); -if (lean_obj_tag(x_6) == 0) -{ -size_t x_7; size_t x_8; -x_7 = 1; -x_8 = lean_usize_add(x_3, x_7); -x_3 = x_8; -goto _start; -} -else -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_6, 0); -lean_inc(x_10); -lean_dec(x_6); -x_11 = l_Lean_LocalDecl_fvarId(x_10); -lean_dec(x_10); -x_12 = l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(x_1, x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -size_t x_13; size_t x_14; -x_13 = 1; -x_14 = lean_usize_add(x_3, x_13); -x_3 = x_14; -goto _start; -} -else -{ -uint8_t x_16; -x_16 = 1; -return x_16; -} -} -} -else -{ -uint8_t x_17; -x_17 = 0; -return x_17; -} -} -} -LEAN_EXPORT uint8_t l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__27(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; uint8_t x_4; -x_3 = lean_ctor_get(x_2, 0); -lean_inc(x_3); -x_4 = l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__28(x_1, x_3); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -lean_dec(x_2); -x_6 = lean_array_get_size(x_5); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_nat_dec_lt(x_7, x_6); -if (x_8 == 0) -{ -uint8_t x_9; -lean_dec(x_6); -lean_dec(x_5); -x_9 = 0; -return x_9; -} -else -{ -uint8_t x_10; -x_10 = lean_nat_dec_le(x_6, x_6); -if (x_10 == 0) -{ -uint8_t x_11; -lean_dec(x_6); -lean_dec(x_5); -x_11 = 0; -return x_11; -} -else -{ -size_t x_12; size_t x_13; uint8_t x_14; -x_12 = 0; -x_13 = lean_usize_of_nat(x_6); -lean_dec(x_6); -x_14 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__31(x_1, x_5, x_12, x_13); -lean_dec(x_5); -return x_14; -} -} -} -else -{ -lean_dec(x_2); -return x_4; -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__25(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -switch (lean_obj_tag(x_2)) { -case 1: -{ -lean_object* x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -lean_dec(x_2); -x_5 = l_Array_contains___at___private_Lean_Class_0__Lean_checkOutParam___spec__1(x_1, x_4); -lean_dec(x_4); -x_6 = lean_box(x_5); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_3); -return x_7; -} -case 2: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_2, 0); -lean_inc(x_8); -lean_dec(x_2); -lean_inc(x_8); -x_9 = l_Lean_getExprMVarAssignment_x3f___at_Lean_exprDependsOn___spec__4(x_8, x_3); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_12 = lean_ctor_get(x_9, 1); -x_13 = lean_ctor_get(x_9, 0); -lean_dec(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -x_15 = l_Lean_MetavarContext_getDecl(x_14, x_8); -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__27(x_1, x_17); -x_19 = lean_box(x_18); -lean_ctor_set(x_9, 0, x_19); -return x_9; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_20 = lean_ctor_get(x_9, 1); -lean_inc(x_20); -lean_dec(x_9); -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -x_22 = l_Lean_MetavarContext_getDecl(x_21, x_8); -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_dec(x_23); -x_25 = l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__27(x_1, x_24); -x_26 = lean_box(x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_20); -return x_27; -} -} -else -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -lean_dec(x_8); -x_28 = lean_ctor_get(x_9, 1); -lean_inc(x_28); -lean_dec(x_9); -x_29 = lean_ctor_get(x_10, 0); -lean_inc(x_29); -lean_dec(x_10); -x_30 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_29, x_28); -return x_30; -} -} -case 5: -{ -lean_object* x_31; uint8_t x_32; -x_31 = l_Lean_Expr_getAppFn(x_2); -x_32 = l_Lean_Expr_isMVar(x_31); -if (x_32 == 0) -{ -lean_object* x_33; -lean_dec(x_31); -x_33 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__26(x_1, x_2, x_3); -return x_33; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; -lean_inc(x_2); -x_34 = l_Lean_instantiateMVars___at_Lean_exprDependsOn___spec__11(x_2, x_3); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = l_Lean_Expr_getAppFn(x_35); -x_38 = lean_expr_eqv(x_37, x_31); -lean_dec(x_31); -lean_dec(x_37); -if (x_38 == 0) -{ -lean_dec(x_2); -x_2 = x_35; -x_3 = x_36; -goto _start; -} -else -{ -lean_object* x_40; -lean_dec(x_35); -x_40 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__26(x_1, x_2, x_36); -return x_40; -} -} -} -case 6: -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; -x_41 = lean_ctor_get(x_2, 1); -lean_inc(x_41); -x_42 = lean_ctor_get(x_2, 2); -lean_inc(x_42); -lean_dec(x_2); -x_43 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_41, x_3); -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_unbox(x_44); -if (x_45 == 0) -{ -lean_object* x_46; lean_object* x_47; -lean_dec(x_44); -x_46 = lean_ctor_get(x_43, 1); -lean_inc(x_46); -lean_dec(x_43); -x_47 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_42, x_46); -return x_47; -} -else -{ -uint8_t x_48; -lean_dec(x_42); -x_48 = !lean_is_exclusive(x_43); -if (x_48 == 0) -{ -lean_object* x_49; -x_49 = lean_ctor_get(x_43, 0); -lean_dec(x_49); -return x_43; -} -else -{ -lean_object* x_50; lean_object* x_51; -x_50 = lean_ctor_get(x_43, 1); -lean_inc(x_50); -lean_dec(x_43); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_44); -lean_ctor_set(x_51, 1, x_50); -return x_51; -} -} -} -case 7: -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; -x_52 = lean_ctor_get(x_2, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_2, 2); -lean_inc(x_53); -lean_dec(x_2); -x_54 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_52, x_3); -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -x_56 = lean_unbox(x_55); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; -lean_dec(x_55); -x_57 = lean_ctor_get(x_54, 1); -lean_inc(x_57); -lean_dec(x_54); -x_58 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_53, x_57); -return x_58; -} -else -{ -uint8_t x_59; -lean_dec(x_53); -x_59 = !lean_is_exclusive(x_54); -if (x_59 == 0) -{ -lean_object* x_60; -x_60 = lean_ctor_get(x_54, 0); -lean_dec(x_60); -return x_54; -} -else -{ -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_54, 1); -lean_inc(x_61); -lean_dec(x_54); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_55); -lean_ctor_set(x_62, 1, x_61); -return x_62; -} -} -} -case 8: -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; -x_63 = lean_ctor_get(x_2, 1); -lean_inc(x_63); -x_64 = lean_ctor_get(x_2, 2); -lean_inc(x_64); -x_65 = lean_ctor_get(x_2, 3); -lean_inc(x_65); -lean_dec(x_2); -x_66 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_63, x_3); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_unbox(x_67); -if (x_68 == 0) -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -lean_dec(x_67); -x_69 = lean_ctor_get(x_66, 1); -lean_inc(x_69); -lean_dec(x_66); -x_70 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_64, x_69); -x_71 = lean_ctor_get(x_70, 0); -lean_inc(x_71); -x_72 = lean_unbox(x_71); -if (x_72 == 0) -{ -lean_object* x_73; lean_object* x_74; -lean_dec(x_71); -x_73 = lean_ctor_get(x_70, 1); -lean_inc(x_73); -lean_dec(x_70); -x_74 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_65, x_73); -return x_74; -} -else -{ -uint8_t x_75; -lean_dec(x_65); -x_75 = !lean_is_exclusive(x_70); -if (x_75 == 0) -{ -lean_object* x_76; -x_76 = lean_ctor_get(x_70, 0); -lean_dec(x_76); -return x_70; -} -else -{ -lean_object* x_77; lean_object* x_78; -x_77 = lean_ctor_get(x_70, 1); -lean_inc(x_77); -lean_dec(x_70); -x_78 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_78, 0, x_71); -lean_ctor_set(x_78, 1, x_77); -return x_78; -} -} -} -else -{ -uint8_t x_79; -lean_dec(x_65); -lean_dec(x_64); -x_79 = !lean_is_exclusive(x_66); -if (x_79 == 0) -{ -lean_object* x_80; -x_80 = lean_ctor_get(x_66, 0); -lean_dec(x_80); -return x_66; -} -else -{ -lean_object* x_81; lean_object* x_82; -x_81 = lean_ctor_get(x_66, 1); -lean_inc(x_81); -lean_dec(x_66); -x_82 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_82, 0, x_67); -lean_ctor_set(x_82, 1, x_81); -return x_82; -} -} -} -case 10: -{ -lean_object* x_83; lean_object* x_84; -x_83 = lean_ctor_get(x_2, 1); -lean_inc(x_83); -lean_dec(x_2); -x_84 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_83, x_3); -return x_84; -} -case 11: -{ -lean_object* x_85; lean_object* x_86; -x_85 = lean_ctor_get(x_2, 2); -lean_inc(x_85); -lean_dec(x_2); -x_86 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_85, x_3); -return x_86; -} -default: -{ -uint8_t x_87; lean_object* x_88; lean_object* x_89; -lean_dec(x_2); -x_87 = 0; -x_88 = lean_box(x_87); -x_89 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_3); -return x_89; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; uint8_t x_6; -lean_inc(x_2); -x_4 = l___private_Lean_MetavarContext_0__Lean_DependsOn_shouldVisit(x_2, x_3); -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -x_6 = lean_unbox(x_5); -lean_dec(x_5); -if (x_6 == 0) -{ -uint8_t x_7; -lean_dec(x_2); -x_7 = !lean_is_exclusive(x_4); -if (x_7 == 0) -{ -lean_object* x_8; uint8_t x_9; lean_object* x_10; -x_8 = lean_ctor_get(x_4, 0); -lean_dec(x_8); -x_9 = 0; -x_10 = lean_box(x_9); -lean_ctor_set(x_4, 0, x_10); -return x_4; -} -else -{ -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_11 = lean_ctor_get(x_4, 1); -lean_inc(x_11); -lean_dec(x_4); -x_12 = 0; -x_13 = lean_box(x_12); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_11); -return x_14; -} -} -else -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_4, 1); -lean_inc(x_15); -lean_dec(x_4); -x_16 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__25(x_1, x_2, x_15); -return x_16; -} -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("_rpcEnc", 7); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_11 = lean_ctor_get(x_2, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_2, 1); -lean_inc(x_12); -x_13 = lean_ctor_get(x_2, 2); -lean_inc(x_13); -x_14 = lean_ctor_get(x_2, 3); -lean_inc(x_14); -x_15 = lean_ctor_get(x_2, 4); -lean_inc(x_15); -x_16 = lean_ctor_get(x_2, 5); -lean_inc(x_16); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -lean_inc(x_11); -x_17 = l_Lean_Meta_DiscrTree_getMatch___rarg(x_11, x_1, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_17) == 0) -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -x_21 = l_Array_isEmpty___rarg(x_19); -lean_dec(x_19); -if (x_21 == 0) -{ -lean_object* x_22; -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_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_2); -lean_ctor_set(x_17, 0, x_22); -return x_17; -} -else -{ -uint8_t x_23; -lean_free_object(x_17); -x_23 = !lean_is_exclusive(x_2); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_24 = lean_ctor_get(x_2, 5); -lean_dec(x_24); -x_25 = lean_ctor_get(x_2, 4); -lean_dec(x_25); -x_26 = lean_ctor_get(x_2, 3); -lean_dec(x_26); -x_27 = lean_ctor_get(x_2, 2); -lean_dec(x_27); -x_28 = lean_ctor_get(x_2, 1); -lean_dec(x_28); -x_29 = lean_ctor_get(x_2, 0); -lean_dec(x_29); -x_30 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__2; -x_31 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_30, x_8, x_9, x_20); -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -x_34 = lean_box(0); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_35 = l_Lean_PrettyPrinter_delab(x_1, x_34, x_6, x_7, x_8, x_9, x_33); -if (lean_obj_tag(x_35) == 0) -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_32); -x_38 = l_Lean_Meta_DiscrTree_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(x_11, x_1, x_32, x_6, x_7, x_8, x_9, x_37); -if (lean_obj_tag(x_38) == 0) -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; 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; uint8_t x_69; -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); -lean_inc(x_8); -x_41 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_40); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = lean_st_ref_get(x_9, x_43); -x_45 = lean_ctor_get(x_44, 1); -lean_inc(x_45); -lean_dec(x_44); -x_46 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; -lean_inc(x_42); -x_47 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_47, 0, x_42); -lean_ctor_set(x_47, 1, x_46); -lean_inc(x_32); -x_48 = lean_mk_syntax_ident(x_32); -x_49 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -lean_inc(x_48); -x_50 = lean_array_push(x_49, x_48); -x_51 = lean_box(2); -x_52 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_53 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_53, 0, x_51); -lean_ctor_set(x_53, 1, x_52); -lean_ctor_set(x_53, 2, x_50); -x_54 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -x_55 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_55, 0, x_42); -lean_ctor_set(x_55, 1, x_54); -x_56 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_57 = lean_array_push(x_56, x_47); -x_58 = lean_array_push(x_57, x_53); -x_59 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_60 = lean_array_push(x_58, x_59); -x_61 = lean_array_push(x_60, x_59); -x_62 = lean_array_push(x_61, x_55); -x_63 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_51); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_45); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -lean_dec(x_65); -x_68 = lean_st_ref_get(x_9, x_67); -lean_dec(x_9); -x_69 = !lean_is_exclusive(x_68); -if (x_69 == 0) -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_70 = lean_ctor_get(x_68, 0); -lean_dec(x_70); -x_71 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; -lean_inc(x_66); -x_72 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_72, 0, x_66); -lean_ctor_set(x_72, 1, x_71); -x_73 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_74 = lean_array_push(x_73, x_36); -x_75 = lean_array_push(x_74, x_48); -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_51); -lean_ctor_set(x_76, 1, x_52); -lean_ctor_set(x_76, 2, x_75); -x_77 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2; -x_78 = lean_array_push(x_77, x_76); -x_79 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_80 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_80, 0, x_51); -lean_ctor_set(x_80, 1, x_79); -lean_ctor_set(x_80, 2, x_78); -x_81 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; -x_82 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_82, 0, x_66); -lean_ctor_set(x_82, 1, x_81); -x_83 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_84 = lean_array_push(x_83, x_72); -x_85 = lean_array_push(x_84, x_59); -x_86 = lean_array_push(x_85, x_80); -x_87 = lean_array_push(x_86, x_82); -x_88 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58; -x_89 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_89, 0, x_51); -lean_ctor_set(x_89, 1, x_88); -lean_ctor_set(x_89, 2, x_87); -x_90 = lean_array_push(x_12, x_32); -x_91 = lean_array_push(x_73, x_64); -x_92 = lean_array_push(x_91, x_89); -x_93 = l_Array_append___rarg(x_13, x_92); -lean_ctor_set(x_2, 2, x_93); -lean_ctor_set(x_2, 1, x_90); -lean_ctor_set(x_2, 0, x_39); -x_94 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_94, 0, x_2); -lean_ctor_set(x_68, 0, x_94); -return x_68; -} -else -{ -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; -x_95 = lean_ctor_get(x_68, 1); -lean_inc(x_95); -lean_dec(x_68); -x_96 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; -lean_inc(x_66); -x_97 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_97, 0, x_66); -lean_ctor_set(x_97, 1, x_96); -x_98 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_99 = lean_array_push(x_98, x_36); -x_100 = lean_array_push(x_99, x_48); -x_101 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_101, 0, x_51); -lean_ctor_set(x_101, 1, x_52); -lean_ctor_set(x_101, 2, x_100); -x_102 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2; -x_103 = lean_array_push(x_102, x_101); -x_104 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_51); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; -x_107 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_107, 0, x_66); -lean_ctor_set(x_107, 1, x_106); -x_108 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_109 = lean_array_push(x_108, x_97); -x_110 = lean_array_push(x_109, x_59); -x_111 = lean_array_push(x_110, x_105); -x_112 = lean_array_push(x_111, x_107); -x_113 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58; -x_114 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_114, 0, x_51); -lean_ctor_set(x_114, 1, x_113); -lean_ctor_set(x_114, 2, x_112); -x_115 = lean_array_push(x_12, x_32); -x_116 = lean_array_push(x_98, x_64); -x_117 = lean_array_push(x_116, x_114); -x_118 = l_Array_append___rarg(x_13, x_117); -lean_ctor_set(x_2, 2, x_118); -lean_ctor_set(x_2, 1, x_115); -lean_ctor_set(x_2, 0, x_39); -x_119 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_119, 0, x_2); -x_120 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_120, 0, x_119); -lean_ctor_set(x_120, 1, x_95); -return x_120; -} -} -else -{ -uint8_t x_121; -lean_dec(x_36); -lean_dec(x_32); -lean_free_object(x_2); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -x_121 = !lean_is_exclusive(x_38); -if (x_121 == 0) -{ -return x_38; -} -else -{ -lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_122 = lean_ctor_get(x_38, 0); -x_123 = lean_ctor_get(x_38, 1); -lean_inc(x_123); -lean_inc(x_122); -lean_dec(x_38); -x_124 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_124, 0, x_122); -lean_ctor_set(x_124, 1, x_123); -return x_124; -} -} -} -else -{ -uint8_t x_125; -lean_dec(x_32); -lean_free_object(x_2); -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_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_125 = !lean_is_exclusive(x_35); -if (x_125 == 0) -{ -return x_35; -} -else -{ -lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_126 = lean_ctor_get(x_35, 0); -x_127 = lean_ctor_get(x_35, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_35); -x_128 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_128, 0, x_126); -lean_ctor_set(x_128, 1, x_127); -return x_128; -} -} -} -else -{ -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; -lean_dec(x_2); -x_129 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__2; -x_130 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_129, x_8, x_9, x_20); -x_131 = lean_ctor_get(x_130, 0); -lean_inc(x_131); -x_132 = lean_ctor_get(x_130, 1); -lean_inc(x_132); -lean_dec(x_130); -x_133 = lean_box(0); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_134 = l_Lean_PrettyPrinter_delab(x_1, x_133, x_6, x_7, x_8, x_9, x_132); -if (lean_obj_tag(x_134) == 0) -{ -lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_135 = lean_ctor_get(x_134, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_134, 1); -lean_inc(x_136); -lean_dec(x_134); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_131); -x_137 = l_Lean_Meta_DiscrTree_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(x_11, x_1, x_131, x_6, x_7, x_8, x_9, x_136); -if (lean_obj_tag(x_137) == 0) -{ -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; -x_138 = lean_ctor_get(x_137, 0); -lean_inc(x_138); -x_139 = lean_ctor_get(x_137, 1); -lean_inc(x_139); -lean_dec(x_137); -lean_inc(x_8); -x_140 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_139); -x_141 = lean_ctor_get(x_140, 0); -lean_inc(x_141); -x_142 = lean_ctor_get(x_140, 1); -lean_inc(x_142); -lean_dec(x_140); -x_143 = lean_st_ref_get(x_9, x_142); -x_144 = lean_ctor_get(x_143, 1); -lean_inc(x_144); -lean_dec(x_143); -x_145 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; -lean_inc(x_141); -x_146 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_146, 0, x_141); -lean_ctor_set(x_146, 1, x_145); -lean_inc(x_131); -x_147 = lean_mk_syntax_ident(x_131); -x_148 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -lean_inc(x_147); -x_149 = lean_array_push(x_148, x_147); -x_150 = lean_box(2); -x_151 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_152 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_152, 0, x_150); -lean_ctor_set(x_152, 1, x_151); -lean_ctor_set(x_152, 2, x_149); -x_153 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -x_154 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_154, 0, x_141); +x_107 = lean_array_get_size(x_106); +x_108 = lean_usize_of_nat(x_107); +lean_dec(x_107); +x_109 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_110 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_111 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18; +x_112 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23; +lean_inc(x_69); +x_113 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(x_109, x_52, x_69, x_81, x_110, x_100, x_111, x_112, x_91, x_108, x_17, x_106); +x_114 = l_Array_append___rarg(x_79, x_113); +x_115 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_115, 0, x_55); +lean_ctor_set(x_115, 1, x_81); +lean_ctor_set(x_115, 2, x_114); +x_116 = lean_array_push(x_91, x_115); +x_117 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33; +x_118 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_118, 0, x_55); +lean_ctor_set(x_118, 1, x_117); +lean_ctor_set(x_118, 2, x_116); +x_119 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +x_120 = lean_array_push(x_119, x_105); +x_121 = lean_array_push(x_120, x_100); +x_122 = lean_array_push(x_121, x_118); +x_123 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_123, 0, x_55); +lean_ctor_set(x_123, 1, x_81); +lean_ctor_set(x_123, 2, x_122); +x_124 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__36; +lean_inc(x_69); +x_125 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_125, 0, x_69); +lean_ctor_set(x_125, 1, x_124); +x_126 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; +lean_inc(x_71); +lean_inc(x_76); +x_127 = l_Lean_addMacroScope(x_76, x_126, x_71); +x_128 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__41; +x_129 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__45; +lean_inc(x_69); +x_130 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_130, 0, x_69); +lean_ctor_set(x_130, 1, x_128); +lean_ctor_set(x_130, 2, x_127); +lean_ctor_set(x_130, 3, x_129); +x_131 = lean_array_push(x_52, x_130); +x_132 = lean_array_push(x_131, x_100); +x_133 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__38; +x_134 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_134, 0, x_55); +lean_ctor_set(x_134, 1, x_133); +lean_ctor_set(x_134, 2, x_132); +x_135 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; +lean_inc(x_69); +x_136 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_136, 0, x_69); +lean_ctor_set(x_136, 1, x_135); +x_137 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50; +lean_inc(x_71); +lean_inc(x_76); +x_138 = l_Lean_addMacroScope(x_76, x_137, x_71); +x_139 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49; +x_140 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53; +lean_inc(x_69); +x_141 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_141, 0, x_69); +lean_ctor_set(x_141, 1, x_139); +lean_ctor_set(x_141, 2, x_138); +lean_ctor_set(x_141, 3, x_140); +x_142 = lean_array_push(x_52, x_141); +x_143 = lean_array_push(x_142, x_100); +x_144 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_144, 0, x_55); +lean_ctor_set(x_144, 1, x_133); +lean_ctor_set(x_144, 2, x_143); +x_145 = lean_array_push(x_119, x_134); +x_146 = lean_array_push(x_145, x_136); +x_147 = lean_array_push(x_146, x_144); +x_148 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_148, 0, x_55); +lean_ctor_set(x_148, 1, x_81); +lean_ctor_set(x_148, 2, x_147); +x_149 = lean_array_push(x_52, x_125); +x_150 = lean_array_push(x_149, x_148); +x_151 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_151, 0, x_55); +lean_ctor_set(x_151, 1, x_81); +lean_ctor_set(x_151, 2, x_150); +x_152 = lean_array_push(x_91, x_151); +x_153 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35; +x_154 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_154, 0, x_55); lean_ctor_set(x_154, 1, x_153); -x_155 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_156 = lean_array_push(x_155, x_146); -x_157 = lean_array_push(x_156, x_152); -x_158 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_159 = lean_array_push(x_157, x_158); -x_160 = lean_array_push(x_159, x_158); -x_161 = lean_array_push(x_160, x_154); -x_162 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; -x_163 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_163, 0, x_150); -lean_ctor_set(x_163, 1, x_162); -lean_ctor_set(x_163, 2, x_161); -x_164 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_144); -x_165 = lean_ctor_get(x_164, 0); -lean_inc(x_165); -x_166 = lean_ctor_get(x_164, 1); -lean_inc(x_166); -lean_dec(x_164); -x_167 = lean_st_ref_get(x_9, x_166); -lean_dec(x_9); -x_168 = lean_ctor_get(x_167, 1); -lean_inc(x_168); -if (lean_is_exclusive(x_167)) { - lean_ctor_release(x_167, 0); - lean_ctor_release(x_167, 1); - x_169 = x_167; -} else { - lean_dec_ref(x_167); - x_169 = lean_box(0); -} -x_170 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; -lean_inc(x_165); -x_171 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_171, 0, x_165); -lean_ctor_set(x_171, 1, x_170); -x_172 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_173 = lean_array_push(x_172, x_135); -x_174 = lean_array_push(x_173, x_147); -x_175 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_175, 0, x_150); -lean_ctor_set(x_175, 1, x_151); -lean_ctor_set(x_175, 2, x_174); -x_176 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2; -x_177 = lean_array_push(x_176, x_175); -x_178 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +lean_ctor_set(x_154, 2, x_152); +x_155 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116; +x_156 = lean_array_push(x_155, x_94); +x_157 = lean_array_push(x_156, x_103); +x_158 = lean_array_push(x_157, x_100); +x_159 = lean_array_push(x_158, x_100); +x_160 = lean_array_push(x_159, x_100); +x_161 = lean_array_push(x_160, x_123); +x_162 = lean_array_push(x_161, x_154); +x_163 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__25; +x_164 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_164, 0, x_55); +lean_ctor_set(x_164, 1, x_163); +lean_ctor_set(x_164, 2, x_162); +x_165 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__54; +x_166 = lean_array_push(x_165, x_164); +x_167 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__10; +x_168 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_168, 0, x_55); +lean_ctor_set(x_168, 1, x_167); +lean_ctor_set(x_168, 2, x_166); +x_169 = lean_array_push(x_119, x_86); +lean_inc(x_88); +x_170 = lean_array_push(x_169, x_88); +x_171 = lean_array_push(x_170, x_168); +x_172 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__13; +x_173 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_173, 0, x_55); +lean_ctor_set(x_173, 1, x_172); +lean_ctor_set(x_173, 2, x_171); +x_174 = l_Array_append___rarg(x_5, x_4); +x_175 = l_Array_append___rarg(x_174, x_6); +x_176 = l_Array_append___rarg(x_79, x_175); +x_177 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_177, 0, x_55); +lean_ctor_set(x_177, 1, x_81); +lean_ctor_set(x_177, 2, x_176); +x_178 = lean_array_push(x_83, x_177); x_179 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_179, 0, x_150); -lean_ctor_set(x_179, 1, x_178); -lean_ctor_set(x_179, 2, x_177); -x_180 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; +lean_ctor_set(x_179, 0, x_55); +lean_ctor_set(x_179, 1, x_85); +lean_ctor_set(x_179, 2, x_178); +x_180 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119; +lean_inc(x_69); x_181 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_181, 0, x_165); +lean_ctor_set(x_181, 0, x_69); lean_ctor_set(x_181, 1, x_180); -x_182 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_183 = lean_array_push(x_182, x_171); -x_184 = lean_array_push(x_183, x_158); -x_185 = lean_array_push(x_184, x_179); -x_186 = lean_array_push(x_185, x_181); -x_187 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58; -x_188 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_188, 0, x_150); -lean_ctor_set(x_188, 1, x_187); -lean_ctor_set(x_188, 2, x_186); -x_189 = lean_array_push(x_12, x_131); -x_190 = lean_array_push(x_172, x_163); -x_191 = lean_array_push(x_190, x_188); -x_192 = l_Array_append___rarg(x_13, x_191); -x_193 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_193, 0, x_138); -lean_ctor_set(x_193, 1, x_189); +x_182 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; +lean_inc(x_69); +x_183 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_183, 0, x_69); +lean_ctor_set(x_183, 1, x_182); +x_184 = lean_array_push(x_52, x_183); +x_185 = lean_array_push(x_184, x_100); +x_186 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__57; +x_187 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_187, 0, x_55); +lean_ctor_set(x_187, 1, x_186); +lean_ctor_set(x_187, 2, x_185); +x_188 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58; +x_189 = lean_array_push(x_188, x_187); +x_190 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__121; +x_191 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_191, 0, x_55); +lean_ctor_set(x_191, 1, x_190); +lean_ctor_set(x_191, 2, x_189); +x_192 = lean_array_push(x_91, x_191); +x_193 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_193, 0, x_55); +lean_ctor_set(x_193, 1, x_81); lean_ctor_set(x_193, 2, x_192); -lean_ctor_set(x_193, 3, x_14); -lean_ctor_set(x_193, 4, x_15); -lean_ctor_set(x_193, 5, x_16); -x_194 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_194, 0, x_193); -if (lean_is_scalar(x_169)) { - x_195 = lean_alloc_ctor(0, 2, 0); -} else { - x_195 = x_169; -} -lean_ctor_set(x_195, 0, x_194); -lean_ctor_set(x_195, 1, x_168); -return x_195; -} -else -{ -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; -lean_dec(x_135); -lean_dec(x_131); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -x_196 = lean_ctor_get(x_137, 0); -lean_inc(x_196); -x_197 = lean_ctor_get(x_137, 1); -lean_inc(x_197); -if (lean_is_exclusive(x_137)) { - lean_ctor_release(x_137, 0); - lean_ctor_release(x_137, 1); - x_198 = x_137; -} else { - lean_dec_ref(x_137); - x_198 = lean_box(0); -} -if (lean_is_scalar(x_198)) { - x_199 = lean_alloc_ctor(1, 2, 0); -} else { - x_199 = x_198; -} -lean_ctor_set(x_199, 0, x_196); -lean_ctor_set(x_199, 1, x_197); -return x_199; -} -} -else -{ -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; -lean_dec(x_131); -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_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_200 = lean_ctor_get(x_134, 0); -lean_inc(x_200); -x_201 = lean_ctor_get(x_134, 1); -lean_inc(x_201); -if (lean_is_exclusive(x_134)) { - lean_ctor_release(x_134, 0); - lean_ctor_release(x_134, 1); - x_202 = x_134; -} else { - lean_dec_ref(x_134); - x_202 = lean_box(0); -} -if (lean_is_scalar(x_202)) { - x_203 = lean_alloc_ctor(1, 2, 0); -} else { - x_203 = x_202; -} -lean_ctor_set(x_203, 0, x_200); -lean_ctor_set(x_203, 1, x_201); -return x_203; -} -} -} -} -else -{ -lean_object* x_204; lean_object* x_205; uint8_t x_206; -x_204 = lean_ctor_get(x_17, 0); -x_205 = lean_ctor_get(x_17, 1); -lean_inc(x_205); -lean_inc(x_204); -lean_dec(x_17); -x_206 = l_Array_isEmpty___rarg(x_204); -lean_dec(x_204); -if (x_206 == 0) -{ -lean_object* x_207; lean_object* x_208; -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_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_207 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_207, 0, x_2); -x_208 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_208, 0, x_207); -lean_ctor_set(x_208, 1, x_205); -return x_208; -} -else -{ -lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; -if (lean_is_exclusive(x_2)) { - lean_ctor_release(x_2, 0); - lean_ctor_release(x_2, 1); - lean_ctor_release(x_2, 2); - lean_ctor_release(x_2, 3); - lean_ctor_release(x_2, 4); - lean_ctor_release(x_2, 5); - x_209 = x_2; -} else { - lean_dec_ref(x_2); - x_209 = lean_box(0); -} -x_210 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__2; -x_211 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_210, x_8, x_9, x_205); -x_212 = lean_ctor_get(x_211, 0); -lean_inc(x_212); -x_213 = lean_ctor_get(x_211, 1); -lean_inc(x_213); -lean_dec(x_211); -x_214 = lean_box(0); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_215 = l_Lean_PrettyPrinter_delab(x_1, x_214, x_6, x_7, x_8, x_9, x_213); -if (lean_obj_tag(x_215) == 0) -{ -lean_object* x_216; lean_object* x_217; lean_object* x_218; -x_216 = lean_ctor_get(x_215, 0); -lean_inc(x_216); -x_217 = lean_ctor_get(x_215, 1); -lean_inc(x_217); -lean_dec(x_215); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_212); -x_218 = l_Lean_Meta_DiscrTree_insert___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(x_11, x_1, x_212, x_6, x_7, x_8, x_9, x_217); -if (lean_obj_tag(x_218) == 0) -{ -lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; -x_219 = lean_ctor_get(x_218, 0); -lean_inc(x_219); -x_220 = lean_ctor_get(x_218, 1); -lean_inc(x_220); -lean_dec(x_218); -lean_inc(x_8); -x_221 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_220); -x_222 = lean_ctor_get(x_221, 0); -lean_inc(x_222); -x_223 = lean_ctor_get(x_221, 1); -lean_inc(x_223); -lean_dec(x_221); -x_224 = lean_st_ref_get(x_9, x_223); -x_225 = lean_ctor_get(x_224, 1); -lean_inc(x_225); -lean_dec(x_224); -x_226 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; -lean_inc(x_222); -x_227 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_227, 0, x_222); -lean_ctor_set(x_227, 1, x_226); -lean_inc(x_212); -x_228 = lean_mk_syntax_ident(x_212); -x_229 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -lean_inc(x_228); -x_230 = lean_array_push(x_229, x_228); -x_231 = lean_box(2); -x_232 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_194 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; +lean_inc(x_69); +x_195 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_195, 0, x_69); +lean_ctor_set(x_195, 1, x_194); +x_196 = lean_array_push(x_119, x_181); +x_197 = lean_array_push(x_196, x_193); +x_198 = lean_array_push(x_197, x_195); +x_199 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__118; +x_200 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_200, 0, x_55); +lean_ctor_set(x_200, 1, x_199); +lean_ctor_set(x_200, 2, x_198); +x_201 = lean_array_push(x_91, x_200); +x_202 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_202, 0, x_55); +lean_ctor_set(x_202, 1, x_81); +lean_ctor_set(x_202, 2, x_201); +x_203 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17; +x_204 = lean_array_push(x_203, x_202); +x_205 = lean_array_push(x_204, x_100); +x_206 = lean_array_push(x_205, x_100); +x_207 = lean_array_push(x_206, x_100); +x_208 = lean_array_push(x_207, x_100); +x_209 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; +x_210 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_210, 0, x_55); +lean_ctor_set(x_210, 1, x_209); +lean_ctor_set(x_210, 2, x_208); +x_211 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23; +lean_inc(x_69); +x_212 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_212, 0, x_69); +lean_ctor_set(x_212, 1, x_211); +x_213 = lean_array_push(x_52, x_67); +x_214 = lean_array_push(x_213, x_100); +x_215 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_215, 0, x_55); +lean_ctor_set(x_215, 1, x_102); +lean_ctor_set(x_215, 2, x_214); +x_216 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; +lean_inc(x_69); +x_217 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_217, 0, x_69); +lean_ctor_set(x_217, 1, x_216); +x_218 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; +lean_inc(x_69); +x_219 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_219, 0, x_69); +lean_ctor_set(x_219, 1, x_218); +x_220 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; +lean_inc(x_71); +lean_inc(x_76); +x_221 = l_Lean_addMacroScope(x_76, x_220, x_71); +x_222 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; +x_223 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5; +lean_inc(x_69); +x_224 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_224, 0, x_69); +lean_ctor_set(x_224, 1, x_222); +lean_ctor_set(x_224, 2, x_221); +lean_ctor_set(x_224, 3, x_223); +x_225 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +lean_inc(x_69); +x_226 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_226, 0, x_69); +lean_ctor_set(x_226, 1, x_225); +x_227 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66; +lean_inc(x_69); +x_228 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_228, 0, x_69); +lean_ctor_set(x_228, 1, x_227); +x_229 = lean_array_push(x_91, x_228); +x_230 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__65; +x_231 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_231, 0, x_55); +lean_ctor_set(x_231, 1, x_230); +lean_ctor_set(x_231, 2, x_229); +x_232 = lean_array_push(x_91, x_231); x_233 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_233, 0, x_231); -lean_ctor_set(x_233, 1, x_232); -lean_ctor_set(x_233, 2, x_230); -x_234 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -x_235 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_235, 0, x_222); -lean_ctor_set(x_235, 1, x_234); -x_236 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_237 = lean_array_push(x_236, x_227); -x_238 = lean_array_push(x_237, x_233); -x_239 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_240 = lean_array_push(x_238, x_239); -x_241 = lean_array_push(x_240, x_239); -x_242 = lean_array_push(x_241, x_235); -x_243 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; -x_244 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_244, 0, x_231); -lean_ctor_set(x_244, 1, x_243); -lean_ctor_set(x_244, 2, x_242); -x_245 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_8, x_9, x_225); -x_246 = lean_ctor_get(x_245, 0); -lean_inc(x_246); -x_247 = lean_ctor_get(x_245, 1); -lean_inc(x_247); -lean_dec(x_245); -x_248 = lean_st_ref_get(x_9, x_247); -lean_dec(x_9); -x_249 = lean_ctor_get(x_248, 1); -lean_inc(x_249); -if (lean_is_exclusive(x_248)) { - lean_ctor_release(x_248, 0); - lean_ctor_release(x_248, 1); - x_250 = x_248; -} else { - lean_dec_ref(x_248); - x_250 = lean_box(0); -} -x_251 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; -lean_inc(x_246); -x_252 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_252, 0, x_246); -lean_ctor_set(x_252, 1, x_251); -x_253 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_254 = lean_array_push(x_253, x_216); -x_255 = lean_array_push(x_254, x_228); -x_256 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_256, 0, x_231); -lean_ctor_set(x_256, 1, x_232); -lean_ctor_set(x_256, 2, x_255); -x_257 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2; -x_258 = lean_array_push(x_257, x_256); -x_259 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_260 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_260, 0, x_231); -lean_ctor_set(x_260, 1, x_259); -lean_ctor_set(x_260, 2, x_258); -x_261 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; -x_262 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_262, 0, x_246); -lean_ctor_set(x_262, 1, x_261); -x_263 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_264 = lean_array_push(x_263, x_252); -x_265 = lean_array_push(x_264, x_239); -x_266 = lean_array_push(x_265, x_260); -x_267 = lean_array_push(x_266, x_262); -x_268 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__58; -x_269 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_269, 0, x_231); -lean_ctor_set(x_269, 1, x_268); -lean_ctor_set(x_269, 2, x_267); -x_270 = lean_array_push(x_12, x_212); -x_271 = lean_array_push(x_253, x_244); -x_272 = lean_array_push(x_271, x_269); -x_273 = l_Array_append___rarg(x_13, x_272); -if (lean_is_scalar(x_209)) { - x_274 = lean_alloc_ctor(0, 6, 0); -} else { - x_274 = x_209; -} -lean_ctor_set(x_274, 0, x_219); -lean_ctor_set(x_274, 1, x_270); -lean_ctor_set(x_274, 2, x_273); -lean_ctor_set(x_274, 3, x_14); -lean_ctor_set(x_274, 4, x_15); -lean_ctor_set(x_274, 5, x_16); -x_275 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_275, 0, x_274); -if (lean_is_scalar(x_250)) { - x_276 = lean_alloc_ctor(0, 2, 0); -} else { - x_276 = x_250; -} -lean_ctor_set(x_276, 0, x_275); -lean_ctor_set(x_276, 1, x_249); -return x_276; -} -else -{ -lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; -lean_dec(x_216); -lean_dec(x_212); -lean_dec(x_209); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -x_277 = lean_ctor_get(x_218, 0); -lean_inc(x_277); -x_278 = lean_ctor_get(x_218, 1); -lean_inc(x_278); -if (lean_is_exclusive(x_218)) { - lean_ctor_release(x_218, 0); - lean_ctor_release(x_218, 1); - x_279 = x_218; -} else { - lean_dec_ref(x_218); - x_279 = lean_box(0); -} -if (lean_is_scalar(x_279)) { - x_280 = lean_alloc_ctor(1, 2, 0); -} else { - x_280 = x_279; -} -lean_ctor_set(x_280, 0, x_277); -lean_ctor_set(x_280, 1, x_278); -return x_280; -} -} -else -{ -lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; -lean_dec(x_212); -lean_dec(x_209); -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_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_281 = lean_ctor_get(x_215, 0); -lean_inc(x_281); -x_282 = lean_ctor_get(x_215, 1); -lean_inc(x_282); -if (lean_is_exclusive(x_215)) { - lean_ctor_release(x_215, 0); - lean_ctor_release(x_215, 1); - x_283 = x_215; -} else { - lean_dec_ref(x_215); - x_283 = lean_box(0); -} -if (lean_is_scalar(x_283)) { - x_284 = lean_alloc_ctor(1, 2, 0); -} else { - x_284 = x_283; -} -lean_ctor_set(x_284, 0, x_281); -lean_ctor_set(x_284, 1, x_282); -return x_284; -} -} -} -} -else -{ -uint8_t x_285; -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); +lean_ctor_set(x_233, 0, x_55); +lean_ctor_set(x_233, 1, x_81); +lean_ctor_set(x_233, 2, x_232); +x_234 = lean_array_push(x_99, x_233); +x_235 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; +x_236 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_236, 0, x_55); +lean_ctor_set(x_236, 1, x_235); +lean_ctor_set(x_236, 2, x_234); +x_237 = lean_array_push(x_52, x_236); +x_238 = lean_array_push(x_237, x_100); +x_239 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_239, 0, x_55); +lean_ctor_set(x_239, 1, x_81); +lean_ctor_set(x_239, 2, x_238); +x_240 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +lean_inc(x_69); +x_241 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_241, 0, x_69); +lean_ctor_set(x_241, 1, x_240); +x_242 = lean_array_push(x_119, x_226); +x_243 = lean_array_push(x_242, x_239); +x_244 = lean_array_push(x_243, x_241); +x_245 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; +x_246 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_246, 0, x_55); +lean_ctor_set(x_246, 1, x_245); +lean_ctor_set(x_246, 2, x_244); +x_247 = lean_array_push(x_52, x_62); +x_248 = lean_array_push(x_247, x_246); +x_249 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_249, 0, x_55); +lean_ctor_set(x_249, 1, x_81); +lean_ctor_set(x_249, 2, x_248); +x_250 = lean_array_push(x_52, x_224); +x_251 = lean_array_push(x_250, x_249); +x_252 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_252, 0, x_55); +lean_ctor_set(x_252, 1, x_235); +lean_ctor_set(x_252, 2, x_251); +x_253 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69; +lean_inc(x_69); +x_254 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_254, 0, x_69); +lean_ctor_set(x_254, 1, x_253); +x_255 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72; +lean_inc(x_69); +x_256 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_256, 0, x_69); +lean_ctor_set(x_256, 1, x_255); +x_257 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86; +lean_inc(x_71); +lean_inc(x_76); +x_258 = l_Lean_addMacroScope(x_76, x_257, x_71); +x_259 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +x_260 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__76; +lean_inc(x_69); +x_261 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_261, 0, x_69); +lean_ctor_set(x_261, 1, x_259); +lean_ctor_set(x_261, 2, x_258); +lean_ctor_set(x_261, 3, x_260); +x_262 = lean_array_push(x_52, x_261); +x_263 = lean_array_push(x_262, x_100); +x_264 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__74; +x_265 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_265, 0, x_55); +lean_ctor_set(x_265, 1, x_264); +lean_ctor_set(x_265, 2, x_263); +x_266 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__77; +lean_inc(x_69); +x_267 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_267, 0, x_69); +lean_ctor_set(x_267, 1, x_266); +x_268 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9; +lean_inc(x_71); +lean_inc(x_76); +x_269 = l_Lean_addMacroScope(x_76, x_268, x_71); +x_270 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8; +lean_inc(x_69); +x_271 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_271, 0, x_69); +lean_ctor_set(x_271, 1, x_270); +lean_ctor_set(x_271, 2, x_269); +lean_ctor_set(x_271, 3, x_46); +x_272 = lean_array_push(x_91, x_271); +x_273 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_273, 0, x_55); +lean_ctor_set(x_273, 1, x_81); +lean_ctor_set(x_273, 2, x_272); +x_274 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__81; +lean_inc(x_69); +x_275 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_275, 0, x_69); +lean_ctor_set(x_275, 1, x_274); +x_276 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__84; +lean_inc(x_69); +x_277 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_277, 0, x_69); +lean_ctor_set(x_277, 1, x_276); +x_278 = lean_array_get_size(x_30); +x_279 = lean_usize_of_nat(x_278); +lean_dec(x_278); +x_280 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__73; +x_281 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_46, x_109, x_280, x_279, x_17, x_30); +x_282 = lean_array_get_size(x_281); +x_283 = lean_usize_of_nat(x_282); +lean_dec(x_282); +x_284 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(x_283, x_17, x_281); +x_285 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__85; +x_286 = l_Lean_mkSepArray(x_284, x_285); +lean_dec(x_284); +x_287 = l_Array_append___rarg(x_79, x_286); +x_288 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_288, 0, x_55); +lean_ctor_set(x_288, 1, x_81); +lean_ctor_set(x_288, 2, x_287); +x_289 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89; +lean_inc(x_69); +x_290 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_290, 0, x_69); +lean_ctor_set(x_290, 1, x_289); +x_291 = lean_array_push(x_111, x_256); +x_292 = lean_array_push(x_291, x_100); +lean_inc(x_292); +x_293 = lean_array_push(x_292, x_288); +x_294 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__88; +x_295 = lean_array_push(x_293, x_294); +x_296 = lean_array_push(x_295, x_100); +lean_inc(x_290); +x_297 = lean_array_push(x_296, x_290); +x_298 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__71; +x_299 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_299, 0, x_55); +lean_ctor_set(x_299, 1, x_298); +lean_ctor_set(x_299, 2, x_297); +x_300 = lean_array_push(x_91, x_299); +x_301 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_301, 0, x_55); +lean_ctor_set(x_301, 1, x_81); +lean_ctor_set(x_301, 2, x_300); +x_302 = lean_array_push(x_52, x_277); +lean_inc(x_302); +x_303 = lean_array_push(x_302, x_301); +x_304 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__83; +x_305 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_305, 0, x_55); +lean_ctor_set(x_305, 1, x_304); +lean_ctor_set(x_305, 2, x_303); +x_306 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_307 = lean_array_push(x_306, x_273); +x_308 = lean_array_push(x_307, x_100); +x_309 = lean_array_push(x_308, x_275); +lean_inc(x_309); +x_310 = lean_array_push(x_309, x_305); +x_311 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__80; +x_312 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_312, 0, x_55); +lean_ctor_set(x_312, 1, x_311); +lean_ctor_set(x_312, 2, x_310); +x_313 = lean_array_push(x_52, x_267); +lean_inc(x_313); +x_314 = lean_array_push(x_313, x_312); +x_315 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__78; +x_316 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_316, 0, x_55); +lean_ctor_set(x_316, 1, x_315); +lean_ctor_set(x_316, 2, x_314); +x_317 = lean_array_push(x_119, x_265); +lean_inc(x_217); +x_318 = lean_array_push(x_317, x_217); +x_319 = lean_array_push(x_318, x_316); +x_320 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_320, 0, x_55); +lean_ctor_set(x_320, 1, x_280); +lean_ctor_set(x_320, 2, x_319); +x_321 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__103; +x_322 = l_Lean_addMacroScope(x_76, x_321, x_71); +x_323 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__102; +x_324 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__91; +x_325 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_325, 0, x_69); +lean_ctor_set(x_325, 1, x_323); +lean_ctor_set(x_325, 2, x_322); +lean_ctor_set(x_325, 3, x_324); +x_326 = lean_array_push(x_52, x_325); +x_327 = lean_array_push(x_326, x_100); +x_328 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_328, 0, x_55); +lean_ctor_set(x_328, 1, x_264); +lean_ctor_set(x_328, 2, x_327); +x_329 = lean_array_get_size(x_34); +x_330 = lean_usize_of_nat(x_329); +lean_dec(x_329); +x_331 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(x_46, x_109, x_280, x_330, x_17, x_34); +x_332 = lean_array_get_size(x_331); +x_333 = lean_usize_of_nat(x_332); +lean_dec(x_332); +x_334 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(x_333, x_17, x_331); +x_335 = l_Lean_mkSepArray(x_334, x_285); +lean_dec(x_334); +x_336 = l_Array_append___rarg(x_79, x_335); +x_337 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_337, 0, x_55); +lean_ctor_set(x_337, 1, x_81); +lean_ctor_set(x_337, 2, x_336); +lean_inc(x_292); +x_338 = lean_array_push(x_292, x_337); +x_339 = lean_array_push(x_338, x_294); +x_340 = lean_array_push(x_339, x_100); +lean_inc(x_290); +x_341 = lean_array_push(x_340, x_290); +x_342 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_342, 0, x_55); +lean_ctor_set(x_342, 1, x_298); +lean_ctor_set(x_342, 2, x_341); +x_343 = lean_array_push(x_91, x_342); +x_344 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_344, 0, x_55); +lean_ctor_set(x_344, 1, x_81); +lean_ctor_set(x_344, 2, x_343); +x_345 = lean_array_push(x_302, x_344); +x_346 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_346, 0, x_55); +lean_ctor_set(x_346, 1, x_304); +lean_ctor_set(x_346, 2, x_345); +x_347 = lean_array_push(x_309, x_346); +x_348 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_348, 0, x_55); +lean_ctor_set(x_348, 1, x_311); +lean_ctor_set(x_348, 2, x_347); +x_349 = lean_array_push(x_313, x_348); +x_350 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_350, 0, x_55); +lean_ctor_set(x_350, 1, x_315); +lean_ctor_set(x_350, 2, x_349); +x_351 = lean_array_push(x_119, x_328); +lean_inc(x_217); +x_352 = lean_array_push(x_351, x_217); +x_353 = lean_array_push(x_352, x_350); +x_354 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_354, 0, x_55); +lean_ctor_set(x_354, 1, x_280); +lean_ctor_set(x_354, 2, x_353); +x_355 = lean_array_push(x_306, x_320); +x_356 = lean_array_push(x_355, x_100); +x_357 = lean_array_push(x_356, x_354); +x_358 = lean_array_push(x_357, x_100); +x_359 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_359, 0, x_55); +lean_ctor_set(x_359, 1, x_81); +lean_ctor_set(x_359, 2, x_358); +x_360 = lean_array_push(x_292, x_359); +x_361 = lean_array_push(x_360, x_294); +x_362 = lean_array_push(x_361, x_100); +x_363 = lean_array_push(x_362, x_290); +x_364 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_364, 0, x_55); +lean_ctor_set(x_364, 1, x_298); +lean_ctor_set(x_364, 2, x_363); +x_365 = lean_array_push(x_52, x_254); +x_366 = lean_array_push(x_365, x_364); +x_367 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__68; +x_368 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_368, 0, x_55); +lean_ctor_set(x_368, 1, x_367); +lean_ctor_set(x_368, 2, x_366); +x_369 = lean_array_push(x_119, x_219); +x_370 = lean_array_push(x_369, x_252); +x_371 = lean_array_push(x_370, x_368); +x_372 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__63; +x_373 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_373, 0, x_55); +lean_ctor_set(x_373, 1, x_372); +lean_ctor_set(x_373, 2, x_371); +x_374 = lean_array_push(x_119, x_217); +x_375 = lean_array_push(x_374, x_373); +x_376 = lean_array_push(x_375, x_100); +x_377 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__150; +x_378 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_378, 0, x_55); +lean_ctor_set(x_378, 1, x_377); +lean_ctor_set(x_378, 2, x_376); +x_379 = lean_array_push(x_155, x_212); +x_380 = lean_array_push(x_379, x_215); +x_381 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__61; +x_382 = lean_array_push(x_380, x_381); +x_383 = lean_array_push(x_382, x_378); +x_384 = lean_array_push(x_383, x_100); +x_385 = lean_array_push(x_384, x_100); +x_386 = lean_array_push(x_385, x_100); +x_387 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__24; +x_388 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_388, 0, x_55); +lean_ctor_set(x_388, 1, x_387); +lean_ctor_set(x_388, 2, x_386); +x_389 = lean_array_push(x_52, x_210); +x_390 = lean_array_push(x_389, x_388); +x_391 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_391, 0, x_55); +lean_ctor_set(x_391, 1, x_167); +lean_ctor_set(x_391, 2, x_390); +x_392 = lean_array_push(x_119, x_179); +x_393 = lean_array_push(x_392, x_88); +x_394 = lean_array_push(x_393, x_391); +x_395 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_395, 0, x_55); +lean_ctor_set(x_395, 1, x_172); +lean_ctor_set(x_395, 2, x_394); +x_396 = lean_array_push(x_52, x_173); +x_397 = lean_array_push(x_396, x_395); +x_398 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_398, 0, x_55); +lean_ctor_set(x_398, 1, x_81); +lean_ctor_set(x_398, 2, x_397); +lean_ctor_set(x_72, 0, x_398); +return x_72; +} +else +{ +lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; size_t x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; lean_object* x_570; lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; size_t x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; size_t x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; size_t x_656; lean_object* x_657; lean_object* x_658; size_t x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; lean_object* x_677; lean_object* x_678; lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; lean_object* x_713; lean_object* x_714; lean_object* x_715; lean_object* x_716; lean_object* x_717; lean_object* x_718; lean_object* x_719; lean_object* x_720; lean_object* x_721; lean_object* x_722; lean_object* x_723; lean_object* x_724; lean_object* x_725; +x_399 = lean_ctor_get(x_72, 0); +x_400 = lean_ctor_get(x_72, 1); +lean_inc(x_400); +lean_inc(x_399); +lean_dec(x_72); +x_401 = lean_ctor_get(x_399, 0); +lean_inc(x_401); +lean_dec(x_399); +x_402 = lean_environment_main_module(x_401); +x_403 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14; +lean_inc(x_69); +x_404 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_404, 0, x_69); +lean_ctor_set(x_404, 1, x_403); +x_405 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +lean_inc(x_4); +x_406 = l_Array_append___rarg(x_405, x_4); +x_407 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_408 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_408, 0, x_55); +lean_ctor_set(x_408, 1, x_407); +lean_ctor_set(x_408, 2, x_406); +x_409 = lean_array_push(x_52, x_404); +lean_inc(x_409); +x_410 = lean_array_push(x_409, x_408); +x_411 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__15; +x_412 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_412, 0, x_55); +lean_ctor_set(x_412, 1, x_411); +lean_ctor_set(x_412, 2, x_410); +x_413 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12; +lean_inc(x_69); +x_414 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_414, 0, x_69); +lean_ctor_set(x_414, 1, x_413); +x_415 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__24; +lean_inc(x_69); +x_416 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_416, 0, x_69); +lean_ctor_set(x_416, 1, x_415); +x_417 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_418 = lean_array_push(x_417, x_416); +x_419 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__27; +x_420 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_420, 0, x_55); +lean_ctor_set(x_420, 1, x_419); +lean_ctor_set(x_420, 2, x_418); +x_421 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__31; +lean_inc(x_71); +lean_inc(x_402); +x_422 = l_Lean_addMacroScope(x_402, x_421, x_71); +x_423 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__30; +lean_inc(x_69); +x_424 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_424, 0, x_69); +lean_ctor_set(x_424, 1, x_423); +lean_ctor_set(x_424, 2, x_422); +lean_ctor_set(x_424, 3, x_46); +x_425 = lean_array_push(x_52, x_424); +x_426 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +lean_inc(x_425); +x_427 = lean_array_push(x_425, x_426); +x_428 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; +x_429 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_429, 0, x_55); +lean_ctor_set(x_429, 1, x_428); +lean_ctor_set(x_429, 2, x_427); +x_430 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__76; +lean_inc(x_69); +x_431 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_431, 0, x_69); +lean_ctor_set(x_431, 1, x_430); +x_432 = l_Array_zip___rarg(x_24, x_23); +lean_dec(x_23); +lean_dec(x_24); +x_433 = lean_array_get_size(x_432); +x_434 = lean_usize_of_nat(x_433); +lean_dec(x_433); +x_435 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_436 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; +x_437 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18; +x_438 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__23; +lean_inc(x_69); +x_439 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(x_435, x_52, x_69, x_407, x_436, x_426, x_437, x_438, x_417, x_434, x_17, x_432); +x_440 = l_Array_append___rarg(x_405, x_439); +x_441 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_441, 0, x_55); +lean_ctor_set(x_441, 1, x_407); +lean_ctor_set(x_441, 2, x_440); +x_442 = lean_array_push(x_417, x_441); +x_443 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33; +x_444 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_444, 0, x_55); +lean_ctor_set(x_444, 1, x_443); +lean_ctor_set(x_444, 2, x_442); +x_445 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +x_446 = lean_array_push(x_445, x_431); +x_447 = lean_array_push(x_446, x_426); +x_448 = lean_array_push(x_447, x_444); +x_449 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_449, 0, x_55); +lean_ctor_set(x_449, 1, x_407); +lean_ctor_set(x_449, 2, x_448); +x_450 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__36; +lean_inc(x_69); +x_451 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_451, 0, x_69); +lean_ctor_set(x_451, 1, x_450); +x_452 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; +lean_inc(x_71); +lean_inc(x_402); +x_453 = l_Lean_addMacroScope(x_402, x_452, x_71); +x_454 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__41; +x_455 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__45; +lean_inc(x_69); +x_456 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_456, 0, x_69); +lean_ctor_set(x_456, 1, x_454); +lean_ctor_set(x_456, 2, x_453); +lean_ctor_set(x_456, 3, x_455); +x_457 = lean_array_push(x_52, x_456); +x_458 = lean_array_push(x_457, x_426); +x_459 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__38; +x_460 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_460, 0, x_55); +lean_ctor_set(x_460, 1, x_459); +lean_ctor_set(x_460, 2, x_458); +x_461 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; +lean_inc(x_69); +x_462 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_462, 0, x_69); +lean_ctor_set(x_462, 1, x_461); +x_463 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50; +lean_inc(x_71); +lean_inc(x_402); +x_464 = l_Lean_addMacroScope(x_402, x_463, x_71); +x_465 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49; +x_466 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53; +lean_inc(x_69); +x_467 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_467, 0, x_69); +lean_ctor_set(x_467, 1, x_465); +lean_ctor_set(x_467, 2, x_464); +lean_ctor_set(x_467, 3, x_466); +x_468 = lean_array_push(x_52, x_467); +x_469 = lean_array_push(x_468, x_426); +x_470 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_470, 0, x_55); +lean_ctor_set(x_470, 1, x_459); +lean_ctor_set(x_470, 2, x_469); +x_471 = lean_array_push(x_445, x_460); +x_472 = lean_array_push(x_471, x_462); +x_473 = lean_array_push(x_472, x_470); +x_474 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_474, 0, x_55); +lean_ctor_set(x_474, 1, x_407); +lean_ctor_set(x_474, 2, x_473); +x_475 = lean_array_push(x_52, x_451); +x_476 = lean_array_push(x_475, x_474); +x_477 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_477, 0, x_55); +lean_ctor_set(x_477, 1, x_407); +lean_ctor_set(x_477, 2, x_476); +x_478 = lean_array_push(x_417, x_477); +x_479 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35; +x_480 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_480, 0, x_55); +lean_ctor_set(x_480, 1, x_479); +lean_ctor_set(x_480, 2, x_478); +x_481 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116; +x_482 = lean_array_push(x_481, x_420); +x_483 = lean_array_push(x_482, x_429); +x_484 = lean_array_push(x_483, x_426); +x_485 = lean_array_push(x_484, x_426); +x_486 = lean_array_push(x_485, x_426); +x_487 = lean_array_push(x_486, x_449); +x_488 = lean_array_push(x_487, x_480); +x_489 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__25; +x_490 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_490, 0, x_55); +lean_ctor_set(x_490, 1, x_489); +lean_ctor_set(x_490, 2, x_488); +x_491 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__54; +x_492 = lean_array_push(x_491, x_490); +x_493 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__10; +x_494 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_494, 0, x_55); +lean_ctor_set(x_494, 1, x_493); +lean_ctor_set(x_494, 2, x_492); +x_495 = lean_array_push(x_445, x_412); +lean_inc(x_414); +x_496 = lean_array_push(x_495, x_414); +x_497 = lean_array_push(x_496, x_494); +x_498 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__13; +x_499 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_499, 0, x_55); +lean_ctor_set(x_499, 1, x_498); +lean_ctor_set(x_499, 2, x_497); +x_500 = l_Array_append___rarg(x_5, x_4); +x_501 = l_Array_append___rarg(x_500, x_6); +x_502 = l_Array_append___rarg(x_405, x_501); +x_503 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_503, 0, x_55); +lean_ctor_set(x_503, 1, x_407); +lean_ctor_set(x_503, 2, x_502); +x_504 = lean_array_push(x_409, x_503); +x_505 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_505, 0, x_55); +lean_ctor_set(x_505, 1, x_411); +lean_ctor_set(x_505, 2, x_504); +x_506 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119; +lean_inc(x_69); +x_507 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_507, 0, x_69); +lean_ctor_set(x_507, 1, x_506); +x_508 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; +lean_inc(x_69); +x_509 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_509, 0, x_69); +lean_ctor_set(x_509, 1, x_508); +x_510 = lean_array_push(x_52, x_509); +x_511 = lean_array_push(x_510, x_426); +x_512 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__57; +x_513 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_513, 0, x_55); +lean_ctor_set(x_513, 1, x_512); +lean_ctor_set(x_513, 2, x_511); +x_514 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58; +x_515 = lean_array_push(x_514, x_513); +x_516 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__121; +x_517 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_517, 0, x_55); +lean_ctor_set(x_517, 1, x_516); +lean_ctor_set(x_517, 2, x_515); +x_518 = lean_array_push(x_417, x_517); +x_519 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_519, 0, x_55); +lean_ctor_set(x_519, 1, x_407); +lean_ctor_set(x_519, 2, x_518); +x_520 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; +lean_inc(x_69); +x_521 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_521, 0, x_69); +lean_ctor_set(x_521, 1, x_520); +x_522 = lean_array_push(x_445, x_507); +x_523 = lean_array_push(x_522, x_519); +x_524 = lean_array_push(x_523, x_521); +x_525 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__118; +x_526 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_526, 0, x_55); +lean_ctor_set(x_526, 1, x_525); +lean_ctor_set(x_526, 2, x_524); +x_527 = lean_array_push(x_417, x_526); +x_528 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_528, 0, x_55); +lean_ctor_set(x_528, 1, x_407); +lean_ctor_set(x_528, 2, x_527); +x_529 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17; +x_530 = lean_array_push(x_529, x_528); +x_531 = lean_array_push(x_530, x_426); +x_532 = lean_array_push(x_531, x_426); +x_533 = lean_array_push(x_532, x_426); +x_534 = lean_array_push(x_533, x_426); +x_535 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; +x_536 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_536, 0, x_55); +lean_ctor_set(x_536, 1, x_535); +lean_ctor_set(x_536, 2, x_534); +x_537 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23; +lean_inc(x_69); +x_538 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_538, 0, x_69); +lean_ctor_set(x_538, 1, x_537); +x_539 = lean_array_push(x_52, x_67); +x_540 = lean_array_push(x_539, x_426); +x_541 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_541, 0, x_55); +lean_ctor_set(x_541, 1, x_428); +lean_ctor_set(x_541, 2, x_540); +x_542 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; +lean_inc(x_69); +x_543 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_543, 0, x_69); +lean_ctor_set(x_543, 1, x_542); +x_544 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; +lean_inc(x_69); +x_545 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_545, 0, x_69); +lean_ctor_set(x_545, 1, x_544); +x_546 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; +lean_inc(x_71); +lean_inc(x_402); +x_547 = l_Lean_addMacroScope(x_402, x_546, x_71); +x_548 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; +x_549 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5; +lean_inc(x_69); +x_550 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_550, 0, x_69); +lean_ctor_set(x_550, 1, x_548); +lean_ctor_set(x_550, 2, x_547); +lean_ctor_set(x_550, 3, x_549); +x_551 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +lean_inc(x_69); +x_552 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_552, 0, x_69); +lean_ctor_set(x_552, 1, x_551); +x_553 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66; +lean_inc(x_69); +x_554 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_554, 0, x_69); +lean_ctor_set(x_554, 1, x_553); +x_555 = lean_array_push(x_417, x_554); +x_556 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__65; +x_557 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_557, 0, x_55); +lean_ctor_set(x_557, 1, x_556); +lean_ctor_set(x_557, 2, x_555); +x_558 = lean_array_push(x_417, x_557); +x_559 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_559, 0, x_55); +lean_ctor_set(x_559, 1, x_407); +lean_ctor_set(x_559, 2, x_558); +x_560 = lean_array_push(x_425, x_559); +x_561 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; +x_562 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_562, 0, x_55); +lean_ctor_set(x_562, 1, x_561); +lean_ctor_set(x_562, 2, x_560); +x_563 = lean_array_push(x_52, x_562); +x_564 = lean_array_push(x_563, x_426); +x_565 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_565, 0, x_55); +lean_ctor_set(x_565, 1, x_407); +lean_ctor_set(x_565, 2, x_564); +x_566 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +lean_inc(x_69); +x_567 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_567, 0, x_69); +lean_ctor_set(x_567, 1, x_566); +x_568 = lean_array_push(x_445, x_552); +x_569 = lean_array_push(x_568, x_565); +x_570 = lean_array_push(x_569, x_567); +x_571 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__51; +x_572 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_572, 0, x_55); +lean_ctor_set(x_572, 1, x_571); +lean_ctor_set(x_572, 2, x_570); +x_573 = lean_array_push(x_52, x_62); +x_574 = lean_array_push(x_573, x_572); +x_575 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_575, 0, x_55); +lean_ctor_set(x_575, 1, x_407); +lean_ctor_set(x_575, 2, x_574); +x_576 = lean_array_push(x_52, x_550); +x_577 = lean_array_push(x_576, x_575); +x_578 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_578, 0, x_55); +lean_ctor_set(x_578, 1, x_561); +lean_ctor_set(x_578, 2, x_577); +x_579 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69; +lean_inc(x_69); +x_580 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_580, 0, x_69); +lean_ctor_set(x_580, 1, x_579); +x_581 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72; +lean_inc(x_69); +x_582 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_582, 0, x_69); +lean_ctor_set(x_582, 1, x_581); +x_583 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86; +lean_inc(x_71); +lean_inc(x_402); +x_584 = l_Lean_addMacroScope(x_402, x_583, x_71); +x_585 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +x_586 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__76; +lean_inc(x_69); +x_587 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_587, 0, x_69); +lean_ctor_set(x_587, 1, x_585); +lean_ctor_set(x_587, 2, x_584); +lean_ctor_set(x_587, 3, x_586); +x_588 = lean_array_push(x_52, x_587); +x_589 = lean_array_push(x_588, x_426); +x_590 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__74; +x_591 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_591, 0, x_55); +lean_ctor_set(x_591, 1, x_590); +lean_ctor_set(x_591, 2, x_589); +x_592 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__77; +lean_inc(x_69); +x_593 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_593, 0, x_69); +lean_ctor_set(x_593, 1, x_592); +x_594 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9; +lean_inc(x_71); +lean_inc(x_402); +x_595 = l_Lean_addMacroScope(x_402, x_594, x_71); +x_596 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8; +lean_inc(x_69); +x_597 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_597, 0, x_69); +lean_ctor_set(x_597, 1, x_596); +lean_ctor_set(x_597, 2, x_595); +lean_ctor_set(x_597, 3, x_46); +x_598 = lean_array_push(x_417, x_597); +x_599 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_599, 0, x_55); +lean_ctor_set(x_599, 1, x_407); +lean_ctor_set(x_599, 2, x_598); +x_600 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__81; +lean_inc(x_69); +x_601 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_601, 0, x_69); +lean_ctor_set(x_601, 1, x_600); +x_602 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__84; +lean_inc(x_69); +x_603 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_603, 0, x_69); +lean_ctor_set(x_603, 1, x_602); +x_604 = lean_array_get_size(x_30); +x_605 = lean_usize_of_nat(x_604); +lean_dec(x_604); +x_606 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__73; +x_607 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_46, x_435, x_606, x_605, x_17, x_30); +x_608 = lean_array_get_size(x_607); +x_609 = lean_usize_of_nat(x_608); +lean_dec(x_608); +x_610 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(x_609, x_17, x_607); +x_611 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__85; +x_612 = l_Lean_mkSepArray(x_610, x_611); +lean_dec(x_610); +x_613 = l_Array_append___rarg(x_405, x_612); +x_614 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_614, 0, x_55); +lean_ctor_set(x_614, 1, x_407); +lean_ctor_set(x_614, 2, x_613); +x_615 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89; +lean_inc(x_69); +x_616 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_616, 0, x_69); +lean_ctor_set(x_616, 1, x_615); +x_617 = lean_array_push(x_437, x_582); +x_618 = lean_array_push(x_617, x_426); +lean_inc(x_618); +x_619 = lean_array_push(x_618, x_614); +x_620 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__88; +x_621 = lean_array_push(x_619, x_620); +x_622 = lean_array_push(x_621, x_426); +lean_inc(x_616); +x_623 = lean_array_push(x_622, x_616); +x_624 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__71; +x_625 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_625, 0, x_55); +lean_ctor_set(x_625, 1, x_624); +lean_ctor_set(x_625, 2, x_623); +x_626 = lean_array_push(x_417, x_625); +x_627 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_627, 0, x_55); +lean_ctor_set(x_627, 1, x_407); +lean_ctor_set(x_627, 2, x_626); +x_628 = lean_array_push(x_52, x_603); +lean_inc(x_628); +x_629 = lean_array_push(x_628, x_627); +x_630 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__83; +x_631 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_631, 0, x_55); +lean_ctor_set(x_631, 1, x_630); +lean_ctor_set(x_631, 2, x_629); +x_632 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_633 = lean_array_push(x_632, x_599); +x_634 = lean_array_push(x_633, x_426); +x_635 = lean_array_push(x_634, x_601); +lean_inc(x_635); +x_636 = lean_array_push(x_635, x_631); +x_637 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__80; +x_638 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_638, 0, x_55); +lean_ctor_set(x_638, 1, x_637); +lean_ctor_set(x_638, 2, x_636); +x_639 = lean_array_push(x_52, x_593); +lean_inc(x_639); +x_640 = lean_array_push(x_639, x_638); +x_641 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__78; +x_642 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_642, 0, x_55); +lean_ctor_set(x_642, 1, x_641); +lean_ctor_set(x_642, 2, x_640); +x_643 = lean_array_push(x_445, x_591); +lean_inc(x_543); +x_644 = lean_array_push(x_643, x_543); +x_645 = lean_array_push(x_644, x_642); +x_646 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_646, 0, x_55); +lean_ctor_set(x_646, 1, x_606); +lean_ctor_set(x_646, 2, x_645); +x_647 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__103; +x_648 = l_Lean_addMacroScope(x_402, x_647, x_71); +x_649 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__102; +x_650 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__91; +x_651 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_651, 0, x_69); +lean_ctor_set(x_651, 1, x_649); +lean_ctor_set(x_651, 2, x_648); +lean_ctor_set(x_651, 3, x_650); +x_652 = lean_array_push(x_52, x_651); +x_653 = lean_array_push(x_652, x_426); +x_654 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_654, 0, x_55); +lean_ctor_set(x_654, 1, x_590); +lean_ctor_set(x_654, 2, x_653); +x_655 = lean_array_get_size(x_34); +x_656 = lean_usize_of_nat(x_655); +lean_dec(x_655); +x_657 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(x_46, x_435, x_606, x_656, x_17, x_34); +x_658 = lean_array_get_size(x_657); +x_659 = lean_usize_of_nat(x_658); +lean_dec(x_658); +x_660 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(x_659, x_17, x_657); +x_661 = l_Lean_mkSepArray(x_660, x_611); +lean_dec(x_660); +x_662 = l_Array_append___rarg(x_405, x_661); +x_663 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_663, 0, x_55); +lean_ctor_set(x_663, 1, x_407); +lean_ctor_set(x_663, 2, x_662); +lean_inc(x_618); +x_664 = lean_array_push(x_618, x_663); +x_665 = lean_array_push(x_664, x_620); +x_666 = lean_array_push(x_665, x_426); +lean_inc(x_616); +x_667 = lean_array_push(x_666, x_616); +x_668 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_668, 0, x_55); +lean_ctor_set(x_668, 1, x_624); +lean_ctor_set(x_668, 2, x_667); +x_669 = lean_array_push(x_417, x_668); +x_670 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_670, 0, x_55); +lean_ctor_set(x_670, 1, x_407); +lean_ctor_set(x_670, 2, x_669); +x_671 = lean_array_push(x_628, x_670); +x_672 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_672, 0, x_55); +lean_ctor_set(x_672, 1, x_630); +lean_ctor_set(x_672, 2, x_671); +x_673 = lean_array_push(x_635, x_672); +x_674 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_674, 0, x_55); +lean_ctor_set(x_674, 1, x_637); +lean_ctor_set(x_674, 2, x_673); +x_675 = lean_array_push(x_639, x_674); +x_676 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_676, 0, x_55); +lean_ctor_set(x_676, 1, x_641); +lean_ctor_set(x_676, 2, x_675); +x_677 = lean_array_push(x_445, x_654); +lean_inc(x_543); +x_678 = lean_array_push(x_677, x_543); +x_679 = lean_array_push(x_678, x_676); +x_680 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_680, 0, x_55); +lean_ctor_set(x_680, 1, x_606); +lean_ctor_set(x_680, 2, x_679); +x_681 = lean_array_push(x_632, x_646); +x_682 = lean_array_push(x_681, x_426); +x_683 = lean_array_push(x_682, x_680); +x_684 = lean_array_push(x_683, x_426); +x_685 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_685, 0, x_55); +lean_ctor_set(x_685, 1, x_407); +lean_ctor_set(x_685, 2, x_684); +x_686 = lean_array_push(x_618, x_685); +x_687 = lean_array_push(x_686, x_620); +x_688 = lean_array_push(x_687, x_426); +x_689 = lean_array_push(x_688, x_616); +x_690 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_690, 0, x_55); +lean_ctor_set(x_690, 1, x_624); +lean_ctor_set(x_690, 2, x_689); +x_691 = lean_array_push(x_52, x_580); +x_692 = lean_array_push(x_691, x_690); +x_693 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__68; +x_694 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_694, 0, x_55); +lean_ctor_set(x_694, 1, x_693); +lean_ctor_set(x_694, 2, x_692); +x_695 = lean_array_push(x_445, x_545); +x_696 = lean_array_push(x_695, x_578); +x_697 = lean_array_push(x_696, x_694); +x_698 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__63; +x_699 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_699, 0, x_55); +lean_ctor_set(x_699, 1, x_698); +lean_ctor_set(x_699, 2, x_697); +x_700 = lean_array_push(x_445, x_543); +x_701 = lean_array_push(x_700, x_699); +x_702 = lean_array_push(x_701, x_426); +x_703 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__150; +x_704 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_704, 0, x_55); +lean_ctor_set(x_704, 1, x_703); +lean_ctor_set(x_704, 2, x_702); +x_705 = lean_array_push(x_481, x_538); +x_706 = lean_array_push(x_705, x_541); +x_707 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__61; +x_708 = lean_array_push(x_706, x_707); +x_709 = lean_array_push(x_708, x_704); +x_710 = lean_array_push(x_709, x_426); +x_711 = lean_array_push(x_710, x_426); +x_712 = lean_array_push(x_711, x_426); +x_713 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__24; +x_714 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_714, 0, x_55); +lean_ctor_set(x_714, 1, x_713); +lean_ctor_set(x_714, 2, x_712); +x_715 = lean_array_push(x_52, x_536); +x_716 = lean_array_push(x_715, x_714); +x_717 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_717, 0, x_55); +lean_ctor_set(x_717, 1, x_493); +lean_ctor_set(x_717, 2, x_716); +x_718 = lean_array_push(x_445, x_505); +x_719 = lean_array_push(x_718, x_414); +x_720 = lean_array_push(x_719, x_717); +x_721 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_721, 0, x_55); +lean_ctor_set(x_721, 1, x_498); +lean_ctor_set(x_721, 2, x_720); +x_722 = lean_array_push(x_52, x_499); +x_723 = lean_array_push(x_722, x_721); +x_724 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_724, 0, x_55); +lean_ctor_set(x_724, 1, x_407); +lean_ctor_set(x_724, 2, x_723); +x_725 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_725, 0, x_724); +lean_ctor_set(x_725, 1, x_400); +return x_725; +} +} +else +{ +uint8_t x_726; +lean_dec(x_34); +lean_dec(x_30); +lean_dec(x_24); +lean_dec(x_23); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_2); -lean_dec(x_1); -x_285 = !lean_is_exclusive(x_17); -if (x_285 == 0) -{ -return x_17; -} -else -{ -lean_object* x_286; lean_object* x_287; lean_object* x_288; -x_286 = lean_ctor_get(x_17, 0); -x_287 = lean_ctor_get(x_17, 1); -lean_inc(x_287); -lean_inc(x_286); -lean_dec(x_17); -x_288 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_288, 0, x_286); -lean_ctor_set(x_288, 1, x_287); -return x_288; -} -} -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("cross-argument dependencies are not supported (", 47); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" : ", 3); -return x_1; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(8u); -x_2 = l_Std_mkHashSetImp___rarg(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_4, x_3); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); lean_dec(x_6); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_5); -lean_ctor_set(x_14, 1, x_12); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_25; -x_15 = lean_array_uget(x_2, x_4); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_15); -x_25 = lean_infer_type(x_15, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_25) == 0) +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_726 = !lean_is_exclusive(x_38); +if (x_726 == 0) { -lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; 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_134; lean_object* x_135; lean_object* x_136; uint8_t x_137; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_53 = lean_st_ref_get(x_11, x_27); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = lean_st_ref_get(x_9, x_54); -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -lean_dec(x_55); -x_134 = lean_ctor_get(x_56, 0); -lean_inc(x_134); -lean_dec(x_56); -x_135 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__6; -x_136 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_136, 0, x_135); -lean_ctor_set(x_136, 1, x_134); -x_137 = l_Lean_Expr_hasFVar(x_26); -if (x_137 == 0) -{ -uint8_t x_138; -x_138 = l_Lean_Expr_hasMVar(x_26); -if (x_138 == 0) -{ -uint8_t x_139; -x_139 = 0; -x_58 = x_139; -x_59 = x_136; -goto block_133; +return x_38; } else { -lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; -lean_inc(x_26); -x_140 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_26, x_136); -x_141 = lean_ctor_get(x_140, 0); -lean_inc(x_141); -x_142 = lean_ctor_get(x_140, 1); -lean_inc(x_142); -lean_dec(x_140); -x_143 = lean_unbox(x_141); -lean_dec(x_141); -x_58 = x_143; -x_59 = x_142; -goto block_133; -} +lean_object* x_727; lean_object* x_728; lean_object* x_729; +x_727 = lean_ctor_get(x_38, 0); +x_728 = lean_ctor_get(x_38, 1); +lean_inc(x_728); +lean_inc(x_727); +lean_dec(x_38); +x_729 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_729, 0, x_727); +lean_ctor_set(x_729, 1, x_728); +return x_729; } -else -{ -lean_object* x_144; lean_object* x_145; lean_object* x_146; uint8_t x_147; -lean_inc(x_26); -x_144 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_26, x_136); -x_145 = lean_ctor_get(x_144, 0); -lean_inc(x_145); -x_146 = lean_ctor_get(x_144, 1); -lean_inc(x_146); -lean_dec(x_144); -x_147 = lean_unbox(x_145); -lean_dec(x_145); -x_58 = x_147; -x_59 = x_146; -goto block_133; } -block_52: -{ -if (x_28 == 0) -{ -lean_object* x_30; lean_object* x_31; -lean_dec(x_15); -x_30 = lean_box(0); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_31 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1(x_26, x_5, x_30, x_6, x_7, x_8, x_9, x_10, x_11, x_29); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; -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_16 = x_32; -x_17 = x_33; -goto block_24; } else { -uint8_t x_34; +uint8_t x_730; +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); lean_dec(x_6); -x_34 = !lean_is_exclusive(x_31); -if (x_34 == 0) -{ -return x_31; -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_31, 0); -x_36 = lean_ctor_get(x_31, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_31); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_dec(x_5); -x_38 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_38, 0, x_15); -x_39 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__2; -x_40 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_38); -x_41 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__4; -x_42 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -x_43 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_43, 0, x_26); -x_44 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -x_45 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__5; -x_46 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -x_47 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__4(x_46, x_6, x_7, x_8, x_9, x_10, x_11, x_29); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -x_48 = !lean_is_exclusive(x_47); -if (x_48 == 0) -{ -return x_47; -} -else -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_47, 0); -x_50 = lean_ctor_get(x_47, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_47); -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; -} -} -} -block_133: -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = lean_st_ref_get(x_11, x_57); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -lean_dec(x_61); -x_63 = lean_st_ref_take(x_9, x_62); -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -x_65 = lean_ctor_get_uint8(x_60, sizeof(void*)*8); -if (x_65 == 0) -{ -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_66 = lean_ctor_get(x_64, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_63, 1); -lean_inc(x_67); -lean_dec(x_63); -x_68 = lean_ctor_get(x_60, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_60, 1); -lean_inc(x_69); -x_70 = lean_ctor_get(x_60, 2); -lean_inc(x_70); -x_71 = lean_ctor_get(x_60, 3); -lean_inc(x_71); -x_72 = lean_ctor_get(x_60, 4); -lean_inc(x_72); -x_73 = lean_ctor_get(x_60, 5); -lean_inc(x_73); -x_74 = lean_ctor_get(x_60, 6); -lean_inc(x_74); -x_75 = lean_ctor_get(x_60, 7); -lean_inc(x_75); -lean_dec(x_60); -x_76 = !lean_is_exclusive(x_64); -if (x_76 == 0) -{ -lean_object* x_77; uint8_t x_78; -x_77 = lean_ctor_get(x_64, 0); -lean_dec(x_77); -x_78 = !lean_is_exclusive(x_66); -if (x_78 == 0) -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_79 = lean_ctor_get(x_66, 7); -lean_dec(x_79); -x_80 = lean_ctor_get(x_66, 6); -lean_dec(x_80); -x_81 = lean_ctor_get(x_66, 5); -lean_dec(x_81); -x_82 = lean_ctor_get(x_66, 4); -lean_dec(x_82); -x_83 = lean_ctor_get(x_66, 3); -lean_dec(x_83); -x_84 = lean_ctor_get(x_66, 2); -lean_dec(x_84); -x_85 = lean_ctor_get(x_66, 1); -lean_dec(x_85); -x_86 = lean_ctor_get(x_66, 0); -lean_dec(x_86); -lean_ctor_set(x_66, 7, x_75); -lean_ctor_set(x_66, 6, x_74); -lean_ctor_set(x_66, 5, x_73); -lean_ctor_set(x_66, 4, x_72); -lean_ctor_set(x_66, 3, x_71); -lean_ctor_set(x_66, 2, x_70); -lean_ctor_set(x_66, 1, x_69); -lean_ctor_set(x_66, 0, x_68); -x_87 = lean_st_ref_set(x_9, x_64, x_67); -x_88 = lean_ctor_get(x_87, 1); -lean_inc(x_88); -lean_dec(x_87); -x_28 = x_58; -x_29 = x_88; -goto block_52; -} -else +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_730 = !lean_is_exclusive(x_19); +if (x_730 == 0) { -uint8_t x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; -x_89 = lean_ctor_get_uint8(x_66, sizeof(void*)*8); -lean_dec(x_66); -x_90 = lean_alloc_ctor(0, 8, 1); -lean_ctor_set(x_90, 0, x_68); -lean_ctor_set(x_90, 1, x_69); -lean_ctor_set(x_90, 2, x_70); -lean_ctor_set(x_90, 3, x_71); -lean_ctor_set(x_90, 4, x_72); -lean_ctor_set(x_90, 5, x_73); -lean_ctor_set(x_90, 6, x_74); -lean_ctor_set(x_90, 7, x_75); -lean_ctor_set_uint8(x_90, sizeof(void*)*8, x_89); -lean_ctor_set(x_64, 0, x_90); -x_91 = lean_st_ref_set(x_9, x_64, x_67); -x_92 = lean_ctor_get(x_91, 1); -lean_inc(x_92); -lean_dec(x_91); -x_28 = x_58; -x_29 = x_92; -goto block_52; -} +return x_19; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_93 = lean_ctor_get(x_64, 1); -x_94 = lean_ctor_get(x_64, 2); -x_95 = lean_ctor_get(x_64, 3); -lean_inc(x_95); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_64); -x_96 = lean_ctor_get_uint8(x_66, sizeof(void*)*8); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - lean_ctor_release(x_66, 2); - lean_ctor_release(x_66, 3); - lean_ctor_release(x_66, 4); - lean_ctor_release(x_66, 5); - lean_ctor_release(x_66, 6); - lean_ctor_release(x_66, 7); - x_97 = x_66; -} else { - lean_dec_ref(x_66); - x_97 = lean_box(0); +lean_object* x_731; lean_object* x_732; lean_object* x_733; +x_731 = lean_ctor_get(x_19, 0); +x_732 = lean_ctor_get(x_19, 1); +lean_inc(x_732); +lean_inc(x_731); +lean_dec(x_19); +x_733 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_733, 0, x_731); +lean_ctor_set(x_733, 1, x_732); +return x_733; } -if (lean_is_scalar(x_97)) { - x_98 = lean_alloc_ctor(0, 8, 1); -} else { - x_98 = x_97; -} -lean_ctor_set(x_98, 0, x_68); -lean_ctor_set(x_98, 1, x_69); -lean_ctor_set(x_98, 2, x_70); -lean_ctor_set(x_98, 3, x_71); -lean_ctor_set(x_98, 4, x_72); -lean_ctor_set(x_98, 5, x_73); -lean_ctor_set(x_98, 6, x_74); -lean_ctor_set(x_98, 7, x_75); -lean_ctor_set_uint8(x_98, sizeof(void*)*8, x_96); -x_99 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_99, 0, x_98); -lean_ctor_set(x_99, 1, x_93); -lean_ctor_set(x_99, 2, x_94); -lean_ctor_set(x_99, 3, x_95); -x_100 = lean_st_ref_set(x_9, x_99, x_67); -x_101 = lean_ctor_get(x_100, 1); -lean_inc(x_101); -lean_dec(x_100); -x_28 = x_58; -x_29 = x_101; -goto block_52; } } -else -{ -lean_object* x_102; uint8_t x_103; -x_102 = lean_ctor_get(x_63, 1); -lean_inc(x_102); -lean_dec(x_63); -x_103 = !lean_is_exclusive(x_60); -if (x_103 == 0) -{ -uint8_t x_104; -x_104 = !lean_is_exclusive(x_64); -if (x_104 == 0) -{ -lean_object* x_105; uint8_t x_106; lean_object* x_107; lean_object* x_108; -x_105 = lean_ctor_get(x_64, 0); -lean_dec(x_105); -x_106 = 1; -lean_ctor_set_uint8(x_60, sizeof(void*)*8, x_106); -lean_ctor_set(x_64, 0, x_60); -x_107 = lean_st_ref_set(x_9, x_64, x_102); -x_108 = lean_ctor_get(x_107, 1); -lean_inc(x_108); -lean_dec(x_107); -x_28 = x_58; -x_29 = x_108; -goto block_52; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__1() { +_start: { -lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_109 = lean_ctor_get(x_64, 1); -x_110 = lean_ctor_get(x_64, 2); -x_111 = lean_ctor_get(x_64, 3); -lean_inc(x_111); -lean_inc(x_110); -lean_inc(x_109); -lean_dec(x_64); -x_112 = 1; -lean_ctor_set_uint8(x_60, sizeof(void*)*8, x_112); -x_113 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_113, 0, x_60); -lean_ctor_set(x_113, 1, x_109); -lean_ctor_set(x_113, 2, x_110); -lean_ctor_set(x_113, 3, x_111); -x_114 = lean_st_ref_set(x_9, x_113, x_102); -x_115 = lean_ctor_get(x_114, 1); -lean_inc(x_115); -lean_dec(x_114); -x_28 = x_58; -x_29 = x_115; -goto block_52; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Elab", 4); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__2() { +_start: { -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; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_116 = lean_ctor_get(x_60, 0); -x_117 = lean_ctor_get(x_60, 1); -x_118 = lean_ctor_get(x_60, 2); -x_119 = lean_ctor_get(x_60, 3); -x_120 = lean_ctor_get(x_60, 4); -x_121 = lean_ctor_get(x_60, 5); -x_122 = lean_ctor_get(x_60, 6); -x_123 = lean_ctor_get(x_60, 7); -lean_inc(x_123); -lean_inc(x_122); -lean_inc(x_121); -lean_inc(x_120); -lean_inc(x_119); -lean_inc(x_118); -lean_inc(x_117); -lean_inc(x_116); -lean_dec(x_60); -x_124 = lean_ctor_get(x_64, 1); -lean_inc(x_124); -x_125 = lean_ctor_get(x_64, 2); -lean_inc(x_125); -x_126 = lean_ctor_get(x_64, 3); -lean_inc(x_126); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - lean_ctor_release(x_64, 2); - lean_ctor_release(x_64, 3); - x_127 = x_64; -} else { - lean_dec_ref(x_64); - x_127 = lean_box(0); -} -x_128 = 1; -x_129 = lean_alloc_ctor(0, 8, 1); -lean_ctor_set(x_129, 0, x_116); -lean_ctor_set(x_129, 1, x_117); -lean_ctor_set(x_129, 2, x_118); -lean_ctor_set(x_129, 3, x_119); -lean_ctor_set(x_129, 4, x_120); -lean_ctor_set(x_129, 5, x_121); -lean_ctor_set(x_129, 6, x_122); -lean_ctor_set(x_129, 7, x_123); -lean_ctor_set_uint8(x_129, sizeof(void*)*8, x_128); -if (lean_is_scalar(x_127)) { - x_130 = lean_alloc_ctor(0, 4, 0); -} else { - x_130 = x_127; -} -lean_ctor_set(x_130, 0, x_129); -lean_ctor_set(x_130, 1, x_124); -lean_ctor_set(x_130, 2, x_125); -lean_ctor_set(x_130, 3, x_126); -x_131 = lean_st_ref_set(x_9, x_130, x_102); -x_132 = lean_ctor_get(x_131, 1); -lean_inc(x_132); -lean_dec(x_131); -x_28 = x_58; -x_29 = x_132; -goto block_52; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Deriving", 8); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__4() { +_start: { -uint8_t x_148; -lean_dec(x_15); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -x_148 = !lean_is_exclusive(x_25); -if (x_148 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__2; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__5() { +_start: { -return x_25; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__4; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__41; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__6() { +_start: { -lean_object* x_149; lean_object* x_150; lean_object* x_151; -x_149 = lean_ctor_get(x_25, 0); -x_150 = lean_ctor_get(x_25, 1); -lean_inc(x_150); -lean_inc(x_149); -lean_dec(x_25); -x_151 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_151, 0, x_149); -lean_ctor_set(x_151, 1, x_150); -return x_151; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("for structure ", 14); +return x_1; } } -block_24: +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__7() { +_start: { -if (lean_obj_tag(x_16) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__6; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__8() { +_start: { -lean_object* x_18; lean_object* x_19; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -return x_19; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(" with params ", 13); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9() { +_start: { -lean_object* x_20; size_t x_21; size_t x_22; -x_20 = lean_ctor_get(x_16, 0); -lean_inc(x_20); -lean_dec(x_16); -x_21 = 1; -x_22 = lean_usize_add(x_4, x_21); -x_4 = x_22; -x_5 = x_20; -x_12 = x_17; -goto _start; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__8; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("", 0); +return x_1; +} } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__10; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__34___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -if (lean_obj_tag(x_4) == 0) +lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_14 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__5; +x_38 = lean_st_ref_get(x_12, x_13); +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_39, 3); +lean_inc(x_40); +lean_dec(x_39); +x_41 = lean_ctor_get_uint8(x_40, sizeof(void*)*1); +lean_dec(x_40); +if (x_41 == 0) { -lean_object* x_13; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_42; uint8_t x_43; +x_42 = lean_ctor_get(x_38, 1); +lean_inc(x_42); +lean_dec(x_38); +x_43 = 0; +x_15 = x_43; +x_16 = x_42; +goto block_37; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; +x_44 = lean_ctor_get(x_38, 1); +lean_inc(x_44); +lean_dec(x_38); +x_45 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_14, x_7, x_8, x_9, x_10, x_11, x_12, x_44); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = lean_unbox(x_46); +lean_dec(x_46); +x_15 = x_48; +x_16 = x_47; +goto block_37; +} +block_37: +{ +if (x_15 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(x_6, x_1, x_2, x_3, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_16); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_5); -lean_ctor_set(x_13, 1, x_12); -return x_13; +return x_18; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_4, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_4, 1); -lean_inc(x_15); -lean_dec(x_4); -lean_inc(x_14); -x_16 = l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1(x_14, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 0); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_19 = lean_ctor_get(x_2, 0); lean_inc(x_19); -lean_dec(x_17); x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); lean_dec(x_19); -lean_inc(x_3); -x_21 = l_Lean_Expr_const___override(x_20, x_3); +x_21 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_21, 0, x_20); +x_22 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__7; +x_23 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +x_24 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9; +x_25 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); lean_inc(x_1); -x_22 = l_Lean_mkAppN(x_21, x_1); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_23 = lean_infer_type(x_22, x_8, x_9, x_10, x_11, x_18); -if (lean_obj_tag(x_23) == 0) +x_26 = lean_array_to_list(lean_box(0), x_1); +x_27 = lean_box(0); +x_28 = l_List_mapTRAux___at_Lean_MessageData_instCoeListExprMessageData___spec__1(x_26, x_27); +x_29 = l_Lean_MessageData_ofList(x_28); +lean_dec(x_28); +x_30 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_30, 0, x_25); +lean_ctor_set(x_30, 1, x_29); +x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__11; +x_32 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_14, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(x_6, x_1, x_2, x_3, x_4, x_5, x_34, x_7, x_8, x_9, x_10, x_11, x_12, x_35); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_34); +lean_dec(x_6); +return x_36; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); +lean_object* x_13; lean_object* x_14; +lean_inc(x_1); lean_inc(x_2); -x_26 = lean_apply_2(x_2, x_5, x_14); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_27 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Elab_Deriving_mkInductArgNames___spec__2___rarg(x_24, x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_25); -if (lean_obj_tag(x_27) == 0) +x_13 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2), 13, 5); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, x_1); +lean_closure_set(x_13, 2, x_4); +lean_closure_set(x_13, 3, x_3); +lean_closure_set(x_13, 4, x_5); +x_14 = l_Lean_Server_RpcEncoding_withFields___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___rarg(x_1, x_2, x_13, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_4 = x_15; -x_5 = x_28; -x_12 = x_29; -goto _start; +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_14; } -else +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -uint8_t x_31; -lean_dec(x_15); +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_27); -if (x_31 == 0) -{ -return x_27; -} -else -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_27, 0); -x_33 = lean_ctor_get(x_27, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_27); -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; -} +return x_15; } } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -uint8_t x_35; -lean_dec(x_15); -lean_dec(x_14); +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__3(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); -lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_35 = !lean_is_exclusive(x_23); -if (x_35 == 0) -{ -return x_23; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_23, 0); -x_37 = lean_ctor_get(x_23, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_23); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} +return x_15; } } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -uint8_t x_39; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_11); -lean_dec(x_10); +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_39 = !lean_is_exclusive(x_16); -if (x_39 == 0) -{ -return x_16; -} -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_16, 0); -x_41 = lean_ctor_get(x_16, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_16); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -return x_42; -} +lean_dec(x_4); +return x_13; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__5(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; } } -LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__34(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__34___rarg), 12, 0); -return x_2; +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_10); +lean_dec(x_10); +x_14 = lean_unbox_usize(x_11); +lean_dec(x_11); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13, x_14, x_12); +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__33___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_13, x_14); -x_16 = lean_ctor_get(x_1, 4); -lean_inc(x_16); +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_17 = l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__34___rarg(x_2, x_3, x_15, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -return x_17; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_17); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; +return x_9; } } -else -{ -uint8_t x_22; -x_22 = !lean_is_exclusive(x_17); -if (x_22 == 0) +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -return x_17; +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__8(x_4, x_5, x_3); +return x_6; } -else +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_17, 0); -x_24 = lean_ctor_get(x_17, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_17); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__9(x_1, x_2, x_3, x_7, x_8, x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_9; } } +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__12(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_2); +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__33(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__33___rarg), 11, 0); -return x_2; +lean_object* x_15; +x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_1); +return x_15; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___closed__1() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_ctors___default() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_levelOne; -x_2 = l_Lean_Expr_sort___override(x_1); -return x_2; +lean_object* x_1; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +return x_1; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encodes___default() { _start: { -lean_object* x_9; lean_object* x_10; -x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_8); -return x_10; +lean_object* x_1; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__1() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_decodes___default() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___boxed), 8, 0); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__2() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__1() { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 0; -x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__1; -x_3 = lean_box(x_1); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); -lean_ctor_set(x_4, 1, x_2); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__4; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l_Lean_Parser_categoryParser(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35(size_t x_1, size_t x_2, lean_object* x_3) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__2() { _start: { -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) -{ -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__1; +x_2 = l_Lean_Parser_Term_matchAlt(x_1); +return x_2; } -else +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF() { +_start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__2; -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_5); -lean_ctor_set(x_9, 1, x_8); -x_10 = 1; -x_11 = lean_usize_add(x_2, x_10); -x_12 = lean_array_uset(x_7, x_2, x_9); -x_2 = x_11; -x_3 = x_12; -goto _start; +lean_object* x_1; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__2; +return x_1; } } +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("explicitBinder", 14); +return x_1; +} } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__36(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; @@ -15870,9 +8029,7 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); +lean_dec(x_2); x_14 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_14, 0, x_5); lean_ctor_set(x_14, 1, x_12); @@ -15880,210 +8037,325 @@ return x_14; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_array_uget(x_2, x_4); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_array_uget(x_5, x_4); +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_array_uset(x_5, x_4, x_16); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_15); -x_16 = lean_infer_type(x_15, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_16) == 0) +x_18 = lean_infer_type(x_15, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_1, 0); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_20 = l_Lean_Meta_DiscrTree_getMatch___rarg(x_19, x_17, x_8, x_9, x_10, x_11, x_18); -if (lean_obj_tag(x_20) == 0) +x_21 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor(x_19, x_8, x_9, x_10, x_11, x_20); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Lean_instInhabitedName; -x_24 = l_Array_back___rarg(x_23, x_21); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); lean_dec(x_21); -x_25 = lean_mk_syntax_ident(x_24); -x_26 = lean_box(0); -x_27 = 1; +x_24 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_28 = l_Lean_Elab_Term_elabTerm(x_25, x_26, x_27, x_27, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +x_25 = l_Lean_PrettyPrinter_delab(x_22, x_24, x_8, x_9, x_10, x_11, x_23); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +lean_inc(x_8); +x_28 = l_Lean_Meta_getFVarLocalDecl(x_15, x_8, x_9, x_10, x_11, x_27); if (lean_obj_tag(x_28) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_object* x_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; size_t x_67; size_t x_68; lean_object* x_69; x_29 = lean_ctor_get(x_28, 0); lean_inc(x_29); x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); lean_dec(x_28); -lean_inc(x_8); -x_31 = l_Lean_Meta_getFVarLocalDecl(x_15, x_8, x_9, x_10, x_11, x_30); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; size_t x_37; size_t x_38; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); +x_31 = l_Lean_LocalDecl_userName(x_29); +lean_dec(x_29); +lean_inc(x_10); +x_32 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_10, x_11, x_30); +x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); -lean_dec(x_31); -x_34 = l_Lean_LocalDecl_userName(x_32); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); lean_dec(x_32); -x_35 = 0; -x_36 = l_Lean_Expr_forallE___override(x_34, x_29, x_5, x_35); -x_37 = 1; -x_38 = lean_usize_add(x_4, x_37); -x_4 = x_38; -x_5 = x_36; -x_12 = x_33; +x_35 = lean_st_ref_get(x_11, x_34); +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +lean_dec(x_35); +x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__5; +lean_inc(x_2); +x_38 = l_Lean_Name_str___override(x_2, x_37); +x_39 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; +x_40 = l_Lean_Name_str___override(x_38, x_39); +x_41 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1; +x_42 = l_Lean_Name_str___override(x_40, x_41); +x_43 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +lean_inc(x_33); +x_44 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_44, 0, x_33); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_mk_syntax_ident(x_31); +x_46 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_47 = lean_array_push(x_46, x_45); +x_48 = lean_box(2); +x_49 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_50 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +lean_ctor_set(x_50, 2, x_47); +x_51 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; +lean_inc(x_33); +x_52 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_52, 0, x_33); +lean_ctor_set(x_52, 1, x_51); +x_53 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_54 = lean_array_push(x_53, x_52); +x_55 = lean_array_push(x_54, x_26); +x_56 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_56, 0, x_48); +lean_ctor_set(x_56, 1, x_49); +lean_ctor_set(x_56, 2, x_55); +x_57 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +x_58 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_58, 0, x_33); +lean_ctor_set(x_58, 1, x_57); +x_59 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; +x_60 = lean_array_push(x_59, x_44); +x_61 = lean_array_push(x_60, x_50); +x_62 = lean_array_push(x_61, x_56); +x_63 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_64 = lean_array_push(x_62, x_63); +x_65 = lean_array_push(x_64, x_58); +x_66 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_66, 0, x_48); +lean_ctor_set(x_66, 1, x_42); +lean_ctor_set(x_66, 2, x_65); +x_67 = 1; +x_68 = lean_usize_add(x_4, x_67); +x_69 = lean_array_uset(x_17, x_4, x_66); +x_4 = x_68; +x_5 = x_69; +x_12 = x_36; goto _start; } else { -uint8_t x_40; -lean_dec(x_29); +uint8_t x_71; +lean_dec(x_26); +lean_dec(x_17); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_40 = !lean_is_exclusive(x_31); -if (x_40 == 0) +lean_dec(x_2); +x_71 = !lean_is_exclusive(x_28); +if (x_71 == 0) { -return x_31; +return x_28; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_31, 0); -x_42 = lean_ctor_get(x_31, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_31); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_72 = lean_ctor_get(x_28, 0); +x_73 = lean_ctor_get(x_28, 1); +lean_inc(x_73); +lean_inc(x_72); +lean_dec(x_28); +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set(x_74, 1, x_73); +return x_74; } } } else { -uint8_t x_44; +uint8_t x_75; +lean_dec(x_17); lean_dec(x_15); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_44 = !lean_is_exclusive(x_28); -if (x_44 == 0) +lean_dec(x_2); +x_75 = !lean_is_exclusive(x_25); +if (x_75 == 0) { -return x_28; +return x_25; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_28, 0); -x_46 = lean_ctor_get(x_28, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_28); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_25, 0); +x_77 = lean_ctor_get(x_25, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_25); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; } } } else { -uint8_t x_48; +uint8_t x_79; +lean_dec(x_17); lean_dec(x_15); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_48 = !lean_is_exclusive(x_20); -if (x_48 == 0) +lean_dec(x_2); +x_79 = !lean_is_exclusive(x_21); +if (x_79 == 0) { -return x_20; +return x_21; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_20, 0); -x_50 = lean_ctor_get(x_20, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_20); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_80 = lean_ctor_get(x_21, 0); +x_81 = lean_ctor_get(x_21, 1); +lean_inc(x_81); +lean_inc(x_80); +lean_dec(x_21); +x_82 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +return x_82; } } } else { -uint8_t x_52; +uint8_t x_83; +lean_dec(x_17); lean_dec(x_15); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_52 = !lean_is_exclusive(x_16); -if (x_52 == 0) +lean_dec(x_2); +x_83 = !lean_is_exclusive(x_18); +if (x_83 == 0) { -return x_16; +return x_18; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_16, 0); -x_54 = lean_ctor_get(x_16, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_16); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -return x_55; +lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_18, 0); +x_85 = lean_ctor_get(x_18, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_18); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +return x_86; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +return x_5; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; +x_7 = lean_array_uget(x_5, x_4); +x_8 = lean_unsigned_to_nat(0u); +x_9 = lean_array_uset(x_5, x_4, x_8); +x_10 = 1; +x_11 = lean_usize_add(x_4, x_10); +x_12 = lean_array_uset(x_9, x_4, x_7); +x_4 = x_11; +x_5 = x_12; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +return x_5; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; +x_7 = lean_array_uget(x_5, x_4); +x_8 = lean_unsigned_to_nat(0u); +x_9 = lean_array_uset(x_5, x_4, x_8); +x_10 = 1; +x_11 = lean_usize_add(x_4, x_10); +x_12 = lean_array_uset(x_9, x_4, x_7); +x_4 = x_11; +x_5 = x_12; +goto _start; +} +} } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; } +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_10 = lean_array_uset(x_7, x_2, x_5); +x_2 = x_9; +x_3 = x_10; +goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__37(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -16151,7 +8423,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__38(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -16175,7 +8447,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__39(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; @@ -16211,14 +8483,14 @@ x_25 = lean_st_ref_get(x_15, x_24); x_26 = lean_ctor_get(x_25, 1); lean_inc(x_26); lean_dec(x_25); -x_27 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1; +x_27 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3; lean_inc(x_3); x_28 = l_Lean_Name_str___override(x_3, x_27); -x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2; +x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; x_30 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_30, 0, x_23); lean_ctor_set(x_30, 1, x_29); -x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; lean_inc(x_3); x_32 = l_Lean_Name_str___override(x_3, x_31); lean_inc(x_6); @@ -16233,53 +8505,29 @@ lean_ctor_set(x_36, 1, x_2); lean_ctor_set(x_36, 2, x_34); lean_inc(x_4); x_37 = lean_array_push(x_4, x_33); -x_38 = lean_array_push(x_37, x_36); -x_39 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_39, 0, x_35); -lean_ctor_set(x_39, 1, x_32); -lean_ctor_set(x_39, 2, x_38); -lean_inc(x_4); -x_40 = lean_array_push(x_4, x_30); -x_41 = lean_array_push(x_40, x_39); -x_42 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_42, 0, x_35); -lean_ctor_set(x_42, 1, x_28); -lean_ctor_set(x_42, 2, x_41); -x_43 = 1; -x_44 = lean_usize_add(x_8, x_43); -x_45 = lean_array_uset(x_21, x_8, x_42); -x_8 = x_44; -x_9 = x_45; -x_16 = x_26; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__40(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { -_start: -{ -uint8_t x_5; -x_5 = lean_usize_dec_lt(x_3, x_2); -if (x_5 == 0) -{ -return x_4; -} -else -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; -x_6 = lean_array_uget(x_4, x_3); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_array_uset(x_4, x_3, x_7); -x_9 = 1; -x_10 = lean_usize_add(x_3, x_9); -x_11 = lean_array_uset(x_8, x_3, x_6); -x_3 = x_10; -x_4 = x_11; +x_38 = lean_array_push(x_37, x_36); +x_39 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_39, 0, x_35); +lean_ctor_set(x_39, 1, x_32); +lean_ctor_set(x_39, 2, x_38); +lean_inc(x_4); +x_40 = lean_array_push(x_4, x_30); +x_41 = lean_array_push(x_40, x_39); +x_42 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_42, 0, x_35); +lean_ctor_set(x_42, 1, x_28); +lean_ctor_set(x_42, 2, x_41); +x_43 = 1; +x_44 = lean_usize_add(x_8, x_43); +x_45 = lean_array_uset(x_21, x_8, x_42); +x_8 = x_44; +x_9 = x_45; +x_16 = x_26; goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__41(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; @@ -16289,10 +8537,10 @@ if (x_17 == 0) lean_object* x_18; lean_dec(x_14); 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_18 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_18, 0, x_9); lean_ctor_set(x_18, 1, x_16); @@ -16315,35 +8563,35 @@ x_25 = lean_st_ref_get(x_15, x_24); x_26 = lean_ctor_get(x_25, 1); lean_inc(x_26); lean_dec(x_25); -x_27 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1; -lean_inc(x_2); -x_28 = l_Lean_Name_str___override(x_2, x_27); -x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2; +x_27 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3; +lean_inc(x_3); +x_28 = l_Lean_Name_str___override(x_3, x_27); +x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; x_30 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_30, 0, x_23); lean_ctor_set(x_30, 1, x_29); -x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; -lean_inc(x_2); -x_32 = l_Lean_Name_str___override(x_2, x_31); +x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; +lean_inc(x_3); +x_32 = l_Lean_Name_str___override(x_3, x_31); lean_inc(x_6); x_33 = lean_mk_syntax_ident(x_6); -lean_inc(x_4); -x_34 = lean_array_push(x_4, x_19); +lean_inc(x_5); +x_34 = lean_array_push(x_5, x_19); x_35 = lean_box(2); -lean_inc(x_1); +lean_inc(x_2); x_36 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_1); +lean_ctor_set(x_36, 1, x_2); lean_ctor_set(x_36, 2, x_34); -lean_inc(x_3); -x_37 = lean_array_push(x_3, x_33); +lean_inc(x_4); +x_37 = lean_array_push(x_4, x_33); x_38 = lean_array_push(x_37, x_36); x_39 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_39, 0, x_35); lean_ctor_set(x_39, 1, x_32); lean_ctor_set(x_39, 2, x_38); -lean_inc(x_3); -x_40 = lean_array_push(x_3, x_30); +lean_inc(x_4); +x_40 = lean_array_push(x_4, x_30); x_41 = lean_array_push(x_40, x_39); x_42 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_42, 0, x_35); @@ -16359,254 +8607,217 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__42(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_6; -x_6 = lean_usize_dec_lt(x_4, x_3); -if (x_6 == 0) +if (lean_obj_tag(x_4) == 0) { -return x_5; +lean_object* x_13; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_5); +lean_ctor_set(x_13, 1, x_12); +return x_13; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; -x_7 = lean_array_uget(x_5, x_4); -x_8 = lean_unsigned_to_nat(0u); -x_9 = lean_array_uset(x_5, x_4, x_8); -x_10 = 1; -x_11 = lean_usize_add(x_4, x_10); -x_12 = lean_array_uset(x_9, x_4, x_7); -x_4 = x_11; -x_5 = x_12; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__43(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { -_start: +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_4, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_4, 1); +lean_inc(x_15); +lean_dec(x_4); +lean_inc(x_14); +x_16 = l_Lean_getConstInfoCtor___at___private_Lean_Meta_WHNF_0__Lean_Meta_toCtorWhenStructure___spec__1(x_14, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_16) == 0) { -uint8_t x_5; -x_5 = lean_usize_dec_lt(x_3, x_2); -if (x_5 == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +lean_dec(x_19); +lean_inc(x_3); +x_21 = l_Lean_Expr_const___override(x_20, x_3); +lean_inc(x_1); +x_22 = l_Lean_mkAppN(x_21, x_1); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +x_23 = lean_infer_type(x_22, x_8, x_9, x_10, x_11, x_18); +if (lean_obj_tag(x_23) == 0) { -return x_4; -} -else +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +lean_inc(x_2); +x_26 = lean_apply_2(x_2, x_5, x_14); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_27 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Elab_Deriving_mkInductArgNames___spec__2___rarg(x_24, x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; -x_6 = lean_array_uget(x_4, x_3); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_array_uset(x_4, x_3, x_7); -x_9 = lean_mk_syntax_ident(x_6); -x_10 = 1; -x_11 = lean_usize_add(x_3, x_10); -x_12 = lean_array_uset(x_8, x_3, x_9); -x_3 = x_11; -x_4 = x_12; +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_4 = x_15; +x_5 = x_28; +x_12 = x_29; goto _start; } -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__44(size_t x_1, size_t x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) -{ -return x_3; -} else { -lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = lean_array_uset(x_7, x_2, x_5); -x_2 = x_9; -x_3 = x_10; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45(size_t x_1, size_t x_2, lean_object* x_3) { -_start: -{ -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) +uint8_t x_31; +lean_dec(x_15); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_31 = !lean_is_exclusive(x_27); +if (x_31 == 0) { -return x_3; +return x_27; } else { -lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = 1; -x_9 = lean_usize_add(x_2, x_8); -x_10 = lean_array_uset(x_7, x_2, x_5); -x_2 = x_9; -x_3 = x_10; -goto _start; -} -} +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_27, 0); +x_33 = lean_ctor_get(x_27, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_27); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47___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) { -_start: -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_array_push(x_1, x_5); -x_14 = l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47___rarg(x_2, x_3, x_4, x_13, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = lean_array_get_size(x_4); -x_13 = lean_array_get_size(x_1); -x_14 = lean_nat_dec_lt(x_12, x_13); -lean_dec(x_13); -if (x_14 == 0) +else { -lean_object* x_15; -lean_dec(x_12); +uint8_t x_35; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_15 = lean_apply_8(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_16 = lean_array_fget(x_1, x_12); -lean_dec(x_12); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); -lean_dec(x_17); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_21 = lean_apply_8(x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47___rarg___lambda__1), 12, 4); -lean_closure_set(x_24, 0, x_4); -lean_closure_set(x_24, 1, x_1); -lean_closure_set(x_24, 2, x_2); -lean_closure_set(x_24, 3, x_3); -x_25 = lean_unbox(x_19); -lean_dec(x_19); -x_26 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__3___rarg(x_18, x_25, x_22, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_23); -return x_26; +x_35 = !lean_is_exclusive(x_23); +if (x_35 == 0) +{ +return x_23; } else { -uint8_t x_27; -lean_dec(x_19); -lean_dec(x_18); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_23, 0); +x_37 = lean_ctor_get(x_23, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_23); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} +} +} +else +{ +uint8_t x_39; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_27 = !lean_is_exclusive(x_21); -if (x_27 == 0) +x_39 = !lean_is_exclusive(x_16); +if (x_39 == 0) { -return x_21; +return x_16; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_21, 0); -x_29 = lean_ctor_get(x_21, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_21); -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_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_16, 0); +x_41 = lean_ctor_get(x_16, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_16); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47___rarg), 11, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__46___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_12 = l_Lean_Meta_withLocalDecls_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__47___rarg(x_2, x_3, x_1, x_11, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__46(lean_object* x_1) { +LEAN_EXPORT lean_object* l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_withLocalDecls___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__46___rarg), 10, 0); +x_2 = lean_alloc_closure((void*)(l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10___rarg), 12, 0); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; -x_11 = lean_array_get_size(x_1); -x_12 = lean_usize_of_nat(x_11); -lean_dec(x_11); -x_13 = 0; -lean_inc(x_6); -lean_inc(x_1); -x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1(x_12, x_13, x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = l_List_mapTRAux___at_Lean_mkConstWithLevelParams___spec__1(x_13, x_14); +x_16 = lean_ctor_get(x_1, 4); lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32(x_15, x_1, x_12, x_13, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_16); lean_dec(x_1); -lean_dec(x_15); +x_17 = l_List_forIn_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__10___rarg(x_2, x_3, x_15, x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_17) == 0) { uint8_t x_18; @@ -16652,758 +8863,587 @@ return x_25; } } } -else -{ -uint8_t x_26; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_26 = !lean_is_exclusive(x_14); -if (x_26 == 0) -{ -return x_14; -} -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_14, 0); -x_28 = lean_ctor_get(x_14, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_14); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; -} -} -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" → ", 5); -return x_1; -} } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9___rarg), 11, 0); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { -uint8_t x_13; lean_object* x_14; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_37 = lean_st_ref_get(x_11, x_12); -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_38, 3); -lean_inc(x_39); -lean_dec(x_38); -x_40 = lean_ctor_get_uint8(x_39, sizeof(void*)*1); -lean_dec(x_39); -if (x_40 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) { -lean_object* x_41; uint8_t x_42; -x_41 = lean_ctor_get(x_37, 1); -lean_inc(x_41); -lean_dec(x_37); -x_42 = 0; -x_13 = x_42; -x_14 = x_41; -goto block_36; +return x_4; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_43 = lean_ctor_get(x_37, 1); -lean_inc(x_43); -lean_dec(x_37); -lean_inc(x_1); -x_44 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_43); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_47 = lean_unbox(x_45); -lean_dec(x_45); -x_13 = x_47; -x_14 = x_46; -goto block_36; +lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_6 = lean_array_uget(x_4, x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_4, x_3, x_7); +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_11 = lean_array_uset(x_8, x_3, x_6); +x_3 = x_10; +x_4 = x_11; +goto _start; } -block_36: +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(size_t x_1, size_t x_2, lean_object* x_3) { +_start: { -if (x_13 == 0) +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) { -lean_object* x_15; lean_object* x_16; -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_1); -x_15 = lean_box(0); -x_16 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1(x_4, x_2, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_14); -lean_dec(x_7); -return x_16; +return x_3; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_17 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_17, 0, x_3); -x_18 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6; -x_19 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__4; -x_21 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -lean_inc(x_4); -x_22 = lean_array_to_list(lean_box(0), x_4); -x_23 = lean_box(0); -x_24 = l_List_mapTRAux___at_Lean_MessageData_instCoeListExprMessageData___spec__1(x_22, x_23); -x_25 = l_Lean_MessageData_ofList(x_24); -lean_dec(x_24); -x_26 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_26, 0, x_21); -lean_ctor_set(x_26, 1, x_25); -x_27 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2; -x_28 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_29, 0, x_5); -x_30 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -x_31 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_18); -x_32 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_1, x_31, x_6, x_7, x_8, x_9, x_10, x_11, x_14); -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); -lean_inc(x_34); -lean_dec(x_32); -x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1(x_4, x_2, x_33, x_6, x_7, x_8, x_9, x_10, x_11, x_34); -lean_dec(x_7); -lean_dec(x_33); -return x_35; -} +lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_10 = lean_array_uset(x_7, x_2, x_5); +x_2 = x_9; +x_3 = x_10; +goto _start; } } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__1() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(size_t x_1, size_t x_2, lean_object* x_3) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("ctor", 4); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__2() { -_start: +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("|", 1); -return x_1; +lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_10 = lean_array_uset(x_7, x_2, x_5); +x_2 = x_9; +x_3 = x_10; +goto _start; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__4() { +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("matchAlt", 8); +x_1 = lean_mk_string_from_bytes("ctor", 4); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__4; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__6() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("=>", 2); +x_1 = lean_mk_string_from_bytes("|", 1); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__3() { _start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; size_t x_20; lean_object* x_21; -lean_inc(x_2); -lean_inc(x_1); -x_17 = l_Lean_Expr_const___override(x_1, x_2); -lean_inc(x_8); -x_18 = l_Array_reverse___rarg(x_8); -x_19 = lean_array_get_size(x_18); -x_20 = lean_usize_of_nat(x_19); -lean_dec(x_19); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_6); -x_21 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__36(x_6, x_18, x_20, x_3, x_17, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_18); -if (lean_obj_tag(x_21) == 0) +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("matchAlt", 8); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { +_start: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_box(0); +lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; +x_20 = lean_array_get_size(x_11); +x_21 = lean_usize_of_nat(x_20); +lean_dec(x_20); +x_22 = 0; +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_25 = l_Lean_PrettyPrinter_delab(x_22, x_24, x_12, x_13, x_14, x_15, x_23); -if (lean_obj_tag(x_25) == 0) +lean_inc(x_11); +lean_inc(x_2); +x_23 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1(x_1, x_2, x_21, x_22, x_11, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; 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; size_t x_73; lean_object* x_74; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; 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; size_t x_55; lean_object* x_56; lean_object* x_57; size_t x_58; lean_object* x_59; lean_object* x_60; size_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +lean_inc(x_17); +x_26 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_17, x_18, x_25); +x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); -lean_dec(x_25); -lean_inc(x_14); -x_28 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_14, x_15, x_27); -x_29 = lean_ctor_get(x_28, 0); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_ctor_get(x_17, 10); lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_st_ref_get(x_15, x_30); -x_32 = lean_ctor_get(x_31, 1); +x_30 = lean_st_ref_get(x_18, x_28); +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_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__3; -lean_inc(x_29); -x_34 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_34, 0, x_29); -lean_ctor_set(x_34, 1, x_33); -x_35 = lean_box(2); -x_36 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_37 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -lean_ctor_set(x_37, 2, x_4); -x_38 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -lean_inc(x_37); -x_39 = lean_array_push(x_38, x_37); -lean_inc(x_37); -x_40 = lean_array_push(x_39, x_37); -lean_inc(x_37); -x_41 = lean_array_push(x_40, x_37); -lean_inc(x_37); -x_42 = lean_array_push(x_41, x_37); -lean_inc(x_37); -x_43 = lean_array_push(x_42, x_37); -lean_inc(x_37); -x_44 = lean_array_push(x_43, x_37); -x_45 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; -x_46 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_46, 0, x_35); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_44); -x_47 = l_Lean_Name_getString_x21(x_7); -x_48 = lean_box(0); -lean_inc(x_47); -x_49 = l_Lean_Name_str___override(x_48, x_47); -x_50 = lean_mk_syntax_ident(x_49); -x_51 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; -x_52 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_52, 0, x_29); -lean_ctor_set(x_52, 1, x_51); -x_53 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_54 = lean_array_push(x_53, x_52); -x_55 = lean_array_push(x_54, x_26); -x_56 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95; -x_57 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_57, 0, x_35); -lean_ctor_set(x_57, 1, x_56); -lean_ctor_set(x_57, 2, x_55); -x_58 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -x_59 = lean_array_push(x_58, x_57); -x_60 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_60, 0, x_35); -lean_ctor_set(x_60, 1, x_36); -lean_ctor_set(x_60, 2, x_59); -x_61 = lean_array_push(x_53, x_37); -x_62 = lean_array_push(x_61, x_60); -x_63 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_35); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_66 = lean_array_push(x_65, x_34); -x_67 = lean_array_push(x_66, x_46); -x_68 = lean_array_push(x_67, x_50); -x_69 = lean_array_push(x_68, x_64); -x_70 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__2; -x_71 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_71, 0, x_35); -lean_ctor_set(x_71, 1, x_70); -lean_ctor_set(x_71, 2, x_69); -x_72 = lean_array_get_size(x_8); -x_73 = lean_usize_of_nat(x_72); -lean_dec(x_72); -lean_inc(x_15); -lean_inc(x_14); -x_74 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__37(x_73, x_3, x_8, x_10, x_11, x_12, x_13, x_14, x_15, x_32); -if (lean_obj_tag(x_74) == 0) +x_34 = lean_environment_main_module(x_33); +x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__5; +x_36 = l_Lean_Name_str___override(x_2, x_35); +x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__7; +lean_inc(x_36); +x_38 = l_Lean_Name_str___override(x_36, x_37); +x_39 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__1; +lean_inc(x_38); +x_40 = l_Lean_Name_str___override(x_38, x_39); +x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__2; +lean_inc(x_27); +x_42 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_42, 0, x_27); +lean_ctor_set(x_42, 1, x_41); +x_43 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; +lean_inc(x_38); +x_44 = l_Lean_Name_str___override(x_38, x_43); +x_45 = lean_box(2); +x_46 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__145; +x_47 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_44); +lean_ctor_set(x_47, 2, x_46); +x_48 = l_Lean_Name_getString_x21(x_10); +x_49 = lean_box(0); +lean_inc(x_48); +x_50 = l_Lean_Name_str___override(x_49, x_48); +x_51 = lean_mk_syntax_ident(x_50); +x_52 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__32; +x_53 = l_Lean_Name_str___override(x_38, x_52); +x_54 = lean_array_get_size(x_24); +x_55 = lean_usize_of_nat(x_54); +lean_dec(x_54); +x_56 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(x_1, x_36, x_55, x_22, x_24); +x_57 = lean_array_get_size(x_56); +x_58 = lean_usize_of_nat(x_57); +lean_dec(x_57); +x_59 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3(x_1, x_36, x_58, x_22, x_56); +x_60 = lean_array_get_size(x_59); +x_61 = lean_usize_of_nat(x_60); +lean_dec(x_60); +x_62 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4(x_61, x_22, x_59); +x_63 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +x_64 = l_Array_append___rarg(x_63, x_62); +x_65 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_66 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_66, 0, x_45); +lean_ctor_set(x_66, 1, x_65); +lean_ctor_set(x_66, 2, x_64); +x_67 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; +x_68 = l_Lean_Name_str___override(x_36, x_67); +x_69 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__36; +lean_inc(x_68); +x_70 = l_Lean_Name_str___override(x_68, x_69); +x_71 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; +lean_inc(x_27); +x_72 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_72, 0, x_27); +lean_ctor_set(x_72, 1, x_71); +x_73 = l_Lean_addMacroScope(x_34, x_3, x_29); +x_74 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_74, 0, x_27); +lean_ctor_set(x_74, 1, x_4); +lean_ctor_set(x_74, 2, x_73); +lean_ctor_set(x_74, 3, x_1); +x_75 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_76 = lean_array_push(x_75, x_72); +x_77 = lean_array_push(x_76, x_74); +x_78 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_78, 0, x_45); +lean_ctor_set(x_78, 1, x_70); +lean_ctor_set(x_78, 2, x_77); +x_79 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +x_80 = lean_array_push(x_79, x_78); +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_45); +lean_ctor_set(x_81, 1, x_65); +lean_ctor_set(x_81, 2, x_80); +x_82 = lean_array_push(x_75, x_66); +x_83 = lean_array_push(x_82, x_81); +x_84 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_84, 0, x_45); +lean_ctor_set(x_84, 1, x_53); +lean_ctor_set(x_84, 2, x_83); +x_85 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_86 = lean_array_push(x_85, x_42); +x_87 = lean_array_push(x_86, x_47); +x_88 = lean_array_push(x_87, x_51); +x_89 = lean_array_push(x_88, x_84); +x_90 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_90, 0, x_45); +lean_ctor_set(x_90, 1, x_40); +lean_ctor_set(x_90, 2, x_89); +lean_inc(x_18); +lean_inc(x_17); +x_91 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5(x_21, x_22, x_11, x_13, x_14, x_15, x_16, x_17, x_18, x_32); +if (lean_obj_tag(x_91) == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; size_t x_78; lean_object* x_79; lean_object* x_80; size_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; 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; uint8_t x_149; -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -lean_dec(x_74); -x_77 = lean_array_get_size(x_75); -x_78 = lean_usize_of_nat(x_77); -lean_dec(x_77); -lean_inc(x_75); -x_79 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__38(x_2, x_78, x_3, x_75); -x_80 = lean_array_get_size(x_79); -x_81 = lean_usize_of_nat(x_80); -lean_dec(x_80); -x_82 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_83 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225; -lean_inc(x_14); -lean_inc(x_79); -x_84 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__39(x_2, x_36, x_82, x_53, x_58, x_83, x_81, x_3, x_79, x_10, x_11, x_12, x_13, x_14, x_15, x_76); -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__9; -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_87); -lean_ctor_set(x_88, 1, x_2); -lean_inc(x_47); -x_89 = l_Lean_Name_str___override(x_1, x_47); -x_90 = lean_mk_syntax_ident(x_89); -lean_inc(x_90); -x_91 = l_Lean_Syntax_mkApp(x_90, x_85); -lean_inc(x_14); -x_92 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_14, x_15, x_86); -x_93 = lean_ctor_get(x_92, 0); +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; size_t x_97; lean_object* x_98; lean_object* x_99; size_t x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; 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; uint8_t x_164; +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_91, 1); lean_inc(x_93); -x_94 = lean_ctor_get(x_92, 1); -lean_inc(x_94); -lean_dec(x_92); -x_95 = lean_st_ref_get(x_15, x_94); -x_96 = lean_ctor_get(x_95, 1); -lean_inc(x_96); -lean_dec(x_95); -x_97 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67; -x_98 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_98, 0, x_93); -lean_ctor_set(x_98, 1, x_97); -x_99 = lean_array_push(x_58, x_91); -x_100 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_100, 0, x_35); -lean_ctor_set(x_100, 1, x_36); -lean_ctor_set(x_100, 2, x_99); -x_101 = lean_array_push(x_53, x_98); -x_102 = lean_array_push(x_101, x_100); -x_103 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66; -x_104 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_104, 0, x_35); -lean_ctor_set(x_104, 1, x_103); -lean_ctor_set(x_104, 2, x_102); -lean_inc(x_14); -x_105 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_14, x_15, x_96); -x_106 = lean_ctor_get(x_105, 0); -lean_inc(x_106); -x_107 = lean_ctor_get(x_105, 1); -lean_inc(x_107); -lean_dec(x_105); -x_108 = lean_st_ref_get(x_15, x_107); -x_109 = lean_ctor_get(x_108, 1); +lean_dec(x_91); +x_94 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; +lean_inc(x_5); +x_95 = l_Lean_Name_str___override(x_5, x_94); +x_96 = lean_array_get_size(x_92); +x_97 = lean_usize_of_nat(x_96); +lean_dec(x_96); +x_98 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6(x_6, x_97, x_22, x_92); +x_99 = lean_array_get_size(x_98); +x_100 = lean_usize_of_nat(x_99); +lean_dec(x_99); +lean_inc(x_17); +lean_inc(x_98); +lean_inc(x_68); +x_101 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(x_6, x_65, x_68, x_75, x_79, x_95, x_100, x_22, x_98, x_13, x_14, x_15, x_16, x_17, x_18, x_93); +x_102 = lean_ctor_get(x_101, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_101, 1); +lean_inc(x_103); +lean_dec(x_101); +lean_inc(x_48); +x_104 = l_Lean_Name_str___override(x_7, x_48); +x_105 = lean_mk_syntax_ident(x_104); +lean_inc(x_105); +x_106 = l_Lean_Syntax_mkApp(x_105, x_102); +lean_inc(x_17); +x_107 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_17, x_18, x_103); +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_107, 1); lean_inc(x_109); -lean_dec(x_108); -lean_inc(x_106); -x_110 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_110, 0, x_106); -lean_ctor_set(x_110, 1, x_33); -x_111 = lean_ctor_get(x_5, 0); +lean_dec(x_107); +x_110 = lean_st_ref_get(x_18, x_109); +x_111 = lean_ctor_get(x_110, 1); lean_inc(x_111); -lean_dec(x_5); -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -lean_dec(x_111); -x_113 = l_Lean_Name_str___override(x_112, x_47); -x_114 = lean_mk_syntax_ident(x_113); -x_115 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__40(x_88, x_78, x_3, x_75); -lean_inc(x_115); -lean_inc(x_114); -x_116 = l_Lean_Syntax_mkApp(x_114, x_115); -x_117 = lean_array_push(x_58, x_116); -x_118 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_118, 0, x_35); -lean_ctor_set(x_118, 1, x_36); -lean_ctor_set(x_118, 2, x_117); -x_119 = lean_array_push(x_58, x_118); +lean_dec(x_110); +x_112 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__82; +lean_inc(x_68); +x_113 = l_Lean_Name_str___override(x_68, x_112); +x_114 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__84; +x_115 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_115, 0, x_108); +lean_ctor_set(x_115, 1, x_114); +x_116 = lean_array_push(x_79, x_106); +x_117 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_117, 0, x_45); +lean_ctor_set(x_117, 1, x_65); +lean_ctor_set(x_117, 2, x_116); +x_118 = lean_array_push(x_75, x_115); +x_119 = lean_array_push(x_118, x_117); +lean_inc(x_113); x_120 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_120, 0, x_35); -lean_ctor_set(x_120, 1, x_36); +lean_ctor_set(x_120, 0, x_45); +lean_ctor_set(x_120, 1, x_113); lean_ctor_set(x_120, 2, x_119); -x_121 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__6; -x_122 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_122, 0, x_106); -lean_ctor_set(x_122, 1, x_121); -x_123 = lean_array_push(x_65, x_110); -x_124 = lean_array_push(x_123, x_120); -x_125 = lean_array_push(x_124, x_122); -x_126 = lean_array_push(x_125, x_104); -x_127 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__5; -x_128 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_128, 0, x_35); -lean_ctor_set(x_128, 1, x_127); -lean_ctor_set(x_128, 2, x_126); -x_129 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232; -lean_inc(x_14); -x_130 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__41(x_36, x_82, x_53, x_58, x_88, x_129, x_81, x_3, x_79, x_10, x_11, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_88); -x_131 = lean_ctor_get(x_130, 0); -lean_inc(x_131); -x_132 = lean_ctor_get(x_130, 1); -lean_inc(x_132); -lean_dec(x_130); -x_133 = l_Lean_Syntax_mkApp(x_114, x_131); -lean_inc(x_14); -x_134 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_14, x_15, x_132); -x_135 = lean_ctor_get(x_134, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_134, 1); -lean_inc(x_136); -lean_dec(x_134); -x_137 = lean_st_ref_get(x_15, x_136); -x_138 = lean_ctor_get(x_137, 1); -lean_inc(x_138); -lean_dec(x_137); -x_139 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_139, 0, x_135); -lean_ctor_set(x_139, 1, x_97); -x_140 = lean_array_push(x_58, x_133); -x_141 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_141, 0, x_35); -lean_ctor_set(x_141, 1, x_36); -lean_ctor_set(x_141, 2, x_140); -x_142 = lean_array_push(x_53, x_139); -x_143 = lean_array_push(x_142, x_141); -x_144 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_144, 0, x_35); -lean_ctor_set(x_144, 1, x_103); -lean_ctor_set(x_144, 2, x_143); -x_145 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_14, x_15, x_138); +lean_inc(x_17); +x_121 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_17, x_18, x_111); +x_122 = lean_ctor_get(x_121, 0); +lean_inc(x_122); +x_123 = lean_ctor_get(x_121, 1); +lean_inc(x_123); +lean_dec(x_121); +x_124 = lean_st_ref_get(x_18, x_123); +x_125 = lean_ctor_get(x_124, 1); +lean_inc(x_125); +lean_dec(x_124); +x_126 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__3; +lean_inc(x_68); +x_127 = l_Lean_Name_str___override(x_68, x_126); +lean_inc(x_122); +x_128 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_128, 0, x_122); +lean_ctor_set(x_128, 1, x_41); +x_129 = l_Lean_Name_str___override(x_8, x_48); +x_130 = lean_mk_syntax_ident(x_129); +lean_inc(x_98); +lean_inc(x_130); +x_131 = l_Lean_Syntax_mkApp(x_130, x_98); +x_132 = lean_array_push(x_79, x_131); +x_133 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_133, 0, x_45); +lean_ctor_set(x_133, 1, x_65); +lean_ctor_set(x_133, 2, x_132); +x_134 = lean_array_push(x_79, x_133); +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_45); +lean_ctor_set(x_135, 1, x_65); +lean_ctor_set(x_135, 2, x_134); +x_136 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__81; +x_137 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_137, 0, x_122); +lean_ctor_set(x_137, 1, x_136); +x_138 = lean_array_push(x_85, x_128); +x_139 = lean_array_push(x_138, x_135); +x_140 = lean_array_push(x_139, x_137); +x_141 = lean_array_push(x_140, x_120); +lean_inc(x_127); +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_45); +lean_ctor_set(x_142, 1, x_127); +lean_ctor_set(x_142, 2, x_141); +x_143 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100; +x_144 = l_Lean_Name_str___override(x_5, x_143); +lean_inc(x_17); +lean_inc(x_98); +x_145 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_6, x_65, x_68, x_75, x_79, x_144, x_100, x_22, x_98, x_13, x_14, x_15, x_16, x_17, x_18, x_125); +lean_dec(x_16); +lean_dec(x_15); x_146 = lean_ctor_get(x_145, 0); lean_inc(x_146); x_147 = lean_ctor_get(x_145, 1); lean_inc(x_147); lean_dec(x_145); -x_148 = lean_st_ref_get(x_15, x_147); -lean_dec(x_15); -x_149 = !lean_is_exclusive(x_148); -if (x_149 == 0) -{ -lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; uint8_t x_163; -x_150 = lean_ctor_get(x_148, 0); -lean_dec(x_150); -lean_inc(x_146); -x_151 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_151, 0, x_146); -lean_ctor_set(x_151, 1, x_33); -x_152 = l_Lean_Syntax_mkApp(x_90, x_115); -x_153 = lean_array_push(x_58, x_152); -x_154 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_154, 0, x_35); -lean_ctor_set(x_154, 1, x_36); -lean_ctor_set(x_154, 2, x_153); -x_155 = lean_array_push(x_58, x_154); +x_148 = l_Lean_Syntax_mkApp(x_130, x_146); +lean_inc(x_17); +x_149 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_17, x_18, x_147); +x_150 = lean_ctor_get(x_149, 0); +lean_inc(x_150); +x_151 = lean_ctor_get(x_149, 1); +lean_inc(x_151); +lean_dec(x_149); +x_152 = lean_st_ref_get(x_18, x_151); +x_153 = lean_ctor_get(x_152, 1); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_154, 0, x_150); +lean_ctor_set(x_154, 1, x_114); +x_155 = lean_array_push(x_79, x_148); x_156 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_156, 0, x_35); -lean_ctor_set(x_156, 1, x_36); +lean_ctor_set(x_156, 0, x_45); +lean_ctor_set(x_156, 1, x_65); lean_ctor_set(x_156, 2, x_155); -x_157 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_157, 0, x_146); -lean_ctor_set(x_157, 1, x_121); -x_158 = lean_array_push(x_65, x_151); -x_159 = lean_array_push(x_158, x_156); -x_160 = lean_array_push(x_159, x_157); -x_161 = lean_array_push(x_160, x_144); -x_162 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_162, 0, x_35); -lean_ctor_set(x_162, 1, x_127); -lean_ctor_set(x_162, 2, x_161); -x_163 = !lean_is_exclusive(x_6); -if (x_163 == 0) -{ -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -x_164 = lean_ctor_get(x_6, 3); -x_165 = lean_ctor_get(x_6, 4); -x_166 = lean_ctor_get(x_6, 5); -x_167 = lean_array_push(x_164, x_71); -x_168 = lean_array_push(x_165, x_128); -x_169 = lean_array_push(x_166, x_162); -lean_ctor_set(x_6, 5, x_169); -lean_ctor_set(x_6, 4, x_168); -lean_ctor_set(x_6, 3, x_167); -lean_ctor_set(x_148, 0, x_6); -return x_148; -} -else -{ -lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_170 = lean_ctor_get(x_6, 0); -x_171 = lean_ctor_get(x_6, 1); -x_172 = lean_ctor_get(x_6, 2); -x_173 = lean_ctor_get(x_6, 3); -x_174 = lean_ctor_get(x_6, 4); -x_175 = lean_ctor_get(x_6, 5); -lean_inc(x_175); -lean_inc(x_174); -lean_inc(x_173); -lean_inc(x_172); -lean_inc(x_171); -lean_inc(x_170); -lean_dec(x_6); -x_176 = lean_array_push(x_173, x_71); -x_177 = lean_array_push(x_174, x_128); -x_178 = lean_array_push(x_175, x_162); -x_179 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_179, 0, x_170); -lean_ctor_set(x_179, 1, x_171); -lean_ctor_set(x_179, 2, x_172); -lean_ctor_set(x_179, 3, x_176); -lean_ctor_set(x_179, 4, x_177); -lean_ctor_set(x_179, 5, x_178); -lean_ctor_set(x_148, 0, x_179); -return x_148; -} -} -else +x_157 = lean_array_push(x_75, x_154); +x_158 = lean_array_push(x_157, x_156); +x_159 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_159, 0, x_45); +lean_ctor_set(x_159, 1, x_113); +lean_ctor_set(x_159, 2, x_158); +x_160 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_17, x_18, x_153); +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = lean_st_ref_get(x_18, x_162); +lean_dec(x_18); +x_164 = !lean_is_exclusive(x_163); +if (x_164 == 0) { -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; -x_180 = lean_ctor_get(x_148, 1); +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; +x_165 = lean_ctor_get(x_163, 0); +lean_dec(x_165); +lean_inc(x_161); +x_166 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_166, 0, x_161); +lean_ctor_set(x_166, 1, x_41); +x_167 = l_Lean_Syntax_mkApp(x_105, x_98); +x_168 = lean_array_push(x_79, x_167); +x_169 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_169, 0, x_45); +lean_ctor_set(x_169, 1, x_65); +lean_ctor_set(x_169, 2, x_168); +x_170 = lean_array_push(x_79, x_169); +x_171 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_171, 0, x_45); +lean_ctor_set(x_171, 1, x_65); +lean_ctor_set(x_171, 2, x_170); +x_172 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_172, 0, x_161); +lean_ctor_set(x_172, 1, x_136); +x_173 = lean_array_push(x_85, x_166); +x_174 = lean_array_push(x_173, x_171); +x_175 = lean_array_push(x_174, x_172); +x_176 = lean_array_push(x_175, x_159); +x_177 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_177, 0, x_45); +lean_ctor_set(x_177, 1, x_127); +lean_ctor_set(x_177, 2, x_176); +x_178 = lean_ctor_get(x_9, 0); +lean_inc(x_178); +x_179 = lean_array_push(x_178, x_90); +x_180 = lean_ctor_get(x_9, 1); lean_inc(x_180); -lean_dec(x_148); -lean_inc(x_146); -x_181 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_181, 0, x_146); -lean_ctor_set(x_181, 1, x_33); -x_182 = l_Lean_Syntax_mkApp(x_90, x_115); -x_183 = lean_array_push(x_58, x_182); -x_184 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_184, 0, x_35); -lean_ctor_set(x_184, 1, x_36); +x_181 = lean_array_push(x_180, x_142); +x_182 = lean_ctor_get(x_9, 2); +lean_inc(x_182); +lean_dec(x_9); +x_183 = lean_array_push(x_182, x_177); +x_184 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_184, 0, x_179); +lean_ctor_set(x_184, 1, x_181); lean_ctor_set(x_184, 2, x_183); -x_185 = lean_array_push(x_58, x_184); -x_186 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_186, 0, x_35); -lean_ctor_set(x_186, 1, x_36); -lean_ctor_set(x_186, 2, x_185); -x_187 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_187, 0, x_146); -lean_ctor_set(x_187, 1, x_121); -x_188 = lean_array_push(x_65, x_181); -x_189 = lean_array_push(x_188, x_186); -x_190 = lean_array_push(x_189, x_187); -x_191 = lean_array_push(x_190, x_144); -x_192 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_192, 0, x_35); -lean_ctor_set(x_192, 1, x_127); -lean_ctor_set(x_192, 2, x_191); -x_193 = lean_ctor_get(x_6, 0); -lean_inc(x_193); -x_194 = lean_ctor_get(x_6, 1); -lean_inc(x_194); -x_195 = lean_ctor_get(x_6, 2); -lean_inc(x_195); -x_196 = lean_ctor_get(x_6, 3); -lean_inc(x_196); -x_197 = lean_ctor_get(x_6, 4); -lean_inc(x_197); -x_198 = lean_ctor_get(x_6, 5); -lean_inc(x_198); -if (lean_is_exclusive(x_6)) { - lean_ctor_release(x_6, 0); - lean_ctor_release(x_6, 1); - lean_ctor_release(x_6, 2); - lean_ctor_release(x_6, 3); - lean_ctor_release(x_6, 4); - lean_ctor_release(x_6, 5); - x_199 = x_6; -} else { - lean_dec_ref(x_6); - x_199 = lean_box(0); -} -x_200 = lean_array_push(x_196, x_71); -x_201 = lean_array_push(x_197, x_128); -x_202 = lean_array_push(x_198, x_192); -if (lean_is_scalar(x_199)) { - x_203 = lean_alloc_ctor(0, 6, 0); -} else { - x_203 = x_199; -} -lean_ctor_set(x_203, 0, x_193); -lean_ctor_set(x_203, 1, x_194); -lean_ctor_set(x_203, 2, x_195); -lean_ctor_set(x_203, 3, x_200); -lean_ctor_set(x_203, 4, x_201); -lean_ctor_set(x_203, 5, x_202); -x_204 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_204, 0, x_203); -lean_ctor_set(x_204, 1, x_180); -return x_204; -} -} -else -{ -uint8_t x_205; -lean_dec(x_71); -lean_dec(x_47); -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_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_205 = !lean_is_exclusive(x_74); -if (x_205 == 0) -{ -return x_74; +lean_ctor_set(x_163, 0, x_184); +return x_163; } else { -lean_object* x_206; lean_object* x_207; lean_object* x_208; -x_206 = lean_ctor_get(x_74, 0); -x_207 = lean_ctor_get(x_74, 1); -lean_inc(x_207); -lean_inc(x_206); -lean_dec(x_74); -x_208 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_208, 0, x_206); -lean_ctor_set(x_208, 1, x_207); -return x_208; -} +lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; +x_185 = lean_ctor_get(x_163, 1); +lean_inc(x_185); +lean_dec(x_163); +lean_inc(x_161); +x_186 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_186, 0, x_161); +lean_ctor_set(x_186, 1, x_41); +x_187 = l_Lean_Syntax_mkApp(x_105, x_98); +x_188 = lean_array_push(x_79, x_187); +x_189 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_189, 0, x_45); +lean_ctor_set(x_189, 1, x_65); +lean_ctor_set(x_189, 2, x_188); +x_190 = lean_array_push(x_79, x_189); +x_191 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_191, 0, x_45); +lean_ctor_set(x_191, 1, x_65); +lean_ctor_set(x_191, 2, x_190); +x_192 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_192, 0, x_161); +lean_ctor_set(x_192, 1, x_136); +x_193 = lean_array_push(x_85, x_186); +x_194 = lean_array_push(x_193, x_191); +x_195 = lean_array_push(x_194, x_192); +x_196 = lean_array_push(x_195, x_159); +x_197 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_197, 0, x_45); +lean_ctor_set(x_197, 1, x_127); +lean_ctor_set(x_197, 2, x_196); +x_198 = lean_ctor_get(x_9, 0); +lean_inc(x_198); +x_199 = lean_array_push(x_198, x_90); +x_200 = lean_ctor_get(x_9, 1); +lean_inc(x_200); +x_201 = lean_array_push(x_200, x_142); +x_202 = lean_ctor_get(x_9, 2); +lean_inc(x_202); +lean_dec(x_9); +x_203 = lean_array_push(x_202, x_197); +x_204 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_204, 0, x_199); +lean_ctor_set(x_204, 1, x_201); +lean_ctor_set(x_204, 2, x_203); +x_205 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_205, 0, x_204); +lean_ctor_set(x_205, 1, x_185); +return x_205; } } else { -uint8_t x_209; +uint8_t x_206; +lean_dec(x_90); +lean_dec(x_68); +lean_dec(x_48); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); -lean_dec(x_6); +lean_dec(x_7); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_209 = !lean_is_exclusive(x_25); -if (x_209 == 0) +x_206 = !lean_is_exclusive(x_91); +if (x_206 == 0) { -return x_25; +return x_91; } -else -{ -lean_object* x_210; lean_object* x_211; lean_object* x_212; -x_210 = lean_ctor_get(x_25, 0); -x_211 = lean_ctor_get(x_25, 1); -lean_inc(x_211); -lean_inc(x_210); -lean_dec(x_25); -x_212 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_212, 0, x_210); -lean_ctor_set(x_212, 1, x_211); -return x_212; +else +{ +lean_object* x_207; lean_object* x_208; lean_object* x_209; +x_207 = lean_ctor_get(x_91, 0); +x_208 = lean_ctor_get(x_91, 1); +lean_inc(x_208); +lean_inc(x_207); +lean_dec(x_91); +x_209 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_209, 0, x_207); +lean_ctor_set(x_209, 1, x_208); +return x_209; } } } else { -uint8_t x_213; +uint8_t x_210; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); -lean_dec(x_6); +lean_dec(x_7); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_213 = !lean_is_exclusive(x_21); -if (x_213 == 0) +x_210 = !lean_is_exclusive(x_23); +if (x_210 == 0) { -return x_21; +return x_23; } else { -lean_object* x_214; lean_object* x_215; lean_object* x_216; -x_214 = lean_ctor_get(x_21, 0); -x_215 = lean_ctor_get(x_21, 1); -lean_inc(x_215); -lean_inc(x_214); -lean_dec(x_21); -x_216 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_216, 0, x_214); -lean_ctor_set(x_216, 1, x_215); -return x_216; +lean_object* x_211; lean_object* x_212; lean_object* x_213; +x_211 = lean_ctor_get(x_23, 0); +x_212 = lean_ctor_get(x_23, 1); +lean_inc(x_212); +lean_inc(x_211); +lean_dec(x_23); +x_213 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_213, 0, x_211); +lean_ctor_set(x_213, 1, x_212); +return x_213; +} } } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +x_2 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +lean_ctor_set(x_2, 2, x_1); +return x_2; +} } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__1() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2() { _start: { lean_object* x_1; @@ -17411,53 +9451,170 @@ x_1 = lean_mk_string_from_bytes("inductive", 9); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__2() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("partial", 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("structInstFieldAbbrev", 21); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("whereDecls", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("letRecDecl", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("implicitBinder", 14); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("m", 1); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__8; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__8; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__9; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__8; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__1; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__8; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__3() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__12() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("fun", 3); +x_1 = lean_mk_string_from_bytes("Monad", 5); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__4() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__12; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__12; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__13; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__5() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("basicFun", 8); +x_1 = lean_mk_string_from_bytes("MonadRpcSession", 15); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__6() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__17; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__5; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__7() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__20() { _start: { lean_object* x_1; @@ -17465,22 +9622,22 @@ x_1 = lean_mk_string_from_bytes("x", 1); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__8() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__21() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__7; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__20; x_2 = lean_string_utf8_byte_size(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__9() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__7; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__20; x_2 = lean_unsigned_to_nat(0u); -x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__8; +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__21; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -17488,53 +9645,139 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__10() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__7; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__20; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__11() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__24() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("match", 5); +x_1 = lean_mk_string_from_bytes("ExceptT", 7); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__12() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__25() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__24; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__26() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__24; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__25; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__27() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__11; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__24; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__13() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__28() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("matchDiscr", 10); +x_1 = lean_mk_string_from_bytes("String", 6); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__14() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__29() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__28; +x_2 = lean_string_utf8_byte_size(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__30() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__28; +x_2 = lean_unsigned_to_nat(0u); +x_3 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__29; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__31() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__13; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__28; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__15() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__32() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("have", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__33() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("haveDecl", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__34() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("haveIdDecl", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__35() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("match", 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__36() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("matchDiscr", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__37() { _start: { lean_object* x_1; @@ -17542,7 +9785,7 @@ x_1 = lean_mk_string_from_bytes("with", 4); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__16() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__38() { _start: { lean_object* x_1; @@ -17550,1761 +9793,2791 @@ x_1 = lean_mk_string_from_bytes("matchAlts", 9); return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__17() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__39() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__16; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__40() { _start: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__15; -x_16 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_15, x_12, x_13, x_14); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_box_usize(x_2); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_1); -lean_inc(x_17); -x_20 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___boxed), 16, 5); -lean_closure_set(x_20, 0, x_17); -lean_closure_set(x_20, 1, x_1); -lean_closure_set(x_20, 2, x_19); -lean_closure_set(x_20, 3, x_3); -lean_closure_set(x_20, 4, x_4); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__39; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23) { +_start: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_inc(x_8); +lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_21 = l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__33___rarg(x_4, x_5, x_20, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_18); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; size_t x_25; lean_object* x_26; -x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_24 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___boxed), 19, 8); +lean_closure_set(x_24, 0, x_1); +lean_closure_set(x_24, 1, x_2); +lean_closure_set(x_24, 2, x_3); +lean_closure_set(x_24, 3, x_4); +lean_closure_set(x_24, 4, x_5); +lean_closure_set(x_24, 5, x_6); +lean_closure_set(x_24, 6, x_7); +lean_closure_set(x_24, 7, x_8); +x_25 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__1; lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_array_get_size(x_5); -x_25 = lean_usize_of_nat(x_24); -lean_dec(x_24); -x_26 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__20(x_25, x_2, x_5, x_8, x_9, x_10, x_11, x_12, x_13, x_23); -lean_dec(x_11); -lean_dec(x_9); -lean_dec(x_8); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_10); +x_26 = l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9___rarg(x_9, x_10, x_24, x_25, x_17, x_18, x_19, x_20, x_21, x_22, x_23); if (lean_obj_tag(x_26) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; 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; size_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; size_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +lean_object* x_27; lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; lean_object* x_32; x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -lean_inc(x_12); -x_29 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_12, x_13, x_28); -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); +x_29 = lean_array_get_size(x_10); +x_30 = lean_usize_of_nat(x_29); lean_dec(x_29); -x_32 = lean_st_ref_get(x_13, x_31); -x_33 = lean_ctor_get(x_32, 1); +x_31 = 0; +x_32 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4(x_30, x_31, x_10, x_17, x_18, x_19, x_20, x_21, x_22, x_28); +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_17); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; 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; size_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; +x_33 = lean_ctor_get(x_32, 0); lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); lean_dec(x_32); -x_34 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__9; -lean_inc(x_1); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_1); -x_36 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__13; -x_37 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_37, 0, x_30); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_ctor_get(x_4, 0); -lean_inc(x_38); -lean_dec(x_4); -x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_21); +x_35 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_21, x_22, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_st_ref_get(x_22, x_37); +x_39 = lean_ctor_get(x_38, 1); lean_inc(x_39); lean_dec(x_38); -x_40 = lean_mk_syntax_ident(x_39); -x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_42 = lean_array_push(x_41, x_37); -x_43 = lean_array_push(x_42, x_40); -x_44 = lean_box(2); -x_45 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12; -x_46 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_43); -x_47 = lean_array_get_size(x_27); -x_48 = lean_usize_of_nat(x_47); -lean_dec(x_47); -x_49 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__42(x_1, x_35, x_48, x_2, x_27); -x_50 = l_Lean_Syntax_mkApp(x_46, x_49); -x_51 = lean_mk_syntax_ident(x_17); -x_52 = lean_ctor_get(x_22, 1); -lean_inc(x_52); -x_53 = lean_array_get_size(x_52); -x_54 = lean_usize_of_nat(x_53); -lean_dec(x_53); -x_55 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__43(x_35, x_54, x_2, x_52); -lean_dec(x_35); -lean_inc(x_51); -x_56 = l_Lean_Syntax_mkApp(x_51, x_55); -lean_inc(x_12); -x_57 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_12, x_13, x_33); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -x_60 = lean_ctor_get(x_12, 10); -lean_inc(x_60); -lean_dec(x_12); -x_61 = lean_st_ref_get(x_13, x_59); -lean_dec(x_13); -x_62 = !lean_is_exclusive(x_61); -if (x_62 == 0) -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; size_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; size_t x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; size_t x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; -x_63 = lean_ctor_get(x_61, 0); +x_40 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__5; +lean_inc(x_2); +x_41 = l_Lean_Name_str___override(x_2, x_40); +x_42 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__34; +lean_inc(x_41); +x_43 = l_Lean_Name_str___override(x_41, x_42); +x_44 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__6; +lean_inc(x_43); +x_45 = l_Lean_Name_str___override(x_43, x_44); +x_46 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__8; +x_47 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_47, 0, x_36); +lean_ctor_set(x_47, 1, x_46); +lean_inc(x_8); +x_48 = lean_mk_syntax_ident(x_8); +x_49 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_50 = lean_array_push(x_49, x_47); +x_51 = lean_array_push(x_50, x_48); +x_52 = lean_box(2); +x_53 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_45); +lean_ctor_set(x_53, 2, x_51); +x_54 = lean_array_get_size(x_33); +x_55 = lean_usize_of_nat(x_54); +lean_dec(x_54); +x_56 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_6, x_55, x_31, x_33); +lean_dec(x_6); +x_57 = l_Lean_Syntax_mkApp(x_53, x_56); +x_58 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__11; +x_59 = lean_name_append_before(x_8, x_58); +x_60 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__10; +x_61 = l_Lean_Name_append(x_60, x_59); +x_62 = lean_mk_syntax_ident(x_61); +lean_inc(x_21); +x_63 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_21, x_22, x_39); x_64 = lean_ctor_get(x_63, 0); lean_inc(x_64); +x_65 = lean_ctor_get(x_63, 1); +lean_inc(x_65); lean_dec(x_63); -x_65 = lean_environment_main_module(x_64); -x_66 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; -lean_inc(x_58); -x_67 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_67, 0, x_58); -lean_ctor_set(x_67, 1, x_66); -x_68 = lean_ctor_get(x_22, 2); -lean_inc(x_68); -lean_inc(x_3); -x_69 = l_Array_append___rarg(x_3, x_68); -x_70 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_71 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_71, 0, x_44); -lean_ctor_set(x_71, 1, x_70); -lean_ctor_set(x_71, 2, x_69); -x_72 = lean_array_push(x_41, x_67); -x_73 = lean_array_push(x_72, x_71); -x_74 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; -x_75 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_75, 0, x_44); -lean_ctor_set(x_75, 1, x_74); -lean_ctor_set(x_75, 2, x_73); -lean_inc(x_3); -x_76 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_76, 0, x_44); -lean_ctor_set(x_76, 1, x_70); -lean_ctor_set(x_76, 2, x_3); -x_77 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -lean_inc(x_76); -x_78 = lean_array_push(x_77, x_76); -lean_inc(x_76); -x_79 = lean_array_push(x_78, x_76); -lean_inc(x_76); -x_80 = lean_array_push(x_79, x_76); -lean_inc(x_76); -x_81 = lean_array_push(x_80, x_76); -lean_inc(x_76); -x_82 = lean_array_push(x_81, x_76); -lean_inc(x_76); -x_83 = lean_array_push(x_82, x_76); -x_84 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; +x_66 = lean_ctor_get(x_21, 10); +lean_inc(x_66); +lean_dec(x_21); +x_67 = lean_st_ref_get(x_22, x_65); +lean_dec(x_22); +x_68 = !lean_is_exclusive(x_67); +if (x_68 == 0) +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; size_t x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; size_t x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; size_t x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; lean_object* x_551; lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; lean_object* x_570; lean_object* x_571; +x_69 = lean_ctor_get(x_67, 0); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +lean_dec(x_69); +x_71 = lean_environment_main_module(x_70); +x_72 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__7; +lean_inc(x_41); +x_73 = l_Lean_Name_str___override(x_41, x_72); +x_74 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12; +lean_inc(x_73); +x_75 = l_Lean_Name_str___override(x_73, x_74); +x_76 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14; +lean_inc(x_73); +x_77 = l_Lean_Name_str___override(x_73, x_76); +lean_inc(x_64); +x_78 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_78, 0, x_64); +lean_ctor_set(x_78, 1, x_76); +x_79 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +lean_inc(x_11); +x_80 = l_Array_append___rarg(x_79, x_11); +x_81 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_82 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_82, 0, x_52); +lean_ctor_set(x_82, 1, x_81); +lean_ctor_set(x_82, 2, x_80); +x_83 = lean_array_push(x_49, x_78); +lean_inc(x_83); +x_84 = lean_array_push(x_83, x_82); +lean_inc(x_77); x_85 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_85, 0, x_44); -lean_ctor_set(x_85, 1, x_84); -lean_ctor_set(x_85, 2, x_83); -x_86 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__1; -lean_inc(x_58); -x_87 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_87, 0, x_58); -lean_ctor_set(x_87, 1, x_86); -x_88 = lean_array_push(x_41, x_51); -lean_inc(x_76); -x_89 = lean_array_push(x_88, x_76); -x_90 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; -x_91 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_91, 0, x_44); -lean_ctor_set(x_91, 1, x_90); -lean_ctor_set(x_91, 2, x_89); -lean_inc(x_76); -x_92 = lean_array_push(x_41, x_76); -lean_inc(x_76); -lean_inc(x_92); -x_93 = lean_array_push(x_92, x_76); -x_94 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56; -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_44); -lean_ctor_set(x_95, 1, x_94); -lean_ctor_set(x_95, 2, x_93); -x_96 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28; -lean_inc(x_58); -x_97 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_97, 0, x_58); -lean_ctor_set(x_97, 1, x_96); -x_98 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; +lean_ctor_set(x_85, 0, x_52); +lean_ctor_set(x_85, 1, x_77); +lean_ctor_set(x_85, 2, x_84); +lean_inc(x_64); +x_86 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_86, 0, x_64); +lean_ctor_set(x_86, 1, x_74); +x_87 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__9; +lean_inc(x_73); +x_88 = l_Lean_Name_str___override(x_73, x_87); +x_89 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; +lean_inc(x_73); +x_90 = l_Lean_Name_str___override(x_73, x_89); +x_91 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__22; +lean_inc(x_90); +x_92 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_92, 0, x_52); +lean_ctor_set(x_92, 1, x_90); +lean_ctor_set(x_92, 2, x_91); +x_93 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2; +lean_inc(x_73); +x_94 = l_Lean_Name_str___override(x_73, x_93); +lean_inc(x_64); +x_95 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_95, 0, x_64); +lean_ctor_set(x_95, 1, x_93); +x_96 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; +lean_inc(x_73); +x_97 = l_Lean_Name_str___override(x_73, x_96); +lean_inc(x_66); +lean_inc(x_71); +x_98 = l_Lean_addMacroScope(x_71, x_3, x_66); +lean_inc(x_1); +lean_inc(x_64); +x_99 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_99, 0, x_64); +lean_ctor_set(x_99, 1, x_4); +lean_ctor_set(x_99, 2, x_98); +lean_ctor_set(x_99, 3, x_1); +x_100 = lean_array_push(x_49, x_99); +x_101 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +lean_inc(x_100); +x_102 = lean_array_push(x_100, x_101); lean_inc(x_97); -x_99 = lean_array_push(x_98, x_97); -x_100 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_100, 0, x_44); -lean_ctor_set(x_100, 1, x_70); -lean_ctor_set(x_100, 2, x_99); -x_101 = lean_ctor_get(x_22, 3); -lean_inc(x_101); -x_102 = lean_array_get_size(x_101); -x_103 = lean_usize_of_nat(x_102); -lean_dec(x_102); -x_104 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__44(x_103, x_2, x_101); -lean_inc(x_3); -x_105 = l_Array_append___rarg(x_3, x_104); -x_106 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_106, 0, x_44); -lean_ctor_set(x_106, 1, x_70); -lean_ctor_set(x_106, 2, x_105); -x_107 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33; -lean_inc(x_58); -x_108 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_108, 0, x_58); -lean_ctor_set(x_108, 1, x_107); -x_109 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; -lean_inc(x_76); -x_110 = lean_array_push(x_109, x_76); -x_111 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35; +x_103 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_103, 0, x_52); +lean_ctor_set(x_103, 1, x_97); +lean_ctor_set(x_103, 2, x_102); +x_104 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__32; +lean_inc(x_73); +x_105 = l_Lean_Name_str___override(x_73, x_104); +x_106 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60; +x_107 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_107, 0, x_52); +lean_ctor_set(x_107, 1, x_105); +lean_ctor_set(x_107, 2, x_106); +x_108 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__76; +lean_inc(x_64); +x_109 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_109, 0, x_64); +lean_ctor_set(x_109, 1, x_108); +x_110 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +lean_inc(x_109); +x_111 = lean_array_push(x_110, x_109); x_112 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_112, 0, x_44); -lean_ctor_set(x_112, 1, x_111); -lean_ctor_set(x_112, 2, x_110); -x_113 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; -lean_inc(x_58); -x_114 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_114, 0, x_58); -lean_ctor_set(x_114, 1, x_113); -x_115 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; -lean_inc(x_76); -x_116 = lean_array_push(x_115, x_76); -x_117 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_117, 0, x_44); -lean_ctor_set(x_117, 1, x_111); -lean_ctor_set(x_117, 2, x_116); -x_118 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; -x_119 = lean_array_push(x_118, x_112); -x_120 = lean_array_push(x_119, x_114); -x_121 = lean_array_push(x_120, x_117); -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_44); -lean_ctor_set(x_122, 1, x_70); -lean_ctor_set(x_122, 2, x_121); -x_123 = lean_array_push(x_41, x_108); -x_124 = lean_array_push(x_123, x_122); -x_125 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_125, 0, x_44); -lean_ctor_set(x_125, 1, x_70); -lean_ctor_set(x_125, 2, x_124); -x_126 = lean_array_push(x_98, x_125); -x_127 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__32; -x_128 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_128, 0, x_44); -lean_ctor_set(x_128, 1, x_127); -lean_ctor_set(x_128, 2, x_126); -x_129 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; -x_130 = lean_array_push(x_129, x_87); -x_131 = lean_array_push(x_130, x_91); -x_132 = lean_array_push(x_131, x_95); -x_133 = lean_array_push(x_132, x_100); -x_134 = lean_array_push(x_133, x_106); -lean_inc(x_76); -x_135 = lean_array_push(x_134, x_76); -x_136 = lean_array_push(x_135, x_128); -x_137 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__2; -x_138 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_138, 0, x_44); -lean_ctor_set(x_138, 1, x_137); -lean_ctor_set(x_138, 2, x_136); -x_139 = lean_array_push(x_41, x_85); -lean_inc(x_139); -x_140 = lean_array_push(x_139, x_138); -x_141 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__37; -x_142 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_142, 0, x_44); -lean_ctor_set(x_142, 1, x_141); -lean_ctor_set(x_142, 2, x_140); -lean_inc(x_76); -x_143 = lean_array_push(x_98, x_76); -x_144 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__124; -x_145 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_145, 0, x_44); -lean_ctor_set(x_145, 1, x_144); -lean_ctor_set(x_145, 2, x_143); -x_146 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205; -lean_inc(x_58); -x_147 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_147, 0, x_58); -lean_ctor_set(x_147, 1, x_146); -x_148 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; -lean_inc(x_58); -x_149 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_149, 0, x_58); -lean_ctor_set(x_149, 1, x_148); -x_150 = lean_array_push(x_41, x_50); -x_151 = lean_array_push(x_150, x_56); -x_152 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_152, 0, x_44); -lean_ctor_set(x_152, 1, x_70); -lean_ctor_set(x_152, 2, x_151); -x_153 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53; -x_154 = lean_array_push(x_153, x_152); -x_155 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_156 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_156, 0, x_44); -lean_ctor_set(x_156, 1, x_155); -lean_ctor_set(x_156, 2, x_154); -x_157 = lean_array_push(x_41, x_149); -x_158 = lean_array_push(x_157, x_156); -x_159 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95; -x_160 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_160, 0, x_44); -lean_ctor_set(x_160, 1, x_159); -lean_ctor_set(x_160, 2, x_158); -lean_inc(x_92); -x_161 = lean_array_push(x_92, x_160); -x_162 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__143; -x_163 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_163, 0, x_44); -lean_ctor_set(x_163, 1, x_162); -lean_ctor_set(x_163, 2, x_161); -x_164 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224; -lean_inc(x_60); -lean_inc(x_65); -x_165 = l_Lean_addMacroScope(x_65, x_164, x_60); -x_166 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225; +lean_ctor_set(x_112, 0, x_52); +lean_ctor_set(x_112, 1, x_81); +lean_ctor_set(x_112, 2, x_111); +x_113 = lean_ctor_get(x_27, 0); +lean_inc(x_113); +x_114 = lean_array_get_size(x_113); +x_115 = lean_usize_of_nat(x_114); +lean_dec(x_114); +x_116 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(x_115, x_31, x_113); +x_117 = l_Array_append___rarg(x_79, x_116); +x_118 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_118, 0, x_52); +lean_ctor_set(x_118, 1, x_81); +lean_ctor_set(x_118, 2, x_117); +x_119 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__34; +lean_inc(x_73); +x_120 = l_Lean_Name_str___override(x_73, x_119); +x_121 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__36; +lean_inc(x_64); +x_122 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_122, 0, x_64); +lean_ctor_set(x_122, 1, x_121); +x_123 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; +lean_inc(x_66); +lean_inc(x_71); +x_124 = l_Lean_addMacroScope(x_71, x_123, x_66); +x_125 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; +lean_inc(x_2); +x_126 = l_Lean_Name_str___override(x_2, x_125); lean_inc(x_1); -x_167 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_167, 0, x_166); -lean_ctor_set(x_167, 1, x_1); +x_127 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_127, 0, x_126); +lean_ctor_set(x_127, 1, x_1); lean_inc(x_1); -x_168 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_168, 0, x_167); -lean_ctor_set(x_168, 1, x_1); -x_169 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223; -lean_inc(x_58); -x_170 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_170, 0, x_58); -lean_ctor_set(x_170, 1, x_169); -lean_ctor_set(x_170, 2, x_165); -lean_ctor_set(x_170, 3, x_168); -x_171 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; -lean_inc(x_58); -x_172 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_172, 0, x_58); -lean_ctor_set(x_172, 1, x_171); -x_173 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__3; -lean_inc(x_58); -x_174 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_174, 0, x_58); -lean_ctor_set(x_174, 1, x_173); -x_175 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__10; -lean_inc(x_60); -lean_inc(x_65); -x_176 = l_Lean_addMacroScope(x_65, x_175, x_60); -x_177 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__9; +x_128 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_128, 0, x_127); +lean_ctor_set(x_128, 1, x_1); +x_129 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__41; +lean_inc(x_64); +x_130 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_130, 0, x_64); +lean_ctor_set(x_130, 1, x_129); +lean_ctor_set(x_130, 2, x_124); +lean_ctor_set(x_130, 3, x_128); +x_131 = lean_array_push(x_49, x_130); +x_132 = lean_array_push(x_131, x_101); +x_133 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__38; +x_134 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_134, 0, x_52); +lean_ctor_set(x_134, 1, x_133); +lean_ctor_set(x_134, 2, x_132); +x_135 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; +lean_inc(x_64); +x_136 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_136, 0, x_64); +lean_ctor_set(x_136, 1, x_135); +x_137 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50; +lean_inc(x_66); +lean_inc(x_71); +x_138 = l_Lean_addMacroScope(x_71, x_137, x_66); +x_139 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47; +x_140 = l_Lean_Name_str___override(x_2, x_139); lean_inc(x_1); -lean_inc(x_58); -x_178 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_178, 0, x_58); -lean_ctor_set(x_178, 1, x_177); -lean_ctor_set(x_178, 2, x_176); -lean_ctor_set(x_178, 3, x_1); -lean_inc(x_178); -x_179 = lean_array_push(x_98, x_178); -x_180 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_180, 0, x_44); -lean_ctor_set(x_180, 1, x_70); -lean_ctor_set(x_180, 2, x_179); -x_181 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__6; -lean_inc(x_58); -x_182 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_182, 0, x_58); -lean_ctor_set(x_182, 1, x_181); -x_183 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__11; -lean_inc(x_58); -x_184 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_184, 0, x_58); -lean_ctor_set(x_184, 1, x_183); -x_185 = lean_array_push(x_92, x_178); -x_186 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__14; -x_187 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_187, 0, x_44); -lean_ctor_set(x_187, 1, x_186); -lean_ctor_set(x_187, 2, x_185); -x_188 = lean_array_push(x_98, x_187); +x_141 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_141, 0, x_140); +lean_ctor_set(x_141, 1, x_1); +lean_inc(x_1); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_141); +lean_ctor_set(x_142, 1, x_1); +x_143 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49; +lean_inc(x_64); +x_144 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_144, 0, x_64); +lean_ctor_set(x_144, 1, x_143); +lean_ctor_set(x_144, 2, x_138); +lean_ctor_set(x_144, 3, x_142); +x_145 = lean_array_push(x_49, x_144); +x_146 = lean_array_push(x_145, x_101); +x_147 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_147, 0, x_52); +lean_ctor_set(x_147, 1, x_133); +lean_ctor_set(x_147, 2, x_146); +x_148 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +x_149 = lean_array_push(x_148, x_134); +lean_inc(x_136); +x_150 = lean_array_push(x_149, x_136); +x_151 = lean_array_push(x_150, x_147); +x_152 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_152, 0, x_52); +lean_ctor_set(x_152, 1, x_81); +lean_ctor_set(x_152, 2, x_151); +x_153 = lean_array_push(x_49, x_122); +x_154 = lean_array_push(x_153, x_152); +x_155 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_155, 0, x_52); +lean_ctor_set(x_155, 1, x_81); +lean_ctor_set(x_155, 2, x_154); +x_156 = lean_array_push(x_110, x_155); +x_157 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_157, 0, x_52); +lean_ctor_set(x_157, 1, x_120); +lean_ctor_set(x_157, 2, x_156); +x_158 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116; +x_159 = lean_array_push(x_158, x_95); +x_160 = lean_array_push(x_159, x_103); +lean_inc(x_107); +x_161 = lean_array_push(x_160, x_107); +x_162 = lean_array_push(x_161, x_112); +x_163 = lean_array_push(x_162, x_118); +x_164 = lean_array_push(x_163, x_101); +x_165 = lean_array_push(x_164, x_157); +x_166 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_166, 0, x_52); +lean_ctor_set(x_166, 1, x_94); +lean_ctor_set(x_166, 2, x_165); +x_167 = lean_array_push(x_49, x_92); +x_168 = lean_array_push(x_167, x_166); +lean_inc(x_88); +x_169 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_169, 0, x_52); +lean_ctor_set(x_169, 1, x_88); +lean_ctor_set(x_169, 2, x_168); +x_170 = lean_array_push(x_148, x_85); +lean_inc(x_86); +x_171 = lean_array_push(x_170, x_86); +x_172 = lean_array_push(x_171, x_169); +lean_inc(x_75); +x_173 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_173, 0, x_52); +lean_ctor_set(x_173, 1, x_75); +lean_ctor_set(x_173, 2, x_172); +x_174 = l_Array_append___rarg(x_12, x_11); +x_175 = l_Array_append___rarg(x_174, x_13); +x_176 = l_Array_append___rarg(x_79, x_175); +x_177 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_177, 0, x_52); +lean_ctor_set(x_177, 1, x_81); +lean_ctor_set(x_177, 2, x_176); +x_178 = lean_array_push(x_83, x_177); +x_179 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_179, 0, x_52); +lean_ctor_set(x_179, 1, x_77); +lean_ctor_set(x_179, 2, x_178); +x_180 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; +lean_inc(x_43); +x_181 = l_Lean_Name_str___override(x_43, x_180); +x_182 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119; +lean_inc(x_64); +x_183 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_183, 0, x_64); +lean_ctor_set(x_183, 1, x_182); +x_184 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__120; +lean_inc(x_43); +x_185 = l_Lean_Name_str___override(x_43, x_184); +x_186 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__122; +lean_inc(x_43); +x_187 = l_Lean_Name_str___override(x_43, x_186); +x_188 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__55; x_189 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_189, 0, x_44); -lean_ctor_set(x_189, 1, x_70); +lean_ctor_set(x_189, 0, x_52); +lean_ctor_set(x_189, 1, x_187); lean_ctor_set(x_189, 2, x_188); -x_190 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__15; -lean_inc(x_58); -x_191 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_191, 0, x_58); -lean_ctor_set(x_191, 1, x_190); -x_192 = lean_ctor_get(x_22, 4); -lean_inc(x_192); -x_193 = lean_array_get_size(x_192); -x_194 = lean_usize_of_nat(x_193); -lean_dec(x_193); -x_195 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45(x_194, x_2, x_192); -lean_inc(x_3); -x_196 = l_Array_append___rarg(x_3, x_195); +x_190 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__126; +x_191 = l_Lean_Name_str___override(x_41, x_190); +x_192 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; +x_193 = l_Lean_Name_str___override(x_191, x_192); +lean_inc(x_64); +x_194 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_194, 0, x_64); +lean_ctor_set(x_194, 1, x_192); +x_195 = lean_array_push(x_49, x_194); +x_196 = lean_array_push(x_195, x_101); x_197 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_197, 0, x_44); -lean_ctor_set(x_197, 1, x_70); +lean_ctor_set(x_197, 0, x_52); +lean_ctor_set(x_197, 1, x_193); lean_ctor_set(x_197, 2, x_196); -x_198 = lean_array_push(x_98, x_197); -x_199 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__17; +x_198 = lean_array_push(x_49, x_189); +x_199 = lean_array_push(x_198, x_197); x_200 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_200, 0, x_44); -lean_ctor_set(x_200, 1, x_199); -lean_ctor_set(x_200, 2, x_198); -x_201 = lean_array_push(x_77, x_184); -lean_inc(x_76); -x_202 = lean_array_push(x_201, x_76); -lean_inc(x_76); -x_203 = lean_array_push(x_202, x_76); -x_204 = lean_array_push(x_203, x_189); -x_205 = lean_array_push(x_204, x_191); -lean_inc(x_205); -x_206 = lean_array_push(x_205, x_200); -x_207 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__12; +lean_ctor_set(x_200, 0, x_52); +lean_ctor_set(x_200, 1, x_185); +lean_ctor_set(x_200, 2, x_199); +x_201 = lean_array_push(x_110, x_200); +x_202 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_202, 0, x_52); +lean_ctor_set(x_202, 1, x_81); +lean_ctor_set(x_202, 2, x_201); +x_203 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; +lean_inc(x_64); +x_204 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_204, 0, x_64); +lean_ctor_set(x_204, 1, x_203); +x_205 = lean_array_push(x_148, x_183); +x_206 = lean_array_push(x_205, x_202); +lean_inc(x_204); +x_207 = lean_array_push(x_206, x_204); x_208 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_208, 0, x_44); -lean_ctor_set(x_208, 1, x_207); -lean_ctor_set(x_208, 2, x_206); -x_209 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_210 = lean_array_push(x_209, x_180); -lean_inc(x_76); -x_211 = lean_array_push(x_210, x_76); -x_212 = lean_array_push(x_211, x_182); -lean_inc(x_212); -x_213 = lean_array_push(x_212, x_208); -x_214 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__6; +lean_ctor_set(x_208, 0, x_52); +lean_ctor_set(x_208, 1, x_181); +lean_ctor_set(x_208, 2, x_207); +x_209 = lean_array_push(x_110, x_208); +x_210 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_210, 0, x_52); +lean_ctor_set(x_210, 1, x_81); +lean_ctor_set(x_210, 2, x_209); +x_211 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__3; +lean_inc(x_73); +x_212 = l_Lean_Name_str___override(x_73, x_211); +lean_inc(x_64); +x_213 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_213, 0, x_64); +lean_ctor_set(x_213, 1, x_211); +x_214 = lean_array_push(x_110, x_213); x_215 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_215, 0, x_44); -lean_ctor_set(x_215, 1, x_214); -lean_ctor_set(x_215, 2, x_213); -x_216 = lean_array_push(x_41, x_174); -lean_inc(x_216); -x_217 = lean_array_push(x_216, x_215); -x_218 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__4; -x_219 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_219, 0, x_44); -lean_ctor_set(x_219, 1, x_218); -lean_ctor_set(x_219, 2, x_217); -x_220 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_221 = lean_array_push(x_220, x_170); -lean_inc(x_76); -x_222 = lean_array_push(x_221, x_76); -lean_inc(x_76); -x_223 = lean_array_push(x_222, x_76); -lean_inc(x_172); -x_224 = lean_array_push(x_223, x_172); -x_225 = lean_array_push(x_224, x_219); -x_226 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; -x_227 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_227, 0, x_44); -lean_ctor_set(x_227, 1, x_226); -lean_ctor_set(x_227, 2, x_225); -x_228 = lean_array_push(x_98, x_227); -x_229 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60; +lean_ctor_set(x_215, 0, x_52); +lean_ctor_set(x_215, 1, x_212); +lean_ctor_set(x_215, 2, x_214); +x_216 = lean_array_push(x_110, x_215); +x_217 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_217, 0, x_52); +lean_ctor_set(x_217, 1, x_81); +lean_ctor_set(x_217, 2, x_216); +x_218 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17; +x_219 = lean_array_push(x_218, x_210); +x_220 = lean_array_push(x_219, x_101); +x_221 = lean_array_push(x_220, x_101); +x_222 = lean_array_push(x_221, x_101); +x_223 = lean_array_push(x_222, x_217); +x_224 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_224, 0, x_52); +lean_ctor_set(x_224, 1, x_90); +lean_ctor_set(x_224, 2, x_223); +x_225 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23; +lean_inc(x_73); +x_226 = l_Lean_Name_str___override(x_73, x_225); +lean_inc(x_64); +x_227 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_227, 0, x_64); +lean_ctor_set(x_227, 1, x_225); +x_228 = lean_array_push(x_49, x_62); +x_229 = lean_array_push(x_228, x_101); x_230 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_230, 0, x_44); -lean_ctor_set(x_230, 1, x_229); -lean_ctor_set(x_230, 2, x_228); -x_231 = lean_array_push(x_98, x_230); -x_232 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58; -x_233 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_233, 0, x_44); -lean_ctor_set(x_233, 1, x_232); -lean_ctor_set(x_233, 2, x_231); -x_234 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231; -x_235 = l_Lean_addMacroScope(x_65, x_234, x_60); -x_236 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232; +lean_ctor_set(x_230, 0, x_52); +lean_ctor_set(x_230, 1, x_97); +lean_ctor_set(x_230, 2, x_229); +x_231 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__149; +x_232 = l_Lean_Name_str___override(x_73, x_231); +x_233 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; +lean_inc(x_64); +x_234 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_234, 0, x_64); +lean_ctor_set(x_234, 1, x_233); +x_235 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; +lean_inc(x_43); +x_236 = l_Lean_Name_str___override(x_43, x_235); +lean_inc(x_64); +x_237 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_237, 0, x_64); +lean_ctor_set(x_237, 1, x_235); +x_238 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; +lean_inc(x_43); +x_239 = l_Lean_Name_str___override(x_43, x_238); +x_240 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; +lean_inc(x_66); +lean_inc(x_71); +x_241 = l_Lean_addMacroScope(x_71, x_240, x_66); lean_inc(x_1); -x_237 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_237, 0, x_236); -lean_ctor_set(x_237, 1, x_1); -x_238 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_238, 0, x_237); -lean_ctor_set(x_238, 1, x_1); -x_239 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230; -x_240 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_240, 0, x_58); -lean_ctor_set(x_240, 1, x_239); -lean_ctor_set(x_240, 2, x_235); -lean_ctor_set(x_240, 3, x_238); -x_241 = lean_ctor_get(x_22, 5); -lean_inc(x_241); -lean_dec(x_22); -x_242 = lean_array_get_size(x_241); -x_243 = lean_usize_of_nat(x_242); -lean_dec(x_242); -x_244 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45(x_243, x_2, x_241); -x_245 = l_Array_append___rarg(x_3, x_244); -x_246 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_246, 0, x_44); -lean_ctor_set(x_246, 1, x_70); -lean_ctor_set(x_246, 2, x_245); -x_247 = lean_array_push(x_98, x_246); -x_248 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_248, 0, x_44); -lean_ctor_set(x_248, 1, x_199); -lean_ctor_set(x_248, 2, x_247); -x_249 = lean_array_push(x_205, x_248); -x_250 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_250, 0, x_44); -lean_ctor_set(x_250, 1, x_207); -lean_ctor_set(x_250, 2, x_249); -x_251 = lean_array_push(x_212, x_250); -x_252 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_252, 0, x_44); -lean_ctor_set(x_252, 1, x_214); -lean_ctor_set(x_252, 2, x_251); -x_253 = lean_array_push(x_216, x_252); -x_254 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_254, 0, x_44); -lean_ctor_set(x_254, 1, x_218); -lean_ctor_set(x_254, 2, x_253); -x_255 = lean_array_push(x_220, x_240); -lean_inc(x_76); -x_256 = lean_array_push(x_255, x_76); -lean_inc(x_76); -x_257 = lean_array_push(x_256, x_76); -x_258 = lean_array_push(x_257, x_172); -x_259 = lean_array_push(x_258, x_254); -x_260 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_260, 0, x_44); -lean_ctor_set(x_260, 1, x_226); -lean_ctor_set(x_260, 2, x_259); -x_261 = lean_array_push(x_98, x_260); +lean_inc(x_5); +x_242 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_242, 0, x_5); +lean_ctor_set(x_242, 1, x_1); +lean_inc(x_1); +x_243 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_243, 0, x_242); +lean_ctor_set(x_243, 1, x_1); +x_244 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; +lean_inc(x_64); +x_245 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_245, 0, x_64); +lean_ctor_set(x_245, 1, x_244); +lean_ctor_set(x_245, 2, x_241); +lean_ctor_set(x_245, 3, x_243); +x_246 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; +lean_inc(x_43); +x_247 = l_Lean_Name_str___override(x_43, x_246); +x_248 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +lean_inc(x_64); +x_249 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_249, 0, x_64); +lean_ctor_set(x_249, 1, x_248); +x_250 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__64; +lean_inc(x_43); +x_251 = l_Lean_Name_str___override(x_43, x_250); +x_252 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66; +lean_inc(x_64); +x_253 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_253, 0, x_64); +lean_ctor_set(x_253, 1, x_252); +x_254 = lean_array_push(x_110, x_253); +x_255 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_255, 0, x_52); +lean_ctor_set(x_255, 1, x_251); +lean_ctor_set(x_255, 2, x_254); +x_256 = lean_array_push(x_110, x_255); +x_257 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_257, 0, x_52); +lean_ctor_set(x_257, 1, x_81); +lean_ctor_set(x_257, 2, x_256); +x_258 = lean_array_push(x_100, x_257); +lean_inc(x_239); +x_259 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_259, 0, x_52); +lean_ctor_set(x_259, 1, x_239); +lean_ctor_set(x_259, 2, x_258); +lean_inc(x_259); +x_260 = lean_array_push(x_49, x_259); +x_261 = lean_array_push(x_260, x_101); x_262 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_262, 0, x_44); -lean_ctor_set(x_262, 1, x_229); +lean_ctor_set(x_262, 0, x_52); +lean_ctor_set(x_262, 1, x_81); lean_ctor_set(x_262, 2, x_261); -x_263 = lean_array_push(x_98, x_262); -x_264 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_264, 0, x_44); -lean_ctor_set(x_264, 1, x_232); -lean_ctor_set(x_264, 2, x_263); -x_265 = lean_array_push(x_209, x_233); -lean_inc(x_76); -x_266 = lean_array_push(x_265, x_76); +x_263 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +lean_inc(x_64); +x_264 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_264, 0, x_64); +lean_ctor_set(x_264, 1, x_263); +lean_inc(x_249); +x_265 = lean_array_push(x_148, x_249); +x_266 = lean_array_push(x_265, x_262); +lean_inc(x_264); x_267 = lean_array_push(x_266, x_264); -lean_inc(x_76); -x_268 = lean_array_push(x_267, x_76); -x_269 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_269, 0, x_44); -lean_ctor_set(x_269, 1, x_70); -lean_ctor_set(x_269, 2, x_268); -x_270 = lean_array_push(x_118, x_97); -x_271 = lean_array_push(x_270, x_269); -lean_inc(x_76); -x_272 = lean_array_push(x_271, x_76); -x_273 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__56; +x_268 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_268, 0, x_52); +lean_ctor_set(x_268, 1, x_247); +lean_ctor_set(x_268, 2, x_267); +lean_inc(x_57); +x_269 = lean_array_push(x_49, x_57); +lean_inc(x_268); +x_270 = lean_array_push(x_269, x_268); +x_271 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_271, 0, x_52); +lean_ctor_set(x_271, 1, x_81); +lean_ctor_set(x_271, 2, x_270); +x_272 = lean_array_push(x_49, x_245); +x_273 = lean_array_push(x_272, x_271); +lean_inc(x_239); x_274 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_274, 0, x_44); -lean_ctor_set(x_274, 1, x_273); -lean_ctor_set(x_274, 2, x_272); -x_275 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238; -x_276 = lean_array_push(x_275, x_145); -x_277 = lean_array_push(x_276, x_147); -lean_inc(x_76); -x_278 = lean_array_push(x_277, x_76); -lean_inc(x_76); -x_279 = lean_array_push(x_278, x_76); -x_280 = lean_array_push(x_279, x_163); -x_281 = lean_array_push(x_280, x_274); -lean_inc(x_76); -x_282 = lean_array_push(x_281, x_76); -x_283 = lean_array_push(x_282, x_76); -x_284 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206; -x_285 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_285, 0, x_44); -lean_ctor_set(x_285, 1, x_284); -lean_ctor_set(x_285, 2, x_283); -x_286 = lean_array_push(x_139, x_285); -x_287 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_287, 0, x_44); -lean_ctor_set(x_287, 1, x_141); -lean_ctor_set(x_287, 2, x_286); -x_288 = lean_array_push(x_118, x_75); -x_289 = lean_array_push(x_288, x_142); -x_290 = lean_array_push(x_289, x_287); -x_291 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_291, 0, x_44); -lean_ctor_set(x_291, 1, x_70); -lean_ctor_set(x_291, 2, x_290); -lean_ctor_set(x_61, 0, x_291); -return x_61; -} -else -{ -lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; size_t x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; size_t x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; size_t x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; -x_292 = lean_ctor_get(x_61, 0); -x_293 = lean_ctor_get(x_61, 1); -lean_inc(x_293); -lean_inc(x_292); -lean_dec(x_61); -x_294 = lean_ctor_get(x_292, 0); -lean_inc(x_294); -lean_dec(x_292); -x_295 = lean_environment_main_module(x_294); -x_296 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; -lean_inc(x_58); -x_297 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_297, 0, x_58); -lean_ctor_set(x_297, 1, x_296); -x_298 = lean_ctor_get(x_22, 2); -lean_inc(x_298); -lean_inc(x_3); -x_299 = l_Array_append___rarg(x_3, x_298); -x_300 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_301 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_301, 0, x_44); -lean_ctor_set(x_301, 1, x_300); -lean_ctor_set(x_301, 2, x_299); -x_302 = lean_array_push(x_41, x_297); -x_303 = lean_array_push(x_302, x_301); -x_304 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; -x_305 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_305, 0, x_44); -lean_ctor_set(x_305, 1, x_304); -lean_ctor_set(x_305, 2, x_303); -lean_inc(x_3); -x_306 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_306, 0, x_44); -lean_ctor_set(x_306, 1, x_300); -lean_ctor_set(x_306, 2, x_3); -x_307 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__42; -lean_inc(x_306); -x_308 = lean_array_push(x_307, x_306); -lean_inc(x_306); -x_309 = lean_array_push(x_308, x_306); -lean_inc(x_306); -x_310 = lean_array_push(x_309, x_306); -lean_inc(x_306); -x_311 = lean_array_push(x_310, x_306); -lean_inc(x_306); -x_312 = lean_array_push(x_311, x_306); -lean_inc(x_306); -x_313 = lean_array_push(x_312, x_306); -x_314 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; -x_315 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_315, 0, x_44); -lean_ctor_set(x_315, 1, x_314); -lean_ctor_set(x_315, 2, x_313); -x_316 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__1; -lean_inc(x_58); -x_317 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_317, 0, x_58); -lean_ctor_set(x_317, 1, x_316); -x_318 = lean_array_push(x_41, x_51); -lean_inc(x_306); -x_319 = lean_array_push(x_318, x_306); -x_320 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; +lean_ctor_set(x_274, 0, x_52); +lean_ctor_set(x_274, 1, x_239); +lean_ctor_set(x_274, 2, x_273); +x_275 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67; +lean_inc(x_43); +x_276 = l_Lean_Name_str___override(x_43, x_275); +x_277 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69; +lean_inc(x_64); +x_278 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_278, 0, x_64); +lean_ctor_set(x_278, 1, x_277); +x_279 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__70; +lean_inc(x_43); +x_280 = l_Lean_Name_str___override(x_43, x_279); +x_281 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72; +lean_inc(x_64); +x_282 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_282, 0, x_64); +lean_ctor_set(x_282, 1, x_281); +x_283 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__4; +lean_inc(x_43); +x_284 = l_Lean_Name_str___override(x_43, x_283); +x_285 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86; +lean_inc(x_66); +lean_inc(x_71); +x_286 = l_Lean_addMacroScope(x_71, x_285, x_66); +x_287 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; +lean_inc(x_5); +x_288 = l_Lean_Name_str___override(x_5, x_287); +lean_inc(x_1); +x_289 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_289, 0, x_288); +lean_ctor_set(x_289, 1, x_1); +lean_inc(x_1); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_1); +x_291 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +lean_inc(x_64); +x_292 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_292, 0, x_64); +lean_ctor_set(x_292, 1, x_291); +lean_ctor_set(x_292, 2, x_286); +lean_ctor_set(x_292, 3, x_290); +lean_inc(x_292); +x_293 = lean_array_push(x_110, x_292); +lean_inc(x_284); +x_294 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_294, 0, x_52); +lean_ctor_set(x_294, 1, x_284); +lean_ctor_set(x_294, 2, x_293); +x_295 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__103; +lean_inc(x_66); +lean_inc(x_71); +x_296 = l_Lean_addMacroScope(x_71, x_295, x_66); +x_297 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100; +x_298 = l_Lean_Name_str___override(x_5, x_297); +lean_inc(x_1); +x_299 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_299, 0, x_298); +lean_ctor_set(x_299, 1, x_1); +lean_inc(x_1); +x_300 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_300, 0, x_299); +lean_ctor_set(x_300, 1, x_1); +x_301 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__102; +lean_inc(x_64); +x_302 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_302, 0, x_64); +lean_ctor_set(x_302, 1, x_301); +lean_ctor_set(x_302, 2, x_296); +lean_ctor_set(x_302, 3, x_300); +lean_inc(x_302); +x_303 = lean_array_push(x_110, x_302); +x_304 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_304, 0, x_52); +lean_ctor_set(x_304, 1, x_284); +lean_ctor_set(x_304, 2, x_303); +x_305 = lean_array_push(x_148, x_294); +x_306 = lean_array_push(x_305, x_136); +x_307 = lean_array_push(x_306, x_304); +x_308 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_308, 0, x_52); +lean_ctor_set(x_308, 1, x_81); +lean_ctor_set(x_308, 2, x_307); +x_309 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__86; +lean_inc(x_43); +x_310 = l_Lean_Name_str___override(x_43, x_309); +x_311 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_311, 0, x_52); +lean_ctor_set(x_311, 1, x_310); +lean_ctor_set(x_311, 2, x_188); +x_312 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89; +lean_inc(x_64); +x_313 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_313, 0, x_64); +lean_ctor_set(x_313, 1, x_312); +x_314 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18; +lean_inc(x_282); +x_315 = lean_array_push(x_314, x_282); +x_316 = lean_array_push(x_315, x_101); +x_317 = lean_array_push(x_316, x_308); +x_318 = lean_array_push(x_317, x_311); +x_319 = lean_array_push(x_318, x_101); +lean_inc(x_313); +x_320 = lean_array_push(x_319, x_313); x_321 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_321, 0, x_44); -lean_ctor_set(x_321, 1, x_320); -lean_ctor_set(x_321, 2, x_319); -lean_inc(x_306); -x_322 = lean_array_push(x_41, x_306); -lean_inc(x_306); -lean_inc(x_322); -x_323 = lean_array_push(x_322, x_306); -x_324 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__56; -x_325 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_325, 0, x_44); -lean_ctor_set(x_325, 1, x_324); -lean_ctor_set(x_325, 2, x_323); -x_326 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__28; -lean_inc(x_58); -x_327 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_327, 0, x_58); -lean_ctor_set(x_327, 1, x_326); -x_328 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -lean_inc(x_327); -x_329 = lean_array_push(x_328, x_327); -x_330 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_330, 0, x_44); -lean_ctor_set(x_330, 1, x_300); -lean_ctor_set(x_330, 2, x_329); -x_331 = lean_ctor_get(x_22, 3); -lean_inc(x_331); -x_332 = lean_array_get_size(x_331); -x_333 = lean_usize_of_nat(x_332); -lean_dec(x_332); -x_334 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__44(x_333, x_2, x_331); -lean_inc(x_3); -x_335 = l_Array_append___rarg(x_3, x_334); -x_336 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_336, 0, x_44); -lean_ctor_set(x_336, 1, x_300); -lean_ctor_set(x_336, 2, x_335); -x_337 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__33; -lean_inc(x_58); -x_338 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_338, 0, x_58); -lean_ctor_set(x_338, 1, x_337); -x_339 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; -lean_inc(x_306); -x_340 = lean_array_push(x_339, x_306); -x_341 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__35; -x_342 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_342, 0, x_44); +lean_ctor_set(x_321, 0, x_52); +lean_ctor_set(x_321, 1, x_280); +lean_ctor_set(x_321, 2, x_320); +x_322 = lean_array_push(x_49, x_278); +lean_inc(x_321); +x_323 = lean_array_push(x_322, x_321); +x_324 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_324, 0, x_52); +lean_ctor_set(x_324, 1, x_276); +lean_ctor_set(x_324, 2, x_323); +x_325 = lean_array_push(x_148, x_237); +lean_inc(x_274); +x_326 = lean_array_push(x_325, x_274); +x_327 = lean_array_push(x_326, x_324); +x_328 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_328, 0, x_52); +lean_ctor_set(x_328, 1, x_236); +lean_ctor_set(x_328, 2, x_327); +x_329 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__5; +lean_inc(x_43); +x_330 = l_Lean_Name_str___override(x_43, x_329); +x_331 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__6; +lean_inc(x_43); +x_332 = l_Lean_Name_str___override(x_43, x_331); +x_333 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; +lean_inc(x_43); +x_334 = l_Lean_Name_str___override(x_43, x_333); +x_335 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__81; +lean_inc(x_43); +x_336 = l_Lean_Name_str___override(x_43, x_335); +x_337 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__7; +lean_inc(x_43); +x_338 = l_Lean_Name_str___override(x_43, x_337); +x_339 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__11; +lean_inc(x_66); +lean_inc(x_71); +x_340 = l_Lean_addMacroScope(x_71, x_339, x_66); +x_341 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__10; +lean_inc(x_1); +lean_inc(x_64); +x_342 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_342, 0, x_64); lean_ctor_set(x_342, 1, x_341); lean_ctor_set(x_342, 2, x_340); -x_343 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; -lean_inc(x_58); -x_344 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_344, 0, x_58); -lean_ctor_set(x_344, 1, x_343); -x_345 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; -lean_inc(x_306); -x_346 = lean_array_push(x_345, x_306); -x_347 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_347, 0, x_44); -lean_ctor_set(x_347, 1, x_341); -lean_ctor_set(x_347, 2, x_346); -x_348 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__33; -x_349 = lean_array_push(x_348, x_342); -x_350 = lean_array_push(x_349, x_344); -x_351 = lean_array_push(x_350, x_347); -x_352 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_352, 0, x_44); -lean_ctor_set(x_352, 1, x_300); -lean_ctor_set(x_352, 2, x_351); -x_353 = lean_array_push(x_41, x_338); -x_354 = lean_array_push(x_353, x_352); -x_355 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_355, 0, x_44); -lean_ctor_set(x_355, 1, x_300); -lean_ctor_set(x_355, 2, x_354); -x_356 = lean_array_push(x_328, x_355); -x_357 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__32; -x_358 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_358, 0, x_44); -lean_ctor_set(x_358, 1, x_357); -lean_ctor_set(x_358, 2, x_356); -x_359 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; -x_360 = lean_array_push(x_359, x_317); -x_361 = lean_array_push(x_360, x_321); -x_362 = lean_array_push(x_361, x_325); -x_363 = lean_array_push(x_362, x_330); -x_364 = lean_array_push(x_363, x_336); -lean_inc(x_306); -x_365 = lean_array_push(x_364, x_306); -x_366 = lean_array_push(x_365, x_358); -x_367 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__2; +lean_ctor_set(x_342, 3, x_1); +lean_inc(x_342); +x_343 = lean_array_push(x_110, x_342); +x_344 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_344, 0, x_52); +lean_ctor_set(x_344, 1, x_81); +lean_ctor_set(x_344, 2, x_343); +x_345 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_346 = lean_array_push(x_345, x_282); +lean_inc(x_344); +x_347 = lean_array_push(x_346, x_344); +x_348 = lean_array_push(x_347, x_101); +x_349 = lean_array_push(x_348, x_313); +x_350 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_350, 0, x_52); +lean_ctor_set(x_350, 1, x_338); +lean_ctor_set(x_350, 2, x_349); +x_351 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__1; +lean_inc(x_43); +x_352 = l_Lean_Name_str___override(x_43, x_351); +x_353 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3; +lean_inc(x_64); +x_354 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_354, 0, x_64); +lean_ctor_set(x_354, 1, x_353); +x_355 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__15; +lean_inc(x_66); +lean_inc(x_71); +x_356 = l_Lean_addMacroScope(x_71, x_355, x_66); +lean_inc(x_1); +x_357 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_357, 0, x_355); +lean_ctor_set(x_357, 1, x_1); +lean_inc(x_1); +x_358 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_358, 0, x_357); +lean_ctor_set(x_358, 1, x_1); +x_359 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__14; +lean_inc(x_64); +x_360 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_360, 0, x_64); +lean_ctor_set(x_360, 1, x_359); +lean_ctor_set(x_360, 2, x_356); +lean_ctor_set(x_360, 3, x_358); +x_361 = lean_array_push(x_49, x_360); +lean_inc(x_344); +x_362 = lean_array_push(x_361, x_344); +lean_inc(x_239); +x_363 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_363, 0, x_52); +lean_ctor_set(x_363, 1, x_239); +lean_ctor_set(x_363, 2, x_362); +x_364 = lean_array_push(x_345, x_354); +x_365 = lean_array_push(x_364, x_101); +lean_inc(x_365); +x_366 = lean_array_push(x_365, x_363); +lean_inc(x_204); +x_367 = lean_array_push(x_366, x_204); +lean_inc(x_352); x_368 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_368, 0, x_44); -lean_ctor_set(x_368, 1, x_367); -lean_ctor_set(x_368, 2, x_366); -x_369 = lean_array_push(x_41, x_315); -lean_inc(x_369); -x_370 = lean_array_push(x_369, x_368); -x_371 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__37; -x_372 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_372, 0, x_44); -lean_ctor_set(x_372, 1, x_371); -lean_ctor_set(x_372, 2, x_370); -lean_inc(x_306); -x_373 = lean_array_push(x_328, x_306); -x_374 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__124; -x_375 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_375, 0, x_44); -lean_ctor_set(x_375, 1, x_374); -lean_ctor_set(x_375, 2, x_373); -x_376 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205; -lean_inc(x_58); -x_377 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_377, 0, x_58); -lean_ctor_set(x_377, 1, x_376); -x_378 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__26; -lean_inc(x_58); -x_379 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_379, 0, x_58); -lean_ctor_set(x_379, 1, x_378); -x_380 = lean_array_push(x_41, x_50); -x_381 = lean_array_push(x_380, x_56); +lean_ctor_set(x_368, 0, x_52); +lean_ctor_set(x_368, 1, x_352); +lean_ctor_set(x_368, 2, x_367); +x_369 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__19; +lean_inc(x_66); +lean_inc(x_71); +x_370 = l_Lean_addMacroScope(x_71, x_369, x_66); +x_371 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16; +x_372 = l_Lean_Name_str___override(x_14, x_371); +lean_inc(x_1); +x_373 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_373, 0, x_372); +lean_ctor_set(x_373, 1, x_1); +lean_inc(x_1); +x_374 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_374, 0, x_373); +lean_ctor_set(x_374, 1, x_1); +x_375 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__18; +lean_inc(x_64); +x_376 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_376, 0, x_64); +lean_ctor_set(x_376, 1, x_375); +lean_ctor_set(x_376, 2, x_370); +lean_ctor_set(x_376, 3, x_374); +x_377 = lean_array_push(x_49, x_376); +x_378 = lean_array_push(x_377, x_344); +lean_inc(x_239); +x_379 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_379, 0, x_52); +lean_ctor_set(x_379, 1, x_239); +lean_ctor_set(x_379, 2, x_378); +x_380 = lean_array_push(x_365, x_379); +x_381 = lean_array_push(x_380, x_204); x_382 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_382, 0, x_44); -lean_ctor_set(x_382, 1, x_300); +lean_ctor_set(x_382, 0, x_52); +lean_ctor_set(x_382, 1, x_352); lean_ctor_set(x_382, 2, x_381); -x_383 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__53; -x_384 = lean_array_push(x_383, x_382); -x_385 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; -x_386 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_386, 0, x_44); -lean_ctor_set(x_386, 1, x_385); -lean_ctor_set(x_386, 2, x_384); -x_387 = lean_array_push(x_41, x_379); -x_388 = lean_array_push(x_387, x_386); -x_389 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__95; +x_383 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1; +lean_inc(x_43); +x_384 = l_Lean_Name_str___override(x_43, x_383); +x_385 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__23; +lean_inc(x_66); +lean_inc(x_71); +x_386 = l_Lean_addMacroScope(x_71, x_385, x_66); +x_387 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__22; +lean_inc(x_1); +lean_inc(x_64); +x_388 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_388, 0, x_64); +lean_ctor_set(x_388, 1, x_387); +lean_ctor_set(x_388, 2, x_386); +lean_ctor_set(x_388, 3, x_1); +lean_inc(x_388); +x_389 = lean_array_push(x_110, x_388); x_390 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_390, 0, x_44); -lean_ctor_set(x_390, 1, x_389); -lean_ctor_set(x_390, 2, x_388); -lean_inc(x_322); -x_391 = lean_array_push(x_322, x_390); -x_392 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__143; -x_393 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_393, 0, x_44); -lean_ctor_set(x_393, 1, x_392); -lean_ctor_set(x_393, 2, x_391); -x_394 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224; -lean_inc(x_60); -lean_inc(x_295); -x_395 = l_Lean_addMacroScope(x_295, x_394, x_60); -x_396 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225; +lean_ctor_set(x_390, 0, x_52); +lean_ctor_set(x_390, 1, x_81); +lean_ctor_set(x_390, 2, x_389); +x_391 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; +lean_inc(x_64); +x_392 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_392, 0, x_64); +lean_ctor_set(x_392, 1, x_391); +x_393 = lean_array_push(x_49, x_392); +lean_inc(x_57); +lean_inc(x_393); +x_394 = lean_array_push(x_393, x_57); +x_395 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_395, 0, x_52); +lean_ctor_set(x_395, 1, x_81); +lean_ctor_set(x_395, 2, x_394); +x_396 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; +x_397 = lean_array_push(x_396, x_249); +x_398 = lean_array_push(x_397, x_390); +lean_inc(x_398); +x_399 = lean_array_push(x_398, x_395); +x_400 = lean_array_push(x_399, x_101); +lean_inc(x_264); +x_401 = lean_array_push(x_400, x_264); +lean_inc(x_384); +x_402 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_402, 0, x_52); +lean_ctor_set(x_402, 1, x_384); +lean_ctor_set(x_402, 2, x_401); +x_403 = lean_array_push(x_345, x_350); +x_404 = lean_array_push(x_403, x_368); +x_405 = lean_array_push(x_404, x_382); +lean_inc(x_405); +x_406 = lean_array_push(x_405, x_402); +x_407 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_407, 0, x_52); +lean_ctor_set(x_407, 1, x_81); +lean_ctor_set(x_407, 2, x_406); +x_408 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__36; +lean_inc(x_43); +x_409 = l_Lean_Name_str___override(x_43, x_408); +x_410 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__27; +lean_inc(x_66); +lean_inc(x_71); +x_411 = l_Lean_addMacroScope(x_71, x_410, x_66); lean_inc(x_1); -x_397 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_397, 0, x_396); -lean_ctor_set(x_397, 1, x_1); +x_412 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_412, 0, x_410); +lean_ctor_set(x_412, 1, x_1); lean_inc(x_1); -x_398 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_398, 0, x_397); -lean_ctor_set(x_398, 1, x_1); -x_399 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223; -lean_inc(x_58); -x_400 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_400, 0, x_58); -lean_ctor_set(x_400, 1, x_399); -lean_ctor_set(x_400, 2, x_395); -lean_ctor_set(x_400, 3, x_398); -x_401 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__109; -lean_inc(x_58); -x_402 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_402, 0, x_58); -lean_ctor_set(x_402, 1, x_401); -x_403 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__3; -lean_inc(x_58); -x_404 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_404, 0, x_58); -lean_ctor_set(x_404, 1, x_403); -x_405 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__10; -lean_inc(x_60); -lean_inc(x_295); -x_406 = l_Lean_addMacroScope(x_295, x_405, x_60); -x_407 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__9; +x_413 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_413, 0, x_412); +lean_ctor_set(x_413, 1, x_1); +x_414 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__26; +lean_inc(x_64); +x_415 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_415, 0, x_64); +lean_ctor_set(x_415, 1, x_414); +lean_ctor_set(x_415, 2, x_411); +lean_ctor_set(x_415, 3, x_413); +x_416 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__31; +lean_inc(x_66); +lean_inc(x_71); +x_417 = l_Lean_addMacroScope(x_71, x_416, x_66); lean_inc(x_1); -lean_inc(x_58); -x_408 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_408, 0, x_58); -lean_ctor_set(x_408, 1, x_407); -lean_ctor_set(x_408, 2, x_406); -lean_ctor_set(x_408, 3, x_1); -lean_inc(x_408); -x_409 = lean_array_push(x_328, x_408); -x_410 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_410, 0, x_44); -lean_ctor_set(x_410, 1, x_300); -lean_ctor_set(x_410, 2, x_409); -x_411 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__6; -lean_inc(x_58); -x_412 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_412, 0, x_58); -lean_ctor_set(x_412, 1, x_411); -x_413 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__11; -lean_inc(x_58); -x_414 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_414, 0, x_58); -lean_ctor_set(x_414, 1, x_413); -x_415 = lean_array_push(x_322, x_408); -x_416 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__14; -x_417 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_417, 0, x_44); -lean_ctor_set(x_417, 1, x_416); -lean_ctor_set(x_417, 2, x_415); -x_418 = lean_array_push(x_328, x_417); -x_419 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_419, 0, x_44); -lean_ctor_set(x_419, 1, x_300); -lean_ctor_set(x_419, 2, x_418); -x_420 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__15; -lean_inc(x_58); -x_421 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_421, 0, x_58); +x_418 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_418, 0, x_416); +lean_ctor_set(x_418, 1, x_1); +lean_inc(x_1); +x_419 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_419, 0, x_418); +lean_ctor_set(x_419, 1, x_1); +x_420 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__30; +lean_inc(x_64); +x_421 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_421, 0, x_64); lean_ctor_set(x_421, 1, x_420); -x_422 = lean_ctor_get(x_22, 4); -lean_inc(x_422); -x_423 = lean_array_get_size(x_422); -x_424 = lean_usize_of_nat(x_423); -lean_dec(x_423); -x_425 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45(x_424, x_2, x_422); -lean_inc(x_3); -x_426 = l_Array_append___rarg(x_3, x_425); -x_427 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_427, 0, x_44); -lean_ctor_set(x_427, 1, x_300); -lean_ctor_set(x_427, 2, x_426); -x_428 = lean_array_push(x_328, x_427); -x_429 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__17; +lean_ctor_set(x_421, 2, x_417); +lean_ctor_set(x_421, 3, x_419); +x_422 = lean_array_push(x_148, x_421); +x_423 = lean_array_push(x_422, x_342); +lean_inc(x_423); +x_424 = lean_array_push(x_423, x_268); +x_425 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_425, 0, x_52); +lean_ctor_set(x_425, 1, x_81); +lean_ctor_set(x_425, 2, x_424); +x_426 = lean_array_push(x_49, x_415); +lean_inc(x_426); +x_427 = lean_array_push(x_426, x_425); +lean_inc(x_239); +x_428 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_428, 0, x_52); +lean_ctor_set(x_428, 1, x_239); +lean_ctor_set(x_428, 2, x_427); +lean_inc(x_393); +x_429 = lean_array_push(x_393, x_428); +lean_inc(x_409); x_430 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_430, 0, x_44); -lean_ctor_set(x_430, 1, x_429); -lean_ctor_set(x_430, 2, x_428); -x_431 = lean_array_push(x_307, x_414); -lean_inc(x_306); -x_432 = lean_array_push(x_431, x_306); -lean_inc(x_306); -x_433 = lean_array_push(x_432, x_306); -x_434 = lean_array_push(x_433, x_419); -x_435 = lean_array_push(x_434, x_421); -lean_inc(x_435); -x_436 = lean_array_push(x_435, x_430); -x_437 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__12; -x_438 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_438, 0, x_44); -lean_ctor_set(x_438, 1, x_437); -lean_ctor_set(x_438, 2, x_436); -x_439 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_440 = lean_array_push(x_439, x_410); -lean_inc(x_306); -x_441 = lean_array_push(x_440, x_306); -x_442 = lean_array_push(x_441, x_412); -lean_inc(x_442); -x_443 = lean_array_push(x_442, x_438); -x_444 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__6; +lean_ctor_set(x_430, 0, x_52); +lean_ctor_set(x_430, 1, x_409); +lean_ctor_set(x_430, 2, x_429); +x_431 = lean_array_push(x_110, x_430); +x_432 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_432, 0, x_52); +lean_ctor_set(x_432, 1, x_81); +lean_ctor_set(x_432, 2, x_431); +x_433 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__32; +lean_inc(x_43); +x_434 = l_Lean_Name_str___override(x_43, x_433); +lean_inc(x_64); +x_435 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_435, 0, x_64); +lean_ctor_set(x_435, 1, x_433); +x_436 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__33; +lean_inc(x_43); +x_437 = l_Lean_Name_str___override(x_43, x_436); +x_438 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__34; +lean_inc(x_43); +x_439 = l_Lean_Name_str___override(x_43, x_438); +x_440 = l_Lean_addMacroScope(x_71, x_15, x_66); +x_441 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__140; +lean_inc(x_64); +x_442 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_442, 0, x_64); +lean_ctor_set(x_442, 1, x_441); +lean_ctor_set(x_442, 2, x_440); +lean_ctor_set(x_442, 3, x_1); +x_443 = lean_array_push(x_49, x_442); +x_444 = lean_array_push(x_443, x_101); x_445 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_445, 0, x_44); -lean_ctor_set(x_445, 1, x_444); -lean_ctor_set(x_445, 2, x_443); -x_446 = lean_array_push(x_41, x_404); -lean_inc(x_446); -x_447 = lean_array_push(x_446, x_445); -x_448 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__4; +lean_ctor_set(x_445, 0, x_52); +lean_ctor_set(x_445, 1, x_81); +lean_ctor_set(x_445, 2, x_444); +lean_inc(x_393); +x_446 = lean_array_push(x_393, x_274); +lean_inc(x_409); +x_447 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_447, 0, x_52); +lean_ctor_set(x_447, 1, x_409); +lean_ctor_set(x_447, 2, x_446); +x_448 = lean_array_push(x_110, x_447); x_449 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_449, 0, x_44); -lean_ctor_set(x_449, 1, x_448); -lean_ctor_set(x_449, 2, x_447); -x_450 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_451 = lean_array_push(x_450, x_400); -lean_inc(x_306); -x_452 = lean_array_push(x_451, x_306); -lean_inc(x_306); -x_453 = lean_array_push(x_452, x_306); -lean_inc(x_402); -x_454 = lean_array_push(x_453, x_402); -x_455 = lean_array_push(x_454, x_449); -x_456 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; -x_457 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_457, 0, x_44); -lean_ctor_set(x_457, 1, x_456); -lean_ctor_set(x_457, 2, x_455); -x_458 = lean_array_push(x_328, x_457); -x_459 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60; -x_460 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_460, 0, x_44); -lean_ctor_set(x_460, 1, x_459); -lean_ctor_set(x_460, 2, x_458); -x_461 = lean_array_push(x_328, x_460); -x_462 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__58; -x_463 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_463, 0, x_44); -lean_ctor_set(x_463, 1, x_462); -lean_ctor_set(x_463, 2, x_461); -x_464 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231; -x_465 = l_Lean_addMacroScope(x_295, x_464, x_60); -x_466 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232; -lean_inc(x_1); -x_467 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_467, 0, x_466); -lean_ctor_set(x_467, 1, x_1); -x_468 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_468, 0, x_467); -lean_ctor_set(x_468, 1, x_1); -x_469 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230; -x_470 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_470, 0, x_58); -lean_ctor_set(x_470, 1, x_469); -lean_ctor_set(x_470, 2, x_465); -lean_ctor_set(x_470, 3, x_468); -x_471 = lean_ctor_get(x_22, 5); +lean_ctor_set(x_449, 0, x_52); +lean_ctor_set(x_449, 1, x_81); +lean_ctor_set(x_449, 2, x_448); +x_450 = lean_array_push(x_345, x_445); +x_451 = lean_array_push(x_450, x_449); +lean_inc(x_234); +x_452 = lean_array_push(x_451, x_234); +x_453 = lean_array_push(x_452, x_321); +x_454 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_454, 0, x_52); +lean_ctor_set(x_454, 1, x_439); +lean_ctor_set(x_454, 2, x_453); +x_455 = lean_array_push(x_110, x_454); +x_456 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_456, 0, x_52); +lean_ctor_set(x_456, 1, x_437); +lean_ctor_set(x_456, 2, x_455); +x_457 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__35; +lean_inc(x_43); +x_458 = l_Lean_Name_str___override(x_43, x_457); +lean_inc(x_64); +x_459 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_459, 0, x_64); +lean_ctor_set(x_459, 1, x_457); +x_460 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__36; +lean_inc(x_43); +x_461 = l_Lean_Name_str___override(x_43, x_460); +x_462 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__59; +x_463 = lean_array_push(x_462, x_388); +x_464 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_464, 0, x_52); +lean_ctor_set(x_464, 1, x_461); +lean_ctor_set(x_464, 2, x_463); +x_465 = lean_array_push(x_110, x_464); +x_466 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_466, 0, x_52); +lean_ctor_set(x_466, 1, x_81); +lean_ctor_set(x_466, 2, x_465); +x_467 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__37; +x_468 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_468, 0, x_64); +lean_ctor_set(x_468, 1, x_467); +x_469 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__38; +x_470 = l_Lean_Name_str___override(x_43, x_469); +x_471 = lean_ctor_get(x_27, 1); lean_inc(x_471); -lean_dec(x_22); x_472 = lean_array_get_size(x_471); x_473 = lean_usize_of_nat(x_472); lean_dec(x_472); -x_474 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45(x_473, x_2, x_471); -x_475 = l_Array_append___rarg(x_3, x_474); +x_474 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(x_473, x_31, x_471); +x_475 = l_Array_append___rarg(x_79, x_474); x_476 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_476, 0, x_44); -lean_ctor_set(x_476, 1, x_300); +lean_ctor_set(x_476, 0, x_52); +lean_ctor_set(x_476, 1, x_81); lean_ctor_set(x_476, 2, x_475); -x_477 = lean_array_push(x_328, x_476); +x_477 = lean_array_push(x_110, x_476); +lean_inc(x_470); x_478 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_478, 0, x_44); -lean_ctor_set(x_478, 1, x_429); +lean_ctor_set(x_478, 0, x_52); +lean_ctor_set(x_478, 1, x_470); lean_ctor_set(x_478, 2, x_477); -x_479 = lean_array_push(x_435, x_478); -x_480 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_480, 0, x_44); -lean_ctor_set(x_480, 1, x_437); -lean_ctor_set(x_480, 2, x_479); -x_481 = lean_array_push(x_442, x_480); -x_482 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_482, 0, x_44); -lean_ctor_set(x_482, 1, x_444); -lean_ctor_set(x_482, 2, x_481); -x_483 = lean_array_push(x_446, x_482); -x_484 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_484, 0, x_44); -lean_ctor_set(x_484, 1, x_448); -lean_ctor_set(x_484, 2, x_483); -x_485 = lean_array_push(x_450, x_470); -lean_inc(x_306); -x_486 = lean_array_push(x_485, x_306); -lean_inc(x_306); -x_487 = lean_array_push(x_486, x_306); -x_488 = lean_array_push(x_487, x_402); -x_489 = lean_array_push(x_488, x_484); +x_479 = lean_array_push(x_314, x_459); +x_480 = lean_array_push(x_479, x_101); +x_481 = lean_array_push(x_480, x_101); +x_482 = lean_array_push(x_481, x_466); +x_483 = lean_array_push(x_482, x_468); +lean_inc(x_483); +x_484 = lean_array_push(x_483, x_478); +lean_inc(x_458); +x_485 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_485, 0, x_52); +lean_ctor_set(x_485, 1, x_458); +lean_ctor_set(x_485, 2, x_484); +x_486 = lean_array_push(x_345, x_435); +x_487 = lean_array_push(x_486, x_456); +x_488 = lean_array_push(x_487, x_101); +lean_inc(x_488); +x_489 = lean_array_push(x_488, x_485); +lean_inc(x_434); x_490 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_490, 0, x_44); -lean_ctor_set(x_490, 1, x_456); +lean_ctor_set(x_490, 0, x_52); +lean_ctor_set(x_490, 1, x_434); lean_ctor_set(x_490, 2, x_489); -x_491 = lean_array_push(x_328, x_490); -x_492 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_492, 0, x_44); -lean_ctor_set(x_492, 1, x_459); -lean_ctor_set(x_492, 2, x_491); -x_493 = lean_array_push(x_328, x_492); -x_494 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_494, 0, x_44); -lean_ctor_set(x_494, 1, x_462); -lean_ctor_set(x_494, 2, x_493); -x_495 = lean_array_push(x_439, x_463); -lean_inc(x_306); -x_496 = lean_array_push(x_495, x_306); -x_497 = lean_array_push(x_496, x_494); -lean_inc(x_306); -x_498 = lean_array_push(x_497, x_306); -x_499 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_499, 0, x_44); -lean_ctor_set(x_499, 1, x_300); -lean_ctor_set(x_499, 2, x_498); -x_500 = lean_array_push(x_348, x_327); -x_501 = lean_array_push(x_500, x_499); -lean_inc(x_306); -x_502 = lean_array_push(x_501, x_306); -x_503 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__56; -x_504 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_504, 0, x_44); -lean_ctor_set(x_504, 1, x_503); -lean_ctor_set(x_504, 2, x_502); -x_505 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238; -x_506 = lean_array_push(x_505, x_375); -x_507 = lean_array_push(x_506, x_377); -lean_inc(x_306); -x_508 = lean_array_push(x_507, x_306); -lean_inc(x_306); -x_509 = lean_array_push(x_508, x_306); -x_510 = lean_array_push(x_509, x_393); -x_511 = lean_array_push(x_510, x_504); -lean_inc(x_306); -x_512 = lean_array_push(x_511, x_306); -x_513 = lean_array_push(x_512, x_306); -x_514 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206; +x_491 = lean_array_push(x_396, x_292); +x_492 = lean_array_push(x_491, x_407); +x_493 = lean_array_push(x_492, x_432); +lean_inc(x_234); +x_494 = lean_array_push(x_493, x_234); +x_495 = lean_array_push(x_494, x_490); +lean_inc(x_336); +x_496 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_496, 0, x_52); +lean_ctor_set(x_496, 1, x_336); +lean_ctor_set(x_496, 2, x_495); +x_497 = lean_array_push(x_110, x_496); +lean_inc(x_334); +x_498 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_498, 0, x_52); +lean_ctor_set(x_498, 1, x_334); +lean_ctor_set(x_498, 2, x_497); +x_499 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__40; +x_500 = lean_array_push(x_499, x_498); +lean_inc(x_332); +x_501 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_501, 0, x_52); +lean_ctor_set(x_501, 1, x_332); +lean_ctor_set(x_501, 2, x_500); +lean_inc(x_393); +x_502 = lean_array_push(x_393, x_259); +x_503 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_503, 0, x_52); +lean_ctor_set(x_503, 1, x_81); +lean_ctor_set(x_503, 2, x_502); +x_504 = lean_array_push(x_398, x_503); +x_505 = lean_array_push(x_504, x_101); +x_506 = lean_array_push(x_505, x_264); +x_507 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_507, 0, x_52); +lean_ctor_set(x_507, 1, x_384); +lean_ctor_set(x_507, 2, x_506); +x_508 = lean_array_push(x_405, x_507); +x_509 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_509, 0, x_52); +lean_ctor_set(x_509, 1, x_81); +lean_ctor_set(x_509, 2, x_508); +x_510 = lean_array_push(x_423, x_57); +x_511 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_511, 0, x_52); +lean_ctor_set(x_511, 1, x_81); +lean_ctor_set(x_511, 2, x_510); +x_512 = lean_array_push(x_426, x_511); +x_513 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_513, 0, x_52); +lean_ctor_set(x_513, 1, x_239); +lean_ctor_set(x_513, 2, x_512); +x_514 = lean_array_push(x_393, x_513); x_515 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_515, 0, x_44); -lean_ctor_set(x_515, 1, x_514); -lean_ctor_set(x_515, 2, x_513); -x_516 = lean_array_push(x_369, x_515); +lean_ctor_set(x_515, 0, x_52); +lean_ctor_set(x_515, 1, x_409); +lean_ctor_set(x_515, 2, x_514); +x_516 = lean_array_push(x_110, x_515); x_517 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_517, 0, x_44); -lean_ctor_set(x_517, 1, x_371); +lean_ctor_set(x_517, 0, x_52); +lean_ctor_set(x_517, 1, x_81); lean_ctor_set(x_517, 2, x_516); -x_518 = lean_array_push(x_348, x_305); -x_519 = lean_array_push(x_518, x_372); -x_520 = lean_array_push(x_519, x_517); -x_521 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_521, 0, x_44); -lean_ctor_set(x_521, 1, x_300); -lean_ctor_set(x_521, 2, x_520); -x_522 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_522, 0, x_521); -lean_ctor_set(x_522, 1, x_293); -return x_522; -} -} -else -{ -uint8_t x_523; -lean_dec(x_22); -lean_dec(x_17); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_523 = !lean_is_exclusive(x_26); -if (x_523 == 0) -{ -return x_26; -} -else -{ -lean_object* x_524; lean_object* x_525; lean_object* x_526; -x_524 = lean_ctor_get(x_26, 0); -x_525 = lean_ctor_get(x_26, 1); -lean_inc(x_525); -lean_inc(x_524); -lean_dec(x_26); -x_526 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_526, 0, x_524); -lean_ctor_set(x_526, 1, x_525); -return x_526; -} -} -} -else -{ -uint8_t x_527; -lean_dec(x_17); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_527 = !lean_is_exclusive(x_21); -if (x_527 == 0) -{ -return x_21; -} -else -{ -lean_object* x_528; lean_object* x_529; lean_object* x_530; -x_528 = lean_ctor_get(x_21, 0); -x_529 = lean_ctor_get(x_21, 1); -lean_inc(x_529); -lean_inc(x_528); -lean_dec(x_21); -x_530 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_530, 0, x_528); -lean_ctor_set(x_530, 1, x_529); -return x_530; -} -} -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("RpcEncoding type binders : ", 27); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -uint8_t x_16; lean_object* x_17; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = lean_st_ref_get(x_14, x_15); -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_33, 3); -lean_inc(x_34); -lean_dec(x_33); -x_35 = lean_ctor_get_uint8(x_34, sizeof(void*)*1); -lean_dec(x_34); -if (x_35 == 0) -{ -lean_object* x_36; uint8_t x_37; -x_36 = lean_ctor_get(x_32, 1); -lean_inc(x_36); -lean_dec(x_32); -x_37 = 0; -x_16 = x_37; -x_17 = x_36; -goto block_31; +x_518 = lean_ctor_get(x_27, 2); +lean_inc(x_518); +lean_dec(x_27); +x_519 = lean_array_get_size(x_518); +x_520 = lean_usize_of_nat(x_519); +lean_dec(x_519); +x_521 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(x_520, x_31, x_518); +x_522 = l_Array_append___rarg(x_79, x_521); +x_523 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_523, 0, x_52); +lean_ctor_set(x_523, 1, x_81); +lean_ctor_set(x_523, 2, x_522); +x_524 = lean_array_push(x_110, x_523); +x_525 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_525, 0, x_52); +lean_ctor_set(x_525, 1, x_470); +lean_ctor_set(x_525, 2, x_524); +x_526 = lean_array_push(x_483, x_525); +x_527 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_527, 0, x_52); +lean_ctor_set(x_527, 1, x_458); +lean_ctor_set(x_527, 2, x_526); +x_528 = lean_array_push(x_488, x_527); +x_529 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_529, 0, x_52); +lean_ctor_set(x_529, 1, x_434); +lean_ctor_set(x_529, 2, x_528); +x_530 = lean_array_push(x_396, x_302); +x_531 = lean_array_push(x_530, x_509); +x_532 = lean_array_push(x_531, x_517); +lean_inc(x_234); +x_533 = lean_array_push(x_532, x_234); +x_534 = lean_array_push(x_533, x_529); +x_535 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_535, 0, x_52); +lean_ctor_set(x_535, 1, x_336); +lean_ctor_set(x_535, 2, x_534); +x_536 = lean_array_push(x_110, x_535); +x_537 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_537, 0, x_52); +lean_ctor_set(x_537, 1, x_334); +lean_ctor_set(x_537, 2, x_536); +x_538 = lean_array_push(x_499, x_537); +x_539 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_539, 0, x_52); +lean_ctor_set(x_539, 1, x_332); +lean_ctor_set(x_539, 2, x_538); +x_540 = lean_array_push(x_345, x_501); +x_541 = lean_array_push(x_540, x_101); +x_542 = lean_array_push(x_541, x_539); +x_543 = lean_array_push(x_542, x_101); +x_544 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_544, 0, x_52); +lean_ctor_set(x_544, 1, x_81); +lean_ctor_set(x_544, 2, x_543); +x_545 = lean_array_push(x_49, x_109); +x_546 = lean_array_push(x_545, x_544); +x_547 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_547, 0, x_52); +lean_ctor_set(x_547, 1, x_330); +lean_ctor_set(x_547, 2, x_546); +x_548 = lean_array_push(x_110, x_547); +x_549 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_549, 0, x_52); +lean_ctor_set(x_549, 1, x_81); +lean_ctor_set(x_549, 2, x_548); +x_550 = lean_array_push(x_148, x_234); +x_551 = lean_array_push(x_550, x_328); +x_552 = lean_array_push(x_551, x_549); +x_553 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_553, 0, x_52); +lean_ctor_set(x_553, 1, x_232); +lean_ctor_set(x_553, 2, x_552); +x_554 = lean_array_push(x_158, x_227); +x_555 = lean_array_push(x_554, x_230); +x_556 = lean_array_push(x_555, x_107); +x_557 = lean_array_push(x_556, x_553); +x_558 = lean_array_push(x_557, x_101); +x_559 = lean_array_push(x_558, x_101); +x_560 = lean_array_push(x_559, x_101); +x_561 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_561, 0, x_52); +lean_ctor_set(x_561, 1, x_226); +lean_ctor_set(x_561, 2, x_560); +x_562 = lean_array_push(x_49, x_224); +x_563 = lean_array_push(x_562, x_561); +x_564 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_564, 0, x_52); +lean_ctor_set(x_564, 1, x_88); +lean_ctor_set(x_564, 2, x_563); +x_565 = lean_array_push(x_148, x_179); +x_566 = lean_array_push(x_565, x_86); +x_567 = lean_array_push(x_566, x_564); +x_568 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_568, 0, x_52); +lean_ctor_set(x_568, 1, x_75); +lean_ctor_set(x_568, 2, x_567); +x_569 = lean_array_push(x_49, x_173); +x_570 = lean_array_push(x_569, x_568); +x_571 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_571, 0, x_52); +lean_ctor_set(x_571, 1, x_81); +lean_ctor_set(x_571, 2, x_570); +lean_ctor_set(x_67, 0, x_571); +return x_67; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; -x_38 = lean_ctor_get(x_32, 1); -lean_inc(x_38); -lean_dec(x_32); -lean_inc(x_7); -x_39 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_7, x_9, x_10, x_11, x_12, x_13, x_14, x_38); -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); +lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; size_t x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; lean_object* x_677; lean_object* x_678; lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; lean_object* x_713; lean_object* x_714; lean_object* x_715; lean_object* x_716; lean_object* x_717; lean_object* x_718; lean_object* x_719; lean_object* x_720; lean_object* x_721; lean_object* x_722; lean_object* x_723; lean_object* x_724; lean_object* x_725; lean_object* x_726; lean_object* x_727; lean_object* x_728; lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; lean_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; lean_object* x_740; lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; lean_object* x_747; lean_object* x_748; lean_object* x_749; lean_object* x_750; lean_object* x_751; lean_object* x_752; lean_object* x_753; lean_object* x_754; lean_object* x_755; lean_object* x_756; lean_object* x_757; lean_object* x_758; lean_object* x_759; lean_object* x_760; lean_object* x_761; lean_object* x_762; lean_object* x_763; lean_object* x_764; lean_object* x_765; lean_object* x_766; lean_object* x_767; lean_object* x_768; lean_object* x_769; lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; lean_object* x_774; lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_796; lean_object* x_797; lean_object* x_798; lean_object* x_799; lean_object* x_800; lean_object* x_801; lean_object* x_802; lean_object* x_803; lean_object* x_804; lean_object* x_805; lean_object* x_806; lean_object* x_807; lean_object* x_808; lean_object* x_809; lean_object* x_810; lean_object* x_811; lean_object* x_812; lean_object* x_813; lean_object* x_814; lean_object* x_815; lean_object* x_816; lean_object* x_817; lean_object* x_818; lean_object* x_819; lean_object* x_820; lean_object* x_821; lean_object* x_822; lean_object* x_823; lean_object* x_824; lean_object* x_825; lean_object* x_826; lean_object* x_827; lean_object* x_828; lean_object* x_829; lean_object* x_830; lean_object* x_831; lean_object* x_832; lean_object* x_833; lean_object* x_834; lean_object* x_835; lean_object* x_836; lean_object* x_837; lean_object* x_838; lean_object* x_839; lean_object* x_840; lean_object* x_841; lean_object* x_842; lean_object* x_843; lean_object* x_844; lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; lean_object* x_849; lean_object* x_850; lean_object* x_851; lean_object* x_852; lean_object* x_853; lean_object* x_854; lean_object* x_855; lean_object* x_856; lean_object* x_857; lean_object* x_858; lean_object* x_859; lean_object* x_860; lean_object* x_861; lean_object* x_862; lean_object* x_863; lean_object* x_864; lean_object* x_865; lean_object* x_866; lean_object* x_867; lean_object* x_868; lean_object* x_869; lean_object* x_870; lean_object* x_871; lean_object* x_872; lean_object* x_873; lean_object* x_874; lean_object* x_875; lean_object* x_876; lean_object* x_877; lean_object* x_878; lean_object* x_879; lean_object* x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; lean_object* x_884; lean_object* x_885; lean_object* x_886; lean_object* x_887; lean_object* x_888; lean_object* x_889; lean_object* x_890; lean_object* x_891; lean_object* x_892; lean_object* x_893; lean_object* x_894; lean_object* x_895; lean_object* x_896; lean_object* x_897; lean_object* x_898; lean_object* x_899; lean_object* x_900; lean_object* x_901; lean_object* x_902; lean_object* x_903; lean_object* x_904; lean_object* x_905; lean_object* x_906; lean_object* x_907; lean_object* x_908; lean_object* x_909; lean_object* x_910; lean_object* x_911; lean_object* x_912; lean_object* x_913; lean_object* x_914; lean_object* x_915; lean_object* x_916; lean_object* x_917; lean_object* x_918; lean_object* x_919; lean_object* x_920; lean_object* x_921; lean_object* x_922; lean_object* x_923; lean_object* x_924; lean_object* x_925; lean_object* x_926; lean_object* x_927; lean_object* x_928; lean_object* x_929; lean_object* x_930; lean_object* x_931; lean_object* x_932; lean_object* x_933; lean_object* x_934; lean_object* x_935; lean_object* x_936; lean_object* x_937; lean_object* x_938; lean_object* x_939; lean_object* x_940; lean_object* x_941; lean_object* x_942; lean_object* x_943; lean_object* x_944; lean_object* x_945; lean_object* x_946; lean_object* x_947; lean_object* x_948; lean_object* x_949; lean_object* x_950; lean_object* x_951; lean_object* x_952; lean_object* x_953; lean_object* x_954; lean_object* x_955; lean_object* x_956; lean_object* x_957; lean_object* x_958; lean_object* x_959; lean_object* x_960; lean_object* x_961; lean_object* x_962; lean_object* x_963; lean_object* x_964; lean_object* x_965; lean_object* x_966; lean_object* x_967; lean_object* x_968; lean_object* x_969; lean_object* x_970; lean_object* x_971; lean_object* x_972; lean_object* x_973; lean_object* x_974; lean_object* x_975; lean_object* x_976; size_t x_977; lean_object* x_978; lean_object* x_979; lean_object* x_980; lean_object* x_981; lean_object* x_982; lean_object* x_983; lean_object* x_984; lean_object* x_985; lean_object* x_986; lean_object* x_987; lean_object* x_988; lean_object* x_989; lean_object* x_990; lean_object* x_991; lean_object* x_992; lean_object* x_993; lean_object* x_994; lean_object* x_995; lean_object* x_996; lean_object* x_997; lean_object* x_998; lean_object* x_999; lean_object* x_1000; lean_object* x_1001; lean_object* x_1002; lean_object* x_1003; lean_object* x_1004; lean_object* x_1005; lean_object* x_1006; lean_object* x_1007; lean_object* x_1008; lean_object* x_1009; lean_object* x_1010; lean_object* x_1011; lean_object* x_1012; lean_object* x_1013; lean_object* x_1014; lean_object* x_1015; lean_object* x_1016; lean_object* x_1017; lean_object* x_1018; lean_object* x_1019; lean_object* x_1020; lean_object* x_1021; lean_object* x_1022; lean_object* x_1023; size_t x_1024; lean_object* x_1025; lean_object* x_1026; lean_object* x_1027; lean_object* x_1028; lean_object* x_1029; lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; lean_object* x_1033; lean_object* x_1034; lean_object* x_1035; lean_object* x_1036; lean_object* x_1037; lean_object* x_1038; lean_object* x_1039; lean_object* x_1040; lean_object* x_1041; lean_object* x_1042; lean_object* x_1043; lean_object* x_1044; lean_object* x_1045; lean_object* x_1046; lean_object* x_1047; lean_object* x_1048; lean_object* x_1049; lean_object* x_1050; lean_object* x_1051; lean_object* x_1052; lean_object* x_1053; lean_object* x_1054; lean_object* x_1055; lean_object* x_1056; lean_object* x_1057; lean_object* x_1058; lean_object* x_1059; lean_object* x_1060; lean_object* x_1061; lean_object* x_1062; lean_object* x_1063; lean_object* x_1064; lean_object* x_1065; lean_object* x_1066; lean_object* x_1067; lean_object* x_1068; lean_object* x_1069; lean_object* x_1070; lean_object* x_1071; lean_object* x_1072; lean_object* x_1073; lean_object* x_1074; lean_object* x_1075; lean_object* x_1076; +x_572 = lean_ctor_get(x_67, 0); +x_573 = lean_ctor_get(x_67, 1); +lean_inc(x_573); +lean_inc(x_572); +lean_dec(x_67); +x_574 = lean_ctor_get(x_572, 0); +lean_inc(x_574); +lean_dec(x_572); +x_575 = lean_environment_main_module(x_574); +x_576 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__7; lean_inc(x_41); -lean_dec(x_39); -x_42 = lean_unbox(x_40); -lean_dec(x_40); -x_16 = x_42; -x_17 = x_41; -goto block_31; -} -block_31: -{ -if (x_16 == 0) -{ -lean_object* x_18; lean_object* x_19; -lean_dec(x_8); -lean_dec(x_7); -x_18 = lean_box(0); -x_19 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_17); -return x_19; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_20 = lean_array_to_list(lean_box(0), x_8); +x_577 = l_Lean_Name_str___override(x_41, x_576); +x_578 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__12; +lean_inc(x_577); +x_579 = l_Lean_Name_str___override(x_577, x_578); +x_580 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__14; +lean_inc(x_577); +x_581 = l_Lean_Name_str___override(x_577, x_580); +lean_inc(x_64); +x_582 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_582, 0, x_64); +lean_ctor_set(x_582, 1, x_580); +x_583 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; +lean_inc(x_11); +x_584 = l_Array_append___rarg(x_583, x_11); +x_585 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_586 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_586, 0, x_52); +lean_ctor_set(x_586, 1, x_585); +lean_ctor_set(x_586, 2, x_584); +x_587 = lean_array_push(x_49, x_582); +lean_inc(x_587); +x_588 = lean_array_push(x_587, x_586); +lean_inc(x_581); +x_589 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_589, 0, x_52); +lean_ctor_set(x_589, 1, x_581); +lean_ctor_set(x_589, 2, x_588); +lean_inc(x_64); +x_590 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_590, 0, x_64); +lean_ctor_set(x_590, 1, x_578); +x_591 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__9; +lean_inc(x_577); +x_592 = l_Lean_Name_str___override(x_577, x_591); +x_593 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; +lean_inc(x_577); +x_594 = l_Lean_Name_str___override(x_577, x_593); +x_595 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__22; +lean_inc(x_594); +x_596 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_596, 0, x_52); +lean_ctor_set(x_596, 1, x_594); +lean_ctor_set(x_596, 2, x_595); +x_597 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2; +lean_inc(x_577); +x_598 = l_Lean_Name_str___override(x_577, x_597); +lean_inc(x_64); +x_599 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_599, 0, x_64); +lean_ctor_set(x_599, 1, x_597); +x_600 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; +lean_inc(x_577); +x_601 = l_Lean_Name_str___override(x_577, x_600); +lean_inc(x_66); +lean_inc(x_575); +x_602 = l_Lean_addMacroScope(x_575, x_3, x_66); +lean_inc(x_1); +lean_inc(x_64); +x_603 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_603, 0, x_64); +lean_ctor_set(x_603, 1, x_4); +lean_ctor_set(x_603, 2, x_602); +lean_ctor_set(x_603, 3, x_1); +x_604 = lean_array_push(x_49, x_603); +x_605 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; +lean_inc(x_604); +x_606 = lean_array_push(x_604, x_605); +lean_inc(x_601); +x_607 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_607, 0, x_52); +lean_ctor_set(x_607, 1, x_601); +lean_ctor_set(x_607, 2, x_606); +x_608 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__32; +lean_inc(x_577); +x_609 = l_Lean_Name_str___override(x_577, x_608); +x_610 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__60; +x_611 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_611, 0, x_52); +lean_ctor_set(x_611, 1, x_609); +lean_ctor_set(x_611, 2, x_610); +x_612 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__76; +lean_inc(x_64); +x_613 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_613, 0, x_64); +lean_ctor_set(x_613, 1, x_612); +x_614 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +lean_inc(x_613); +x_615 = lean_array_push(x_614, x_613); +x_616 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_616, 0, x_52); +lean_ctor_set(x_616, 1, x_585); +lean_ctor_set(x_616, 2, x_615); +x_617 = lean_ctor_get(x_27, 0); +lean_inc(x_617); +x_618 = lean_array_get_size(x_617); +x_619 = lean_usize_of_nat(x_618); +lean_dec(x_618); +x_620 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(x_619, x_31, x_617); +x_621 = l_Array_append___rarg(x_583, x_620); +x_622 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_622, 0, x_52); +lean_ctor_set(x_622, 1, x_585); +lean_ctor_set(x_622, 2, x_621); +x_623 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__34; +lean_inc(x_577); +x_624 = l_Lean_Name_str___override(x_577, x_623); +x_625 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__36; +lean_inc(x_64); +x_626 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_626, 0, x_64); +lean_ctor_set(x_626, 1, x_625); +x_627 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__42; +lean_inc(x_66); +lean_inc(x_575); +x_628 = l_Lean_addMacroScope(x_575, x_627, x_66); +x_629 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__39; +lean_inc(x_2); +x_630 = l_Lean_Name_str___override(x_2, x_629); +lean_inc(x_1); +x_631 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_631, 0, x_630); +lean_ctor_set(x_631, 1, x_1); +lean_inc(x_1); +x_632 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_632, 0, x_631); +lean_ctor_set(x_632, 1, x_1); +x_633 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__41; +lean_inc(x_64); +x_634 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_634, 0, x_64); +lean_ctor_set(x_634, 1, x_633); +lean_ctor_set(x_634, 2, x_628); +lean_ctor_set(x_634, 3, x_632); +x_635 = lean_array_push(x_49, x_634); +x_636 = lean_array_push(x_635, x_605); +x_637 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__38; +x_638 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_638, 0, x_52); +lean_ctor_set(x_638, 1, x_637); +lean_ctor_set(x_638, 2, x_636); +x_639 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__46; +lean_inc(x_64); +x_640 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_640, 0, x_64); +lean_ctor_set(x_640, 1, x_639); +x_641 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__50; +lean_inc(x_66); +lean_inc(x_575); +x_642 = l_Lean_addMacroScope(x_575, x_641, x_66); +x_643 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__47; +x_644 = l_Lean_Name_str___override(x_2, x_643); +lean_inc(x_1); +x_645 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_645, 0, x_644); +lean_ctor_set(x_645, 1, x_1); +lean_inc(x_1); +x_646 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_646, 0, x_645); +lean_ctor_set(x_646, 1, x_1); +x_647 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__49; +lean_inc(x_64); +x_648 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_648, 0, x_64); +lean_ctor_set(x_648, 1, x_647); +lean_ctor_set(x_648, 2, x_642); +lean_ctor_set(x_648, 3, x_646); +x_649 = lean_array_push(x_49, x_648); +x_650 = lean_array_push(x_649, x_605); +x_651 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_651, 0, x_52); +lean_ctor_set(x_651, 1, x_637); +lean_ctor_set(x_651, 2, x_650); +x_652 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__61; +x_653 = lean_array_push(x_652, x_638); +lean_inc(x_640); +x_654 = lean_array_push(x_653, x_640); +x_655 = lean_array_push(x_654, x_651); +x_656 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_656, 0, x_52); +lean_ctor_set(x_656, 1, x_585); +lean_ctor_set(x_656, 2, x_655); +x_657 = lean_array_push(x_49, x_626); +x_658 = lean_array_push(x_657, x_656); +x_659 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_659, 0, x_52); +lean_ctor_set(x_659, 1, x_585); +lean_ctor_set(x_659, 2, x_658); +x_660 = lean_array_push(x_614, x_659); +x_661 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_661, 0, x_52); +lean_ctor_set(x_661, 1, x_624); +lean_ctor_set(x_661, 2, x_660); +x_662 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__116; +x_663 = lean_array_push(x_662, x_599); +x_664 = lean_array_push(x_663, x_607); +lean_inc(x_611); +x_665 = lean_array_push(x_664, x_611); +x_666 = lean_array_push(x_665, x_616); +x_667 = lean_array_push(x_666, x_622); +x_668 = lean_array_push(x_667, x_605); +x_669 = lean_array_push(x_668, x_661); +x_670 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_670, 0, x_52); +lean_ctor_set(x_670, 1, x_598); +lean_ctor_set(x_670, 2, x_669); +x_671 = lean_array_push(x_49, x_596); +x_672 = lean_array_push(x_671, x_670); +lean_inc(x_592); +x_673 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_673, 0, x_52); +lean_ctor_set(x_673, 1, x_592); +lean_ctor_set(x_673, 2, x_672); +x_674 = lean_array_push(x_652, x_589); +lean_inc(x_590); +x_675 = lean_array_push(x_674, x_590); +x_676 = lean_array_push(x_675, x_673); +lean_inc(x_579); +x_677 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_677, 0, x_52); +lean_ctor_set(x_677, 1, x_579); +lean_ctor_set(x_677, 2, x_676); +x_678 = l_Array_append___rarg(x_12, x_11); +x_679 = l_Array_append___rarg(x_678, x_13); +x_680 = l_Array_append___rarg(x_583, x_679); +x_681 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_681, 0, x_52); +lean_ctor_set(x_681, 1, x_585); +lean_ctor_set(x_681, 2, x_680); +x_682 = lean_array_push(x_587, x_681); +x_683 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_683, 0, x_52); +lean_ctor_set(x_683, 1, x_581); +lean_ctor_set(x_683, 2, x_682); +x_684 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__117; +lean_inc(x_43); +x_685 = l_Lean_Name_str___override(x_43, x_684); +x_686 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__119; +lean_inc(x_64); +x_687 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_687, 0, x_64); +lean_ctor_set(x_687, 1, x_686); +x_688 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__120; +lean_inc(x_43); +x_689 = l_Lean_Name_str___override(x_43, x_688); +x_690 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__122; +lean_inc(x_43); +x_691 = l_Lean_Name_str___override(x_43, x_690); +x_692 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__55; +x_693 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_693, 0, x_52); +lean_ctor_set(x_693, 1, x_691); +lean_ctor_set(x_693, 2, x_692); +x_694 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__126; +x_695 = l_Lean_Name_str___override(x_41, x_694); +x_696 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__147; +x_697 = l_Lean_Name_str___override(x_695, x_696); +lean_inc(x_64); +x_698 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_698, 0, x_64); +lean_ctor_set(x_698, 1, x_696); +x_699 = lean_array_push(x_49, x_698); +x_700 = lean_array_push(x_699, x_605); +x_701 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_701, 0, x_52); +lean_ctor_set(x_701, 1, x_697); +lean_ctor_set(x_701, 2, x_700); +x_702 = lean_array_push(x_49, x_693); +x_703 = lean_array_push(x_702, x_701); +x_704 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_704, 0, x_52); +lean_ctor_set(x_704, 1, x_689); +lean_ctor_set(x_704, 2, x_703); +x_705 = lean_array_push(x_614, x_704); +x_706 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_706, 0, x_52); +lean_ctor_set(x_706, 1, x_585); +lean_ctor_set(x_706, 2, x_705); +x_707 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; +lean_inc(x_64); +x_708 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_708, 0, x_64); +lean_ctor_set(x_708, 1, x_707); +x_709 = lean_array_push(x_652, x_687); +x_710 = lean_array_push(x_709, x_706); +lean_inc(x_708); +x_711 = lean_array_push(x_710, x_708); +x_712 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_712, 0, x_52); +lean_ctor_set(x_712, 1, x_685); +lean_ctor_set(x_712, 2, x_711); +x_713 = lean_array_push(x_614, x_712); +x_714 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_714, 0, x_52); +lean_ctor_set(x_714, 1, x_585); +lean_ctor_set(x_714, 2, x_713); +x_715 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__3; +lean_inc(x_577); +x_716 = l_Lean_Name_str___override(x_577, x_715); +lean_inc(x_64); +x_717 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_717, 0, x_64); +lean_ctor_set(x_717, 1, x_715); +x_718 = lean_array_push(x_614, x_717); +x_719 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_719, 0, x_52); +lean_ctor_set(x_719, 1, x_716); +lean_ctor_set(x_719, 2, x_718); +x_720 = lean_array_push(x_614, x_719); +x_721 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_721, 0, x_52); +lean_ctor_set(x_721, 1, x_585); +lean_ctor_set(x_721, 2, x_720); +x_722 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__17; +x_723 = lean_array_push(x_722, x_714); +x_724 = lean_array_push(x_723, x_605); +x_725 = lean_array_push(x_724, x_605); +x_726 = lean_array_push(x_725, x_605); +x_727 = lean_array_push(x_726, x_721); +x_728 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_728, 0, x_52); +lean_ctor_set(x_728, 1, x_594); +lean_ctor_set(x_728, 2, x_727); +x_729 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__23; +lean_inc(x_577); +x_730 = l_Lean_Name_str___override(x_577, x_729); +lean_inc(x_64); +x_731 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_731, 0, x_64); +lean_ctor_set(x_731, 1, x_729); +x_732 = lean_array_push(x_49, x_62); +x_733 = lean_array_push(x_732, x_605); +x_734 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_734, 0, x_52); +lean_ctor_set(x_734, 1, x_601); +lean_ctor_set(x_734, 2, x_733); +x_735 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__149; +x_736 = l_Lean_Name_str___override(x_577, x_735); +x_737 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__90; +lean_inc(x_64); +x_738 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_738, 0, x_64); +lean_ctor_set(x_738, 1, x_737); +x_739 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__62; +lean_inc(x_43); +x_740 = l_Lean_Name_str___override(x_43, x_739); +lean_inc(x_64); +x_741 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_741, 0, x_64); +lean_ctor_set(x_741, 1, x_739); +x_742 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__39; +lean_inc(x_43); +x_743 = l_Lean_Name_str___override(x_43, x_742); +x_744 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; +lean_inc(x_66); +lean_inc(x_575); +x_745 = l_Lean_addMacroScope(x_575, x_744, x_66); +lean_inc(x_1); +lean_inc(x_5); +x_746 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_746, 0, x_5); +lean_ctor_set(x_746, 1, x_1); +lean_inc(x_1); +x_747 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_747, 0, x_746); +lean_ctor_set(x_747, 1, x_1); +x_748 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; +lean_inc(x_64); +x_749 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_749, 0, x_64); +lean_ctor_set(x_749, 1, x_748); +lean_ctor_set(x_749, 2, x_745); +lean_ctor_set(x_749, 3, x_747); +x_750 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__50; +lean_inc(x_43); +x_751 = l_Lean_Name_str___override(x_43, x_750); +x_752 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +lean_inc(x_64); +x_753 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_753, 0, x_64); +lean_ctor_set(x_753, 1, x_752); +x_754 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__64; +lean_inc(x_43); +x_755 = l_Lean_Name_str___override(x_43, x_754); +x_756 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__66; +lean_inc(x_64); +x_757 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_757, 0, x_64); +lean_ctor_set(x_757, 1, x_756); +x_758 = lean_array_push(x_614, x_757); +x_759 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_759, 0, x_52); +lean_ctor_set(x_759, 1, x_755); +lean_ctor_set(x_759, 2, x_758); +x_760 = lean_array_push(x_614, x_759); +x_761 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_761, 0, x_52); +lean_ctor_set(x_761, 1, x_585); +lean_ctor_set(x_761, 2, x_760); +x_762 = lean_array_push(x_604, x_761); +lean_inc(x_743); +x_763 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_763, 0, x_52); +lean_ctor_set(x_763, 1, x_743); +lean_ctor_set(x_763, 2, x_762); +lean_inc(x_763); +x_764 = lean_array_push(x_49, x_763); +x_765 = lean_array_push(x_764, x_605); +x_766 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_766, 0, x_52); +lean_ctor_set(x_766, 1, x_585); +lean_ctor_set(x_766, 2, x_765); +x_767 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +lean_inc(x_64); +x_768 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_768, 0, x_64); +lean_ctor_set(x_768, 1, x_767); +lean_inc(x_753); +x_769 = lean_array_push(x_652, x_753); +x_770 = lean_array_push(x_769, x_766); +lean_inc(x_768); +x_771 = lean_array_push(x_770, x_768); +x_772 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_772, 0, x_52); +lean_ctor_set(x_772, 1, x_751); +lean_ctor_set(x_772, 2, x_771); +lean_inc(x_57); +x_773 = lean_array_push(x_49, x_57); +lean_inc(x_772); +x_774 = lean_array_push(x_773, x_772); +x_775 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_775, 0, x_52); +lean_ctor_set(x_775, 1, x_585); +lean_ctor_set(x_775, 2, x_774); +x_776 = lean_array_push(x_49, x_749); +x_777 = lean_array_push(x_776, x_775); +lean_inc(x_743); +x_778 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_778, 0, x_52); +lean_ctor_set(x_778, 1, x_743); +lean_ctor_set(x_778, 2, x_777); +x_779 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__67; +lean_inc(x_43); +x_780 = l_Lean_Name_str___override(x_43, x_779); +x_781 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__69; +lean_inc(x_64); +x_782 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_782, 0, x_64); +lean_ctor_set(x_782, 1, x_781); +x_783 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__70; +lean_inc(x_43); +x_784 = l_Lean_Name_str___override(x_43, x_783); +x_785 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72; +lean_inc(x_64); +x_786 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_786, 0, x_64); +lean_ctor_set(x_786, 1, x_785); +x_787 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__4; +lean_inc(x_43); +x_788 = l_Lean_Name_str___override(x_43, x_787); +x_789 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__86; +lean_inc(x_66); +lean_inc(x_575); +x_790 = l_Lean_addMacroScope(x_575, x_789, x_66); +x_791 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__83; +lean_inc(x_5); +x_792 = l_Lean_Name_str___override(x_5, x_791); +lean_inc(x_1); +x_793 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_793, 0, x_792); +lean_ctor_set(x_793, 1, x_1); +lean_inc(x_1); +x_794 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_794, 0, x_793); +lean_ctor_set(x_794, 1, x_1); +x_795 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__85; +lean_inc(x_64); +x_796 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_796, 0, x_64); +lean_ctor_set(x_796, 1, x_795); +lean_ctor_set(x_796, 2, x_790); +lean_ctor_set(x_796, 3, x_794); +lean_inc(x_796); +x_797 = lean_array_push(x_614, x_796); +lean_inc(x_788); +x_798 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_798, 0, x_52); +lean_ctor_set(x_798, 1, x_788); +lean_ctor_set(x_798, 2, x_797); +x_799 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__103; +lean_inc(x_66); +lean_inc(x_575); +x_800 = l_Lean_addMacroScope(x_575, x_799, x_66); +x_801 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__100; +x_802 = l_Lean_Name_str___override(x_5, x_801); +lean_inc(x_1); +x_803 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_803, 0, x_802); +lean_ctor_set(x_803, 1, x_1); +lean_inc(x_1); +x_804 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_804, 0, x_803); +lean_ctor_set(x_804, 1, x_1); +x_805 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__102; +lean_inc(x_64); +x_806 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_806, 0, x_64); +lean_ctor_set(x_806, 1, x_805); +lean_ctor_set(x_806, 2, x_800); +lean_ctor_set(x_806, 3, x_804); +lean_inc(x_806); +x_807 = lean_array_push(x_614, x_806); +x_808 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_808, 0, x_52); +lean_ctor_set(x_808, 1, x_788); +lean_ctor_set(x_808, 2, x_807); +x_809 = lean_array_push(x_652, x_798); +x_810 = lean_array_push(x_809, x_640); +x_811 = lean_array_push(x_810, x_808); +x_812 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_812, 0, x_52); +lean_ctor_set(x_812, 1, x_585); +lean_ctor_set(x_812, 2, x_811); +x_813 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__86; +lean_inc(x_43); +x_814 = l_Lean_Name_str___override(x_43, x_813); +x_815 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_815, 0, x_52); +lean_ctor_set(x_815, 1, x_814); +lean_ctor_set(x_815, 2, x_692); +x_816 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89; +lean_inc(x_64); +x_817 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_817, 0, x_64); +lean_ctor_set(x_817, 1, x_816); +x_818 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__18; +lean_inc(x_786); +x_819 = lean_array_push(x_818, x_786); +x_820 = lean_array_push(x_819, x_605); +x_821 = lean_array_push(x_820, x_812); +x_822 = lean_array_push(x_821, x_815); +x_823 = lean_array_push(x_822, x_605); +lean_inc(x_817); +x_824 = lean_array_push(x_823, x_817); +x_825 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_825, 0, x_52); +lean_ctor_set(x_825, 1, x_784); +lean_ctor_set(x_825, 2, x_824); +x_826 = lean_array_push(x_49, x_782); +lean_inc(x_825); +x_827 = lean_array_push(x_826, x_825); +x_828 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_828, 0, x_52); +lean_ctor_set(x_828, 1, x_780); +lean_ctor_set(x_828, 2, x_827); +x_829 = lean_array_push(x_652, x_741); +lean_inc(x_778); +x_830 = lean_array_push(x_829, x_778); +x_831 = lean_array_push(x_830, x_828); +x_832 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_832, 0, x_52); +lean_ctor_set(x_832, 1, x_740); +lean_ctor_set(x_832, 2, x_831); +x_833 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__5; +lean_inc(x_43); +x_834 = l_Lean_Name_str___override(x_43, x_833); +x_835 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__6; +lean_inc(x_43); +x_836 = l_Lean_Name_str___override(x_43, x_835); +x_837 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; +lean_inc(x_43); +x_838 = l_Lean_Name_str___override(x_43, x_837); +x_839 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__81; +lean_inc(x_43); +x_840 = l_Lean_Name_str___override(x_43, x_839); +x_841 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__7; +lean_inc(x_43); +x_842 = l_Lean_Name_str___override(x_43, x_841); +x_843 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__11; +lean_inc(x_66); +lean_inc(x_575); +x_844 = l_Lean_addMacroScope(x_575, x_843, x_66); +x_845 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__10; lean_inc(x_1); -x_21 = l_List_mapTRAux___at_Lean_MessageData_instCoeListExprMessageData___spec__1(x_20, x_1); -x_22 = l_Lean_MessageData_ofList(x_21); -lean_dec(x_21); -x_23 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__2; -x_24 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_22); -x_25 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6; -x_26 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -x_27 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_7, x_26, x_9, x_10, x_11, x_12, x_13, x_14, x_17); -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_28, x_9, x_10, x_11, x_12, x_13, x_14, x_29); -lean_dec(x_28); -return x_30; -} -} -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6___boxed__const__1() { -_start: -{ -size_t x_1; lean_object* x_2; -x_1 = 0; -x_2 = lean_box_usize(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -lean_dec(x_4); +lean_inc(x_64); +x_846 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_846, 0, x_64); +lean_ctor_set(x_846, 1, x_845); +lean_ctor_set(x_846, 2, x_844); +lean_ctor_set(x_846, 3, x_1); +lean_inc(x_846); +x_847 = lean_array_push(x_614, x_846); +x_848 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_848, 0, x_52); +lean_ctor_set(x_848, 1, x_585); +lean_ctor_set(x_848, 2, x_847); +x_849 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_850 = lean_array_push(x_849, x_786); +lean_inc(x_848); +x_851 = lean_array_push(x_850, x_848); +x_852 = lean_array_push(x_851, x_605); +x_853 = lean_array_push(x_852, x_817); +x_854 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_854, 0, x_52); +lean_ctor_set(x_854, 1, x_842); +lean_ctor_set(x_854, 2, x_853); +x_855 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__1; +lean_inc(x_43); +x_856 = l_Lean_Name_str___override(x_43, x_855); +x_857 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3; +lean_inc(x_64); +x_858 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_858, 0, x_64); +lean_ctor_set(x_858, 1, x_857); +x_859 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__15; +lean_inc(x_66); +lean_inc(x_575); +x_860 = l_Lean_addMacroScope(x_575, x_859, x_66); lean_inc(x_1); -x_12 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2), 12, 1); -lean_closure_set(x_12, 0, x_1); -x_13 = l_Lean_Server_RpcEncoding_instInhabitedCtorState___closed__1; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_3); -lean_inc(x_2); -x_14 = l_Lean_Server_RpcEncoding_foldWithConstructors___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__33___rarg(x_2, x_3, x_12, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); +x_861 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_861, 0, x_859); +lean_ctor_set(x_861, 1, x_1); +lean_inc(x_1); +x_862 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_862, 0, x_861); +lean_ctor_set(x_862, 1, x_1); +x_863 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__14; +lean_inc(x_64); +x_864 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_864, 0, x_64); +lean_ctor_set(x_864, 1, x_863); +lean_ctor_set(x_864, 2, x_860); +lean_ctor_set(x_864, 3, x_862); +x_865 = lean_array_push(x_49, x_864); +lean_inc(x_848); +x_866 = lean_array_push(x_865, x_848); +lean_inc(x_743); +x_867 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_867, 0, x_52); +lean_ctor_set(x_867, 1, x_743); +lean_ctor_set(x_867, 2, x_866); +x_868 = lean_array_push(x_849, x_858); +x_869 = lean_array_push(x_868, x_605); +lean_inc(x_869); +x_870 = lean_array_push(x_869, x_867); +lean_inc(x_708); +x_871 = lean_array_push(x_870, x_708); +lean_inc(x_856); +x_872 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_872, 0, x_52); +lean_ctor_set(x_872, 1, x_856); +lean_ctor_set(x_872, 2, x_871); +x_873 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__19; +lean_inc(x_66); +lean_inc(x_575); +x_874 = l_Lean_addMacroScope(x_575, x_873, x_66); +x_875 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16; +x_876 = l_Lean_Name_str___override(x_14, x_875); +lean_inc(x_1); +x_877 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_877, 0, x_876); +lean_ctor_set(x_877, 1, x_1); +lean_inc(x_1); +x_878 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_878, 0, x_877); +lean_ctor_set(x_878, 1, x_1); +x_879 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__18; +lean_inc(x_64); +x_880 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_880, 0, x_64); +lean_ctor_set(x_880, 1, x_879); +lean_ctor_set(x_880, 2, x_874); +lean_ctor_set(x_880, 3, x_878); +x_881 = lean_array_push(x_49, x_880); +x_882 = lean_array_push(x_881, x_848); +lean_inc(x_743); +x_883 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_883, 0, x_52); +lean_ctor_set(x_883, 1, x_743); +lean_ctor_set(x_883, 2, x_882); +x_884 = lean_array_push(x_869, x_883); +x_885 = lean_array_push(x_884, x_708); +x_886 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_886, 0, x_52); +lean_ctor_set(x_886, 1, x_856); +lean_ctor_set(x_886, 2, x_885); +x_887 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1; +lean_inc(x_43); +x_888 = l_Lean_Name_str___override(x_43, x_887); +x_889 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__23; +lean_inc(x_66); +lean_inc(x_575); +x_890 = l_Lean_addMacroScope(x_575, x_889, x_66); +x_891 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__22; +lean_inc(x_1); +lean_inc(x_64); +x_892 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_892, 0, x_64); +lean_ctor_set(x_892, 1, x_891); +lean_ctor_set(x_892, 2, x_890); +lean_ctor_set(x_892, 3, x_1); +lean_inc(x_892); +x_893 = lean_array_push(x_614, x_892); +x_894 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_894, 0, x_52); +lean_ctor_set(x_894, 1, x_585); +lean_ctor_set(x_894, 2, x_893); +x_895 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; +lean_inc(x_64); +x_896 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_896, 0, x_64); +lean_ctor_set(x_896, 1, x_895); +x_897 = lean_array_push(x_49, x_896); +lean_inc(x_57); +lean_inc(x_897); +x_898 = lean_array_push(x_897, x_57); +x_899 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_899, 0, x_52); +lean_ctor_set(x_899, 1, x_585); +lean_ctor_set(x_899, 2, x_898); +x_900 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; +x_901 = lean_array_push(x_900, x_753); +x_902 = lean_array_push(x_901, x_894); +lean_inc(x_902); +x_903 = lean_array_push(x_902, x_899); +x_904 = lean_array_push(x_903, x_605); +lean_inc(x_768); +x_905 = lean_array_push(x_904, x_768); +lean_inc(x_888); +x_906 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_906, 0, x_52); +lean_ctor_set(x_906, 1, x_888); +lean_ctor_set(x_906, 2, x_905); +x_907 = lean_array_push(x_849, x_854); +x_908 = lean_array_push(x_907, x_872); +x_909 = lean_array_push(x_908, x_886); +lean_inc(x_909); +x_910 = lean_array_push(x_909, x_906); +x_911 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_911, 0, x_52); +lean_ctor_set(x_911, 1, x_585); +lean_ctor_set(x_911, 2, x_910); +x_912 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__36; +lean_inc(x_43); +x_913 = l_Lean_Name_str___override(x_43, x_912); +x_914 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__27; +lean_inc(x_66); +lean_inc(x_575); +x_915 = l_Lean_addMacroScope(x_575, x_914, x_66); +lean_inc(x_1); +x_916 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_916, 0, x_914); +lean_ctor_set(x_916, 1, x_1); +lean_inc(x_1); +x_917 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_917, 0, x_916); +lean_ctor_set(x_917, 1, x_1); +x_918 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__26; +lean_inc(x_64); +x_919 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_919, 0, x_64); +lean_ctor_set(x_919, 1, x_918); +lean_ctor_set(x_919, 2, x_915); +lean_ctor_set(x_919, 3, x_917); +x_920 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__31; +lean_inc(x_66); +lean_inc(x_575); +x_921 = l_Lean_addMacroScope(x_575, x_920, x_66); +lean_inc(x_1); +x_922 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_922, 0, x_920); +lean_ctor_set(x_922, 1, x_1); +lean_inc(x_1); +x_923 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_923, 0, x_922); +lean_ctor_set(x_923, 1, x_1); +x_924 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__30; +lean_inc(x_64); +x_925 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_925, 0, x_64); +lean_ctor_set(x_925, 1, x_924); +lean_ctor_set(x_925, 2, x_921); +lean_ctor_set(x_925, 3, x_923); +x_926 = lean_array_push(x_652, x_925); +x_927 = lean_array_push(x_926, x_846); +lean_inc(x_927); +x_928 = lean_array_push(x_927, x_772); +x_929 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_929, 0, x_52); +lean_ctor_set(x_929, 1, x_585); +lean_ctor_set(x_929, 2, x_928); +x_930 = lean_array_push(x_49, x_919); +lean_inc(x_930); +x_931 = lean_array_push(x_930, x_929); +lean_inc(x_743); +x_932 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_932, 0, x_52); +lean_ctor_set(x_932, 1, x_743); +lean_ctor_set(x_932, 2, x_931); +lean_inc(x_897); +x_933 = lean_array_push(x_897, x_932); +lean_inc(x_913); +x_934 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_934, 0, x_52); +lean_ctor_set(x_934, 1, x_913); +lean_ctor_set(x_934, 2, x_933); +x_935 = lean_array_push(x_614, x_934); +x_936 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_936, 0, x_52); +lean_ctor_set(x_936, 1, x_585); +lean_ctor_set(x_936, 2, x_935); +x_937 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__32; +lean_inc(x_43); +x_938 = l_Lean_Name_str___override(x_43, x_937); +lean_inc(x_64); +x_939 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_939, 0, x_64); +lean_ctor_set(x_939, 1, x_937); +x_940 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__33; +lean_inc(x_43); +x_941 = l_Lean_Name_str___override(x_43, x_940); +x_942 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__34; +lean_inc(x_43); +x_943 = l_Lean_Name_str___override(x_43, x_942); +x_944 = l_Lean_addMacroScope(x_575, x_15, x_66); +x_945 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__140; +lean_inc(x_64); +x_946 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_946, 0, x_64); +lean_ctor_set(x_946, 1, x_945); +lean_ctor_set(x_946, 2, x_944); +lean_ctor_set(x_946, 3, x_1); +x_947 = lean_array_push(x_49, x_946); +x_948 = lean_array_push(x_947, x_605); +x_949 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_949, 0, x_52); +lean_ctor_set(x_949, 1, x_585); +lean_ctor_set(x_949, 2, x_948); +lean_inc(x_897); +x_950 = lean_array_push(x_897, x_778); +lean_inc(x_913); +x_951 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_951, 0, x_52); +lean_ctor_set(x_951, 1, x_913); +lean_ctor_set(x_951, 2, x_950); +x_952 = lean_array_push(x_614, x_951); +x_953 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_953, 0, x_52); +lean_ctor_set(x_953, 1, x_585); +lean_ctor_set(x_953, 2, x_952); +x_954 = lean_array_push(x_849, x_949); +x_955 = lean_array_push(x_954, x_953); +lean_inc(x_738); +x_956 = lean_array_push(x_955, x_738); +x_957 = lean_array_push(x_956, x_825); +x_958 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_958, 0, x_52); +lean_ctor_set(x_958, 1, x_943); +lean_ctor_set(x_958, 2, x_957); +x_959 = lean_array_push(x_614, x_958); +x_960 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_960, 0, x_52); +lean_ctor_set(x_960, 1, x_941); +lean_ctor_set(x_960, 2, x_959); +x_961 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__35; +lean_inc(x_43); +x_962 = l_Lean_Name_str___override(x_43, x_961); +lean_inc(x_64); +x_963 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_963, 0, x_64); +lean_ctor_set(x_963, 1, x_961); +x_964 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__36; +lean_inc(x_43); +x_965 = l_Lean_Name_str___override(x_43, x_964); +x_966 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__59; +x_967 = lean_array_push(x_966, x_892); +x_968 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_968, 0, x_52); +lean_ctor_set(x_968, 1, x_965); +lean_ctor_set(x_968, 2, x_967); +x_969 = lean_array_push(x_614, x_968); +x_970 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_970, 0, x_52); +lean_ctor_set(x_970, 1, x_585); +lean_ctor_set(x_970, 2, x_969); +x_971 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__37; +x_972 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_972, 0, x_64); +lean_ctor_set(x_972, 1, x_971); +x_973 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__38; +x_974 = l_Lean_Name_str___override(x_43, x_973); +x_975 = lean_ctor_get(x_27, 1); +lean_inc(x_975); +x_976 = lean_array_get_size(x_975); +x_977 = lean_usize_of_nat(x_976); +lean_dec(x_976); +x_978 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(x_977, x_31, x_975); +x_979 = l_Array_append___rarg(x_583, x_978); +x_980 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_980, 0, x_52); +lean_ctor_set(x_980, 1, x_585); +lean_ctor_set(x_980, 2, x_979); +x_981 = lean_array_push(x_614, x_980); +lean_inc(x_974); +x_982 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_982, 0, x_52); +lean_ctor_set(x_982, 1, x_974); +lean_ctor_set(x_982, 2, x_981); +x_983 = lean_array_push(x_818, x_963); +x_984 = lean_array_push(x_983, x_605); +x_985 = lean_array_push(x_984, x_605); +x_986 = lean_array_push(x_985, x_970); +x_987 = lean_array_push(x_986, x_972); +lean_inc(x_987); +x_988 = lean_array_push(x_987, x_982); +lean_inc(x_962); +x_989 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_989, 0, x_52); +lean_ctor_set(x_989, 1, x_962); +lean_ctor_set(x_989, 2, x_988); +x_990 = lean_array_push(x_849, x_939); +x_991 = lean_array_push(x_990, x_960); +x_992 = lean_array_push(x_991, x_605); +lean_inc(x_992); +x_993 = lean_array_push(x_992, x_989); +lean_inc(x_938); +x_994 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_994, 0, x_52); +lean_ctor_set(x_994, 1, x_938); +lean_ctor_set(x_994, 2, x_993); +x_995 = lean_array_push(x_900, x_796); +x_996 = lean_array_push(x_995, x_911); +x_997 = lean_array_push(x_996, x_936); +lean_inc(x_738); +x_998 = lean_array_push(x_997, x_738); +x_999 = lean_array_push(x_998, x_994); +lean_inc(x_840); +x_1000 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1000, 0, x_52); +lean_ctor_set(x_1000, 1, x_840); +lean_ctor_set(x_1000, 2, x_999); +x_1001 = lean_array_push(x_614, x_1000); +lean_inc(x_838); +x_1002 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1002, 0, x_52); +lean_ctor_set(x_1002, 1, x_838); +lean_ctor_set(x_1002, 2, x_1001); +x_1003 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__40; +x_1004 = lean_array_push(x_1003, x_1002); +lean_inc(x_836); +x_1005 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1005, 0, x_52); +lean_ctor_set(x_1005, 1, x_836); +lean_ctor_set(x_1005, 2, x_1004); +lean_inc(x_897); +x_1006 = lean_array_push(x_897, x_763); +x_1007 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1007, 0, x_52); +lean_ctor_set(x_1007, 1, x_585); +lean_ctor_set(x_1007, 2, x_1006); +x_1008 = lean_array_push(x_902, x_1007); +x_1009 = lean_array_push(x_1008, x_605); +x_1010 = lean_array_push(x_1009, x_768); +x_1011 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1011, 0, x_52); +lean_ctor_set(x_1011, 1, x_888); +lean_ctor_set(x_1011, 2, x_1010); +x_1012 = lean_array_push(x_909, x_1011); +x_1013 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1013, 0, x_52); +lean_ctor_set(x_1013, 1, x_585); +lean_ctor_set(x_1013, 2, x_1012); +x_1014 = lean_array_push(x_927, x_57); +x_1015 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1015, 0, x_52); +lean_ctor_set(x_1015, 1, x_585); +lean_ctor_set(x_1015, 2, x_1014); +x_1016 = lean_array_push(x_930, x_1015); +x_1017 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1017, 0, x_52); +lean_ctor_set(x_1017, 1, x_743); +lean_ctor_set(x_1017, 2, x_1016); +x_1018 = lean_array_push(x_897, x_1017); +x_1019 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1019, 0, x_52); +lean_ctor_set(x_1019, 1, x_913); +lean_ctor_set(x_1019, 2, x_1018); +x_1020 = lean_array_push(x_614, x_1019); +x_1021 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1021, 0, x_52); +lean_ctor_set(x_1021, 1, x_585); +lean_ctor_set(x_1021, 2, x_1020); +x_1022 = lean_ctor_get(x_27, 2); +lean_inc(x_1022); +lean_dec(x_27); +x_1023 = lean_array_get_size(x_1022); +x_1024 = lean_usize_of_nat(x_1023); +lean_dec(x_1023); +x_1025 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(x_1024, x_31, x_1022); +x_1026 = l_Array_append___rarg(x_583, x_1025); +x_1027 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1027, 0, x_52); +lean_ctor_set(x_1027, 1, x_585); +lean_ctor_set(x_1027, 2, x_1026); +x_1028 = lean_array_push(x_614, x_1027); +x_1029 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1029, 0, x_52); +lean_ctor_set(x_1029, 1, x_974); +lean_ctor_set(x_1029, 2, x_1028); +x_1030 = lean_array_push(x_987, x_1029); +x_1031 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1031, 0, x_52); +lean_ctor_set(x_1031, 1, x_962); +lean_ctor_set(x_1031, 2, x_1030); +x_1032 = lean_array_push(x_992, x_1031); +x_1033 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1033, 0, x_52); +lean_ctor_set(x_1033, 1, x_938); +lean_ctor_set(x_1033, 2, x_1032); +x_1034 = lean_array_push(x_900, x_806); +x_1035 = lean_array_push(x_1034, x_1013); +x_1036 = lean_array_push(x_1035, x_1021); +lean_inc(x_738); +x_1037 = lean_array_push(x_1036, x_738); +x_1038 = lean_array_push(x_1037, x_1033); +x_1039 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1039, 0, x_52); +lean_ctor_set(x_1039, 1, x_840); +lean_ctor_set(x_1039, 2, x_1038); +x_1040 = lean_array_push(x_614, x_1039); +x_1041 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1041, 0, x_52); +lean_ctor_set(x_1041, 1, x_838); +lean_ctor_set(x_1041, 2, x_1040); +x_1042 = lean_array_push(x_1003, x_1041); +x_1043 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1043, 0, x_52); +lean_ctor_set(x_1043, 1, x_836); +lean_ctor_set(x_1043, 2, x_1042); +x_1044 = lean_array_push(x_849, x_1005); +x_1045 = lean_array_push(x_1044, x_605); +x_1046 = lean_array_push(x_1045, x_1043); +x_1047 = lean_array_push(x_1046, x_605); +x_1048 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1048, 0, x_52); +lean_ctor_set(x_1048, 1, x_585); +lean_ctor_set(x_1048, 2, x_1047); +x_1049 = lean_array_push(x_49, x_613); +x_1050 = lean_array_push(x_1049, x_1048); +x_1051 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1051, 0, x_52); +lean_ctor_set(x_1051, 1, x_834); +lean_ctor_set(x_1051, 2, x_1050); +x_1052 = lean_array_push(x_614, x_1051); +x_1053 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1053, 0, x_52); +lean_ctor_set(x_1053, 1, x_585); +lean_ctor_set(x_1053, 2, x_1052); +x_1054 = lean_array_push(x_652, x_738); +x_1055 = lean_array_push(x_1054, x_832); +x_1056 = lean_array_push(x_1055, x_1053); +x_1057 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1057, 0, x_52); +lean_ctor_set(x_1057, 1, x_736); +lean_ctor_set(x_1057, 2, x_1056); +x_1058 = lean_array_push(x_662, x_731); +x_1059 = lean_array_push(x_1058, x_734); +x_1060 = lean_array_push(x_1059, x_611); +x_1061 = lean_array_push(x_1060, x_1057); +x_1062 = lean_array_push(x_1061, x_605); +x_1063 = lean_array_push(x_1062, x_605); +x_1064 = lean_array_push(x_1063, x_605); +x_1065 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1065, 0, x_52); +lean_ctor_set(x_1065, 1, x_730); +lean_ctor_set(x_1065, 2, x_1064); +x_1066 = lean_array_push(x_49, x_728); +x_1067 = lean_array_push(x_1066, x_1065); +x_1068 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1068, 0, x_52); +lean_ctor_set(x_1068, 1, x_592); +lean_ctor_set(x_1068, 2, x_1067); +x_1069 = lean_array_push(x_652, x_683); +x_1070 = lean_array_push(x_1069, x_590); +x_1071 = lean_array_push(x_1070, x_1068); +x_1072 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1072, 0, x_52); +lean_ctor_set(x_1072, 1, x_579); +lean_ctor_set(x_1072, 2, x_1071); +x_1073 = lean_array_push(x_49, x_677); +x_1074 = lean_array_push(x_1073, x_1072); +x_1075 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1075, 0, x_52); +lean_ctor_set(x_1075, 1, x_585); +lean_ctor_set(x_1075, 2, x_1074); +x_1076 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1076, 0, x_1075); +lean_ctor_set(x_1076, 1, x_573); +return x_1076; +} +} +else +{ +uint8_t x_1077; +lean_dec(x_27); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_15); lean_dec(x_14); -x_17 = lean_box(0); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -x_19 = lean_array_get_size(x_18); -x_20 = lean_usize_of_nat(x_19); -lean_dec(x_19); -x_21 = 0; -x_22 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35(x_20, x_21, x_18); -x_23 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -x_24 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6___boxed__const__1; -x_25 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___boxed), 15, 7); -lean_closure_set(x_25, 0, x_17); -lean_closure_set(x_25, 1, x_24); -lean_closure_set(x_25, 2, x_23); -lean_closure_set(x_25, 3, x_2); -lean_closure_set(x_25, 4, x_3); -lean_closure_set(x_25, 5, x_15); -lean_closure_set(x_25, 6, x_1); -x_26 = lean_box(0); -x_27 = l_Lean_Meta_withLocalDecls___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__46___rarg(x_26, x_22, x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_16); -return x_27; -} -else -{ -uint8_t x_28; -lean_dec(x_10); -lean_dec(x_9); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_28 = !lean_is_exclusive(x_14); -if (x_28 == 0) +x_1077 = !lean_is_exclusive(x_32); +if (x_1077 == 0) { -return x_14; +return x_32; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_14, 0); -x_30 = lean_ctor_get(x_14, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_14); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; -} -} -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("for inductive ", 14); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_10 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__5; -x_34 = lean_st_ref_get(x_8, x_9); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_35, 3); -lean_inc(x_36); -lean_dec(x_35); -x_37 = lean_ctor_get_uint8(x_36, sizeof(void*)*1); -lean_dec(x_36); -if (x_37 == 0) -{ -lean_object* x_38; uint8_t x_39; -x_38 = lean_ctor_get(x_34, 1); -lean_inc(x_38); -lean_dec(x_34); -x_39 = 0; -x_11 = x_39; -x_12 = x_38; -goto block_33; +lean_object* x_1078; lean_object* x_1079; lean_object* x_1080; +x_1078 = lean_ctor_get(x_32, 0); +x_1079 = lean_ctor_get(x_32, 1); +lean_inc(x_1079); +lean_inc(x_1078); +lean_dec(x_32); +x_1080 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1080, 0, x_1078); +lean_ctor_set(x_1080, 1, x_1079); +return x_1080; } -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_40 = lean_ctor_get(x_34, 1); -lean_inc(x_40); -lean_dec(x_34); -x_41 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_10, x_3, x_4, x_5, x_6, x_7, x_8, x_40); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_44 = lean_unbox(x_42); -lean_dec(x_42); -x_11 = x_44; -x_12 = x_43; -goto block_33; } -block_33: -{ -if (x_11 == 0) -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_box(0); -x_14 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6(x_10, x_1, x_2, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -return x_14; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_15 = lean_ctor_get(x_1, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); +uint8_t x_1081; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); lean_dec(x_15); -x_17 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_17, 0, x_16); -x_18 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__2; -x_19 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -x_20 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9; -x_21 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -lean_inc(x_2); -x_22 = lean_array_to_list(lean_box(0), x_2); -x_23 = lean_box(0); -x_24 = l_List_mapTRAux___at_Lean_MessageData_instCoeListExprMessageData___spec__1(x_22, x_23); -x_25 = l_Lean_MessageData_ofList(x_24); -lean_dec(x_24); -x_26 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_26, 0, x_21); -lean_ctor_set(x_26, 1, x_25); -x_27 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6; -x_28 = lean_alloc_ctor(10, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_10, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6(x_10, x_1, x_2, x_30, x_3, x_4, x_5, x_6, x_7, x_8, x_31); -return x_32; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_12 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -lean_dec(x_4); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; lean_object* x_5; -x_4 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_5 = l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5(x_1, x_4, x_3); -lean_dec(x_3); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -size_t x_7; lean_object* x_8; -x_7 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_8 = l_Std_PersistentHashMap_insertAux_traverse___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__9(x_7, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_3); -lean_dec(x_2); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_7 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_8 = l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_1, x_6, x_7, x_4, x_5); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Init_Data_Array_BinSearch_0__Array_binInsertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__14(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_1); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Array_binInsertM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_1); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_5; -} -} -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__18(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__21(x_1, x_2, x_5, x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; -} +x_1081 = !lean_is_exclusive(x_26); +if (x_1081 == 0) +{ +return x_26; } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__22(x_1, x_2, x_5, x_6); -lean_dec(x_2); -lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; +lean_object* x_1082; lean_object* x_1083; lean_object* x_1084; +x_1082 = lean_ctor_get(x_26, 0); +x_1083 = lean_ctor_get(x_26, 1); +lean_inc(x_1083); +lean_inc(x_1082); +lean_dec(x_26); +x_1084 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1084, 0, x_1082); +lean_ctor_set(x_1084, 1, x_1083); +return x_1084; } } -LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__20___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__20(x_1, x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__1() { _start: { -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__23(x_1, x_2, x_5, x_6); -lean_dec(x_2); -lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } } -LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__19___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__19(x_1, x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_14 = lean_st_ref_get(x_12, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +lean_inc(x_11); +x_18 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_11, x_12, x_16); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_ctor_get(x_11, 10); +lean_inc(x_21); +x_22 = lean_st_ref_get(x_12, x_20); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_environment_main_module(x_25); +x_27 = lean_box(0); +x_28 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__31; +x_29 = l_Lean_addMacroScope(x_26, x_28, x_21); +x_30 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__30; +x_31 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_31, 0, x_19); +lean_ctor_set(x_31, 1, x_30); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_27); +x_32 = l_Lean_Syntax_getId(x_31); +lean_dec(x_31); +x_33 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__1; +lean_inc(x_32); +x_34 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_27); +lean_ctor_set(x_34, 2, x_33); +x_35 = 1; +x_36 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set_uint8(x_36, sizeof(void*)*1, x_35); +x_37 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_37, 0, x_36); +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_38 = l_Lean_addDecl___at_Lean_Elab_Term_declareTacticSyntax___spec__1(x_37, x_7, x_8, x_9, x_10, x_11, x_12, x_24); +if (lean_obj_tag(x_38) == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; lean_object* x_54; +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +lean_dec(x_38); +lean_inc(x_32); +x_40 = l_Lean_Expr_const___override(x_32, x_27); +x_41 = lean_ctor_get(x_1, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +lean_dec(x_41); +lean_inc(x_42); +x_43 = l_Lean_Expr_const___override(x_42, x_27); +lean_inc(x_2); +x_44 = l_Lean_mkAppN(x_43, x_2); +x_45 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__1; +x_46 = l_Lean_mkAppB(x_45, x_44, x_40); +x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; +x_48 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; +x_49 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__5; +x_50 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__46; +x_51 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__141; +x_52 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___boxed), 23, 15); +lean_closure_set(x_52, 0, x_27); +lean_closure_set(x_52, 1, x_47); +lean_closure_set(x_52, 2, x_28); +lean_closure_set(x_52, 3, x_30); +lean_closure_set(x_52, 4, x_48); +lean_closure_set(x_52, 5, x_49); +lean_closure_set(x_52, 6, x_32); +lean_closure_set(x_52, 7, x_42); +lean_closure_set(x_52, 8, x_1); +lean_closure_set(x_52, 9, x_2); +lean_closure_set(x_52, 10, x_3); +lean_closure_set(x_52, 11, x_4); +lean_closure_set(x_52, 12, x_5); +lean_closure_set(x_52, 13, x_50); +lean_closure_set(x_52, 14, x_51); +x_53 = 3; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_54 = l_Lean_Meta_withLocalDecl___at_Lean_Elab_Term_withAuxDecl___spec__3___rarg(x_51, x_53, x_46, x_52, x_7, x_8, x_9, x_10, x_11, x_12, x_39); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +lean_dec(x_54); +x_57 = l_Lean_setEnv___at_Lean_Elab_Term_expandDeclId___spec__7(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_56); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) +{ +lean_object* x_59; +x_59 = lean_ctor_get(x_57, 0); +lean_dec(x_59); +lean_ctor_set(x_57, 0, x_55); +return x_57; } -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__17(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; +lean_object* x_60; lean_object* x_61; +x_60 = lean_ctor_get(x_57, 1); +lean_inc(x_60); +lean_dec(x_57); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_55); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__16(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} +lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; +x_62 = lean_ctor_get(x_54, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_54, 1); +lean_inc(x_63); +lean_dec(x_54); +x_64 = l_Lean_setEnv___at_Lean_Elab_Term_expandDeclId___spec__7(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_63); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_65 = !lean_is_exclusive(x_64); +if (x_65 == 0) +{ +lean_object* x_66; +x_66 = lean_ctor_get(x_64, 0); +lean_dec(x_66); +lean_ctor_set_tag(x_64, 1); +lean_ctor_set(x_64, 0, x_62); +return x_64; } -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__26(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; +lean_object* x_67; lean_object* x_68; +x_67 = lean_ctor_get(x_64, 1); +lean_inc(x_67); +lean_dec(x_64); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_62); +lean_ctor_set(x_68, 1, x_67); +return x_68; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +} +else { -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); +lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +lean_dec(x_32); +lean_dec(x_5); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__29(x_1, x_2, x_5, x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; -} +x_69 = lean_ctor_get(x_38, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_38, 1); +lean_inc(x_70); +lean_dec(x_38); +x_71 = l_Lean_setEnv___at_Lean_Elab_Term_expandDeclId___spec__7(x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_70); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_72 = !lean_is_exclusive(x_71); +if (x_72 == 0) +{ +lean_object* x_73; +x_73 = lean_ctor_get(x_71, 0); +lean_dec(x_73); +lean_ctor_set_tag(x_71, 1); +lean_ctor_set(x_71, 0, x_69); +return x_71; } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +else { -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__30(x_1, x_2, x_5, x_6); -lean_dec(x_2); -lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; +lean_object* x_74; lean_object* x_75; +x_74 = lean_ctor_get(x_71, 1); +lean_inc(x_74); +lean_dec(x_71); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_69); +lean_ctor_set(x_75, 1, x_74); +return x_75; } } -LEAN_EXPORT lean_object* l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__28___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_PersistentArray_anyMAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__28(x_1, x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__31___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__1() { _start: { -size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_6 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__31(x_1, x_2, x_5, x_6); -lean_dec(x_2); -lean_dec(x_1); -x_8 = lean_box(x_7); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("for inductive ", 14); +return x_1; } } -LEAN_EXPORT lean_object* l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__27___boxed(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__2() { _start: { -uint8_t x_3; lean_object* x_4; -x_3 = l_Std_PersistentArray_anyM___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__27(x_1, x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_4; -x_4 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__25(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; +lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_13 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__5; +x_37 = lean_st_ref_get(x_11, x_12); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_38, 3); +lean_inc(x_39); +lean_dec(x_38); +x_40 = lean_ctor_get_uint8(x_39, sizeof(void*)*1); +lean_dec(x_39); +if (x_40 == 0) +{ +lean_object* x_41; uint8_t x_42; +x_41 = lean_ctor_get(x_37, 1); +lean_inc(x_41); +lean_dec(x_37); +x_42 = 0; +x_14 = x_42; +x_15 = x_41; +goto block_36; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_43 = lean_ctor_get(x_37, 1); +lean_inc(x_43); +lean_dec(x_37); +x_44 = l___private_Lean_Util_Trace_0__Lean_checkTraceOptionM___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__2(x_13, x_6, x_7, x_8, x_9, x_10, x_11, x_43); +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = lean_unbox(x_45); +lean_dec(x_45); +x_14 = x_47; +x_15 = x_46; +goto block_36; } +block_36: +{ +if (x_14 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_box(0); +x_17 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3(x_1, x_2, x_4, x_3, x_5, x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +return x_17; } -LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__24(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; +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; +x_18 = lean_ctor_get(x_1, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +lean_dec(x_18); +x_20 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_20, 0, x_19); +x_21 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__2; +x_22 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +x_23 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9; +x_24 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +lean_inc(x_2); +x_25 = lean_array_to_list(lean_box(0), x_2); +x_26 = lean_box(0); +x_27 = l_List_mapTRAux___at_Lean_MessageData_instCoeListExprMessageData___spec__1(x_25, x_26); +x_28 = l_Lean_MessageData_ofList(x_27); +lean_dec(x_27); +x_29 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_29, 0, x_24); +lean_ctor_set(x_29, 1, x_28); +x_30 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__11; +x_31 = lean_alloc_ctor(10, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_addTrace___at___private_Lean_Elab_Term_0__Lean_Elab_Term_tryCoe___spec__1(x_13, x_31, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3(x_1, x_2, x_4, x_3, x_5, x_33, x_6, x_7, x_8, x_9, x_10, x_11, x_34); +lean_dec(x_33); +return x_35; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_11; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { size_t x_13; size_t x_14; lean_object* x_15; @@ -19312,29 +12585,42 @@ x_13 = lean_unbox_usize(x_3); lean_dec(x_3); x_14 = lean_unbox_usize(x_4); lean_dec(x_4); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); -lean_dec(x_2); +lean_dec(x_6); lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_9; -x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__2(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__3(x_1, x_2, x_6, x_7, x_5); lean_dec(x_2); lean_dec(x_1); -return x_9; +return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -19342,24 +12628,11 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__4(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__36___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_14 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_15 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__36(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_2); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__37___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -19367,7 +12640,7 @@ x_11 = lean_unbox_usize(x_1); lean_dec(x_1); x_12 = lean_unbox_usize(x_2); lean_dec(x_2); -x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__37(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__5(x_11, x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -19375,7 +12648,7 @@ lean_dec(x_4); return x_13; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__38___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -19383,12 +12656,12 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__38(x_1, x_5, x_6, x_4); +x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__6(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__39___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { size_t x_17; size_t x_18; lean_object* x_19; @@ -19396,7 +12669,7 @@ x_17 = lean_unbox_usize(x_7); lean_dec(x_7); x_18 = lean_unbox_usize(x_8); lean_dec(x_8); -x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__39(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__7(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_13); lean_dec(x_12); @@ -19406,20 +12679,7 @@ lean_dec(x_1); return x_19; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__40___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -size_t x_5; size_t x_6; lean_object* x_7; -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__40(x_1, x_5, x_6, x_4); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__41___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { size_t x_17; size_t x_18; lean_object* x_19; @@ -19427,31 +12687,17 @@ x_17 = lean_unbox_usize(x_7); lean_dec(x_7); x_18 = lean_unbox_usize(x_8); lean_dec(x_8); -x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__41(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -lean_dec(x_5); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__42___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__42(x_1, x_2, x_6, x_7, x_5); -lean_dec(x_2); lean_dec(x_1); -return x_8; +return x_19; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__43___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -19459,12 +12705,12 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__43(x_1, x_5, x_6, x_4); +x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__11(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__44___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -19472,11 +12718,11 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__44(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__12(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -19484,51 +12730,81 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__45(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__13(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_3); -return x_11; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -size_t x_17; lean_object* x_18; -x_17 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_18 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3(x_1, x_2, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_9); -lean_dec(x_7); -return x_18; +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +_start: +{ +lean_object* x_20; +x_20 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_6); +return x_20; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -size_t x_15; lean_object* x_16; -x_15 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_16 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4(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); -lean_dec(x_7); -return x_16; +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; +lean_object* x_21 = _args[20]; +lean_object* x_22 = _args[21]; +lean_object* x_23 = _args[22]; +_start: +{ +lean_object* x_24; +x_24 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22, x_23); +lean_dec(x_16); +return x_24; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___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: { -size_t x_16; lean_object* x_17; -x_16 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_17 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5(x_1, x_16, 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); -return x_17; +lean_object* x_14; +x_14 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_6); +return x_14; } } LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { @@ -19712,795 +12988,1057 @@ return x_25; } } } -static lean_object* _init_l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1() { _start: { -lean_object* x_1; -x_1 = l_Lean_Elab_Term_instInhabitedTermElabM(lean_box(0)); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__2() { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1; -x_10 = lean_panic_fn(x_9, x_1); -x_11 = lean_apply_7(x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Packet", 6); +return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__1() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("hole", 4); +x_1 = lean_mk_string_from_bytes("type", 4); return x_1; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__2() { +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; +x_2 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__5() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("_", 1); +x_1 = lean_mk_string_from_bytes("Type", 4); return x_1; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_lt(x_3, x_2); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_4); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_22; +x_14 = lean_array_uget(x_1, x_3); +x_22 = !lean_is_exclusive(x_4); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_4, 0); +x_24 = lean_ctor_get(x_4, 1); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +lean_inc(x_7); +lean_inc(x_14); +x_27 = l_Lean_Meta_getFVarLocalDecl(x_14, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = l_Lean_LocalDecl_userName(x_28); +lean_dec(x_28); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_14); +x_31 = lean_infer_type(x_14, x_7, x_8, x_9, x_10, x_29); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = lean_box(0); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_35 = l_Lean_PrettyPrinter_delab(x_32, x_34, x_7, x_8, x_9, x_10, x_33); +if (lean_obj_tag(x_35) == 0) +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; 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; +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +lean_inc(x_9); +x_38 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_37); +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = lean_st_ref_get(x_10, x_40); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_43 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +lean_inc(x_39); +x_44 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_44, 0, x_39); +lean_ctor_set(x_44, 1, x_43); +lean_inc(x_30); +x_45 = lean_mk_syntax_ident(x_30); +x_46 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +lean_inc(x_45); +x_47 = lean_array_push(x_46, x_45); +x_48 = lean_box(2); +x_49 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_50 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +lean_ctor_set(x_50, 2, x_47); +x_51 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; +lean_inc(x_39); +x_52 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_52, 0, x_39); +lean_ctor_set(x_52, 1, x_51); +x_53 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_54 = lean_array_push(x_53, x_52); +x_55 = lean_array_push(x_54, x_36); +x_56 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_56, 0, x_48); +lean_ctor_set(x_56, 1, x_49); +lean_ctor_set(x_56, 2, x_55); +x_57 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +x_58 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_58, 0, x_39); +lean_ctor_set(x_58, 1, x_57); +x_59 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; +x_60 = lean_array_push(x_59, x_44); +x_61 = lean_array_push(x_60, x_50); +x_62 = lean_array_push(x_61, x_56); +x_63 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_64 = lean_array_push(x_62, x_63); +x_65 = lean_array_push(x_64, x_58); +x_66 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1; +x_67 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_67, 0, x_48); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set(x_67, 2, x_65); +x_68 = lean_array_push(x_26, x_67); +x_69 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__2; +x_70 = lean_name_append_after(x_30, x_69); +x_71 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_70, x_9, x_10, x_42); +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = lean_mk_syntax_ident(x_72); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_75 = lean_infer_type(x_14, x_7, x_8, x_9, x_10, x_73); +if (lean_obj_tag(x_75) == 0) +{ +lean_object* x_76; lean_object* x_77; uint8_t x_78; +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_75, 1); +lean_inc(x_77); +lean_dec(x_75); +x_78 = l_Lean_Expr_isType(x_76); +lean_dec(x_76); +if (x_78 == 0) +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +lean_dec(x_74); +lean_dec(x_45); +x_79 = lean_box(0); +x_80 = l_Array_back___rarg(x_79, x_68); +x_81 = lean_array_push(x_25, x_80); +lean_ctor_set(x_4, 1, x_68); +lean_ctor_set(x_4, 0, x_81); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_23); +lean_ctor_set(x_82, 1, x_4); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_82); +x_15 = x_83; +x_16 = x_77; +goto block_21; +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; 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_inc(x_9); +x_84 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_77); +x_85 = lean_ctor_get(x_84, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_84, 1); +lean_inc(x_86); +lean_dec(x_84); +x_87 = lean_st_ref_get(x_10, x_86); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); +lean_inc(x_85); +x_89 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_89, 0, x_85); +lean_ctor_set(x_89, 1, x_43); +lean_inc(x_74); +x_90 = lean_array_push(x_46, x_74); +x_91 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_91, 0, x_48); +lean_ctor_set(x_91, 1, x_49); +lean_ctor_set(x_91, 2, x_90); +lean_inc(x_85); +x_92 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_92, 0, x_85); +lean_ctor_set(x_92, 1, x_51); +x_93 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__5; +lean_inc(x_85); +x_94 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_94, 0, x_85); +lean_ctor_set(x_94, 1, x_93); +x_95 = lean_array_push(x_53, x_94); +x_96 = lean_array_push(x_95, x_63); +x_97 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__4; +x_98 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_98, 0, x_48); +lean_ctor_set(x_98, 1, x_97); +lean_ctor_set(x_98, 2, x_96); +x_99 = lean_array_push(x_53, x_92); +x_100 = lean_array_push(x_99, x_98); +x_101 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_101, 0, x_48); +lean_ctor_set(x_101, 1, x_49); +lean_ctor_set(x_101, 2, x_100); +x_102 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_102, 0, x_85); +lean_ctor_set(x_102, 1, x_57); +x_103 = lean_array_push(x_59, x_89); +x_104 = lean_array_push(x_103, x_91); +x_105 = lean_array_push(x_104, x_101); +x_106 = lean_array_push(x_105, x_63); +x_107 = lean_array_push(x_106, x_102); +x_108 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_108, 0, x_48); +lean_ctor_set(x_108, 1, x_66); +lean_ctor_set(x_108, 2, x_107); +x_109 = lean_array_push(x_25, x_108); +lean_inc(x_9); +x_110 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_88); +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +lean_dec(x_110); +x_113 = lean_ctor_get(x_9, 10); +lean_inc(x_113); +x_114 = lean_st_ref_get(x_10, x_112); +x_115 = lean_ctor_get(x_114, 0); +lean_inc(x_115); +x_116 = lean_ctor_get(x_114, 1); +lean_inc(x_116); +lean_dec(x_114); +x_117 = lean_ctor_get(x_115, 0); +lean_inc(x_117); +lean_dec(x_115); +x_118 = lean_environment_main_module(x_117); +x_119 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3; +lean_inc(x_111); +x_120 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_120, 0, x_111); +lean_ctor_set(x_120, 1, x_119); +x_121 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; +x_122 = l_Lean_addMacroScope(x_118, x_121, x_113); +x_123 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; +x_124 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5; +lean_inc(x_111); +x_125 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_125, 0, x_111); +lean_ctor_set(x_125, 1, x_123); +lean_ctor_set(x_125, 2, x_122); +lean_ctor_set(x_125, 3, x_124); +x_126 = lean_array_push(x_53, x_45); +x_127 = lean_array_push(x_126, x_74); +x_128 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_128, 0, x_48); +lean_ctor_set(x_128, 1, x_49); +lean_ctor_set(x_128, 2, x_127); +x_129 = lean_array_push(x_53, x_125); +x_130 = lean_array_push(x_129, x_128); +x_131 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; +x_132 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_132, 0, x_48); +lean_ctor_set(x_132, 1, x_131); +lean_ctor_set(x_132, 2, x_130); +x_133 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; +x_134 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_134, 0, x_111); +lean_ctor_set(x_134, 1, x_133); +x_135 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_136 = lean_array_push(x_135, x_120); +x_137 = lean_array_push(x_136, x_63); +x_138 = lean_array_push(x_137, x_132); +x_139 = lean_array_push(x_138, x_134); +x_140 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__2; +x_141 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_141, 0, x_48); +lean_ctor_set(x_141, 1, x_140); +lean_ctor_set(x_141, 2, x_139); +x_142 = lean_array_push(x_23, x_141); +lean_ctor_set(x_4, 1, x_68); +lean_ctor_set(x_4, 0, x_109); +x_143 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_143, 0, x_142); +lean_ctor_set(x_143, 1, x_4); +x_144 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_144, 0, x_143); +x_15 = x_144; +x_16 = x_116; +goto block_21; +} +} +else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_16 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_13, x_14, x_15); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_st_ref_get(x_14, x_18); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +uint8_t x_145; +lean_dec(x_74); +lean_dec(x_68); +lean_dec(x_45); +lean_dec(x_25); +lean_free_object(x_4); +lean_dec(x_23); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_145 = !lean_is_exclusive(x_75); +if (x_145 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; 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; -x_21 = lean_ctor_get(x_19, 0); -lean_dec(x_21); -x_22 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__57; -lean_inc(x_1); -x_23 = l_Lean_Name_str___override(x_1, x_22); -x_24 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; -lean_inc(x_17); -x_25 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_25, 0, x_17); -lean_ctor_set(x_25, 1, x_24); -x_26 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; -lean_inc(x_1); -x_27 = l_Lean_Name_str___override(x_1, x_26); -x_28 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__73; -x_29 = l_Lean_Name_str___override(x_2, x_28); -x_30 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207; -x_31 = l_Lean_Name_str___override(x_29, x_30); -x_32 = lean_mk_syntax_ident(x_31); -x_33 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__1; -x_34 = l_Lean_Name_str___override(x_1, x_33); -x_35 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__2; -lean_inc(x_17); -x_36 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_36, 0, x_17); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_array_push(x_3, x_36); -x_38 = lean_box(2); -x_39 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_34); -lean_ctor_set(x_39, 2, x_37); -x_40 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_41 = lean_array_push(x_40, x_4); -x_42 = lean_array_push(x_41, x_39); -x_43 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_43, 0, x_38); -lean_ctor_set(x_43, 1, x_5); -lean_ctor_set(x_43, 2, x_42); -x_44 = lean_array_push(x_40, x_32); -x_45 = lean_array_push(x_44, x_43); -x_46 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_46, 0, x_38); -lean_ctor_set(x_46, 1, x_27); -lean_ctor_set(x_46, 2, x_45); -x_47 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; -x_48 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_48, 0, x_17); -lean_ctor_set(x_48, 1, x_47); -x_49 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_50 = lean_array_push(x_49, x_25); -x_51 = lean_array_push(x_50, x_6); -x_52 = lean_array_push(x_51, x_46); -x_53 = lean_array_push(x_52, x_48); -x_54 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_54, 0, x_38); -lean_ctor_set(x_54, 1, x_23); -lean_ctor_set(x_54, 2, x_53); -x_55 = lean_array_push(x_7, x_54); -x_56 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_19, 0, x_56); -return x_19; +return x_75; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_57 = lean_ctor_get(x_19, 1); -lean_inc(x_57); -lean_dec(x_19); -x_58 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__57; -lean_inc(x_1); -x_59 = l_Lean_Name_str___override(x_1, x_58); -x_60 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__59; -lean_inc(x_17); -x_61 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_61, 0, x_17); -lean_ctor_set(x_61, 1, x_60); -x_62 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; -lean_inc(x_1); -x_63 = l_Lean_Name_str___override(x_1, x_62); -x_64 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__73; -x_65 = l_Lean_Name_str___override(x_2, x_64); -x_66 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207; -x_67 = l_Lean_Name_str___override(x_65, x_66); -x_68 = lean_mk_syntax_ident(x_67); -x_69 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__1; -x_70 = l_Lean_Name_str___override(x_1, x_69); -x_71 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__2; -lean_inc(x_17); -x_72 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_72, 0, x_17); -lean_ctor_set(x_72, 1, x_71); -x_73 = lean_array_push(x_3, x_72); -x_74 = lean_box(2); -x_75 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_75, 0, x_74); -lean_ctor_set(x_75, 1, x_70); -lean_ctor_set(x_75, 2, x_73); -x_76 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_77 = lean_array_push(x_76, x_4); -x_78 = lean_array_push(x_77, x_75); -x_79 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_79, 0, x_74); -lean_ctor_set(x_79, 1, x_5); -lean_ctor_set(x_79, 2, x_78); -x_80 = lean_array_push(x_76, x_68); -x_81 = lean_array_push(x_80, x_79); -x_82 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_82, 0, x_74); -lean_ctor_set(x_82, 1, x_63); -lean_ctor_set(x_82, 2, x_81); -x_83 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__68; -x_84 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_84, 0, x_17); -lean_ctor_set(x_84, 1, x_83); -x_85 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_86 = lean_array_push(x_85, x_61); -x_87 = lean_array_push(x_86, x_6); -x_88 = lean_array_push(x_87, x_82); -x_89 = lean_array_push(x_88, x_84); -x_90 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_90, 0, x_74); -lean_ctor_set(x_90, 1, x_59); -lean_ctor_set(x_90, 2, x_89); -x_91 = lean_array_push(x_7, x_90); -x_92 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_92, 0, x_91); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_57); -return x_93; +lean_object* x_146; lean_object* x_147; lean_object* x_148; +x_146 = lean_ctor_get(x_75, 0); +x_147 = lean_ctor_get(x_75, 1); +lean_inc(x_147); +lean_inc(x_146); +lean_dec(x_75); +x_148 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_148, 0, x_146); +lean_ctor_set(x_148, 1, x_147); +return x_148; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; -x_12 = lean_usize_dec_lt(x_3, x_2); -if (x_12 == 0) +else { -lean_object* x_13; +uint8_t x_149; +lean_dec(x_30); +lean_dec(x_26); +lean_dec(x_25); +lean_free_object(x_4); +lean_dec(x_23); +lean_dec(x_14); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_4); -lean_ctor_set(x_13, 1, x_11); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_22; -x_14 = lean_array_uget(x_1, x_3); -lean_inc(x_7); -lean_inc(x_14); -x_22 = l_Lean_Meta_getFVarLocalDecl(x_14, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_22) == 0) +x_149 = !lean_is_exclusive(x_35); +if (x_149 == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = l_Lean_LocalDecl_userName(x_23); -lean_dec(x_23); -lean_inc(x_9); -x_26 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, 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); -lean_dec(x_26); -x_29 = lean_st_ref_get(x_10, x_28); -x_30 = lean_ctor_get(x_29, 1); -lean_inc(x_30); -lean_dec(x_29); -x_31 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__80; -lean_inc(x_27); -x_32 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_32, 0, x_27); -lean_ctor_set(x_32, 1, x_31); -x_33 = lean_mk_syntax_ident(x_25); -x_34 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__25; -lean_inc(x_33); -x_35 = lean_array_push(x_34, x_33); -x_36 = lean_box(2); -x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -x_39 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__92; -x_40 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_40, 0, x_27); -lean_ctor_set(x_40, 1, x_39); -x_41 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__93; -x_42 = lean_array_push(x_41, x_32); -x_43 = lean_array_push(x_42, x_38); -x_44 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__12; -x_45 = lean_array_push(x_43, x_44); -x_46 = lean_array_push(x_45, x_44); -x_47 = lean_array_push(x_46, x_40); -x_48 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__79; -x_49 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_49, 0, x_36); -lean_ctor_set(x_49, 1, x_48); -lean_ctor_set(x_49, 2, x_47); -x_50 = lean_array_push(x_4, x_49); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_51 = lean_infer_type(x_14, x_7, x_8, x_9, x_10, x_30); -if (lean_obj_tag(x_51) == 0) -{ -lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -x_54 = l_Lean_Expr_isType(x_52); -lean_dec(x_52); -if (x_54 == 0) -{ -lean_object* x_55; -lean_dec(x_33); -x_55 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_55, 0, x_50); -x_15 = x_55; -x_16 = x_53; -goto block_21; +return x_35; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_56 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; -x_57 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__4; -x_58 = lean_box(0); -lean_inc(x_9); -x_59 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1(x_56, x_57, x_34, x_33, x_37, x_44, x_50, x_58, x_5, x_6, x_7, x_8, x_9, x_10, x_53); -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); -lean_dec(x_59); -x_15 = x_60; -x_16 = x_61; -goto block_21; +lean_object* x_150; lean_object* x_151; lean_object* x_152; +x_150 = lean_ctor_get(x_35, 0); +x_151 = lean_ctor_get(x_35, 1); +lean_inc(x_151); +lean_inc(x_150); +lean_dec(x_35); +x_152 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_152, 0, x_150); +lean_ctor_set(x_152, 1, x_151); +return x_152; +} } } else { -uint8_t x_62; -lean_dec(x_50); -lean_dec(x_33); +uint8_t x_153; +lean_dec(x_30); +lean_dec(x_26); +lean_dec(x_25); +lean_free_object(x_4); +lean_dec(x_23); +lean_dec(x_14); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -x_62 = !lean_is_exclusive(x_51); -if (x_62 == 0) +x_153 = !lean_is_exclusive(x_31); +if (x_153 == 0) { -return x_51; +return x_31; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_51, 0); -x_64 = lean_ctor_get(x_51, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_51); -x_65 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -return x_65; +lean_object* x_154; lean_object* x_155; lean_object* x_156; +x_154 = lean_ctor_get(x_31, 0); +x_155 = lean_ctor_get(x_31, 1); +lean_inc(x_155); +lean_inc(x_154); +lean_dec(x_31); +x_156 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_156, 0, x_154); +lean_ctor_set(x_156, 1, x_155); +return x_156; } } } else { -uint8_t x_66; +uint8_t x_157; +lean_dec(x_26); +lean_dec(x_25); +lean_free_object(x_4); +lean_dec(x_23); lean_dec(x_14); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_4); -x_66 = !lean_is_exclusive(x_22); -if (x_66 == 0) +x_157 = !lean_is_exclusive(x_27); +if (x_157 == 0) { -return x_22; +return x_27; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_22, 0); -x_68 = lean_ctor_get(x_22, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_22); -x_69 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -return x_69; -} -} -block_21: -{ -lean_object* x_17; size_t x_18; size_t x_19; -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -lean_dec(x_15); -x_18 = 1; -x_19 = lean_usize_add(x_3, x_18); -x_3 = x_19; -x_4 = x_17; -x_11 = x_16; -goto _start; -} -} +lean_object* x_158; lean_object* x_159; lean_object* x_160; +x_158 = lean_ctor_get(x_27, 0); +x_159 = lean_ctor_get(x_27, 1); +lean_inc(x_159); +lean_inc(x_158); +lean_dec(x_27); +x_160 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_160, 0, x_158); +lean_ctor_set(x_160, 1, x_159); +return x_160; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__5(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -uint8_t x_8; -x_8 = lean_usize_dec_lt(x_3, x_2); -if (x_8 == 0) -{ -lean_object* x_9; -lean_dec(x_6); -lean_dec(x_5); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_4); -lean_ctor_set(x_9, 1, x_7); -return x_9; } else { -lean_object* x_10; lean_object* x_11; +lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_161 = lean_ctor_get(x_4, 0); +x_162 = lean_ctor_get(x_4, 1); +lean_inc(x_162); +lean_inc(x_161); lean_dec(x_4); -x_10 = lean_array_uget(x_1, x_3); -lean_inc(x_6); -lean_inc(x_5); -x_11 = l_Lean_Elab_Command_elabCommand(x_10, x_5, x_6, x_7); -if (lean_obj_tag(x_11) == 0) +x_163 = lean_ctor_get(x_162, 0); +lean_inc(x_163); +x_164 = lean_ctor_get(x_162, 1); +lean_inc(x_164); +lean_dec(x_162); +lean_inc(x_7); +lean_inc(x_14); +x_165 = l_Lean_Meta_getFVarLocalDecl(x_14, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_165) == 0) { -lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = 1; -x_14 = lean_usize_add(x_3, x_13); -x_15 = lean_box(0); -x_3 = x_14; -x_4 = x_15; -x_7 = x_12; -goto _start; +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_166 = lean_ctor_get(x_165, 0); +lean_inc(x_166); +x_167 = lean_ctor_get(x_165, 1); +lean_inc(x_167); +lean_dec(x_165); +x_168 = l_Lean_LocalDecl_userName(x_166); +lean_dec(x_166); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_14); +x_169 = lean_infer_type(x_14, x_7, x_8, x_9, x_10, x_167); +if (lean_obj_tag(x_169) == 0) +{ +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_170 = lean_ctor_get(x_169, 0); +lean_inc(x_170); +x_171 = lean_ctor_get(x_169, 1); +lean_inc(x_171); +lean_dec(x_169); +x_172 = lean_box(0); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_173 = l_Lean_PrettyPrinter_delab(x_170, x_172, x_7, x_8, x_9, x_10, x_171); +if (lean_obj_tag(x_173) == 0) +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; +x_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_173, 1); +lean_inc(x_175); +lean_dec(x_173); +lean_inc(x_9); +x_176 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_175); +x_177 = lean_ctor_get(x_176, 0); +lean_inc(x_177); +x_178 = lean_ctor_get(x_176, 1); +lean_inc(x_178); +lean_dec(x_176); +x_179 = lean_st_ref_get(x_10, x_178); +x_180 = lean_ctor_get(x_179, 1); +lean_inc(x_180); +lean_dec(x_179); +x_181 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__52; +lean_inc(x_177); +x_182 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_182, 0, x_177); +lean_ctor_set(x_182, 1, x_181); +lean_inc(x_168); +x_183 = lean_mk_syntax_ident(x_168); +x_184 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__17; +lean_inc(x_183); +x_185 = lean_array_push(x_184, x_183); +x_186 = lean_box(2); +x_187 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; +x_188 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_188, 0, x_186); +lean_ctor_set(x_188, 1, x_187); +lean_ctor_set(x_188, 2, x_185); +x_189 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__38; +lean_inc(x_177); +x_190 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_190, 0, x_177); +lean_ctor_set(x_190, 1, x_189); +x_191 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__31; +x_192 = lean_array_push(x_191, x_190); +x_193 = lean_array_push(x_192, x_174); +x_194 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_194, 0, x_186); +lean_ctor_set(x_194, 1, x_187); +lean_ctor_set(x_194, 2, x_193); +x_195 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__60; +x_196 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_196, 0, x_177); +lean_ctor_set(x_196, 1, x_195); +x_197 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__99; +x_198 = lean_array_push(x_197, x_182); +x_199 = lean_array_push(x_198, x_188); +x_200 = lean_array_push(x_199, x_194); +x_201 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; +x_202 = lean_array_push(x_200, x_201); +x_203 = lean_array_push(x_202, x_196); +x_204 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1; +x_205 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_205, 0, x_186); +lean_ctor_set(x_205, 1, x_204); +lean_ctor_set(x_205, 2, x_203); +x_206 = lean_array_push(x_164, x_205); +x_207 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__2; +x_208 = lean_name_append_after(x_168, x_207); +x_209 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_208, x_9, x_10, x_180); +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = lean_mk_syntax_ident(x_210); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_213 = lean_infer_type(x_14, x_7, x_8, x_9, x_10, x_211); +if (lean_obj_tag(x_213) == 0) +{ +lean_object* x_214; lean_object* x_215; uint8_t x_216; +x_214 = lean_ctor_get(x_213, 0); +lean_inc(x_214); +x_215 = lean_ctor_get(x_213, 1); +lean_inc(x_215); +lean_dec(x_213); +x_216 = l_Lean_Expr_isType(x_214); +lean_dec(x_214); +if (x_216 == 0) +{ +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; +lean_dec(x_212); +lean_dec(x_183); +x_217 = lean_box(0); +x_218 = l_Array_back___rarg(x_217, x_206); +x_219 = lean_array_push(x_163, x_218); +x_220 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_220, 0, x_219); +lean_ctor_set(x_220, 1, x_206); +x_221 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_221, 0, x_161); +lean_ctor_set(x_221, 1, x_220); +x_222 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_222, 0, x_221); +x_15 = x_222; +x_16 = x_215; +goto block_21; } else { -uint8_t x_17; -lean_dec(x_6); -lean_dec(x_5); -x_17 = !lean_is_exclusive(x_11); -if (x_17 == 0) -{ -return x_11; +lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; +lean_inc(x_9); +x_223 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_215); +x_224 = lean_ctor_get(x_223, 0); +lean_inc(x_224); +x_225 = lean_ctor_get(x_223, 1); +lean_inc(x_225); +lean_dec(x_223); +x_226 = lean_st_ref_get(x_10, x_225); +x_227 = lean_ctor_get(x_226, 1); +lean_inc(x_227); +lean_dec(x_226); +lean_inc(x_224); +x_228 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_228, 0, x_224); +lean_ctor_set(x_228, 1, x_181); +lean_inc(x_212); +x_229 = lean_array_push(x_184, x_212); +x_230 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_230, 0, x_186); +lean_ctor_set(x_230, 1, x_187); +lean_ctor_set(x_230, 2, x_229); +lean_inc(x_224); +x_231 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_231, 0, x_224); +lean_ctor_set(x_231, 1, x_189); +x_232 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__5; +lean_inc(x_224); +x_233 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_233, 0, x_224); +lean_ctor_set(x_233, 1, x_232); +x_234 = lean_array_push(x_191, x_233); +x_235 = lean_array_push(x_234, x_201); +x_236 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__4; +x_237 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_237, 0, x_186); +lean_ctor_set(x_237, 1, x_236); +lean_ctor_set(x_237, 2, x_235); +x_238 = lean_array_push(x_191, x_231); +x_239 = lean_array_push(x_238, x_237); +x_240 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_240, 0, x_186); +lean_ctor_set(x_240, 1, x_187); +lean_ctor_set(x_240, 2, x_239); +x_241 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_241, 0, x_224); +lean_ctor_set(x_241, 1, x_195); +x_242 = lean_array_push(x_197, x_228); +x_243 = lean_array_push(x_242, x_230); +x_244 = lean_array_push(x_243, x_240); +x_245 = lean_array_push(x_244, x_201); +x_246 = lean_array_push(x_245, x_241); +x_247 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_247, 0, x_186); +lean_ctor_set(x_247, 1, x_204); +lean_ctor_set(x_247, 2, x_246); +x_248 = lean_array_push(x_163, x_247); +lean_inc(x_9); +x_249 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_227); +x_250 = lean_ctor_get(x_249, 0); +lean_inc(x_250); +x_251 = lean_ctor_get(x_249, 1); +lean_inc(x_251); +lean_dec(x_249); +x_252 = lean_ctor_get(x_9, 10); +lean_inc(x_252); +x_253 = lean_st_ref_get(x_10, x_251); +x_254 = lean_ctor_get(x_253, 0); +lean_inc(x_254); +x_255 = lean_ctor_get(x_253, 1); +lean_inc(x_255); +lean_dec(x_253); +x_256 = lean_ctor_get(x_254, 0); +lean_inc(x_256); +lean_dec(x_254); +x_257 = lean_environment_main_module(x_256); +x_258 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3; +lean_inc(x_250); +x_259 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_259, 0, x_250); +lean_ctor_set(x_259, 1, x_258); +x_260 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__44; +x_261 = l_Lean_addMacroScope(x_257, x_260, x_252); +x_262 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__43; +x_263 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5; +lean_inc(x_250); +x_264 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_264, 0, x_250); +lean_ctor_set(x_264, 1, x_262); +lean_ctor_set(x_264, 2, x_261); +lean_ctor_set(x_264, 3, x_263); +x_265 = lean_array_push(x_191, x_183); +x_266 = lean_array_push(x_265, x_212); +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_186); +lean_ctor_set(x_267, 1, x_187); +lean_ctor_set(x_267, 2, x_266); +x_268 = lean_array_push(x_191, x_264); +x_269 = lean_array_push(x_268, x_267); +x_270 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__40; +x_271 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_271, 0, x_186); +lean_ctor_set(x_271, 1, x_270); +lean_ctor_set(x_271, 2, x_269); +x_272 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__135; +x_273 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_273, 0, x_250); +lean_ctor_set(x_273, 1, x_272); +x_274 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__115; +x_275 = lean_array_push(x_274, x_259); +x_276 = lean_array_push(x_275, x_201); +x_277 = lean_array_push(x_276, x_271); +x_278 = lean_array_push(x_277, x_273); +x_279 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__2; +x_280 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_280, 0, x_186); +lean_ctor_set(x_280, 1, x_279); +lean_ctor_set(x_280, 2, x_278); +x_281 = lean_array_push(x_161, x_280); +x_282 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_282, 0, x_248); +lean_ctor_set(x_282, 1, x_206); +x_283 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_283, 0, x_281); +lean_ctor_set(x_283, 1, x_282); +x_284 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_284, 0, x_283); +x_15 = x_284; +x_16 = x_255; +goto block_21; +} } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_11, 0); -x_19 = lean_ctor_get(x_11, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_11); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; +lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; +lean_dec(x_212); +lean_dec(x_206); +lean_dec(x_183); +lean_dec(x_163); +lean_dec(x_161); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_285 = lean_ctor_get(x_213, 0); +lean_inc(x_285); +x_286 = lean_ctor_get(x_213, 1); +lean_inc(x_286); +if (lean_is_exclusive(x_213)) { + lean_ctor_release(x_213, 0); + lean_ctor_release(x_213, 1); + x_287 = x_213; +} else { + lean_dec_ref(x_213); + x_287 = lean_box(0); +} +if (lean_is_scalar(x_287)) { + x_288 = lean_alloc_ctor(1, 2, 0); +} else { + x_288 = x_287; +} +lean_ctor_set(x_288, 0, x_285); +lean_ctor_set(x_288, 1, x_286); +return x_288; +} } +else +{ +lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; +lean_dec(x_168); +lean_dec(x_164); +lean_dec(x_163); +lean_dec(x_161); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_289 = lean_ctor_get(x_173, 0); +lean_inc(x_289); +x_290 = lean_ctor_get(x_173, 1); +lean_inc(x_290); +if (lean_is_exclusive(x_173)) { + lean_ctor_release(x_173, 0); + lean_ctor_release(x_173, 1); + x_291 = x_173; +} else { + lean_dec_ref(x_173); + x_291 = lean_box(0); } +if (lean_is_scalar(x_291)) { + x_292 = lean_alloc_ctor(1, 2, 0); +} else { + x_292 = x_291; } +lean_ctor_set(x_292, 0, x_289); +lean_ctor_set(x_292, 1, x_290); +return x_292; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("assertion violation: ", 21); -return x_1; +lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; +lean_dec(x_168); +lean_dec(x_164); +lean_dec(x_163); +lean_dec(x_161); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_293 = lean_ctor_get(x_169, 0); +lean_inc(x_293); +x_294 = lean_ctor_get(x_169, 1); +lean_inc(x_294); +if (lean_is_exclusive(x_169)) { + lean_ctor_release(x_169, 0); + lean_ctor_release(x_169, 1); + x_295 = x_169; +} else { + lean_dec_ref(x_169); + x_295 = lean_box(0); } +if (lean_is_scalar(x_295)) { + x_296 = lean_alloc_ctor(1, 2, 0); +} else { + x_296 = x_295; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("params.size == indVal.numParams\n\n -- bind every parameter and *some* (not named) `RpcEncoding` for it\n ", 113); -return x_1; +lean_ctor_set(x_296, 0, x_293); +lean_ctor_set(x_296, 1, x_294); +return x_296; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__3() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__1; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__2; -x_3 = lean_string_append(x_1, x_2); -return x_3; +lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; +lean_dec(x_164); +lean_dec(x_163); +lean_dec(x_161); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +x_297 = lean_ctor_get(x_165, 0); +lean_inc(x_297); +x_298 = lean_ctor_get(x_165, 1); +lean_inc(x_298); +if (lean_is_exclusive(x_165)) { + lean_ctor_release(x_165, 0); + lean_ctor_release(x_165, 1); + x_299 = x_165; +} else { + lean_dec_ref(x_165); + x_299 = lean_box(0); } +if (lean_is_scalar(x_299)) { + x_300 = lean_alloc_ctor(1, 2, 0); +} else { + x_300 = x_299; } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("Lean.Server.Rpc.Deriving", 24); -return x_1; +lean_ctor_set(x_300, 0, x_297); +lean_ctor_set(x_300, 1, x_298); +return x_300; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__5() { -_start: +block_21: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("_private.Lean.Server.Rpc.Deriving.0.Lean.Server.RpcEncoding.deriveInstance", 74); -return x_1; +lean_object* x_17; size_t x_18; size_t x_19; +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +x_18 = 1; +x_19 = lean_usize_add(x_3, x_18); +x_3 = x_19; +x_4 = x_17; +x_11 = x_16; +goto _start; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__4; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(261u); -x_4 = lean_unsigned_to_nat(6u); -x_5 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__3; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_12; lean_object* x_13; uint8_t x_14; -lean_dec(x_4); -x_12 = lean_array_get_size(x_3); -x_13 = lean_ctor_get(x_1, 1); -lean_inc(x_13); -x_14 = lean_nat_dec_eq(x_12, x_13); -lean_dec(x_13); -if (x_14 == 0) +lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_array_get_size(x_1); +x_11 = lean_usize_of_nat(x_10); +lean_dec(x_10); +x_12 = 0; +x_13 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__2; +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3(x_1, x_11, x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_15; lean_object* x_16; -lean_dec(x_12); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__6; -x_16 = l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3(x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_16; +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_14, 0); +lean_dec(x_18); +x_19 = lean_ctor_get(x_15, 0); +lean_inc(x_19); +lean_dec(x_15); +x_20 = lean_ctor_get(x_16, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_16, 1); +lean_inc(x_21); +lean_dec(x_16); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_19); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_14, 0, x_23); +return x_14; } else { -size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; -x_17 = lean_usize_of_nat(x_12); -lean_dec(x_12); -x_18 = 0; -x_19 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__11; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_20 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4(x_3, x_17, x_18, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; 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; uint8_t x_55; lean_object* x_56; lean_object* x_57; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -lean_inc(x_9); -x_23 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_22); -x_24 = lean_ctor_get(x_23, 0); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_14, 1); lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); +lean_dec(x_14); +x_25 = lean_ctor_get(x_15, 0); lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_st_ref_get(x_10, x_25); -x_27 = lean_ctor_get(x_26, 1); +lean_dec(x_15); +x_26 = lean_ctor_get(x_16, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_16, 1); lean_inc(x_27); -lean_dec(x_26); -x_28 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__9; -x_29 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_29, 0, x_24); +lean_dec(x_16); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_25); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); -x_30 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__13; -x_31 = lean_array_push(x_30, x_29); -x_32 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__16; -x_33 = lean_array_push(x_31, x_32); -x_34 = lean_box(2); -x_35 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__10; -x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -lean_ctor_set(x_36, 2, x_33); -lean_inc(x_9); -x_37 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_27); -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_37, 1); -lean_inc(x_39); -lean_dec(x_37); -x_40 = lean_st_ref_get(x_10, x_39); -x_41 = lean_ctor_get(x_40, 1); -lean_inc(x_41); -lean_dec(x_40); -x_42 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__14; -x_43 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_43, 0, x_38); -lean_ctor_set(x_43, 1, x_42); -x_44 = l_Array_append___rarg(x_19, x_21); -x_45 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__2; -x_46 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_46, 0, x_34); -lean_ctor_set(x_46, 1, x_45); -lean_ctor_set(x_46, 2, x_44); -x_47 = lean_array_push(x_30, x_43); -x_48 = lean_array_push(x_47, x_46); -x_49 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__15; -x_50 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_50, 0, x_34); -lean_ctor_set(x_50, 1, x_49); -lean_ctor_set(x_50, 2, x_48); -x_51 = lean_st_ref_get(x_10, x_41); -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -x_54 = lean_ctor_get(x_52, 0); -lean_inc(x_54); -lean_dec(x_52); -x_55 = l_Lean_isStructure(x_54, x_2); -if (x_55 == 0) -{ -lean_object* x_89; -lean_inc(x_10); -lean_inc(x_9); -x_89 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance(x_1, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_53); -if (lean_obj_tag(x_89) == 0) -{ -lean_object* x_90; lean_object* x_91; -x_90 = lean_ctor_get(x_89, 0); -lean_inc(x_90); -x_91 = lean_ctor_get(x_89, 1); -lean_inc(x_91); -lean_dec(x_89); -x_56 = x_90; -x_57 = x_91; -goto block_88; -} -else -{ -uint8_t x_92; -lean_dec(x_50); -lean_dec(x_36); -lean_dec(x_10); -lean_dec(x_9); -x_92 = !lean_is_exclusive(x_89); -if (x_92 == 0) -{ -return x_89; -} -else -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_89, 0); -x_94 = lean_ctor_get(x_89, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_89); -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -return x_95; -} +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_24); +return x_30; } } else { -lean_object* x_96; -lean_inc(x_10); -lean_inc(x_9); -x_96 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance(x_1, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_53); -if (lean_obj_tag(x_96) == 0) +uint8_t x_31; +x_31 = !lean_is_exclusive(x_14); +if (x_31 == 0) { -lean_object* x_97; lean_object* x_98; -x_97 = lean_ctor_get(x_96, 0); -lean_inc(x_97); -x_98 = lean_ctor_get(x_96, 1); -lean_inc(x_98); -lean_dec(x_96); -x_56 = x_97; -x_57 = x_98; -goto block_88; +return x_14; } else { -uint8_t x_99; -lean_dec(x_50); -lean_dec(x_36); -lean_dec(x_10); -lean_dec(x_9); -x_99 = !lean_is_exclusive(x_96); -if (x_99 == 0) -{ -return x_96; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_14, 0); +x_33 = lean_ctor_get(x_14, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_14); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } -else -{ -lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_100 = lean_ctor_get(x_96, 0); -x_101 = lean_ctor_get(x_96, 1); -lean_inc(x_101); -lean_inc(x_100); -lean_dec(x_96); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_100); -lean_ctor_set(x_102, 1, x_101); -return x_102; } } } -block_88: +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_58 = l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(x_9, x_10, x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -lean_dec(x_58); -x_61 = lean_st_ref_get(x_10, x_60); -lean_dec(x_10); -x_62 = !lean_is_exclusive(x_61); -if (x_62 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_14 = lean_array_get_size(x_1); +x_15 = lean_unsigned_to_nat(0u); +x_16 = l_Array_toSubarray___rarg(x_6, x_15, x_14); +x_17 = lean_st_ref_get(x_12, x_13); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_ctor_get(x_18, 0); +lean_inc(x_20); +lean_dec(x_18); +x_21 = l_Lean_isStructure(x_20, x_2); +if (x_21 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_63 = lean_ctor_get(x_61, 0); -lean_dec(x_63); -x_64 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241; -x_65 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_65, 0, x_59); -lean_ctor_set(x_65, 1, x_64); -x_66 = lean_array_push(x_30, x_65); -x_67 = lean_array_push(x_66, x_32); -x_68 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__242; -x_69 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_69, 0, x_34); -lean_ctor_set(x_69, 1, x_68); -lean_ctor_set(x_69, 2, x_67); -x_70 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_71 = lean_array_push(x_70, x_36); -x_72 = lean_array_push(x_71, x_50); -x_73 = lean_array_push(x_72, x_56); -x_74 = lean_array_push(x_73, x_69); -lean_ctor_set(x_61, 0, x_74); -return x_61; +lean_object* x_22; lean_object* x_23; +x_22 = l_Array_ofSubarray___rarg(x_16); +x_23 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance(x_3, x_22, x_1, x_4, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_19); +return x_23; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_75 = lean_ctor_get(x_61, 1); -lean_inc(x_75); -lean_dec(x_61); -x_76 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241; -x_77 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_77, 0, x_59); -lean_ctor_set(x_77, 1, x_76); -x_78 = lean_array_push(x_30, x_77); -x_79 = lean_array_push(x_78, x_32); -x_80 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__242; -x_81 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_81, 0, x_34); -lean_ctor_set(x_81, 1, x_80); -lean_ctor_set(x_81, 2, x_79); -x_82 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__35; -x_83 = lean_array_push(x_82, x_36); -x_84 = lean_array_push(x_83, x_50); -x_85 = lean_array_push(x_84, x_56); -x_86 = lean_array_push(x_85, x_81); -x_87 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_75); -return x_87; -} +lean_object* x_24; lean_object* x_25; +x_24 = l_Array_ofSubarray___rarg(x_16); +x_25 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance(x_3, x_24, x_1, x_4, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_19); +return x_25; } } -else -{ -uint8_t x_103; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_103 = !lean_is_exclusive(x_20); -if (x_103 == 0) -{ -return x_20; } -else +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__1() { +_start: { -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_20, 0); -x_105 = lean_ctor_get(x_20, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_20); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_104); -lean_ctor_set(x_106, 1, x_105); -return x_106; -} -} -} +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___boxed), 9, 0); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; @@ -20510,9 +14048,7 @@ lean_inc(x_8); x_9 = lean_ctor_get(x_8, 2); lean_inc(x_9); lean_dec(x_8); -x_10 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1), 11, 2); -lean_closure_set(x_10, 0, x_1); -lean_closure_set(x_10, 1, x_2); +x_10 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__1; x_11 = lean_alloc_closure((void*)(l_Lean_Meta_forallTelescopeReducing___at_Lean_Elab_Deriving_mkInductArgNames___spec__2___rarg), 9, 2); lean_closure_set(x_11, 0, x_9); lean_closure_set(x_11, 1, x_10); @@ -20520,97 +14056,152 @@ lean_inc(x_4); x_12 = l_Lean_Elab_Command_liftTermElabM___rarg(x_7, x_11, x_4, x_5, x_6); if (lean_obj_tag(x_12) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_array_get_size(x_13); -x_16 = lean_usize_of_nat(x_15); -lean_dec(x_15); -x_17 = 0; -x_18 = lean_box(0); -x_19 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__5(x_13, x_16, x_17, x_18, x_4, x_5, x_14); -lean_dec(x_13); -if (lean_obj_tag(x_19) == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_dec(x_12); +x_16 = lean_ctor_get(x_13, 0); +lean_inc(x_16); +lean_dec(x_13); +x_17 = lean_ctor_get(x_14, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +lean_inc(x_17); +lean_inc(x_16); +x_19 = l_Array_append___rarg(x_16, x_17); +lean_inc(x_18); +x_20 = l_Array_append___rarg(x_19, x_18); +x_21 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2), 13, 5); +lean_closure_set(x_21, 0, x_16); +lean_closure_set(x_21, 1, x_2); +lean_closure_set(x_21, 2, x_1); +lean_closure_set(x_21, 3, x_17); +lean_closure_set(x_21, 4, x_18); +x_22 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabBinders___rarg), 9, 2); +lean_closure_set(x_22, 0, x_20); +lean_closure_set(x_22, 1, x_21); +lean_inc(x_4); +x_23 = l_Lean_Elab_Command_liftTermElabM___rarg(x_7, x_22, x_4, x_5, x_15); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l_Lean_Elab_Command_elabCommand(x_24, x_4, x_5, x_25); +if (lean_obj_tag(x_26) == 0) +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) +{ +lean_object* x_28; uint8_t x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_26, 0); +lean_dec(x_28); +x_29 = 1; +x_30 = lean_box(x_29); +lean_ctor_set(x_26, 0, x_30); +return x_26; +} +else +{ +lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_26, 1); +lean_inc(x_31); +lean_dec(x_26); +x_32 = 1; +x_33 = lean_box(x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_31); +return x_34; +} +} +else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +uint8_t x_35; +x_35 = !lean_is_exclusive(x_26); +if (x_35 == 0) { -lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_19, 0); -lean_dec(x_21); -x_22 = 1; -x_23 = lean_box(x_22); -lean_ctor_set(x_19, 0, x_23); -return x_19; +return x_26; } else { -lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_19, 1); -lean_inc(x_24); -lean_dec(x_19); -x_25 = 1; -x_26 = lean_box(x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_26, 0); +x_37 = lean_ctor_get(x_26, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_26); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} } } else { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_19); -if (x_28 == 0) +uint8_t x_39; +lean_dec(x_5); +lean_dec(x_4); +x_39 = !lean_is_exclusive(x_23); +if (x_39 == 0) { -return x_19; +return x_23; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_19, 0); -x_30 = lean_ctor_get(x_19, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_19); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_23, 0); +x_41 = lean_ctor_get(x_23, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_23); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; } } } else { -uint8_t x_32; +uint8_t x_43; lean_dec(x_5); lean_dec(x_4); -x_32 = !lean_is_exclusive(x_12); -if (x_32 == 0) +lean_dec(x_2); +lean_dec(x_1); +x_43 = !lean_is_exclusive(x_12); +if (x_43 == 0) { return x_12; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_12, 0); -x_34 = lean_ctor_get(x_12, 1); -lean_inc(x_34); -lean_inc(x_33); +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_12, 0); +x_45 = lean_ctor_get(x_12, 1); +lean_inc(x_45); +lean_inc(x_44); lean_dec(x_12); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } } } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__1() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -20618,16 +14209,16 @@ x_1 = lean_mk_string_from_bytes("indexed inductive families are not supported", return x_1; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__2() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__1; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; uint8_t x_9; uint8_t x_10; @@ -20642,7 +14233,7 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; x_11 = lean_box(0); -x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2(x_1, x_2, x_11, x_4, x_5, x_6); +x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3(x_1, x_2, x_11, x_4, x_5, x_6); return x_12; } else @@ -20650,7 +14241,7 @@ else lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_dec(x_2); lean_dec(x_1); -x_13 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__2; +x_13 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__2; x_14 = l_Lean_throwError___at_Lean_Elab_Command_expandDeclId___spec__4(x_13, x_4, x_5, x_6); lean_dec(x_5); x_15 = !lean_is_exclusive(x_14); @@ -20719,7 +14310,7 @@ if (x_13 == 0) { lean_object* x_14; lean_object* x_15; x_14 = lean_box(0); -x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3(x_6, x_1, x_14, x_2, x_3, x_7); +x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4(x_6, x_1, x_14, x_2, x_3, x_7); return x_15; } else @@ -20795,21 +14386,7 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -lean_object* x_16; -x_16 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___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); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_16; -} -} -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { size_t x_12; size_t x_13; lean_object* x_14; @@ -20817,35 +14394,71 @@ x_12 = lean_unbox_usize(x_2); lean_dec(x_2); x_13 = lean_unbox_usize(x_3); lean_dec(x_3); -x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_14 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); return x_14; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -size_t x_8; size_t x_9; lean_object* x_10; -x_8 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_9 = lean_unbox_usize(x_3); +lean_object* x_10; +x_10 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); lean_dec(x_3); -x_10 = l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__5(x_1, x_8, x_9, x_4, x_5, x_6, x_7); +lean_dec(x_2); lean_dec(x_1); return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_3); return x_7; } } +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Init.Util", 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("getElem!", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("index out of bounds", 19); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__1; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__2; +x_3 = lean_unsigned_to_nat(69u); +x_4 = lean_unsigned_to_nat(36u); +x_5 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -20859,7 +14472,7 @@ lean_dec(x_6); if (x_8 == 0) { lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; +x_9 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__4; x_10 = l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(x_9); x_11 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance(x_10, x_3, x_4, x_5); return x_11; @@ -20882,7 +14495,7 @@ lean_dec(x_14); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4; +x_17 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__4; x_18 = l_panic___at___private_Init_Prelude_0__Lean_assembleParts___spec__1(x_17); x_19 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance(x_18, x_3, x_4, x_5); return x_19; @@ -20952,7 +14565,7 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("_args", 5); +x_1 = lean_mk_string_from_bytes("DerivingParams", 14); return x_1; } } @@ -20960,7 +14573,7 @@ static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_Rp _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; @@ -20969,46 +14582,18 @@ return x_3; static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__2; -x_2 = lean_alloc_closure((void*)(l_Lean_Core_mkFreshUserName___boxed), 4, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("DerivingParams", 14); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__4; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__6() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__5; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__7() { +static lean_object* _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__6; +x_1 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__3; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; @@ -21027,190 +14612,54 @@ return x_8; } else { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_2); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_2, 0); -x_11 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__3; -lean_inc(x_4); -x_12 = l_Lean_Elab_Command_liftCoreM___rarg(x_11, x_4, x_5, x_6); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -lean_ctor_set(x_2, 0, x_13); -x_15 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__7; -x_16 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__5; -x_17 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__2), 10, 3); -lean_closure_set(x_17, 0, x_10); -lean_closure_set(x_17, 1, x_15); -lean_closure_set(x_17, 2, x_16); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_box(0); +x_11 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__4; +x_12 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__2; +x_13 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__2), 10, 3); +lean_closure_set(x_13, 0, x_9); +lean_closure_set(x_13, 1, x_11); +lean_closure_set(x_13, 2, x_12); lean_inc(x_4); -x_18 = l_Lean_Elab_Command_liftTermElabM___rarg(x_2, x_17, x_4, x_5, x_14); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_unbox(x_19); -lean_dec(x_19); -x_22 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1(x_1, x_21, x_4, x_5, x_20); -return x_22; -} -else -{ -uint8_t x_23; -lean_dec(x_5); -lean_dec(x_4); -x_23 = !lean_is_exclusive(x_18); -if (x_23 == 0) +x_14 = l_Lean_Elab_Command_liftTermElabM___rarg(x_10, x_13, x_4, x_5, x_6); +if (lean_obj_tag(x_14) == 0) { +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_unbox(x_15); +lean_dec(x_15); +x_18 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1(x_1, x_17, x_4, x_5, x_16); return x_18; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_18, 0); -x_25 = lean_ctor_get(x_18, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_18); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; -} -} -} -else -{ -uint8_t x_27; -lean_free_object(x_2); -lean_dec(x_10); +uint8_t x_19; lean_dec(x_5); lean_dec(x_4); -x_27 = !lean_is_exclusive(x_12); -if (x_27 == 0) -{ -return x_12; -} -else -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_12, 0); -x_29 = lean_ctor_get(x_12, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_12); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; -} -} -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_2, 0); -lean_inc(x_31); -lean_dec(x_2); -x_32 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__3; -lean_inc(x_4); -x_33 = l_Lean_Elab_Command_liftCoreM___rarg(x_32, x_4, x_5, x_6); -if (lean_obj_tag(x_33) == 0) -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_34); -x_37 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__7; -x_38 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__5; -x_39 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__2), 10, 3); -lean_closure_set(x_39, 0, x_31); -lean_closure_set(x_39, 1, x_37); -lean_closure_set(x_39, 2, x_38); -lean_inc(x_4); -x_40 = l_Lean_Elab_Command_liftTermElabM___rarg(x_36, x_39, x_4, x_5, x_35); -if (lean_obj_tag(x_40) == 0) -{ -lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); -x_43 = lean_unbox(x_41); -lean_dec(x_41); -x_44 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1(x_1, x_43, x_4, x_5, x_42); -return x_44; -} -else +x_19 = !lean_is_exclusive(x_14); +if (x_19 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -lean_dec(x_5); -lean_dec(x_4); -x_45 = lean_ctor_get(x_40, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_40, 1); -lean_inc(x_46); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_47 = x_40; -} else { - lean_dec_ref(x_40); - x_47 = lean_box(0); -} -if (lean_is_scalar(x_47)) { - x_48 = lean_alloc_ctor(1, 2, 0); -} else { - x_48 = x_47; -} -lean_ctor_set(x_48, 0, x_45); -lean_ctor_set(x_48, 1, x_46); -return x_48; -} +return x_14; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -lean_dec(x_31); -lean_dec(x_5); -lean_dec(x_4); -x_49 = lean_ctor_get(x_33, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_33, 1); -lean_inc(x_50); -if (lean_is_exclusive(x_33)) { - lean_ctor_release(x_33, 0); - lean_ctor_release(x_33, 1); - x_51 = x_33; -} else { - lean_dec_ref(x_33); - x_51 = lean_box(0); -} -if (lean_is_scalar(x_51)) { - x_52 = lean_alloc_ctor(1, 2, 0); -} else { - x_52 = x_51; -} -lean_ctor_set(x_52, 0, x_49); -lean_ctor_set(x_52, 1, x_50); -return x_52; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_14, 0); +x_21 = lean_ctor_get(x_14, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_14); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } } @@ -21276,7 +14725,7 @@ lean_dec(x_1); return x_6; } } -static lean_object* _init_l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944____closed__1() { +static lean_object* _init_l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985____closed__1() { _start: { lean_object* x_1; @@ -21284,12 +14733,12 @@ x_1 = lean_alloc_closure((void*)(l___private_Lean_Server_Rpc_Deriving_0__Lean_Se return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211; -x_3 = l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944____closed__1; +x_2 = l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__47; +x_3 = l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985____closed__1; x_4 = l_Lean_Elab_registerBuiltinDerivingHandlerWithArgs(x_2, x_3, x_1); if (lean_obj_tag(x_4) == 0) { @@ -21672,276 +15121,48 @@ l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefIns lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__156); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__157 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__157(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__157); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__158 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__158(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__158); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__159 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__159(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__159); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__160 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__160(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__160); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__161 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__161(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__161); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__162 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__162(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__162); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__163 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__163(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__163); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__164 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__164(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__164); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__165 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__165(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__165); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__166 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__166(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__166); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__167 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__167(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__167); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__168 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__168(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__168); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__169 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__169(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__169); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__170 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__170(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__170); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__171 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__171(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__171); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__172 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__172(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__172); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__173 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__173(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__173); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__174 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__174(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__174); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__175 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__175(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__175); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__176 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__176(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__176); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__177 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__177(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__177); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__178 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__178(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__178); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__179 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__179(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__179); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__180 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__180(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__180); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__181 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__181(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__181); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__182 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__182(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__182); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__183 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__183(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__183); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__184 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__184(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__184); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__185 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__185(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__185); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__186 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__186(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__186); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__187 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__187(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__187); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__188 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__188(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__188); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__189 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__189(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__189); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__190); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__191 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__191(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__191); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__192 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__192(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__192); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__193 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__193(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__193); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__194 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__194(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__194); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__195 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__195(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__195); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__196 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__196(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__196); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__197 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__197(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__197); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__198 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__198(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__198); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__199 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__199(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__199); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__200 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__200(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__200); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__201 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__201(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__201); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__202 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__202(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__202); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__203 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__203(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__203); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__204 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__204(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__204); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__205); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__206); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__207); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__208 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__208(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__208); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__209 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__209(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__209); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__210 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__210(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__210); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__211); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__212 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__212(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__212); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__213 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__213(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__213); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__214 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__214(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__214); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__215 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__215(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__215); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__216 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__216(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__216); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__217 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__217(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__217); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__218 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__218(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__218); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__219 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__219(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__219); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__220 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__220(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__220); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__221); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__222 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__222(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__222); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__223); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__224); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__225); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__226 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__226(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__226); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__227 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__227(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__227); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__228); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__229 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__229(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__229); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__230); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__231); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__232); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__233 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__233(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__233); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__234 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__234(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__234); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__235 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__235(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__235); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__236 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__236(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__236); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__237 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__237(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__237); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__238); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__239 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__239(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__239); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__240 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__240(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__240); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__241); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__242 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__242(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__242); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__243 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__243(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__243); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__244 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__244(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__244); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__245 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__245(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__245); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__246 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__246(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveWithRefInstance___closed__246); l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__1 = _init_l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__1(); lean_mark_persistent(l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__1); l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2 = _init_l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2(); lean_mark_persistent(l_Lean_Server_RpcEncoding_withFieldsAux___rarg___closed__2); l_Lean_Server_RpcEncoding_withFields___rarg___closed__1 = _init_l_Lean_Server_RpcEncoding_withFields___rarg___closed__1(); lean_mark_persistent(l_Lean_Server_RpcEncoding_withFields___rarg___closed__1); -l_Lean_Server_RpcEncoding_isOptField___closed__1 = _init_l_Lean_Server_RpcEncoding_isOptField___closed__1(); -lean_mark_persistent(l_Lean_Server_RpcEncoding_isOptField___closed__1); -l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__1 = _init_l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__1(); -l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2 = _init_l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__4___closed__2(); -l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1 = _init_l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1(); -lean_mark_persistent(l_Std_PersistentHashMap_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__7___closed__1); -l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__1 = _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__1(); -lean_mark_persistent(l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__1); -l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2 = _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2(); -lean_mark_persistent(l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__2); -l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3 = _init_l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3(); -lean_mark_persistent(l___private_Lean_Meta_DiscrTree_0__Lean_Meta_DiscrTree_insertAux___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__10___closed__3); -l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16___closed__1 = _init_l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16___closed__1(); -lean_mark_persistent(l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__16___closed__1); -l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1 = _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1); -l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2 = _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2); -l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3 = _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3); -l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4 = _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4); -l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5 = _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5); -l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6 = _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6); -l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7 = _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7); -l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8 = _init_l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8(); -lean_mark_persistent(l_Lean_Meta_DiscrTree_insertCore___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__3); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__4); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__5); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__6 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__1___closed__6); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___lambda__2___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__3); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__4); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__5); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__6); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__7 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__7(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__7); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__8 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__8(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__8); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__9 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__9(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__9); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__10 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__10(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__10); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__11 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__11(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__11); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__12 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__12(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__17___closed__12); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__1); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__2); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__3(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__3); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__4 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__4(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__4); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__5 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__5(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__5); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__6); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__18___closed__7); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__23___closed__1); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__1(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__1); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__2(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__2); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__3 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__3(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_getRpcPacketFor___closed__3); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__1); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__2); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__3); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__4); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__1___closed__5); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__3); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__4); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__5); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__6); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__7); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__8); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__2___closed__9); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___spec__6___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__2(); @@ -22086,6 +15307,44 @@ l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureI lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__71); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__72); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__73 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__73(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__73); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__74 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__74(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__74); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__75 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__75(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__75); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__76 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__76(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__76); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__77 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__77(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__77); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__78 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__78(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__78); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__79 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__79(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__79); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__80 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__80(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__80); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__81 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__81(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__81); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__82 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__82(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__82); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__83 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__83(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__83); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__84 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__84(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__84); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__85 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__85(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__85); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__86 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__86(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__86); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__87 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__87(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__87); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__88 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__88(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__88); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__89); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__90 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__90(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__90); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__91 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__91(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__1___closed__91); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__2(); @@ -22104,106 +15363,112 @@ l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureI lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__8); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__9); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encArgTypes___default = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encArgTypes___default(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encArgTypes___default); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_uniqEncArgTypes___default = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_uniqEncArgTypes___default(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_uniqEncArgTypes___default); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_binders___default = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_binders___default(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_binders___default); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__10 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__10(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__10); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__11 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__11(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveStructureInstance___lambda__2___closed__11); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_ctors___default = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_ctors___default(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_ctors___default); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encodes___default = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encodes___default(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_encodes___default); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_decodes___default = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_decodes___default(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_CtorState_decodes___default); -l_Lean_Server_RpcEncoding_instInhabitedCtorState___closed__1 = _init_l_Lean_Server_RpcEncoding_instInhabitedCtorState___closed__1(); -lean_mark_persistent(l_Lean_Server_RpcEncoding_instInhabitedCtorState___closed__1); -l_Lean_Server_RpcEncoding_instInhabitedCtorState = _init_l_Lean_Server_RpcEncoding_instInhabitedCtorState(); -lean_mark_persistent(l_Lean_Server_RpcEncoding_instInhabitedCtorState); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__2(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF___closed__2); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_matchF); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___lambda__1___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__2); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__3(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__3); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__4(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__4); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__5(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__5); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__6 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__6(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__32___closed__6); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___lambda__1___closed__1); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__1); -l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__2(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__35___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___spec__1___closed__1); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__1); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__2); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__3 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__3(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__1___closed__3); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__2); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__3 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__3); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__4 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__4(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__4); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__5 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__5(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__5); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__6 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__6(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__6); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__7 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__7(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__7); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__8 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__8(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__8); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__9 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__9(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__9); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__10 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__10(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__10); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__11 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__11(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__11); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__12 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__12(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__12); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__13 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__13(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__13); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__14 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__14(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__14); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__15 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__15(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__15); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__16); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__17 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__17(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__17); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__18 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__18(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__18); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__19 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__19(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__19); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__20 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__20(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__20); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__21 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__21(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__21); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__22 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__22(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__22); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__23 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__23(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__23); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__24 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__24(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__24); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__25 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__25(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__25); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__26 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__26(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__26); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__27 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__27(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__27); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__28 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__28(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__28); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__29 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__29(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__29); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__30 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__30(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__30); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__31 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__31(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__31); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__32 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__32(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__32); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__33 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__33(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__33); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__34 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__34(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__34); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__35 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__35(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__35); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__36 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__36(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__36); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__37 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__37(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__37); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__38 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__38(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__38); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__39 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__39(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__39); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__40 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__40(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__2___closed__40); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__1); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__2(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__2); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__3 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__3(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__3); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__4 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__4(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__4); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__5 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__5(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__5); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__6 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__6(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__3___closed__6); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__1(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__1); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__2(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__2); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__3 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__3(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__3); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__4 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__4(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__4); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__5 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__5(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__5); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__6 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__6(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__6); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__7 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__7(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__7); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__8 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__8(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__8); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__9 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__9(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__9); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__10 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__10(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__10); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__11 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__11(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__11); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__12 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__12(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__12); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__13 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__13(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__13); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__14 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__14(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__14); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__15 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__15(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__15); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__16 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__16(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__16); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__17 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__17(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__4___closed__17); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__1(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__1); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__2(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__5___closed__2); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6___boxed__const__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6___boxed__const__1(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___lambda__6___boxed__const__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInductiveInstance___closed__2(); @@ -22216,32 +15481,34 @@ l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server lean_mark_persistent(l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___closed__3); l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___closed__4 = _init_l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___closed__4(); lean_mark_persistent(l_Lean_getConstInfoInduct___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__1___closed__4); -l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1 = _init_l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1(); -lean_mark_persistent(l_panic___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__1(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__1); -l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__2(); -lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__4___lambda__1___closed__2); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__1(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__1); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__2(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__2); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__3 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__3(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__3); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__4 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__4(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__4); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__5 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__5(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__5); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__6 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__6(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__1___closed__6); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__1); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__2 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__2(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__2); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__3 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__3(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__3); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__4 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__4(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__4); +l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__5 = _init_l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__5(); +lean_mark_persistent(l_Array_forInUnsafe_loop___at___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___spec__3___closed__5); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__1); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__2(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__3___closed__2); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__1(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__1); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__2(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___lambda__4___closed__2); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___closed__2(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_deriveInstance___closed__2); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__1); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__2); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__3 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__3(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__3); +l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__4 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__4(); +lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__1___closed__4); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__1 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__1(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__1); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__2 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__2(); @@ -22250,15 +15517,9 @@ l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveIn lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__3); l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__4 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__4(); lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__4); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__5 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__5(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__5); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__6 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__6(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__6); -l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__7 = _init_l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__7(); -lean_mark_persistent(l___private_Lean_Server_Rpc_Deriving_0__Lean_Server_RpcEncoding_dispatchDeriveInstanceUnsafe___lambda__3___closed__7); -l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944____closed__1 = _init_l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944____closed__1(); -lean_mark_persistent(l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944____closed__1); -res = l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_8944_(lean_io_mk_world()); +l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985____closed__1 = _init_l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985____closed__1(); +lean_mark_persistent(l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985____closed__1); +res = l_Lean_Server_RpcEncoding_initFn____x40_Lean_Server_Rpc_Deriving___hyg_7985_(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/Server/Rpc/RequestHandling.c b/stage0/stdlib/Lean/Server/Rpc/RequestHandling.c index ae5da4cfb735..c8aefe9c55b9 100644 --- a/stage0/stdlib/Lean/Server/Rpc/RequestHandling.c +++ b/stage0/stdlib/Lean/Server/Rpc/RequestHandling.c @@ -15,6 +15,7 @@ extern "C" { #endif static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_find_x3f___at___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___spec__1(lean_object*, lean_object*); +lean_object* l_Lean_initializing(lean_object*); lean_object* l_Lean_throwError___at_Lean_KeyedDeclsAttribute_ExtensionState_erase___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isRecCore(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___closed__2; @@ -26,20 +27,22 @@ static lean_object* l_Lean_addDecl___at_Lean_Server_registerRpcProcedure___spec_ static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___lambda__2___closed__2; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___closed__1; size_t lean_usize_add(size_t, size_t); -static lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___closed__2; LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__11; +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__4___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__9___closed__3; +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__6; lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_throwError___at_Lean_declareBuiltin___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); uint8_t lean_uint64_dec_eq(uint64_t, uint64_t); static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___closed__1; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__24; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__22; LEAN_EXPORT lean_object* l_Lean_Server_registerRpcProcedure___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___lambda__2___closed__1; @@ -48,25 +51,26 @@ lean_object* lean_io_error_to_string(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_32_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_72_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__18; lean_object* l_Lean_Server_FileWorker_instMonadRpcSession___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__19; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__5; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addDecl___at_Lean_Server_registerRpcProcedure___spec__2___closed__1; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_32____closed__1; +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1___closed__4; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__15; LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___at_Lean_Server_registerRpcProcedure___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_setEnv___at_Lean_Meta_unfoldDeclsFrom___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_72____closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__1; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__3; size_t lean_usize_sub(size_t, size_t); +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__4___closed__2; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__11; uint8_t l_Lean_isCasesOnRecursor(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_id___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_Server_registerBuiltinRpcProcedure___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); @@ -75,14 +79,15 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Serve uint8_t lean_name_eq(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__12; LEAN_EXPORT lean_object* l_Lean_Server_builtinRpcProcedures; -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__1(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); lean_object* l_Std_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__2; lean_object* lean_string_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static size_t l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___spec__2___closed__2; lean_object* l_Lean_Elab_Term_TermElabM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__14; @@ -94,9 +99,9 @@ LEAN_EXPORT uint8_t l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__ size_t lean_usize_shift_right(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2(lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1___closed__3; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__25; uint8_t l___private_Lean_Message_0__Lean_beqMessageSeverity____x40_Lean_Message___hyg_101_(uint8_t, uint8_t); lean_object* lean_nat_add(lean_object*, lean_object*); @@ -104,20 +109,21 @@ static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling_ LEAN_EXPORT lean_object* l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Declaration_foldExprM___at_Lean_Server_registerRpcProcedure___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Server_registerRpcProcedure___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___closed__1; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__21; size_t lean_uint64_to_usize(uint64_t); lean_object* l_Lean_Expr_FindImpl_findUnsafe_x3f(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2(lean_object*); LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__3___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__3; lean_object* l_Lean_MapDeclarationExtension_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_compileDecl___at_Lean_Server_registerRpcProcedure___spec__6(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__2; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__20; uint64_t l_Lean_Name_hash___override(lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__10; +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__6; lean_object* l_Except_map___rarg(lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); @@ -128,14 +134,12 @@ static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__13; LEAN_EXPORT lean_object* l_Lean_Server_userRpcProcedures; lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__23; -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_compress(lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___spec__2___boxed(lean_object*, lean_object*, lean_object*); static size_t l_Std_PersistentHashMap_findAux___at___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___spec__2___closed__1; LEAN_EXPORT uint8_t l_Lean_Server_registerRpcProcedure___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__6___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__5; LEAN_EXPORT lean_object* l_Lean_addDecl___at_Lean_Server_registerRpcProcedure___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_instInhabitedRpcProcedure___rarg___closed__2; lean_object* l_Lean_KernelException_toMessageData(lean_object*, lean_object*); @@ -148,10 +152,10 @@ lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_replaceRef(lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint64_t, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_insert___at_Lean_Server_registerLspRequestHandler___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__21; -LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwKernelException___at_Lean_Server_registerRpcProcedure___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkMapDeclarationExtension___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_containsAtAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -162,7 +166,9 @@ static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_h static lean_object* l_Lean_Server_registerRpcProcedure___closed__4; lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__1; +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1___closed__2; uint8_t lean_uint64_dec_lt(uint64_t, uint64_t); +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1; extern lean_object* l_Lean_Server_requestHandlers; extern lean_object* l_Lean_Expr_instHashableExpr; LEAN_EXPORT lean_object* l_Lean_logAt___at_Lean_Server_registerRpcProcedure___spec__5(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); @@ -172,7 +178,6 @@ static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__24; lean_object* l_Lean_Server_RequestM_bindTask___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); uint8_t l_Std_PersistentHashMap_contains___at_Lean_Server_registerLspRequestHandler___spec__6(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_left(size_t, size_t); lean_object* l_Lean_Meta_InfoCacheKey_instHashableInfoCacheKey___boxed(lean_object*); @@ -182,9 +187,10 @@ LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Ser static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_32____closed__2; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__16; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__3; -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_instInhabitedRpcProcedure___rarg___closed__4; +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__2; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__5; lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); @@ -207,35 +213,31 @@ lean_object* l_Lean_Server_RequestM_bindWaitFindSnap___rarg(lean_object*, lean_o static lean_object* l_Lean_Server_registerRpcProcedure___lambda__4___closed__3; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__18; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__15; -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__22; lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_instInhabitedRpcProcedure___rarg___closed__1; -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__2; size_t lean_usize_land(size_t, size_t); lean_object* l_Lean_Environment_evalConstCheck___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__19; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__17; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); uint8_t l_Array_contains___at___private_Lean_Meta_Match_Value_0__Lean_Meta_isUIntTypeName___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwKernelException___at_Lean_Server_registerRpcProcedure___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_String_intercalate(lean_object*, lean_object*); -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__7; lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentHashMap_containsAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__6(lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint64_t, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___closed__3; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__22; LEAN_EXPORT lean_object* l_Lean_Server_registerRpcProcedure___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MonadEnv_0__Lean_checkUnsupported___at_Lean_Server_registerRpcProcedure___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__3___closed__2; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__14; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__26; lean_object* lean_environment_main_module(lean_object*); @@ -248,25 +250,26 @@ uint8_t lean_usize_dec_le(size_t, size_t); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_log___at_Lean_Server_registerRpcProcedure___spec__4(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__5; lean_object* l_Lean_Name_append(lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__11; +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__4; lean_object* l_Lean_quoteNameMk(lean_object*); -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__1; -static lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_Command_instInhabitedScope; uint8_t lean_is_aux_recursor(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1___boxed(lean_object*, lean_object*); lean_object* l_Lean_MonadRef_mkInfoFromRefPos___at_Lean_Elab_Term_exprToSyntax___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentHashMap_findAtAux___at___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__6; +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__3___closed__1; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__12; -LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(lean_object*, uint64_t); +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1___closed__5; +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__1; LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__19; -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__1; -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__6; lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); @@ -274,14 +277,12 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Serve lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_Snapshots_Snapshot_endPos(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__1; LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__2___closed__1; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__23; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__25; -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__4; LEAN_EXPORT lean_object* l_Lean_Server_instInhabitedRpcProcedure___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_StateT_instMonadStateT___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_instInhabitedRpcProcedure___rarg(lean_object*); @@ -290,6 +291,7 @@ lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_ uint8_t l_Lean_MapDeclarationExtension_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__20; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); +static lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_addDecl___at_Lean_Server_registerRpcProcedure___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_addDecl___at_Lean_Server_registerRpcProcedure___spec__2___closed__3; @@ -299,23 +301,24 @@ lean_object* l_Lean_Elab_Term_withoutErrToSorry___rarg(lean_object*, lean_object static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__10; lean_object* lean_io_initializing(lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___closed__3; -static lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__6; +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__5; +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__9___closed__4; lean_object* lean_mk_syntax_ident(lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__21; -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__2___closed__2; static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___lambda__4___closed__1; static lean_object* l_List_foldlM___at_Lean_Server_registerRpcProcedure___spec__9___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__13; lean_object* l_Lean_Server_RequestM_asTask___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__3; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__16; static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__10; lean_object* l_Lean_Environment_compileDecl(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_PersistentHashMap_containsAtAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__6; +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(lean_object*, uint64_t); lean_object* l_instMonadStateOfStateT___rarg(lean_object*); uint8_t l_Std_PersistentArray_anyM___at_Lean_MessageLog_hasErrors___spec__1(lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__8; @@ -325,14 +328,13 @@ lean_object* lean_usize_to_nat(size_t); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____closed__1; static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___lambda__3___closed__1; static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___lambda__4___closed__2; -LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__3(lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcCallParams____x40_Lean_Data_Lsp_Extra___hyg_1296_(lean_object*); -static lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__4___closed__4; -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_parseRequestParams___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Server_instInhabitedRpcProcedure___rarg___closed__3; +static lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__7; static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334____spec__1___lambda__3___closed__2; lean_object* l_Lean_Server_Snapshots_Snapshot_env(lean_object*); LEAN_EXPORT lean_object* l_Lean_addAndCompile___at_Lean_Server_registerRpcProcedure___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -344,6 +346,7 @@ static lean_object* l_Lean_Server_registerRpcProcedure___lambda__1___closed__16; static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___closed__3; lean_object* l_Lean_Server_RequestM_readDoc(lean_object*, lean_object*); static lean_object* l_Lean_Server_registerRpcProcedure___lambda__3___closed__4; +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__7; LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerRpcProcedure___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1714,7 +1717,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Serve _start: { lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_io_initializing(x_3); +x_4 = l_Lean_initializing(x_3); x_5 = lean_ctor_get(x_4, 0); lean_inc(x_5); x_6 = lean_unbox(x_5); @@ -1816,7 +1819,7 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(lean_object* x_1, uint64_t x_2) { +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(lean_object* x_1, uint64_t x_2) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1872,7 +1875,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1897,15 +1900,15 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2___rarg___boxed), 3, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; @@ -1948,15 +1951,15 @@ return x_12; } } } -LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__3___rarg), 4, 0); +x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 0); return x_3; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1() { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -1965,7 +1968,7 @@ x_2 = l_StateT_instMonadStateT___rarg(x_1); return x_2; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__2() { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; @@ -1974,17 +1977,17 @@ x_2 = l_instMonadStateOfStateT___rarg(x_1); return x_2; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__3() { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1; -x_2 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__2; +x_1 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1; +x_2 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__2; x_3 = l_Lean_Server_FileWorker_instMonadRpcSession___rarg(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__4() { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__4() { _start: { lean_object* x_1; @@ -1992,7 +1995,7 @@ x_1 = lean_mk_string_from_bytes("Cannot decode params in RPC call '", 34); return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__5() { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__5() { _start: { lean_object* x_1; @@ -2000,7 +2003,7 @@ x_1 = lean_mk_string_from_bytes("(", 1); return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__6() { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__6() { _start: { lean_object* x_1; @@ -2008,7 +2011,7 @@ x_1 = lean_mk_string_from_bytes(")'\n", 3); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; uint8_t x_10; @@ -2021,8 +2024,8 @@ if (x_10 == 0) { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_11 = lean_ctor_get(x_9, 0); -x_12 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1; -x_13 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__3; +x_12 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1; +x_13 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__3; x_14 = lean_apply_5(x_8, lean_box(0), x_12, x_13, x_5, x_11); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); @@ -2035,15 +2038,15 @@ lean_inc(x_16); lean_dec(x_15); x_17 = 1; x_18 = l_Lean_Name_toString(x_3, x_17); -x_19 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__4; +x_19 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__4; x_20 = lean_string_append(x_19, x_18); lean_dec(x_18); -x_21 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__5; +x_21 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__5; x_22 = lean_string_append(x_20, x_21); x_23 = l_Lean_Json_compress(x_4); x_24 = lean_string_append(x_22, x_23); lean_dec(x_23); -x_25 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__6; +x_25 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__6; x_26 = lean_string_append(x_24, x_25); x_27 = lean_string_append(x_26, x_16); lean_dec(x_16); @@ -2077,8 +2080,8 @@ x_34 = lean_ctor_get(x_9, 1); lean_inc(x_34); lean_inc(x_33); lean_dec(x_9); -x_35 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1; -x_36 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__3; +x_35 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1; +x_36 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__3; x_37 = lean_apply_5(x_8, lean_box(0), x_35, x_36, x_5, x_33); x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); @@ -2091,15 +2094,15 @@ lean_inc(x_39); lean_dec(x_38); x_40 = 1; x_41 = l_Lean_Name_toString(x_3, x_40); -x_42 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__4; +x_42 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__4; x_43 = lean_string_append(x_42, x_41); lean_dec(x_41); -x_44 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__5; +x_44 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__5; x_45 = lean_string_append(x_43, x_44); x_46 = l_Lean_Json_compress(x_4); x_47 = lean_string_append(x_45, x_46); lean_dec(x_46); -x_48 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__6; +x_48 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__6; x_49 = lean_string_append(x_47, x_48); x_50 = lean_string_append(x_49, x_39); lean_dec(x_39); @@ -2130,7 +2133,7 @@ return x_57; } } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { if (lean_obj_tag(x_2) == 0) @@ -2157,72 +2160,177 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__3___closed__1() { _start: { -if (lean_obj_tag(x_4) == 0) +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Cannot encode result of RPC call '", 34); +return x_1; +} +} +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__3___closed__2() { +_start: { -lean_object* x_7; lean_object* x_8; -lean_dec(x_3); -lean_dec(x_1); -x_7 = lean_ctor_get(x_4, 0); -lean_inc(x_7); +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("'\n", 2); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_dec(x_4); -x_8 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -return x_8; +lean_dec(x_3); +lean_dec(x_2); +x_27 = lean_ctor_get(x_5, 0); +lean_inc(x_27); +lean_dec(x_5); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_7); +return x_28; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_9 = lean_ctor_get(x_4, 0); -lean_inc(x_9); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_29 = lean_ctor_get(x_5, 0); +lean_inc(x_29); +lean_dec(x_5); +x_30 = lean_st_ref_take(x_1, x_7); +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_2, 0); +lean_inc(x_33); +lean_dec(x_2); +x_34 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1; +x_35 = l_Lean_Server_wrapRpcProcedure___lambda__1___closed__3; +lean_inc(x_31); +x_36 = lean_apply_5(x_33, lean_box(0), x_34, x_35, x_29, x_31); +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +if (lean_obj_tag(x_37) == 0) +{ +uint8_t x_38; +lean_dec(x_36); +x_38 = !lean_is_exclusive(x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +x_39 = lean_st_ref_set(x_1, x_31, x_32); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_8 = x_37; +x_9 = x_40; +goto block_26; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_41 = lean_ctor_get(x_37, 0); +lean_inc(x_41); +lean_dec(x_37); +x_42 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_42, 0, x_41); +x_43 = lean_st_ref_set(x_1, x_31, x_32); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +x_8 = x_42; +x_9 = x_44; +goto block_26; +} +} +else +{ +lean_object* x_45; uint8_t x_46; +lean_dec(x_31); +x_45 = lean_ctor_get(x_36, 1); +lean_inc(x_45); +lean_dec(x_36); +x_46 = !lean_is_exclusive(x_37); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; +x_47 = lean_st_ref_set(x_1, x_45, x_32); +x_48 = lean_ctor_get(x_47, 1); +lean_inc(x_48); +lean_dec(x_47); +x_8 = x_37; +x_9 = x_48; +goto block_26; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_49 = lean_ctor_get(x_37, 0); +lean_inc(x_49); +lean_dec(x_37); +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +x_51 = lean_st_ref_set(x_1, x_45, x_32); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +lean_dec(x_51); +x_8 = x_50; +x_9 = x_52; +goto block_26; +} +} +} +block_26: +{ +if (lean_obj_tag(x_8) == 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; uint8_t x_20; lean_object* x_21; lean_object* x_22; lean_dec(x_4); -x_10 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_8, 0); lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_st_ref_take(x_2, x_6); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1; -x_15 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__3; -x_16 = lean_apply_5(x_10, lean_box(0), x_14, x_15, x_9, x_12); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_st_ref_set(x_2, x_18, x_13); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_19, 0); -lean_dec(x_21); -x_22 = lean_apply_1(x_3, x_17); -lean_ctor_set(x_19, 0, x_22); -return x_19; +lean_dec(x_8); +x_11 = 1; +x_12 = l_Lean_Name_toString(x_3, x_11); +x_13 = l_Lean_Server_wrapRpcProcedure___lambda__3___closed__1; +x_14 = lean_string_append(x_13, x_12); +lean_dec(x_12); +x_15 = l_Lean_Server_wrapRpcProcedure___lambda__3___closed__2; +x_16 = lean_string_append(x_14, x_15); +x_17 = lean_string_append(x_16, x_10); +lean_dec(x_10); +x_18 = l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__22; +x_19 = lean_string_append(x_17, x_18); +x_20 = 3; +x_21 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set_uint8(x_21, sizeof(void*)*1, x_20); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_9); +return x_22; } else { lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_19, 1); +lean_dec(x_3); +x_23 = lean_ctor_get(x_8, 0); lean_inc(x_23); -lean_dec(x_19); -x_24 = lean_apply_1(x_3, x_17); +lean_dec(x_8); +x_24 = lean_apply_1(x_4, x_23); x_25 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_23); +lean_ctor_set(x_25, 1, x_9); return x_25; } } } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___elambda__1___closed__1() { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -2230,83 +2338,85 @@ x_1 = lean_mk_string_from_bytes("Outdated RPC session", 20); return x_1; } } -static lean_object* _init_l_Lean_Server_wrapRpcProcedure___elambda__1___closed__2() { +static lean_object* _init_l_Lean_Server_wrapRpcProcedure___lambda__4___closed__2() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; x_1 = 9; -x_2 = l_Lean_Server_wrapRpcProcedure___elambda__1___closed__1; +x_2 = l_Lean_Server_wrapRpcProcedure___lambda__4___closed__1; x_3 = lean_alloc_ctor(0, 1, 1); lean_ctor_set(x_3, 0, x_2); lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, uint64_t x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___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, uint64_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_13, 0); -lean_inc(x_15); -x_16 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(x_15, x_11); -if (lean_obj_tag(x_16) == 0) +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +x_12 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_11, x_7); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_17; lean_object* x_18; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_10); +lean_object* x_13; lean_object* x_14; lean_dec(x_9); lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_17 = l_Lean_Server_wrapRpcProcedure___elambda__1___closed__2; -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_14); -return x_18; +x_13 = l_Lean_Server_wrapRpcProcedure___lambda__4___closed__2; +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_10); +return x_14; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_19 = lean_ctor_get(x_16, 0); -lean_inc(x_19); -lean_dec(x_16); -lean_inc(x_12); -x_20 = l_Lean_Server_parseRequestParams___rarg(x_6, x_12); -x_21 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2___rarg___boxed), 3, 1); -lean_closure_set(x_21, 0, x_20); -lean_inc(x_19); -x_22 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___boxed), 7, 4); -lean_closure_set(x_22, 0, x_5); -lean_closure_set(x_22, 1, x_19); -lean_closure_set(x_22, 2, x_1); -lean_closure_set(x_22, 3, x_12); -x_23 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__3___rarg), 4, 2); -lean_closure_set(x_23, 0, x_21); -lean_closure_set(x_23, 1, x_22); -lean_inc(x_13); -x_24 = l_Lean_Server_RequestM_asTask___rarg(x_23, x_13, 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; +x_15 = lean_ctor_get(x_12, 0); +lean_inc(x_15); +lean_dec(x_12); +lean_inc(x_8); +x_16 = l_Lean_Server_parseRequestParams___rarg(x_1, x_8); +x_17 = lean_alloc_closure((void*)(l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2___rarg___boxed), 3, 1); +lean_closure_set(x_17, 0, x_16); +lean_inc(x_3); +lean_inc(x_15); +x_18 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___lambda__1___boxed), 7, 4); +lean_closure_set(x_18, 0, x_2); +lean_closure_set(x_18, 1, x_15); +lean_closure_set(x_18, 2, x_3); +lean_closure_set(x_18, 3, x_8); +x_19 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Server_wrapRpcProcedure___spec__3___rarg), 4, 2); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_18); +lean_inc(x_9); +x_20 = l_Lean_Server_RequestM_asTask___rarg(x_19, x_9, x_10); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___lambda__2), 4, 1); +lean_closure_set(x_23, 0, x_4); +lean_inc(x_9); +x_24 = l_Lean_Server_RequestM_bindTask___rarg(x_21, x_23, x_9, x_22); x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); x_26 = lean_ctor_get(x_24, 1); lean_inc(x_26); lean_dec(x_24); -x_27 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__2), 4, 1); -lean_closure_set(x_27, 0, x_10); -lean_inc(x_13); -x_28 = l_Lean_Server_RequestM_bindTask___rarg(x_25, x_27, x_13, x_26); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__3___boxed), 6, 3); -lean_closure_set(x_31, 0, x_8); -lean_closure_set(x_31, 1, x_19); -lean_closure_set(x_31, 2, x_9); -x_32 = l_Lean_Server_RequestM_mapTask___rarg(x_29, x_31, x_13, x_30); -return x_32; +x_27 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___lambda__3___boxed), 7, 4); +lean_closure_set(x_27, 0, x_15); +lean_closure_set(x_27, 1, x_5); +lean_closure_set(x_27, 2, x_3); +lean_closure_set(x_27, 3, x_6); +x_28 = l_Lean_Server_RequestM_mapTask___rarg(x_25, x_27, x_9, x_26); +return x_28; } } } @@ -2314,68 +2424,64 @@ LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure(lean_object* x_1, lean_o _start: { lean_object* x_11; -x_11 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___boxed), 14, 10); -lean_closure_set(x_11, 0, x_1); -lean_closure_set(x_11, 1, lean_box(0)); -lean_closure_set(x_11, 2, lean_box(0)); -lean_closure_set(x_11, 3, lean_box(0)); -lean_closure_set(x_11, 4, x_5); -lean_closure_set(x_11, 5, x_6); -lean_closure_set(x_11, 6, lean_box(0)); -lean_closure_set(x_11, 7, x_8); -lean_closure_set(x_11, 8, x_9); -lean_closure_set(x_11, 9, x_10); +x_11 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___lambda__4___boxed), 10, 6); +lean_closure_set(x_11, 0, x_6); +lean_closure_set(x_11, 1, x_5); +lean_closure_set(x_11, 2, x_1); +lean_closure_set(x_11, 3, x_10); +lean_closure_set(x_11, 4, x_8); +lean_closure_set(x_11, 5, x_9); return x_11; } } -LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint64_t x_3; lean_object* x_4; x_3 = lean_unbox_uint64(x_2); lean_dec(x_2); -x_4 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__1(x_1, x_3); +x_4 = l_Std_RBNode_find___at_Lean_Server_wrapRpcProcedure___spec__1(x_1, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l_liftExcept___at_Lean_Server_wrapRpcProcedure___elambda__1___spec__2___rarg(x_1, x_2, x_3); +x_4 = l_liftExcept___at_Lean_Server_wrapRpcProcedure___spec__2___rarg(x_1, x_2, x_3); lean_dec(x_2); lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; -x_8 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +x_8 = l_Lean_Server_wrapRpcProcedure___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_7; -x_7 = l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_2); -return x_7; +lean_object* x_8; +x_8 = l_Lean_Server_wrapRpcProcedure___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_1); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___elambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Server_wrapRpcProcedure___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint64_t x_15; lean_object* x_16; -x_15 = lean_unbox_uint64(x_11); -lean_dec(x_11); -x_16 = l_Lean_Server_wrapRpcProcedure___elambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15, x_12, x_13, x_14); -return x_16; +uint64_t x_11; lean_object* x_12; +x_11 = lean_unbox_uint64(x_7); +lean_dec(x_7); +x_12 = l_Lean_Server_wrapRpcProcedure___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_11, x_8, x_9, x_10); +return x_12; } } LEAN_EXPORT lean_object* l_Std_PersistentHashMap_insertAux_traverse___at_Lean_Server_registerBuiltinRpcProcedure___spec__3(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -3041,18 +3147,14 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerBuiltinRpcProcedure___lambda__1(l _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -lean_inc(x_1); -x_9 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___elambda__1___boxed), 14, 10); +lean_inc(x_3); +x_9 = lean_alloc_closure((void*)(l_Lean_Server_wrapRpcProcedure___lambda__4___boxed), 10, 6); lean_closure_set(x_9, 0, x_1); -lean_closure_set(x_9, 1, lean_box(0)); -lean_closure_set(x_9, 2, lean_box(0)); -lean_closure_set(x_9, 3, lean_box(0)); -lean_closure_set(x_9, 4, x_2); -lean_closure_set(x_9, 5, x_3); -lean_closure_set(x_9, 6, lean_box(0)); -lean_closure_set(x_9, 7, x_4); -lean_closure_set(x_9, 8, x_5); -lean_closure_set(x_9, 9, x_6); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_3); +lean_closure_set(x_9, 3, x_4); +lean_closure_set(x_9, 4, x_5); +lean_closure_set(x_9, 5, x_6); x_10 = l___private_Lean_Server_Rpc_RequestHandling_0__Lean_Server_handleRpcCallUnsafe___lambda__3___closed__1; x_11 = lean_st_ref_take(x_10, x_8); x_12 = lean_ctor_get(x_11, 0); @@ -3060,7 +3162,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_12, x_1, x_9); +x_14 = l_Std_PersistentHashMap_insert___at_Lean_Server_registerBuiltinRpcProcedure___spec__1(x_12, x_3, x_9); x_15 = lean_st_ref_set(x_10, x_14, x_13); x_16 = !lean_is_exclusive(x_15); if (x_16 == 0) @@ -3103,8 +3205,8 @@ if (x_12 == 0) lean_object* x_13; lean_object* x_14; uint8_t x_15; x_13 = lean_ctor_get(x_11, 0); x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_1); -x_15 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_13, x_1); +lean_inc(x_3); +x_15 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_13, x_3); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; @@ -3143,8 +3245,8 @@ x_24 = lean_ctor_get(x_11, 1); lean_inc(x_24); lean_inc(x_23); lean_dec(x_11); -lean_inc(x_1); -x_25 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_23, x_1); +lean_inc(x_3); +x_25 = l_Std_PersistentHashMap_contains___at_Lean_Server_registerBuiltinRpcProcedure___spec__5(x_23, x_3); if (x_25 == 0) { lean_object* x_26; lean_object* x_27; @@ -3270,7 +3372,7 @@ x_35 = lean_ctor_get(x_18, 1); lean_inc(x_35); lean_dec(x_18); x_36 = lean_box(0); -x_37 = l_Lean_Server_registerBuiltinRpcProcedure___lambda__2(x_1, x_5, x_6, x_8, x_9, x_10, x_17, x_36, x_35); +x_37 = l_Lean_Server_registerBuiltinRpcProcedure___lambda__2(x_6, x_5, x_1, x_10, x_8, x_9, x_17, x_36, x_35); return x_37; } } @@ -6200,12 +6302,13 @@ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(0); x_2 = lean_box(0); x_3 = l_Lean_Server_registerRpcProcedure___lambda__3___closed__10; -x_4 = lean_alloc_ctor(0, 5, 0); +x_4 = lean_alloc_ctor(0, 6, 0); lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_1); -lean_ctor_set(x_4, 2, x_2); -lean_ctor_set(x_4, 3, x_1); -lean_ctor_set(x_4, 4, x_3); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_1); +lean_ctor_set(x_4, 3, x_2); +lean_ctor_set(x_4, 4, x_1); +lean_ctor_set(x_4, 5, x_3); return x_4; } } @@ -6868,7 +6971,7 @@ lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; @@ -6876,7 +6979,7 @@ x_7 = l_Lean_Server_registerRpcProcedure(x_1, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__1() { _start: { lean_object* x_1; @@ -6884,25 +6987,25 @@ x_1 = lean_mk_string_from_bytes("attribute cannot be erased", 26); return x_1; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__2() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__1; +x_1 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__2; +x_5 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__2; x_6 = l_Lean_throwError___at_Lean_AttributeImpl_erase___default___spec__1(x_5, x_2, x_3, x_4); return x_6; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__1() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__1() { _start: { lean_object* x_1; @@ -6910,17 +7013,17 @@ x_1 = lean_mk_string_from_bytes("serverRpcMethod", 15); return x_1; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__2() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__1; +x_2 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__3() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__3() { _start: { lean_object* x_1; @@ -6928,12 +7031,12 @@ x_1 = lean_mk_string_from_bytes("Marks a function as a Lean server RPC method.\n return x_1; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__4() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__4() { _start: { lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; -x_1 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__2; -x_2 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__3; +x_1 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__2; +x_2 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__3; x_3 = 1; x_4 = lean_alloc_ctor(0, 2, 1); lean_ctor_set(x_4, 0, x_1); @@ -6942,29 +7045,29 @@ lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__5() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__1___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__1___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__6() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__7() { +static lean_object* _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__4; -x_2 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__5; -x_3 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__6; +x_1 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__4; +x_2 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__5; +x_3 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__6; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -6972,31 +7075,31 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__7; +x_2 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__7; x_3 = l_Lean_registerBuiltinAttribute(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); -x_8 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); @@ -7129,22 +7232,26 @@ lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling res = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_334_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__1); -l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__2); -l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__3); -l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__4 = _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__4); -l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__5 = _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__5); -l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__6 = _init_l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___elambda__1___lambda__1___closed__6); -l_Lean_Server_wrapRpcProcedure___elambda__1___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___elambda__1___closed__1(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___elambda__1___closed__1); -l_Lean_Server_wrapRpcProcedure___elambda__1___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___elambda__1___closed__2(); -lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___elambda__1___closed__2); +l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__1___closed__1); +l_Lean_Server_wrapRpcProcedure___lambda__1___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__1___closed__2); +l_Lean_Server_wrapRpcProcedure___lambda__1___closed__3 = _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__1___closed__3); +l_Lean_Server_wrapRpcProcedure___lambda__1___closed__4 = _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__1___closed__4); +l_Lean_Server_wrapRpcProcedure___lambda__1___closed__5 = _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__1___closed__5); +l_Lean_Server_wrapRpcProcedure___lambda__1___closed__6 = _init_l_Lean_Server_wrapRpcProcedure___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__1___closed__6); +l_Lean_Server_wrapRpcProcedure___lambda__3___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__3___closed__1); +l_Lean_Server_wrapRpcProcedure___lambda__3___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__3___closed__2); +l_Lean_Server_wrapRpcProcedure___lambda__4___closed__1 = _init_l_Lean_Server_wrapRpcProcedure___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__4___closed__1); +l_Lean_Server_wrapRpcProcedure___lambda__4___closed__2 = _init_l_Lean_Server_wrapRpcProcedure___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Server_wrapRpcProcedure___lambda__4___closed__2); l_Std_PersistentHashMap_insertAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__2___closed__1 = _init_l_Std_PersistentHashMap_insertAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__2___closed__1(); lean_mark_persistent(l_Std_PersistentHashMap_insertAux___at_Lean_Server_registerBuiltinRpcProcedure___spec__2___closed__1); l_Lean_Server_registerBuiltinRpcProcedure___lambda__2___closed__1 = _init_l_Lean_Server_registerBuiltinRpcProcedure___lambda__2___closed__1(); @@ -7289,25 +7396,25 @@ l_Lean_Server_registerRpcProcedure___closed__3 = _init_l_Lean_Server_registerRpc lean_mark_persistent(l_Lean_Server_registerRpcProcedure___closed__3); l_Lean_Server_registerRpcProcedure___closed__4 = _init_l_Lean_Server_registerRpcProcedure___closed__4(); lean_mark_persistent(l_Lean_Server_registerRpcProcedure___closed__4); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__1 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__1); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__2 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____lambda__2___closed__2); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__1 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__1(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__1); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__2 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__2(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__2); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__3 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__3(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__3); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__4 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__4(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__4); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__5 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__5(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__5); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__6 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__6(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__6); -l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__7 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__7(); -lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289____closed__7); -res = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1289_(lean_io_mk_world()); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__1 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__1); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__2 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____lambda__2___closed__2); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__1 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__1(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__1); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__2 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__2(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__2); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__3 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__3(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__3); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__4 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__4(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__4); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__5 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__5(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__5); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__6 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__6(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__6); +l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__7 = _init_l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__7(); +lean_mark_persistent(l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406____closed__7); +res = l_Lean_Server_initFn____x40_Lean_Server_Rpc_RequestHandling___hyg_1406_(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/Server/Snapshots.c b/stage0/stdlib/Lean/Server/Snapshots.c index c9fe711da08d..0c8977a85b49 100644 --- a/stage0/stdlib/Lean/Server/Snapshots.c +++ b/stage0/stdlib/Lean/Server/Snapshots.c @@ -19,6 +19,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Snapshots_Snaps lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_compileNextCmd___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_Snapshots_compileNextCmd_withNewInteractiveDiags___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static uint32_t l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__6; @@ -28,14 +29,13 @@ LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_server_stderrAsMessages; static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_6____closed__3; static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__3; lean_object* lean_st_ref_get(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_parseAhead_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__3; lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_Snapshot_infoTree(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_parseAhead_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Snapshots_Snapshot_infoTree___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Snapshots_Snapshot_diagnostics___spec__4(size_t, size_t, lean_object*); +static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__6; static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__14; lean_object* l_List_head_x21___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_withStdout___at_Lean_Server_Snapshots_compileNextCmd___spec__2(lean_object*, lean_object*, lean_object*); @@ -48,7 +48,6 @@ LEAN_EXPORT lean_object* l_IO_withStderr___at_Lean_Server_Snapshots_compileNextC lean_object* l_IO_FS_Stream_ofBuffer(lean_object*); lean_object* lean_get_set_stderr(lean_object*, lean_object*); static lean_object* l_IO_FS_withIsolatedStreams___at_Lean_Server_Snapshots_compileNextCmd___spec__1___closed__1; -static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__2; static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_6____closed__2; LEAN_EXPORT lean_object* l_IO_withStdin___at_Lean_Server_Snapshots_compileNextCmd___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__5; @@ -56,12 +55,11 @@ static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__15; lean_object* l_panic___at_Lean_FileMap_toPosition_loop___spec__1(lean_object*); static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__18; extern lean_object* l_ByteArray_empty; +static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__5; static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__16; lean_object* l_Lean_Widget_msgToInteractiveDiagnostic(lean_object*, lean_object*, uint8_t, lean_object*); uint8_t l_Lean_Option_get___at_Lean_getSanitizeNames___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_parseAhead(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Lean_initFn____x40_Lean_PrettyPrinter_Delaborator_Options___hyg_6____spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__1; static lean_object* l_Lean_Server_Snapshots_Snapshot_infoTree___closed__6; lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__7; @@ -74,20 +72,19 @@ LEAN_EXPORT lean_object* l_IO_FS_withIsolatedStreams___at_Lean_Server_Snapshots_ lean_object* l_Std_mkHashMapImp___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_compileNextCmd___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedMessage; -static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__5; lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); static lean_object* l_Lean_Server_Snapshots_compileNextCmd___closed__6; -static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__3; -lean_object* l_Lean_Elab_Command_withLogging(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__1; lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Snapshots_Snapshot_infoTree___closed__9; extern lean_object* l_Lean_firstFrontendMacroScope; LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot; LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_Snapshot_endPos___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_6_(lean_object*); +static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__2; size_t lean_usize_of_nat(lean_object*); lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_Snapshot_diagnostics(lean_object*); @@ -99,12 +96,10 @@ lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); lean_object* l_Std_PersistentArray_push___rarg(lean_object*, lean_object*); extern lean_object* l_Lean_Elab_instInhabitedInfoTree; uint8_t l_String_isEmpty(lean_object*); -static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__6; uint8_t l_Lean_Parser_isExitCommand(lean_object*); static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__12; static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_6____closed__1; static lean_object* l_Lean_Server_Snapshots_Snapshot_infoTree___closed__4; -static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__4; static lean_object* l_Lean_Server_Snapshots_compileNextCmd___closed__5; LEAN_EXPORT lean_object* l_Std_PersistentArray_mapM___at_Lean_Server_Snapshots_Snapshot_diagnostics___spec__1(lean_object*); static lean_object* l_Lean_Server_Snapshots_compileNextCmd___closed__3; @@ -123,6 +118,7 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_Server_Snapshots_Snapshot_infoTree___ LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_compileNextCmd___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); lean_object* l_Lean_Elab_Command_elabCommandTopLevel(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__4; static lean_object* l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__4; LEAN_EXPORT lean_object* l_List_forIn_loop___at_Lean_Server_Snapshots_compileNextCmd_withNewInteractiveDiags___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_Snapshot_msgLog(lean_object*); @@ -817,7 +813,7 @@ static lean_object* _init_l_Lean_Server_Snapshots_Snapshot_infoTree___closed__10 lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Server_Snapshots_Snapshot_infoTree___closed__7; x_2 = l_Lean_Server_Snapshots_Snapshot_infoTree___closed__8; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Server_Snapshots_Snapshot_infoTree___closed__9; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -947,108 +943,7 @@ lean_ctor_set(x_17, 1, x_3); return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_parseAhead_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_7 = l_Lean_Server_Snapshots_Snapshot_msgLog(x_1); -lean_inc(x_3); -lean_inc(x_2); -x_8 = l_Lean_Parser_parseCommand(x_2, x_3, x_4, x_7); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 0); -lean_inc(x_10); -lean_dec(x_8); -x_11 = lean_ctor_get(x_9, 0); -lean_inc(x_11); -lean_dec(x_9); -lean_inc(x_10); -x_12 = l_Lean_Parser_isEOI(x_10); -if (x_12 == 0) -{ -uint8_t x_13; -lean_inc(x_10); -x_13 = l_Lean_Parser_isExitCommand(x_10); -if (x_13 == 0) -{ -lean_object* x_14; -x_14 = lean_array_push(x_5, x_10); -x_4 = x_11; -x_5 = x_14; -goto _start; -} -else -{ -lean_object* x_16; lean_object* x_17; -lean_dec(x_11); -lean_dec(x_3); -lean_dec(x_2); -x_16 = lean_array_push(x_5, x_10); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_6); -return x_17; -} -} -else -{ -lean_object* x_18; lean_object* x_19; -lean_dec(x_11); -lean_dec(x_3); -lean_dec(x_2); -x_18 = lean_array_push(x_5, x_10); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_6); -return x_19; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_parseAhead_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Lean_Server_Snapshots_parseAhead_go(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_parseAhead(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_4 = lean_ctor_get(x_2, 3); -lean_inc(x_4); -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(x_4, 2); -lean_inc(x_6); -lean_dec(x_4); -x_7 = l_Lean_Elab_Command_instInhabitedScope; -x_8 = l_List_head_x21___rarg(x_7, x_6); -lean_dec(x_6); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 2); -lean_inc(x_10); -x_11 = lean_ctor_get(x_8, 3); -lean_inc(x_11); -lean_dec(x_8); -x_12 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_12, 0, x_5); -lean_ctor_set(x_12, 1, x_9); -lean_ctor_set(x_12, 2, x_10); -lean_ctor_set(x_12, 3, x_11); -x_13 = lean_ctor_get(x_2, 2); -lean_inc(x_13); -x_14 = l_Lean_Server_Snapshots_instInhabitedSnapshot___closed__5; -x_15 = l_Lean_Server_Snapshots_parseAhead_go(x_2, x_1, x_12, x_13, x_14, x_3); -lean_dec(x_2); -return x_15; -} -} -static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__1() { +static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__1() { _start: { lean_object* x_1; @@ -1056,17 +951,17 @@ x_1 = lean_mk_string_from_bytes("server", 6); return x_1; } } -static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__2() { +static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__1; +x_2 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__3() { +static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__3() { _start: { lean_object* x_1; @@ -1074,17 +969,17 @@ x_1 = lean_mk_string_from_bytes("stderrAsMessages", 16); return x_1; } } -static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__4() { +static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__2; -x_2 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__3; +x_1 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__2; +x_2 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__5() { +static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__5() { _start: { lean_object* x_1; @@ -1092,13 +987,13 @@ x_1 = lean_mk_string_from_bytes("(server) capture output to the Lean stderr chan return x_1; } } -static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__6() { +static lean_object* _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__6() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 1; -x_2 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__1; -x_3 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__5; +x_2 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__1; +x_3 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__5; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -1107,12 +1002,12 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__4; -x_3 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__6; +x_2 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__4; +x_3 = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__6; x_4 = l_Lean_Option_register___at_Lean_initFn____x40_Lean_PrettyPrinter_Delaborator_Options___hyg_6____spec__1(x_2, x_3, x_1); return x_4; } @@ -1651,7 +1546,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_Snapshots_compileNextCmd___lambda__2(lean _start: { lean_object* x_5; -x_5 = l_Lean_Elab_Command_withLogging(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_withLogging___at_Lean_Elab_Command_elabCommand___spec__2(x_1, x_2, x_3, x_4); if (lean_obj_tag(x_5) == 0) { uint8_t x_6; @@ -2693,19 +2588,19 @@ l_Lean_Server_Snapshots_Snapshot_infoTree___closed__9 = _init_l_Lean_Server_Snap lean_mark_persistent(l_Lean_Server_Snapshots_Snapshot_infoTree___closed__9); l_Lean_Server_Snapshots_Snapshot_infoTree___closed__10 = _init_l_Lean_Server_Snapshots_Snapshot_infoTree___closed__10(); lean_mark_persistent(l_Lean_Server_Snapshots_Snapshot_infoTree___closed__10); -l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__1 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__1(); -lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__1); -l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__2 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__2(); -lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__2); -l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__3 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__3(); -lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__3); -l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__4 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__4(); -lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__4); -l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__5 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__5(); -lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__5); -l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__6 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__6(); -lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373____closed__6); -if (builtin) {res = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_373_(lean_io_mk_world()); +l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__1 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__1(); +lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__1); +l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__2 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__2(); +lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__2); +l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__3 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__3(); +lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__3); +l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__4 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__4(); +lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__4); +l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__5 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__5(); +lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__5); +l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__6 = _init_l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__6(); +lean_mark_persistent(l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251____closed__6); +if (builtin) {res = l_Lean_Server_Snapshots_initFn____x40_Lean_Server_Snapshots___hyg_251_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Server_Snapshots_server_stderrAsMessages = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Server_Snapshots_server_stderrAsMessages); diff --git a/stage0/stdlib/Lean/Server/Watchdog.c b/stage0/stdlib/Lean/Server/Watchdog.c index b9bac26a4ba9..0e1e0c381d40 100644 --- a/stage0/stdlib/Lean/Server/Watchdog.c +++ b/stage0/stdlib/Lean/Server/Watchdog.c @@ -73,6 +73,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_terminateFileWorker___boxed(lean double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Server_Watchdog_startFileWorker___closed__3; static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_Watchdog_initAndRunWatchdog___spec__2___closed__2; +extern lean_object* l_Lean_Lsp_SemanticTokenModifier_names; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_forwardRequestToWorker___spec__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_RBNode_forIn_visit___at_Lean_Server_Watchdog_mainLoop___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspResponse___at_Lean_Server_Watchdog_handleRequest___spec__2(lean_object*, lean_object*, lean_object*); @@ -19347,7 +19348,7 @@ static lean_object* _init_l_Lean_Server_Watchdog_mkLeanServerCapabilities___clos { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Lsp_SemanticTokenType_names; -x_2 = l_Lean_Server_Watchdog_startFileWorker___closed__4; +x_2 = l_Lean_Lsp_SemanticTokenModifier_names; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); diff --git a/stage0/stdlib/Lean/Structure.c b/stage0/stdlib/Lean/Structure.c index 62acd97f61e6..318c315a17fc 100644 --- a/stage0/stdlib/Lean/Structure.c +++ b/stage0/stdlib/Lean/Structure.c @@ -21,7 +21,7 @@ size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_StructureInfo_getProjFn_x3f___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_62____closed__24; LEAN_EXPORT lean_object* l_Lean_instInhabitedStructureDescr; -lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); @@ -641,7 +641,7 @@ x_51 = lean_ctor_get(x_27, 0); lean_inc(x_51); lean_dec(x_27); x_52 = lean_unsigned_to_nat(1024u); -x_53 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2803_(x_51, x_52); +x_53 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_2766_(x_51, x_52); x_54 = l___private_Lean_Structure_0__Lean_reprStructureFieldInfo____x40_Lean_Structure___hyg_62____closed__26; x_55 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_55, 0, x_54); diff --git a/stage0/stdlib/Lean/SubExpr.c b/stage0/stdlib/Lean/SubExpr.c index 59f8979dce75..927e76ffc136 100644 --- a/stage0/stdlib/Lean/SubExpr.c +++ b/stage0/stdlib/Lean/SubExpr.c @@ -54,7 +54,6 @@ LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushLetValue___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushBindingBody(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushLetBody(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushBindingDomain(lean_object*); -lean_object* l_Lean_Expr_updateApp_x21(lean_object*, lean_object*, lean_object*); lean_object* l_String_splitOn(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushAppFn___boxed(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); @@ -145,6 +144,7 @@ static lean_object* l_Lean_SubExpr_Pos_toArray___closed__1; LEAN_EXPORT lean_object* l___private_Lean_SubExpr_0__Lean_SubExpr_Pos_ofStringCoord(lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_ofArray___boxed(lean_object*); static lean_object* l_Lean_SubExpr_Pos_push___closed__2; +lean_object* l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_push___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_SubExpr_Pos_pushLetVarType(lean_object*); static lean_object* l_Lean_SubExpr_Pos_push___closed__1; @@ -1739,7 +1739,7 @@ lean_dec(x_7); x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); lean_dec(x_9); -x_11 = lean_alloc_closure((void*)(l_Lean_Expr_updateApp_x21), 3, 1); +x_11 = lean_alloc_closure((void*)(l___private_Lean_Expr_0__Lean_Expr_updateApp_x21Impl___boxed), 3, 1); lean_closure_set(x_11, 0, x_4); x_12 = lean_unsigned_to_nat(0u); x_13 = l_Lean_SubExpr_Pos_push(x_3, x_12); diff --git a/stage0/stdlib/Lean/Syntax.c b/stage0/stdlib/Lean/Syntax.c index 7750e39063c2..42e8352caabf 100644 --- a/stage0/stdlib/Lean/Syntax.c +++ b/stage0/stdlib/Lean/Syntax.c @@ -2105,7 +2105,7 @@ static lean_object* _init_l_Lean_Syntax_updateTrailing___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Syntax_updateTrailing___closed__1; x_2 = l_Lean_Syntax_updateTrailing___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Lean_Syntax_updateTrailing___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Util/HasConstCache.c b/stage0/stdlib/Lean/Util/HasConstCache.c index 1c993a90eba0..67c1cf484935 100644 --- a/stage0/stdlib/Lean/Util/HasConstCache.c +++ b/stage0/stdlib/Lean/Util/HasConstCache.c @@ -16,6 +16,7 @@ extern "C" { LEAN_EXPORT lean_object* l_Lean_HasConstCache_containsUnsafe(lean_object*, lean_object*, lean_object*); lean_object* l___private_Std_Data_HashMap_0__Std_numBucketsForCapacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_HasConstCache_containsUnsafe___boxed(lean_object*, lean_object*, lean_object*); +uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_HasConstCache_containsUnsafe_cache___boxed(lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -24,7 +25,6 @@ uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_foldlM___at_Lean_HasConstCache_containsUnsafe_cache___spec__4(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_HasConstCache_containsUnsafe_cache___rarg___boxed(lean_object*, lean_object*, lean_object*); -uint8_t l_Lean_Expr_ptrEq(lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Std_HashMapImp_expand___at_Lean_HasConstCache_containsUnsafe_cache___spec__2(lean_object*, lean_object*); @@ -39,6 +39,7 @@ LEAN_EXPORT lean_object* l_Std_AssocList_find_x3f___at_Lean_HasConstCache_contai LEAN_EXPORT lean_object* l_Lean_HasConstCache_cache___default; size_t lean_usize_modn(size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_AssocList_replace___at_Lean_HasConstCache_containsUnsafe_cache___spec__5(lean_object*, uint8_t, lean_object*); +size_t lean_ptr_addr(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Lean_HasConstCache_cache___default___closed__1; lean_object* lean_nat_mul(lean_object*, lean_object*); @@ -76,20 +77,22 @@ return x_3; } else { -lean_object* x_4; lean_object* x_5; uint8_t x_6; +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; uint8_t x_8; x_4 = lean_ctor_get(x_2, 0); x_5 = lean_ctor_get(x_2, 2); -x_6 = l_Lean_Expr_ptrEq(x_4, x_1); -if (x_6 == 0) +x_6 = lean_ptr_addr(x_4); +x_7 = lean_ptr_addr(x_1); +x_8 = lean_usize_dec_eq(x_6, x_7); +if (x_8 == 0) { x_2 = x_5; goto _start; } else { -uint8_t x_8; -x_8 = 1; -return x_8; +uint8_t x_10; +x_10 = 1; +return x_10; } } } @@ -214,61 +217,65 @@ uint8_t x_5; x_5 = !lean_is_exclusive(x_3); if (x_5 == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; uint8_t x_11; x_6 = lean_ctor_get(x_3, 0); x_7 = lean_ctor_get(x_3, 1); x_8 = lean_ctor_get(x_3, 2); -x_9 = l_Lean_Expr_ptrEq(x_6, x_1); -if (x_9 == 0) -{ -lean_object* x_10; -x_10 = l_Std_AssocList_replace___at_Lean_HasConstCache_containsUnsafe_cache___spec__5(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_10); +x_9 = lean_ptr_addr(x_6); +x_10 = lean_ptr_addr(x_1); +x_11 = lean_usize_dec_eq(x_9, x_10); +if (x_11 == 0) +{ +lean_object* x_12; +x_12 = l_Std_AssocList_replace___at_Lean_HasConstCache_containsUnsafe_cache___spec__5(x_1, x_2, x_8); +lean_ctor_set(x_3, 2, x_12); return x_3; } else { -lean_object* x_11; +lean_object* x_13; lean_dec(x_7); lean_dec(x_6); -x_11 = lean_box(x_2); -lean_ctor_set(x_3, 1, x_11); +x_13 = lean_box(x_2); +lean_ctor_set(x_3, 1, x_13); lean_ctor_set(x_3, 0, x_1); return x_3; } } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_12 = lean_ctor_get(x_3, 0); -x_13 = lean_ctor_get(x_3, 1); -x_14 = lean_ctor_get(x_3, 2); +lean_object* x_14; lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; uint8_t x_19; +x_14 = lean_ctor_get(x_3, 0); +x_15 = lean_ctor_get(x_3, 1); +x_16 = lean_ctor_get(x_3, 2); +lean_inc(x_16); +lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); lean_dec(x_3); -x_15 = l_Lean_Expr_ptrEq(x_12, x_1); -if (x_15 == 0) +x_17 = lean_ptr_addr(x_14); +x_18 = lean_ptr_addr(x_1); +x_19 = lean_usize_dec_eq(x_17, x_18); +if (x_19 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = l_Std_AssocList_replace___at_Lean_HasConstCache_containsUnsafe_cache___spec__5(x_1, x_2, x_14); -x_17 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_17, 0, x_12); -lean_ctor_set(x_17, 1, x_13); -lean_ctor_set(x_17, 2, x_16); -return x_17; +lean_object* x_20; lean_object* x_21; +x_20 = l_Std_AssocList_replace___at_Lean_HasConstCache_containsUnsafe_cache___spec__5(x_1, x_2, x_16); +x_21 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_21, 0, x_14); +lean_ctor_set(x_21, 1, x_15); +lean_ctor_set(x_21, 2, x_20); +return x_21; } else { -lean_object* x_18; lean_object* x_19; -lean_dec(x_13); -lean_dec(x_12); -x_18 = lean_box(x_2); -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_1); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set(x_19, 2, x_14); -return x_19; +lean_object* x_22; lean_object* x_23; +lean_dec(x_15); +lean_dec(x_14); +x_22 = lean_box(x_2); +x_23 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_23, 0, x_1); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_23, 2, x_16); +return x_23; } } } @@ -473,23 +480,25 @@ return x_3; } else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; x_4 = lean_ctor_get(x_2, 0); x_5 = lean_ctor_get(x_2, 1); x_6 = lean_ctor_get(x_2, 2); -x_7 = l_Lean_Expr_ptrEq(x_4, x_1); -if (x_7 == 0) +x_7 = lean_ptr_addr(x_4); +x_8 = lean_ptr_addr(x_1); +x_9 = lean_usize_dec_eq(x_7, x_8); +if (x_9 == 0) { x_2 = x_6; goto _start; } else { -lean_object* x_9; +lean_object* x_11; lean_inc(x_5); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_5); -return x_9; +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_5); +return x_11; } } } diff --git a/stage0/stdlib/Lean/Util/Recognizers.c b/stage0/stdlib/Lean/Util/Recognizers.c index 1828d2da343f..e4eb56b7311d 100644 --- a/stage0/stdlib/Lean/Util/Recognizers.c +++ b/stage0/stdlib/Lean/Util/Recognizers.c @@ -63,6 +63,7 @@ LEAN_EXPORT lean_object* l_Lean_Expr_isConstructorApp___boxed(lean_object*, lean static lean_object* l_Lean_Expr_iff_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Expr_heq_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app4_x3f___boxed(lean_object*, lean_object*); +lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_eq_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_iff_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_natAdd_x3f(lean_object*); @@ -87,7 +88,6 @@ static lean_object* l_Lean_Expr_natAdd_x3f___closed__4; LEAN_EXPORT lean_object* l_Lean_Expr_app1_x3f___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_app2_x3f___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Expr_constructorApp_x3f___closed__1; -lean_object* l_Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_arrow_x3f(lean_object*); LEAN_EXPORT uint8_t l_Lean_Expr_isDIte(lean_object*); static lean_object* l_Lean_Expr_ne_x3f___closed__2; @@ -1334,7 +1334,7 @@ x_19 = lean_nat_add(x_17, x_18); lean_dec(x_18); lean_dec(x_17); x_20 = lean_unsigned_to_nat(0u); -x_21 = l_Lean_Expr_getAppNumArgsAux(x_2, x_20); +x_21 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_20); x_22 = lean_nat_dec_eq(x_19, x_21); lean_dec(x_21); lean_dec(x_19); @@ -1365,7 +1365,7 @@ x_27 = lean_nat_add(x_25, x_26); lean_dec(x_26); lean_dec(x_25); x_28 = lean_unsigned_to_nat(0u); -x_29 = l_Lean_Expr_getAppNumArgsAux(x_2, x_28); +x_29 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_28); x_30 = lean_nat_dec_eq(x_27, x_29); lean_dec(x_29); lean_dec(x_27); @@ -1429,7 +1429,7 @@ x_42 = lean_nat_add(x_40, x_41); lean_dec(x_41); lean_dec(x_40); x_43 = lean_unsigned_to_nat(0u); -x_44 = l_Lean_Expr_getAppNumArgsAux(x_2, x_43); +x_44 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_43); x_45 = lean_nat_dec_eq(x_42, x_44); lean_dec(x_44); lean_dec(x_42); @@ -1460,7 +1460,7 @@ x_50 = lean_nat_add(x_48, x_49); lean_dec(x_49); lean_dec(x_48); x_51 = lean_unsigned_to_nat(0u); -x_52 = l_Lean_Expr_getAppNumArgsAux(x_2, x_51); +x_52 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_51); x_53 = lean_nat_dec_eq(x_50, x_52); lean_dec(x_52); lean_dec(x_50); @@ -1707,7 +1707,7 @@ x_45 = lean_nat_add(x_43, x_44); lean_dec(x_44); lean_dec(x_43); x_46 = lean_unsigned_to_nat(0u); -x_47 = l_Lean_Expr_getAppNumArgsAux(x_2, x_46); +x_47 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_46); x_48 = lean_nat_dec_eq(x_45, x_47); lean_dec(x_45); if (x_48 == 0) @@ -1751,7 +1751,7 @@ x_59 = lean_nat_add(x_57, x_58); lean_dec(x_58); lean_dec(x_57); x_60 = lean_unsigned_to_nat(0u); -x_61 = l_Lean_Expr_getAppNumArgsAux(x_2, x_60); +x_61 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_60); x_62 = lean_nat_dec_eq(x_59, x_61); lean_dec(x_59); if (x_62 == 0) @@ -1828,7 +1828,7 @@ x_80 = lean_nat_add(x_78, x_79); lean_dec(x_79); lean_dec(x_78); x_81 = lean_unsigned_to_nat(0u); -x_82 = l_Lean_Expr_getAppNumArgsAux(x_2, x_81); +x_82 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_81); x_83 = lean_nat_dec_eq(x_80, x_82); lean_dec(x_80); if (x_83 == 0) @@ -1872,7 +1872,7 @@ x_94 = lean_nat_add(x_92, x_93); lean_dec(x_93); lean_dec(x_92); x_95 = lean_unsigned_to_nat(0u); -x_96 = l_Lean_Expr_getAppNumArgsAux(x_2, x_95); +x_96 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_95); x_97 = lean_nat_dec_eq(x_94, x_96); lean_dec(x_94); if (x_97 == 0) diff --git a/stage0/stdlib/Lean/Util/ReplaceExpr.c b/stage0/stdlib/Lean/Util/ReplaceExpr.c index f9d773f0d6e7..82fcbc218a00 100644 --- a/stage0/stdlib/Lean/Util/ReplaceExpr.c +++ b/stage0/stdlib/Lean/Util/ReplaceExpr.c @@ -13,29 +13,30 @@ #ifdef __cplusplus extern "C" { #endif -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Expr_ReplaceImpl_initCache___closed__1; +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceImpl_cache___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_ReplaceImpl_initCache___closed__2; +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceImpl_replaceUnsafe(lean_object*, lean_object*); static lean_object* l_Lean_Expr_ReplaceImpl_initCache___closed__4; LEAN_EXPORT size_t l_Lean_Expr_ReplaceImpl_cacheSize; lean_object* l_Lean_Expr_bvar___override(lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceImpl_replaceUnsafeM(lean_object*, size_t, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceImpl_cache(size_t, lean_object*, lean_object*, lean_object*); size_t lean_usize_mod(size_t, size_t); size_t lean_ptr_addr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceImpl_replaceUnsafeM___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); -lean_object* lean_expr_update_app(lean_object*, lean_object*, lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_ReplaceImpl_initCache___closed__3; LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(lean_object*, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceImpl_initCache; @@ -122,11 +123,12 @@ if (lean_obj_tag(x_11) == 0) switch (lean_obj_tag(x_3)) { case 5: { -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_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; size_t x_20; size_t x_21; uint8_t x_22; x_12 = lean_ctor_get(x_3, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_3, 1); lean_inc(x_13); +lean_inc(x_12); lean_inc(x_1); x_14 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_12, x_4); x_15 = lean_ctor_get(x_14, 0); @@ -134,170 +136,411 @@ lean_inc(x_15); x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); lean_dec(x_14); +lean_inc(x_13); x_17 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_13, x_16); x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -lean_inc(x_3); -x_20 = lean_expr_update_app(x_3, x_15, x_18); -x_21 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_20, x_19); -return x_21; +x_20 = lean_ptr_addr(x_12); +lean_dec(x_12); +x_21 = lean_ptr_addr(x_15); +x_22 = lean_usize_dec_eq(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_13); +x_23 = l_Lean_Expr_app___override(x_15, x_18); +x_24 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_23, x_19); +return x_24; } -case 6: +else { -lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_22 = lean_ctor_get(x_3, 1); -lean_inc(x_22); -x_23 = lean_ctor_get(x_3, 2); -lean_inc(x_23); -x_24 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); -lean_inc(x_1); -x_25 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_22, x_4); -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_23, x_27); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); +size_t x_25; size_t x_26; uint8_t x_27; +x_25 = lean_ptr_addr(x_13); +lean_dec(x_13); +x_26 = lean_ptr_addr(x_18); +x_27 = lean_usize_dec_eq(x_25, x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = l_Lean_Expr_app___override(x_15, x_18); +x_29 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_28, x_19); +return x_29; +} +else +{ +lean_object* x_30; +lean_dec(x_18); +lean_dec(x_15); lean_inc(x_3); -x_31 = lean_expr_update_lambda(x_3, x_24, x_26, x_29); -x_32 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_31, x_30); -return x_32; +x_30 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_3, x_19); +return x_30; } -case 7: +} +} +case 6: { -lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_33 = lean_ctor_get(x_3, 1); +lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; size_t x_42; size_t x_43; uint8_t x_44; +x_31 = lean_ctor_get(x_3, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_3, 1); +lean_inc(x_32); +x_33 = lean_ctor_get(x_3, 2); lean_inc(x_33); -x_34 = lean_ctor_get(x_3, 2); -lean_inc(x_34); -x_35 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +x_34 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +lean_inc(x_32); lean_inc(x_1); -x_36 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_33, x_4); -x_37 = lean_ctor_get(x_36, 0); +x_35 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_32, x_4); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); lean_inc(x_37); -x_38 = lean_ctor_get(x_36, 1); -lean_inc(x_38); -lean_dec(x_36); -x_39 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_34, x_38); -x_40 = lean_ctor_get(x_39, 0); +lean_dec(x_35); +lean_inc(x_33); +x_38 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_33, x_37); +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); -lean_inc(x_41); +lean_dec(x_38); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +x_41 = l_Lean_Expr_lam___override(x_31, x_32, x_33, x_34); +x_42 = lean_ptr_addr(x_32); +lean_dec(x_32); +x_43 = lean_ptr_addr(x_36); +x_44 = lean_usize_dec_eq(x_42, x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +lean_dec(x_41); +lean_dec(x_33); +x_45 = l_Lean_Expr_lam___override(x_31, x_36, x_39, x_34); +x_46 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_45, x_40); +return x_46; +} +else +{ +size_t x_47; size_t x_48; uint8_t x_49; +x_47 = lean_ptr_addr(x_33); +lean_dec(x_33); +x_48 = lean_ptr_addr(x_39); +x_49 = lean_usize_dec_eq(x_47, x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; +lean_dec(x_41); +x_50 = l_Lean_Expr_lam___override(x_31, x_36, x_39, x_34); +x_51 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_50, x_40); +return x_51; +} +else +{ +uint8_t x_52; +x_52 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_34, x_34); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; +lean_dec(x_41); +x_53 = l_Lean_Expr_lam___override(x_31, x_36, x_39, x_34); +x_54 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_53, x_40); +return x_54; +} +else +{ +lean_object* x_55; lean_dec(x_39); -lean_inc(x_3); -x_42 = lean_expr_update_forall(x_3, x_35, x_37, x_40); -x_43 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_42, x_41); -return x_43; +lean_dec(x_36); +lean_dec(x_31); +x_55 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_41, x_40); +return x_55; +} +} +} +} +case 7: +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; size_t x_67; size_t x_68; uint8_t x_69; +x_56 = lean_ctor_get(x_3, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_3, 1); +lean_inc(x_57); +x_58 = lean_ctor_get(x_3, 2); +lean_inc(x_58); +x_59 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +lean_inc(x_57); +lean_inc(x_1); +x_60 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_57, x_4); +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_60, 1); +lean_inc(x_62); +lean_dec(x_60); +lean_inc(x_58); +x_63 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_58, x_62); +x_64 = lean_ctor_get(x_63, 0); +lean_inc(x_64); +x_65 = lean_ctor_get(x_63, 1); +lean_inc(x_65); +lean_dec(x_63); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +x_66 = l_Lean_Expr_forallE___override(x_56, x_57, x_58, x_59); +x_67 = lean_ptr_addr(x_57); +lean_dec(x_57); +x_68 = lean_ptr_addr(x_61); +x_69 = lean_usize_dec_eq(x_67, x_68); +if (x_69 == 0) +{ +lean_object* x_70; lean_object* x_71; +lean_dec(x_66); +lean_dec(x_58); +x_70 = l_Lean_Expr_forallE___override(x_56, x_61, x_64, x_59); +x_71 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_70, x_65); +return x_71; +} +else +{ +size_t x_72; size_t x_73; uint8_t x_74; +x_72 = lean_ptr_addr(x_58); +lean_dec(x_58); +x_73 = lean_ptr_addr(x_64); +x_74 = lean_usize_dec_eq(x_72, x_73); +if (x_74 == 0) +{ +lean_object* x_75; lean_object* x_76; +lean_dec(x_66); +x_75 = l_Lean_Expr_forallE___override(x_56, x_61, x_64, x_59); +x_76 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_75, x_65); +return x_76; +} +else +{ +uint8_t x_77; +x_77 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_59, x_59); +if (x_77 == 0) +{ +lean_object* x_78; lean_object* x_79; +lean_dec(x_66); +x_78 = l_Lean_Expr_forallE___override(x_56, x_61, x_64, x_59); +x_79 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_78, x_65); +return x_79; +} +else +{ +lean_object* x_80; +lean_dec(x_64); +lean_dec(x_61); +lean_dec(x_56); +x_80 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_66, x_65); +return x_80; +} +} +} } case 8: { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_44 = lean_ctor_get(x_3, 1); -lean_inc(x_44); -x_45 = lean_ctor_get(x_3, 2); -lean_inc(x_45); -x_46 = lean_ctor_get(x_3, 3); -lean_inc(x_46); +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; size_t x_95; size_t x_96; uint8_t x_97; +x_81 = lean_ctor_get(x_3, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_3, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_3, 2); +lean_inc(x_83); +x_84 = lean_ctor_get(x_3, 3); +lean_inc(x_84); +x_85 = lean_ctor_get_uint8(x_3, sizeof(void*)*4 + 8); +lean_inc(x_82); lean_inc(x_1); -x_47 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_44, x_4); -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); -lean_inc(x_49); -lean_dec(x_47); +x_86 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_82, x_4); +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +lean_inc(x_83); lean_inc(x_1); -x_50 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_45, x_49); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -lean_dec(x_50); -x_53 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_46, x_52); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); +x_89 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_83, x_88); +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +lean_inc(x_84); +x_92 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_84, x_91); +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +lean_dec(x_92); +x_95 = lean_ptr_addr(x_82); +lean_dec(x_82); +x_96 = lean_ptr_addr(x_87); +x_97 = lean_usize_dec_eq(x_95, x_96); +if (x_97 == 0) +{ +lean_object* x_98; lean_object* x_99; +lean_dec(x_84); +lean_dec(x_83); +x_98 = l_Lean_Expr_letE___override(x_81, x_87, x_90, x_93, x_85); +x_99 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_98, x_94); +return x_99; +} +else +{ +size_t x_100; size_t x_101; uint8_t x_102; +x_100 = lean_ptr_addr(x_83); +lean_dec(x_83); +x_101 = lean_ptr_addr(x_90); +x_102 = lean_usize_dec_eq(x_100, x_101); +if (x_102 == 0) +{ +lean_object* x_103; lean_object* x_104; +lean_dec(x_84); +x_103 = l_Lean_Expr_letE___override(x_81, x_87, x_90, x_93, x_85); +x_104 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_103, x_94); +return x_104; +} +else +{ +size_t x_105; size_t x_106; uint8_t x_107; +x_105 = lean_ptr_addr(x_84); +lean_dec(x_84); +x_106 = lean_ptr_addr(x_93); +x_107 = lean_usize_dec_eq(x_105, x_106); +if (x_107 == 0) +{ +lean_object* x_108; lean_object* x_109; +x_108 = l_Lean_Expr_letE___override(x_81, x_87, x_90, x_93, x_85); +x_109 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_108, x_94); +return x_109; +} +else +{ +lean_object* x_110; +lean_dec(x_93); +lean_dec(x_90); +lean_dec(x_87); +lean_dec(x_81); lean_inc(x_3); -x_56 = lean_expr_update_let(x_3, x_48, x_51, x_54); -x_57 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_56, x_55); -return x_57; +x_110 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_3, x_94); +return x_110; +} +} +} } case 10: { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_58 = lean_ctor_get(x_3, 1); -lean_inc(x_58); -x_59 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_58, x_4); -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); -lean_dec(x_59); +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; size_t x_116; size_t x_117; uint8_t x_118; +x_111 = lean_ctor_get(x_3, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_3, 1); +lean_inc(x_112); +lean_inc(x_112); +x_113 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_112, x_4); +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); +x_116 = lean_ptr_addr(x_112); +lean_dec(x_112); +x_117 = lean_ptr_addr(x_114); +x_118 = lean_usize_dec_eq(x_116, x_117); +if (x_118 == 0) +{ +lean_object* x_119; lean_object* x_120; +x_119 = l_Lean_Expr_mdata___override(x_111, x_114); +x_120 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_119, x_115); +return x_120; +} +else +{ +lean_object* x_121; +lean_dec(x_114); +lean_dec(x_111); lean_inc(x_3); -x_62 = lean_expr_update_mdata(x_3, x_60); -x_63 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_62, x_61); -return x_63; +x_121 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_3, x_115); +return x_121; +} } case 11: { -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_64 = lean_ctor_get(x_3, 2); -lean_inc(x_64); -x_65 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_64, x_4); -x_66 = lean_ctor_get(x_65, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_65, 1); -lean_inc(x_67); -lean_dec(x_65); +lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; size_t x_128; size_t x_129; uint8_t x_130; +x_122 = lean_ctor_get(x_3, 0); +lean_inc(x_122); +x_123 = lean_ctor_get(x_3, 1); +lean_inc(x_123); +x_124 = lean_ctor_get(x_3, 2); +lean_inc(x_124); +lean_inc(x_124); +x_125 = l_Lean_Expr_ReplaceImpl_replaceUnsafeM_visit(x_1, x_2, x_124, x_4); +x_126 = lean_ctor_get(x_125, 0); +lean_inc(x_126); +x_127 = lean_ctor_get(x_125, 1); +lean_inc(x_127); +lean_dec(x_125); +x_128 = lean_ptr_addr(x_124); +lean_dec(x_124); +x_129 = lean_ptr_addr(x_126); +x_130 = lean_usize_dec_eq(x_128, x_129); +if (x_130 == 0) +{ +lean_object* x_131; lean_object* x_132; +x_131 = l_Lean_Expr_proj___override(x_122, x_123, x_126); +x_132 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_131, x_127); +return x_132; +} +else +{ +lean_object* x_133; +lean_dec(x_126); +lean_dec(x_123); +lean_dec(x_122); lean_inc(x_3); -x_68 = lean_expr_update_proj(x_3, x_66); -x_69 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_68, x_67); -return x_69; +x_133 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_3, x_127); +return x_133; +} } default: { -lean_object* x_70; +lean_object* x_134; lean_dec(x_1); -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_3); -lean_ctor_set(x_70, 1, x_4); -return x_70; +x_134 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_134, 0, x_3); +lean_ctor_set(x_134, 1, x_4); +return x_134; } } } else { -lean_object* x_71; lean_object* x_72; +lean_object* x_135; lean_object* x_136; lean_dec(x_1); -x_71 = lean_ctor_get(x_11, 0); -lean_inc(x_71); +x_135 = lean_ctor_get(x_11, 0); +lean_inc(x_135); lean_dec(x_11); -x_72 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_71, x_4); -return x_72; +x_136 = l_Lean_Expr_ReplaceImpl_cache(x_6, x_3, x_135, x_4); +return x_136; } } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; +lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_dec(x_3); lean_dec(x_1); -x_73 = lean_ctor_get(x_4, 1); -lean_inc(x_73); -x_74 = lean_array_uget(x_73, x_6); -lean_dec(x_73); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_74); -lean_ctor_set(x_75, 1, x_4); -return x_75; +x_137 = lean_ctor_get(x_4, 1); +lean_inc(x_137); +x_138 = lean_array_uget(x_137, x_6); +lean_dec(x_137); +x_139 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_4); +return x_139; } } } diff --git a/stage0/stdlib/Lean/Util/ReplaceLevel.c b/stage0/stdlib/Lean/Util/ReplaceLevel.c index 1a8639cbc1a3..165122be8ee6 100644 --- a/stage0/stdlib/Lean/Util/ReplaceLevel.c +++ b/stage0/stdlib/Lean/Util/ReplaceLevel.c @@ -14,38 +14,40 @@ extern "C" { #endif lean_object* l_List_reverse___rarg(lean_object*); -lean_object* lean_expr_update_forall(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); +lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); uint8_t lean_usize_dec_eq(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); -lean_object* lean_expr_update_mdata(lean_object*, lean_object*); lean_object* l_Lean_Level_succ___override(lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(lean_object*, size_t, lean_object*, lean_object*); static lean_object* l_Lean_Expr_ReplaceLevelImpl_initCache___closed__3; +lean_object* l_Lean_Expr_mdata___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceLevelImpl_cache(size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_letE___override(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +uint8_t l_ptrEqList___rarg(lean_object*, lean_object*); LEAN_EXPORT size_t l_Lean_Expr_ReplaceLevelImpl_cacheSize; -lean_object* lean_level_mk_max_simp(lean_object*, lean_object*); -lean_object* lean_level_mk_imax_simp(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelMax_x27(lean_object*, lean_object*); +lean_object* l_Lean_mkLevelIMax_x27(lean_object*, lean_object*); +lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceLevelImpl_replaceUnsafe(lean_object*, lean_object*); static lean_object* l_Lean_Expr_ReplaceLevelImpl_initCache___closed__1; lean_object* l_Lean_Expr_bvar___override(lean_object*); -lean_object* lean_expr_update_let(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_proj(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Level_replace(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceLevelImpl_cache___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_mod(size_t, size_t); size_t lean_ptr_addr(lean_object*); -lean_object* lean_expr_update_sort(lean_object*, lean_object*); +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM(lean_object*, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_ReplaceLevelImpl_initCache; -lean_object* lean_expr_update_lambda(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); +uint8_t l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(uint8_t, uint8_t); +lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_ReplaceLevelImpl_initCache___closed__2; -lean_object* lean_expr_update_app(lean_object*, lean_object*, lean_object*); -lean_object* lean_expr_update_const(lean_object*, lean_object*); static lean_object* l_Lean_Expr_ReplaceLevelImpl_initCache___closed__4; LEAN_EXPORT lean_object* l_Lean_Level_replace(lean_object* x_1, lean_object* x_2) { _start: @@ -78,7 +80,7 @@ lean_dec(x_2); lean_inc(x_1); x_9 = l_Lean_Level_replace(x_1, x_7); x_10 = l_Lean_Level_replace(x_1, x_8); -x_11 = lean_level_mk_max_simp(x_9, x_10); +x_11 = l_Lean_mkLevelMax_x27(x_9, x_10); return x_11; } case 3: @@ -92,7 +94,7 @@ lean_dec(x_2); lean_inc(x_1); x_14 = l_Lean_Level_replace(x_1, x_12); x_15 = l_Lean_Level_replace(x_1, x_13); -x_16 = lean_level_mk_imax_simp(x_14, x_15); +x_16 = l_Lean_mkLevelIMax_x27(x_14, x_15); return x_16; } default: @@ -222,194 +224,469 @@ if (x_10 == 0) switch (lean_obj_tag(x_3)) { case 3: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; uint8_t x_15; x_11 = lean_ctor_get(x_3, 0); lean_inc(x_11); +lean_inc(x_11); x_12 = l_Lean_Level_replace(x_1, x_11); -lean_inc(x_3); -x_13 = lean_expr_update_sort(x_3, x_12); -x_14 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_13, x_4); -return x_14; +x_13 = lean_ptr_addr(x_11); +lean_dec(x_11); +x_14 = lean_ptr_addr(x_12); +x_15 = lean_usize_dec_eq(x_13, x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = l_Lean_Expr_sort___override(x_12); +x_17 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_16, x_4); +return x_17; } -case 4: +else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_15 = lean_ctor_get(x_3, 1); -lean_inc(x_15); -x_16 = lean_box(0); -x_17 = l_List_mapTRAux___at_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit___spec__1(x_1, x_15, x_16); +lean_object* x_18; +lean_dec(x_12); lean_inc(x_3); -x_18 = lean_expr_update_const(x_3, x_17); -x_19 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_18, x_4); -return x_19; +x_18 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_3, x_4); +return x_18; } -case 5: +} +case 4: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_20 = lean_ctor_get(x_3, 0); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_19 = lean_ctor_get(x_3, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_3, 1); lean_inc(x_20); -x_21 = lean_ctor_get(x_3, 1); -lean_inc(x_21); -lean_inc(x_1); -x_22 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_20, x_4); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); +x_21 = lean_box(0); +lean_inc(x_20); +x_22 = l_List_mapTRAux___at_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit___spec__1(x_1, x_20, x_21); +x_23 = l_ptrEqList___rarg(x_20, x_22); +lean_dec(x_20); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = l_Lean_Expr_const___override(x_19, x_22); +x_25 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_24, x_4); +return x_25; +} +else +{ +lean_object* x_26; lean_dec(x_22); -x_25 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_21, x_24); -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); +lean_dec(x_19); lean_inc(x_3); -x_28 = lean_expr_update_app(x_3, x_23, x_26); -x_29 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_28, x_27); -return x_29; +x_26 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_3, x_4); +return x_26; } -case 6: +} +case 5: { -lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_30 = lean_ctor_get(x_3, 1); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; uint8_t x_37; +x_27 = lean_ctor_get(x_3, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_3, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_1); +x_29 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_27, x_4); +x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); -x_31 = lean_ctor_get(x_3, 2); +x_31 = lean_ctor_get(x_29, 1); lean_inc(x_31); -x_32 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); -lean_inc(x_1); -x_33 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_30, x_4); -x_34 = lean_ctor_get(x_33, 0); +lean_dec(x_29); +lean_inc(x_28); +x_32 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_28, x_31); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); +lean_dec(x_32); +x_35 = lean_ptr_addr(x_27); +lean_dec(x_27); +x_36 = lean_ptr_addr(x_30); +x_37 = lean_usize_dec_eq(x_35, x_36); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; +lean_dec(x_28); +x_38 = l_Lean_Expr_app___override(x_30, x_33); +x_39 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_38, x_34); +return x_39; +} +else +{ +size_t x_40; size_t x_41; uint8_t x_42; +x_40 = lean_ptr_addr(x_28); +lean_dec(x_28); +x_41 = lean_ptr_addr(x_33); +x_42 = lean_usize_dec_eq(x_40, x_41); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; +x_43 = l_Lean_Expr_app___override(x_30, x_33); +x_44 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_43, x_34); +return x_44; +} +else +{ +lean_object* x_45; lean_dec(x_33); -x_36 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_31, x_35); -x_37 = lean_ctor_get(x_36, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_36, 1); -lean_inc(x_38); -lean_dec(x_36); +lean_dec(x_30); lean_inc(x_3); -x_39 = lean_expr_update_lambda(x_3, x_32, x_34, x_37); -x_40 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_39, x_38); -return x_40; +x_45 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_3, x_34); +return x_45; } -case 7: +} +} +case 6: { -lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_41 = lean_ctor_get(x_3, 1); -lean_inc(x_41); -x_42 = lean_ctor_get(x_3, 2); -lean_inc(x_42); -x_43 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); -lean_inc(x_1); -x_44 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_41, x_4); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; size_t x_57; size_t x_58; uint8_t x_59; +x_46 = lean_ctor_get(x_3, 0); lean_inc(x_46); -lean_dec(x_44); -x_47 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_42, x_46); -x_48 = lean_ctor_get(x_47, 0); +x_47 = lean_ctor_get(x_3, 1); +lean_inc(x_47); +x_48 = lean_ctor_get(x_3, 2); +lean_inc(x_48); +x_49 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +lean_inc(x_47); +lean_inc(x_1); +x_50 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_47, x_4); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +lean_inc(x_48); +x_53 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_48, x_52); +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +lean_dec(x_53); lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); -lean_inc(x_49); +lean_inc(x_47); +lean_inc(x_46); +x_56 = l_Lean_Expr_lam___override(x_46, x_47, x_48, x_49); +x_57 = lean_ptr_addr(x_47); lean_dec(x_47); -lean_inc(x_3); -x_50 = lean_expr_update_forall(x_3, x_43, x_45, x_48); -x_51 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_50, x_49); -return x_51; +x_58 = lean_ptr_addr(x_51); +x_59 = lean_usize_dec_eq(x_57, x_58); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; +lean_dec(x_56); +lean_dec(x_48); +x_60 = l_Lean_Expr_lam___override(x_46, x_51, x_54, x_49); +x_61 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_60, x_55); +return x_61; +} +else +{ +size_t x_62; size_t x_63; uint8_t x_64; +x_62 = lean_ptr_addr(x_48); +lean_dec(x_48); +x_63 = lean_ptr_addr(x_54); +x_64 = lean_usize_dec_eq(x_62, x_63); +if (x_64 == 0) +{ +lean_object* x_65; lean_object* x_66; +lean_dec(x_56); +x_65 = l_Lean_Expr_lam___override(x_46, x_51, x_54, x_49); +x_66 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_65, x_55); +return x_66; +} +else +{ +uint8_t x_67; +x_67 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_49, x_49); +if (x_67 == 0) +{ +lean_object* x_68; lean_object* x_69; +lean_dec(x_56); +x_68 = l_Lean_Expr_lam___override(x_46, x_51, x_54, x_49); +x_69 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_68, x_55); +return x_69; +} +else +{ +lean_object* x_70; +lean_dec(x_54); +lean_dec(x_51); +lean_dec(x_46); +x_70 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_56, x_55); +return x_70; +} +} +} +} +case 7: +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; size_t x_82; size_t x_83; uint8_t x_84; +x_71 = lean_ctor_get(x_3, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_3, 1); +lean_inc(x_72); +x_73 = lean_ctor_get(x_3, 2); +lean_inc(x_73); +x_74 = lean_ctor_get_uint8(x_3, sizeof(void*)*3 + 8); +lean_inc(x_72); +lean_inc(x_1); +x_75 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_72, x_4); +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_75, 1); +lean_inc(x_77); +lean_dec(x_75); +lean_inc(x_73); +x_78 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_73, x_77); +x_79 = lean_ctor_get(x_78, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +lean_dec(x_78); +lean_inc(x_73); +lean_inc(x_72); +lean_inc(x_71); +x_81 = l_Lean_Expr_forallE___override(x_71, x_72, x_73, x_74); +x_82 = lean_ptr_addr(x_72); +lean_dec(x_72); +x_83 = lean_ptr_addr(x_76); +x_84 = lean_usize_dec_eq(x_82, x_83); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; +lean_dec(x_81); +lean_dec(x_73); +x_85 = l_Lean_Expr_forallE___override(x_71, x_76, x_79, x_74); +x_86 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_85, x_80); +return x_86; +} +else +{ +size_t x_87; size_t x_88; uint8_t x_89; +x_87 = lean_ptr_addr(x_73); +lean_dec(x_73); +x_88 = lean_ptr_addr(x_79); +x_89 = lean_usize_dec_eq(x_87, x_88); +if (x_89 == 0) +{ +lean_object* x_90; lean_object* x_91; +lean_dec(x_81); +x_90 = l_Lean_Expr_forallE___override(x_71, x_76, x_79, x_74); +x_91 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_90, x_80); +return x_91; +} +else +{ +uint8_t x_92; +x_92 = l___private_Lean_Expr_0__Lean_beqBinderInfo____x40_Lean_Expr___hyg_362_(x_74, x_74); +if (x_92 == 0) +{ +lean_object* x_93; lean_object* x_94; +lean_dec(x_81); +x_93 = l_Lean_Expr_forallE___override(x_71, x_76, x_79, x_74); +x_94 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_93, x_80); +return x_94; +} +else +{ +lean_object* x_95; +lean_dec(x_79); +lean_dec(x_76); +lean_dec(x_71); +x_95 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_81, x_80); +return x_95; +} +} +} } case 8: { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_52 = lean_ctor_get(x_3, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_3, 2); -lean_inc(x_53); -x_54 = lean_ctor_get(x_3, 3); -lean_inc(x_54); +lean_object* x_96; lean_object* x_97; lean_object* x_98; 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_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; size_t x_110; size_t x_111; uint8_t x_112; +x_96 = lean_ctor_get(x_3, 0); +lean_inc(x_96); +x_97 = lean_ctor_get(x_3, 1); +lean_inc(x_97); +x_98 = lean_ctor_get(x_3, 2); +lean_inc(x_98); +x_99 = lean_ctor_get(x_3, 3); +lean_inc(x_99); +x_100 = lean_ctor_get_uint8(x_3, sizeof(void*)*4 + 8); +lean_inc(x_97); lean_inc(x_1); -x_55 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_52, x_4); -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -lean_dec(x_55); +x_101 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_97, x_4); +x_102 = lean_ctor_get(x_101, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_101, 1); +lean_inc(x_103); +lean_dec(x_101); +lean_inc(x_98); lean_inc(x_1); -x_58 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_53, x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -lean_dec(x_58); -x_61 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_54, 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_104 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_98, x_103); +x_105 = lean_ctor_get(x_104, 0); +lean_inc(x_105); +x_106 = lean_ctor_get(x_104, 1); +lean_inc(x_106); +lean_dec(x_104); +lean_inc(x_99); +x_107 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_99, x_106); +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +x_110 = lean_ptr_addr(x_97); +lean_dec(x_97); +x_111 = lean_ptr_addr(x_102); +x_112 = lean_usize_dec_eq(x_110, x_111); +if (x_112 == 0) +{ +lean_object* x_113; lean_object* x_114; +lean_dec(x_99); +lean_dec(x_98); +x_113 = l_Lean_Expr_letE___override(x_96, x_102, x_105, x_108, x_100); +x_114 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_113, x_109); +return x_114; +} +else +{ +size_t x_115; size_t x_116; uint8_t x_117; +x_115 = lean_ptr_addr(x_98); +lean_dec(x_98); +x_116 = lean_ptr_addr(x_105); +x_117 = lean_usize_dec_eq(x_115, x_116); +if (x_117 == 0) +{ +lean_object* x_118; lean_object* x_119; +lean_dec(x_99); +x_118 = l_Lean_Expr_letE___override(x_96, x_102, x_105, x_108, x_100); +x_119 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_118, x_109); +return x_119; +} +else +{ +size_t x_120; size_t x_121; uint8_t x_122; +x_120 = lean_ptr_addr(x_99); +lean_dec(x_99); +x_121 = lean_ptr_addr(x_108); +x_122 = lean_usize_dec_eq(x_120, x_121); +if (x_122 == 0) +{ +lean_object* x_123; lean_object* x_124; +x_123 = l_Lean_Expr_letE___override(x_96, x_102, x_105, x_108, x_100); +x_124 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_123, x_109); +return x_124; +} +else +{ +lean_object* x_125; +lean_dec(x_108); +lean_dec(x_105); +lean_dec(x_102); +lean_dec(x_96); lean_inc(x_3); -x_64 = lean_expr_update_let(x_3, x_56, x_59, x_62); -x_65 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_64, x_63); -return x_65; +x_125 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_3, x_109); +return x_125; +} +} +} } case 10: { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_66 = lean_ctor_get(x_3, 1); -lean_inc(x_66); -x_67 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_66, x_4); -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); +lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; size_t x_131; size_t x_132; uint8_t x_133; +x_126 = lean_ctor_get(x_3, 0); +lean_inc(x_126); +x_127 = lean_ctor_get(x_3, 1); +lean_inc(x_127); +lean_inc(x_127); +x_128 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_127, x_4); +x_129 = lean_ctor_get(x_128, 0); +lean_inc(x_129); +x_130 = lean_ctor_get(x_128, 1); +lean_inc(x_130); +lean_dec(x_128); +x_131 = lean_ptr_addr(x_127); +lean_dec(x_127); +x_132 = lean_ptr_addr(x_129); +x_133 = lean_usize_dec_eq(x_131, x_132); +if (x_133 == 0) +{ +lean_object* x_134; lean_object* x_135; +x_134 = l_Lean_Expr_mdata___override(x_126, x_129); +x_135 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_134, x_130); +return x_135; +} +else +{ +lean_object* x_136; +lean_dec(x_129); +lean_dec(x_126); lean_inc(x_3); -x_70 = lean_expr_update_mdata(x_3, x_68); -x_71 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_70, x_69); -return x_71; +x_136 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_3, x_130); +return x_136; +} } case 11: { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_72 = lean_ctor_get(x_3, 2); -lean_inc(x_72); -x_73 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_72, x_4); -x_74 = lean_ctor_get(x_73, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_73, 1); -lean_inc(x_75); -lean_dec(x_73); +lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; size_t x_143; size_t x_144; uint8_t x_145; +x_137 = lean_ctor_get(x_3, 0); +lean_inc(x_137); +x_138 = lean_ctor_get(x_3, 1); +lean_inc(x_138); +x_139 = lean_ctor_get(x_3, 2); +lean_inc(x_139); +lean_inc(x_139); +x_140 = l_Lean_Expr_ReplaceLevelImpl_replaceUnsafeM_visit(x_1, x_2, x_139, x_4); +x_141 = lean_ctor_get(x_140, 0); +lean_inc(x_141); +x_142 = lean_ctor_get(x_140, 1); +lean_inc(x_142); +lean_dec(x_140); +x_143 = lean_ptr_addr(x_139); +lean_dec(x_139); +x_144 = lean_ptr_addr(x_141); +x_145 = lean_usize_dec_eq(x_143, x_144); +if (x_145 == 0) +{ +lean_object* x_146; lean_object* x_147; +x_146 = l_Lean_Expr_proj___override(x_137, x_138, x_141); +x_147 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_146, x_142); +return x_147; +} +else +{ +lean_object* x_148; +lean_dec(x_141); +lean_dec(x_138); +lean_dec(x_137); lean_inc(x_3); -x_76 = lean_expr_update_proj(x_3, x_74); -x_77 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_76, x_75); -return x_77; +x_148 = l_Lean_Expr_ReplaceLevelImpl_cache(x_6, x_3, x_3, x_142); +return x_148; +} } default: { -lean_object* x_78; +lean_object* x_149; lean_dec(x_1); -x_78 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_78, 0, x_3); -lean_ctor_set(x_78, 1, x_4); -return x_78; +x_149 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_149, 0, x_3); +lean_ctor_set(x_149, 1, x_4); +return x_149; } } } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_dec(x_3); lean_dec(x_1); -x_79 = lean_ctor_get(x_4, 1); -lean_inc(x_79); -x_80 = lean_array_uget(x_79, x_6); -lean_dec(x_79); -x_81 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_81, 1, x_4); -return x_81; +x_150 = lean_ctor_get(x_4, 1); +lean_inc(x_150); +x_151 = lean_array_uget(x_150, x_6); +lean_dec(x_150); +x_152 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_152, 0, x_151); +lean_ctor_set(x_152, 1, x_4); +return x_152; } } } diff --git a/stage0/stdlib/Lean/Util/Trace.c b/stage0/stdlib/Lean/Util/Trace.c index 463d48a25f98..5da92b6b2374 100644 --- a/stage0/stdlib/Lean/Util/Trace.c +++ b/stage0/stdlib/Lean/Util/Trace.c @@ -5154,7 +5154,7 @@ static lean_object* _init_l___private_Lean_Util_Trace_0__Lean_withNestedTracesFi 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_Util_Trace_0__Lean_withNestedTracesFinalizer___rarg___lambda__1___closed__1; x_2 = l___private_Lean_Util_Trace_0__Lean_withNestedTracesFinalizer___rarg___lambda__1___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Util_Trace_0__Lean_withNestedTracesFinalizer___rarg___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Widget/Basic.c b/stage0/stdlib/Lean/Widget/Basic.c index 484b5b55c122..efce0635e032 100644 --- a/stage0/stdlib/Lean/Widget/Basic.c +++ b/stage0/stdlib/Lean/Widget/Basic.c @@ -16,79 +16,77 @@ extern "C" { static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__1; lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonFVarId(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -static lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___lambda__1(size_t); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__17; +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1(lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__8; static lean_object* l_Lean_Widget_instFromJsonFVarId___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg(lean_object*, lean_object*, size_t); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__6; +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__1; +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_getStr_x3f(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg(lean_object*, lean_object*, size_t); lean_object* lean_string_append(lean_object*, lean_object*); +static lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___closed__1; +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__3; LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedInfoWithCtx; -static lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__3; -static lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__4; -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__2; +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___spec__1(lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__11; -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__3; +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___lambda__1___boxed(lean_object*); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__2; lean_object* l_Lean_Name_toString(lean_object*, uint8_t); static lean_object* l_Lean_Widget_instFromJsonFVarId___closed__3; lean_object* l_Std_mkHashMapImp___rarg(lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__10; LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonMVarId(lean_object*); -static lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__2(lean_object*, lean_object*, lean_object*, size_t); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__1; +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__13; -static lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__3; -static lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__5; -static lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__1; +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__4; +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__3; static lean_object* l_Lean_Widget_instFromJsonFVarId___closed__4; +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4_; +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76_; static uint32_t l_Lean_Widget_instInhabitedInfoWithCtx___closed__7; -static lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instFromJsonFVarId___closed__5; -static lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__6; LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonMVarId(lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__16; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; static lean_object* l_Lean_Widget_instFromJsonFVarId___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__4; +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__1; static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__9; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg(lean_object*, lean_object*, size_t); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__19; lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__6; lean_object* l_Lean_Syntax_decodeNameLit(lean_object*); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__2; static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__15; static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__18; static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__5; static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__14; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__5; LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonFVarId(lean_object*); -static lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__1; -static lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__2(lean_object*, lean_object*, lean_object*, size_t); uint32_t lean_uint32_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg(lean_object*, lean_object*, size_t); static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__2; -static lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__3; lean_object* l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; -static lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___boxed(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__3; static lean_object* l_Lean_Widget_instInhabitedInfoWithCtx___closed__12; uint8_t lean_string_dec_eq(lean_object*, lean_object*); static lean_object* _init_l_Lean_Widget_instInhabitedInfoWithCtx___closed__1() { @@ -342,7 +340,7 @@ x_1 = l_Lean_Widget_instInhabitedInfoWithCtx___closed__19; return x_1; } } -static lean_object* _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__1() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__1() { _start: { lean_object* x_1; @@ -350,17 +348,17 @@ x_1 = lean_mk_string_from_bytes("Lean", 4); return x_1; } } -static lean_object* _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__2() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__1; +x_2 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__3() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__3() { _start: { lean_object* x_1; @@ -368,17 +366,17 @@ x_1 = lean_mk_string_from_bytes("Widget", 6); return x_1; } } -static lean_object* _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__4() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__2; -x_2 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__3; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__2; +x_2 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__5() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__5() { _start: { lean_object* x_1; @@ -386,141 +384,163 @@ x_1 = lean_mk_string_from_bytes("InfoWithCtx", 11); return x_1; } } -static lean_object* _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__6() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__4; -x_2 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__5; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__4; +x_2 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg(lean_object* x_1, lean_object* x_2, size_t x_3) { _start: { lean_object* x_4; lean_object* x_5; -x_4 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__6; -x_5 = l_Lean_Server_WithRpcRef_encodeUnsafe___rarg(x_2, lean_box(0), x_1, x_4, x_3); +x_4 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__6; +x_5 = l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg(x_1, x_2, lean_box(0), x_4, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___boxed), 3, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___lambda__1(size_t x_1) { _start: { -lean_object* x_4; -x_4 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; +lean_object* x_2; lean_object* x_3; +x_2 = lean_box_usize(x_1); +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg(lean_object* x_1, lean_object* x_2, size_t x_3) { +static lean_object* _init_l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___closed__1() { _start: { -lean_object* x_4; lean_object* x_5; -x_4 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__6; -x_5 = l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg(x_1, x_2, lean_box(0), x_4, x_3); -return x_5; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___lambda__1___boxed), 1, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___boxed), 3, 0); -return x_2; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_apply_2(x_5, x_3, x_4); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +lean_dec(x_8); +x_10 = l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___closed__1; +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_10, x_6); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1(lean_object* x_1) { _start: { -size_t x_4; lean_object* x_5; -x_4 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_5 = l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg(x_1, x_2, x_4); -return x_5; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg), 4, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; -x_5 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg(x_2, x_3, x_4); +lean_object* x_4; lean_object* x_5; +x_4 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__6; +x_5 = l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg(x_1, x_2, x_4, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4) { +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2(lean_object* x_1) { _start: { -lean_object* x_5; -x_5 = l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg(x_2, x_3, x_4); -return x_5; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___rarg), 3, 0); +return x_2; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__1() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__2() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__2___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__3() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__1; -x_2 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__2; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__1; +x_2 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__2; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4_() { _start: { lean_object* x_1; -x_1 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__3; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__3; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___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_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; -x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_2); +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg(x_1, x_2, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___lambda__1___boxed(lean_object* x_1) { _start: { -size_t x_5; lean_object* x_6; -x_5 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_6 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___lambda__2(x_1, x_2, x_3, x_5); -return x_6; +size_t x_2; lean_object* x_3; +x_2 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_3 = l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___lambda__1(x_2); +return x_3; } } -static lean_object* _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__1() { +static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4_; +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__1() { _start: { lean_object* x_1; @@ -528,138 +548,132 @@ x_1 = lean_mk_string_from_bytes("MessageData", 11); return x_1; } } -static lean_object* _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__2() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__2; -x_2 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__1; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__2; +x_2 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg(lean_object* x_1, lean_object* x_2, size_t x_3) { _start: { lean_object* x_4; lean_object* x_5; -x_4 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__2; -x_5 = l_Lean_Server_WithRpcRef_encodeUnsafe___rarg(x_2, lean_box(0), x_1, x_4, x_3); +x_4 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__2; +x_5 = l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg(x_1, x_2, lean_box(0), x_4, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___boxed), 3, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_4; -x_4 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg(x_1, x_2, x_3); +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_apply_2(x_5, x_3, x_4); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg(lean_object* x_1, lean_object* x_2, size_t x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; -x_4 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__2; -x_5 = l_Lean_Server_WithRpcRef_decodeUnsafeAs___rarg(x_1, x_2, lean_box(0), x_4, x_3); -return x_5; +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +lean_dec(x_8); +x_10 = l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___closed__1; +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_10, x_6); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___spec__1___rarg), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -size_t x_4; lean_object* x_5; -x_4 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_5 = l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg(x_1, x_2, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; -x_5 = l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg(x_2, x_3, x_4); +lean_object* x_4; lean_object* x_5; +x_4 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__2; +x_5 = l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___spec__1___rarg(x_1, x_2, x_4, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4) { +LEAN_EXPORT lean_object* l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2(lean_object* x_1) { _start: { -lean_object* x_5; -x_5 = l_Lean_Widget_decodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg(x_2, x_3, x_4); -return x_5; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2___rarg), 3, 0); +return x_2; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__1() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__1___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__2), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__2() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__2___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1), 1, 0); return x_1; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__3() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__1; -x_2 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__2; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__1; +x_2 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__2; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef() { +static lean_object* _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76_() { _start: { lean_object* x_1; -x_1 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__3; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__3; return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___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_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; -x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__1(x_1, x_2, x_3, x_4); -lean_dec(x_2); +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg(x_1, x_2, x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef() { _start: { -size_t x_5; lean_object* x_6; -x_5 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_6 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___lambda__2(x_1, x_2, x_3, x_5); -return x_6; +lean_object* x_1; +x_1 = l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76_; +return x_1; } } LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonFVarId(lean_object* x_1) { @@ -1046,36 +1060,42 @@ l_Lean_Widget_instInhabitedInfoWithCtx___closed__19 = _init_l_Lean_Widget_instIn lean_mark_persistent(l_Lean_Widget_instInhabitedInfoWithCtx___closed__19); l_Lean_Widget_instInhabitedInfoWithCtx = _init_l_Lean_Widget_instInhabitedInfoWithCtx(); lean_mark_persistent(l_Lean_Widget_instInhabitedInfoWithCtx); -l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__1 = _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__1(); -lean_mark_persistent(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__1); -l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__2 = _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__2(); -lean_mark_persistent(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__2); -l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__3 = _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__3(); -lean_mark_persistent(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__3); -l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__4 = _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__4(); -lean_mark_persistent(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__4); -l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__5 = _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__5(); -lean_mark_persistent(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__5); -l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__6 = _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__6(); -lean_mark_persistent(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_4____rarg___closed__6); -l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__1 = _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__1(); -lean_mark_persistent(l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__1); -l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__2 = _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__2(); -lean_mark_persistent(l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__2); -l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__3 = _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__3(); -lean_mark_persistent(l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef___closed__3); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__1 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__1(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__1); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__2 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__2(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__2); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__3 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__3(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__3); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__4 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__4(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__4); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__5 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__5(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__5); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__6 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__6(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__1___rarg___closed__6); +l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___closed__1 = _init_l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___closed__1(); +lean_mark_persistent(l_Lean_Server_WithRpcRef_encodeUnsafe___at_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____elambda__2___spec__1___rarg___closed__1); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__1 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__1(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__1); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__2 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__2(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__2); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__3 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__3(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4____closed__3); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4_ = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4_(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_4_); l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef = _init_l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef(); lean_mark_persistent(l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef); -l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__1 = _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__1(); -lean_mark_persistent(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__1); -l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__2 = _init_l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__2(); -lean_mark_persistent(l_Lean_Widget_encodeUnsafe____x40_Lean_Widget_Basic___hyg_144____rarg___closed__2); -l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__1 = _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__1(); -lean_mark_persistent(l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__1); -l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__2 = _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__2(); -lean_mark_persistent(l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__2); -l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__3 = _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__3(); -lean_mark_persistent(l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef___closed__3); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__1 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__1(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__1); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__2 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__2(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____elambda__1___rarg___closed__2); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__1 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__1(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__1); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__2 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__2(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__2); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__3 = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__3(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76____closed__3); +l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76_ = _init_l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76_(); +lean_mark_persistent(l_Lean_Widget_unsafeInst____x40_Lean_Widget_Basic___hyg_76_); l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef = _init_l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef(); lean_mark_persistent(l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef); l_Lean_Widget_instFromJsonFVarId___closed__1 = _init_l_Lean_Widget_instFromJsonFVarId___closed__1(); diff --git a/stage0/stdlib/Lean/Widget/InteractiveCode.c b/stage0/stdlib/Lean/Widget/InteractiveCode.c index f7b98749b88e..08205fcb3970 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveCode.c +++ b/stage0/stdlib/Lean/Widget/InteractiveCode.c @@ -13,93 +13,110 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__2___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___closed__3; lean_object* l_Lean_KVMap_setBool(lean_object*, lean_object*, uint8_t); static lean_object* l_Lean_Widget_ppExprTagged___closed__6; lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__19; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_ppExprTagged(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Json_getObjValAs_x3f(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Std_Format_defWidth; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket(lean_object*); lean_object* l_Lean_Widget_TaggedText_prettyTagged(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_RBMap_ofList___at_Lean_Widget_ppExprTagged___spec__1(lean_object*); +lean_object* l_Lean_SubExpr_Pos_toString(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__2(lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_RBNode_insert___at_Lean_Widget_ppExprTagged___spec__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket___closed__1; +lean_object* l_Lean_Json_getStr_x3f(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket; +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60_(lean_object*); lean_object* l_List_join___rarg(lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__11; extern lean_object* l_Lean_SubExpr_Pos_root; lean_object* l_Lean_Widget_TaggedText_stripTags___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo; static lean_object* l_Lean_Widget_ppExprTagged___closed__7; static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__13; static lean_object* l_Lean_Widget_ppExprTagged___closed__10; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__1(size_t, lean_object*, lean_object*); lean_object* l_Std_RBNode_setBlack___rarg(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__3___rarg(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_Widget_instInhabitedSubexprInfo___closed__12; static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__6; static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__1; lean_object* l_Lean_Widget_TaggedText_rewrite___rarg(lean_object*, lean_object*); +lean_object* l_Lean_SubExpr_Pos_fromString_x3f(lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__2(lean_object*, lean_object*, size_t); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__17; LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Widget_tagExprInfos_go___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_tagExprInfos(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_tagExprInfos_go(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__8; static lean_object* l_Lean_Widget_ppExprTagged___closed__5; static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__4; lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__2; +static lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___closed__2; static uint32_t l_Lean_Widget_instInhabitedSubexprInfo___closed__7; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1065_(size_t); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_CodeWithInfos_pretty(lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket___closed__1; static lean_object* l_Lean_Widget_ppExprTagged___closed__12; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__9; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__2; static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__3; static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__15; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_tagExprInfos_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_RBNode_find___at_Lean_Widget_tagExprInfos_go___spec__1___boxed(lean_object*, lean_object*); +extern lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__5; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__2(lean_object*); +lean_object* l_Lean_Json_getObjValD(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__5___boxed(lean_object*, lean_object*, lean_object*); uint8_t l_Std_RBNode_isRed___rarg(lean_object*); extern lean_object* l_Lean_KVMap_empty; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__4(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__18; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__3(lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__14; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_194____rarg(lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1027_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_RBNode_ins___at_Lean_Widget_ppExprTagged___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedSubexprInfo; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__10; static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__20; static lean_object* l_Lean_Widget_ppExprTagged___closed__2; static lean_object* l_Lean_Widget_ppExprTagged___closed__4; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____boxed(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__1; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Widget_ppExprTagged___closed__9; +static lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__2; static lean_object* l_Lean_Widget_ppExprTagged___closed__8; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__4(lean_object*); static lean_object* l_Lean_Widget_ppExprTagged___closed__3; static lean_object* l_Lean_Widget_ppExprTagged___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_ppExprTagged___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1(lean_object*, lean_object*); uint32_t lean_uint32_of_nat(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_ppExprTagged___closed__11; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedSubexprInfo___closed__16; lean_object* l_Lean_PrettyPrinter_ppExprWithInfos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_194_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_115_(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* _init_l_Lean_Widget_instInhabitedSubexprInfo___closed__1() { _start: @@ -364,7 +381,53 @@ x_1 = l_Lean_Widget_instInhabitedSubexprInfo___closed__20; return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +x_4 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1027_(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +x_4 = l_Lean_Json_getStr_x3f(x_3); +lean_dec(x_3); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_5; +x_5 = !lean_is_exclusive(x_4); +if (x_5 == 0) +{ +return x_4; +} +else +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_7, 0, x_6); +return x_7; +} +} +else +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_4, 0); +lean_inc(x_8); +lean_dec(x_4); +x_9 = l_Lean_SubExpr_Pos_fromString_x3f(x_8); +return x_9; +} +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__1() { _start: { lean_object* x_1; @@ -372,7 +435,7 @@ x_1 = lean_mk_string_from_bytes("info", 4); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__2() { +static lean_object* _init_l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__2() { _start: { lean_object* x_1; @@ -380,190 +443,251 @@ x_1 = lean_mk_string_from_bytes("subexprPos", 10); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60_(lean_object* x_1) { _start: { -lean_object* x_4; lean_object* x_5; -x_4 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__1; -x_5 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_1, x_4); -if (lean_obj_tag(x_5) == 0) +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1(x_1, x_2); +if (lean_obj_tag(x_3) == 0) { -uint8_t x_6; -lean_dec(x_2); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) { -return x_5; +return x_3; } else { -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -lean_dec(x_5); -x_10 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__2; -x_11 = l_Lean_Json_getObjValAs_x3f(x_3, lean_box(0), x_2, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +x_8 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__2; +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__2(x_1, x_8); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_12; -lean_dec(x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_10; +lean_dec(x_7); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -return x_11; +return x_9; } else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_11); -if (x_15 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_9); +if (x_13 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_11, 0); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_9); -lean_ctor_set(x_17, 1, x_16); -lean_ctor_set(x_11, 0, x_17); -return x_11; +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_9, 0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_7); +lean_ctor_set(x_15, 1, x_14); +lean_ctor_set(x_9, 0, x_15); +return x_9; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_11, 0); -lean_inc(x_18); -lean_dec(x_11); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_9); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_20, 0, x_19); -return x_20; +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_9, 0); +lean_inc(x_16); +lean_dec(x_9); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_7); +lean_ctor_set(x_17, 1, x_16); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; } } } } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___boxed), 3, 0); +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_4; -x_4 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg(x_1, x_2, x_3); -lean_dec(x_3); -return x_4; +lean_object* x_3; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____spec__2(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____boxed(lean_object* x_1) { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___boxed), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; +lean_object* x_2; +x_2 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60_(x_1); +lean_dec(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket___closed__1() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket___rarg), 2, 0); -return x_3; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____boxed), 1, 0); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_194____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket() { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_4 = lean_ctor_get(x_3, 0); -lean_inc(x_4); -x_5 = lean_apply_1(x_1, x_4); -x_6 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__1; -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_9, 0, x_7); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_ctor_get(x_3, 1); -lean_inc(x_10); -lean_dec(x_3); -x_11 = lean_apply_1(x_2, x_10); -x_12 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__2; +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_115_(lean_object* x_1) { +_start: +{ +lean_object* x_2; size_t x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_4 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1065_(x_3); +x_5 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__1; +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_5); +lean_ctor_set(x_6, 1, x_4); +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_6); +lean_ctor_set(x_8, 1, x_7); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +lean_dec(x_1); +x_10 = l_Lean_SubExpr_Pos_toString(x_9); +x_11 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__2; x_13 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_13, 0, x_12); lean_ctor_set(x_13, 1, x_11); x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_8); +lean_ctor_set(x_14, 1, x_7); x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_8); +lean_ctor_set(x_15, 1, x_7); x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_9); +lean_ctor_set(x_16, 0, x_8); lean_ctor_set(x_16, 1, x_15); x_17 = l_List_join___rarg(x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_194_(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket___closed__1() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_194____rarg), 3, 0); -return x_3; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_115_), 1, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2) { +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket() { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_194____rarg), 3, 2); -lean_closure_set(x_3, 0, x_1); -lean_closure_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket___closed__1; +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket___rarg), 2, 0); -return x_3; +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__1___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -613,15 +737,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__1___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__2___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -671,114 +795,203 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__2___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__3___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; lean_dec(x_4); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_2); -lean_ctor_set(x_6, 1, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_1, 0); lean_inc(x_7); lean_dec(x_1); -x_8 = lean_ctor_get(x_2, 1); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); -lean_dec(x_2); -lean_inc(x_3); -x_9 = lean_apply_4(x_7, lean_box(0), x_3, x_4, x_8); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__1), 3, 2); -lean_closure_set(x_10, 0, x_3); -lean_closure_set(x_10, 1, x_6); -x_11 = lean_apply_4(x_5, lean_box(0), lean_box(0), x_9, x_10); -return x_11; +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: +} +else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_7 = lean_ctor_get(x_4, 1); -lean_inc(x_7); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_15; lean_object* x_16; lean_dec(x_1); -x_9 = lean_ctor_get(x_6, 0); -lean_inc(x_9); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_box_usize(x_1); +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_2, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__2(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); lean_inc(x_4); -x_10 = lean_apply_4(x_8, lean_box(0), x_4, x_5, x_9); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__1___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_4, 0); lean_inc(x_7); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__2), 6, 5); +lean_inc(x_2); +x_8 = lean_apply_4(x_6, lean_box(0), x_2, x_3, x_7); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__2___boxed), 3, 2); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_2); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__2___rarg), 5, 4); lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, x_6); -lean_closure_set(x_11, 2, x_4); -lean_closure_set(x_11, 3, x_5); -lean_closure_set(x_11, 4, x_7); -x_12 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_10, x_11); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +x_6 = lean_apply_2(x_2, lean_box(0), x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); x_5 = lean_ctor_get(x_2, 0); lean_inc(x_5); -lean_dec(x_2); x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); lean_dec(x_5); +lean_inc(x_4); x_7 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__4), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__3___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_6 = lean_ctor_get(x_1, 1); +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_5 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_6 = lean_ctor_get(x_5, 1); lean_inc(x_6); -lean_dec(x_1); -x_7 = lean_ctor_get(x_2, 1); +x_7 = lean_ctor_get(x_4, 0); lean_inc(x_7); -lean_dec(x_2); -lean_inc(x_3); -x_8 = lean_apply_4(x_6, lean_box(0), x_3, x_4, x_7); -lean_inc(x_3); -x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__4), 3, 2); -lean_closure_set(x_9, 0, x_5); -lean_closure_set(x_9, 1, x_3); -x_10 = lean_ctor_get(x_3, 1); +lean_inc(x_2); +x_8 = lean_apply_4(x_6, lean_box(0), x_2, x_3, x_7); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__5___boxed), 3, 2); +lean_closure_set(x_9, 0, x_4); +lean_closure_set(x_9, 1, x_2); +x_10 = lean_ctor_get(x_2, 1); lean_inc(x_10); -x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_11, 0, x_3); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfo___spec__4___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); lean_closure_set(x_11, 1, lean_box(0)); lean_closure_set(x_11, 2, lean_box(0)); lean_closure_set(x_11, 3, x_9); @@ -786,59 +999,70 @@ x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingSubexprInfo___closed__1() { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__3), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingSubexprInfo___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__6), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingSubexprInfo___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingSubexprInfo___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingSubexprInfo___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingSubexprInfo() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingSubexprInfo___closed__3; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_1); lean_dec(x_1); -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_inc(x_5); -lean_inc(x_4); -x_9 = lean_apply_4(x_7, lean_box(0), x_4, x_5, x_8); -lean_inc(x_4); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__5), 5, 4); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_6); -lean_closure_set(x_10, 2, x_4); -lean_closure_set(x_10, 3, x_5); -x_11 = lean_ctor_get(x_4, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_12, 0, x_4); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); -return x_13; +x_5 = l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__1(x_4, x_2, x_3); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__2___boxed(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_inc(x_3); -lean_inc(x_1); -x_4 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__3), 6, 2); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_3); -x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg___lambda__6), 6, 2); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_3); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_4); -lean_ctor_set(x_6, 1, x_5); -return x_6; +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__2(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingSubexprInfoRpcEncodingPacket___rarg), 3, 0); -return x_2; +lean_object* x_4; +x_4 = l_Lean_Widget_instRpcEncodingSubexprInfo___lambda__5(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; } } LEAN_EXPORT lean_object* l_Lean_Widget_CodeWithInfos_pretty(lean_object* x_1) { @@ -3817,10 +4041,26 @@ l_Lean_Widget_instInhabitedSubexprInfo___closed__20 = _init_l_Lean_Widget_instIn lean_mark_persistent(l_Lean_Widget_instInhabitedSubexprInfo___closed__20); l_Lean_Widget_instInhabitedSubexprInfo = _init_l_Lean_Widget_instInhabitedSubexprInfo(); lean_mark_persistent(l_Lean_Widget_instInhabitedSubexprInfo); -l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__1); -l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__2 = _init_l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__2(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_93____rarg___closed__2); +l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__1 = _init_l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__1); +l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__2 = _init_l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__2(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60____closed__2); +l_Lean_Widget_instFromJsonRpcEncodingPacket___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket); +l_Lean_Widget_instToJsonRpcEncodingPacket___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket = _init_l_Lean_Widget_instToJsonRpcEncodingPacket(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket); +l_Lean_Widget_instRpcEncodingSubexprInfo___closed__1 = _init_l_Lean_Widget_instRpcEncodingSubexprInfo___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingSubexprInfo___closed__1); +l_Lean_Widget_instRpcEncodingSubexprInfo___closed__2 = _init_l_Lean_Widget_instRpcEncodingSubexprInfo___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingSubexprInfo___closed__2); +l_Lean_Widget_instRpcEncodingSubexprInfo___closed__3 = _init_l_Lean_Widget_instRpcEncodingSubexprInfo___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingSubexprInfo___closed__3); +l_Lean_Widget_instRpcEncodingSubexprInfo = _init_l_Lean_Widget_instRpcEncodingSubexprInfo(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingSubexprInfo); l_Lean_Widget_ppExprTagged___closed__1 = _init_l_Lean_Widget_ppExprTagged___closed__1(); lean_mark_persistent(l_Lean_Widget_ppExprTagged___closed__1); l_Lean_Widget_ppExprTagged___closed__2 = _init_l_Lean_Widget_ppExprTagged___closed__2(); diff --git a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c index 716adf67191a..56b0078470d0 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c +++ b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c @@ -13,258 +13,623 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__20___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___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_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedEmbedFmt; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__3; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29(lean_object*); size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11(lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed___closed__1; +lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractive___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46(lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__6; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52(lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__3; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1(lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(lean_object*, size_t, size_t, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9; static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__5; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__11(lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); extern lean_object* l_Std_Format_defWidth; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getNat_x3f(lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_TaggedText_prettyTagged(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1642_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__6; +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Except_orElseLazy___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__21(lean_object*); static lean_object* l_Lean_Widget_msgToInteractive___lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___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_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__9(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__5(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10; +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_rewriteM___at_Lean_Widget_msgToInteractive___spec__2(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getStr_x3f(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__5(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__4; +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17(lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__8; +lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_msgToInteractive___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_msgToInteractive___lambda__1___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__9; -static lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_withIgnoreTags(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__2; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__5(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractive___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_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___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__3; static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); lean_object* l_List_join___rarg(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__5; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_TaggedText_stripTags___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__11(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___closed__5; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___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_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__5; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static uint32_t l_Lean_Widget_instInhabitedEmbedFmt___closed__7; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_InteractiveGoal_pretty(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8(lean_object*); lean_object* l_Lean_ppGoal(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___closed__3; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__8(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__5___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractiveDiagnostic(lean_object*, lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__11(lean_object*, lean_object*); static lean_object* l_Lean_Widget_msgToInteractive___lambda__1___closed__4; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__20(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__15; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__2(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25(lean_object*); lean_object* l_Lean_Json_parseTagged(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14(lean_object*); lean_object* l_Lean_Expr_mvar___override(lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__5; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52(lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__8; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__15(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__8; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_TaggedText_rewrite___rarg(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Json_setObjVal_x21___spec__1(lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__4; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__8; -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__4; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2(lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7; +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1036____spec__3(lean_object*, lean_object*); lean_object* l_Std_mkHashMapImp___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2(lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__18; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37(lean_object*); lean_object* l_Lean_Widget_tagExprInfos_go(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__14; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__6(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__9; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__8(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__3(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__2(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2161____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___boxed(lean_object*, lean_object*); lean_object* lean_format_pretty(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__4; +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_pure___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___spec__1(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_pushEmbed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__3; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__5; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__22(lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__5___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__19(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49(lean_object*); lean_object* lean_expr_dbg_to_string(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__8(lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__3; -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__5; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34(lean_object*); +lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1065_(size_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1(size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__5(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21(lean_object*); static lean_object* l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50(lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1036____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedMsgEmbed___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__6(lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__12; -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux___closed__1; size_t lean_usize_of_nat(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractive(lean_object*, uint8_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__12(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__5; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__20(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__19; -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +extern lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4(lean_object*, lean_object*, size_t); static lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___closed__4; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__1; static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__20; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__22___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__4; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__23(lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__10; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__6(lean_object*); -lean_object* l_Lean_Json_opt___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Json_getObjValD(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__1; +lean_object* l_Lean_JsonNumber_fromNat(lean_object*); static lean_object* l_panic___at_Lean_Widget_msgToInteractive___spec__1___closed__1; -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__16(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__6; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__12(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__10(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__7(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__10; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_lift___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___spec__3(lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__6; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__6(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_mkPPContext___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__16; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___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_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__18(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320____closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5(lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); static lean_object* l_Lean_Widget_instInhabitedMsgEmbed___closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9(lean_object*); +lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1027_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10(lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2131____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); lean_object* l_Lean_ppTerm(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, uint8_t); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___spec__4(uint8_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1(lean_object*); lean_object* l_EStateM_instInhabitedEStateM___rarg(lean_object*, lean_object*); +lean_object* l_Lean_Syntax_decodeNameLit(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13(lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__7___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1642____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__12(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__6___rarg(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed___closed__3; static lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14(lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocation____x40_Lean_Data_Lsp_Basic___hyg_940____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___spec__2(uint8_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedMsgEmbed; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__24(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_mkPPContext(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__3(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__7(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__6___rarg(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8; +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__7; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed; static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__13; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__5; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4(lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Widget_msgToInteractive___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4(lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(lean_object*); extern lean_object* l_IO_instInhabitedError; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_leanPosToLspPos(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive___spec__3(lean_object*, size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___lambda__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_pure___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___spec__1___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13(lean_object*, lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1036____spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31(lean_object*); uint32_t lean_uint32_of_nat(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____rarg(lean_object*, lean_object*); lean_object* l_Lean_Elab_ContextInfo_runMetaM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1036____spec__5(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___closed__7; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__11; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__5(lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__2(lean_object*, lean_object*); lean_object* l_Lean_Level_format(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +extern lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_StateT_lift___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___spec__3___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36(lean_object*); size_t lean_usize_of_nat(lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__7; lean_object* lean_nat_to_int(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__18(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_formatStxAux(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___lambda__1___closed__1; +static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__7(lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedEmbedFmt___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19(lean_object*); lean_object* l_Lean_PrettyPrinter_ppExprWithInfos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__13(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Widget_msgToInteractiveDiagnostic___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___lambda__1(lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static size_t l_Lean_Widget_instInhabitedEmbedFmt___closed__17; static lean_object* _init_l_Lean_Widget_instInhabitedMsgEmbed___closed__1() { _start: @@ -302,7 +667,7 @@ x_1 = l_Lean_Widget_instInhabitedMsgEmbed___closed__3; return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__1() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -310,25 +675,25 @@ x_1 = lean_mk_string_from_bytes("no inductive constructor matched", 32); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__2() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__1; +x_1 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__1; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__2; +x_2 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__2; return x_2; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__1() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__1() { _start: { lean_object* x_1; @@ -336,15 +701,15 @@ x_1 = lean_mk_string_from_bytes("lazyTrace", 9); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___boxed), 1, 0); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__3() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__3() { _start: { lean_object* x_1; @@ -352,7 +717,7 @@ x_1 = lean_mk_string_from_bytes("Init.Util", 9); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__4() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__4() { _start: { lean_object* x_1; @@ -360,7 +725,7 @@ x_1 = lean_mk_string_from_bytes("getElem!", 8); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__5() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__5() { _start: { lean_object* x_1; @@ -368,720 +733,974 @@ x_1 = lean_mk_string_from_bytes("index out of bounds", 19); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__3; -x_2 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_1 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__3; +x_2 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__4; +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); -x_5 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__5; +x_5 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7() { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__1; -x_8 = lean_unsigned_to_nat(3u); -x_9 = l_Lean_Json_parseTagged(x_1, x_7, x_8, x_2); -if (lean_obj_tag(x_9) == 0) -{ -uint8_t x_10; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_12 = l_Except_orElseLazy___rarg(x_9, x_11); -return x_12; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("[anonymous]", 11); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8() { +_start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_9, 0); -lean_inc(x_13); -lean_dec(x_9); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_16 = l_Except_orElseLazy___rarg(x_14, x_15); -return x_16; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("`", 1); +return x_1; } } -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_87; uint8_t x_88; -x_17 = lean_ctor_get(x_9, 0); -lean_inc(x_17); -lean_dec(x_9); -x_18 = lean_array_get_size(x_17); -x_87 = lean_unsigned_to_nat(0u); -x_88 = lean_nat_dec_lt(x_87, x_18); -if (x_88 == 0) +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9() { +_start: { -lean_object* x_89; lean_object* x_90; -x_89 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6; -x_90 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_89); -x_19 = x_90; -goto block_86; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("expected a `Name`, got '", 24); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10() { +_start: { -lean_object* x_91; -x_91 = lean_array_fget(x_17, x_87); -x_19 = x_91; -goto block_86; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("'", 1); +return x_1; } -block_86: +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -lean_object* x_20; -x_20 = lean_apply_1(x_3, x_19); -if (lean_obj_tag(x_20) == 0) +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__1; +x_5 = lean_unsigned_to_nat(3u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +if (lean_obj_tag(x_6) == 0) { -uint8_t x_21; -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_5); -lean_dec(x_4); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_23 = l_Except_orElseLazy___rarg(x_20, x_22); -return x_23; +lean_object* x_8; lean_object* x_9; +x_8 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_9 = l_Except_orElseLazy___rarg(x_6, x_8); +return x_9; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_20, 0); -lean_inc(x_24); -lean_dec(x_20); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -x_26 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_27 = l_Except_orElseLazy___rarg(x_25, x_26); -return x_27; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_13 = l_Except_orElseLazy___rarg(x_11, x_12); +return x_13; } } else { -lean_object* x_28; lean_object* x_29; lean_object* x_81; uint8_t x_82; -x_28 = lean_ctor_get(x_20, 0); -lean_inc(x_28); -lean_dec(x_20); -x_81 = lean_unsigned_to_nat(1u); -x_82 = lean_nat_dec_lt(x_81, x_18); -if (x_82 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_159; uint8_t x_160; +x_14 = lean_ctor_get(x_6, 0); +lean_inc(x_14); +lean_dec(x_6); +x_15 = lean_array_get_size(x_14); +x_159 = lean_unsigned_to_nat(0u); +x_160 = lean_nat_dec_lt(x_159, x_15); +if (x_160 == 0) { -lean_object* x_83; lean_object* x_84; -x_83 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6; -x_84 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_83); -x_29 = x_84; -goto block_80; +lean_object* x_161; lean_object* x_162; +x_161 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6; +x_162 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_161); +x_16 = x_162; +goto block_158; } else { -lean_object* x_85; -x_85 = lean_array_fget(x_17, x_81); -x_29 = x_85; -goto block_80; +lean_object* x_163; +x_163 = lean_array_fget(x_14, x_159); +x_16 = x_163; +goto block_158; } -block_80: +block_158: { -lean_object* x_30; -x_30 = lean_apply_1(x_4, x_29); -if (lean_obj_tag(x_30) == 0) +lean_object* x_17; +x_17 = l_Lean_Json_getNat_x3f(x_16); +lean_dec(x_16); +if (lean_obj_tag(x_17) == 0) { -uint8_t x_31; -lean_dec(x_28); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_5); -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) +uint8_t x_18; +lean_dec(x_15); +lean_dec(x_14); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_33 = l_Except_orElseLazy___rarg(x_30, x_32); -return x_33; +lean_object* x_19; lean_object* x_20; +x_19 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_20 = l_Except_orElseLazy___rarg(x_17, x_19); +return x_20; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_30, 0); -lean_inc(x_34); -lean_dec(x_30); -x_35 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_35, 0, x_34); -x_36 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_37 = l_Except_orElseLazy___rarg(x_35, x_36); -return x_37; +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_17, 0); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_24 = l_Except_orElseLazy___rarg(x_22, x_23); +return x_24; } } else { -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = lean_ctor_get(x_30, 0); -lean_inc(x_38); -lean_dec(x_30); -x_39 = lean_unsigned_to_nat(2u); -x_40 = lean_nat_dec_lt(x_39, x_18); -lean_dec(x_18); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_object* x_25; lean_object* x_26; lean_object* x_69; uint8_t x_70; +x_25 = lean_ctor_get(x_17, 0); +lean_inc(x_25); lean_dec(x_17); -x_41 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6; -x_42 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_41); -x_43 = lean_apply_1(x_5, x_42); -if (lean_obj_tag(x_43) == 0) +x_69 = lean_unsigned_to_nat(1u); +x_70 = lean_nat_dec_lt(x_69, x_15); +if (x_70 == 0) { -uint8_t x_44; -lean_dec(x_38); -lean_dec(x_28); -x_44 = !lean_is_exclusive(x_43); -if (x_44 == 0) +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6; +x_72 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_71); +x_73 = l_Lean_Json_getStr_x3f(x_72); +if (lean_obj_tag(x_73) == 0) { -lean_object* x_45; lean_object* x_46; -x_45 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_46 = l_Except_orElseLazy___rarg(x_43, x_45); -return x_46; +uint8_t x_74; +lean_dec(x_72); +lean_dec(x_25); +lean_dec(x_15); +lean_dec(x_14); +x_74 = !lean_is_exclusive(x_73); +if (x_74 == 0) +{ +lean_object* x_75; lean_object* x_76; +x_75 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_76 = l_Except_orElseLazy___rarg(x_73, x_75); +return x_76; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_47 = lean_ctor_get(x_43, 0); -lean_inc(x_47); -lean_dec(x_43); -x_48 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_48, 0, x_47); -x_49 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_50 = l_Except_orElseLazy___rarg(x_48, x_49); -return x_50; +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_77 = lean_ctor_get(x_73, 0); +lean_inc(x_77); +lean_dec(x_73); +x_78 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_78, 0, x_77); +x_79 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_80 = l_Except_orElseLazy___rarg(x_78, x_79); +return x_80; } } else { -uint8_t x_51; -x_51 = !lean_is_exclusive(x_43); -if (x_51 == 0) +uint8_t x_81; +x_81 = !lean_is_exclusive(x_73); +if (x_81 == 0) { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_43, 0); -x_53 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_53, 0, x_28); -lean_ctor_set(x_53, 1, x_38); -lean_ctor_set(x_53, 2, x_52); -lean_ctor_set(x_43, 0, x_53); -x_54 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_55 = l_Except_orElseLazy___rarg(x_43, x_54); -return x_55; +lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_82 = lean_ctor_get(x_73, 0); +x_83 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7; +x_84 = lean_string_dec_eq(x_82, x_83); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8; +x_86 = lean_string_append(x_85, x_82); +lean_dec(x_82); +x_87 = l_Lean_Syntax_decodeNameLit(x_86); +if (lean_obj_tag(x_87) == 0) +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +lean_dec(x_25); +lean_dec(x_15); +lean_dec(x_14); +x_88 = lean_unsigned_to_nat(80u); +x_89 = l_Lean_Json_pretty(x_72, x_88); +x_90 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9; +x_91 = lean_string_append(x_90, x_89); +lean_dec(x_89); +x_92 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10; +x_93 = lean_string_append(x_91, x_92); +lean_ctor_set_tag(x_73, 0); +lean_ctor_set(x_73, 0, x_93); +x_94 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_95 = l_Except_orElseLazy___rarg(x_73, x_94); +return x_95; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_56 = lean_ctor_get(x_43, 0); -lean_inc(x_56); -lean_dec(x_43); -x_57 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_57, 0, x_28); -lean_ctor_set(x_57, 1, x_38); -lean_ctor_set(x_57, 2, x_56); -x_58 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_58, 0, x_57); -x_59 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_60 = l_Except_orElseLazy___rarg(x_58, x_59); -return x_60; -} +lean_object* x_96; +lean_free_object(x_73); +lean_dec(x_72); +x_96 = lean_ctor_get(x_87, 0); +lean_inc(x_96); +lean_dec(x_87); +x_26 = x_96; +goto block_68; } } else { -lean_object* x_61; lean_object* x_62; -x_61 = lean_array_fget(x_17, x_39); -lean_dec(x_17); -x_62 = lean_apply_1(x_5, x_61); -if (lean_obj_tag(x_62) == 0) -{ -uint8_t x_63; -lean_dec(x_38); -lean_dec(x_28); -x_63 = !lean_is_exclusive(x_62); -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; -x_64 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_65 = l_Except_orElseLazy___rarg(x_62, x_64); -return x_65; +lean_object* x_97; +lean_free_object(x_73); +lean_dec(x_82); +lean_dec(x_72); +x_97 = lean_box(0); +x_26 = x_97; +goto block_68; +} } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_66 = lean_ctor_get(x_62, 0); -lean_inc(x_66); -lean_dec(x_62); -x_67 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_67, 0, x_66); -x_68 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_69 = l_Except_orElseLazy___rarg(x_67, x_68); -return x_69; -} +lean_object* x_98; lean_object* x_99; uint8_t x_100; +x_98 = lean_ctor_get(x_73, 0); +lean_inc(x_98); +lean_dec(x_73); +x_99 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7; +x_100 = lean_string_dec_eq(x_98, x_99); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_101 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8; +x_102 = lean_string_append(x_101, x_98); +lean_dec(x_98); +x_103 = l_Lean_Syntax_decodeNameLit(x_102); +if (lean_obj_tag(x_103) == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +lean_dec(x_25); +lean_dec(x_15); +lean_dec(x_14); +x_104 = lean_unsigned_to_nat(80u); +x_105 = l_Lean_Json_pretty(x_72, x_104); +x_106 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9; +x_107 = lean_string_append(x_106, x_105); +lean_dec(x_105); +x_108 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10; +x_109 = lean_string_append(x_107, x_108); +x_110 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_110, 0, x_109); +x_111 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_112 = l_Except_orElseLazy___rarg(x_110, x_111); +return x_112; } else { -uint8_t x_70; -x_70 = !lean_is_exclusive(x_62); -if (x_70 == 0) -{ -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_71 = lean_ctor_get(x_62, 0); -x_72 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_72, 0, x_28); -lean_ctor_set(x_72, 1, x_38); -lean_ctor_set(x_72, 2, x_71); -lean_ctor_set(x_62, 0, x_72); -x_73 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_74 = l_Except_orElseLazy___rarg(x_62, x_73); -return x_74; +lean_object* x_113; +lean_dec(x_72); +x_113 = lean_ctor_get(x_103, 0); +lean_inc(x_113); +lean_dec(x_103); +x_26 = x_113; +goto block_68; +} } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_75 = lean_ctor_get(x_62, 0); -lean_inc(x_75); -lean_dec(x_62); -x_76 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_76, 0, x_28); -lean_ctor_set(x_76, 1, x_38); -lean_ctor_set(x_76, 2, x_75); -x_77 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_77, 0, x_76); -x_78 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2; -x_79 = l_Except_orElseLazy___rarg(x_77, x_78); -return x_79; +lean_object* x_114; +lean_dec(x_98); +lean_dec(x_72); +x_114 = lean_box(0); +x_26 = x_114; +goto block_68; } } } } +else +{ +lean_object* x_115; lean_object* x_116; +x_115 = lean_array_fget(x_14, x_69); +x_116 = l_Lean_Json_getStr_x3f(x_115); +if (lean_obj_tag(x_116) == 0) +{ +uint8_t x_117; +lean_dec(x_115); +lean_dec(x_25); +lean_dec(x_15); +lean_dec(x_14); +x_117 = !lean_is_exclusive(x_116); +if (x_117 == 0) +{ +lean_object* x_118; lean_object* x_119; +x_118 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_119 = l_Except_orElseLazy___rarg(x_116, x_118); +return x_119; } +else +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; +x_120 = lean_ctor_get(x_116, 0); +lean_inc(x_120); +lean_dec(x_116); +x_121 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_121, 0, x_120); +x_122 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_123 = l_Except_orElseLazy___rarg(x_121, x_122); +return x_123; } } +else +{ +uint8_t x_124; +x_124 = !lean_is_exclusive(x_116); +if (x_124 == 0) +{ +lean_object* x_125; lean_object* x_126; uint8_t x_127; +x_125 = lean_ctor_get(x_116, 0); +x_126 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7; +x_127 = lean_string_dec_eq(x_125, x_126); +if (x_127 == 0) +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8; +x_129 = lean_string_append(x_128, x_125); +lean_dec(x_125); +x_130 = l_Lean_Syntax_decodeNameLit(x_129); +if (lean_obj_tag(x_130) == 0) +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; +lean_dec(x_25); +lean_dec(x_15); +lean_dec(x_14); +x_131 = lean_unsigned_to_nat(80u); +x_132 = l_Lean_Json_pretty(x_115, x_131); +x_133 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9; +x_134 = lean_string_append(x_133, x_132); +lean_dec(x_132); +x_135 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10; +x_136 = lean_string_append(x_134, x_135); +lean_ctor_set_tag(x_116, 0); +lean_ctor_set(x_116, 0, x_136); +x_137 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_138 = l_Except_orElseLazy___rarg(x_116, x_137); +return x_138; } +else +{ +lean_object* x_139; +lean_free_object(x_116); +lean_dec(x_115); +x_139 = lean_ctor_get(x_130, 0); +lean_inc(x_139); +lean_dec(x_130); +x_26 = x_139; +goto block_68; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("expr", 4); -return x_1; +lean_object* x_140; +lean_free_object(x_116); +lean_dec(x_125); +lean_dec(x_115); +x_140 = lean_box(0); +x_26 = x_140; +goto block_68; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___closed__1; -x_9 = lean_unsigned_to_nat(1u); -x_10 = l_Lean_Json_parseTagged(x_1, x_8, x_9, x_2); -x_11 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___boxed), 6, 5); -lean_closure_set(x_11, 0, x_1); -lean_closure_set(x_11, 1, x_2); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_4); -lean_closure_set(x_11, 4, x_5); -if (lean_obj_tag(x_10) == 0) +lean_object* x_141; lean_object* x_142; uint8_t x_143; +x_141 = lean_ctor_get(x_116, 0); +lean_inc(x_141); +lean_dec(x_116); +x_142 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7; +x_143 = lean_string_dec_eq(x_141, x_142); +if (x_143 == 0) { -uint8_t x_12; -lean_dec(x_6); -x_12 = !lean_is_exclusive(x_10); -if (x_12 == 0) +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8; +x_145 = lean_string_append(x_144, x_141); +lean_dec(x_141); +x_146 = l_Lean_Syntax_decodeNameLit(x_145); +if (lean_obj_tag(x_146) == 0) { -lean_object* x_13; -x_13 = l_Except_orElseLazy___rarg(x_10, x_11); -return x_13; +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_dec(x_25); +lean_dec(x_15); +lean_dec(x_14); +x_147 = lean_unsigned_to_nat(80u); +x_148 = l_Lean_Json_pretty(x_115, x_147); +x_149 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9; +x_150 = lean_string_append(x_149, x_148); +lean_dec(x_148); +x_151 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10; +x_152 = lean_string_append(x_150, x_151); +x_153 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_153, 0, x_152); +x_154 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_155 = l_Except_orElseLazy___rarg(x_153, x_154); +return x_155; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_10, 0); -lean_inc(x_14); -lean_dec(x_10); -x_15 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_15, 0, x_14); -x_16 = l_Except_orElseLazy___rarg(x_15, x_11); -return x_16; +lean_object* x_156; +lean_dec(x_115); +x_156 = lean_ctor_get(x_146, 0); +lean_inc(x_156); +lean_dec(x_146); +x_26 = x_156; +goto block_68; } } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_ctor_get(x_10, 0); -lean_inc(x_17); -lean_dec(x_10); -x_18 = lean_array_get_size(x_17); -x_19 = lean_unsigned_to_nat(0u); -x_20 = lean_nat_dec_lt(x_19, x_18); -lean_dec(x_18); -if (x_20 == 0) +lean_object* x_157; +lean_dec(x_141); +lean_dec(x_115); +x_157 = lean_box(0); +x_26 = x_157; +goto block_68; +} +} +} +} +block_68: { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -lean_dec(x_17); -x_21 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6; -x_22 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_21); -x_23 = lean_apply_1(x_6, x_22); -if (lean_obj_tag(x_23) == 0) +lean_object* x_27; uint8_t x_28; +x_27 = lean_unsigned_to_nat(2u); +x_28 = lean_nat_dec_lt(x_27, x_15); +lean_dec(x_15); +if (x_28 == 0) { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_14); +x_29 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6; +x_30 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_29); +x_31 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1027_(x_30); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_25; -x_25 = l_Except_orElseLazy___rarg(x_23, x_11); -return x_25; +uint8_t x_32; +lean_dec(x_26); +lean_dec(x_25); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; +x_33 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_34 = l_Except_orElseLazy___rarg(x_31, x_33); +return x_34; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_23, 0); -lean_inc(x_26); -lean_dec(x_23); -x_27 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_27, 0, x_26); -x_28 = l_Except_orElseLazy___rarg(x_27, x_11); -return x_28; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_35 = lean_ctor_get(x_31, 0); +lean_inc(x_35); +lean_dec(x_31); +x_36 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_36, 0, x_35); +x_37 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_38 = l_Except_orElseLazy___rarg(x_36, x_37); +return x_38; } } else { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_23); -if (x_29 == 0) +uint8_t x_39; +x_39 = !lean_is_exclusive(x_31); +if (x_39 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_23, 0); -x_31 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_23, 0, x_31); -x_32 = l_Except_orElseLazy___rarg(x_23, x_11); -return x_32; +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_40 = lean_ctor_get(x_31, 0); +x_41 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_41, 0, x_25); +lean_ctor_set(x_41, 1, x_26); +lean_ctor_set(x_41, 2, x_40); +lean_ctor_set(x_31, 0, x_41); +x_42 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_43 = l_Except_orElseLazy___rarg(x_31, x_42); +return x_43; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_33 = lean_ctor_get(x_23, 0); -lean_inc(x_33); -lean_dec(x_23); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -x_36 = l_Except_orElseLazy___rarg(x_35, x_11); -return x_36; +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_44 = lean_ctor_get(x_31, 0); +lean_inc(x_44); +lean_dec(x_31); +x_45 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_45, 0, x_25); +lean_ctor_set(x_45, 1, x_26); +lean_ctor_set(x_45, 2, x_44); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_48 = l_Except_orElseLazy___rarg(x_46, x_47); +return x_48; } } } else { -lean_object* x_37; lean_object* x_38; -x_37 = lean_array_fget(x_17, x_19); -lean_dec(x_17); -x_38 = lean_apply_1(x_6, x_37); -if (lean_obj_tag(x_38) == 0) +lean_object* x_49; lean_object* x_50; +x_49 = lean_array_fget(x_14, x_27); +lean_dec(x_14); +x_50 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1027_(x_49); +if (lean_obj_tag(x_50) == 0) { -uint8_t x_39; -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +uint8_t x_51; +lean_dec(x_26); +lean_dec(x_25); +x_51 = !lean_is_exclusive(x_50); +if (x_51 == 0) { -lean_object* x_40; -x_40 = l_Except_orElseLazy___rarg(x_38, x_11); -return x_40; +lean_object* x_52; lean_object* x_53; +x_52 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_53 = l_Except_orElseLazy___rarg(x_50, x_52); +return x_53; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_38, 0); -lean_inc(x_41); -lean_dec(x_38); -x_42 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_42, 0, x_41); -x_43 = l_Except_orElseLazy___rarg(x_42, x_11); -return x_43; +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_54 = lean_ctor_get(x_50, 0); +lean_inc(x_54); +lean_dec(x_50); +x_55 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_55, 0, x_54); +x_56 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_57 = l_Except_orElseLazy___rarg(x_55, x_56); +return x_57; } } else { -uint8_t x_44; -x_44 = !lean_is_exclusive(x_38); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_38, 0); -x_46 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_38, 0, x_46); -x_47 = l_Except_orElseLazy___rarg(x_38, x_11); -return x_47; +uint8_t x_58; +x_58 = !lean_is_exclusive(x_50); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_59 = lean_ctor_get(x_50, 0); +x_60 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_60, 0, x_25); +lean_ctor_set(x_60, 1, x_26); +lean_ctor_set(x_60, 2, x_59); +lean_ctor_set(x_50, 0, x_60); +x_61 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_62 = l_Except_orElseLazy___rarg(x_50, x_61); +return x_62; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = lean_ctor_get(x_38, 0); -lean_inc(x_48); -lean_dec(x_38); -x_49 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_49, 0, x_48); -x_50 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_50, 0, x_49); -x_51 = l_Except_orElseLazy___rarg(x_50, x_11); -return x_51; +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_63 = lean_ctor_get(x_50, 0); +lean_inc(x_63); +lean_dec(x_50); +x_64 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_64, 0, x_25); +lean_ctor_set(x_64, 1, x_26); +lean_ctor_set(x_64, 2, x_63); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2; +x_67 = l_Except_orElseLazy___rarg(x_65, x_66); +return x_67; } } } } } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___closed__1() { +} +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("goal", 4); +x_1 = lean_mk_string_from_bytes("expr", 4); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_box(0); -x_8 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___closed__1; -x_9 = lean_unsigned_to_nat(1u); -x_10 = l_Lean_Json_parseTagged(x_6, x_8, x_9, x_7); -x_11 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___boxed), 7, 6); -lean_closure_set(x_11, 0, x_6); -lean_closure_set(x_11, 1, x_7); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_4); -lean_closure_set(x_11, 4, x_5); -lean_closure_set(x_11, 5, x_1); -if (lean_obj_tag(x_10) == 0) +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___closed__1; +x_5 = lean_unsigned_to_nat(1u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) { -uint8_t x_12; -lean_dec(x_2); -x_12 = !lean_is_exclusive(x_10); -if (x_12 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) { -lean_object* x_13; -x_13 = l_Except_orElseLazy___rarg(x_10, x_11); -return x_13; +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); +return x_9; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_10, 0); -lean_inc(x_14); -lean_dec(x_10); -x_15 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_15, 0, x_14); -x_16 = l_Except_orElseLazy___rarg(x_15, x_11); -return x_16; +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; } } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_ctor_get(x_10, 0); -lean_inc(x_17); -lean_dec(x_10); -x_18 = lean_array_get_size(x_17); -x_19 = lean_unsigned_to_nat(0u); -x_20 = lean_nat_dec_lt(x_19, x_18); -lean_dec(x_18); -if (x_20 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = lean_ctor_get(x_6, 0); +lean_inc(x_13); +lean_dec(x_6); +x_14 = lean_array_get_size(x_13); +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_nat_dec_lt(x_15, x_14); +lean_dec(x_14); +if (x_16 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -lean_dec(x_17); -x_21 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6; -x_22 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_21); -x_23 = lean_apply_1(x_2, x_22); -if (lean_obj_tag(x_23) == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_dec(x_13); +x_17 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6; +x_18 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_17); +x_19 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_18); +if (lean_obj_tag(x_19) == 0) { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) { -lean_object* x_25; -x_25 = l_Except_orElseLazy___rarg(x_23, x_11); -return x_25; +lean_object* x_21; +x_21 = l_Except_orElseLazy___rarg(x_19, x_7); +return x_21; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_19, 0); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_23, 0, x_22); +x_24 = l_Except_orElseLazy___rarg(x_23, x_7); +return x_24; +} } else { +uint8_t x_25; +x_25 = !lean_is_exclusive(x_19); +if (x_25 == 0) +{ lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_23, 0); -lean_inc(x_26); -lean_dec(x_23); +x_26 = lean_ctor_get(x_19, 0); x_27 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_27, 0, x_26); -x_28 = l_Except_orElseLazy___rarg(x_27, x_11); +lean_ctor_set(x_19, 0, x_27); +x_28 = l_Except_orElseLazy___rarg(x_19, x_7); return x_28; } -} else { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_23); -if (x_29 == 0) -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_23, 0); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_19, 0); +lean_inc(x_29); +lean_dec(x_19); +x_30 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_30, 0, x_29); x_31 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_23, 0, x_31); -x_32 = l_Except_orElseLazy___rarg(x_23, x_11); +x_32 = l_Except_orElseLazy___rarg(x_31, x_7); return x_32; } -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_33 = lean_ctor_get(x_23, 0); -lean_inc(x_33); -lean_dec(x_23); -x_34 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_34, 0, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -x_36 = l_Except_orElseLazy___rarg(x_35, x_11); -return x_36; -} } } else { -lean_object* x_37; lean_object* x_38; -x_37 = lean_array_fget(x_17, x_19); -lean_dec(x_17); -x_38 = lean_apply_1(x_2, x_37); -if (lean_obj_tag(x_38) == 0) +lean_object* x_33; lean_object* x_34; +x_33 = lean_array_fget(x_13, x_15); +lean_dec(x_13); +x_34 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_33); +if (lean_obj_tag(x_34) == 0) { -uint8_t x_39; -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +uint8_t x_35; +x_35 = !lean_is_exclusive(x_34); +if (x_35 == 0) { -lean_object* x_40; -x_40 = l_Except_orElseLazy___rarg(x_38, x_11); -return x_40; +lean_object* x_36; +x_36 = l_Except_orElseLazy___rarg(x_34, x_7); +return x_36; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_34, 0); +lean_inc(x_37); +lean_dec(x_34); +x_38 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = l_Except_orElseLazy___rarg(x_38, x_7); +return x_39; +} } else { +uint8_t x_40; +x_40 = !lean_is_exclusive(x_34); +if (x_40 == 0) +{ lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_38, 0); -lean_inc(x_41); -lean_dec(x_38); +x_41 = lean_ctor_get(x_34, 0); x_42 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_42, 0, x_41); -x_43 = l_Except_orElseLazy___rarg(x_42, x_11); +lean_ctor_set(x_34, 0, x_42); +x_43 = l_Except_orElseLazy___rarg(x_34, x_7); return x_43; } -} else { -uint8_t x_44; -x_44 = !lean_is_exclusive(x_38); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_38, 0); +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_34, 0); +lean_inc(x_44); +lean_dec(x_34); +x_45 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_45, 0, x_44); x_46 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_38, 0, x_46); -x_47 = l_Except_orElseLazy___rarg(x_38, x_11); +x_47 = l_Except_orElseLazy___rarg(x_46, x_7); return x_47; } +} +} +} +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("goal", 4); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = lean_box(0); +x_3 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____closed__1; +x_4 = lean_unsigned_to_nat(1u); +x_5 = l_Lean_Json_parseTagged(x_1, x_3, x_4, x_2); +x_6 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___boxed), 3, 2); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; +x_8 = l_Except_orElseLazy___rarg(x_5, x_6); +return x_8; +} else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = lean_ctor_get(x_38, 0); -lean_inc(x_48); -lean_dec(x_38); -x_49 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_49, 0, x_48); -x_50 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_50, 0, x_49); -x_51 = l_Except_orElseLazy___rarg(x_50, x_11); -return x_51; +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_5, 0); +lean_inc(x_9); +lean_dec(x_5); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = l_Except_orElseLazy___rarg(x_10, x_6); +return x_11; +} +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_ctor_get(x_5, 0); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_array_get_size(x_12); +x_14 = lean_unsigned_to_nat(0u); +x_15 = lean_nat_dec_lt(x_14, x_13); +lean_dec(x_13); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_dec(x_12); +x_16 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6; +x_17 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_16); +x_18 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696_(x_17); +if (lean_obj_tag(x_18) == 0) +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) +{ +lean_object* x_20; +x_20 = l_Except_orElseLazy___rarg(x_18, x_6); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_18, 0); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Except_orElseLazy___rarg(x_22, x_6); +return x_23; +} } +else +{ +uint8_t x_24; +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_18, 0); +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_18, 0, x_26); +x_27 = l_Except_orElseLazy___rarg(x_18, x_6); +return x_27; } +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = lean_ctor_get(x_18, 0); +lean_inc(x_28); +lean_dec(x_18); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = l_Except_orElseLazy___rarg(x_30, x_6); +return x_31; } } } +else +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_array_fget(x_12, x_14); +lean_dec(x_12); +x_33 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696_(x_32); +if (lean_obj_tag(x_33) == 0) +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +lean_object* x_35; +x_35 = l_Except_orElseLazy___rarg(x_33, x_6); +return x_35; } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; -x_6 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg), 6, 0); -return x_6; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_33, 0); +lean_inc(x_36); +lean_dec(x_33); +x_37 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_37, 0, x_36); +x_38 = l_Except_orElseLazy___rarg(x_37, x_6); +return x_38; +} +} +else +{ +uint8_t x_39; +x_39 = !lean_is_exclusive(x_33); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_33, 0); +x_41 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_33, 0, x_41); +x_42 = l_Except_orElseLazy___rarg(x_33, x_6); +return x_42; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_43 = lean_ctor_get(x_33, 0); +lean_inc(x_43); +lean_dec(x_33); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_46 = l_Except_orElseLazy___rarg(x_45, x_6); +return x_46; +} +} +} +} } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1(x_1); +x_2 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_7; -x_7 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_6); +lean_object* x_4; +x_4 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2(x_1, x_2, x_3); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_7; +return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_8; -x_8 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_7); -return x_8; +lean_object* x_4; +x_4 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__5___closed__1() { _start: { -lean_object* x_6; -x_6 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg), 6, 5); -lean_closure_set(x_6, 0, x_1); -lean_closure_set(x_6, 1, x_2); -lean_closure_set(x_6, 2, x_3); -lean_closure_set(x_6, 3, x_4); -lean_closure_set(x_6, 4, x_5); -return x_6; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125_), 1, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__5() { _start: { -lean_object* x_6; -x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__5___rarg), 5, 0); -return x_6; +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket__5___closed__1; +return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg___closed__1() { +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320____closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -1090,119 +1709,103 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320_(lean_object* x_1) { _start: { -switch (lean_obj_tag(x_6)) { +switch (lean_obj_tag(x_1)) { case 0: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_7 = lean_ctor_get(x_6, 0); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_apply_1(x_1, x_7); -x_9 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_8); -x_11 = lean_box(0); -x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_11); -x_13 = l_Lean_Json_mkObj(x_12); -return x_13; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +lean_dec(x_1); +x_3 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_2); +x_4 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___closed__1; +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_box(0); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_6); +x_8 = l_Lean_Json_mkObj(x_7); +return x_8; } case 1: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_9 = lean_ctor_get(x_1, 0); +lean_inc(x_9); lean_dec(x_1); -x_14 = lean_ctor_get(x_6, 0); -lean_inc(x_14); -lean_dec(x_6); -x_15 = lean_apply_1(x_2, x_14); -x_16 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___closed__1; -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -x_18 = lean_box(0); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -x_20 = l_Lean_Json_mkObj(x_19); -return x_20; +x_10 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802_(x_9); +x_11 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____closed__1; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +x_15 = l_Lean_Json_mkObj(x_14); +return x_15; } default: { -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_dec(x_2); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; size_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_16 = lean_ctor_get(x_1, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_1, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_1, 2); +lean_inc(x_18); lean_dec(x_1); -x_21 = lean_ctor_get(x_6, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_6, 1); -lean_inc(x_22); -x_23 = lean_ctor_get(x_6, 2); -lean_inc(x_23); -lean_dec(x_6); -x_24 = lean_apply_1(x_3, x_21); -x_25 = lean_apply_1(x_4, x_22); -x_26 = lean_apply_1(x_5, x_23); -x_27 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg___closed__1; -x_28 = lean_array_push(x_27, x_24); +x_19 = l_Lean_JsonNumber_fromNat(x_16); +x_20 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_20, 0, x_19); +x_21 = 1; +x_22 = l_Lean_Name_toString(x_17, x_21); +x_23 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_23, 0, x_22); +x_24 = lean_unbox_usize(x_18); +lean_dec(x_18); +x_25 = l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcRef____x40_Lean_Data_Lsp_Extra___hyg_1065_(x_24); +x_26 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320____closed__1; +x_27 = lean_array_push(x_26, x_20); +x_28 = lean_array_push(x_27, x_23); x_29 = lean_array_push(x_28, x_25); -x_30 = lean_array_push(x_29, x_26); -x_31 = lean_alloc_ctor(4, 1, 0); -lean_ctor_set(x_31, 0, x_30); -x_32 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__1; -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -x_34 = lean_box(0); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -x_36 = l_Lean_Json_mkObj(x_35); -return x_36; -} -} +x_30 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__1; +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +x_33 = lean_box(0); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean_Json_mkObj(x_34); +return x_35; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg), 6, 0); -return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__5___closed__1() { _start: { -lean_object* x_6; -x_6 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg), 6, 5); -lean_closure_set(x_6, 0, x_1); -lean_closure_set(x_6, 1, x_2); -lean_closure_set(x_6, 2, x_3); -lean_closure_set(x_6, 3, x_4); -lean_closure_set(x_6, 4, x_5); -return x_6; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320_), 1, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__5() { _start: { -lean_object* x_6; -x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__5___rarg), 5, 0); -return x_6; +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket__5___closed__1; +return x_1; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -1252,15 +1855,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__1___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -1310,15 +1913,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__2___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -1368,15 +1971,84 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__3___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___boxed), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -1426,15 +2098,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__4___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -1484,191 +2156,77 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__5___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_5, 0, x_2); -x_6 = lean_apply_2(x_4, lean_box(0), x_5); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2) { -_start: +if (lean_obj_tag(x_5) == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_5, 0, x_2); -x_6 = lean_apply_2(x_4, lean_box(0), x_5); -return x_6; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_7, 0, x_2); -lean_ctor_set(x_7, 1, x_3); -lean_ctor_set(x_7, 2, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_1, 0); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); -lean_dec(x_1); -lean_inc(x_2); -x_9 = lean_apply_4(x_8, lean_box(0), x_2, x_3, x_4); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__3), 4, 3); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_5); -lean_closure_set(x_10, 2, x_7); -x_11 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_9, x_10); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -lean_dec(x_1); -lean_inc(x_3); -lean_inc(x_2); -x_10 = lean_apply_4(x_9, lean_box(0), x_2, x_3, x_4); -lean_inc(x_7); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__4), 7, 6); -lean_closure_set(x_11, 0, x_5); -lean_closure_set(x_11, 1, x_2); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_6); -lean_closure_set(x_11, 4, x_8); -lean_closure_set(x_11, 5, x_7); -x_12 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_10, x_11); -return x_12; -} +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -switch (lean_obj_tag(x_9)) { -case 0: +else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_10 = lean_ctor_get(x_9, 0); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_ctor_get(x_7, 1); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); lean_dec(x_1); -lean_inc(x_7); -x_13 = lean_apply_4(x_12, lean_box(0), x_7, x_8, x_10); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__1), 2, 1); -lean_closure_set(x_14, 0, x_7); -x_15 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_13, x_14); -return x_15; +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } -case 1: -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_16 = lean_ctor_get(x_9, 0); -lean_inc(x_16); -lean_dec(x_9); -x_17 = lean_ctor_get(x_7, 1); -lean_inc(x_17); -x_18 = lean_ctor_get(x_2, 0); -lean_inc(x_18); -lean_dec(x_2); -lean_inc(x_7); -x_19 = lean_apply_4(x_18, lean_box(0), x_7, x_8, x_16); -x_20 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__2), 2, 1); -lean_closure_set(x_20, 0, x_7); -x_21 = lean_apply_4(x_17, lean_box(0), lean_box(0), x_19, x_20); -return x_21; } -default: +else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_dec(x_2); +lean_object* x_15; lean_object* x_16; lean_dec(x_1); -x_22 = lean_ctor_get(x_9, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_9, 1); -lean_inc(x_23); -x_24 = lean_ctor_get(x_9, 2); -lean_inc(x_24); -lean_dec(x_9); -x_25 = lean_ctor_get(x_7, 1); -lean_inc(x_25); -x_26 = lean_ctor_get(x_3, 0); -lean_inc(x_26); -lean_dec(x_3); -lean_inc(x_8); -lean_inc(x_7); -x_27 = lean_apply_4(x_26, lean_box(0), x_7, x_8, x_22); -lean_inc(x_25); -x_28 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__5), 8, 7); -lean_closure_set(x_28, 0, x_4); -lean_closure_set(x_28, 1, x_7); -lean_closure_set(x_28, 2, x_8); -lean_closure_set(x_28, 3, x_23); -lean_closure_set(x_28, 4, x_5); -lean_closure_set(x_28, 5, x_24); -lean_closure_set(x_28, 6, x_25); -x_29 = lean_apply_4(x_25, lean_box(0), lean_box(0), x_27, x_28); -return x_29; +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8___rarg), 5, 0); +return x_2; +} } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__7(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_alloc_ctor(0, 1, 0); +x_3 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_3, 0, x_2); x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); @@ -1682,151 +2240,108 @@ x_7 = lean_apply_2(x_5, lean_box(0), x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__8(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_3, 0, x_2); -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_4 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_ctor_get(x_2, 0); lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_6, 0, x_3); -x_7 = lean_apply_2(x_5, lean_box(0), x_6); -return x_7; +lean_dec(x_2); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_5 = lean_alloc_ctor(2, 3, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_4); -x_6 = lean_ctor_get(x_3, 0); -lean_inc(x_6); -lean_dec(x_3); -x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_8, 0, x_5); -x_9 = lean_apply_2(x_7, lean_box(0), x_8); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -lean_dec(x_1); -lean_inc(x_2); -x_8 = lean_apply_4(x_7, lean_box(0), x_2, x_3, x_4); -lean_inc(x_2); -x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__9), 4, 3); -lean_closure_set(x_9, 0, x_5); -lean_closure_set(x_9, 1, x_6); -lean_closure_set(x_9, 2, x_2); -x_10 = lean_ctor_get(x_2, 1); -lean_inc(x_10); -x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__3___rarg), 5, 4); -lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, lean_box(0)); -lean_closure_set(x_11, 2, lean_box(0)); -lean_closure_set(x_11, 3, x_9); -x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +switch (lean_obj_tag(x_3)) { +case 0: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); lean_dec(x_1); -lean_inc(x_3); -lean_inc(x_2); -x_9 = lean_apply_4(x_8, lean_box(0), x_2, x_3, x_4); -lean_inc(x_2); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__10), 6, 5); -lean_closure_set(x_10, 0, x_5); -lean_closure_set(x_10, 1, x_2); -lean_closure_set(x_10, 2, x_3); -lean_closure_set(x_10, 3, x_6); -lean_closure_set(x_10, 4, x_7); -x_11 = lean_ctor_get(x_2, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__4___rarg), 5, 4); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); -return x_13; -} +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -switch (lean_obj_tag(x_9)) { -case 0: +else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_5); -lean_dec(x_4); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); lean_dec(x_3); -lean_dec(x_2); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_ctor_get(x_1, 1); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); lean_dec(x_1); -lean_inc(x_7); -x_12 = lean_apply_4(x_11, lean_box(0), x_7, x_8, x_10); -lean_inc(x_7); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__7), 2, 1); -lean_closure_set(x_13, 0, x_7); -x_14 = lean_ctor_get(x_7, 1); -lean_inc(x_14); -x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_15, 0, x_7); -lean_closure_set(x_15, 1, lean_box(0)); -lean_closure_set(x_15, 2, lean_box(0)); -lean_closure_set(x_15, 3, x_13); -x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); -return x_16; +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} } case 1: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -lean_dec(x_5); -lean_dec(x_4); +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); lean_dec(x_3); -lean_dec(x_1); -x_17 = lean_ctor_get(x_9, 0); -lean_inc(x_17); -lean_dec(x_9); -x_18 = lean_ctor_get(x_2, 1); -lean_inc(x_18); -lean_dec(x_2); -lean_inc(x_7); -x_19 = lean_apply_4(x_18, lean_box(0), x_7, x_8, x_17); -lean_inc(x_7); -x_20 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__8), 2, 1); -lean_closure_set(x_20, 0, x_7); -x_21 = lean_ctor_get(x_7, 1); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); lean_inc(x_21); -x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_22, 0, x_7); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); lean_closure_set(x_22, 1, lean_box(0)); lean_closure_set(x_22, 2, lean_box(0)); lean_closure_set(x_22, 3, x_20); @@ -1835,1040 +2350,660 @@ return x_23; } default: { -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_dec(x_2); -lean_dec(x_1); -x_24 = lean_ctor_get(x_9, 0); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); lean_inc(x_24); -x_25 = lean_ctor_get(x_9, 1); +x_25 = lean_ctor_get(x_3, 1); lean_inc(x_25); -x_26 = lean_ctor_get(x_9, 2); -lean_inc(x_26); -lean_dec(x_9); -x_27 = lean_ctor_get(x_3, 1); -lean_inc(x_27); lean_dec(x_3); -lean_inc(x_8); -lean_inc(x_7); -x_28 = lean_apply_4(x_27, lean_box(0), x_7, x_8, x_24); -lean_inc(x_7); -x_29 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__11), 7, 6); -lean_closure_set(x_29, 0, x_4); -lean_closure_set(x_29, 1, x_7); -lean_closure_set(x_29, 2, x_8); -lean_closure_set(x_29, 3, x_25); -lean_closure_set(x_29, 4, x_5); -lean_closure_set(x_29, 5, x_26); -x_30 = lean_ctor_get(x_7, 1); -lean_inc(x_30); -x_31 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___spec__5___rarg), 5, 4); -lean_closure_set(x_31, 0, x_7); -lean_closure_set(x_31, 1, lean_box(0)); -lean_closure_set(x_31, 2, lean_box(0)); -lean_closure_set(x_31, 3, x_29); -x_32 = lean_apply_4(x_30, lean_box(0), lean_box(0), x_28, x_31); -return x_32; -} -} +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__3), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; -lean_inc(x_9); -lean_inc(x_7); -lean_inc(x_5); -lean_inc(x_3); -lean_inc(x_1); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__6), 9, 5); -lean_closure_set(x_10, 0, x_1); -lean_closure_set(x_10, 1, x_3); -lean_closure_set(x_10, 2, x_5); -lean_closure_set(x_10, 3, x_7); -lean_closure_set(x_10, 4, x_9); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg___lambda__12), 9, 5); -lean_closure_set(x_11, 0, x_1); -lean_closure_set(x_11, 1, x_3); -lean_closure_set(x_11, 2, x_5); -lean_closure_set(x_11, 3, x_7); -lean_closure_set(x_11, 4, x_9); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_11); -return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbedRpcEncodingPacket___rarg), 9, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg), 3, 0); return x_2; } } -static lean_object* _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1() { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +if (lean_obj_tag(x_5) == 0) { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValD(x_2, x_3); -if (lean_obj_tag(x_4) == 0) +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_5; +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -return x_5; -} -else -{ -lean_object* x_6; -x_6 = lean_apply_1(x_1, x_4); -if (lean_obj_tag(x_6) == 0) -{ -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) -{ -return x_6; -} -else -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); return x_9; } -} else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_6); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_6, 0); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_6, 0, x_12); -return x_6; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_6, 0); -lean_inc(x_13); -lean_dec(x_6); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; -} -} +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValD(x_2, x_3); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; -lean_dec(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -return x_5; -} -else -{ -lean_object* x_6; -x_6 = lean_apply_1(x_1, x_4); -if (lean_obj_tag(x_6) == 0) +if (lean_obj_tag(x_5) == 0) { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -return x_6; +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); -return x_9; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_6); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_6, 0); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_6, 0, x_12); -return x_6; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_6, 0); -lean_inc(x_13); -lean_dec(x_6); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; -} -} +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { _start: { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValD(x_2, x_3); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; -lean_dec(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -return x_5; -} -else -{ -lean_object* x_6; -x_6 = lean_apply_1(x_1, x_4); -if (lean_obj_tag(x_6) == 0) -{ -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) -{ -return x_6; -} -else -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(x_3, x_4, x_7, x_8); return x_9; } } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_6); -if (x_10 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_6, 0); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_6, 0, x_12); -return x_6; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_6, 0); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); lean_inc(x_13); -lean_dec(x_6); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; -} -} +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___boxed), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValD(x_2, x_3); -if (lean_obj_tag(x_4) == 0) +if (lean_obj_tag(x_5) == 0) { -lean_object* x_5; +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -return x_5; +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_6; -x_6 = lean_apply_1(x_1, x_4); -if (lean_obj_tag(x_6) == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13(lean_object* x_1) { +_start: { -return x_6; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13___rarg), 5, 0); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(x_3, x_4, x_7, x_8); return x_9; } } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_6); -if (x_10 == 0) +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_6, 0); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_6, 0, x_12); -return x_6; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_6, 0); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); lean_inc(x_13); -lean_dec(x_6); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; -} -} +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___boxed), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValD(x_2, x_3); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; -lean_dec(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -return x_5; -} -else -{ -lean_object* x_6; -x_6 = lean_apply_1(x_1, x_4); -if (lean_obj_tag(x_6) == 0) -{ -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +if (lean_obj_tag(x_5) == 0) { -return x_6; -} -else +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); return x_9; } -} else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_6); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_6, 0); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_6, 0, x_12); -return x_6; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_6, 0); -lean_inc(x_13); -lean_dec(x_6); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; -} -} +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14___rarg), 5, 0); return x_2; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__1() { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("range", 5); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__2() { -_start: +if (lean_obj_tag(x_5) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("fullRange", 9); -return x_1; +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("severity", 8); -return x_1; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__4() { +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("code", 4); -return x_1; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15___rarg), 5, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__5() { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("source", 6); -return x_1; +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__6() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("message", 7); -return x_1; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__7() { +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("tags", 4); -return x_1; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18___rarg), 5, 0); +return x_2; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__8() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("relatedInformation", 18); -return x_1; +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { -lean_object* x_9; lean_object* x_10; -x_9 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__1; -lean_inc(x_1); -x_10 = l_Lean_Json_getObjValAs_x3f(x_8, lean_box(0), x_1, x_9); -if (lean_obj_tag(x_10) == 0) +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) { -uint8_t x_11; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); return x_10; } else { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_10, 0); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; } } -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_10, 0); -lean_inc(x_14); -lean_dec(x_10); -x_15 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__2; -x_16 = l_Lean_Json_getObjValAs_x3f(x_8, lean_box(0), x_1, x_15); -if (lean_obj_tag(x_16) == 0) -{ -uint8_t x_17; -lean_dec(x_14); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -return x_16; } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17(lean_object* x_1) { +_start: { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___boxed), 5, 0); +return x_2; } } -else +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_16, 0); -lean_inc(x_20); -lean_dec(x_16); -x_21 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__3; -x_22 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg(x_2, x_8, x_21); -if (lean_obj_tag(x_22) == 0) +if (lean_obj_tag(x_5) == 0) { -uint8_t x_23; -lean_dec(x_20); -lean_dec(x_14); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +uint8_t x_6; lean_dec(x_4); -lean_dec(x_3); -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -return x_22; +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_22, 0); -lean_inc(x_26); -lean_dec(x_22); -x_27 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__4; -x_28 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2___rarg(x_3, x_8, x_27); -if (lean_obj_tag(x_28) == 0) -{ -uint8_t x_29; -lean_dec(x_26); -lean_dec(x_20); -lean_dec(x_14); -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); lean_dec(x_5); -lean_dec(x_4); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) -{ -return x_28; +x_16 = lean_apply_1(x_4, x_15); +return x_16; } -else -{ -lean_object* x_30; lean_object* x_31; -x_30 = lean_ctor_get(x_28, 0); -lean_inc(x_30); -lean_dec(x_28); -x_31 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_31, 0, x_30); -return x_31; } } -else +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19(lean_object* x_1) { +_start: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_28, 0); -lean_inc(x_32); -lean_dec(x_28); -x_33 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__5; -x_34 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3___rarg(x_4, x_8, x_33); -if (lean_obj_tag(x_34) == 0) -{ -uint8_t x_35; -lean_dec(x_32); -lean_dec(x_26); -lean_dec(x_20); -lean_dec(x_14); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) -{ -return x_34; -} -else -{ -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_37, 0, x_36); -return x_37; -} -} -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_34, 0); -lean_inc(x_38); -lean_dec(x_34); -x_39 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__6; -x_40 = l_Lean_Json_getObjValAs_x3f(x_8, lean_box(0), x_5, x_39); -if (lean_obj_tag(x_40) == 0) -{ -uint8_t x_41; -lean_dec(x_38); -lean_dec(x_32); -lean_dec(x_26); -lean_dec(x_20); -lean_dec(x_14); -lean_dec(x_7); -lean_dec(x_6); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -return x_40; -} -else -{ -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_40, 0); -lean_inc(x_42); -lean_dec(x_40); -x_43 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_43, 0, x_42); -return x_43; -} -} -else -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_40, 0); -lean_inc(x_44); -lean_dec(x_40); -x_45 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__7; -x_46 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4___rarg(x_6, x_8, x_45); -if (lean_obj_tag(x_46) == 0) -{ -uint8_t x_47; -lean_dec(x_44); -lean_dec(x_38); -lean_dec(x_32); -lean_dec(x_26); -lean_dec(x_20); -lean_dec(x_14); -lean_dec(x_7); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) -{ -return x_46; -} -else -{ -lean_object* x_48; lean_object* x_49; -x_48 = lean_ctor_get(x_46, 0); -lean_inc(x_48); -lean_dec(x_46); -x_49 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_49, 0, x_48); -return x_49; -} -} -else -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_46, 0); -lean_inc(x_50); -lean_dec(x_46); -x_51 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__8; -x_52 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5___rarg(x_7, x_8, x_51); -if (lean_obj_tag(x_52) == 0) -{ -uint8_t x_53; -lean_dec(x_50); -lean_dec(x_44); -lean_dec(x_38); -lean_dec(x_32); -lean_dec(x_26); -lean_dec(x_20); -lean_dec(x_14); -x_53 = !lean_is_exclusive(x_52); -if (x_53 == 0) -{ -return x_52; -} -else -{ -lean_object* x_54; lean_object* x_55; -x_54 = lean_ctor_get(x_52, 0); -lean_inc(x_54); -lean_dec(x_52); -x_55 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_55, 0, x_54); -return x_55; -} -} -else -{ -uint8_t x_56; -x_56 = !lean_is_exclusive(x_52); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; -x_57 = lean_ctor_get(x_52, 0); -x_58 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_58, 0, x_14); -lean_ctor_set(x_58, 1, x_20); -lean_ctor_set(x_58, 2, x_26); -lean_ctor_set(x_58, 3, x_32); -lean_ctor_set(x_58, 4, x_38); -lean_ctor_set(x_58, 5, x_44); -lean_ctor_set(x_58, 6, x_50); -lean_ctor_set(x_58, 7, x_57); -lean_ctor_set(x_52, 0, x_58); -return x_52; -} -else -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_52, 0); -lean_inc(x_59); -lean_dec(x_52); -x_60 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_60, 0, x_14); -lean_ctor_set(x_60, 1, x_20); -lean_ctor_set(x_60, 2, x_26); -lean_ctor_set(x_60, 3, x_32); -lean_ctor_set(x_60, 4, x_38); -lean_ctor_set(x_60, 5, x_44); -lean_ctor_set(x_60, 6, x_50); -lean_ctor_set(x_60, 7, x_59); -x_61 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_61, 0, x_60); -return x_61; -} -} -} -} -} -} -} -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___boxed), 8, 0); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__2___rarg(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__3___rarg(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__4___rarg(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__5___rarg(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_8); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___boxed), 8, 7); -lean_closure_set(x_8, 0, x_1); -lean_closure_set(x_8, 1, x_2); -lean_closure_set(x_8, 2, x_3); -lean_closure_set(x_8, 3, x_4); -lean_closure_set(x_8, 4, x_5); -lean_closure_set(x_8, 5, x_6); -lean_closure_set(x_8, 6, x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__6___rarg), 7, 0); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1642____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; lean_object* x_10; 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; -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -lean_inc(x_1); -x_10 = lean_apply_1(x_1, x_9); -x_11 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__1; -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); -x_13 = lean_box(0); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_12); -lean_ctor_set(x_14, 1, x_13); -x_15 = lean_ctor_get(x_8, 1); -lean_inc(x_15); -x_16 = lean_apply_1(x_1, x_15); -x_17 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__2; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_13); -x_20 = lean_ctor_get(x_8, 2); -lean_inc(x_20); -x_21 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__3; -x_22 = l_Lean_Json_opt___rarg(x_2, x_21, x_20); -x_23 = lean_ctor_get(x_8, 3); -lean_inc(x_23); -x_24 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__4; -x_25 = l_Lean_Json_opt___rarg(x_3, x_24, x_23); -x_26 = lean_ctor_get(x_8, 4); -lean_inc(x_26); -x_27 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__5; -x_28 = l_Lean_Json_opt___rarg(x_4, x_27, x_26); -x_29 = lean_ctor_get(x_8, 5); -lean_inc(x_29); -x_30 = lean_apply_1(x_5, x_29); -x_31 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__6; -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_30); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_13); -x_34 = lean_ctor_get(x_8, 6); -lean_inc(x_34); -x_35 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__7; -x_36 = l_Lean_Json_opt___rarg(x_6, x_35, x_34); -x_37 = lean_ctor_get(x_8, 7); -lean_inc(x_37); -lean_dec(x_8); -x_38 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__8; -x_39 = l_Lean_Json_opt___rarg(x_7, x_38, x_37); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_13); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_36); -lean_ctor_set(x_41, 1, x_40); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_33); -lean_ctor_set(x_42, 1, x_41); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_28); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_25); -lean_ctor_set(x_44, 1, x_43); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_22); -lean_ctor_set(x_45, 1, x_44); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_19); -lean_ctor_set(x_46, 1, x_45); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_14); -lean_ctor_set(x_47, 1, x_46); -x_48 = l_List_join___rarg(x_47); -x_49 = l_Lean_Json_mkObj(x_48); -return x_49; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1642_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1642____rarg), 8, 0); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1642____rarg), 8, 7); -lean_closure_set(x_8, 0, x_1); -lean_closure_set(x_8, 1, x_2); -lean_closure_set(x_8, 2, x_3); -lean_closure_set(x_8, 3, x_4); -lean_closure_set(x_8, 4, x_5); -lean_closure_set(x_8, 5, x_6); -lean_closure_set(x_8, 6, x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__6___rarg), 7, 0); -return x_8; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -2918,15 +3053,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__1___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -2976,18 +3111,143 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__2___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -if (lean_obj_tag(x_5) == 0) +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) { uint8_t x_6; lean_dec(x_4); @@ -3034,15 +3294,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__3___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -3092,15 +3352,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__4___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -3150,15 +3410,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__5___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -3208,15 +3468,84 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__6(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__6___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___boxed), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -3266,15 +3595,15 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__7(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__7___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -3324,494 +3653,602 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__8(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__8___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -x_11 = lean_ctor_get(x_10, 1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); -lean_dec(x_10); -x_12 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_12, 0, x_2); -lean_ctor_set(x_12, 1, x_3); -lean_ctor_set(x_12, 2, x_4); -lean_ctor_set(x_12, 3, x_5); -lean_ctor_set(x_12, 4, x_6); -lean_ctor_set(x_12, 5, x_7); -lean_ctor_set(x_12, 6, x_8); -lean_ctor_set(x_12, 7, x_9); -x_13 = lean_apply_2(x_11, lean_box(0), x_12); -return x_13; +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__2(lean_object* x_1) { +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30___rarg), 5, 0); return x_2; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__2), 1, 0); -return x_1; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_1, 7); -lean_inc(x_13); -lean_dec(x_1); -lean_inc(x_2); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__1), 9, 8); -lean_closure_set(x_14, 0, x_2); -lean_closure_set(x_14, 1, x_3); -lean_closure_set(x_14, 2, x_4); -lean_closure_set(x_14, 3, x_5); -lean_closure_set(x_14, 4, x_6); -lean_closure_set(x_14, 5, x_7); -lean_closure_set(x_14, 6, x_8); -lean_closure_set(x_14, 7, x_12); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -lean_dec(x_11); -lean_dec(x_10); -x_15 = lean_ctor_get(x_2, 0); -lean_inc(x_15); +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; lean_dec(x_2); -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_box(0); -x_18 = lean_apply_2(x_16, lean_box(0), x_17); -x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_18, x_14); -return x_19; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_20 = lean_ctor_get(x_13, 0); -lean_inc(x_20); -lean_dec(x_13); -x_21 = lean_ctor_get(x_2, 0); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); lean_inc(x_21); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_10, 0); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); lean_inc(x_24); -lean_dec(x_10); -x_25 = lean_apply_4(x_24, lean_box(0), x_2, x_11, x_20); -x_26 = l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1; -x_27 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_26, x_25); -x_28 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_27, x_14); -return x_28; +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25(lean_object* x_1) { _start: { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_1, 6); -lean_inc(x_13); -lean_inc(x_10); -lean_inc(x_8); -lean_inc(x_2); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3), 12, 11); -lean_closure_set(x_14, 0, x_1); -lean_closure_set(x_14, 1, x_2); -lean_closure_set(x_14, 2, x_3); -lean_closure_set(x_14, 3, x_4); -lean_closure_set(x_14, 4, x_5); -lean_closure_set(x_14, 5, x_6); -lean_closure_set(x_14, 6, x_7); -lean_closure_set(x_14, 7, x_12); -lean_closure_set(x_14, 8, x_8); -lean_closure_set(x_14, 9, x_9); -lean_closure_set(x_14, 10, x_10); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -lean_dec(x_11); -lean_dec(x_10); -x_15 = lean_ctor_get(x_2, 0); -lean_inc(x_15); -lean_dec(x_2); -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_box(0); -x_18 = lean_apply_2(x_16, lean_box(0), x_17); -x_19 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_18, x_14); -return x_19; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_20 = lean_ctor_get(x_13, 0); -lean_inc(x_20); -lean_dec(x_13); -x_21 = lean_ctor_get(x_2, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_11, 0); -lean_inc(x_24); -lean_dec(x_11); -x_25 = lean_apply_4(x_24, lean_box(0), x_2, x_10, x_20); -x_26 = l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1; -x_27 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_26, x_25); -x_28 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_27, x_14); -return x_28; -} +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg), 3, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_1, 0); -lean_inc(x_13); -lean_dec(x_1); -x_14 = lean_ctor_get(x_2, 5); -lean_inc(x_14); -lean_inc(x_4); -lean_inc(x_3); -x_15 = lean_apply_4(x_13, lean_box(0), x_3, x_4, x_14); -lean_inc(x_9); -x_16 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__4), 12, 11); -lean_closure_set(x_16, 0, x_2); -lean_closure_set(x_16, 1, x_3); -lean_closure_set(x_16, 2, x_5); -lean_closure_set(x_16, 3, x_6); -lean_closure_set(x_16, 4, x_7); -lean_closure_set(x_16, 5, x_8); -lean_closure_set(x_16, 6, x_12); -lean_closure_set(x_16, 7, x_9); -lean_closure_set(x_16, 8, x_10); -lean_closure_set(x_16, 9, x_4); -lean_closure_set(x_16, 10, x_11); -x_17 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_15, x_16); -return x_17; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +if (lean_obj_tag(x_5) == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_1, 4); -lean_inc(x_13); -lean_inc(x_8); -lean_inc(x_4); -lean_inc(x_3); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__5), 12, 11); -lean_closure_set(x_14, 0, x_2); -lean_closure_set(x_14, 1, x_1); -lean_closure_set(x_14, 2, x_3); -lean_closure_set(x_14, 3, x_4); -lean_closure_set(x_14, 4, x_5); -lean_closure_set(x_14, 5, x_6); -lean_closure_set(x_14, 6, x_7); -lean_closure_set(x_14, 7, x_12); -lean_closure_set(x_14, 8, x_8); -lean_closure_set(x_14, 9, x_9); -lean_closure_set(x_14, 10, x_10); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -lean_dec(x_11); +uint8_t x_6; lean_dec(x_4); -x_15 = lean_ctor_get(x_3, 0); -lean_inc(x_15); -lean_dec(x_3); -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_box(0); -x_18 = lean_apply_2(x_16, lean_box(0), x_17); -x_19 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_18, x_14); -return x_19; +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_20 = lean_ctor_get(x_13, 0); -lean_inc(x_20); -lean_dec(x_13); -x_21 = lean_ctor_get(x_3, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_11, 0); -lean_inc(x_24); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); lean_dec(x_11); -x_25 = lean_apply_4(x_24, lean_box(0), x_3, x_4, x_20); -x_26 = l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1; -x_27 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_26, x_25); -x_28 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_27, x_14); -return x_28; -} +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_1, 3); -lean_inc(x_13); -lean_inc(x_7); -lean_inc(x_4); -lean_inc(x_3); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__6), 12, 11); -lean_closure_set(x_14, 0, x_1); -lean_closure_set(x_14, 1, x_2); -lean_closure_set(x_14, 2, x_3); -lean_closure_set(x_14, 3, x_4); -lean_closure_set(x_14, 4, x_5); -lean_closure_set(x_14, 5, x_6); -lean_closure_set(x_14, 6, x_12); -lean_closure_set(x_14, 7, x_7); -lean_closure_set(x_14, 8, x_8); -lean_closure_set(x_14, 9, x_9); -lean_closure_set(x_14, 10, x_10); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -lean_dec(x_11); -lean_dec(x_4); -x_15 = lean_ctor_get(x_3, 0); +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); lean_inc(x_15); -lean_dec(x_3); -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_box(0); -x_18 = lean_apply_2(x_16, lean_box(0), x_17); -x_19 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_14); -return x_19; +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} } -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_20 = lean_ctor_get(x_13, 0); -lean_inc(x_20); -lean_dec(x_13); -x_21 = lean_ctor_get(x_3, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_11, 0); -lean_inc(x_24); -lean_dec(x_11); -x_25 = lean_apply_4(x_24, lean_box(0), x_3, x_4, x_20); -x_26 = l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1; -x_27 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_26, x_25); -x_28 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_27, x_14); -return x_28; } +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_1, 2); -lean_inc(x_13); -lean_inc(x_6); -lean_inc(x_4); -lean_inc(x_3); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__7), 12, 11); -lean_closure_set(x_14, 0, x_1); -lean_closure_set(x_14, 1, x_2); -lean_closure_set(x_14, 2, x_3); -lean_closure_set(x_14, 3, x_4); -lean_closure_set(x_14, 4, x_5); -lean_closure_set(x_14, 5, x_12); -lean_closure_set(x_14, 6, x_6); -lean_closure_set(x_14, 7, x_7); -lean_closure_set(x_14, 8, x_8); -lean_closure_set(x_14, 9, x_9); -lean_closure_set(x_14, 10, x_10); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -lean_dec(x_11); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; lean_dec(x_4); -x_15 = lean_ctor_get(x_3, 0); -lean_inc(x_15); -lean_dec(x_3); -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_box(0); -x_18 = lean_apply_2(x_16, lean_box(0), x_17); -x_19 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_18, x_14); -return x_19; +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_20 = lean_ctor_get(x_13, 0); -lean_inc(x_20); -lean_dec(x_13); -x_21 = lean_ctor_get(x_3, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -lean_dec(x_21); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -lean_dec(x_22); -x_24 = lean_ctor_get(x_11, 0); -lean_inc(x_24); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); lean_dec(x_11); -x_25 = lean_apply_4(x_24, lean_box(0), x_3, x_4, x_20); -x_26 = l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1; -x_27 = lean_apply_4(x_23, lean_box(0), lean_box(0), x_26, x_25); -x_28 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_27, x_14); -return x_28; -} +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_1, 1); -lean_inc(x_13); -lean_inc(x_4); -lean_inc(x_3); -x_14 = lean_apply_4(x_2, lean_box(0), x_3, x_4, x_13); -lean_inc(x_6); -x_15 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__8), 12, 11); -lean_closure_set(x_15, 0, x_1); -lean_closure_set(x_15, 1, x_5); -lean_closure_set(x_15, 2, x_3); -lean_closure_set(x_15, 3, x_4); -lean_closure_set(x_15, 4, x_12); -lean_closure_set(x_15, 5, x_6); -lean_closure_set(x_15, 6, x_7); -lean_closure_set(x_15, 7, x_8); -lean_closure_set(x_15, 8, x_9); -lean_closure_set(x_15, 9, x_10); -lean_closure_set(x_15, 10, x_11); -x_16 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_14, x_15); +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, 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_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32(lean_object* x_1) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_12 = lean_ctor_get(x_9, 1); -lean_inc(x_12); -x_13 = lean_ctor_get(x_1, 0); -lean_inc(x_13); -lean_dec(x_1); -x_14 = lean_ctor_get(x_11, 0); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_10); -lean_inc(x_9); -x_15 = lean_apply_4(x_13, lean_box(0), x_9, x_10, x_14); -lean_inc(x_12); -x_16 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__9), 12, 11); -lean_closure_set(x_16, 0, x_11); -lean_closure_set(x_16, 1, x_13); -lean_closure_set(x_16, 2, x_9); -lean_closure_set(x_16, 3, x_10); -lean_closure_set(x_16, 4, x_2); -lean_closure_set(x_16, 5, x_12); -lean_closure_set(x_16, 6, x_3); -lean_closure_set(x_16, 7, x_4); -lean_closure_set(x_16, 8, x_5); -lean_closure_set(x_16, 9, x_6); -lean_closure_set(x_16, 10, x_7); -x_17 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_15, x_16); -return x_17; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_10, 0, x_1); -lean_ctor_set(x_10, 1, x_2); -lean_ctor_set(x_10, 2, x_3); -lean_ctor_set(x_10, 3, x_4); -lean_ctor_set(x_10, 4, x_5); -lean_ctor_set(x_10, 5, x_6); -lean_ctor_set(x_10, 6, x_7); -lean_ctor_set(x_10, 7, x_9); -x_11 = lean_ctor_get(x_8, 0); +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); -lean_dec(x_8); +lean_dec(x_1); x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); -x_13 = lean_alloc_ctor(1, 1, 0); +x_13 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_13, 0, x_10); x_14 = lean_apply_2(x_12, lean_box(0), x_13); return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__12(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -uint8_t x_3; -x_3 = !lean_is_exclusive(x_2); -if (x_3 == 0) +else { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); +lean_object* x_15; lean_object* x_16; lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_apply_2(x_5, lean_box(0), x_2); -return x_6; +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } -else +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33(lean_object* x_1) { +_start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_box_usize(x_1); +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_2, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_2); +lean_ctor_set(x_8, 2, x_3); +lean_ctor_set(x_8, 3, x_4); +lean_ctor_set_uint8(x_8, sizeof(void*)*4, x_5); +lean_ctor_set_uint8(x_8, sizeof(void*)*4 + 1, x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +x_10 = lean_apply_2(x_6, lean_box(0), x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__7(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_apply_2(x_5, lean_box(0), x_2); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; x_7 = lean_ctor_get(x_2, 0); lean_inc(x_7); lean_dec(x_2); @@ -3869,292 +4306,8814 @@ return x_23; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1() { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_1, 7); -lean_inc(x_12); -lean_dec(x_1); -lean_inc(x_8); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__11), 9, 8); -lean_closure_set(x_13, 0, x_2); -lean_closure_set(x_13, 1, x_3); -lean_closure_set(x_13, 2, x_4); -lean_closure_set(x_13, 3, x_5); -lean_closure_set(x_13, 4, x_6); -lean_closure_set(x_13, 5, x_7); -lean_closure_set(x_13, 6, x_11); -lean_closure_set(x_13, 7, x_8); -x_14 = lean_ctor_get(x_8, 1); -lean_inc(x_14); -lean_inc(x_8); -x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_15, 0, x_8); -lean_closure_set(x_15, 1, lean_box(0)); -lean_closure_set(x_15, 2, lean_box(0)); -lean_closure_set(x_15, 3, x_13); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_10); -lean_dec(x_9); -x_16 = lean_ctor_get(x_8, 0); -lean_inc(x_16); -lean_dec(x_8); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -x_19 = lean_apply_2(x_17, lean_box(0), x_18); -x_20 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_19, x_15); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_12, 0); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_ctor_get(x_9, 1); -lean_inc(x_22); -lean_dec(x_9); -lean_inc(x_8); -x_23 = lean_apply_4(x_22, lean_box(0), x_8, x_10, x_21); -x_24 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__12), 2, 1); -lean_closure_set(x_24, 0, x_8); -lean_inc(x_14); -x_25 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_23, x_24); -x_26 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_25, x_15); -return x_26; -} +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_1, 6); -lean_inc(x_12); -lean_inc(x_9); -lean_inc(x_7); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__13), 11, 10); -lean_closure_set(x_13, 0, x_1); -lean_closure_set(x_13, 1, x_2); -lean_closure_set(x_13, 2, x_3); -lean_closure_set(x_13, 3, x_4); -lean_closure_set(x_13, 4, x_5); -lean_closure_set(x_13, 5, x_6); -lean_closure_set(x_13, 6, x_11); -lean_closure_set(x_13, 7, x_7); -lean_closure_set(x_13, 8, x_8); -lean_closure_set(x_13, 9, x_9); -x_14 = lean_ctor_get(x_7, 1); -lean_inc(x_14); +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); lean_inc(x_7); -x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_15, 0, x_7); -lean_closure_set(x_15, 1, lean_box(0)); -lean_closure_set(x_15, 2, lean_box(0)); -lean_closure_set(x_15, 3, x_13); -if (lean_obj_tag(x_12) == 0) +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__6), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_10); -lean_dec(x_9); x_16 = lean_ctor_get(x_7, 0); lean_inc(x_16); lean_dec(x_7); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -x_19 = lean_apply_2(x_17, lean_box(0), x_18); -x_20 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_19, x_15); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); return x_20; } -else -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_12, 0); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); -lean_dec(x_10); -lean_inc(x_7); -x_23 = lean_apply_4(x_22, lean_box(0), x_7, x_9, x_21); -x_24 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__12), 2, 1); -lean_closure_set(x_24, 0, x_7); -lean_inc(x_14); -x_25 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_23, x_24); -x_26 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_25, x_15); -return x_26; -} } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_12 = lean_ctor_get(x_1, 1); -lean_inc(x_12); -lean_dec(x_1); -x_13 = lean_ctor_get(x_2, 5); +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__3), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__11(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(x_1, x_16, x_17, x_14); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1; +lean_inc(x_2); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10___boxed), 5, 4); +lean_closure_set(x_20, 0, x_11); +lean_closure_set(x_20, 1, x_1); +lean_closure_set(x_20, 2, x_19); +lean_closure_set(x_20, 3, x_2); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +lean_inc(x_21); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_18, x_22); +x_24 = lean_box_usize(x_4); +x_25 = lean_box_usize(x_3); +lean_inc(x_1); +x_26 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__11___boxed), 6, 5); +lean_closure_set(x_26, 0, x_24); +lean_closure_set(x_26, 1, x_13); +lean_closure_set(x_26, 2, x_1); +lean_closure_set(x_26, 3, x_2); +lean_closure_set(x_26, 4, x_25); +x_27 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35___rarg), 5, 4); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, lean_box(0)); +lean_closure_set(x_27, 2, lean_box(0)); +lean_closure_set(x_27, 3, x_26); +x_28 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_23, x_27); +return x_28; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__3(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_3 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_7, 0, x_1); +lean_ctor_set(x_7, 1, x_2); +lean_ctor_set(x_7, 2, x_3); +lean_ctor_set(x_7, 3, x_4); +lean_ctor_set(x_7, 4, x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_apply_2(x_5, lean_box(0), x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; +x_4 = lean_apply_2(x_1, lean_box(0), x_2); +return x_4; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_1, lean_box(0), x_6); +return x_7; +} +} +else +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_2); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_2, 0, x_10); +x_11 = lean_apply_2(x_1, lean_box(0), x_2); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); +lean_dec(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = lean_apply_2(x_1, lean_box(0), x_14); +return x_15; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 4); +lean_inc(x_5); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__6), 6, 5); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_7); +lean_closure_set(x_9, 4, x_5); +x_10 = lean_ctor_get(x_6, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44___rarg), 5, 4); +lean_closure_set(x_11, 0, x_6); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_13 = lean_apply_2(x_5, lean_box(0), x_12); +x_14 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_13, x_11); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_8, 0); +lean_inc(x_15); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_inc(x_5); +x_17 = lean_apply_2(x_5, lean_box(0), x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_5); +lean_inc(x_10); +x_19 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_11); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 3); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_6); +lean_inc(x_8); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8___boxed), 7, 6); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_3); +lean_closure_set(x_11, 2, x_4); +lean_closure_set(x_11, 3, x_5); +lean_closure_set(x_11, 4, x_8); +lean_closure_set(x_11, 5, x_2); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__10(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; +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__9), 5, 4); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +lean_closure_set(x_6, 2, x_3); +lean_closure_set(x_6, 3, x_4); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_14); +lean_inc(x_16); +x_18 = lean_apply_2(x_16, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_19, 0, x_16); +lean_inc(x_7); +x_20 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_20, x_8); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__5), 3, 2); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_3); +lean_inc(x_2); +x_7 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(x_2, x_6, x_5); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__10), 4, 3); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__12(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_box_usize(x_4); +x_6 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_6, 0, x_1); +lean_ctor_set(x_6, 1, x_2); +lean_ctor_set(x_6, 2, x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_6); +x_8 = lean_apply_2(x_3, lean_box(0), x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_7 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +lean_inc(x_1); +x_9 = lean_apply_4(x_8, lean_box(0), x_1, x_2, x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13___boxed), 4, 3); +lean_closure_set(x_10, 0, x_4); +lean_closure_set(x_10, 1, x_6); +lean_closure_set(x_10, 2, x_5); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50___rarg), 5, 4); +lean_closure_set(x_12, 0, x_1); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_1); +lean_inc(x_2); +x_8 = lean_apply_2(x_2, lean_box(0), x_7); +lean_inc(x_3); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14), 6, 5); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_4); +lean_closure_set(x_9, 2, x_5); +lean_closure_set(x_9, 3, x_6); +lean_closure_set(x_9, 4, x_2); +x_10 = lean_ctor_get(x_3, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51___rarg), 5, 4); +lean_closure_set(x_11, 0, x_3); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +lean_inc(x_1); +x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__2), 3, 2); +lean_closure_set(x_5, 0, x_1); +lean_closure_set(x_5, 1, x_2); +lean_inc(x_1); +x_6 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(x_1, x_5, x_4); +lean_inc(x_1); +x_7 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__3), 2, 1); +lean_closure_set(x_7, 0, x_1); +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); +x_9 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9___rarg), 5, 4); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, lean_box(0)); +lean_closure_set(x_9, 2, lean_box(0)); +lean_closure_set(x_9, 3, x_7); +x_10 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_6, x_9); +return x_10; +} +case 1: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_11 = lean_ctor_get(x_3, 0); +lean_inc(x_11); +lean_dec(x_3); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_array_get_size(x_12); +x_14 = lean_usize_of_nat(x_13); +lean_dec(x_13); +x_15 = 0; +lean_inc(x_2); +lean_inc(x_1); +x_16 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(x_1, x_2, x_14, x_15, x_12); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__11), 4, 3); +lean_closure_set(x_17, 0, x_11); +lean_closure_set(x_17, 1, x_1); +lean_closure_set(x_17, 2, x_2); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +lean_inc(x_18); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_16, x_19); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__12), 2, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_21); +x_23 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_20, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +x_26 = lean_ctor_get(x_3, 2); +lean_inc(x_26); +lean_dec(x_3); +x_27 = lean_ctor_get(x_1, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_24); +lean_inc(x_28); +x_30 = lean_apply_2(x_28, lean_box(0), x_29); +lean_inc(x_1); +x_31 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__15), 6, 5); +lean_closure_set(x_31, 0, x_25); +lean_closure_set(x_31, 1, x_28); +lean_closure_set(x_31, 2, x_1); +lean_closure_set(x_31, 3, x_2); +lean_closure_set(x_31, 4, x_26); +x_32 = lean_ctor_get(x_1, 1); +lean_inc(x_32); +x_33 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52___rarg), 5, 4); +lean_closure_set(x_33, 0, x_1); +lean_closure_set(x_33, 1, lean_box(0)); +lean_closure_set(x_33, 2, lean_box(0)); +lean_closure_set(x_33, 3, x_31); +x_34 = lean_apply_4(x_32, lean_box(0), lean_box(0), x_30, x_33); +return x_34; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4_(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__5___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__7___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__6___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__8___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__11___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__13___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__18___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__20___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__19___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__21___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__27___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__29___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__28___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__30___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +x_6 = lean_apply_2(x_2, lean_box(0), x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__14___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__15___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_2); +lean_ctor_set(x_8, 2, x_3); +lean_ctor_set(x_8, 3, x_4); +lean_ctor_set_uint8(x_8, sizeof(void*)*4, x_5); +lean_ctor_set_uint8(x_8, sizeof(void*)*4 + 1, x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +x_10 = lean_apply_2(x_6, lean_box(0), x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__22___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__23___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__6), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__24___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__25___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__3), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__16___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__7), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__31___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__32___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(x_1, x_16, x_17, x_14); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1; +lean_inc(x_2); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9___boxed), 5, 4); +lean_closure_set(x_20, 0, x_11); +lean_closure_set(x_20, 1, x_1); +lean_closure_set(x_20, 2, x_19); +lean_closure_set(x_20, 3, x_2); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__33___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +lean_inc(x_21); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_18, x_22); +x_24 = lean_box_usize(x_4); +x_25 = lean_box_usize(x_3); +lean_inc(x_1); +x_26 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10___boxed), 6, 5); +lean_closure_set(x_26, 0, x_24); +lean_closure_set(x_26, 1, x_13); +lean_closure_set(x_26, 2, x_1); +lean_closure_set(x_26, 3, x_2); +lean_closure_set(x_26, 4, x_25); +x_27 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__35___rarg), 5, 4); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, lean_box(0)); +lean_closure_set(x_27, 2, lean_box(0)); +lean_closure_set(x_27, 3, x_26); +x_28 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_23, x_27); +return x_28; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__40___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__42___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__41___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__43___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__1___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__2___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__3(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_3 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__36___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__37___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_7, 0, x_1); +lean_ctor_set(x_7, 1, x_2); +lean_ctor_set(x_7, 2, x_3); +lean_ctor_set(x_7, 3, x_4); +lean_ctor_set(x_7, 4, x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_apply_2(x_5, lean_box(0), x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 4); +lean_inc(x_5); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__6), 6, 5); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_7); +lean_closure_set(x_9, 4, x_5); +x_10 = lean_ctor_get(x_6, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__44___rarg), 5, 4); +lean_closure_set(x_11, 0, x_6); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_13 = lean_apply_2(x_5, lean_box(0), x_12); +x_14 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_13, x_11); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_8, 0); +lean_inc(x_15); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_inc(x_5); +x_17 = lean_apply_2(x_5, lean_box(0), x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_5); +lean_inc(x_10); +x_19 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_11); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 3); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_6); +lean_inc(x_8); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7___boxed), 7, 6); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_3); +lean_closure_set(x_11, 2, x_4); +lean_closure_set(x_11, 3, x_5); +lean_closure_set(x_11, 4, x_8); +lean_closure_set(x_11, 5, x_2); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__45___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8), 5, 4); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +lean_closure_set(x_6, 2, x_3); +lean_closure_set(x_6, 3, x_4); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__46___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_14); +lean_inc(x_16); +x_18 = lean_apply_2(x_16, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_19, 0, x_16); +lean_inc(x_7); +x_20 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_20, x_8); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__5), 3, 2); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_3); +lean_inc(x_2); +x_7 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__38___rarg(x_2, x_6, x_5); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__9), 4, 3); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__47___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__11(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_alloc_ctor(2, 3, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_3, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_7 = l_Lean_Widget_instRpcEncodingWithRpcRefMessageDataRpcRef; +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +x_9 = lean_box_usize(x_3); +lean_inc(x_1); +x_10 = lean_apply_4(x_8, lean_box(0), x_1, x_2, x_9); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__12), 4, 3); +lean_closure_set(x_11, 0, x_4); +lean_closure_set(x_11, 1, x_6); +lean_closure_set(x_11, 2, x_5); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__50___rarg), 5, 4); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_1); +lean_inc(x_2); +x_8 = lean_apply_2(x_2, lean_box(0), x_7); +x_9 = lean_box_usize(x_5); +lean_inc(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13___boxed), 6, 5); +lean_closure_set(x_10, 0, x_3); +lean_closure_set(x_10, 1, x_4); +lean_closure_set(x_10, 2, x_9); +lean_closure_set(x_10, 3, x_6); +lean_closure_set(x_10, 4, x_2); +x_11 = lean_ctor_get(x_3, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__51___rarg), 5, 4); +lean_closure_set(x_12, 0, x_3); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +lean_inc(x_1); +x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__2), 3, 2); +lean_closure_set(x_5, 0, x_1); +lean_closure_set(x_5, 1, x_2); +lean_inc(x_1); +x_6 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__3___rarg(x_1, x_5, x_4); +lean_inc(x_1); +x_7 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__3), 2, 1); +lean_closure_set(x_7, 0, x_1); +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); +x_9 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__9___rarg), 5, 4); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, lean_box(0)); +lean_closure_set(x_9, 2, lean_box(0)); +lean_closure_set(x_9, 3, x_7); +x_10 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_6, x_9); +return x_10; +} +case 1: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_11 = lean_ctor_get(x_3, 0); +lean_inc(x_11); +lean_dec(x_3); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_array_get_size(x_12); +x_14 = lean_usize_of_nat(x_13); +lean_dec(x_13); +x_15 = 0; +lean_inc(x_2); +lean_inc(x_1); +x_16 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(x_1, x_2, x_14, x_15, x_12); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__10), 4, 3); +lean_closure_set(x_17, 0, x_11); +lean_closure_set(x_17, 1, x_1); +lean_closure_set(x_17, 2, x_2); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__48___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +lean_inc(x_18); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_16, x_19); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__11), 2, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__49___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_21); +x_23 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_20, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +x_26 = lean_ctor_get(x_3, 2); +lean_inc(x_26); +lean_dec(x_3); +x_27 = lean_ctor_get(x_1, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_24); +lean_inc(x_28); +x_30 = lean_apply_2(x_28, lean_box(0), x_29); +lean_inc(x_1); +x_31 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14___boxed), 6, 5); +lean_closure_set(x_31, 0, x_25); +lean_closure_set(x_31, 1, x_28); +lean_closure_set(x_31, 2, x_1); +lean_closure_set(x_31, 3, x_2); +lean_closure_set(x_31, 4, x_26); +x_32 = lean_ctor_get(x_1, 1); +lean_inc(x_32); +x_33 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__52___rarg), 5, 4); +lean_closure_set(x_33, 0, x_1); +lean_closure_set(x_33, 1, lean_box(0)); +lean_closure_set(x_33, 2, lean_box(0)); +lean_closure_set(x_33, 3, x_31); +x_34 = lean_apply_4(x_32, lean_box(0), lean_box(0), x_30, x_33); +return x_34; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4_(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__1(x_4, x_2, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +uint8_t x_8; uint8_t x_9; lean_object* x_10; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = lean_unbox(x_7); +lean_dec(x_7); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4(x_1, x_2, x_3, x_4, x_8, x_6, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__11(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; lean_object* x_6; +x_5 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_6 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13(x_1, x_2, x_3, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__4___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__10___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__12___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__17___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__26___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__2(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +uint8_t x_8; uint8_t x_9; lean_object* x_10; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = lean_unbox(x_7); +lean_dec(x_7); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__4(x_1, x_2, x_3, x_4, x_8, x_6, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__9(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__10(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__39___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__4(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; lean_object* x_8; +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__13(x_1, x_2, x_7, x_4, x_5, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; lean_object* x_8; +x_7 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_8 = l_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__14(x_1, x_2, x_3, x_4, x_7, x_6); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed___lambda__1(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_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg(x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingMsgEmbed___lambda__2(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_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg(x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgEmbed___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed___lambda__1), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgEmbed___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed___lambda__2), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgEmbed___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingMsgEmbed___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingMsgEmbed___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingMsgEmbed() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingMsgEmbed___closed__3; +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("range", 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("fullRange", 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("severity", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("code", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("source", 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("message", 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("tags", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("relatedInformation", 18); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__1; +x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocation____x40_Lean_Data_Lsp_Basic___hyg_940____spec__2(x_2, x_3); +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_5; +lean_dec(x_1); +x_5 = !lean_is_exclusive(x_4); +if (x_5 == 0) +{ +return x_4; +} +else +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_4, 0); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_7, 0, x_6); +return x_7; +} +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_4, 0); +lean_inc(x_8); +lean_dec(x_4); +x_9 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__2; +x_10 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocation____x40_Lean_Data_Lsp_Basic___hyg_940____spec__2(x_2, x_9); +if (lean_obj_tag(x_10) == 0) +{ +uint8_t x_11; +lean_dec(x_8); +lean_dec(x_1); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +return x_10; +} +else +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_10, 0); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_12); +return x_13; +} +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_10, 0); +lean_inc(x_14); +lean_dec(x_10); +x_15 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__3; +x_16 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1036____spec__1(x_2, x_15); +if (lean_obj_tag(x_16) == 0) +{ +uint8_t x_17; +lean_dec(x_14); +lean_dec(x_8); +lean_dec(x_1); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +return x_16; +} +else +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_19, 0, x_18); +return x_19; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_16, 0); +lean_inc(x_20); +lean_dec(x_16); +x_21 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__4; +x_22 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1036____spec__2(x_2, x_21); +if (lean_obj_tag(x_22) == 0) +{ +uint8_t x_23; +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_8); +lean_dec(x_1); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) +{ +return x_22; +} +else +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_22, 0); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_25, 0, x_24); +return x_25; +} +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_22, 0); +lean_inc(x_26); +lean_dec(x_22); +x_27 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__5; +x_28 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2161____spec__1(x_2, x_27); +if (lean_obj_tag(x_28) == 0) +{ +uint8_t x_29; +lean_dec(x_26); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_8); +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) +{ +return x_28; +} +else +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_28, 0); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_31, 0, x_30); +return x_31; +} +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_28, 0); +lean_inc(x_32); +lean_dec(x_28); +x_33 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__6; +x_34 = l_Lean_Json_getObjValAs_x3f(x_2, lean_box(0), x_1, x_33); +if (lean_obj_tag(x_34) == 0) +{ +uint8_t x_35; +lean_dec(x_32); +lean_dec(x_26); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_8); +x_35 = !lean_is_exclusive(x_34); +if (x_35 == 0) +{ +return x_34; +} +else +{ +lean_object* x_36; lean_object* x_37; +x_36 = lean_ctor_get(x_34, 0); +lean_inc(x_36); +lean_dec(x_34); +x_37 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_37, 0, x_36); +return x_37; +} +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_34, 0); +lean_inc(x_38); +lean_dec(x_34); +x_39 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__7; +x_40 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1036____spec__3(x_2, x_39); +if (lean_obj_tag(x_40) == 0) +{ +uint8_t x_41; +lean_dec(x_38); +lean_dec(x_32); +lean_dec(x_26); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_8); +x_41 = !lean_is_exclusive(x_40); +if (x_41 == 0) +{ +return x_40; +} +else +{ +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_40, 0); +lean_inc(x_42); +lean_dec(x_40); +x_43 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_43, 0, x_42); +return x_43; +} +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_40, 0); +lean_inc(x_44); +lean_dec(x_40); +x_45 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__8; +x_46 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_fromJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_1036____spec__5(x_2, x_45); +if (lean_obj_tag(x_46) == 0) +{ +uint8_t x_47; +lean_dec(x_44); +lean_dec(x_38); +lean_dec(x_32); +lean_dec(x_26); +lean_dec(x_20); +lean_dec(x_14); +lean_dec(x_8); +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) +{ +return x_46; +} +else +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_46, 0); +lean_inc(x_48); +lean_dec(x_46); +x_49 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_49, 0, x_48); +return x_49; +} +} +else +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_46); +if (x_50 == 0) +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_46, 0); +x_52 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_52, 0, x_8); +lean_ctor_set(x_52, 1, x_14); +lean_ctor_set(x_52, 2, x_20); +lean_ctor_set(x_52, 3, x_26); +lean_ctor_set(x_52, 4, x_32); +lean_ctor_set(x_52, 5, x_38); +lean_ctor_set(x_52, 6, x_44); +lean_ctor_set(x_52, 7, x_51); +lean_ctor_set(x_46, 0, x_52); +return x_46; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_46, 0); +lean_inc(x_53); +lean_dec(x_46); +x_54 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_54, 0, x_8); +lean_ctor_set(x_54, 1, x_14); +lean_ctor_set(x_54, 2, x_20); +lean_ctor_set(x_54, 3, x_26); +lean_ctor_set(x_54, 4, x_32); +lean_ctor_set(x_54, 5, x_38); +lean_ctor_set(x_54, 6, x_44); +lean_ctor_set(x_54, 7, x_53); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_54); +return x_55; +} +} +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867_(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___boxed), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__6___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___boxed), 2, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__6(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__6___rarg), 1, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; 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; +x_3 = lean_ctor_get(x_2, 0); +lean_inc(x_3); +x_4 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(x_3); +x_5 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__1; +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_5); +lean_ctor_set(x_6, 1, x_4); +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_6); +lean_ctor_set(x_8, 1, x_7); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(x_9); +x_11 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__2; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_7); +x_14 = lean_ctor_get(x_2, 2); +lean_inc(x_14); +x_15 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__3; +x_16 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__1(x_15, x_14); +lean_dec(x_14); +x_17 = lean_ctor_get(x_2, 3); +lean_inc(x_17); +x_18 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__4; +x_19 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__2(x_18, x_17); +lean_dec(x_17); +x_20 = lean_ctor_get(x_2, 4); +lean_inc(x_20); +x_21 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__5; +x_22 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2131____spec__1(x_21, x_20); +lean_dec(x_20); +x_23 = lean_ctor_get(x_2, 5); +lean_inc(x_23); +x_24 = lean_apply_1(x_1, x_23); +x_25 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__6; +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_24); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_7); +x_28 = lean_ctor_get(x_2, 6); +lean_inc(x_28); +x_29 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__7; +x_30 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__3(x_29, x_28); +x_31 = lean_ctor_get(x_2, 7); +lean_inc(x_31); +lean_dec(x_2); +x_32 = l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__8; +x_33 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Diagnostics_0__Lean_Lsp_toJsonDiagnosticWith____x40_Lean_Data_Lsp_Diagnostics___hyg_953____spec__5(x_32, x_31); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_7); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_30); +lean_ctor_set(x_35, 1, x_34); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_27); +lean_ctor_set(x_36, 1, x_35); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_22); +lean_ctor_set(x_37, 1, x_36); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_19); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_16); +lean_ctor_set(x_39, 1, x_38); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_13); +lean_ctor_set(x_40, 1, x_39); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_8); +lean_ctor_set(x_41, 1, x_40); +x_42 = l_List_join___rarg(x_41); +x_43 = l_Lean_Json_mkObj(x_42); +return x_43; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038_(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__6___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1038____rarg), 2, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__6(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__6___rarg), 1, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__1___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__3___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_11); +lean_inc(x_2); +x_15 = lean_apply_2(x_2, lean_box(0), x_14); +x_16 = lean_box_usize(x_4); +x_17 = lean_box_usize(x_3); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_13); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__3___rarg), 5, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_15, x_20); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__6(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__6___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, uint8_t x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_box(x_6); +x_10 = lean_array_uset(x_2, x_1, x_9); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg(x_3, x_4, x_5, x_8, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_11); +lean_inc(x_2); +x_15 = lean_apply_2(x_2, lean_box(0), x_14); +x_16 = lean_box_usize(x_4); +x_17 = lean_box_usize(x_3); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_13); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__6___rarg), 5, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_15, x_20); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__7(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__7___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__8(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__8___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__9(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__9___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__10(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__10___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__11___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__12___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__12(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__12___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__13___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__13(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__13___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__15___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__15(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__15___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_11); +lean_inc(x_2); +x_15 = lean_apply_2(x_2, lean_box(0), x_14); +x_16 = lean_box_usize(x_4); +x_17 = lean_box_usize(x_3); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_13); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__15___rarg), 5, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_15, x_20); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__16___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__16(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__16___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__18___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__18(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__18___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, uint8_t x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_box(x_6); +x_10 = lean_array_uset(x_2, x_1, x_9); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg(x_3, x_4, x_5, x_8, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_11); +lean_inc(x_2); +x_15 = lean_apply_2(x_2, lean_box(0), x_14); +x_16 = lean_box_usize(x_4); +x_17 = lean_box_usize(x_3); +lean_inc(x_1); +x_18 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_18, 0, x_16); +lean_closure_set(x_18, 1, x_13); +lean_closure_set(x_18, 2, x_1); +lean_closure_set(x_18, 3, x_2); +lean_closure_set(x_18, 4, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +x_20 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__18___rarg), 5, 4); +lean_closure_set(x_20, 0, x_1); +lean_closure_set(x_20, 1, lean_box(0)); +lean_closure_set(x_20, 2, lean_box(0)); +lean_closure_set(x_20, 3, x_18); +x_21 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_15, x_20); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__19___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__19(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__19___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__20(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__20___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__21(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__21___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__22___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__22(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__22___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__23___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__23(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__23___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__24___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__24(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__24___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_2); +lean_ctor_set(x_10, 2, x_3); +lean_ctor_set(x_10, 3, x_4); +lean_ctor_set(x_10, 4, x_5); +lean_ctor_set(x_10, 5, x_6); +lean_ctor_set(x_10, 6, x_7); +lean_ctor_set(x_10, 7, x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = lean_apply_2(x_8, lean_box(0), x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_ctor_get(x_1, 7); +lean_inc(x_11); +lean_dec(x_1); +lean_inc(x_8); +x_12 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__1), 9, 8); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, x_3); +lean_closure_set(x_12, 2, x_4); +lean_closure_set(x_12, 3, x_5); +lean_closure_set(x_12, 4, x_6); +lean_closure_set(x_12, 5, x_7); +lean_closure_set(x_12, 6, x_10); +lean_closure_set(x_12, 7, x_8); +x_13 = lean_ctor_get(x_9, 1); lean_inc(x_13); -lean_inc(x_4); +lean_inc(x_9); +x_14 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__1___rarg), 5, 4); +lean_closure_set(x_14, 0, x_9); +lean_closure_set(x_14, 1, lean_box(0)); +lean_closure_set(x_14, 2, lean_box(0)); +lean_closure_set(x_14, 3, x_12); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_dec(x_9); +x_15 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_16 = lean_apply_2(x_8, lean_box(0), x_15); +x_17 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_16, x_14); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_18 = lean_ctor_get(x_11, 0); +lean_inc(x_18); +lean_dec(x_11); +x_19 = lean_array_get_size(x_18); +x_20 = lean_usize_of_nat(x_19); +lean_dec(x_19); +x_21 = 0; +lean_inc(x_8); +x_22 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg(x_9, x_8, x_20, x_21, x_18); +x_23 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_23, 0, x_8); +lean_inc(x_13); +x_24 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_22, x_23); +x_25 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_24, x_14); +return x_25; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_1, 6); +lean_inc(x_10); +lean_inc(x_8); +lean_inc(x_7); +x_11 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__2), 10, 9); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_2); +lean_closure_set(x_11, 2, x_3); +lean_closure_set(x_11, 3, x_4); +lean_closure_set(x_11, 4, x_5); +lean_closure_set(x_11, 5, x_6); +lean_closure_set(x_11, 6, x_9); +lean_closure_set(x_11, 7, x_7); +lean_closure_set(x_11, 8, x_8); +x_12 = lean_ctor_get(x_8, 1); +lean_inc(x_12); +lean_inc(x_8); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__4___rarg), 5, 4); +lean_closure_set(x_13, 0, x_8); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_8); +x_14 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_15 = lean_apply_2(x_7, lean_box(0), x_14); +x_16 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_15, x_13); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_17 = lean_ctor_get(x_10, 0); +lean_inc(x_17); +lean_dec(x_10); +x_18 = lean_array_get_size(x_17); +x_19 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_20 = 0; +lean_inc(x_7); +x_21 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg(x_8, x_7, x_19, x_20, x_17); +x_22 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_22, 0, x_7); +lean_inc(x_12); +x_23 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_21, x_22); +x_24 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_23, x_13); +return x_24; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_2, 5); +lean_inc(x_12); lean_inc(x_3); -x_14 = lean_apply_4(x_12, lean_box(0), x_3, x_4, x_13); +x_13 = lean_apply_4(x_11, lean_box(0), x_3, x_4, x_12); lean_inc(x_3); -x_15 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__14), 11, 10); -lean_closure_set(x_15, 0, x_2); -lean_closure_set(x_15, 1, x_5); -lean_closure_set(x_15, 2, x_6); -lean_closure_set(x_15, 3, x_7); -lean_closure_set(x_15, 4, x_8); -lean_closure_set(x_15, 5, x_11); -lean_closure_set(x_15, 6, x_3); -lean_closure_set(x_15, 7, x_9); -lean_closure_set(x_15, 8, x_4); -lean_closure_set(x_15, 9, x_10); -x_16 = lean_ctor_get(x_3, 1); -lean_inc(x_16); -x_17 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__3___rarg), 5, 4); -lean_closure_set(x_17, 0, x_3); -lean_closure_set(x_17, 1, lean_box(0)); -lean_closure_set(x_17, 2, lean_box(0)); -lean_closure_set(x_17, 3, x_15); -x_18 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_14, x_17); -return x_18; +x_14 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__3), 9, 8); +lean_closure_set(x_14, 0, x_2); +lean_closure_set(x_14, 1, x_5); +lean_closure_set(x_14, 2, x_6); +lean_closure_set(x_14, 3, x_7); +lean_closure_set(x_14, 4, x_8); +lean_closure_set(x_14, 5, x_10); +lean_closure_set(x_14, 6, x_9); +lean_closure_set(x_14, 7, x_3); +x_15 = lean_ctor_get(x_3, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__7___rarg), 5, 4); +lean_closure_set(x_16, 0, x_3); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_13, x_16); +return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_1, 4); -lean_inc(x_12); -lean_inc(x_4); -lean_inc(x_3); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__15), 11, 10); -lean_closure_set(x_13, 0, x_2); -lean_closure_set(x_13, 1, x_1); -lean_closure_set(x_13, 2, x_3); -lean_closure_set(x_13, 3, x_4); -lean_closure_set(x_13, 4, x_5); -lean_closure_set(x_13, 5, x_6); -lean_closure_set(x_13, 6, x_7); -lean_closure_set(x_13, 7, x_11); -lean_closure_set(x_13, 8, x_8); -lean_closure_set(x_13, 9, x_9); -x_14 = lean_ctor_get(x_3, 1); -lean_inc(x_14); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_1, 4); +lean_inc(x_10); +lean_inc(x_8); lean_inc(x_3); -x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__4___rarg), 5, 4); -lean_closure_set(x_15, 0, x_3); -lean_closure_set(x_15, 1, lean_box(0)); -lean_closure_set(x_15, 2, lean_box(0)); -lean_closure_set(x_15, 3, x_13); -if (lean_obj_tag(x_12) == 0) +x_11 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__4), 10, 9); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, x_1); +lean_closure_set(x_11, 2, x_3); +lean_closure_set(x_11, 3, x_4); +lean_closure_set(x_11, 4, x_5); +lean_closure_set(x_11, 5, x_6); +lean_closure_set(x_11, 6, x_7); +lean_closure_set(x_11, 7, x_9); +lean_closure_set(x_11, 8, x_8); +x_12 = lean_ctor_get(x_3, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__8___rarg), 5, 4); +lean_closure_set(x_13, 0, x_3); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_10); -lean_dec(x_4); -x_16 = lean_ctor_get(x_3, 0); -lean_inc(x_16); -lean_dec(x_3); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -x_19 = lean_apply_2(x_17, lean_box(0), x_18); -x_20 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_19, x_15); -return x_20; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_15 = lean_apply_2(x_8, lean_box(0), x_14); +x_16 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_15, x_13); +return x_16; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_12, 0); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_17 = lean_ctor_get(x_10, 0); +lean_inc(x_17); lean_dec(x_10); -lean_inc(x_3); -x_23 = lean_apply_4(x_22, lean_box(0), x_3, x_4, x_21); -x_24 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__12), 2, 1); -lean_closure_set(x_24, 0, x_3); -lean_inc(x_14); -x_25 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_23, x_24); -x_26 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_25, x_15); -return x_26; +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_17); +lean_inc(x_8); +x_19 = lean_apply_2(x_8, lean_box(0), x_18); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_20, 0, x_8); +lean_inc(x_12); +x_21 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_19, x_20); +x_22 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_21, x_13); +return x_22; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_1, 3); -lean_inc(x_12); -lean_inc(x_4); -lean_inc(x_3); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__16), 11, 10); -lean_closure_set(x_13, 0, x_1); -lean_closure_set(x_13, 1, x_2); -lean_closure_set(x_13, 2, x_3); -lean_closure_set(x_13, 3, x_4); -lean_closure_set(x_13, 4, x_5); -lean_closure_set(x_13, 5, x_6); -lean_closure_set(x_13, 6, x_11); -lean_closure_set(x_13, 7, x_7); -lean_closure_set(x_13, 8, x_8); -lean_closure_set(x_13, 9, x_9); -x_14 = lean_ctor_get(x_3, 1); -lean_inc(x_14); +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_1, 3); +lean_inc(x_9); +lean_inc(x_7); lean_inc(x_3); -x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__5___rarg), 5, 4); -lean_closure_set(x_15, 0, x_3); -lean_closure_set(x_15, 1, lean_box(0)); -lean_closure_set(x_15, 2, lean_box(0)); -lean_closure_set(x_15, 3, x_13); -if (lean_obj_tag(x_12) == 0) +x_10 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__5), 9, 8); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_3); +lean_closure_set(x_10, 3, x_4); +lean_closure_set(x_10, 4, x_5); +lean_closure_set(x_10, 5, x_6); +lean_closure_set(x_10, 6, x_8); +lean_closure_set(x_10, 7, x_7); +x_11 = lean_ctor_get(x_3, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__9___rarg), 5, 4); +lean_closure_set(x_12, 0, x_3); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +if (lean_obj_tag(x_9) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_10); -lean_dec(x_4); -x_16 = lean_ctor_get(x_3, 0); -lean_inc(x_16); -lean_dec(x_3); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -x_19 = lean_apply_2(x_17, lean_box(0), x_18); -x_20 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_19, x_15); -return x_20; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_14 = lean_apply_2(x_7, lean_box(0), x_13); +x_15 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_14, x_12); +return x_15; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_12, 0); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); -lean_dec(x_10); -lean_inc(x_3); -x_23 = lean_apply_4(x_22, lean_box(0), x_3, x_4, x_21); -x_24 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__12), 2, 1); -lean_closure_set(x_24, 0, x_3); -lean_inc(x_14); -x_25 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_23, x_24); -x_26 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_25, x_15); -return x_26; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_16 = lean_ctor_get(x_9, 0); +lean_inc(x_16); +lean_dec(x_9); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_16); +lean_inc(x_7); +x_18 = lean_apply_2(x_7, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_19, 0, x_7); +lean_inc(x_11); +x_20 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_20, x_12); +return x_21; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__18(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__7(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -4163,163 +13122,318 @@ uint8_t x_3; x_3 = !lean_is_exclusive(x_2); if (x_3 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_apply_2(x_5, lean_box(0), x_2); -return x_6; +lean_object* x_4; +x_4 = lean_apply_2(x_1, lean_box(0), x_2); +return x_4; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); lean_dec(x_2); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_10, 0, x_7); -x_11 = lean_apply_2(x_9, lean_box(0), x_10); -return x_11; +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_1, lean_box(0), x_6); +return x_7; } } else { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_2); -if (x_12 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_2); +if (x_8 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_2, 0); -x_14 = lean_ctor_get(x_1, 0); -lean_inc(x_14); -lean_dec(x_1); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_13); -lean_ctor_set(x_2, 0, x_16); -x_17 = lean_apply_2(x_15, lean_box(0), x_2); -return x_17; +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_2, 0, x_10); +x_11 = lean_apply_2(x_1, lean_box(0), x_2); +return x_11; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_18 = lean_ctor_get(x_2, 0); -lean_inc(x_18); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); lean_dec(x_2); -x_19 = lean_ctor_get(x_1, 0); -lean_inc(x_19); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = lean_apply_2(x_1, lean_box(0), x_14); +return x_15; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 2); +lean_inc(x_8); +lean_inc(x_6); +lean_inc(x_3); +x_9 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__6), 8, 7); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_3); +lean_closure_set(x_9, 3, x_4); +lean_closure_set(x_9, 4, x_5); +lean_closure_set(x_9, 5, x_7); +lean_closure_set(x_9, 6, x_6); +x_10 = lean_ctor_get(x_3, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__10___rarg), 5, 4); +lean_closure_set(x_11, 0, x_3); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_13 = lean_apply_2(x_6, lean_box(0), x_12); +x_14 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_13, x_11); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_8, 0); +lean_inc(x_15); +lean_dec(x_8); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_inc(x_6); +x_17 = lean_apply_2(x_6, lean_box(0), x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_6); +lean_inc(x_10); +x_19 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_11); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_7); +lean_inc(x_2); +x_9 = lean_apply_2(x_2, lean_box(0), x_8); +lean_inc(x_4); +x_10 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__8), 7, 6); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_3); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +lean_closure_set(x_10, 4, x_6); +lean_closure_set(x_10, 5, x_2); +x_11 = lean_ctor_get(x_4, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__11___rarg), 5, 4); +lean_closure_set(x_12, 0, x_4); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_6); +lean_inc(x_8); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +lean_inc(x_3); +x_11 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__9), 6, 5); +lean_closure_set(x_11, 0, x_5); +lean_closure_set(x_11, 1, x_8); +lean_closure_set(x_11, 2, x_1); +lean_closure_set(x_11, 3, x_3); +lean_closure_set(x_11, 4, x_4); +x_12 = lean_ctor_get(x_3, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__12___rarg), 5, 4); +lean_closure_set(x_13, 0, x_3); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_2); +lean_ctor_set(x_10, 2, x_3); +lean_ctor_set(x_10, 3, x_4); +lean_ctor_set(x_10, 4, x_5); +lean_ctor_set(x_10, 5, x_6); +lean_ctor_set(x_10, 6, x_7); +lean_ctor_set(x_10, 7, x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = lean_apply_2(x_8, lean_box(0), x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_ctor_get(x_1, 7); +lean_inc(x_11); lean_dec(x_1); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_21, 0, x_18); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_21); -x_23 = lean_apply_2(x_20, lean_box(0), x_22); -return x_23; +lean_inc(x_8); +x_12 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__11), 9, 8); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, x_3); +lean_closure_set(x_12, 2, x_4); +lean_closure_set(x_12, 3, x_5); +lean_closure_set(x_12, 4, x_6); +lean_closure_set(x_12, 5, x_7); +lean_closure_set(x_12, 6, x_10); +lean_closure_set(x_12, 7, x_8); +x_13 = lean_ctor_get(x_9, 1); +lean_inc(x_13); +lean_inc(x_9); +x_14 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__13___rarg), 5, 4); +lean_closure_set(x_14, 0, x_9); +lean_closure_set(x_14, 1, lean_box(0)); +lean_closure_set(x_14, 2, lean_box(0)); +lean_closure_set(x_14, 3, x_12); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_dec(x_9); +x_15 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_16 = lean_apply_2(x_8, lean_box(0), x_15); +x_17 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_16, x_14); +return x_17; } +else +{ +lean_object* x_18; lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_18 = lean_ctor_get(x_11, 0); +lean_inc(x_18); +lean_dec(x_11); +x_19 = lean_array_get_size(x_18); +x_20 = lean_usize_of_nat(x_19); +lean_dec(x_19); +x_21 = 0; +lean_inc(x_8); +x_22 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg(x_9, x_8, x_20, x_21, x_18); +x_23 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_23, 0, x_8); +lean_inc(x_13); +x_24 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_22, x_23); +x_25 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_24, x_14); +return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_1, 2); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_1, 6); +lean_inc(x_10); +lean_inc(x_8); +lean_inc(x_7); +x_11 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__12), 10, 9); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_2); +lean_closure_set(x_11, 2, x_3); +lean_closure_set(x_11, 3, x_4); +lean_closure_set(x_11, 4, x_5); +lean_closure_set(x_11, 5, x_6); +lean_closure_set(x_11, 6, x_9); +lean_closure_set(x_11, 7, x_7); +lean_closure_set(x_11, 8, x_8); +x_12 = lean_ctor_get(x_8, 1); lean_inc(x_12); -lean_inc(x_4); -lean_inc(x_3); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__17), 11, 10); -lean_closure_set(x_13, 0, x_1); -lean_closure_set(x_13, 1, x_2); -lean_closure_set(x_13, 2, x_3); -lean_closure_set(x_13, 3, x_4); -lean_closure_set(x_13, 4, x_5); -lean_closure_set(x_13, 5, x_11); -lean_closure_set(x_13, 6, x_6); -lean_closure_set(x_13, 7, x_7); -lean_closure_set(x_13, 8, x_8); -lean_closure_set(x_13, 9, x_9); -x_14 = lean_ctor_get(x_3, 1); -lean_inc(x_14); -lean_inc(x_3); -x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__6___rarg), 5, 4); -lean_closure_set(x_15, 0, x_3); -lean_closure_set(x_15, 1, lean_box(0)); -lean_closure_set(x_15, 2, lean_box(0)); -lean_closure_set(x_15, 3, x_13); -if (lean_obj_tag(x_12) == 0) +lean_inc(x_8); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__16___rarg), 5, 4); +lean_closure_set(x_13, 0, x_8); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_10); -lean_dec(x_4); -x_16 = lean_ctor_get(x_3, 0); -lean_inc(x_16); -lean_dec(x_3); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1; -x_19 = lean_apply_2(x_17, lean_box(0), x_18); -x_20 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_19, x_15); -return x_20; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_8); +x_14 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_15 = lean_apply_2(x_7, lean_box(0), x_14); +x_16 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_15, x_13); +return x_16; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_12, 0); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_ctor_get(x_10, 1); -lean_inc(x_22); +lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_17 = lean_ctor_get(x_10, 0); +lean_inc(x_17); lean_dec(x_10); -lean_inc(x_3); -x_23 = lean_apply_4(x_22, lean_box(0), x_3, x_4, x_21); -x_24 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__18), 2, 1); -lean_closure_set(x_24, 0, x_3); -lean_inc(x_14); -x_25 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_23, x_24); -x_26 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_25, x_15); -return x_26; +x_18 = lean_array_get_size(x_17); +x_19 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_20 = 0; +lean_inc(x_7); +x_21 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg(x_8, x_7, x_19, x_20, x_17); +x_22 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_22, 0, x_7); +lean_inc(x_12); +x_23 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_21, x_22); +x_24 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_23, x_13); +return x_24; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__20(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_12 = lean_ctor_get(x_1, 1); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_2, 5); lean_inc(x_12); -lean_inc(x_4); lean_inc(x_3); -x_13 = lean_apply_4(x_2, lean_box(0), x_3, x_4, x_12); +x_13 = lean_apply_4(x_11, lean_box(0), x_3, x_4, x_12); lean_inc(x_3); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__19), 11, 10); -lean_closure_set(x_14, 0, x_1); +x_14 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__13), 9, 8); +lean_closure_set(x_14, 0, x_2); lean_closure_set(x_14, 1, x_5); -lean_closure_set(x_14, 2, x_3); -lean_closure_set(x_14, 3, x_4); -lean_closure_set(x_14, 4, x_11); -lean_closure_set(x_14, 5, x_6); -lean_closure_set(x_14, 6, x_7); -lean_closure_set(x_14, 7, x_8); -lean_closure_set(x_14, 8, x_9); -lean_closure_set(x_14, 9, x_10); +lean_closure_set(x_14, 2, x_6); +lean_closure_set(x_14, 3, x_7); +lean_closure_set(x_14, 4, x_8); +lean_closure_set(x_14, 5, x_10); +lean_closure_set(x_14, 6, x_9); +lean_closure_set(x_14, 7, x_3); x_15 = lean_ctor_get(x_3, 1); lean_inc(x_15); -x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__7___rarg), 5, 4); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__19___rarg), 5, 4); lean_closure_set(x_16, 0, x_3); lean_closure_set(x_16, 1, lean_box(0)); lean_closure_set(x_16, 2, lean_box(0)); @@ -4328,83 +13442,344 @@ x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_13, x_16); return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__21(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_12 = lean_ctor_get(x_1, 1); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_1, 4); +lean_inc(x_10); +lean_inc(x_8); +lean_inc(x_3); +x_11 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__14), 10, 9); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, x_1); +lean_closure_set(x_11, 2, x_3); +lean_closure_set(x_11, 3, x_4); +lean_closure_set(x_11, 4, x_5); +lean_closure_set(x_11, 5, x_6); +lean_closure_set(x_11, 6, x_7); +lean_closure_set(x_11, 7, x_9); +lean_closure_set(x_11, 8, x_8); +x_12 = lean_ctor_get(x_3, 1); lean_inc(x_12); -lean_dec(x_1); -x_13 = lean_ctor_get(x_11, 0); -lean_inc(x_13); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__20___rarg), 5, 4); +lean_closure_set(x_13, 0, x_3); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_15 = lean_apply_2(x_8, lean_box(0), x_14); +x_16 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_15, x_13); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_17 = lean_ctor_get(x_10, 0); +lean_inc(x_17); +lean_dec(x_10); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_17); +lean_inc(x_8); +x_19 = lean_apply_2(x_8, lean_box(0), x_18); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_20, 0, x_8); lean_inc(x_12); -lean_inc(x_10); -lean_inc(x_9); -x_14 = lean_apply_4(x_12, lean_box(0), x_9, x_10, x_13); +x_21 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_19, x_20); +x_22 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_21, x_13); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_1, 3); lean_inc(x_9); -x_15 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__20), 11, 10); -lean_closure_set(x_15, 0, x_11); -lean_closure_set(x_15, 1, x_12); -lean_closure_set(x_15, 2, x_9); -lean_closure_set(x_15, 3, x_10); -lean_closure_set(x_15, 4, x_2); -lean_closure_set(x_15, 5, x_3); -lean_closure_set(x_15, 6, x_4); -lean_closure_set(x_15, 7, x_5); -lean_closure_set(x_15, 8, x_6); -lean_closure_set(x_15, 9, x_7); -x_16 = lean_ctor_get(x_9, 1); +lean_inc(x_7); +lean_inc(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__15), 9, 8); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_3); +lean_closure_set(x_10, 3, x_4); +lean_closure_set(x_10, 4, x_5); +lean_closure_set(x_10, 5, x_6); +lean_closure_set(x_10, 6, x_8); +lean_closure_set(x_10, 7, x_7); +x_11 = lean_ctor_get(x_3, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__21___rarg), 5, 4); +lean_closure_set(x_12, 0, x_3); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_14 = lean_apply_2(x_7, lean_box(0), x_13); +x_15 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_14, x_12); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_16 = lean_ctor_get(x_9, 0); lean_inc(x_16); -x_17 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___spec__8___rarg), 5, 4); -lean_closure_set(x_17, 0, x_9); -lean_closure_set(x_17, 1, lean_box(0)); -lean_closure_set(x_17, 2, lean_box(0)); -lean_closure_set(x_17, 3, x_15); -x_18 = lean_apply_4(x_16, lean_box(0), lean_box(0), x_14, x_17); -return x_18; +lean_dec(x_9); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_16); +lean_inc(x_7); +x_18 = lean_apply_2(x_7, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____rarg___lambda__7), 2, 1); +lean_closure_set(x_19, 0, x_7); +lean_inc(x_11); +x_20 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_20, x_12); +return x_21; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 2); +lean_inc(x_8); +lean_inc(x_6); lean_inc(x_3); -lean_inc(x_5); +x_9 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__16), 8, 7); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_3); +lean_closure_set(x_9, 3, x_4); +lean_closure_set(x_9, 4, x_5); +lean_closure_set(x_9, 5, x_7); +lean_closure_set(x_9, 6, x_6); +x_10 = lean_ctor_get(x_3, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__22___rarg), 5, 4); +lean_closure_set(x_11, 0, x_3); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1; +x_13 = lean_apply_2(x_6, lean_box(0), x_12); +x_14 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_13, x_11); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_8, 0); +lean_inc(x_15); +lean_dec(x_8); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_inc(x_6); +x_17 = lean_apply_2(x_6, lean_box(0), x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_6); +lean_inc(x_10); +x_19 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_11); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_7 = lean_ctor_get(x_1, 1); lean_inc(x_7); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_7); +lean_inc(x_2); +x_9 = lean_apply_2(x_2, lean_box(0), x_8); +lean_inc(x_4); +x_10 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__17), 7, 6); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_3); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +lean_closure_set(x_10, 4, x_6); +lean_closure_set(x_10, 5, x_2); +x_11 = lean_ctor_get(x_4, 1); lean_inc(x_11); -lean_inc(x_13); -lean_inc(x_9); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__23___rarg), 5, 4); +lean_closure_set(x_12, 0, x_4); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_6); +lean_inc(x_8); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +lean_inc(x_3); +x_11 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__18), 6, 5); +lean_closure_set(x_11, 0, x_5); +lean_closure_set(x_11, 1, x_8); +lean_closure_set(x_11, 2, x_1); +lean_closure_set(x_11, 3, x_3); +lean_closure_set(x_11, 4, x_4); +x_12 = lean_ctor_get(x_3, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__24___rarg), 5, 4); +lean_closure_set(x_13, 0, x_3); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_inc(x_1); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__10), 11, 7); -lean_closure_set(x_14, 0, x_1); -lean_closure_set(x_14, 1, x_9); -lean_closure_set(x_14, 2, x_13); -lean_closure_set(x_14, 3, x_11); -lean_closure_set(x_14, 4, x_7); -lean_closure_set(x_14, 5, x_5); -lean_closure_set(x_14, 6, x_3); -x_15 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__21), 11, 7); -lean_closure_set(x_15, 0, x_1); -lean_closure_set(x_15, 1, x_9); -lean_closure_set(x_15, 2, x_13); -lean_closure_set(x_15, 3, x_11); -lean_closure_set(x_15, 4, x_7); -lean_closure_set(x_15, 5, x_5); -lean_closure_set(x_15, 6, x_3); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -return x_16; +x_2 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__10), 5, 1); +lean_closure_set(x_2, 0, x_1); +x_3 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg___lambda__19), 5, 1); +lean_closure_set(x_3, 0, x_1); +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Lsp_instRpcEncodingDiagnosticWith(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg), 13, 0); +x_3 = lean_alloc_closure((void*)(l_Lean_Lsp_instRpcEncodingDiagnosticWith___rarg), 1, 0); return x_3; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__2___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; uint8_t x_9; lean_object* x_10; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = lean_unbox(x_6); +lean_dec(x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__5___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__14___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; uint8_t x_9; lean_object* x_10; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = lean_unbox(x_6); +lean_dec(x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Lsp_instRpcEncodingDiagnosticWith___spec__17___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -7927,48 +17302,74 @@ l_Lean_Widget_instInhabitedMsgEmbed___closed__3 = _init_l_Lean_Widget_instInhabi lean_mark_persistent(l_Lean_Widget_instInhabitedMsgEmbed___closed__3); l_Lean_Widget_instInhabitedMsgEmbed = _init_l_Lean_Widget_instInhabitedMsgEmbed(); lean_mark_persistent(l_Lean_Widget_instInhabitedMsgEmbed); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__1); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__2 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__2(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__1___closed__2); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__1); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__2); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__3 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__3(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__3); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__4 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__4(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__4); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__5 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__5(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__5); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__2___closed__6); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___lambda__3___closed__1); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_225____rarg___closed__1); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_532____rarg___closed__1); -l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1 = _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1(); -lean_mark_persistent(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____spec__1___rarg___closed__1); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__1); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__2 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__2(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__2); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__3 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__3(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__3); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__4 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__4(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__4); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__5 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__5(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__5); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__6 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__6(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__6); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__7 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__7(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__7); -l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__8 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__8(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_1317____rarg___closed__8); -l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1 = _init_l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Widget_instRpcEncodingDiagnosticWithRpcEncodingPacket___rarg___lambda__3___closed__1); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__1); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__2 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__1___closed__2); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__1); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__2); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__3 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__3); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__4 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__4(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__4); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__5 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__5(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__5); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__6); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__7); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__8); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__9); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__2___closed__10); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____lambda__3___closed__1); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_125____closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__5___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__5___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__5___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__5 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__5(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__5); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320____closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320____closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_320____closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__5___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__5___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__5___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__5 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__5(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__5); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___lambda__8___closed__1); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcEncode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingMsgEmbed_rpcDecode____x40_Lean_Widget_InteractiveDiagnostic___hyg_4____spec__34___rarg___boxed__const__1); +l_Lean_Widget_instRpcEncodingMsgEmbed___closed__1 = _init_l_Lean_Widget_instRpcEncodingMsgEmbed___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgEmbed___closed__1); +l_Lean_Widget_instRpcEncodingMsgEmbed___closed__2 = _init_l_Lean_Widget_instRpcEncodingMsgEmbed___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgEmbed___closed__2); +l_Lean_Widget_instRpcEncodingMsgEmbed___closed__3 = _init_l_Lean_Widget_instRpcEncodingMsgEmbed___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgEmbed___closed__3); +l_Lean_Widget_instRpcEncodingMsgEmbed = _init_l_Lean_Widget_instRpcEncodingMsgEmbed(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingMsgEmbed); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__1); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__2 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__2(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__2); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__3 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__3(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__3); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__4 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__4(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__4); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__5 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__5(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__5); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__6 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__6(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__6); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__7 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__7(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__7); +l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__8 = _init_l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__8(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_867____rarg___closed__8); l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___closed__1 = _init_l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___closed__1(); lean_mark_persistent(l_Lean_Widget_InteractiveDiagnostic_toDiagnostic_prettyTt___closed__1); l_Lean_Widget_instInhabitedEmbedFmt___closed__1 = _init_l_Lean_Widget_instInhabitedEmbedFmt___closed__1(); diff --git a/stage0/stdlib/Lean/Widget/InteractiveGoal.c b/stage0/stdlib/Lean/Widget/InteractiveGoal.c index 22ddba2c8a07..d9f59eb81762 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveGoal.c +++ b/stage0/stdlib/Lean/Widget/InteractiveGoal.c @@ -14,265 +14,1139 @@ extern "C" { #endif lean_object* l_List_reverse___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1(size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__63(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__34(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Widget_goalToInteractive___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_Widget_goalToInteractive___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedInteractiveHypothesisBundle; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__48(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__59(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__72(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__23(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__77___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__56(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__66___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__65(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__22___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_erase_macro_scopes(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__31___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__22___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__19(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__43___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__49___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__22(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__63___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__11(lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__4(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__6(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__8(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__39___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__14(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__72___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__2(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Widget_ppExprTagged(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__76(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3; uint8_t l_Lean_LocalDecl_isAuxDecl(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__52___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__18(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__1(lean_object*, lean_object*, size_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__54___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__12(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__57(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__18(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__36(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__34___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__36(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__6(lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__2; static lean_object* l_Lean_Widget_goalToInteractive___closed__3; -lean_object* l_Lean_Json_getObjValAs_x3f(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__74___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__38___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__21(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__21(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__50(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__26(lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__6(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__6(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__44(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__53(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__26___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__7(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__9(lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__10(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__76(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__55(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_pp_auxDecls; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__7(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__18(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__70(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__28(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed__const__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__39___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29(lean_object*); +lean_object* l_Except_orElseLazy___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__33___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__58(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__1___closed__1; static lean_object* l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__3; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__20___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__73___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__19(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__3; +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__5; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___boxed(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_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__32(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__52(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__22(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__84(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__56___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_addInteractiveHypothesisBundle___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__75___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__51___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____closed__1; static lean_object* l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__34___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__3; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_InteractiveGoal_pretty___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__61(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__60(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_addInteractiveHypothesisBundle___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_Widget_instFromJsonRpcEncodingPacket__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getStr_x3f(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__3; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__73(lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__74(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42(lean_object*); lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__73___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__7___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66(lean_object*); +lean_object* lean_string_append(lean_object*, lean_object*); lean_object* l_Lean_Meta_isClass_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_Widget_goalToInteractive___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__13___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__7(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40(lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__4; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__5___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__22___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__68___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__24(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__47(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__70___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237_(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414_(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2236_(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2648_(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed__const__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__24(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1563_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__5(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__39___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16(lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__beqOption____x40_Init_Data_Option_Basic___hyg_803____at_Lean_Meta_ppGoal_ppVars___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__31(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__26___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__6; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__33___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__12(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__41(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__55___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__37___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__80___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_join___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed__const__1; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_addInteractiveHypothesisBundle___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__7(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__37___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__39(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__29(lean_object*); LEAN_EXPORT lean_object* l_List_filterTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__1(lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__63___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__46___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__3; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__45___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40(lean_object*); lean_object* l_Lean_Widget_TaggedText_stripTags___rarg(lean_object*); static lean_object* l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__15(lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__43(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__37(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__70___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__23(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__7(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__72(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__61(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__10___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__74___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__65(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__77(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__34___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__64___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__43___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__13(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveGoal_pretty(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveHypothesisBundle_val_x3f___default; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__68(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__39(lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__34___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__4(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__1(lean_object*, lean_object*, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_addInteractiveHypothesisBundle___spec__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__57___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__71(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Widget_goalToInteractive___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__59___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__7(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__57___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__47(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__31(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__33(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_fget(lean_object*, lean_object*); uint8_t l_Lean_Option_get___at_Lean_getSanitizeNames___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__55___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_parseTagged(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__24(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__61___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__8(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__31(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__5(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__75___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__32___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__22(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__63___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__44___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__33___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__26___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__56(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__30___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__4; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11___boxed__const__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__13(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__31___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_addInteractiveHypothesisBundle___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedInteractiveGoal; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__9(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__8(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__51(lean_object*); +static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__27(lean_object*); static lean_object* l_Lean_Widget_InteractiveGoal_pretty___closed__3; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_panic___at_Lean_Json_setObjVal_x21___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_goalToInteractive___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__37___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__42___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__72___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__53___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__57___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_goalToInteractive___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__3___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__4; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__39(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__10(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__53(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__10(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__26___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__54(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_RBNode_findCore___at_Lean_Meta_removeUnused___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__10(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__44(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__28(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__9(lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_Widget_goalToInteractive___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___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_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Widget_goalToInteractive___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__58___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__4; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__14(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__31___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__5; -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLCtx___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__21(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2161____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__13(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__69(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__26(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__36(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__74(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__80(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__77___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_addInteractiveHypothesisBundle___spec__1(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__45(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__4(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__8(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__67___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__75(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__4(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__49___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__50___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__20___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__42___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_JsonRpc_instFromJsonMessage___spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__76___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__71___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845____spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_Widget_goalToInteractive___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_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__37___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__54(lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__7; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__4(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__66(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__64(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed__const__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__70(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__1(lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__22___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__44___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__9(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__56___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__46(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__61(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__15___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__51___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__28(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__45___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__65___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__8(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__3; LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__2(lean_object*, lean_object*); +lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__27(lean_object*); uint8_t l_Array_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__52___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__10(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__9(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__51(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__33___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__43(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__6(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__4(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2648____rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__38(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__26(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__78___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__60(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__8(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__52(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__32(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__57(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__4; +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__3; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__62___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45(lean_object*); size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__1; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__9___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__4___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__61___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__14(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__30(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__47___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_fvarId(lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__69(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__78(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__49(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__1(lean_object*, lean_object*, size_t); lean_object* l_Lean_throwError___at_Lean_Meta_mkSimpCongrTheorem___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__71___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__4___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__4(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__47___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__7(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__23(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__48(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__83___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38(lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__2(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_addInteractiveHypothesisBundle___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__29___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +extern lean_object* l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_Widget_goalToInteractive___spec__2(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_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__5(lean_object*); static lean_object* l_Lean_Widget_goalToInteractive___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__63(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__46___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__81(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_String_intercalate(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__34(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__69___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__60___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__10; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Json_opt___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3(lean_object*, lean_object*); lean_object* l_Lean_Json_getObjValD(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__3(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__4___rarg(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___closed__1; -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__46(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__33(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__75(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__14(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__43(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__2(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__37(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_addInteractiveHypothesisBundle(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_Widget_goalToInteractive___spec__3(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__41(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__42(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__83(lean_object*); static lean_object* l_Lean_Widget_goalToInteractive___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__12(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__73(lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__35(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__71(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__20(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491____closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket(lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__2___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__20___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__5(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__67(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__43___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Name_isAnonymous(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__3___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__35(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__60___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__15(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__39___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__6(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__12(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__47(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__70___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__20(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7(lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__78___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845____spec__1(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__65(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__15(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__46___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21___boxed__const__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__6; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__19___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__19(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__79(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedInteractiveTermGoal; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__58___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MetavarContext_findDecl_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2131____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__47___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forInAux___at_Lean_Widget_goalToInteractive___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__66___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__7(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__10(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__44(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__41___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3(lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__2___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__70(lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__55(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__14___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__13___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__27(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__42(lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__5(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041_(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096_(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199_(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586_(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__51(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__34(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136_(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491_(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__5___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__1(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__52___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__5(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__28(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__81___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__66(lean_object*); +lean_object* l_Lean_Syntax_decodeNameLit(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__59(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed__const__1; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__24(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__84___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__22(lean_object*); static lean_object* l_Lean_Widget_goalToInteractive___closed__4; +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__32___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__65___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_addInteractiveHypothesisBundle___spec__2(size_t, size_t, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__4; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__19(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__18___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__3; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__35(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_InteractiveGoal_pretty___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__9; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__52(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__20(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__32(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__53___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__59___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_goalToInteractive___lambda__1(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_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocation____x40_Lean_Data_Lsp_Basic___hyg_940____spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); static lean_object* l_Lean_Widget_instInhabitedInteractiveGoal___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Json_getBool_x3f(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__68(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__4; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__33(lean_object*); +static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__5; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__20(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__69___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__8; -static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__35(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__48___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__48___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__3(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__74(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__5(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__42(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__73(lean_object*); lean_object* l_Lean_Meta_ToHide_collect(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__4___rarg(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__5(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__32___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__33(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__13(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__74___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__37(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__5(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveGoal_mvarId_x3f___default; -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__34(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__48___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(lean_object*); lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_mkLeveErrorMessageCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__8(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__39(lean_object*); lean_object* lean_simp_macro_scopes(lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__3; -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__6; -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___closed__1; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__4(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__23(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__12(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__58(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__4___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__20___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__76___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__18(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__54___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__42___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__68___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__38___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__64(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__77(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__73___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__62(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__48___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__79___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__1___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__48(lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__4; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__61___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getGoalPrefix(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__2(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__64___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__20(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__62___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__60___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__37(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__65___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__38(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__2; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_PersistentArray_forIn___at_Lean_Widget_goalToInteractive___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3; -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__38___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___lambda__1(size_t, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__44___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__50___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__36(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__51___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__48(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__62(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__78(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__2; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__49(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__57(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__15(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed__const__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__26(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__7(lean_object*, lean_object*, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__41(lean_object*); +static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__4; +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__6___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__12(lean_object*); lean_object* lean_nat_to_int(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2236____rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__36___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__14(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__4___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__21(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__50(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__28___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__1(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__1(lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__24___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_Format_isNil(lean_object*); -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__35___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__2(lean_object*, lean_object*, size_t); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); uint8_t l_Lean_Expr_isSort(lean_object*); +lean_object* l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_115_(lean_object*); lean_object* l_Lean_LocalContext_sanitizeNames(lean_object*, lean_object*); -static lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__5; -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__45(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__63(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__1(lean_object*, lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Widget_goalToInteractive(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__38(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25(lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__13(lean_object*); +uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__41___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__60(lean_object*); +static lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__1; +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_goalToInteractive___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__46(lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__41___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lean_Widget_InteractiveHypothesisBundle_val_x3f___default() { _start: { @@ -334,2155 +1208,2374 @@ x_1 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__4; return x_1; } } -static lean_object* _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1() { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("[anonymous]", 11); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2() { _start: { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValD(x_2, x_3); -if (lean_obj_tag(x_4) == 0) +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("`", 1); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("expected a `Name`, got '", 24); +return x_1; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("'", 1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) { lean_object* x_5; -lean_dec(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1; +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_3); return x_5; } else { -lean_object* x_6; -x_6 = lean_apply_1(x_1, x_4); -if (lean_obj_tag(x_6) == 0) +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_array_uget(x_3, x_2); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_3, x_2, x_7); +x_9 = l_Lean_Json_getStr_x3f(x_6); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +uint8_t x_10; +lean_dec(x_8); +lean_dec(x_6); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -return x_6; +return x_9; } else { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); -return x_9; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_6); -if (x_10 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_9); +if (x_13 == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_6, 0); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_6, 0, x_12); -return x_6; +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_9, 0); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1; +x_16 = lean_string_dec_eq(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2; +x_18 = lean_string_append(x_17, x_14); +lean_dec(x_14); +x_19 = l_Lean_Syntax_decodeNameLit(x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_dec(x_8); +x_20 = lean_unsigned_to_nat(80u); +x_21 = l_Lean_Json_pretty(x_6, x_20); +x_22 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3; +x_23 = lean_string_append(x_22, x_21); +lean_dec(x_21); +x_24 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_25 = lean_string_append(x_23, x_24); +lean_ctor_set_tag(x_9, 0); +lean_ctor_set(x_9, 0, x_25); +return x_9; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_6, 0); -lean_inc(x_13); +lean_object* x_26; size_t x_27; size_t x_28; lean_object* x_29; +lean_free_object(x_9); lean_dec(x_6); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; -} -} -} +x_26 = lean_ctor_get(x_19, 0); +lean_inc(x_26); +lean_dec(x_19); +x_27 = 1; +x_28 = lean_usize_add(x_2, x_27); +x_29 = lean_array_uset(x_8, x_2, x_26); +x_2 = x_28; +x_3 = x_29; +goto _start; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___boxed), 3, 0); -return x_2; +size_t x_31; size_t x_32; lean_object* x_33; lean_object* x_34; +lean_free_object(x_9); +lean_dec(x_14); +lean_dec(x_6); +x_31 = 1; +x_32 = lean_usize_add(x_2, x_31); +x_33 = lean_box(0); +x_34 = lean_array_uset(x_8, x_2, x_33); +x_2 = x_32; +x_3 = x_34; +goto _start; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("names", 5); -return x_1; -} +lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_36 = lean_ctor_get(x_9, 0); +lean_inc(x_36); +lean_dec(x_9); +x_37 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1; +x_38 = lean_string_dec_eq(x_36, x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2; +x_40 = lean_string_append(x_39, x_36); +lean_dec(x_36); +x_41 = l_Lean_Syntax_decodeNameLit(x_40); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +lean_dec(x_8); +x_42 = lean_unsigned_to_nat(80u); +x_43 = l_Lean_Json_pretty(x_6, x_42); +x_44 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3; +x_45 = lean_string_append(x_44, x_43); +lean_dec(x_43); +x_46 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_47 = lean_string_append(x_45, x_46); +x_48 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_48, 0, x_47); +return x_48; } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__2() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("fvarIds", 7); -return x_1; +lean_object* x_49; size_t x_50; size_t x_51; lean_object* x_52; +lean_dec(x_6); +x_49 = lean_ctor_get(x_41, 0); +lean_inc(x_49); +lean_dec(x_41); +x_50 = 1; +x_51 = lean_usize_add(x_2, x_50); +x_52 = lean_array_uset(x_8, x_2, x_49); +x_2 = x_51; +x_3 = x_52; +goto _start; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("type", 4); -return x_1; +size_t x_54; size_t x_55; lean_object* x_56; lean_object* x_57; +lean_dec(x_36); +lean_dec(x_6); +x_54 = 1; +x_55 = lean_usize_add(x_2, x_54); +x_56 = lean_box(0); +x_57 = lean_array_uset(x_8, x_2, x_56); +x_2 = x_55; +x_3 = x_57; +goto _start; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("val", 3); -return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("isInstance", 10); -return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__6() { +static lean_object* _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("isType", 6); +x_1 = lean_mk_string_from_bytes("expected JSON array, got '", 26); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_6; lean_object* x_7; -x_6 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__1; -x_7 = l_Lean_Json_getObjValAs_x3f(x_5, lean_box(0), x_1, x_6); -if (lean_obj_tag(x_7) == 0) -{ -uint8_t x_8; -lean_dec(x_4); -lean_dec(x_3); +lean_object* x_3; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); lean_dec(x_2); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) +lean_dec(x_1); +if (lean_obj_tag(x_3) == 4) { -return x_7; +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_array_get_size(x_4); +x_6 = lean_usize_of_nat(x_5); +lean_dec(x_5); +x_7 = 0; +x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2(x_6, x_7, x_4); +return x_8; } else { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -lean_dec(x_7); -x_10 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_9 = lean_unsigned_to_nat(80u); +x_10 = l_Lean_Json_pretty(x_3, x_9); +x_11 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; +} } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__4(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_7, 0); -lean_inc(x_11); -lean_dec(x_7); -x_12 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__2; -x_13 = l_Lean_Json_getObjValAs_x3f(x_5, lean_box(0), x_2, x_12); -if (lean_obj_tag(x_13) == 0) +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_array_uget(x_3, x_2); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_3, x_2, x_7); +x_9 = l_Lean_Json_getStr_x3f(x_6); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_14; -lean_dec(x_11); -lean_dec(x_4); -lean_dec(x_3); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +uint8_t x_10; +lean_dec(x_8); +lean_dec(x_6); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -return x_13; +return x_9; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_13, 0); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_16, 0, x_15); -return x_16; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { +uint8_t x_13; +x_13 = !lean_is_exclusive(x_9); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_9, 0); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1; +x_16 = lean_string_dec_eq(x_14, x_15); +if (x_16 == 0) +{ lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_13, 0); -lean_inc(x_17); -lean_dec(x_13); -x_18 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3; -lean_inc(x_3); -x_19 = l_Lean_Json_getObjValAs_x3f(x_5, lean_box(0), x_3, x_18); +x_17 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2; +x_18 = lean_string_append(x_17, x_14); +lean_dec(x_14); +x_19 = l_Lean_Syntax_decodeNameLit(x_18); if (lean_obj_tag(x_19) == 0) { -uint8_t x_20; -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_4); -lean_dec(x_3); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) -{ -return 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_dec(x_8); +x_20 = lean_unsigned_to_nat(80u); +x_21 = l_Lean_Json_pretty(x_6, x_20); +x_22 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3; +x_23 = lean_string_append(x_22, x_21); +lean_dec(x_21); +x_24 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_25 = lean_string_append(x_23, x_24); +lean_ctor_set_tag(x_9, 0); +lean_ctor_set(x_9, 0, x_25); +return x_9; } else { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_19, 0); -lean_inc(x_21); +lean_object* x_26; size_t x_27; size_t x_28; lean_object* x_29; +lean_free_object(x_9); +lean_dec(x_6); +x_26 = lean_ctor_get(x_19, 0); +lean_inc(x_26); lean_dec(x_19); -x_22 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_22, 0, x_21); -return x_22; +x_27 = 1; +x_28 = lean_usize_add(x_2, x_27); +x_29 = lean_array_uset(x_8, x_2, x_26); +x_2 = x_28; +x_3 = x_29; +goto _start; } } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_19, 0); -lean_inc(x_23); -lean_dec(x_19); -x_24 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__4; -x_25 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg(x_3, x_5, x_24); -if (lean_obj_tag(x_25) == 0) +size_t x_31; size_t x_32; lean_object* x_33; lean_object* x_34; +lean_free_object(x_9); +lean_dec(x_14); +lean_dec(x_6); +x_31 = 1; +x_32 = lean_usize_add(x_2, x_31); +x_33 = lean_box(0); +x_34 = lean_array_uset(x_8, x_2, x_33); +x_2 = x_32; +x_3 = x_34; +goto _start; +} +} +else { -uint8_t x_26; -lean_dec(x_23); -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_4); -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) +lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_36 = lean_ctor_get(x_9, 0); +lean_inc(x_36); +lean_dec(x_9); +x_37 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1; +x_38 = lean_string_dec_eq(x_36, x_37); +if (x_38 == 0) { -return x_25; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2; +x_40 = lean_string_append(x_39, x_36); +lean_dec(x_36); +x_41 = l_Lean_Syntax_decodeNameLit(x_40); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +lean_dec(x_8); +x_42 = lean_unsigned_to_nat(80u); +x_43 = l_Lean_Json_pretty(x_6, x_42); +x_44 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3; +x_45 = lean_string_append(x_44, x_43); +lean_dec(x_43); +x_46 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_47 = lean_string_append(x_45, x_46); +x_48 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_48, 0, x_47); +return x_48; } else { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_25, 0); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_28, 0, x_27); -return x_28; +lean_object* x_49; size_t x_50; size_t x_51; lean_object* x_52; +lean_dec(x_6); +x_49 = lean_ctor_get(x_41, 0); +lean_inc(x_49); +lean_dec(x_41); +x_50 = 1; +x_51 = lean_usize_add(x_2, x_50); +x_52 = lean_array_uset(x_8, x_2, x_49); +x_2 = x_51; +x_3 = x_52; +goto _start; } } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_25, 0); -lean_inc(x_29); -lean_dec(x_25); -x_30 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__5; -lean_inc(x_4); -x_31 = l_Lean_Json_getObjValAs_x3f(x_5, lean_box(0), x_4, x_30); -if (lean_obj_tag(x_31) == 0) +size_t x_54; size_t x_55; lean_object* x_56; lean_object* x_57; +lean_dec(x_36); +lean_dec(x_6); +x_54 = 1; +x_55 = lean_usize_add(x_2, x_54); +x_56 = lean_box(0); +x_57 = lean_array_uset(x_8, x_2, x_56); +x_2 = x_55; +x_3 = x_57; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__3(lean_object* x_1, lean_object* x_2) { +_start: { -uint8_t x_32; -lean_dec(x_29); -lean_dec(x_23); -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_4); -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) +lean_object* x_3; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +if (lean_obj_tag(x_3) == 4) { -return x_31; +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_array_get_size(x_4); +x_6 = lean_usize_of_nat(x_5); +lean_dec(x_5); +x_7 = 0; +x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__4(x_6, x_7, x_4); +return x_8; } else { -lean_object* x_33; lean_object* x_34; -x_33 = lean_ctor_get(x_31, 0); -lean_inc(x_33); -lean_dec(x_31); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_9 = lean_unsigned_to_nat(80u); +x_10 = l_Lean_Json_pretty(x_3, x_9); +x_11 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } } -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_31, 0); -lean_inc(x_35); -lean_dec(x_31); -x_36 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__6; -x_37 = l_Lean_Json_getObjValAs_x3f(x_5, lean_box(0), x_4, x_36); -if (lean_obj_tag(x_37) == 0) +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7(size_t x_1, size_t x_2, lean_object* x_3) { +_start: { -uint8_t x_38; -lean_dec(x_35); -lean_dec(x_29); -lean_dec(x_23); -lean_dec(x_17); -lean_dec(x_11); -x_38 = !lean_is_exclusive(x_37); -if (x_38 == 0) +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) { -return x_37; +lean_object* x_5; +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_3); +return x_5; } else { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_37, 0); -lean_inc(x_39); -lean_dec(x_37); -x_40 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_40, 0, x_39); -return x_40; -} -} -else +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_array_uget(x_3, x_2); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_3, x_2, x_7); +x_9 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_6); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_41; -x_41 = !lean_is_exclusive(x_37); -if (x_41 == 0) +uint8_t x_10; +lean_dec(x_8); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_37, 0); -x_43 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_43, 0, x_11); -lean_ctor_set(x_43, 1, x_17); -lean_ctor_set(x_43, 2, x_23); -lean_ctor_set(x_43, 3, x_29); -lean_ctor_set(x_43, 4, x_35); -lean_ctor_set(x_43, 5, x_42); -lean_ctor_set(x_37, 0, x_43); -return x_37; +return x_9; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_37, 0); -lean_inc(x_44); -lean_dec(x_37); -x_45 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_45, 0, x_11); -lean_ctor_set(x_45, 1, x_17); -lean_ctor_set(x_45, 2, x_23); -lean_ctor_set(x_45, 3, x_29); -lean_ctor_set(x_45, 4, x_35); -lean_ctor_set(x_45, 5, x_44); -x_46 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_46, 0, x_45); -return x_46; -} -} -} +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } +else +{ +lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = 1; +x_15 = lean_usize_add(x_2, x_14); +x_16 = lean_array_uset(x_8, x_2, x_13); +x_2 = x_15; +x_3 = x_16; +goto _start; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__1() { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___boxed), 5, 0); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("no inductive constructor matched", 32); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__2() { _start: { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1(lean_object* x_1) { _start: { -lean_object* x_6; -x_6 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); -return x_6; +lean_object* x_2; +x_2 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__2; +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__1() { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___boxed), 5, 4); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_2); -lean_closure_set(x_5, 2, x_3); -lean_closure_set(x_5, 3, x_4); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("tag", 3); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2() { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__1___rarg), 4, 0); -return x_5; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___boxed), 1, 0); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__3() { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; 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; -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_apply_1(x_1, x_6); -x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__1; -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -x_10 = lean_box(0); -x_11 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_11, 0, x_9); -lean_ctor_set(x_11, 1, x_10); -x_12 = lean_ctor_get(x_5, 1); -lean_inc(x_12); -x_13 = lean_apply_1(x_2, x_12); -x_14 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__2; -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_10); -x_17 = lean_ctor_get(x_5, 2); -lean_inc(x_17); -lean_inc(x_3); -x_18 = lean_apply_1(x_3, x_17); -x_19 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3; -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_10); -x_22 = lean_ctor_get(x_5, 3); -lean_inc(x_22); -x_23 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__4; -x_24 = l_Lean_Json_opt___rarg(x_3, x_23, x_22); -x_25 = lean_ctor_get(x_5, 4); -lean_inc(x_25); -lean_inc(x_4); -x_26 = lean_apply_1(x_4, x_25); -x_27 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__5; -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_10); -x_30 = lean_ctor_get(x_5, 5); -lean_inc(x_30); -lean_dec(x_5); -x_31 = lean_apply_1(x_4, x_30); -x_32 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__6; -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_10); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_10); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_29); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_24); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_21); -lean_ctor_set(x_38, 1, x_37); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_16); -lean_ctor_set(x_39, 1, x_38); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_11); -lean_ctor_set(x_40, 1, x_39); -x_41 = l_List_join___rarg(x_40); -x_42 = l_Lean_Json_mkObj(x_41); -return x_42; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("Init.Util", 9); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__4() { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414____rarg), 5, 0); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("getElem!", 8); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__5() { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_414____rarg), 5, 4); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_2); -lean_closure_set(x_5, 2, x_3); -lean_closure_set(x_5, 3, x_4); -return x_5; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("index out of bounds", 19); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6() { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__1___rarg), 4, 0); -return x_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; +x_1 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__3; +x_2 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__4; +x_3 = lean_unsigned_to_nat(69u); +x_4 = lean_unsigned_to_nat(36u); +x_5 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__5; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -if (lean_obj_tag(x_5) == 0) +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__1; +x_5 = lean_unsigned_to_nat(2u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +if (lean_obj_tag(x_6) == 0) { -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); +lean_object* x_8; lean_object* x_9; +x_8 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_9 = l_Except_orElseLazy___rarg(x_6, x_8); return x_9; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 0); lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_13 = l_Except_orElseLazy___rarg(x_11, x_12); +return x_13; } } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; -} -} -} -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__1(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__1___rarg), 5, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_6, 0); +lean_inc(x_14); +lean_dec(x_6); +x_15 = lean_array_get_size(x_14); +x_16 = lean_unsigned_to_nat(0u); +x_17 = lean_nat_dec_lt(x_16, x_15); +if (x_17 == 0) { -if (lean_obj_tag(x_5) == 0) +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6; +x_19 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_18); +x_20 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60_(x_19); +lean_dec(x_19); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_21; +lean_dec(x_15); +lean_dec(x_14); +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +lean_object* x_22; lean_object* x_23; +x_22 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_23 = l_Except_orElseLazy___rarg(x_20, x_22); +return x_23; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_20, 0); +lean_inc(x_24); +lean_dec(x_20); +x_25 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_25, 0, x_24); +x_26 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_27 = l_Except_orElseLazy___rarg(x_25, x_26); +return x_27; } } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; +lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_28 = lean_ctor_get(x_20, 0); +lean_inc(x_28); +lean_dec(x_20); +x_29 = lean_unsigned_to_nat(1u); +x_30 = lean_nat_dec_lt(x_29, x_15); +lean_dec(x_15); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +lean_dec(x_14); +x_31 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_18); +x_32 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_31); +if (lean_obj_tag(x_32) == 0) +{ +uint8_t x_33; +lean_dec(x_28); +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_35 = l_Except_orElseLazy___rarg(x_32, x_34); +return x_35; } +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_32, 0); +lean_inc(x_36); +lean_dec(x_32); +x_37 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_37, 0, x_36); +x_38 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_39 = l_Except_orElseLazy___rarg(x_37, x_38); +return x_39; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__2(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__2___rarg), 5, 0); -return x_2; +uint8_t x_40; +x_40 = !lean_is_exclusive(x_32); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_41 = lean_ctor_get(x_32, 0); +x_42 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_42, 0, x_28); +lean_ctor_set(x_42, 1, x_41); +lean_ctor_set(x_32, 0, x_42); +x_43 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_44 = l_Except_orElseLazy___rarg(x_32, x_43); +return x_44; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_45 = lean_ctor_get(x_32, 0); +lean_inc(x_45); +lean_dec(x_32); +x_46 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_46, 0, x_28); +lean_ctor_set(x_46, 1, x_45); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_49 = l_Except_orElseLazy___rarg(x_47, x_48); +return x_49; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +} +else { -if (lean_obj_tag(x_5) == 0) +lean_object* x_50; lean_object* x_51; +x_50 = lean_array_fget(x_14, x_29); +lean_dec(x_14); +x_51 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_50); +if (lean_obj_tag(x_51) == 0) { -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_52; +lean_dec(x_28); +x_52 = !lean_is_exclusive(x_51); +if (x_52 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +lean_object* x_53; lean_object* x_54; +x_53 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_54 = l_Except_orElseLazy___rarg(x_51, x_53); +return x_54; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_55 = lean_ctor_get(x_51, 0); +lean_inc(x_55); +lean_dec(x_51); +x_56 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_56, 0, x_55); +x_57 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_58 = l_Except_orElseLazy___rarg(x_56, x_57); +return x_58; } } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; +uint8_t x_59; +x_59 = !lean_is_exclusive(x_51); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_60 = lean_ctor_get(x_51, 0); +x_61 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_61, 0, x_28); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_51, 0, x_61); +x_62 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_63 = l_Except_orElseLazy___rarg(x_51, x_62); +return x_63; +} +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_64 = lean_ctor_get(x_51, 0); +lean_inc(x_64); +lean_dec(x_51); +x_65 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_65, 0, x_28); +lean_ctor_set(x_65, 1, x_64); +x_66 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_66, 0, x_65); +x_67 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_68 = l_Except_orElseLazy___rarg(x_66, x_67); +return x_68; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__3(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__3___rarg), 5, 0); -return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -if (lean_obj_tag(x_5) == 0) +lean_object* x_69; lean_object* x_70; +x_69 = lean_array_fget(x_14, x_16); +x_70 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_60_(x_69); +lean_dec(x_69); +if (lean_obj_tag(x_70) == 0) { -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_71; +lean_dec(x_15); +lean_dec(x_14); +x_71 = !lean_is_exclusive(x_70); +if (x_71 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +lean_object* x_72; lean_object* x_73; +x_72 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_73 = l_Except_orElseLazy___rarg(x_70, x_72); +return x_73; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_74 = lean_ctor_get(x_70, 0); +lean_inc(x_74); +lean_dec(x_70); +x_75 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_75, 0, x_74); +x_76 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_77 = l_Except_orElseLazy___rarg(x_75, x_76); +return x_77; } } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; +lean_object* x_78; lean_object* x_79; uint8_t x_80; +x_78 = lean_ctor_get(x_70, 0); +lean_inc(x_78); +lean_dec(x_70); +x_79 = lean_unsigned_to_nat(1u); +x_80 = lean_nat_dec_lt(x_79, x_15); +lean_dec(x_15); +if (x_80 == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; +lean_dec(x_14); +x_81 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6; +x_82 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_81); +x_83 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_82); +if (lean_obj_tag(x_83) == 0) +{ +uint8_t x_84; +lean_dec(x_78); +x_84 = !lean_is_exclusive(x_83); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; +x_85 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_86 = l_Except_orElseLazy___rarg(x_83, x_85); +return x_86; } +else +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_87 = lean_ctor_get(x_83, 0); +lean_inc(x_87); +lean_dec(x_83); +x_88 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_88, 0, x_87); +x_89 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_90 = l_Except_orElseLazy___rarg(x_88, x_89); +return x_90; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__4(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__4___rarg), 5, 0); -return x_2; +uint8_t x_91; +x_91 = !lean_is_exclusive(x_83); +if (x_91 == 0) +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_92 = lean_ctor_get(x_83, 0); +x_93 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_93, 0, x_78); +lean_ctor_set(x_93, 1, x_92); +lean_ctor_set(x_83, 0, x_93); +x_94 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_95 = l_Except_orElseLazy___rarg(x_83, x_94); +return x_95; } +else +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_96 = lean_ctor_get(x_83, 0); +lean_inc(x_96); +lean_dec(x_83); +x_97 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_97, 0, x_78); +lean_ctor_set(x_97, 1, x_96); +x_98 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_98, 0, x_97); +x_99 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_100 = l_Except_orElseLazy___rarg(x_98, x_99); +return x_100; } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +} +} +else { -if (lean_obj_tag(x_5) == 0) +lean_object* x_101; lean_object* x_102; +x_101 = lean_array_fget(x_14, x_79); +lean_dec(x_14); +x_102 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_101); +if (lean_obj_tag(x_102) == 0) { -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_103; +lean_dec(x_78); +x_103 = !lean_is_exclusive(x_102); +if (x_103 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +lean_object* x_104; lean_object* x_105; +x_104 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_105 = l_Except_orElseLazy___rarg(x_102, x_104); +return x_105; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_106 = lean_ctor_get(x_102, 0); +lean_inc(x_106); +lean_dec(x_102); +x_107 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_107, 0, x_106); +x_108 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_109 = l_Except_orElseLazy___rarg(x_107, x_108); +return x_109; } } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; +uint8_t x_110; +x_110 = !lean_is_exclusive(x_102); +if (x_110 == 0) +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_111 = lean_ctor_get(x_102, 0); +x_112 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_112, 0, x_78); +lean_ctor_set(x_112, 1, x_111); +lean_ctor_set(x_102, 0, x_112); +x_113 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_114 = l_Except_orElseLazy___rarg(x_102, x_113); +return x_114; +} +else +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_115 = lean_ctor_get(x_102, 0); +lean_inc(x_115); +lean_dec(x_102); +x_116 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_116, 0, x_78); +lean_ctor_set(x_116, 1, x_115); +x_117 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_117, 0, x_116); +x_118 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2; +x_119 = l_Except_orElseLazy___rarg(x_117, x_118); +return x_119; +} +} } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__5(lean_object* x_1) { +} +} +} +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___closed__1() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__5___rarg), 5, 0); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("text", 4); +return x_1; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -if (lean_obj_tag(x_5) == 0) +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___closed__1; +x_5 = lean_unsigned_to_nat(1u); +x_6 = l_Lean_Json_parseTagged(x_1, x_4, x_5, x_2); +x_7 = lean_alloc_closure((void*)(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___boxed), 3, 2); +lean_closure_set(x_7, 0, x_1); +lean_closure_set(x_7, 1, x_2); +if (lean_obj_tag(x_6) == 0) { -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); +lean_object* x_9; +x_9 = l_Except_orElseLazy___rarg(x_6, x_7); return x_9; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_6, 0); lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_dec(x_6); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Except_orElseLazy___rarg(x_11, x_7); +return x_12; } } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; -} -} -} -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__6(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__6___rarg), 5, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = lean_ctor_get(x_6, 0); +lean_inc(x_13); +lean_dec(x_6); +x_14 = lean_array_get_size(x_13); +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_nat_dec_lt(x_15, x_14); +lean_dec(x_14); +if (x_16 == 0) { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_10, 0, x_2); -lean_ctor_set(x_10, 1, x_3); -lean_ctor_set(x_10, 2, x_4); -lean_ctor_set(x_10, 3, x_5); -lean_ctor_set(x_10, 4, x_6); -lean_ctor_set(x_10, 5, x_7); -x_11 = lean_apply_2(x_9, lean_box(0), x_10); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_dec(x_13); +x_17 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6; +x_18 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_17); +x_19 = l_Lean_Json_getStr_x3f(x_18); +lean_dec(x_18); +if (lean_obj_tag(x_19) == 0) { -uint8_t x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); -x_12 = lean_box(x_11); -lean_inc(x_3); -x_13 = lean_apply_4(x_2, lean_box(0), x_3, x_4, x_12); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__1), 7, 6); -lean_closure_set(x_14, 0, x_3); -lean_closure_set(x_14, 1, x_5); -lean_closure_set(x_14, 2, x_6); -lean_closure_set(x_14, 3, x_7); -lean_closure_set(x_14, 4, x_8); -lean_closure_set(x_14, 5, x_10); -x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_13, x_14); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +uint8_t x_20; +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 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; -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_ctor_get_uint8(x_2, sizeof(void*)*4); -x_12 = lean_box(x_11); -lean_inc(x_10); -lean_inc(x_4); -lean_inc(x_3); -x_13 = lean_apply_4(x_10, lean_box(0), x_3, x_4, x_12); -lean_inc(x_8); -x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__2___boxed), 10, 9); -lean_closure_set(x_14, 0, x_2); -lean_closure_set(x_14, 1, x_10); -lean_closure_set(x_14, 2, x_3); -lean_closure_set(x_14, 3, x_4); -lean_closure_set(x_14, 4, x_5); -lean_closure_set(x_14, 5, x_6); -lean_closure_set(x_14, 6, x_7); -lean_closure_set(x_14, 7, x_9); -lean_closure_set(x_14, 8, x_8); -x_15 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_13, x_14); -return x_15; -} +lean_object* x_21; +x_21 = l_Except_orElseLazy___rarg(x_19, x_7); +return x_21; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__4(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_19, 0); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_23, 0, x_22); +x_24 = l_Except_orElseLazy___rarg(x_23, x_7); +return x_24; } } -static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__4), 1, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +uint8_t x_25; +x_25 = !lean_is_exclusive(x_19); +if (x_25 == 0) { -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_1, 3); -lean_inc(x_10); -lean_inc(x_7); -lean_inc(x_4); -lean_inc(x_3); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__3), 9, 8); -lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, x_1); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_4); -lean_closure_set(x_11, 4, x_5); -lean_closure_set(x_11, 5, x_6); -lean_closure_set(x_11, 6, x_9); -lean_closure_set(x_11, 7, x_7); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_8); -lean_dec(x_4); -x_12 = lean_ctor_get(x_3, 0); -lean_inc(x_12); -lean_dec(x_3); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_2(x_13, lean_box(0), x_14); -x_16 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_15, x_11); -return x_16; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_19, 0); +x_27 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_19, 0, x_27); +x_28 = l_Except_orElseLazy___rarg(x_19, x_7); +return x_28; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_17 = lean_ctor_get(x_10, 0); -lean_inc(x_17); -lean_dec(x_10); -x_18 = lean_ctor_get(x_3, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_ctor_get(x_19, 0); +lean_inc(x_29); lean_dec(x_19); -x_21 = lean_apply_4(x_8, lean_box(0), x_3, x_4, x_17); -x_22 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5___closed__1; -x_23 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_22, x_21); -x_24 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_23, x_11); -return x_24; +x_30 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_30); +x_32 = l_Except_orElseLazy___rarg(x_31, x_7); +return x_32; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -lean_dec(x_1); -x_10 = lean_ctor_get(x_2, 2); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_4); -lean_inc(x_3); -x_11 = lean_apply_4(x_9, lean_box(0), x_3, x_4, x_10); -lean_inc(x_7); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5), 9, 8); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_5); -lean_closure_set(x_12, 2, x_3); -lean_closure_set(x_12, 3, x_4); -lean_closure_set(x_12, 4, x_6); -lean_closure_set(x_12, 5, x_8); -lean_closure_set(x_12, 6, x_7); -lean_closure_set(x_12, 7, x_9); -x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_11, x_12); -return x_13; -} +lean_object* x_33; lean_object* x_34; +x_33 = lean_array_fget(x_13, x_15); +lean_dec(x_13); +x_34 = l_Lean_Json_getStr_x3f(x_33); +lean_dec(x_33); +if (lean_obj_tag(x_34) == 0) +{ +uint8_t x_35; +x_35 = !lean_is_exclusive(x_34); +if (x_35 == 0) +{ +lean_object* x_36; +x_36 = l_Except_orElseLazy___rarg(x_34, x_7); +return x_36; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -lean_dec(x_1); -x_10 = lean_ctor_get(x_2, 1); -lean_inc(x_10); -lean_inc(x_4); -lean_inc(x_3); -x_11 = lean_apply_4(x_9, lean_box(0), x_3, x_4, x_10); -lean_inc(x_7); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__6), 8, 7); -lean_closure_set(x_12, 0, x_5); -lean_closure_set(x_12, 1, x_2); -lean_closure_set(x_12, 2, x_3); -lean_closure_set(x_12, 3, x_4); -lean_closure_set(x_12, 4, x_6); -lean_closure_set(x_12, 5, x_8); -lean_closure_set(x_12, 6, x_7); -x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_11, x_12); -return x_13; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_34, 0); +lean_inc(x_37); +lean_dec(x_34); +x_38 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = l_Except_orElseLazy___rarg(x_38, x_7); +return x_39; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_ctor_get(x_8, 0); -lean_inc(x_11); -lean_inc(x_7); -lean_inc(x_6); -x_12 = lean_apply_4(x_10, lean_box(0), x_6, x_7, x_11); -lean_inc(x_9); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__7), 8, 7); -lean_closure_set(x_13, 0, x_2); -lean_closure_set(x_13, 1, x_8); -lean_closure_set(x_13, 2, x_6); -lean_closure_set(x_13, 3, x_7); -lean_closure_set(x_13, 4, x_3); -lean_closure_set(x_13, 5, x_4); -lean_closure_set(x_13, 6, x_9); -x_14 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_12, x_13); -return x_14; -} +uint8_t x_40; +x_40 = !lean_is_exclusive(x_34); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_34, 0); +x_42 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_34, 0, x_42); +x_43 = l_Except_orElseLazy___rarg(x_34, x_7); +return x_43; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7) { -_start: +else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_alloc_ctor(0, 4, 2); -lean_ctor_set(x_8, 0, x_1); -lean_ctor_set(x_8, 1, x_2); -lean_ctor_set(x_8, 2, x_3); -lean_ctor_set(x_8, 3, x_4); -lean_ctor_set_uint8(x_8, sizeof(void*)*4, x_5); -lean_ctor_set_uint8(x_8, sizeof(void*)*4 + 1, x_7); -x_9 = lean_ctor_get(x_6, 0); -lean_inc(x_9); -lean_dec(x_6); -x_10 = lean_ctor_get(x_9, 1); -lean_inc(x_10); -lean_dec(x_9); -x_11 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_11, 0, x_8); -x_12 = lean_apply_2(x_10, lean_box(0), x_11); -return x_12; +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_34, 0); +lean_inc(x_44); +lean_dec(x_34); +x_45 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = l_Except_orElseLazy___rarg(x_46, x_7); +return x_47; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_10 = lean_ctor_get(x_1, 5); -lean_inc(x_10); -lean_dec(x_1); -lean_inc(x_3); -x_11 = lean_apply_4(x_2, lean_box(0), x_3, x_4, x_10); -x_12 = lean_box(x_9); -lean_inc(x_3); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__9___boxed), 7, 6); -lean_closure_set(x_13, 0, x_5); -lean_closure_set(x_13, 1, x_6); -lean_closure_set(x_13, 2, x_7); -lean_closure_set(x_13, 3, x_8); -lean_closure_set(x_13, 4, x_12); -lean_closure_set(x_13, 5, x_3); -x_14 = lean_ctor_get(x_3, 1); -lean_inc(x_14); -x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_15, 0, x_3); -lean_closure_set(x_15, 1, lean_box(0)); -lean_closure_set(x_15, 2, lean_box(0)); -lean_closure_set(x_15, 3, x_13); -x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_11, x_15); -return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +} +} +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___closed__1() { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); -lean_dec(x_1); -x_10 = lean_ctor_get(x_2, 4); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_4); -lean_inc(x_3); -x_11 = lean_apply_4(x_9, lean_box(0), x_3, x_4, x_10); -lean_inc(x_3); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__10___boxed), 9, 8); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_9); -lean_closure_set(x_12, 2, x_3); -lean_closure_set(x_12, 3, x_4); -lean_closure_set(x_12, 4, x_5); -lean_closure_set(x_12, 5, x_6); -lean_closure_set(x_12, 6, x_7); -lean_closure_set(x_12, 7, x_8); -x_13 = lean_ctor_get(x_3, 1); -lean_inc(x_13); -x_14 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_14, 0, x_3); -lean_closure_set(x_14, 1, lean_box(0)); -lean_closure_set(x_14, 2, lean_box(0)); -lean_closure_set(x_14, 3, x_12); -x_15 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_11, x_14); -return x_15; +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("append", 6); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__12(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(lean_object* x_1) { _start: { -if (lean_obj_tag(x_2) == 0) +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = lean_box(0); +x_3 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___closed__1; +x_4 = lean_unsigned_to_nat(1u); +x_5 = l_Lean_Json_parseTagged(x_1, x_3, x_4, x_2); +x_6 = lean_alloc_closure((void*)(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___boxed), 3, 2); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +if (lean_obj_tag(x_5) == 0) { -uint8_t x_3; -x_3 = !lean_is_exclusive(x_2); -if (x_3 == 0) +uint8_t x_7; +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 1); -lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_apply_2(x_5, lean_box(0), x_2); -return x_6; +lean_object* x_8; +x_8 = l_Except_orElseLazy___rarg(x_5, x_6); +return x_8; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); -lean_dec(x_2); -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_8, 1); +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_5, 0); lean_inc(x_9); -lean_dec(x_8); +lean_dec(x_5); x_10 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_10, 0, x_7); -x_11 = lean_apply_2(x_9, lean_box(0), x_10); +lean_ctor_set(x_10, 0, x_9); +x_11 = l_Except_orElseLazy___rarg(x_10, x_6); return x_11; } } else { uint8_t x_12; -x_12 = !lean_is_exclusive(x_2); +x_12 = !lean_is_exclusive(x_5); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_2, 0); -x_14 = lean_ctor_get(x_1, 0); -lean_inc(x_14); -lean_dec(x_1); -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = lean_ctor_get(x_5, 0); +x_14 = lean_array_get_size(x_13); +x_15 = lean_unsigned_to_nat(0u); +x_16 = lean_nat_dec_lt(x_15, x_14); lean_dec(x_14); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_13); -lean_ctor_set(x_2, 0, x_16); -x_17 = lean_apply_2(x_15, lean_box(0), x_2); -return x_17; -} -else +if (x_16 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_18 = lean_ctor_get(x_2, 0); -lean_inc(x_18); -lean_dec(x_2); -x_19 = lean_ctor_get(x_1, 0); +lean_object* x_17; lean_object* x_18; +lean_dec(x_13); +x_17 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6; +x_18 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_17); +if (lean_obj_tag(x_18) == 4) +{ +lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; +lean_free_object(x_5); +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_1); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_21, 0, x_18); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_21); -x_23 = lean_apply_2(x_20, lean_box(0), x_22); -return x_23; -} +lean_dec(x_18); +x_20 = lean_array_get_size(x_19); +x_21 = lean_usize_of_nat(x_20); +lean_dec(x_20); +x_22 = 0; +x_23 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7(x_21, x_22, x_19); +if (lean_obj_tag(x_23) == 0) +{ +uint8_t x_24; +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; +x_25 = l_Except_orElseLazy___rarg(x_23, x_6); +return x_25; } +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_23, 0); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_27, 0, x_26); +x_28 = l_Except_orElseLazy___rarg(x_27, x_6); +return x_28; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_1, 3); -lean_inc(x_9); -lean_inc(x_4); -lean_inc(x_3); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__11), 8, 7); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_1); -lean_closure_set(x_10, 2, x_3); -lean_closure_set(x_10, 3, x_4); -lean_closure_set(x_10, 4, x_5); -lean_closure_set(x_10, 5, x_6); -lean_closure_set(x_10, 6, x_8); -x_11 = lean_ctor_get(x_3, 1); -lean_inc(x_11); -lean_inc(x_3); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__3___rarg), 5, 4); -lean_closure_set(x_12, 0, x_3); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -if (lean_obj_tag(x_9) == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_23); +if (x_29 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -lean_dec(x_7); -lean_dec(x_4); -x_13 = lean_ctor_get(x_3, 0); -lean_inc(x_13); -lean_dec(x_3); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1; -x_16 = lean_apply_2(x_14, lean_box(0), x_15); -x_17 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_16, x_12); -return x_17; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_23, 0); +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_23, 0, x_31); +x_32 = l_Except_orElseLazy___rarg(x_23, x_6); +return x_32; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_18 = lean_ctor_get(x_9, 0); -lean_inc(x_18); -lean_dec(x_9); -lean_inc(x_3); -x_19 = lean_apply_4(x_7, lean_box(0), x_3, x_4, x_18); -x_20 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__12), 2, 1); -lean_closure_set(x_20, 0, x_3); -lean_inc(x_11); -x_21 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_19, x_20); -x_22 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_21, x_12); -return x_22; +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_33 = lean_ctor_get(x_23, 0); +lean_inc(x_33); +lean_dec(x_23); +x_34 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_34, 0, x_33); +x_35 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_35, 0, x_34); +x_36 = l_Except_orElseLazy___rarg(x_35, x_6); +return x_36; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_2, 2); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_4); -lean_inc(x_3); -x_10 = lean_apply_4(x_8, lean_box(0), x_3, x_4, x_9); -lean_inc(x_3); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__13), 8, 7); -lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, x_5); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_4); -lean_closure_set(x_11, 4, x_6); -lean_closure_set(x_11, 5, x_7); -lean_closure_set(x_11, 6, x_8); -x_12 = lean_ctor_get(x_3, 1); -lean_inc(x_12); -x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__4___rarg), 5, 4); -lean_closure_set(x_13, 0, x_3); -lean_closure_set(x_13, 1, lean_box(0)); -lean_closure_set(x_13, 2, lean_box(0)); -lean_closure_set(x_13, 3, x_11); -x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); -return x_14; +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_37 = lean_unsigned_to_nat(80u); +x_38 = l_Lean_Json_pretty(x_18, x_37); +x_39 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +x_40 = lean_string_append(x_39, x_38); +lean_dec(x_38); +x_41 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_42 = lean_string_append(x_40, x_41); +lean_ctor_set_tag(x_5, 0); +lean_ctor_set(x_5, 0, x_42); +x_43 = l_Except_orElseLazy___rarg(x_5, x_6); +return x_43; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_2, 1); -lean_inc(x_9); -lean_inc(x_4); -lean_inc(x_3); -x_10 = lean_apply_4(x_8, lean_box(0), x_3, x_4, x_9); -lean_inc(x_3); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__14), 7, 6); -lean_closure_set(x_11, 0, x_5); -lean_closure_set(x_11, 1, x_2); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_4); -lean_closure_set(x_11, 4, x_6); -lean_closure_set(x_11, 5, x_7); -x_12 = lean_ctor_get(x_3, 1); -lean_inc(x_12); -x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__5___rarg), 5, 4); -lean_closure_set(x_13, 0, x_3); -lean_closure_set(x_13, 1, lean_box(0)); -lean_closure_set(x_13, 2, lean_box(0)); -lean_closure_set(x_13, 3, x_11); -x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); -return x_14; -} +lean_object* x_44; +x_44 = lean_array_fget(x_13, x_15); +lean_dec(x_13); +if (lean_obj_tag(x_44) == 4) +{ +lean_object* x_45; lean_object* x_46; size_t x_47; size_t x_48; lean_object* x_49; +lean_free_object(x_5); +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +lean_dec(x_44); +x_46 = lean_array_get_size(x_45); +x_47 = lean_usize_of_nat(x_46); +lean_dec(x_46); +x_48 = 0; +x_49 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7(x_47, x_48, x_45); +if (lean_obj_tag(x_49) == 0) +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_49); +if (x_50 == 0) +{ +lean_object* x_51; +x_51 = l_Except_orElseLazy___rarg(x_49, x_6); +return x_51; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); -lean_dec(x_1); -x_10 = lean_ctor_get(x_8, 0); -lean_inc(x_10); -lean_inc(x_7); -lean_inc(x_6); -x_11 = lean_apply_4(x_9, lean_box(0), x_6, x_7, x_10); -lean_inc(x_6); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__15), 7, 6); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_8); -lean_closure_set(x_12, 2, x_6); -lean_closure_set(x_12, 3, x_7); -lean_closure_set(x_12, 4, x_3); -lean_closure_set(x_12, 5, x_4); -x_13 = lean_ctor_get(x_6, 1); -lean_inc(x_13); -x_14 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___spec__6___rarg), 5, 4); -lean_closure_set(x_14, 0, x_6); -lean_closure_set(x_14, 1, lean_box(0)); -lean_closure_set(x_14, 2, lean_box(0)); -lean_closure_set(x_14, 3, x_12); -x_15 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_11, x_14); -return x_15; +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_49, 0); +lean_inc(x_52); +lean_dec(x_49); +x_53 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_53, 0, x_52); +x_54 = l_Except_orElseLazy___rarg(x_53, x_6); +return x_54; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; -lean_inc(x_7); -lean_inc(x_5); -lean_inc(x_3); -lean_inc(x_1); -x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__8), 8, 4); -lean_closure_set(x_8, 0, x_1); -lean_closure_set(x_8, 1, x_3); -lean_closure_set(x_8, 2, x_5); -lean_closure_set(x_8, 3, x_7); -x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__16), 8, 4); -lean_closure_set(x_9, 0, x_1); -lean_closure_set(x_9, 1, x_3); -lean_closure_set(x_9, 2, x_5); -lean_closure_set(x_9, 3, x_7); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -return x_10; -} +uint8_t x_55; +x_55 = !lean_is_exclusive(x_49); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_49, 0); +x_57 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_49, 0, x_57); +x_58 = l_Except_orElseLazy___rarg(x_49, x_6); +return x_58; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg), 7, 0); -return x_2; +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_59 = lean_ctor_get(x_49, 0); +lean_inc(x_59); +lean_dec(x_49); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_59); +x_61 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_61, 0, x_60); +x_62 = l_Except_orElseLazy___rarg(x_61, x_6); +return x_62; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +} +else { -lean_object* x_11; -x_11 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); -return x_11; +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_63 = lean_unsigned_to_nat(80u); +x_64 = l_Lean_Json_pretty(x_44, x_63); +x_65 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +x_66 = lean_string_append(x_65, x_64); +lean_dec(x_64); +x_67 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_68 = lean_string_append(x_66, x_67); +lean_ctor_set_tag(x_5, 0); +lean_ctor_set(x_5, 0, x_68); +x_69 = l_Except_orElseLazy___rarg(x_5, x_6); +return x_69; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: +} +else { -uint8_t x_8; uint8_t x_9; lean_object* x_10; -x_8 = lean_unbox(x_5); +lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; +x_70 = lean_ctor_get(x_5, 0); +lean_inc(x_70); lean_dec(x_5); -x_9 = lean_unbox(x_7); -lean_dec(x_7); -x_10 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__9(x_1, x_2, x_3, x_4, x_8, x_6, x_9); -return x_10; -} +x_71 = lean_array_get_size(x_70); +x_72 = lean_unsigned_to_nat(0u); +x_73 = lean_nat_dec_lt(x_72, x_71); +lean_dec(x_71); +if (x_73 == 0) +{ +lean_object* x_74; lean_object* x_75; +lean_dec(x_70); +x_74 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6; +x_75 = l_panic___at_Lean_Json_setObjVal_x21___spec__1(x_74); +if (lean_obj_tag(x_75) == 4) +{ +lean_object* x_76; lean_object* x_77; size_t x_78; size_t x_79; lean_object* x_80; +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +lean_dec(x_75); +x_77 = lean_array_get_size(x_76); +x_78 = lean_usize_of_nat(x_77); +lean_dec(x_77); +x_79 = 0; +x_80 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7(x_78, x_79, x_76); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + x_82 = x_80; +} else { + lean_dec_ref(x_80); + x_82 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -uint8_t x_10; lean_object* x_11; -x_10 = lean_unbox(x_9); -lean_dec(x_9); -x_11 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_10); -return x_11; +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(0, 1, 0); +} else { + x_83 = x_82; } +lean_ctor_set(x_83, 0, x_81); +x_84 = l_Except_orElseLazy___rarg(x_83, x_6); +return x_84; } -static lean_object* _init_l_Lean_Widget_InteractiveGoal_mvarId_x3f___default() { -_start: +else { -lean_object* x_1; -x_1 = lean_box(0); -return x_1; +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_85 = lean_ctor_get(x_80, 0); +lean_inc(x_85); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + x_86 = x_80; +} else { + lean_dec_ref(x_80); + x_86 = lean_box(0); } +x_87 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_87, 0, x_85); +if (lean_is_scalar(x_86)) { + x_88 = lean_alloc_ctor(1, 1, 0); +} else { + x_88 = x_86; } -static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveGoal___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = lean_box(0); -x_2 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__1; -x_3 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__3; -x_4 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; -x_5 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_5, 0, x_2); -lean_ctor_set(x_5, 1, x_3); -lean_ctor_set(x_5, 2, x_1); -lean_ctor_set(x_5, 3, x_4); -lean_ctor_set(x_5, 4, x_1); -return x_5; +lean_ctor_set(x_88, 0, x_87); +x_89 = l_Except_orElseLazy___rarg(x_88, x_6); +return x_89; } } -static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveGoal() { -_start: +else { -lean_object* x_1; -x_1 = l_Lean_Widget_instInhabitedInteractiveGoal___closed__1; -return x_1; -} +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_90 = lean_unsigned_to_nat(80u); +x_91 = l_Lean_Json_pretty(x_75, x_90); +x_92 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +x_93 = lean_string_append(x_92, x_91); +lean_dec(x_91); +x_94 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_95 = lean_string_append(x_93, x_94); +x_96 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_96, 0, x_95); +x_97 = l_Except_orElseLazy___rarg(x_96, x_6); +return x_97; } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Json_getObjValD(x_2, x_3); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; -lean_dec(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1; -return x_5; } else { -lean_object* x_6; -x_6 = lean_apply_1(x_1, x_4); -if (lean_obj_tag(x_6) == 0) +lean_object* x_98; +x_98 = lean_array_fget(x_70, x_72); +lean_dec(x_70); +if (lean_obj_tag(x_98) == 4) { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +lean_object* x_99; lean_object* x_100; size_t x_101; size_t x_102; lean_object* x_103; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_array_get_size(x_99); +x_101 = lean_usize_of_nat(x_100); +lean_dec(x_100); +x_102 = 0; +x_103 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7(x_101, x_102, x_99); +if (lean_obj_tag(x_103) == 0) { -return x_6; +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_104 = lean_ctor_get(x_103, 0); +lean_inc(x_104); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + x_105 = x_103; +} else { + lean_dec_ref(x_103); + x_105 = lean_box(0); } -else -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); -return x_9; +if (lean_is_scalar(x_105)) { + x_106 = lean_alloc_ctor(0, 1, 0); +} else { + x_106 = x_105; } +lean_ctor_set(x_106, 0, x_104); +x_107 = l_Except_orElseLazy___rarg(x_106, x_6); +return x_107; } else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_6); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_6, 0); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_6, 0, x_12); -return x_6; +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_108 = lean_ctor_get(x_103, 0); +lean_inc(x_108); +if (lean_is_exclusive(x_103)) { + lean_ctor_release(x_103, 0); + x_109 = x_103; +} else { + lean_dec_ref(x_103); + x_109 = lean_box(0); +} +x_110 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_110, 0, x_108); +if (lean_is_scalar(x_109)) { + x_111 = lean_alloc_ctor(1, 1, 0); +} else { + x_111 = x_109; +} +lean_ctor_set(x_111, 0, x_110); +x_112 = l_Except_orElseLazy___rarg(x_111, x_6); +return x_112; +} } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_6, 0); -lean_inc(x_13); -lean_dec(x_6); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_113 = lean_unsigned_to_nat(80u); +x_114 = l_Lean_Json_pretty(x_98, x_113); +x_115 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +x_116 = lean_string_append(x_115, x_114); +lean_dec(x_114); +x_117 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_118 = lean_string_append(x_116, x_117); +x_119 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_119, 0, x_118); +x_120 = l_Except_orElseLazy___rarg(x_119, x_6); +return x_120; +} } } } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__5(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1___rarg___boxed), 3, 0); -return x_2; +lean_object* x_3; lean_object* x_4; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +lean_dec(x_1); +x_4 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +static lean_object* _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1() { _start: { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValD(x_2, x_3); -if (lean_obj_tag(x_4) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_5; -lean_dec(x_1); -x_5 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1; -return x_5; +lean_object* x_3; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; +x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +return x_4; } else { -lean_object* x_6; -x_6 = lean_apply_1(x_1, x_4); -if (lean_obj_tag(x_6) == 0) +lean_object* x_5; +x_5 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6(x_3); +if (lean_obj_tag(x_5) == 0) { -uint8_t x_7; -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +uint8_t x_6; +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -return x_6; +return x_5; } else { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); -lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); -return x_9; +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +return x_8; } } else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_6); -if (x_10 == 0) +uint8_t x_9; +x_9 = !lean_is_exclusive(x_5); +if (x_9 == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_6, 0); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_6, 0, x_12); -return x_6; +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_5, 0); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_5, 0, x_11); +return x_5; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_6, 0); -lean_inc(x_13); -lean_dec(x_6); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_5, 0); +lean_inc(x_12); +lean_dec(x_5); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); x_14 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_14, 0, x_13); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +return x_14; } } } } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__9(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2___rarg___boxed), 3, 0); -return x_2; +lean_object* x_3; lean_object* x_4; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +x_4 = l_Lean_Json_getBool_x3f(x_3); +lean_dec(x_3); +return x_4; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1() { +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("hyps", 4); +x_1 = lean_mk_string_from_bytes("names", 5); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__2() { +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("userName", 8); +x_1 = lean_mk_string_from_bytes("fvarIds", 7); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__3() { +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("goalPrefix", 10); +x_1 = lean_mk_string_from_bytes("type", 4); return x_1; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__4() { +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_from_bytes("mvarId", 6); +x_1 = lean_mk_string_from_bytes("val", 3); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__5() { _start: { -lean_object* x_6; lean_object* x_7; -x_6 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1; -x_7 = l_Lean_Json_getObjValAs_x3f(x_5, lean_box(0), x_1, x_6); -if (lean_obj_tag(x_7) == 0) +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("isInstance", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__6() { +_start: { -uint8_t x_8; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_8 = !lean_is_exclusive(x_7); -if (x_8 == 0) +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("isType", 6); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136_(lean_object* x_1) { +_start: { -return x_7; +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__1; +lean_inc(x_1); +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +lean_dec(x_1); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +return x_3; } else { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -lean_dec(x_7); -x_10 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_7, 0); -lean_inc(x_11); -lean_dec(x_7); -x_12 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3; -x_13 = l_Lean_Json_getObjValAs_x3f(x_5, lean_box(0), x_2, x_12); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -lean_dec(x_11); -lean_dec(x_4); +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); lean_dec(x_3); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__2; +lean_inc(x_1); +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__3(x_1, x_8); +if (lean_obj_tag(x_9) == 0) { -return x_13; +uint8_t x_10; +lean_dec(x_7); +lean_dec(x_1); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_13, 0); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_16, 0, x_15); -return x_16; +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_13, 0); -lean_inc(x_17); -lean_dec(x_13); -x_18 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__2; -lean_inc(x_3); -x_19 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1___rarg(x_3, x_5, x_18); -if (lean_obj_tag(x_19) == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3; +lean_inc(x_1); +x_15 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__5(x_1, x_14); +if (lean_obj_tag(x_15) == 0) { -uint8_t x_20; -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_4); -lean_dec(x_3); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +uint8_t x_16; +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_1); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) { -return x_19; +return x_15; } else { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_19, 0); -lean_inc(x_21); -lean_dec(x_19); -x_22 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_22, 0, x_21); -return x_22; +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; } } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_19, 0); -lean_inc(x_23); -lean_dec(x_19); -x_24 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__3; -x_25 = l_Lean_Json_getObjValAs_x3f(x_5, lean_box(0), x_3, x_24); -if (lean_obj_tag(x_25) == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_15, 0); +lean_inc(x_19); +lean_dec(x_15); +x_20 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__4; +x_21 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8(x_1, x_20); +if (lean_obj_tag(x_21) == 0) { -uint8_t x_26; -lean_dec(x_23); -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_4); -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) +uint8_t x_22; +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) { -return x_25; +return x_21; } else { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_25, 0); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_28, 0, x_27); -return x_28; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_24, 0, x_23); +return x_24; } } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_25, 0); -lean_inc(x_29); -lean_dec(x_25); -x_30 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__4; -x_31 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2___rarg(x_4, x_5, x_30); -if (lean_obj_tag(x_31) == 0) +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__5; +x_27 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__9(x_1, x_26); +if (lean_obj_tag(x_27) == 0) { -uint8_t x_32; -lean_dec(x_29); -lean_dec(x_23); -lean_dec(x_17); -lean_dec(x_11); -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) +uint8_t x_28; +lean_dec(x_25); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_1); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) { -return x_31; +return x_27; } else { -lean_object* x_33; lean_object* x_34; -x_33 = lean_ctor_get(x_31, 0); -lean_inc(x_33); -lean_dec(x_31); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_27, 0); +lean_inc(x_29); +lean_dec(x_27); +x_30 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_30, 0, x_29); +return x_30; } } else { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_31); -if (x_35 == 0) +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_27, 0); +lean_inc(x_31); +lean_dec(x_27); +x_32 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__6; +x_33 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__9(x_1, x_32); +lean_dec(x_1); +if (lean_obj_tag(x_33) == 0) +{ +uint8_t x_34; +lean_dec(x_31); +lean_dec(x_25); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_7); +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_31, 0); -x_37 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_37, 0, x_11); -lean_ctor_set(x_37, 1, x_17); -lean_ctor_set(x_37, 2, x_23); -lean_ctor_set(x_37, 3, x_29); -lean_ctor_set(x_37, 4, x_36); -lean_ctor_set(x_31, 0, x_37); -return x_31; +return x_33; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_31, 0); -lean_inc(x_38); -lean_dec(x_31); -x_39 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_39, 0, x_11); -lean_ctor_set(x_39, 1, x_17); -lean_ctor_set(x_39, 2, x_23); -lean_ctor_set(x_39, 3, x_29); -lean_ctor_set(x_39, 4, x_38); -x_40 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_40, 0, x_39); -return x_40; -} +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_33, 0); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_36, 0, x_35); +return x_36; } } +else +{ +uint8_t x_37; +x_37 = !lean_is_exclusive(x_33); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; uint8_t x_40; uint8_t x_41; +x_38 = lean_ctor_get(x_33, 0); +x_39 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_39, 0, x_7); +lean_ctor_set(x_39, 1, x_13); +lean_ctor_set(x_39, 2, x_19); +lean_ctor_set(x_39, 3, x_25); +x_40 = lean_unbox(x_31); +lean_dec(x_31); +lean_ctor_set_uint8(x_39, sizeof(void*)*4, x_40); +x_41 = lean_unbox(x_38); +lean_dec(x_38); +lean_ctor_set_uint8(x_39, sizeof(void*)*4 + 1, x_41); +lean_ctor_set(x_33, 0, x_39); +return x_33; } +else +{ +lean_object* x_42; lean_object* x_43; uint8_t x_44; uint8_t x_45; lean_object* x_46; +x_42 = lean_ctor_get(x_33, 0); +lean_inc(x_42); +lean_dec(x_33); +x_43 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_43, 0, x_7); +lean_ctor_set(x_43, 1, x_13); +lean_ctor_set(x_43, 2, x_19); +lean_ctor_set(x_43, 3, x_25); +x_44 = lean_unbox(x_31); +lean_dec(x_31); +lean_ctor_set_uint8(x_43, sizeof(void*)*4, x_44); +x_45 = lean_unbox(x_42); +lean_dec(x_42); +lean_ctor_set_uint8(x_43, sizeof(void*)*4 + 1, x_45); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_43); +return x_46; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___boxed), 5, 0); -return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__1___rarg(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; -x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____spec__2___rarg(x_1, x_2, x_3); -lean_dec(x_3); +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -return x_4; +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2(x_4, x_5, x_3); +return x_6; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_6; -x_6 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__4(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___boxed), 5, 4); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_2); -lean_closure_set(x_5, 2, x_3); -lean_closure_set(x_5, 3, x_4); -return x_5; +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__7(x_4, x_5, x_3); +return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___boxed(lean_object* x_1) { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__2___rarg), 4, 0); -return x_5; +lean_object* x_2; +x_2 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1(x_1); +lean_dec(x_1); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_apply_1(x_1, x_6); -x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1; -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -x_10 = lean_box(0); -x_11 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_11, 0, x_9); -lean_ctor_set(x_11, 1, x_10); -x_12 = lean_ctor_get(x_5, 1); -lean_inc(x_12); -x_13 = lean_apply_1(x_2, x_12); -x_14 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3; -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_10); -x_17 = lean_ctor_get(x_5, 2); -lean_inc(x_17); -x_18 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__2; -lean_inc(x_3); -x_19 = l_Lean_Json_opt___rarg(x_3, x_18, x_17); -x_20 = lean_ctor_get(x_5, 3); -lean_inc(x_20); -x_21 = lean_apply_1(x_3, x_20); -x_22 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__3; -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_10); -x_25 = lean_ctor_get(x_5, 4); -lean_inc(x_25); -lean_dec(x_5); -x_26 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__4; -x_27 = l_Lean_Json_opt___rarg(x_4, x_26, x_25); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_10); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_24); -lean_ctor_set(x_29, 1, x_28); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_19); -lean_ctor_set(x_30, 1, x_29); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_16); -lean_ctor_set(x_31, 1, x_30); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_11); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_List_join___rarg(x_32); -x_34 = l_Lean_Json_mkObj(x_33); -return x_34; +lean_object* x_4; +x_4 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237_(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237____rarg), 5, 0); -return x_5; +lean_object* x_4; +x_4 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__5___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1237____rarg), 5, 4); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_2); -lean_closure_set(x_5, 2, x_3); -lean_closure_set(x_5, 3, x_4); -return x_5; +lean_object* x_3; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__5(x_1, x_2); +lean_dec(x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__2___rarg), 4, 0); -return x_5; +lean_object* x_3; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__9___boxed(lean_object* x_1, lean_object* x_2) { _start: { -if (lean_obj_tag(x_5) == 0) -{ -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); +lean_object* x_3; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__9(x_1, x_2); +lean_dec(x_2); lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +return x_3; } -else +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__1___closed__1() { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136_), 1, 0); +return x_1; } } -else +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__1() { +_start: { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; -} +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket__1___closed__1; +return x_1; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__1(size_t x_1, size_t x_2, lean_object* x_3) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__1___rarg), 5, 0); -return x_2; +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = 1; +x_9 = l_Lean_Name_toString(x_5, x_8); +x_10 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_2, x_11); +x_13 = lean_array_uset(x_7, x_2, x_10); +x_2 = x_12; +x_3 = x_13; +goto _start; +} } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__2(size_t x_1, size_t x_2, lean_object* x_3) { _start: { -if (lean_obj_tag(x_5) == 0) -{ -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +return x_3; } else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = 1; +x_9 = l_Lean_Name_toString(x_5, x_8); +x_10 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = 1; +x_12 = lean_usize_add(x_2, x_11); +x_13 = lean_array_uset(x_7, x_2, x_10); +x_2 = x_12; +x_3 = x_13; +goto _start; +} +} } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__4(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; } else { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__2(lean_object* x_1) { +static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3___closed__1() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__2___rarg), 5, 0); +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(2u); +x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(lean_object* x_1) { _start: { -if (lean_obj_tag(x_5) == 0) -{ -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +switch (lean_obj_tag(x_1)) { +case 0: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); +x_3 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___closed__1; +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_box(0); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_6); +x_8 = l_Lean_Json_mkObj(x_7); +return x_8; +} +case 1: +{ +lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_9 = lean_ctor_get(x_1, 0); +lean_inc(x_9); +lean_dec(x_1); +x_10 = lean_array_get_size(x_9); +x_11 = lean_usize_of_nat(x_10); +lean_dec(x_10); +x_12 = 0; +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__4(x_11, x_12, x_9); +x_14 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___closed__1; +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean_Json_mkObj(x_18); +return x_19; +} +default: +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_dec(x_1); +x_22 = l___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveCode___hyg_115_(x_20); +x_23 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_21); +x_24 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3___closed__1; +x_25 = lean_array_push(x_24, x_22); +x_26 = lean_array_push(x_25, x_23); +x_27 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_27, 0, x_26); +x_28 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__1; +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +x_30 = lean_box(0); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_Json_mkObj(x_31); +return x_32; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__5(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +lean_dec(x_1); +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_4 = lean_ctor_get(x_2, 0); +lean_inc(x_4); +lean_dec(x_2); +x_5 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_4); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_1); +lean_ctor_set(x_6, 1, x_5); +x_7 = lean_box(0); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_6); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = lean_array_get_size(x_2); +x_4 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_5 = 0; +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__1(x_4, x_5, x_2); +x_7 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_7, 0, x_6); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__1; +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +x_13 = lean_array_get_size(x_12); +x_14 = lean_usize_of_nat(x_13); +lean_dec(x_13); +x_15 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__2(x_14, x_5, x_12); +x_16 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_16, 0, x_15); +x_17 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__2; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_10); +x_20 = lean_ctor_get(x_1, 2); +lean_inc(x_20); +x_21 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_20); +x_22 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_10); +x_25 = lean_ctor_get(x_1, 3); +lean_inc(x_25); +x_26 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__4; +x_27 = l_Lean_Json_opt___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__5(x_26, x_25); +x_28 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_29 = lean_alloc_ctor(1, 0, 1); +lean_ctor_set_uint8(x_29, 0, x_28); +x_30 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__5; +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_29); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_10); +x_33 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +lean_dec(x_1); +x_34 = lean_alloc_ctor(1, 0, 1); +lean_ctor_set_uint8(x_34, 0, x_33); +x_35 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__6; +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_34); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_10); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_10); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_32); +lean_ctor_set(x_39, 1, x_38); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_27); +lean_ctor_set(x_40, 1, x_39); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_24); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_19); +lean_ctor_set(x_42, 1, x_41); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_11); +lean_ctor_set(x_43, 1, x_42); +x_44 = l_List_join___rarg(x_43); +x_45 = l_Lean_Json_mkObj(x_44); +return x_45; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__1(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__2(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__4(x_4, x_5, x_3); +return x_6; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket__1___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); x_9 = lean_apply_2(x_8, lean_box(0), x_5); @@ -2518,15 +3611,87 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__3(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__2___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__2___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__3___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___boxed), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -2576,15 +3741,87 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__4___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__4___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___boxed), 4, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -2634,808 +3871,11712 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__5(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__5(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__5___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__5___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___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_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; x_7 = lean_ctor_get(x_1, 0); lean_inc(x_7); lean_dec(x_1); x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); -x_9 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_9, 0, x_2); -lean_ctor_set(x_9, 1, x_3); -lean_ctor_set(x_9, 2, x_4); -lean_ctor_set(x_9, 3, x_5); -lean_ctor_set(x_9, 4, x_6); -x_10 = lean_apply_2(x_8, lean_box(0), x_9); -return x_10; -} +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_1, 4); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); lean_inc(x_10); -lean_dec(x_1); -lean_inc(x_2); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__1), 6, 5); -lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, x_3); -lean_closure_set(x_11, 2, x_4); -lean_closure_set(x_11, 3, x_5); -lean_closure_set(x_11, 4, x_9); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -lean_dec(x_8); -lean_dec(x_7); -x_12 = lean_ctor_get(x_2, 0); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); -lean_dec(x_2); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_2(x_13, lean_box(0), x_14); -x_16 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_15, x_11); -return x_16; +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_17 = lean_ctor_get(x_10, 0); -lean_inc(x_17); -lean_dec(x_10); -x_18 = lean_ctor_get(x_2, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -lean_dec(x_19); -x_21 = lean_ctor_get(x_7, 0); -lean_inc(x_21); -lean_dec(x_7); -x_22 = lean_apply_4(x_21, lean_box(0), x_2, x_8, x_17); -x_23 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5___closed__1; -x_24 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_23, x_22); -x_25 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_24, x_11); -return x_25; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__6(lean_object* x_1) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_ctor_get(x_2, 3); -lean_inc(x_11); -lean_inc(x_4); -lean_inc(x_3); -x_12 = lean_apply_4(x_10, lean_box(0), x_3, x_4, x_11); -lean_inc(x_7); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__2), 9, 8); -lean_closure_set(x_13, 0, x_2); -lean_closure_set(x_13, 1, x_3); -lean_closure_set(x_13, 2, x_5); -lean_closure_set(x_13, 3, x_6); -lean_closure_set(x_13, 4, x_9); -lean_closure_set(x_13, 5, x_7); -lean_closure_set(x_13, 6, x_8); -lean_closure_set(x_13, 7, x_4); -x_14 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_13); -return x_14; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__6___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_1, 2); -lean_inc(x_9); -lean_inc(x_6); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__3), 9, 8); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_1); -lean_closure_set(x_10, 2, x_3); -lean_closure_set(x_10, 3, x_4); -lean_closure_set(x_10, 4, x_5); -lean_closure_set(x_10, 5, x_8); -lean_closure_set(x_10, 6, x_6); -lean_closure_set(x_10, 7, x_7); -if (lean_obj_tag(x_9) == 0) +if (lean_obj_tag(x_5) == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +uint8_t x_6; lean_dec(x_4); -lean_dec(x_2); -x_11 = lean_ctor_get(x_3, 0); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); -lean_dec(x_3); +lean_dec(x_1); x_12 = lean_ctor_get(x_11, 1); lean_inc(x_12); lean_dec(x_11); -x_13 = lean_box(0); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); x_14 = lean_apply_2(x_12, lean_box(0), x_13); -x_15 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_14, x_10); -return x_15; +return x_14; +} } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_16 = lean_ctor_get(x_9, 0); -lean_inc(x_16); -lean_dec(x_9); -x_17 = lean_ctor_get(x_3, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -lean_dec(x_17); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -lean_dec(x_18); -x_20 = lean_ctor_get(x_2, 0); -lean_inc(x_20); -lean_dec(x_2); -x_21 = lean_apply_4(x_20, lean_box(0), x_3, x_4, x_16); -x_22 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5___closed__1; -x_23 = lean_apply_4(x_19, lean_box(0), lean_box(0), x_22, x_21); -x_24 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_23, x_10); -return x_24; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__9(lean_object* x_1) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -lean_dec(x_1); -x_10 = lean_ctor_get(x_2, 1); -lean_inc(x_10); -lean_inc(x_4); -lean_inc(x_3); -x_11 = lean_apply_4(x_9, lean_box(0), x_3, x_4, x_10); -lean_inc(x_6); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__4), 8, 7); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_5); -lean_closure_set(x_12, 2, x_3); -lean_closure_set(x_12, 3, x_4); -lean_closure_set(x_12, 4, x_8); -lean_closure_set(x_12, 5, x_6); -lean_closure_set(x_12, 6, x_7); -x_13 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_11, x_12); -return x_13; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__9___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = lean_ctor_get(x_8, 0); -lean_inc(x_11); -lean_inc(x_7); -lean_inc(x_6); -x_12 = lean_apply_4(x_10, lean_box(0), x_6, x_7, x_11); -lean_inc(x_9); -x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__5), 8, 7); -lean_closure_set(x_13, 0, x_2); -lean_closure_set(x_13, 1, x_8); -lean_closure_set(x_13, 2, x_6); -lean_closure_set(x_13, 3, x_7); -lean_closure_set(x_13, 4, x_3); -lean_closure_set(x_13, 5, x_9); -lean_closure_set(x_13, 6, x_4); -x_14 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_12, x_13); -return x_14; +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_7, 0, x_1); -lean_ctor_set(x_7, 1, x_2); -lean_ctor_set(x_7, 2, x_3); -lean_ctor_set(x_7, 3, x_4); -lean_ctor_set(x_7, 4, x_6); -x_8 = lean_ctor_get(x_5, 0); -lean_inc(x_8); -lean_dec(x_5); -x_9 = lean_ctor_get(x_8, 1); -lean_inc(x_9); -lean_dec(x_8); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_7); -x_11 = lean_apply_2(x_9, lean_box(0), x_10); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_1, 4); -lean_inc(x_9); +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -lean_inc(x_5); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__7), 6, 5); -lean_closure_set(x_10, 0, x_2); -lean_closure_set(x_10, 1, x_3); -lean_closure_set(x_10, 2, x_4); -lean_closure_set(x_10, 3, x_8); -lean_closure_set(x_10, 4, x_5); -x_11 = lean_ctor_get(x_5, 1); -lean_inc(x_11); -lean_inc(x_5); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_12, 0, x_5); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); lean_dec(x_7); -lean_dec(x_6); -x_13 = lean_ctor_get(x_5, 0); -lean_inc(x_13); -lean_dec(x_5); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1; -x_16 = lean_apply_2(x_14, lean_box(0), x_15); -x_17 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_16, x_12); -return x_17; +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_18 = lean_ctor_get(x_9, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); lean_inc(x_18); -lean_dec(x_9); -x_19 = lean_ctor_get(x_6, 1); -lean_inc(x_19); -lean_dec(x_6); -lean_inc(x_5); -x_20 = lean_apply_4(x_19, lean_box(0), x_5, x_7, x_18); -x_21 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__12), 2, 1); -lean_closure_set(x_21, 0, x_5); -lean_inc(x_11); -x_22 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_20, x_21); -x_23 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_22, x_12); -return x_23; +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__9___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; } } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8(lean_object* x_1) { _start: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); -lean_dec(x_1); -x_10 = lean_ctor_get(x_2, 3); -lean_inc(x_10); -lean_inc(x_4); -lean_inc(x_3); -x_11 = lean_apply_4(x_9, lean_box(0), x_3, x_4, x_10); -lean_inc(x_3); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__8), 8, 7); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_5); -lean_closure_set(x_12, 2, x_6); -lean_closure_set(x_12, 3, x_8); -lean_closure_set(x_12, 4, x_3); -lean_closure_set(x_12, 5, x_7); -lean_closure_set(x_12, 6, x_4); -x_13 = lean_ctor_get(x_3, 1); -lean_inc(x_13); -x_14 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_14, 0, x_3); -lean_closure_set(x_14, 1, lean_box(0)); -lean_closure_set(x_14, 2, lean_box(0)); -lean_closure_set(x_14, 3, x_12); -x_15 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_11, x_14); -return x_15; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___boxed), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_8 = lean_ctor_get(x_1, 2); -lean_inc(x_8); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__9), 8, 7); -lean_closure_set(x_9, 0, x_2); -lean_closure_set(x_9, 1, x_1); -lean_closure_set(x_9, 2, x_3); -lean_closure_set(x_9, 3, x_4); -lean_closure_set(x_9, 4, x_5); -lean_closure_set(x_9, 5, x_7); -lean_closure_set(x_9, 6, x_6); -x_10 = lean_ctor_get(x_3, 1); -lean_inc(x_10); -lean_inc(x_3); -x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__3___rarg), 5, 4); -lean_closure_set(x_11, 0, x_3); -lean_closure_set(x_11, 1, lean_box(0)); -lean_closure_set(x_11, 2, lean_box(0)); -lean_closure_set(x_11, 3, x_9); -if (lean_obj_tag(x_8) == 0) +if (lean_obj_tag(x_5) == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +uint8_t x_6; lean_dec(x_4); -lean_dec(x_2); -x_12 = lean_ctor_get(x_3, 0); -lean_inc(x_12); -lean_dec(x_3); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1; -x_15 = lean_apply_2(x_13, lean_box(0), x_14); -x_16 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_15, x_11); -return x_16; +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_8, 0); -lean_inc(x_17); -lean_dec(x_8); -x_18 = lean_ctor_get(x_2, 1); -lean_inc(x_18); -lean_dec(x_2); -lean_inc(x_3); -x_19 = lean_apply_4(x_18, lean_box(0), x_3, x_4, x_17); -x_20 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__12), 2, 1); -lean_closure_set(x_20, 0, x_3); -lean_inc(x_10); -x_21 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_20); -x_22 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_21, x_11); -return x_22; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = lean_ctor_get(x_2, 1); -lean_inc(x_9); -lean_inc(x_4); -lean_inc(x_3); -x_10 = lean_apply_4(x_8, lean_box(0), x_3, x_4, x_9); -lean_inc(x_3); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__10), 7, 6); -lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, x_5); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_4); -lean_closure_set(x_11, 4, x_7); -lean_closure_set(x_11, 5, x_6); -x_12 = lean_ctor_get(x_3, 1); -lean_inc(x_12); -x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__4___rarg), 5, 4); -lean_closure_set(x_13, 0, x_3); -lean_closure_set(x_13, 1, lean_box(0)); -lean_closure_set(x_13, 2, lean_box(0)); -lean_closure_set(x_13, 3, x_11); -x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: +else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_9 = lean_ctor_get(x_1, 1); -lean_inc(x_9); +lean_object* x_15; lean_object* x_16; lean_dec(x_1); -x_10 = lean_ctor_get(x_8, 0); -lean_inc(x_10); -lean_inc(x_7); -lean_inc(x_6); -x_11 = lean_apply_4(x_9, lean_box(0), x_6, x_7, x_10); -lean_inc(x_6); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__11), 7, 6); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_8); -lean_closure_set(x_12, 2, x_6); -lean_closure_set(x_12, 3, x_7); -lean_closure_set(x_12, 4, x_3); -lean_closure_set(x_12, 5, x_4); -x_13 = lean_ctor_get(x_6, 1); -lean_inc(x_13); -x_14 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___spec__5___rarg), 5, 4); -lean_closure_set(x_14, 0, x_6); -lean_closure_set(x_14, 1, lean_box(0)); -lean_closure_set(x_14, 2, lean_box(0)); -lean_closure_set(x_14, 3, x_12); -x_15 = lean_apply_4(x_13, lean_box(0), lean_box(0), x_11, x_14); -return x_15; -} +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; -lean_inc(x_7); -lean_inc(x_5); -lean_inc(x_3); -lean_inc(x_1); -x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__6), 8, 4); -lean_closure_set(x_8, 0, x_1); -lean_closure_set(x_8, 1, x_3); -lean_closure_set(x_8, 2, x_5); -lean_closure_set(x_8, 3, x_7); -x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg___lambda__12), 8, 4); -lean_closure_set(x_9, 0, x_1); -lean_closure_set(x_9, 1, x_3); -lean_closure_set(x_9, 2, x_5); -lean_closure_set(x_9, 3, x_7); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__10(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalRpcEncodingPacket___rarg), 7, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__10___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(lean_object* x_1) { -_start: -{ -uint8_t x_2; -x_2 = l_Std_Format_isNil(x_1); -if (x_2 == 0) -{ -lean_object* x_3; lean_object* x_4; -x_3 = lean_box(1); -x_4 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_3); -return x_4; -} -else -{ -return x_1; -} -} -} -LEAN_EXPORT lean_object* l_List_filterTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_3; -x_3 = l_List_reverse___rarg(x_2); -return x_3; -} -else -{ -uint8_t x_4; -x_4 = !lean_is_exclusive(x_1); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_1, 1); -x_7 = l_Lean_Name_isAnonymous(x_5); -if (x_7 == 0) +if (lean_obj_tag(x_5) == 0) { -lean_ctor_set(x_1, 1, x_2); +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* _tmp_0 = x_6; -lean_object* _tmp_1 = x_1; -x_1 = _tmp_0; -x_2 = _tmp_1; -} -goto _start; +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_free_object(x_1); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); lean_dec(x_5); -x_1 = x_6; -goto _start; -} -} -else -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_1, 0); -x_11 = lean_ctor_get(x_1, 1); +x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); -lean_inc(x_10); lean_dec(x_1); -x_12 = l_Lean_Name_isAnonymous(x_10); -if (x_12 == 0) -{ -lean_object* x_13; -x_13 = lean_alloc_ctor(1, 2, 0); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_13, 0, x_10); -lean_ctor_set(x_13, 1, x_2); -x_1 = x_11; -x_2 = x_13; -goto _start; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} } else { -lean_dec(x_10); -x_1 = x_11; -goto _start; -} -} +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__11(lean_object* x_1) { _start: { -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_3; -x_3 = l_List_reverse___rarg(x_2); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__11___rarg), 5, 0); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__12___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_1); -if (x_4 == 0) +if (lean_obj_tag(x_5) == 0) { -lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_1, 1); -x_7 = 1; -x_8 = l_Lean_Name_toString(x_5, x_7); -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_8); +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* _tmp_0 = x_6; -lean_object* _tmp_1 = x_1; -x_1 = _tmp_0; -x_2 = _tmp_1; -} -goto _start; +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_1, 0); -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_12 = 1; -x_13 = l_Lean_Name_toString(x_10, x_12); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_2); -x_1 = x_11; -x_2 = x_14; -goto _start; -} -} +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" ", 1); -return x_1; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2() { +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__12(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__12___rarg), 5, 0); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" :", 2); -return x_1; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_3 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_3, 0, x_2); +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_3); +x_7 = lean_apply_2(x_5, lean_box(0), x_6); +return x_7; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__4() { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__3; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_4 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__5() { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" : ", 3); -return x_1; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__11___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__6() { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__5; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__7() { -_start: +case 1: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(" :=", 3); -return x_1; +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__10___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__3), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__12___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__8() { +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__7; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg), 3, 0); return x_2; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__9() { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__13___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes(":", 1); -return x_1; +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__10() { +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__13(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__9; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__13___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__14___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { +if (lean_obj_tag(x_5) == 0) +{ uint8_t x_6; -x_6 = lean_usize_dec_lt(x_4, x_3); +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); if (x_6 == 0) { +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -return x_5; +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_7 = lean_array_uget(x_2, x_4); -x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(x_5); -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -x_10 = lean_array_to_list(lean_box(0), x_9); -x_11 = lean_box(0); -x_12 = l_List_filterTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__1(x_10, x_11); -x_13 = l_List_mapTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__2(x_12, x_11); -x_14 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1; -x_15 = l_String_intercalate(x_14, x_13); -x_16 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; -x_17 = lean_string_dec_eq(x_15, x_16); -if (x_17 == 0) -{ -lean_object* x_18; -x_18 = lean_ctor_get(x_7, 3); -lean_inc(x_18); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; -x_19 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_19, 0, x_15); -x_20 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; -x_21 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__4; -x_23 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -x_24 = lean_ctor_get(x_7, 2); -lean_inc(x_24); -lean_dec(x_7); -x_25 = l_Lean_Widget_TaggedText_stripTags___rarg(x_24); -x_26 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_26, 0, x_25); -x_27 = lean_box(1); -x_28 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -lean_inc(x_1); -x_29 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_29, 0, x_1); -lean_ctor_set(x_29, 1, x_28); -x_30 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_30, 0, x_23); -lean_ctor_set(x_30, 1, x_29); -x_31 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_20); -x_32 = 0; -x_33 = lean_alloc_ctor(5, 1, 1); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); -x_34 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_34, 0, x_8); -lean_ctor_set(x_34, 1, x_33); -x_35 = 1; -x_36 = lean_usize_add(x_4, x_35); -x_4 = x_36; -x_5 = x_34; -goto _start; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; -x_38 = lean_ctor_get(x_18, 0); -lean_inc(x_38); -lean_dec(x_18); -x_39 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_39, 0, x_15); -x_40 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; -x_41 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_41, 0, x_40); +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__14(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__14___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__15___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__15(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__15___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__18___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__18(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__18___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__18___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__19___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__19(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__19___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__20(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__20___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__21(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__21___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__20___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__19___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__21___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__22___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__22(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__22___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__23___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__23(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__23___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__24___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__24(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__24___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__26___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__26(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__26___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__26___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__28___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__28(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__28___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__28___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__29___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__29(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__29___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__30___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__30(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__30___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__33___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__33(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__33___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__33___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__34___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__34(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__34___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__35___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__35(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__35___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__36___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__36(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__36___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__35___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__34___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__36___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__37___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__37(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__37___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__38___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__38(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__38___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__39___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__39(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__39___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__42___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__42(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__42___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__42___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__43___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__43(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__43___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__44___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__44(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__44___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__45___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__45(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__45___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__44___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__43___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__45___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__46___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__46(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__46___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__47___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__47(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__47___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__48___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__48(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__48___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_box_usize(x_1); +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_3); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_2, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__2(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__5___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__2___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__6___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_2); +lean_ctor_set(x_8, 2, x_3); +lean_ctor_set(x_8, 3, x_4); +lean_ctor_set_uint8(x_8, sizeof(void*)*4, x_5); +lean_ctor_set_uint8(x_8, sizeof(void*)*4 + 1, x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +x_10 = lean_apply_2(x_6, lean_box(0), x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__4___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__13___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__5___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__14___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_dec(x_4); +x_6 = lean_apply_2(x_5, lean_box(0), x_2); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +lean_dec(x_1); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_7); +x_11 = lean_apply_2(x_9, lean_box(0), x_10); +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_2); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_2, 0); +x_14 = lean_ctor_get(x_1, 0); +lean_inc(x_14); +lean_dec(x_1); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_13); +lean_ctor_set(x_2, 0, x_16); +x_17 = lean_apply_2(x_15, lean_box(0), x_2); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +lean_dec(x_2); +x_19 = lean_ctor_get(x_1, 0); +lean_inc(x_19); +lean_dec(x_1); +x_20 = lean_ctor_get(x_19, 1); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_21, 0, x_18); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = lean_apply_2(x_20, lean_box(0), x_22); +return x_23; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__6), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__15___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__16___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__3), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__8), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__22___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__10(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__9), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__23___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11(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; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_array_get_size(x_5); +x_7 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_8 = 0; +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg(x_2, x_7, x_8, x_5); +x_10 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11___boxed__const__1; +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__10___boxed), 5, 4); +lean_closure_set(x_11, 0, x_4); +lean_closure_set(x_11, 1, x_2); +lean_closure_set(x_11, 2, x_10); +lean_closure_set(x_11, 3, x_3); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__24___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_9, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +x_6 = lean_apply_2(x_2, lean_box(0), x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__29___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__13___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__30___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, uint8_t x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_alloc_ctor(0, 4, 2); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_2); +lean_ctor_set(x_8, 2, x_3); +lean_ctor_set(x_8, 3, x_4); +lean_ctor_set_uint8(x_8, sizeof(void*)*4, x_5); +lean_ctor_set_uint8(x_8, sizeof(void*)*4 + 1, x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +x_10 = lean_apply_2(x_6, lean_box(0), x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__37___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__16___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__38___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__17), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__39___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__40___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__14), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__31___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__18), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__46___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__20(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__19), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__47___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21(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; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_array_get_size(x_5); +x_7 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_8 = 0; +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg(x_2, x_7, x_8, x_5); +x_10 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21___boxed__const__1; +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__20___boxed), 5, 4); +lean_closure_set(x_11, 0, x_4); +lean_closure_set(x_11, 1, x_2); +lean_closure_set(x_11, 2, x_10); +lean_closure_set(x_11, 3, x_3); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__48___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_9, x_13); +return x_14; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__3; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__1___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__3___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__8___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__17___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__25___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__27___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__32___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__41___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1(x_4, x_2, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__2(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___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) { +_start: +{ +uint8_t x_8; uint8_t x_9; lean_object* x_10; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = lean_unbox(x_7); +lean_dec(x_7); +x_10 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__4(x_1, x_2, x_3, x_4, x_8, x_6, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__10(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__13(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +uint8_t x_8; uint8_t x_9; lean_object* x_10; +x_8 = lean_unbox(x_5); +lean_dec(x_5); +x_9 = lean_unbox(x_7); +lean_dec(x_7); +x_10 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15(x_1, x_2, x_3, x_4, x_8, x_6, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__16(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__20(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +static lean_object* _init_l_Lean_Widget_InteractiveGoal_mvarId_x3f___default() { +_start: +{ +lean_object* x_1; +x_1 = lean_box(0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveGoal___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = lean_box(0); +x_2 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__1; +x_3 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__3; +x_4 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; +x_5 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_5, 0, x_2); +lean_ctor_set(x_5, 1, x_3); +lean_ctor_set(x_5, 2, x_1); +lean_ctor_set(x_5, 3, x_4); +lean_ctor_set(x_5, 4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveGoal() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instInhabitedInteractiveGoal___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__2(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_array_uget(x_3, x_2); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_3, x_2, x_7); +x_9 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136_(x_6); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +lean_dec(x_8); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; +} +} +else +{ +lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = 1; +x_15 = lean_usize_add(x_2, x_14); +x_16 = lean_array_uset(x_8, x_2, x_13); +x_2 = x_15; +x_3 = x_16; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +if (lean_obj_tag(x_3) == 4) +{ +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_array_get_size(x_4); +x_6 = lean_usize_of_nat(x_5); +lean_dec(x_5); +x_7 = 0; +x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__2(x_6, x_7, x_4); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_9 = lean_unsigned_to_nat(80u); +x_10 = l_Lean_Json_pretty(x_3, x_9); +x_11 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; +} +} +} +static lean_object* _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__1; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; +x_4 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +return x_4; +} +else +{ +lean_object* x_5; +x_5 = l_Lean_Json_getStr_x3f(x_3); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_3); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +return x_5; +} +else +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +return x_8; +} +} +else +{ +uint8_t x_9; +x_9 = !lean_is_exclusive(x_5); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_5, 0); +x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1; +x_12 = lean_string_dec_eq(x_10, x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2; +x_14 = lean_string_append(x_13, x_10); +lean_dec(x_10); +x_15 = l_Lean_Syntax_decodeNameLit(x_14); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_16 = lean_unsigned_to_nat(80u); +x_17 = l_Lean_Json_pretty(x_3, x_16); +x_18 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3; +x_19 = lean_string_append(x_18, x_17); +lean_dec(x_17); +x_20 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_21 = lean_string_append(x_19, x_20); +lean_ctor_set_tag(x_5, 0); +lean_ctor_set(x_5, 0, x_21); +return x_5; +} +else +{ +uint8_t x_22; +lean_dec(x_3); +x_22 = !lean_is_exclusive(x_15); +if (x_22 == 0) +{ +lean_ctor_set(x_5, 0, x_15); +return x_5; +} +else +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_15, 0); +lean_inc(x_23); +lean_dec(x_15); +x_24 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_5, 0, x_24); +return x_5; +} +} +} +else +{ +lean_object* x_25; +lean_free_object(x_5); +lean_dec(x_10); +lean_dec(x_3); +x_25 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__2; +return x_25; +} +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = lean_ctor_get(x_5, 0); +lean_inc(x_26); +lean_dec(x_5); +x_27 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1; +x_28 = lean_string_dec_eq(x_26, x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2; +x_30 = lean_string_append(x_29, x_26); +lean_dec(x_26); +x_31 = l_Lean_Syntax_decodeNameLit(x_30); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_32 = lean_unsigned_to_nat(80u); +x_33 = l_Lean_Json_pretty(x_3, x_32); +x_34 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3; +x_35 = lean_string_append(x_34, x_33); +lean_dec(x_33); +x_36 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_37 = lean_string_append(x_35, x_36); +x_38 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_38, 0, x_37); +return x_38; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +lean_dec(x_3); +x_39 = lean_ctor_get(x_31, 0); +lean_inc(x_39); +if (lean_is_exclusive(x_31)) { + lean_ctor_release(x_31, 0); + x_40 = x_31; +} else { + lean_dec_ref(x_31); + x_40 = lean_box(0); +} +if (lean_is_scalar(x_40)) { + x_41 = lean_alloc_ctor(1, 1, 0); +} else { + x_41 = x_40; +} +lean_ctor_set(x_41, 0, x_39); +x_42 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_42, 0, x_41); +return x_42; +} +} +else +{ +lean_object* x_43; +lean_dec(x_26); +lean_dec(x_3); +x_43 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__2; +return x_43; +} +} +} +} +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("hyps", 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("userName", 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("goalPrefix", 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("mvarId", 6); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1; +lean_inc(x_1); +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__1(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +lean_dec(x_1); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3; +lean_inc(x_1); +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__5(x_1, x_8); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +lean_dec(x_7); +lean_dec(x_1); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__2; +x_15 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2161____spec__1(x_1, x_14); +if (lean_obj_tag(x_15) == 0) +{ +uint8_t x_16; +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_1); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +return x_15; +} +else +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; +} +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_15, 0); +lean_inc(x_19); +lean_dec(x_15); +x_20 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__3; +x_21 = l_Lean_Json_getObjValAs_x3f___at_Lean_JsonRpc_instFromJsonMessage___spec__3(x_1, x_20); +if (lean_obj_tag(x_21) == 0) +{ +uint8_t x_22; +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +return x_21; +} +else +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_24, 0, x_23); +return x_24; +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_21, 0); +lean_inc(x_25); +lean_dec(x_21); +x_26 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__4; +x_27 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3(x_1, x_26); +lean_dec(x_1); +if (lean_obj_tag(x_27) == 0) +{ +uint8_t x_28; +lean_dec(x_25); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_7); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +return x_27; +} +else +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_27, 0); +lean_inc(x_29); +lean_dec(x_27); +x_30 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_30, 0, x_29); +return x_30; +} +} +else +{ +uint8_t x_31; +x_31 = !lean_is_exclusive(x_27); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_27, 0); +x_33 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_33, 0, x_7); +lean_ctor_set(x_33, 1, x_13); +lean_ctor_set(x_33, 2, x_19); +lean_ctor_set(x_33, 3, x_25); +lean_ctor_set(x_33, 4, x_32); +lean_ctor_set(x_27, 0, x_33); +return x_27; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_27, 0); +lean_inc(x_34); +lean_dec(x_27); +x_35 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_35, 0, x_7); +lean_ctor_set(x_35, 1, x_13); +lean_ctor_set(x_35, 2, x_19); +lean_ctor_set(x_35, 3, x_25); +lean_ctor_set(x_35, 4, x_34); +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_35); +return x_36; +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__2(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__2() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket__2___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__1(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259_(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Json_opt___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +lean_dec(x_1); +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_4 = lean_ctor_get(x_2, 0); +lean_inc(x_4); +lean_dec(x_2); +x_5 = 1; +x_6 = l_Lean_Name_toString(x_4, x_5); +x_7 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_7, 0, x_6); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_7); +x_9 = lean_box(0); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +return x_10; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = lean_array_get_size(x_2); +x_4 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_5 = 0; +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__1(x_4, x_5, x_2); +x_7 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_7, 0, x_6); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1; +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +x_13 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_12); +x_14 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3; +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_10); +x_17 = lean_ctor_get(x_1, 2); +lean_inc(x_17); +x_18 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__2; +x_19 = l_Lean_Json_opt___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonDocumentFilter____x40_Lean_Data_Lsp_Basic___hyg_2131____spec__1(x_18, x_17); +lean_dec(x_17); +x_20 = lean_ctor_get(x_1, 3); +lean_inc(x_20); +x_21 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_21, 0, x_20); +x_22 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__3; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_10); +x_25 = lean_ctor_get(x_1, 4); +lean_inc(x_25); +lean_dec(x_1); +x_26 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__4; +x_27 = l_Lean_Json_opt___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__2(x_26, x_25); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_10); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_24); +lean_ctor_set(x_29, 1, x_28); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_19); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_16); +lean_ctor_set(x_31, 1, x_30); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_11); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_List_join___rarg(x_32); +x_34 = l_Lean_Json_mkObj(x_33); +return x_34; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__1(x_4, x_5, x_3); +return x_6; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__2() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket__2___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__2___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__2___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__4___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__5___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__6(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__6___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__9(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__9___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__9___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__10(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__10___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__11___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__12___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__12(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__12___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__11___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__10___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__12___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__13___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__13(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__13___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__14___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__14(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__14___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__15___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__15(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__15___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__18___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__18(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__18___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__18___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__19___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__19(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__19___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__20(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__20___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__21(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__21___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__20___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__19___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__21___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__22___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__22(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__22___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__23___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__23(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__23___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__24___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__24(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__24___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__26___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__26(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__26___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__1(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__5___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__6___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__4___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__13___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__14___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__4), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__15___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__16___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__2), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__7___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__5), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__22___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__7(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__6), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__23___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__8(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg(x_1, x_16, x_17, x_14); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed__const__1; +lean_inc(x_2); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__7___boxed), 5, 4); +lean_closure_set(x_20, 0, x_11); +lean_closure_set(x_20, 1, x_1); +lean_closure_set(x_20, 2, x_19); +lean_closure_set(x_20, 3, x_2); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__24___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +lean_inc(x_21); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_18, x_22); +x_24 = lean_box_usize(x_4); +x_25 = lean_box_usize(x_3); +lean_inc(x_1); +x_26 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__8___boxed), 6, 5); +lean_closure_set(x_26, 0, x_24); +lean_closure_set(x_26, 1, x_13); +lean_closure_set(x_26, 2, x_1); +lean_closure_set(x_26, 3, x_2); +lean_closure_set(x_26, 4, x_25); +x_27 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__26___rarg), 5, 4); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, lean_box(0)); +lean_closure_set(x_27, 2, lean_box(0)); +lean_closure_set(x_27, 3, x_26); +x_28 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_23, x_27); +return x_28; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__27(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__27___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__28___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__28(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__28___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__31___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__31(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__31___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__31___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__32___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__32(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__32___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__33___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__33(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__33___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__34___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__34(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__34___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__33___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__32___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__34___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__35___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__35(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__35___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__36___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__36(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__36___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__37___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__37(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__37___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__38___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__38(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__38___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__39___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__39(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__39___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__41___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__41(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__41___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__41___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__43___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__43(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__43___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__43___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__44___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__44(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__44___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__45___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__45(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__45___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__48___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__48(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__48___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__48___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__49___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__49(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__49___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__50___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__50(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__50___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__51___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__51(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__51___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__50___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__49___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__51___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__52___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__52(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__52___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__53___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__53(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__53___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__54___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__54(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__54___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__57___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__57(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__57___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__57___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__58___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__58(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__58___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__59___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__59(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__59___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__60___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__60(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__60___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__59___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__58___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__60___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__61___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__61(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__61___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__62___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__62(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__62___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__63___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__63(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__63___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__65___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__65(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__65___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__44___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__45___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__52___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__53___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__4), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__54___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__55___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__2), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__46___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__5), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__61___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__7(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__6), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__62___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__8(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg(x_1, x_16, x_17, x_14); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed__const__1; +lean_inc(x_2); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__7___boxed), 5, 4); +lean_closure_set(x_20, 0, x_11); +lean_closure_set(x_20, 1, x_1); +lean_closure_set(x_20, 2, x_19); +lean_closure_set(x_20, 3, x_2); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__63___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +lean_inc(x_21); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_18, x_22); +x_24 = lean_box_usize(x_4); +x_25 = lean_box_usize(x_3); +lean_inc(x_1); +x_26 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__8___boxed), 6, 5); +lean_closure_set(x_26, 0, x_24); +lean_closure_set(x_26, 1, x_13); +lean_closure_set(x_26, 2, x_1); +lean_closure_set(x_26, 3, x_2); +lean_closure_set(x_26, 4, x_25); +x_27 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__65___rarg), 5, 4); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, lean_box(0)); +lean_closure_set(x_27, 2, lean_box(0)); +lean_closure_set(x_27, 3, x_26); +x_28 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_23, x_27); +return x_28; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__66___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__66(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__66___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__67___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__67(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__67___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__70___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__70(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__70___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__70___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__71___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__71(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__71___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__72___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__72(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__72___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__73___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__73(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__73___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__72___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__71___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__73___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__74___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__74(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__74___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__75___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__75(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__75___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__76___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__76(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__76___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__77___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__77(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__77___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__78___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__78(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__78___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__1(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__27___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__28___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_7, 0, x_1); +lean_ctor_set(x_7, 1, x_2); +lean_ctor_set(x_7, 2, x_3); +lean_ctor_set(x_7, 3, x_4); +lean_ctor_set(x_7, 4, x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_apply_2(x_5, lean_box(0), x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; +x_4 = lean_apply_2(x_1, lean_box(0), x_2); +return x_4; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_1, lean_box(0), x_6); +return x_7; +} +} +else +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_2); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_2, 0, x_10); +x_11 = lean_apply_2(x_1, lean_box(0), x_2); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); +lean_dec(x_2); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = lean_apply_2(x_1, lean_box(0), x_14); +return x_15; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 4); +lean_inc(x_5); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__3), 6, 5); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_7); +lean_closure_set(x_9, 4, x_5); +x_10 = lean_ctor_get(x_6, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__35___rarg), 5, 4); +lean_closure_set(x_11, 0, x_6); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_13 = lean_apply_2(x_5, lean_box(0), x_12); +x_14 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_13, x_11); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_8, 0); +lean_inc(x_15); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_inc(x_5); +x_17 = lean_apply_2(x_5, lean_box(0), x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4), 2, 1); +lean_closure_set(x_18, 0, x_5); +lean_inc(x_10); +x_19 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_11); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 3); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_6); +lean_inc(x_8); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__5___boxed), 7, 6); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_3); +lean_closure_set(x_11, 2, x_4); +lean_closure_set(x_11, 3, x_5); +lean_closure_set(x_11, 4, x_8); +lean_closure_set(x_11, 5, x_2); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__36___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__7(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; +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__6), 5, 4); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +lean_closure_set(x_6, 2, x_3); +lean_closure_set(x_6, 3, x_4); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__37___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_14); +lean_inc(x_16); +x_18 = lean_apply_2(x_16, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4), 2, 1); +lean_closure_set(x_19, 0, x_16); +lean_inc(x_7); +x_20 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_20, x_8); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_3); +lean_inc(x_2); +x_7 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__29___rarg(x_2, x_6, x_5); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__7), 4, 3); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__38___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_array_get_size(x_5); +x_7 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_8 = 0; +lean_inc(x_3); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg(x_2, x_3, x_7, x_8, x_5); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__8), 4, 3); +lean_closure_set(x_10, 0, x_4); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_3); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__39___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__66___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__10___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__67___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_7, 0, x_1); +lean_ctor_set(x_7, 1, x_2); +lean_ctor_set(x_7, 2, x_3); +lean_ctor_set(x_7, 3, x_4); +lean_ctor_set(x_7, 4, x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_apply_2(x_5, lean_box(0), x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 4); +lean_inc(x_5); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__12), 6, 5); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_7); +lean_closure_set(x_9, 4, x_5); +x_10 = lean_ctor_get(x_6, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__74___rarg), 5, 4); +lean_closure_set(x_11, 0, x_6); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_13 = lean_apply_2(x_5, lean_box(0), x_12); +x_14 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_13, x_11); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_8, 0); +lean_inc(x_15); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_inc(x_5); +x_17 = lean_apply_2(x_5, lean_box(0), x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4), 2, 1); +lean_closure_set(x_18, 0, x_5); +lean_inc(x_10); +x_19 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_11); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__14(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 3); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_6); +lean_inc(x_8); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__13___boxed), 7, 6); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_3); +lean_closure_set(x_11, 2, x_4); +lean_closure_set(x_11, 3, x_5); +lean_closure_set(x_11, 4, x_8); +lean_closure_set(x_11, 5, x_2); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__75___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__15(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; +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__14), 5, 4); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +lean_closure_set(x_6, 2, x_3); +lean_closure_set(x_6, 3, x_4); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__76___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_14); +lean_inc(x_16); +x_18 = lean_apply_2(x_16, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4), 2, 1); +lean_closure_set(x_19, 0, x_16); +lean_inc(x_7); +x_20 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_20, x_8); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__11), 3, 2); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_3); +lean_inc(x_2); +x_7 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__68___rarg(x_2, x_6, x_5); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__15), 4, 3); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__77___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__17(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; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_array_get_size(x_5); +x_7 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_8 = 0; +lean_inc(x_3); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg(x_2, x_3, x_7, x_8, x_5); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__16), 4, 3); +lean_closure_set(x_10, 0, x_4); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_3); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__78___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__9), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__17), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveGoal() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__3; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__1___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__3___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__8___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__17___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__1(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__7(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___lambda__8(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__30___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__40___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__42___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__47___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__56___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__7(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___lambda__8(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__69___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__1(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__10(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__13(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = l_Std_Format_isNil(x_1); +if (x_2 == 0) +{ +lean_object* x_3; lean_object* x_4; +x_3 = lean_box(1); +x_4 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +return x_4; +} +else +{ +return x_1; +} +} +} +LEAN_EXPORT lean_object* l_List_filterTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; +x_3 = l_List_reverse___rarg(x_2); +return x_3; +} +else +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_1); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_1, 1); +x_7 = l_Lean_Name_isAnonymous(x_5); +if (x_7 == 0) +{ +lean_ctor_set(x_1, 1, x_2); +{ +lean_object* _tmp_0 = x_6; +lean_object* _tmp_1 = x_1; +x_1 = _tmp_0; +x_2 = _tmp_1; +} +goto _start; +} +else +{ +lean_free_object(x_1); +lean_dec(x_5); +x_1 = x_6; +goto _start; +} +} +else +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_1, 0); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_inc(x_10); +lean_dec(x_1); +x_12 = l_Lean_Name_isAnonymous(x_10); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_10); +lean_ctor_set(x_13, 1, x_2); +x_1 = x_11; +x_2 = x_13; +goto _start; +} +else +{ +lean_dec(x_10); +x_1 = x_11; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_List_mapTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; +x_3 = l_List_reverse___rarg(x_2); +return x_3; +} +else +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_1); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_1, 1); +x_7 = 1; +x_8 = l_Lean_Name_toString(x_5, x_7); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set(x_1, 0, x_8); +{ +lean_object* _tmp_0 = x_6; +lean_object* _tmp_1 = x_1; +x_1 = _tmp_0; +x_2 = _tmp_1; +} +goto _start; +} +else +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_1, 0); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_inc(x_10); +lean_dec(x_1); +x_12 = 1; +x_13 = l_Lean_Name_toString(x_10, x_12); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_2); +x_1 = x_11; +x_2 = x_14; +goto _start; +} +} +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(" ", 1); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(" :", 2); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__3; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(" : ", 3); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__5; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(" :=", 3); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__7; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes(":", 1); +return x_1; +} +} +static lean_object* _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__9; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_dec(x_1); +return x_5; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_7 = lean_array_uget(x_2, x_4); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(x_5); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +x_10 = lean_array_to_list(lean_box(0), x_9); +x_11 = lean_box(0); +x_12 = l_List_filterTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__1(x_10, x_11); +x_13 = l_List_mapTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__2(x_12, x_11); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1; +x_15 = l_String_intercalate(x_14, x_13); +x_16 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; +x_17 = lean_string_dec_eq(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_7, 3); +lean_inc(x_18); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; +x_19 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_19, 0, x_15); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; +x_21 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +x_22 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__4; +x_23 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_ctor_get(x_7, 2); +lean_inc(x_24); +lean_dec(x_7); +x_25 = l_Lean_Widget_TaggedText_stripTags___rarg(x_24); +x_26 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_27 = lean_box(1); +x_28 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +lean_inc(x_1); +x_29 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_29, 0, x_1); +lean_ctor_set(x_29, 1, x_28); +x_30 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_30, 0, x_23); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_20); +x_32 = 0; +x_33 = lean_alloc_ctor(5, 1, 1); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); +x_34 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_34, 0, x_8); +lean_ctor_set(x_34, 1, x_33); +x_35 = 1; +x_36 = lean_usize_add(x_4, x_35); +x_4 = x_36; +x_5 = x_34; +goto _start; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; +x_38 = lean_ctor_get(x_18, 0); +lean_inc(x_38); +lean_dec(x_18); +x_39 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_39, 0, x_15); +x_40 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; +x_41 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_39); +x_42 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__6; +x_43 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_ctor_get(x_7, 2); +lean_inc(x_44); +lean_dec(x_7); +x_45 = l_Lean_Widget_TaggedText_stripTags___rarg(x_44); +x_46 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_47, 0, x_43); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__8; +x_49 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_Widget_TaggedText_stripTags___rarg(x_38); +x_51 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_51, 0, x_50); +x_52 = lean_box(1); +x_53 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +lean_inc(x_1); +x_54 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_54, 0, x_1); +lean_ctor_set(x_54, 1, x_53); +x_55 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_55, 0, x_49); +lean_ctor_set(x_55, 1, x_54); +x_56 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_40); +x_57 = 0; +x_58 = lean_alloc_ctor(5, 1, 1); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set_uint8(x_58, sizeof(void*)*1, x_57); +x_59 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_59, 0, x_8); +lean_ctor_set(x_59, 1, x_58); +x_60 = 1; +x_61 = lean_usize_add(x_4, x_60); +x_4 = x_61; +x_5 = x_59; +goto _start; +} +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; size_t x_76; size_t x_77; +lean_dec(x_15); +x_63 = lean_ctor_get(x_7, 2); +lean_inc(x_63); +lean_dec(x_7); +x_64 = l_Lean_Widget_TaggedText_stripTags___rarg(x_63); +x_65 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = lean_box(1); +x_67 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_65); +lean_inc(x_1); +x_68 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_68, 0, x_1); +lean_ctor_set(x_68, 1, x_67); +x_69 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__10; +x_70 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_68); +x_71 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; +x_72 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +x_73 = 0; +x_74 = lean_alloc_ctor(5, 1, 1); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set_uint8(x_74, sizeof(void*)*1, x_73); +x_75 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_75, 0, x_8); +lean_ctor_set(x_75, 1, x_74); +x_76 = 1; +x_77 = lean_usize_add(x_4, x_76); +x_4 = x_77; +x_5 = x_75; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_dec(x_1); +return x_5; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_7 = lean_array_uget(x_2, x_4); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(x_5); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +x_10 = lean_array_to_list(lean_box(0), x_9); +x_11 = lean_box(0); +x_12 = l_List_filterTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__1(x_10, x_11); +x_13 = l_List_mapTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__2(x_12, x_11); +x_14 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1; +x_15 = l_String_intercalate(x_14, x_13); +x_16 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; +x_17 = lean_string_dec_eq(x_15, x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_7, 3); +lean_inc(x_18); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; +x_19 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_19, 0, x_15); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; +x_21 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +x_22 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__4; +x_23 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_ctor_get(x_7, 2); +lean_inc(x_24); +lean_dec(x_7); +x_25 = l_Lean_Widget_TaggedText_stripTags___rarg(x_24); +x_26 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_27 = lean_box(1); +x_28 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +lean_inc(x_1); +x_29 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_29, 0, x_1); +lean_ctor_set(x_29, 1, x_28); +x_30 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_30, 0, x_23); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_20); +x_32 = 0; +x_33 = lean_alloc_ctor(5, 1, 1); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); +x_34 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_34, 0, x_8); +lean_ctor_set(x_34, 1, x_33); +x_35 = 1; +x_36 = lean_usize_add(x_4, x_35); +x_4 = x_36; +x_5 = x_34; +goto _start; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; +x_38 = lean_ctor_get(x_18, 0); +lean_inc(x_38); +lean_dec(x_18); +x_39 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_39, 0, x_15); +x_40 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; +x_41 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_41, 0, x_40); lean_ctor_set(x_41, 1, x_39); x_42 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__6; x_43 = lean_alloc_ctor(4, 2, 0); @@ -3444,681 +15585,12887 @@ lean_ctor_set(x_43, 1, x_42); x_44 = lean_ctor_get(x_7, 2); lean_inc(x_44); lean_dec(x_7); -x_45 = l_Lean_Widget_TaggedText_stripTags___rarg(x_44); -x_46 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_46, 0, x_45); -x_47 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_47, 0, x_43); -lean_ctor_set(x_47, 1, x_46); -x_48 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__8; -x_49 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); -x_50 = l_Lean_Widget_TaggedText_stripTags___rarg(x_38); -x_51 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_51, 0, x_50); -x_52 = lean_box(1); -x_53 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_51); +x_45 = l_Lean_Widget_TaggedText_stripTags___rarg(x_44); +x_46 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_47, 0, x_43); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__8; +x_49 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_Widget_TaggedText_stripTags___rarg(x_38); +x_51 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_51, 0, x_50); +x_52 = lean_box(1); +x_53 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +lean_inc(x_1); +x_54 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_54, 0, x_1); +lean_ctor_set(x_54, 1, x_53); +x_55 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_55, 0, x_49); +lean_ctor_set(x_55, 1, x_54); +x_56 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_40); +x_57 = 0; +x_58 = lean_alloc_ctor(5, 1, 1); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set_uint8(x_58, sizeof(void*)*1, x_57); +x_59 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_59, 0, x_8); +lean_ctor_set(x_59, 1, x_58); +x_60 = 1; +x_61 = lean_usize_add(x_4, x_60); +x_4 = x_61; +x_5 = x_59; +goto _start; +} +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; size_t x_76; size_t x_77; +lean_dec(x_15); +x_63 = lean_ctor_get(x_7, 2); +lean_inc(x_63); +lean_dec(x_7); +x_64 = l_Lean_Widget_TaggedText_stripTags___rarg(x_63); +x_65 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = lean_box(1); +x_67 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_65); +lean_inc(x_1); +x_68 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_68, 0, x_1); +lean_ctor_set(x_68, 1, x_67); +x_69 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__10; +x_70 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_68); +x_71 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; +x_72 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +x_73 = 0; +x_74 = lean_alloc_ctor(5, 1, 1); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set_uint8(x_74, sizeof(void*)*1, x_73); +x_75 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_75, 0, x_8); +lean_ctor_set(x_75, 1, x_74); +x_76 = 1; +x_77 = lean_usize_add(x_4, x_76); +x_4 = x_77; +x_5 = x_75; +goto _start; +} +} +} +} +static lean_object* _init_l_Lean_Widget_InteractiveGoal_pretty___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(2u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Widget_InteractiveGoal_pretty___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("case ", 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_InteractiveGoal_pretty___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Widget_InteractiveGoal_pretty___closed__2; +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveGoal_pretty(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_2 = lean_ctor_get(x_1, 2); +lean_inc(x_2); +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_array_get_size(x_3); +x_5 = lean_usize_of_nat(x_4); +lean_dec(x_4); +x_6 = 0; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +x_8 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; +x_10 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +x_11 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +lean_dec(x_1); +x_13 = l_Lean_Widget_TaggedText_stripTags___rarg(x_12); +x_14 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = l_Lean_Widget_InteractiveGoal_pretty___closed__1; +x_16 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +x_17 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_17, 0, x_11); +lean_ctor_set(x_17, 1, x_16); +x_18 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_9); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_box(0); +x_20 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3(x_15, x_3, x_5, x_6, x_19); +lean_dec(x_3); +x_21 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(x_20); +x_22 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_18); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_23 = lean_ctor_get(x_2, 0); +lean_inc(x_23); +lean_dec(x_2); +x_24 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_24, 0, x_23); +x_25 = l_Lean_Widget_InteractiveGoal_pretty___closed__3; +x_26 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_24); +x_27 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_9); +x_28 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4(x_15, x_3, x_5, x_6, x_27); +lean_dec(x_3); +x_29 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(x_28); +x_30 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_18); +return x_30; +} +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_2); +return x_8; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__1; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__1; +x_2 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__3; +x_3 = l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__2; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveTermGoal() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__3; +return x_1; +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("range", 5); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1; +lean_inc(x_1); +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__1(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +lean_dec(x_1); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_3, 0); +lean_inc(x_7); +lean_dec(x_3); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3; +lean_inc(x_1); +x_9 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__5(x_1, x_8); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +lean_dec(x_7); +lean_dec(x_1); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; +} +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491____closed__1; +x_15 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonLocation____x40_Lean_Data_Lsp_Basic___hyg_940____spec__2(x_1, x_14); +lean_dec(x_1); +if (lean_obj_tag(x_15) == 0) +{ +uint8_t x_16; +lean_dec(x_13); +lean_dec(x_7); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +return x_15; +} +else +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_15); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_15, 0); +x_21 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_21, 0, x_7); +lean_ctor_set(x_21, 1, x_13); +lean_ctor_set(x_21, 2, x_20); +lean_ctor_set(x_15, 0, x_21); +return x_15; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 0); +lean_inc(x_22); +lean_dec(x_15); +x_23 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_23, 0, x_7); +lean_ctor_set(x_23, 1, x_13); +lean_ctor_set(x_23, 2, x_22); +x_24 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_24, 0, x_23); +return x_24; +} +} +} +} +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket__3___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1563_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +x_3 = lean_array_get_size(x_2); +x_4 = lean_usize_of_nat(x_3); +lean_dec(x_3); +x_5 = 0; +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802____spec__1(x_4, x_5, x_2); +x_7 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_7, 0, x_6); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1; +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_12); +x_13 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3(x_12); +x_14 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3; +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_10); +x_17 = lean_ctor_get(x_1, 2); +lean_inc(x_17); +lean_dec(x_1); +x_18 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_623_(x_17); +x_19 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491____closed__1; +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_10); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_10); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_16); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_11); +lean_ctor_set(x_24, 1, x_23); +x_25 = l_List_join___rarg(x_24); +x_26 = l_Lean_Json_mkObj(x_25); +return x_26; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1563_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket__3___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__2___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__2___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__4___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__5___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__6(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__6___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__9(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__9___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__9___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__10(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__10___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__11___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__12___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__12(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__12___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__11___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__10___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__12___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__13___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__13(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__13___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__14___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__14(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__14___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__15___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__15(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__15___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__18___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__18(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__18___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__18___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__19___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__19(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__19___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__20(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__20___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__21(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__21___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__20___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__19___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__21___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__22___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__22(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__22___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__23___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__23(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__23___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__24___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__24(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__24___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__26___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__26(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__26___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__1(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__5___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__6___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__4___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__13___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__14___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__4), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__15___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__16___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__2), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__7___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__5), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__22___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__7(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__6), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__23___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__8(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg(x_1, x_16, x_17, x_14); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed__const__1; +lean_inc(x_2); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__7___boxed), 5, 4); +lean_closure_set(x_20, 0, x_11); +lean_closure_set(x_20, 1, x_1); +lean_closure_set(x_20, 2, x_19); +lean_closure_set(x_20, 3, x_2); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__24___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +lean_inc(x_21); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_18, x_22); +x_24 = lean_box_usize(x_4); +x_25 = lean_box_usize(x_3); +lean_inc(x_1); +x_26 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__8___boxed), 6, 5); +lean_closure_set(x_26, 0, x_24); +lean_closure_set(x_26, 1, x_13); +lean_closure_set(x_26, 2, x_1); +lean_closure_set(x_26, 3, x_2); +lean_closure_set(x_26, 4, x_25); +x_27 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__26___rarg), 5, 4); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, lean_box(0)); +lean_closure_set(x_27, 2, lean_box(0)); +lean_closure_set(x_27, 3, x_26); +x_28 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_23, x_27); +return x_28; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__27(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__27___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__28___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__28(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__28___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__31___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__31(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__31___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__31___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__32___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__32(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__32___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__33___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__33(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__33___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__34___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__34(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__34___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__33___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__32___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__34___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__35___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__35(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__35___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__36___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__36(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__36___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__37___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__37(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__37___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__39___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__39(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__39___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__39___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__41___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__41(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__41___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__41___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__42___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__42(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__42___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__43___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__43(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__43___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__46___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__46(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__46___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__46___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__47___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__47(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__47___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__48___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__48(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__48___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__49___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__49(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__49___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__48___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__47___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__49___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__50___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__50(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__50___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__51___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__51(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__51___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__52___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__52(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__52___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__55___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__55(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__55___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__55___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__56___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__56(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__56___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__57___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__57(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__57___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__58___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__58(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__58___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__57___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__56___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__58___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__59___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__59(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__59___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__60___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__60(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__60___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__61___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__61(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__61___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__63___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__63(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__63___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__42___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__43___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__50___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__51___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__4), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__52___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__53___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__2), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__44___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__5), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__59___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__7(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__6), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__60___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__8(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg(x_1, x_16, x_17, x_14); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed__const__1; +lean_inc(x_2); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__7___boxed), 5, 4); +lean_closure_set(x_20, 0, x_11); +lean_closure_set(x_20, 1, x_1); +lean_closure_set(x_20, 2, x_19); +lean_closure_set(x_20, 3, x_2); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__61___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +lean_inc(x_21); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_18, x_22); +x_24 = lean_box_usize(x_4); +x_25 = lean_box_usize(x_3); +lean_inc(x_1); +x_26 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__8___boxed), 6, 5); +lean_closure_set(x_26, 0, x_24); +lean_closure_set(x_26, 1, x_13); +lean_closure_set(x_26, 2, x_1); +lean_closure_set(x_26, 3, x_2); +lean_closure_set(x_26, 4, x_25); +x_27 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__63___rarg), 5, 4); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, lean_box(0)); +lean_closure_set(x_27, 2, lean_box(0)); +lean_closure_set(x_27, 3, x_26); +x_28 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_23, x_27); +return x_28; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__64___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__64(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__64___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__65___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__65(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__65___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__68___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__68(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__68___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__68___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__69___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__69(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__69___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__70___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__70(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__70___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__71___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__71(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__71___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__70___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__69___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__71___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__72___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__72(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__72___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__73___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__73(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__73___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__74___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__74(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__74___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__1(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__27___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__28___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_3, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_5 = lean_ctor_get(x_1, 2); +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +lean_inc(x_5); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_5); +lean_inc(x_7); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__3), 4, 3); +lean_closure_set(x_10, 0, x_3); +lean_closure_set(x_10, 1, x_4); +lean_closure_set(x_10, 2, x_7); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__35___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_3); +lean_inc(x_2); +x_7 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__29___rarg(x_2, x_6, x_5); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__4___boxed), 4, 3); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__36___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_array_get_size(x_5); +x_7 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_8 = 0; +lean_inc(x_3); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg(x_2, x_3, x_7, x_8, x_5); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__5), 4, 3); +lean_closure_set(x_10, 0, x_4); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_3); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__37___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__64___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__7___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__65___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_apply_2(x_3, lean_box(0), x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_5 = lean_ctor_get(x_1, 2); +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +lean_inc(x_5); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_5); +lean_inc(x_7); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__9), 4, 3); +lean_closure_set(x_10, 0, x_3); +lean_closure_set(x_10, 1, x_4); +lean_closure_set(x_10, 2, x_7); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__72___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__8), 3, 2); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_3); +lean_inc(x_2); +x_7 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__66___rarg(x_2, x_6, x_5); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__10___boxed), 4, 3); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__73___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__12(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; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_array_get_size(x_5); +x_7 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_8 = 0; +lean_inc(x_3); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg(x_2, x_3, x_7, x_8, x_5); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__11), 4, 3); +lean_closure_set(x_10, 0, x_4); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_3); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__74___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__6), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__12), 4, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveTermGoal() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__3; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__1___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__3___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__8___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__17___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__1(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__7(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___lambda__8(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__30___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__38___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__40___rarg(x_1, x_5, x_6, x_4); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__45___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__54___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__1(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__7(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___lambda__8(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__67___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__1(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__4(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__7(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoal___lambda__10___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_Widget_instRpcEncodingInteractiveTermGoal___lambda__10(x_1, x_2, x_3, x_4); +lean_dec(x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("⊢ ", 4); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_2 = lean_ctor_get(x_1, 0); +x_3 = lean_ctor_get(x_1, 1); +x_4 = lean_box(0); +x_5 = l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___closed__1; +lean_inc(x_3); +lean_inc(x_2); +x_6 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_6, 0, x_2); +lean_ctor_set(x_6, 1, x_3); +lean_ctor_set(x_6, 2, x_4); +lean_ctor_set(x_6, 3, x_5); +lean_ctor_set(x_6, 4, x_4); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__2(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_array_uget(x_3, x_2); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_3, x_2, x_7); +x_9 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696_(x_6); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +lean_dec(x_8); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; +} +} +else +{ +lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_9, 0); +lean_inc(x_13); +lean_dec(x_9); +x_14 = 1; +x_15 = lean_usize_add(x_2, x_14); +x_16 = lean_array_uset(x_8, x_2, x_13); +x_2 = x_15; +x_3 = x_16; +goto _start; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Json_getObjValD(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +if (lean_obj_tag(x_3) == 4) +{ +lean_object* x_4; lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_array_get_size(x_4); +x_6 = lean_usize_of_nat(x_5); +lean_dec(x_5); +x_7 = 0; +x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__2(x_6, x_7, x_4); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_9 = lean_unsigned_to_nat(80u); +x_10 = l_Lean_Json_pretty(x_3, x_9); +x_11 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1; +x_12 = lean_string_append(x_11, x_10); +lean_dec(x_10); +x_13 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4; +x_14 = lean_string_append(x_12, x_13); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; +} +} +} +static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_from_bytes("goals", 5); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____closed__1; +x_3 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__1(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +else +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_3); +if (x_7 == 0) +{ +return x_3; +} +else +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +lean_dec(x_3); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_8); +return x_9; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____spec__2(x_4, x_5, x_3); +return x_6; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__4() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instFromJsonRpcEncodingPacket__4___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845____spec__1(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_802_(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845_(lean_object* x_1) { +_start: +{ +lean_object* x_2; size_t x_3; size_t x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_2 = lean_array_get_size(x_1); +x_3 = lean_usize_of_nat(x_2); +lean_dec(x_2); +x_4 = 0; +x_5 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845____spec__1(x_3, x_4, x_1); +x_6 = lean_alloc_ctor(4, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____closed__1; +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_6); +x_9 = lean_box(0); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +x_12 = l_List_join___rarg(x_11); +x_13 = l_Lean_Json_mkObj(x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845____spec__1(x_4, x_5, x_3); +return x_6; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1845_), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Widget_instToJsonRpcEncodingPacket__4() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Widget_instToJsonRpcEncodingPacket__4___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__2___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__2___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__4___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__4___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__5___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__5(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__5___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__6(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__6___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__9(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__9___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__9___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__10(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__10___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__11___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__12___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__12(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__12___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__11___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__10___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__12___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__13___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__13(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__13___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__14___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__14(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__14___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__15___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__15(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__15___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__18___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__18(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__18___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__18___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__19___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__19(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__19___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__20___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__20(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__20___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__21___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__21(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__21___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__20___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__19___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__21___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__22___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__22(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__22___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__23___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__23(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__23___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__24___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__24(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__24___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__26___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__26(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__26___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__1(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__5___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__6___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__4___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__13___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__14___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__4), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__15___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__16___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__2), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__7___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__5), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__22___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__7(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__6), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__23___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__8(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg(x_1, x_16, x_17, x_14); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed__const__1; +lean_inc(x_2); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__7___boxed), 5, 4); +lean_closure_set(x_20, 0, x_11); +lean_closure_set(x_20, 1, x_1); +lean_closure_set(x_20, 2, x_19); +lean_closure_set(x_20, 3, x_2); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__24___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +lean_inc(x_21); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_18, x_22); +x_24 = lean_box_usize(x_4); +x_25 = lean_box_usize(x_3); +lean_inc(x_1); +x_26 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__8___boxed), 6, 5); +lean_closure_set(x_26, 0, x_24); +lean_closure_set(x_26, 1, x_13); +lean_closure_set(x_26, 2, x_1); +lean_closure_set(x_26, 3, x_2); +lean_closure_set(x_26, 4, x_25); +x_27 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__26___rarg), 5, 4); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, lean_box(0)); +lean_closure_set(x_27, 2, lean_box(0)); +lean_closure_set(x_27, 3, x_26); +x_28 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_23, x_27); +return x_28; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__27___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__27(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__27___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__28___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__28(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__28___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__31___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__31(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__31___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__31___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__32___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__32(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__32___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__33___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__33(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__33___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__34___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__34(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__34___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__33___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__32___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__34___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__35___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__35(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__35___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__36___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__36(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__36___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__37___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__37(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__37___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__38___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__38(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__38___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__39___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__39(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__39___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__41___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__41(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__41___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__1(lean_object* x_1, lean_object* x_2, size_t x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_box_usize(x_3); +x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__1___boxed), 3, 2); +lean_closure_set(x_10, 0, x_9); +lean_closure_set(x_10, 1, x_6); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__27___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_8, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__28___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 4); +lean_inc(x_5); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__3), 6, 5); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_7); +lean_closure_set(x_9, 4, x_5); +x_10 = lean_ctor_get(x_6, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__35___rarg), 5, 4); +lean_closure_set(x_11, 0, x_6); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_13 = lean_apply_2(x_5, lean_box(0), x_12); +x_14 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_13, x_11); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_8, 0); +lean_inc(x_15); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_inc(x_5); +x_17 = lean_apply_2(x_5, lean_box(0), x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4), 2, 1); +lean_closure_set(x_18, 0, x_5); +lean_inc(x_10); +x_19 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_11); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 3); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_6); +lean_inc(x_8); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__3___boxed), 7, 6); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_3); +lean_closure_set(x_11, 2, x_4); +lean_closure_set(x_11, 3, x_5); +lean_closure_set(x_11, 4, x_8); +lean_closure_set(x_11, 5, x_2); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__36___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__5(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; +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__4), 5, 4); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +lean_closure_set(x_6, 2, x_3); +lean_closure_set(x_6, 3, x_4); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__37___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_14); +lean_inc(x_16); +x_18 = lean_apply_2(x_16, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4), 2, 1); +lean_closure_set(x_19, 0, x_16); +lean_inc(x_7); +x_20 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_20, x_8); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_3); +lean_inc(x_2); +x_7 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__29___rarg(x_2, x_6, x_5); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__5), 4, 3); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__38___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__7(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_2); +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg(x_1, x_2, x_16, x_17, x_14); +lean_inc(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__6), 4, 3); +lean_closure_set(x_19, 0, x_11); +lean_closure_set(x_19, 1, x_1); +lean_closure_set(x_19, 2, x_2); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__39___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +lean_inc(x_20); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_18, x_21); +x_23 = lean_box_usize(x_4); +x_24 = lean_box_usize(x_3); +lean_inc(x_1); +x_25 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__7___boxed), 6, 5); +lean_closure_set(x_25, 0, x_23); +lean_closure_set(x_25, 1, x_13); +lean_closure_set(x_25, 2, x_1); +lean_closure_set(x_25, 3, x_2); +lean_closure_set(x_25, 4, x_24); +x_26 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__41___rarg), 5, 4); +lean_closure_set(x_26, 0, x_1); +lean_closure_set(x_26, 1, lean_box(0)); +lean_closure_set(x_26, 2, lean_box(0)); +lean_closure_set(x_26, 3, x_25); +x_27 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_22, x_26); +return x_27; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__42___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__42(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__42___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__44___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__44(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__44___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__44___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__46___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__46(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__46___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, size_t x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; +x_6 = 1; +x_7 = lean_usize_add(x_1, x_6); +x_8 = lean_array_uset(x_2, x_1, x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg(x_3, x_4, x_7, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_6 = lean_ctor_get(x_1, 0); +lean_inc(x_6); +lean_dec(x_1); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_8, 0, x_4); +x_9 = lean_apply_2(x_7, lean_box(0), x_8); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_10 = lean_array_uget(x_4, x_3); +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_array_uset(x_4, x_3, x_11); +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_10); +x_16 = lean_apply_2(x_14, lean_box(0), x_15); +x_17 = lean_box_usize(x_3); +x_18 = lean_box_usize(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___lambda__1___boxed), 5, 4); +lean_closure_set(x_19, 0, x_17); +lean_closure_set(x_19, 1, x_12); +lean_closure_set(x_19, 2, x_1); +lean_closure_set(x_19, 3, x_18); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__46___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_16, x_21); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__47___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__47(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__47___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__48___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__48(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__48___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__51___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__51(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__51___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__51___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__52___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__52(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__52___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__53___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__53(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__53___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__54___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__54(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__54___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__53___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__52___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__54___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__55___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__55(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__55___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__56___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__56(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__56___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__57___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__57(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__57___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__60___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__60(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__60___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__60___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__61___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__61(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__61___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__62___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__62(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__62___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__63___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__63(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__63___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__62___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__61___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__63___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__64___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__64(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__64___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__65___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__65(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__65___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__66___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__66(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__66___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__68___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__68(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__68___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__47___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__48___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8) { +_start: +{ +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; +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*4 + 1); +x_10 = lean_box(x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_2); +x_12 = lean_apply_2(x_2, lean_box(0), x_11); +x_13 = lean_box(x_8); +x_14 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__15___boxed), 7, 6); +lean_closure_set(x_14, 0, x_3); +lean_closure_set(x_14, 1, x_4); +lean_closure_set(x_14, 2, x_5); +lean_closure_set(x_14, 3, x_6); +lean_closure_set(x_14, 4, x_13); +lean_closure_set(x_14, 5, x_2); +x_15 = lean_ctor_get(x_7, 1); +lean_inc(x_15); +x_16 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__55___rarg), 5, 4); +lean_closure_set(x_16, 0, x_7); +lean_closure_set(x_16, 1, lean_box(0)); +lean_closure_set(x_16, 2, lean_box(0)); +lean_closure_set(x_16, 3, x_14); +x_17 = lean_apply_4(x_15, lean_box(0), lean_box(0), x_12, x_16); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*4); +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_box(x_7); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +lean_inc(x_9); +x_12 = lean_apply_2(x_9, lean_box(0), x_11); +lean_inc(x_2); +x_13 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__3___boxed), 8, 7); +lean_closure_set(x_13, 0, x_1); +lean_closure_set(x_13, 1, x_9); +lean_closure_set(x_13, 2, x_3); +lean_closure_set(x_13, 3, x_4); +lean_closure_set(x_13, 4, x_5); +lean_closure_set(x_13, 5, x_6); +lean_closure_set(x_13, 6, x_2); +x_14 = lean_ctor_get(x_2, 1); +lean_inc(x_14); +x_15 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__56___rarg), 5, 4); +lean_closure_set(x_15, 0, x_2); +lean_closure_set(x_15, 1, lean_box(0)); +lean_closure_set(x_15, 2, lean_box(0)); +lean_closure_set(x_15, 3, x_13); +x_16 = lean_apply_4(x_14, lean_box(0), lean_box(0), x_12, x_15); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_1, 3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__4), 6, 5); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_3); +lean_closure_set(x_8, 3, x_4); +lean_closure_set(x_8, 4, x_6); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__57___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_dec(x_5); +x_11 = lean_ctor_get(x_2, 0); +lean_inc(x_11); +lean_dec(x_2); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +x_15 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_14, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_7, 0); +lean_inc(x_16); +lean_dec(x_7); +lean_inc(x_2); +x_17 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__58___rarg(x_2, x_5, x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__7), 2, 1); +lean_closure_set(x_18, 0, x_2); +lean_inc(x_9); +x_19 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_19, x_10); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_inc(x_2); +x_7 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__2), 3, 2); +lean_closure_set(x_7, 0, x_2); +lean_closure_set(x_7, 1, x_3); +lean_inc(x_7); +lean_inc(x_2); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__49___rarg(x_2, x_7, x_6); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__5), 6, 5); +lean_closure_set(x_9, 0, x_1); +lean_closure_set(x_9, 1, x_2); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_5); +lean_closure_set(x_9, 4, x_7); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__64___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__7(lean_object* x_1, lean_object* x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_6); +x_8 = lean_usize_of_nat(x_7); +lean_dec(x_7); +lean_inc(x_2); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg(x_2, x_8, x_3, x_6); +lean_inc(x_2); +x_10 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__6), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +lean_closure_set(x_10, 2, x_4); +lean_closure_set(x_10, 3, x_5); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); +x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__65___rarg), 5, 4); +lean_closure_set(x_12, 0, x_2); +lean_closure_set(x_12, 1, lean_box(0)); +lean_closure_set(x_12, 2, lean_box(0)); +lean_closure_set(x_12, 3, x_10); +x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__8(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed__const__1() { +_start: +{ +size_t x_1; lean_object* x_2; +x_1 = 0; +x_2 = lean_box_usize(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; lean_inc(x_1); -x_54 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_54, 0, x_1); -lean_ctor_set(x_54, 1, x_53); -x_55 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_55, 0, x_49); -lean_ctor_set(x_55, 1, x_54); -x_56 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_40); -x_57 = 0; -x_58 = lean_alloc_ctor(5, 1, 1); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set_uint8(x_58, sizeof(void*)*1, x_57); -x_59 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_59, 0, x_8); -lean_ctor_set(x_59, 1, x_58); -x_60 = 1; -x_61 = lean_usize_add(x_4, x_60); -x_4 = x_61; -x_5 = x_59; -goto _start; +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg(x_1, x_16, x_17, x_14); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed__const__1; +lean_inc(x_2); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__7___boxed), 5, 4); +lean_closure_set(x_20, 0, x_11); +lean_closure_set(x_20, 1, x_1); +lean_closure_set(x_20, 2, x_19); +lean_closure_set(x_20, 3, x_2); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +lean_inc(x_1); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__66___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +lean_inc(x_21); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_18, x_22); +x_24 = lean_box_usize(x_4); +x_25 = lean_box_usize(x_3); +lean_inc(x_1); +x_26 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__8___boxed), 6, 5); +lean_closure_set(x_26, 0, x_24); +lean_closure_set(x_26, 1, x_13); +lean_closure_set(x_26, 2, x_1); +lean_closure_set(x_26, 3, x_2); +lean_closure_set(x_26, 4, x_25); +x_27 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__68___rarg), 5, 4); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, lean_box(0)); +lean_closure_set(x_27, 2, lean_box(0)); +lean_closure_set(x_27, 3, x_26); +x_28 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_23, x_27); +return x_28; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__69___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__69(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__69___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__70___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__70(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__70___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__73___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } -else +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__73(lean_object* x_1) { +_start: { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; size_t x_76; size_t x_77; -lean_dec(x_15); -x_63 = lean_ctor_get(x_7, 2); -lean_inc(x_63); -lean_dec(x_7); -x_64 = l_Lean_Widget_TaggedText_stripTags___rarg(x_63); -x_65 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_65, 0, x_64); -x_66 = lean_box(1); -x_67 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_65); -lean_inc(x_1); -x_68 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_68, 0, x_1); -lean_ctor_set(x_68, 1, x_67); -x_69 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__10; -x_70 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_68); -x_71 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; -x_72 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -x_73 = 0; -x_74 = lean_alloc_ctor(5, 1, 1); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set_uint8(x_74, sizeof(void*)*1, x_73); -x_75 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_75, 0, x_8); -lean_ctor_set(x_75, 1, x_74); -x_76 = 1; -x_77 = lean_usize_add(x_4, x_76); -x_4 = x_77; -x_5 = x_75; -goto _start; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__73___rarg), 5, 0); +return x_2; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { _start: { uint8_t x_6; x_6 = lean_usize_dec_lt(x_4, x_3); if (x_6 == 0) { +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -return x_5; +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_7 = lean_array_uget(x_2, x_4); -x_8 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(x_5); -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -x_10 = lean_array_to_list(lean_box(0), x_9); -x_11 = lean_box(0); -x_12 = l_List_filterTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__1(x_10, x_11); -x_13 = l_List_mapTRAux___at_Lean_Widget_InteractiveGoal_pretty___spec__2(x_12, x_11); -x_14 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1; -x_15 = l_String_intercalate(x_14, x_13); -x_16 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__2; -x_17 = lean_string_dec_eq(x_15, x_16); -if (x_17 == 0) -{ -lean_object* x_18; -x_18 = lean_ctor_get(x_7, 3); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); lean_inc(x_18); -if (lean_obj_tag(x_18) == 0) +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__73___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72(lean_object* x_1) { +_start: { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; -x_19 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_19, 0, x_15); -x_20 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; -x_21 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -x_22 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__4; -x_23 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -x_24 = lean_ctor_get(x_7, 2); -lean_inc(x_24); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__74___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); lean_dec(x_7); -x_25 = l_Lean_Widget_TaggedText_stripTags___rarg(x_24); -x_26 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_26, 0, x_25); -x_27 = lean_box(1); -x_28 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -lean_inc(x_1); -x_29 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_29, 0, x_1); -lean_ctor_set(x_29, 1, x_28); -x_30 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_30, 0, x_23); -lean_ctor_set(x_30, 1, x_29); -x_31 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_20); -x_32 = 0; -x_33 = lean_alloc_ctor(5, 1, 1); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); -x_34 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_34, 0, x_8); -lean_ctor_set(x_34, 1, x_33); -x_35 = 1; -x_36 = lean_usize_add(x_4, x_35); -x_4 = x_36; -x_5 = x_34; -goto _start; +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; -x_38 = lean_ctor_get(x_18, 0); -lean_inc(x_38); -lean_dec(x_18); -x_39 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_39, 0, x_15); -x_40 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; -x_41 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_39); -x_42 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__6; -x_43 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_ctor_get(x_7, 2); -lean_inc(x_44); -lean_dec(x_7); -x_45 = l_Lean_Widget_TaggedText_stripTags___rarg(x_44); -x_46 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_46, 0, x_45); -x_47 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_47, 0, x_43); -lean_ctor_set(x_47, 1, x_46); -x_48 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__8; -x_49 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); -x_50 = l_Lean_Widget_TaggedText_stripTags___rarg(x_38); -x_51 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_51, 0, x_50); -x_52 = lean_box(1); -x_53 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_51); -lean_inc(x_1); -x_54 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_54, 0, x_1); -lean_ctor_set(x_54, 1, x_53); -x_55 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_55, 0, x_49); -lean_ctor_set(x_55, 1, x_54); -x_56 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_40); -x_57 = 0; -x_58 = lean_alloc_ctor(5, 1, 1); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set_uint8(x_58, sizeof(void*)*1, x_57); -x_59 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_59, 0, x_8); -lean_ctor_set(x_59, 1, x_58); -x_60 = 1; -x_61 = lean_usize_add(x_4, x_60); -x_4 = x_61; -x_5 = x_59; -goto _start; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; size_t x_76; size_t x_77; -lean_dec(x_15); -x_63 = lean_ctor_get(x_7, 2); -lean_inc(x_63); -lean_dec(x_7); -x_64 = l_Lean_Widget_TaggedText_stripTags___rarg(x_63); -x_65 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_65, 0, x_64); -x_66 = lean_box(1); -x_67 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_65); -lean_inc(x_1); -x_68 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_68, 0, x_1); -lean_ctor_set(x_68, 1, x_67); -x_69 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__10; -x_70 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_68); -x_71 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; -x_72 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -x_73 = 0; -x_74 = lean_alloc_ctor(5, 1, 1); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set_uint8(x_74, sizeof(void*)*1, x_73); -x_75 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_75, 0, x_8); -lean_ctor_set(x_75, 1, x_74); -x_76 = 1; -x_77 = lean_usize_add(x_4, x_76); -x_4 = x_77; -x_5 = x_75; -goto _start; -} +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -static lean_object* _init_l_Lean_Widget_InteractiveGoal_pretty___closed__1() { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__74(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(2u); -x_2 = lean_nat_to_int(x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__74___rarg), 5, 0); return x_2; } } -static lean_object* _init_l_Lean_Widget_InteractiveGoal_pretty___closed__2() { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__75___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("case ", 5); -return x_1; +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -static lean_object* _init_l_Lean_Widget_InteractiveGoal_pretty___closed__3() { +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__75(lean_object* x_1) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Widget_InteractiveGoal_pretty___closed__2; -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__75___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveGoal_pretty(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__76___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; size_t x_5; size_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_2 = lean_ctor_get(x_1, 2); -lean_inc(x_2); -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -x_4 = lean_array_get_size(x_3); -x_5 = lean_usize_of_nat(x_4); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; lean_dec(x_4); -x_6 = 0; -x_7 = lean_ctor_get(x_1, 3); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); lean_inc(x_7); -x_8 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_8, 0, x_7); -x_9 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2; -x_10 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_8); -x_11 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_9); -x_12 = lean_ctor_get(x_1, 1); -lean_inc(x_12); lean_dec(x_1); -x_13 = l_Lean_Widget_TaggedText_stripTags___rarg(x_12); -x_14 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = l_Lean_Widget_InteractiveGoal_pretty___closed__1; -x_16 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -x_17 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_17, 0, x_11); -lean_ctor_set(x_17, 1, x_16); -x_18 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_9); -if (lean_obj_tag(x_2) == 0) +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_box(0); -x_20 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3(x_15, x_3, x_5, x_6, x_19); -lean_dec(x_3); -x_21 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(x_20); -x_22 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_18); -return x_22; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_23 = lean_ctor_get(x_2, 0); -lean_inc(x_23); -lean_dec(x_2); -x_24 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_24, 0, x_23); -x_25 = l_Lean_Widget_InteractiveGoal_pretty___closed__3; -x_26 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -x_27 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_9); -x_28 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4(x_15, x_3, x_5, x_6, x_27); -lean_dec(x_3); -x_29 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_InteractiveGoal_addLine(x_28); -x_30 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_18); -return x_30; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__76(lean_object* x_1) { _start: { -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_8 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3(x_1, x_2, x_6, x_7, x_5); -lean_dec(x_2); -return x_8; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__76___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_8 = l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__4(x_1, x_2, x_6, x_7, x_5); -lean_dec(x_2); -return x_8; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__75___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; } } -static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(0u); -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__2() { -_start: +case 1: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__1; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___spec__7___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__74___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__76___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg), 3, 0); return x_2; } } -static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__3() { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__77___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__1; -x_2 = l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__3; -x_3 = l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__2; -x_4 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_2); -lean_ctor_set(x_4, 2, x_3); -return x_4; +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -static lean_object* _init_l_Lean_Widget_instInhabitedInteractiveTermGoal() { -_start: +else { -lean_object* x_1; -x_1 = l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__3; -return x_1; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___closed__1() { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__77(lean_object* x_1) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("range", 5); -return x_1; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__77___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__78___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_5; lean_object* x_6; -x_5 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1; -x_6 = l_Lean_Json_getObjValAs_x3f(x_4, lean_box(0), x_1, x_5); -if (lean_obj_tag(x_6) == 0) -{ -uint8_t x_7; -lean_dec(x_3); -lean_dec(x_2); -x_7 = !lean_is_exclusive(x_6); -if (x_7 == 0) +if (lean_obj_tag(x_5) == 0) { -return x_6; -} -else +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) { -lean_object* x_8; lean_object* x_9; -x_8 = lean_ctor_get(x_6, 0); +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); -lean_dec(x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); return x_9; } -} else { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_6, 0); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); lean_inc(x_10); -lean_dec(x_6); -x_11 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3; -x_12 = l_Lean_Json_getObjValAs_x3f(x_4, lean_box(0), x_2, x_11); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_13; -lean_dec(x_10); -lean_dec(x_3); -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) -{ -return x_12; +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} } else { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_12, 0); -lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_12, 0); -lean_inc(x_16); -lean_dec(x_12); -x_17 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___closed__1; -x_18 = l_Lean_Json_getObjValAs_x3f(x_4, lean_box(0), x_3, x_17); -if (lean_obj_tag(x_18) == 0) -{ -uint8_t x_19; -lean_dec(x_16); -lean_dec(x_10); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) -{ -return x_18; } -else +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__78(lean_object* x_1) { +_start: { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_18, 0); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_21, 0, x_20); -return x_21; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__78___rarg), 5, 0); +return x_2; } } -else +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__79___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_18); -if (x_22 == 0) +if (lean_obj_tag(x_5) == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_18, 0); -x_24 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_24, 0, x_10); -lean_ctor_set(x_24, 1, x_16); -lean_ctor_set(x_24, 2, x_23); -lean_ctor_set(x_18, 0, x_24); -return x_18; +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_18, 0); -lean_inc(x_25); -lean_dec(x_18); -x_26 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_26, 0, x_10); -lean_ctor_set(x_26, 1, x_16); -lean_ctor_set(x_26, 2, x_25); -x_27 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_27, 0, x_26); -return x_27; -} +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__79(lean_object* x_1) { _start: { -lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___boxed), 4, 0); -return x_4; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__79___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__80___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_5; -x_5 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg(x_1, x_2, x_3, x_4); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; lean_dec(x_4); -return x_5; +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +} +else { -lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___boxed), 4, 3); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_2); -lean_closure_set(x_4, 2, x_3); -return x_4; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__80(lean_object* x_1) { _start: -{ -lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__3___rarg), 3, 0); -return x_4; +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__80___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2236____rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__81___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; 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; -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -x_6 = lean_apply_1(x_1, x_5); -x_7 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1; -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -x_9 = lean_box(0); -x_10 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_ctor_get(x_4, 1); -lean_inc(x_11); -x_12 = lean_apply_1(x_2, x_11); -x_13 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3; -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -x_15 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_9); -x_16 = lean_ctor_get(x_4, 2); -lean_inc(x_16); +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; lean_dec(x_4); -x_17 = lean_apply_1(x_3, x_16); -x_18 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___closed__1; -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_9); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_9); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_15); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_10); -lean_ctor_set(x_23, 1, x_22); -x_24 = l_List_join___rarg(x_23); -x_25 = l_Lean_Json_mkObj(x_24); -return x_25; -} +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2236_(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2236____rarg), 4, 0); -return x_4; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2236____rarg), 4, 3); -lean_closure_set(x_4, 0, x_1); -lean_closure_set(x_4, 1, x_2); -lean_closure_set(x_4, 2, x_3); -return x_4; +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__81(lean_object* x_1) { _start: { -lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__3___rarg), 3, 0); -return x_4; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__81___rarg), 5, 0); +return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__83___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -4168,15 +28515,325 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__83(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__83___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +lean_inc(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_4); +lean_inc(x_6); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__12), 3, 2); +lean_closure_set(x_9, 0, x_3); +lean_closure_set(x_9, 1, x_6); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__69___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_4 = l_Lean_Widget_instRpcEncodingWithRpcRefInfoWithCtxRpcRef; +x_5 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_inc(x_1); +x_7 = lean_apply_4(x_5, lean_box(0), x_1, x_2, x_6); +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__1___boxed), 3, 2); +lean_closure_set(x_8, 0, x_3); +lean_closure_set(x_8, 1, x_1); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__70___rarg), 5, 4); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_8 = lean_ctor_get(x_1, 4); +lean_inc(x_5); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__12), 6, 5); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 2, x_4); +lean_closure_set(x_9, 3, x_7); +lean_closure_set(x_9, 4, x_5); +x_10 = lean_ctor_get(x_6, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__77___rarg), 5, 4); +lean_closure_set(x_11, 0, x_6); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_13 = lean_apply_2(x_5, lean_box(0), x_12); +x_14 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_13, x_11); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_8, 0); +lean_inc(x_15); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +lean_inc(x_5); +x_17 = lean_apply_2(x_5, lean_box(0), x_16); +x_18 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4), 2, 1); +lean_closure_set(x_18, 0, x_5); +lean_inc(x_10); +x_19 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_17, x_18); +x_20 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_19, x_11); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_6 = lean_ctor_get(x_1, 3); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_6); +lean_inc(x_8); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +lean_inc(x_2); +x_11 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__3___boxed), 7, 6); +lean_closure_set(x_11, 0, x_1); +lean_closure_set(x_11, 1, x_3); +lean_closure_set(x_11, 2, x_4); +lean_closure_set(x_11, 3, x_5); +lean_closure_set(x_11, 4, x_8); +lean_closure_set(x_11, 5, x_2); +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); +x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__78___rarg), 5, 4); +lean_closure_set(x_13, 0, x_2); +lean_closure_set(x_13, 1, lean_box(0)); +lean_closure_set(x_13, 2, lean_box(0)); +lean_closure_set(x_13, 3, x_11); +x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__5(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; +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__4), 5, 4); +lean_closure_set(x_6, 0, x_1); +lean_closure_set(x_6, 1, x_2); +lean_closure_set(x_6, 2, x_3); +lean_closure_set(x_6, 3, x_4); +x_7 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__79___rarg), 5, 4); +lean_closure_set(x_8, 0, x_2); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_ctor_get(x_9, 1); +lean_inc(x_10); +lean_dec(x_9); +x_11 = l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1; +x_12 = lean_apply_2(x_10, lean_box(0), x_11); +x_13 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_12, x_8); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); +lean_dec(x_5); +x_15 = lean_ctor_get(x_2, 0); +lean_inc(x_15); +lean_dec(x_2); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_14); +lean_inc(x_16); +x_18 = lean_apply_2(x_16, lean_box(0), x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoal___lambda__4), 2, 1); +lean_closure_set(x_19, 0, x_16); +lean_inc(x_7); +x_20 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_18, x_19); +x_21 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_20, x_8); +return x_21; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +lean_inc(x_2); +x_6 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_2); +lean_closure_set(x_6, 1, x_3); +lean_inc(x_2); +x_7 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__71___rarg(x_2, x_6, x_5); +lean_inc(x_2); +x_8 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__5), 4, 3); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, x_2); +lean_closure_set(x_8, 2, x_4); +x_9 = lean_ctor_get(x_2, 1); +lean_inc(x_9); +x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__80___rarg), 5, 4); +lean_closure_set(x_10, 0, x_2); +lean_closure_set(x_10, 1, lean_box(0)); +lean_closure_set(x_10, 2, lean_box(0)); +lean_closure_set(x_10, 3, x_8); +x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__7(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_array_get_size(x_14); +x_16 = lean_usize_of_nat(x_15); +lean_dec(x_15); +x_17 = 0; +lean_inc(x_2); +lean_inc(x_1); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg(x_1, x_2, x_16, x_17, x_14); +lean_inc(x_2); +lean_inc(x_1); +x_19 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__6), 4, 3); +lean_closure_set(x_19, 0, x_11); +lean_closure_set(x_19, 1, x_1); +lean_closure_set(x_19, 2, x_2); +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__81___rarg), 5, 4); +lean_closure_set(x_21, 0, x_1); +lean_closure_set(x_21, 1, lean_box(0)); +lean_closure_set(x_21, 2, lean_box(0)); +lean_closure_set(x_21, 3, x_19); +lean_inc(x_20); +x_22 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_18, x_21); +x_23 = lean_box_usize(x_4); +x_24 = lean_box_usize(x_3); +lean_inc(x_1); +x_25 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__7___boxed), 6, 5); +lean_closure_set(x_25, 0, x_23); +lean_closure_set(x_25, 1, x_13); +lean_closure_set(x_25, 2, x_1); +lean_closure_set(x_25, 3, x_2); +lean_closure_set(x_25, 4, x_24); +x_26 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__83___rarg), 5, 4); +lean_closure_set(x_26, 0, x_1); +lean_closure_set(x_26, 1, lean_box(0)); +lean_closure_set(x_26, 2, lean_box(0)); +lean_closure_set(x_26, 3, x_25); +x_27 = lean_apply_4(x_20, lean_box(0), lean_box(0), x_22, x_26); +return x_27; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__1___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___boxed), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__84___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { if (lean_obj_tag(x_5) == 0) @@ -4226,616 +28883,548 @@ return x_16; } } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__2(lean_object* x_1) { +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__84(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__2___rarg), 5, 0); +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__84___rarg), 5, 0); return x_2; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { -if (lean_obj_tag(x_5) == 0) -{ -uint8_t x_6; -lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +x_4 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_2); +x_6 = lean_apply_2(x_4, lean_box(0), x_5); +return x_6; } -else +} +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); +lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_5 = lean_array_get_size(x_4); +x_6 = lean_usize_of_nat(x_5); lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +x_7 = 0; +lean_inc(x_2); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg(x_2, x_3, x_6, x_7, x_4); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__1), 2, 1); +lean_closure_set(x_9, 0, x_2); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__42___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; } } -else +LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_15; lean_object* x_16; -lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); +lean_object* x_5; size_t x_6; size_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_5 = lean_array_get_size(x_4); +x_6 = lean_usize_of_nat(x_5); lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; -} +x_7 = 0; +lean_inc(x_2); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg(x_2, x_3, x_6, x_7, x_4); +lean_inc(x_2); +x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__1), 2, 1); +lean_closure_set(x_9, 0, x_2); +x_10 = lean_ctor_get(x_2, 1); +lean_inc(x_10); +x_11 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__84___rarg), 5, 4); +lean_closure_set(x_11, 0, x_2); +lean_closure_set(x_11, 1, lean_box(0)); +lean_closure_set(x_11, 2, lean_box(0)); +lean_closure_set(x_11, 3, x_9); +x_12 = lean_apply_4(x_10, lean_box(0), lean_box(0), x_8, x_11); +return x_12; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__3(lean_object* x_1) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__1() { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__3___rarg), 5, 0); -return x_2; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__2), 4, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__2() { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_ctor_get(x_1, 0); -lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -x_7 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_7, 0, x_2); -lean_ctor_set(x_7, 1, x_3); -lean_ctor_set(x_7, 2, x_4); -x_8 = lean_apply_2(x_6, lean_box(0), x_7); -return x_8; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoals___lambda__3), 4, 0); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__3() { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_2, 2); -lean_inc(x_9); -lean_dec(x_2); -lean_inc(x_3); -x_10 = lean_apply_4(x_8, lean_box(0), x_3, x_4, x_9); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__1), 4, 3); -lean_closure_set(x_11, 0, x_3); -lean_closure_set(x_11, 1, x_5); -lean_closure_set(x_11, 2, x_7); -x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); -return x_12; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__1; +x_2 = l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +static lean_object* _init_l_Lean_Widget_instRpcEncodingInteractiveGoals() { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = lean_ctor_get(x_2, 1); -lean_inc(x_9); -lean_inc(x_4); -lean_inc(x_3); -x_10 = lean_apply_4(x_8, lean_box(0), x_3, x_4, x_9); -lean_inc(x_6); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__2), 7, 6); -lean_closure_set(x_11, 0, x_5); -lean_closure_set(x_11, 1, x_2); -lean_closure_set(x_11, 2, x_3); -lean_closure_set(x_11, 3, x_4); -lean_closure_set(x_11, 4, x_7); -lean_closure_set(x_11, 5, x_6); -x_12 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_10, x_11); -return x_12; +lean_object* x_1; +x_1 = l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__3; +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_5, 1); -lean_inc(x_8); -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); lean_dec(x_1); -x_10 = lean_ctor_get(x_7, 0); -lean_inc(x_10); -lean_inc(x_6); -lean_inc(x_5); -x_11 = lean_apply_4(x_9, lean_box(0), x_5, x_6, x_10); -lean_inc(x_8); -x_12 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__3), 7, 6); -lean_closure_set(x_12, 0, x_2); -lean_closure_set(x_12, 1, x_7); -lean_closure_set(x_12, 2, x_5); -lean_closure_set(x_12, 3, x_6); -lean_closure_set(x_12, 4, x_3); -lean_closure_set(x_12, 5, x_8); -x_13 = lean_apply_4(x_8, lean_box(0), lean_box(0), x_11, x_12); -return x_13; +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg___boxed(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; -x_5 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_4); -x_6 = lean_ctor_get(x_3, 0); -lean_inc(x_6); +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_8, 0, x_5); -x_9 = lean_apply_2(x_7, lean_box(0), x_8); -return x_9; +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__1___rarg(x_1, x_5, x_6, x_4); +return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); lean_dec(x_1); -x_8 = lean_ctor_get(x_2, 2); -lean_inc(x_8); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -lean_inc(x_3); -x_9 = lean_apply_4(x_7, lean_box(0), x_3, x_4, x_8); -lean_inc(x_3); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__5), 4, 3); -lean_closure_set(x_10, 0, x_5); -lean_closure_set(x_10, 1, x_6); -lean_closure_set(x_10, 2, x_3); -x_11 = lean_ctor_get(x_3, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_12, 0, x_3); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); -return x_13; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__3___rarg(x_1, x_5, x_6, x_4); +return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); lean_dec(x_1); -x_8 = lean_ctor_get(x_2, 1); -lean_inc(x_8); -lean_inc(x_4); -lean_inc(x_3); -x_9 = lean_apply_4(x_7, lean_box(0), x_3, x_4, x_8); -lean_inc(x_3); -x_10 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__6), 6, 5); -lean_closure_set(x_10, 0, x_5); -lean_closure_set(x_10, 1, x_2); -lean_closure_set(x_10, 2, x_3); -lean_closure_set(x_10, 3, x_4); -lean_closure_set(x_10, 4, x_6); -x_11 = lean_ctor_get(x_3, 1); -lean_inc(x_11); -x_12 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__2___rarg), 5, 4); -lean_closure_set(x_12, 0, x_3); -lean_closure_set(x_12, 1, lean_box(0)); -lean_closure_set(x_12, 2, lean_box(0)); -lean_closure_set(x_12, 3, x_10); -x_13 = lean_apply_4(x_11, lean_box(0), lean_box(0), x_9, x_12); -return x_13; +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_8 = lean_ctor_get(x_1, 1); -lean_inc(x_8); +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__8___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); lean_dec(x_1); -x_9 = lean_ctor_get(x_7, 0); -lean_inc(x_9); -lean_inc(x_6); -lean_inc(x_5); -x_10 = lean_apply_4(x_8, lean_box(0), x_5, x_6, x_9); -lean_inc(x_5); -x_11 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__7), 6, 5); -lean_closure_set(x_11, 0, x_2); -lean_closure_set(x_11, 1, x_7); -lean_closure_set(x_11, 2, x_5); -lean_closure_set(x_11, 3, x_6); -lean_closure_set(x_11, 4, x_3); -x_12 = lean_ctor_get(x_5, 1); -lean_inc(x_12); -x_13 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___spec__3___rarg), 5, 4); -lean_closure_set(x_13, 0, x_5); -lean_closure_set(x_13, 1, lean_box(0)); -lean_closure_set(x_13, 2, lean_box(0)); -lean_closure_set(x_13, 3, x_11); -x_14 = lean_apply_4(x_12, lean_box(0), lean_box(0), x_10, x_13); -return x_14; +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; -lean_inc(x_5); -lean_inc(x_3); -lean_inc(x_1); -x_6 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__4), 7, 3); -lean_closure_set(x_6, 0, x_1); -lean_closure_set(x_6, 1, x_3); -lean_closure_set(x_6, 2, x_5); -x_7 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg___lambda__8), 7, 3); -lean_closure_set(x_7, 0, x_1); -lean_closure_set(x_7, 1, x_3); -lean_closure_set(x_7, 2, x_5); -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_6); -lean_ctor_set(x_8, 1, x_7); +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__17___rarg(x_1, x_2, x_6, x_7, x_5); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveTermGoalRpcEncodingPacket___rarg), 5, 0); -return x_2; +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__1(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; } } -static lean_object* _init_l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___closed__1() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("⊢ ", 4); -return x_1; +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); +lean_dec(x_1); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = lean_ctor_get(x_1, 0); -x_3 = lean_ctor_get(x_1, 1); -x_4 = lean_box(0); -x_5 = l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___closed__1; -lean_inc(x_3); -lean_inc(x_2); -x_6 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_6, 0, x_2); -lean_ctor_set(x_6, 1, x_3); -lean_ctor_set(x_6, 2, x_4); -lean_ctor_set(x_6, 3, x_5); -lean_ctor_set(x_6, 4, x_4); -return x_6; +{ +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__7(x_1, x_2, x_6, x_4, x_5); +return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_2; -x_2 = l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal(x_1); +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); lean_dec(x_1); -return x_2; +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___lambda__8(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -static lean_object* _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___closed__1() { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_from_bytes("goals", 5); -return x_1; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_3; lean_object* x_4; -x_3 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___closed__1; -x_4 = l_Lean_Json_getObjValAs_x3f(x_2, lean_box(0), x_1, x_3); -if (lean_obj_tag(x_4) == 0) -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_4); -if (x_5 == 0) -{ -return x_4; +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } -else +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -lean_object* x_6; lean_object* x_7; -x_6 = lean_ctor_get(x_4, 0); -lean_inc(x_6); +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); lean_dec(x_4); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__30___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; } } -else -{ -uint8_t x_8; -x_8 = !lean_is_exclusive(x_4); -if (x_8 == 0) +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -return x_4; +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_5 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__1(x_1, x_2, x_4); +lean_dec(x_1); +return x_5; } -else +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_4, 0); -lean_inc(x_9); -lean_dec(x_4); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +lean_object* x_8; +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_8; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___lambda__7(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___boxed), 2, 0); -return x_2; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__40___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_3; -x_3 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg(x_1, x_2); -lean_dec(x_2); -return x_3; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__4___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___boxed), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__43___rarg(x_1, x_5, x_6, x_4); +return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonRpcEncodingPacket__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instFromJsonRpcEncodingPacket__4___rarg), 1, 0); -return x_2; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___lambda__1(x_6, x_2, x_3, x_7, x_5); +return x_8; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2648____rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_3 = lean_apply_1(x_1, x_2); -x_4 = l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___closed__1; -x_5 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_5, 0, x_4); -lean_ctor_set(x_5, 1, x_3); -x_6 = lean_box(0); -x_7 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_7, 0, x_5); -lean_ctor_set(x_7, 1, x_6); -x_8 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -x_9 = l_List_join___rarg(x_8); -x_10 = l_Lean_Json_mkObj(x_9); -return x_10; +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__45___rarg(x_1, x_5, x_6, x_4); +return x_7; } } -LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2648_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2648____rarg), 2, 0); -return x_2; +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__4___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2648____rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__50___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instToJsonRpcEncodingPacket__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instToJsonRpcEncodingPacket__4___rarg), 1, 0); -return x_2; +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -if (lean_obj_tag(x_5) == 0) -{ -uint8_t x_6; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); lean_dec(x_4); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__59___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); +lean_object* x_4; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__1(x_1, x_2, x_3); lean_dec(x_1); -x_8 = lean_ctor_get(x_7, 1); -lean_inc(x_8); -lean_dec(x_7); -x_9 = lean_apply_2(x_8, lean_box(0), x_5); -return x_9; +return x_4; } -else +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = lean_ctor_get(x_5, 0); -lean_inc(x_10); -lean_dec(x_5); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_8); +lean_dec(x_8); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_9); lean_dec(x_1); -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_10); -x_14 = lean_apply_2(x_12, lean_box(0), x_13); -return x_14; +return x_10; } } -else +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -lean_object* x_15; lean_object* x_16; +size_t x_6; lean_object* x_7; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__7(x_1, x_2, x_6, x_4, x_5); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); lean_dec(x_1); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); +x_8 = lean_unbox_usize(x_5); lean_dec(x_5); -x_16 = lean_apply_1(x_4, x_15); -return x_16; -} +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___lambda__8(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___spec__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___spec__1___rarg), 5, 0); -return x_2; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_apply_2(x_4, lean_box(0), x_2); -return x_5; +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_6 = lean_ctor_get(x_3, 1); -lean_inc(x_6); -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -lean_dec(x_1); -lean_inc(x_3); -x_8 = lean_apply_4(x_7, lean_box(0), x_3, x_4, x_5); -x_9 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__1), 2, 1); -lean_closure_set(x_9, 0, x_3); -x_10 = lean_apply_4(x_6, lean_box(0), lean_box(0), x_8, x_9); -return x_10; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__72___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); +lean_object* x_4; +x_4 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__1(x_1, x_2, x_3); lean_dec(x_1); -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -lean_dec(x_3); -x_5 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_5, 0, x_2); -x_6 = lean_apply_2(x_4, lean_box(0), x_5); -return x_6; +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); +lean_object* x_8; +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_1); -lean_inc(x_3); -x_7 = lean_apply_4(x_6, lean_box(0), x_3, x_4, x_5); -lean_inc(x_3); -x_8 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__3), 2, 1); -lean_closure_set(x_8, 0, x_3); -x_9 = lean_ctor_get(x_3, 1); -lean_inc(x_9); -x_10 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___spec__1___rarg), 5, 4); -lean_closure_set(x_10, 0, x_3); -lean_closure_set(x_10, 1, lean_box(0)); -lean_closure_set(x_10, 2, lean_box(0)); -lean_closure_set(x_10, 3, x_8); -x_11 = lean_apply_4(x_9, lean_box(0), lean_box(0), x_7, x_10); -return x_11; +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -lean_inc(x_1); -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__2), 5, 1); -lean_closure_set(x_2, 0, x_1); -x_3 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg___lambda__4), 5, 1); -lean_closure_set(x_3, 0, x_1); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_3); -return x_4; +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___lambda__7(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Widget_instRpcEncodingInteractiveGoalsRpcEncodingPacket___rarg), 1, 0); -return x_2; +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__82___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; } } LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_addInteractiveHypothesisBundle___spec__1(size_t x_1, size_t x_2, lean_object* x_3) { @@ -8680,36 +33269,110 @@ l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__4 = _init_l_Lea lean_mark_persistent(l_Lean_Widget_instInhabitedInteractiveHypothesisBundle___closed__4); l_Lean_Widget_instInhabitedInteractiveHypothesisBundle = _init_l_Lean_Widget_instInhabitedInteractiveHypothesisBundle(); lean_mark_persistent(l_Lean_Widget_instInhabitedInteractiveHypothesisBundle); -l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1 = _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1(); -lean_mark_persistent(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____spec__1___rarg___closed__1); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__1); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__2 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__2(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__2); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__3); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__4 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__4(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__4); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__5 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__5(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__5); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__6 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__6(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_199____rarg___closed__6); -l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5___closed__1 = _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundleRpcEncodingPacket___rarg___lambda__5___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__2); +l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__3); +l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__2___closed__4); +l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1 = _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1(); +lean_mark_persistent(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__1___closed__1); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__1 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__1); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__2 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__1___closed__2); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__1 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__1); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__2); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__3 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__3); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__4 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__4(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__4); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__5 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__5(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__5); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__2___closed__6); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___closed__1 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___lambda__3___closed__1); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___closed__1 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__6___closed__1); +l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1 = _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1(); +lean_mark_persistent(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____spec__8___closed__1); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__1 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__1); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__2 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__2(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__2); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__3); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__4 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__4(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__4); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__5 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__5(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__5); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__6 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__6(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_136____closed__6); +l_Lean_Widget_instFromJsonRpcEncodingPacket__1___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__1___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__1___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__1); +l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3___closed__1 = _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3___closed__1(); +lean_mark_persistent(l___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_toJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_259____spec__3___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__1___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__1___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__1___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__1); +l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11___boxed__const__1 = _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11___boxed__const__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__11___boxed__const__1); +l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21___boxed__const__1 = _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21___boxed__const__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___lambda__21___boxed__const__1); +l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__1 = _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__1); +l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__2 = _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__2); +l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__3 = _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle___closed__3); +l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle = _init_l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveHypothesisBundle); l_Lean_Widget_InteractiveGoal_mvarId_x3f___default = _init_l_Lean_Widget_InteractiveGoal_mvarId_x3f___default(); lean_mark_persistent(l_Lean_Widget_InteractiveGoal_mvarId_x3f___default); l_Lean_Widget_instInhabitedInteractiveGoal___closed__1 = _init_l_Lean_Widget_instInhabitedInteractiveGoal___closed__1(); lean_mark_persistent(l_Lean_Widget_instInhabitedInteractiveGoal___closed__1); l_Lean_Widget_instInhabitedInteractiveGoal = _init_l_Lean_Widget_instInhabitedInteractiveGoal(); lean_mark_persistent(l_Lean_Widget_instInhabitedInteractiveGoal); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__1); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__2 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__2(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__2); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__3 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__3(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__3); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__4 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__4(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1041____rarg___closed__4); +l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__1 = _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__1(); +lean_mark_persistent(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__1); +l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__2 = _init_l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__2(); +lean_mark_persistent(l_Lean_Json_getObjValAs_x3f___at___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____spec__3___closed__2); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__1); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__2 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__2(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__2); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__3 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__3(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__3); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__4 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__4(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_696____closed__4); +l_Lean_Widget_instFromJsonRpcEncodingPacket__2___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__2___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__2___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__2 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__2(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__2); +l_Lean_Widget_instToJsonRpcEncodingPacket__2___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__2___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__2___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__2 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__2(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__2); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed__const__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__25___rarg___boxed__const__1); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed__const__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoal___spec__64___rarg___boxed__const__1); +l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__1 = _init_l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__1); +l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__2 = _init_l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__2); +l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__3 = _init_l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveGoal___closed__3); +l_Lean_Widget_instRpcEncodingInteractiveGoal = _init_l_Lean_Widget_instRpcEncodingInteractiveGoal(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveGoal); l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1 = _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1(); lean_mark_persistent(l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__1); l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2 = _init_l_Array_forInUnsafe_loop___at_Lean_Widget_InteractiveGoal_pretty___spec__3___closed__2(); @@ -8744,12 +33407,52 @@ l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__3 = _init_l_Lean_Widget lean_mark_persistent(l_Lean_Widget_instInhabitedInteractiveTermGoal___closed__3); l_Lean_Widget_instInhabitedInteractiveTermGoal = _init_l_Lean_Widget_instInhabitedInteractiveTermGoal(); lean_mark_persistent(l_Lean_Widget_instInhabitedInteractiveTermGoal); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2096____rarg___closed__1); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491____closed__1 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491____closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1491____closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__3___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__3___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__3___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__3 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__3(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__3); +l_Lean_Widget_instToJsonRpcEncodingPacket__3___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__3___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__3___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__3 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__3(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__3); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed__const__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__25___rarg___boxed__const__1); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed__const__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveTermGoal___spec__62___rarg___boxed__const__1); +l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__1 = _init_l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__1); +l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__2 = _init_l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__2); +l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__3 = _init_l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveTermGoal___closed__3); +l_Lean_Widget_instRpcEncodingInteractiveTermGoal = _init_l_Lean_Widget_instRpcEncodingInteractiveTermGoal(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveTermGoal); l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___closed__1 = _init_l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___closed__1(); lean_mark_persistent(l_Lean_Widget_InteractiveTermGoal_toInteractiveGoal___closed__1); -l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___closed__1 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_2586____rarg___closed__1); +l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____closed__1 = _init_l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____closed__1(); +lean_mark_persistent(l___private_Lean_Widget_InteractiveGoal_0__Lean_Widget_fromJsonRpcEncodingPacket____x40_Lean_Widget_InteractiveGoal___hyg_1807____closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__4___closed__1 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__4___closed__1(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__4___closed__1); +l_Lean_Widget_instFromJsonRpcEncodingPacket__4 = _init_l_Lean_Widget_instFromJsonRpcEncodingPacket__4(); +lean_mark_persistent(l_Lean_Widget_instFromJsonRpcEncodingPacket__4); +l_Lean_Widget_instToJsonRpcEncodingPacket__4___closed__1 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__4___closed__1(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__4___closed__1); +l_Lean_Widget_instToJsonRpcEncodingPacket__4 = _init_l_Lean_Widget_instToJsonRpcEncodingPacket__4(); +lean_mark_persistent(l_Lean_Widget_instToJsonRpcEncodingPacket__4); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed__const__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__25___rarg___boxed__const__1); +l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed__const__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed__const__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodingInteractiveGoals___spec__67___rarg___boxed__const__1); +l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__1 = _init_l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__1(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__1); +l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__2 = _init_l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__2(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__2); +l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__3 = _init_l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__3(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveGoals___closed__3); +l_Lean_Widget_instRpcEncodingInteractiveGoals = _init_l_Lean_Widget_instRpcEncodingInteractiveGoals(); +lean_mark_persistent(l_Lean_Widget_instRpcEncodingInteractiveGoals); l_Lean_Widget_addInteractiveHypothesisBundle___closed__1 = _init_l_Lean_Widget_addInteractiveHypothesisBundle___closed__1(); lean_mark_persistent(l_Lean_Widget_addInteractiveHypothesisBundle___closed__1); l_Lean_Widget_addInteractiveHypothesisBundle___closed__2 = _init_l_Lean_Widget_addInteractiveHypothesisBundle___closed__2(); diff --git a/stage0/stdlib/Lean/Widget/TaggedText.c b/stage0/stdlib/Lean/Widget/TaggedText.c index 0a9e0ef69e69..19394c909281 100644 --- a/stage0/stdlib/Lean/Widget/TaggedText.c +++ b/stage0/stdlib/Lean/Widget/TaggedText.c @@ -47,6 +47,7 @@ LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_stripTags_go___rarg(lean_objec static lean_object* l_panic___at_Lean_Widget_TaggedText_prettyTagged___spec__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_TaggedText_instInhabitedTaggedState___closed__1; LEAN_EXPORT lean_object* l_Std_Format_prettyM___at_Lean_Widget_TaggedText_prettyTagged___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Format_Basic_0__Std_Format_pushGroup___at_Lean_Widget_TaggedText_prettyTagged___spec__3(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); @@ -65,9 +66,11 @@ static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTa LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_rewrite___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__1___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__11; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8(lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Data_Format_Basic_0__Std_Format_spaceUptoLine_x27(lean_object*, lean_object*); static lean_object* l_Lean_Widget_TaggedText_instMonadPrettyFormatStateMTaggedState___closed__1; LEAN_EXPORT lean_object* l_panic___at_Lean_Widget_TaggedText_prettyTagged___spec__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____spec__2___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Widget_TaggedText_prettyTagged___spec__4___closed__1; lean_object* l_Lean_Json_getStr_x3f(lean_object*); @@ -110,9 +113,11 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_rewr lean_object* lean_nat_sub(lean_object*, lean_object*); uint8_t l___private_Init_Data_Format_Basic_0__Std_Format_beqFlattenBehavior____x40_Init_Data_Format_Basic___hyg_18_(uint8_t, uint8_t); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____rarg___lambda__2___closed__6; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__10___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_rewrite___rarg(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Json_setObjVal_x21___spec__1(lean_object*); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____rarg___lambda__2___closed__4; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__12(lean_object*); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__21; lean_object* l_instInhabited___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__23; @@ -125,6 +130,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_inst lean_object* lean_array_to_list(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__2; static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__1; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__9(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_TaggedText_TaggedState_out___default; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instFromJsonTaggedText(lean_object*); @@ -136,7 +142,9 @@ lean_object* l_Array_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instBEqTaggedText___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_mapM___spec__1___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_stripTags_go(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_TaggedText_instMonadPrettyFormatStateMTaggedState___closed__3; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__11(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_TaggedText_0__Lean_Widget_toJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_594____spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__25; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__2(lean_object*, lean_object*, lean_object*); @@ -154,6 +162,7 @@ lean_object* l_Int_toNat(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Lean_Widget_TaggedText_instMonadPrettyFormatStateMTaggedState___spec__3(lean_object*, lean_object*); static lean_object* l_Lean_Widget_TaggedText_instMonadPrettyFormatStateMTaggedState___closed__5; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_rewriteM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__10(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____spec__1(lean_object*); lean_object* l_List_drop___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_beqTaggedText____x40_Lean_Widget_TaggedText___hyg_76_(lean_object*); @@ -187,6 +196,8 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_Tagge LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____spec__3(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_rewrite___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_rewrite___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__12___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_rewriteM(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____spec__3___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__1___rarg___lambda__2(lean_object*, lean_object*, lean_object*); @@ -194,6 +205,7 @@ LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___rarg___lambda__3(lean_o lean_object* l_Lean_Json_mkObj(lean_object*); lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_map___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Format_Basic_0__Std_Format_pushGroup___at_Lean_Widget_TaggedText_prettyTagged___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_instRpcEncodingTaggedText___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -201,6 +213,7 @@ static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTagged static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__24; lean_object* lean_panic_fn(lean_object*, lean_object*); lean_object* l_StateT_instMonadStateT___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_Widget_TaggedText_instMonadPrettyFormatStateMTaggedState___spec__2___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_array_pop(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__2___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -218,12 +231,15 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_Tagge lean_object* l_List_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateT_bind___at_Lean_Widget_TaggedText_instMonadPrettyFormatStateMTaggedState___spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__10; +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_reprTaggedText____x40_Lean_Widget_TaggedText___hyg_223____rarg___closed__20; static lean_object* l_Lean_Widget_instInhabitedTaggedText___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_instRpcEncodingTaggedText(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__11___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instInhabitedTaggedText(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_map___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_instReprTaggedText___rarg(lean_object*); LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_appendText___rarg(lean_object*, lean_object*); @@ -1344,7 +1360,7 @@ static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_from 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_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____rarg___lambda__2___closed__3; x_2 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____rarg___lambda__2___closed__4; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l___private_Lean_Widget_TaggedText_0__Lean_Widget_fromJsonTaggedText____x40_Lean_Widget_TaggedText___hyg_398____rarg___lambda__2___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4010,6 +4026,432 @@ x_4 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_ return x_4; } } +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__9___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__9(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__9___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___lambda__1(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_add(x_1, x_7); +x_9 = lean_array_uset(x_2, x_1, x_6); +x_10 = l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg(x_3, x_4, x_5, x_8, x_9); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_lt(x_4, x_3); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +x_10 = lean_apply_2(x_8, lean_box(0), x_9); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_11 = lean_array_uget(x_5, x_4); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_5, x_4, x_12); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg(x_1, x_2, x_11); +x_15 = lean_box_usize(x_4); +x_16 = lean_box_usize(x_3); +lean_inc(x_1); +x_17 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___lambda__1___boxed), 6, 5); +lean_closure_set(x_17, 0, x_15); +lean_closure_set(x_17, 1, x_13); +lean_closure_set(x_17, 2, x_1); +lean_closure_set(x_17, 3, x_2); +lean_closure_set(x_17, 4, x_16); +x_18 = lean_ctor_get(x_1, 1); +lean_inc(x_18); +x_19 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__9___rarg), 5, 4); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, lean_box(0)); +lean_closure_set(x_19, 2, lean_box(0)); +lean_closure_set(x_19, 3, x_17); +x_20 = lean_apply_4(x_18, lean_box(0), lean_box(0), x_14, x_19); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___boxed), 5, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__10___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__10(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__10___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__11___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__11(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__11___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__12___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +uint8_t x_6; +lean_dec(x_4); +x_6 = !lean_is_exclusive(x_5); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 1); +lean_inc(x_8); +lean_dec(x_7); +x_9 = lean_apply_2(x_8, lean_box(0), x_5); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_5, 0); +lean_inc(x_10); +lean_dec(x_5); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +else +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_15 = lean_ctor_get(x_5, 0); +lean_inc(x_15); +lean_dec(x_5); +x_16 = lean_apply_1(x_4, x_15); +return x_16; +} +} +} +LEAN_EXPORT lean_object* l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__12(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__12___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; +lean_inc(x_1); +x_5 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg(x_1, x_2, x_3); +lean_inc(x_1); +x_6 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__1___rarg___lambda__2), 3, 2); +lean_closure_set(x_6, 0, x_4); +lean_closure_set(x_6, 1, x_1); +x_7 = lean_ctor_get(x_1, 1); +lean_inc(x_7); +x_8 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__11___rarg), 5, 4); +lean_closure_set(x_8, 0, x_1); +lean_closure_set(x_8, 1, lean_box(0)); +lean_closure_set(x_8, 2, lean_box(0)); +lean_closure_set(x_8, 3, x_6); +x_9 = lean_apply_4(x_7, lean_box(0), lean_box(0), x_5, x_8); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +switch (lean_obj_tag(x_3)) { +case 0: +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +lean_dec(x_1); +x_6 = lean_ctor_get(x_5, 1); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +x_8 = lean_apply_2(x_6, lean_box(0), x_7); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_9 = lean_ctor_get(x_3, 0); +lean_inc(x_9); +lean_dec(x_3); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_10); +x_14 = lean_apply_2(x_12, lean_box(0), x_13); +return x_14; +} +} +case 1: +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = lean_ctor_get(x_3, 0); +lean_inc(x_15); +lean_dec(x_3); +x_16 = lean_array_get_size(x_15); +x_17 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_18 = 0; +lean_inc(x_1); +x_19 = l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg(x_1, x_2, x_17, x_18, x_15); +lean_inc(x_1); +x_20 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__1___rarg___lambda__1), 2, 1); +lean_closure_set(x_20, 0, x_1); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); +x_22 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__10___rarg), 5, 4); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, lean_box(0)); +lean_closure_set(x_22, 2, lean_box(0)); +lean_closure_set(x_22, 3, x_20); +x_23 = lean_apply_4(x_21, lean_box(0), lean_box(0), x_19, x_22); +return x_23; +} +default: +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_3, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_3, 1); +lean_inc(x_25); +lean_dec(x_3); +lean_inc(x_2); +x_26 = lean_apply_1(x_2, x_24); +lean_inc(x_1); +x_27 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg___lambda__1), 4, 3); +lean_closure_set(x_27, 0, x_1); +lean_closure_set(x_27, 1, x_2); +lean_closure_set(x_27, 2, x_25); +x_28 = lean_ctor_get(x_1, 1); +lean_inc(x_28); +x_29 = lean_alloc_closure((void*)(l_ExceptT_bindCont___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__12___rarg), 5, 4); +lean_closure_set(x_29, 0, x_1); +lean_closure_set(x_29, 1, lean_box(0)); +lean_closure_set(x_29, 2, lean_box(0)); +lean_closure_set(x_29, 3, x_27); +x_30 = lean_apply_4(x_28, lean_box(0), lean_box(0), x_26, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg), 3, 0); +return x_4; +} +} LEAN_EXPORT lean_object* l_Lean_Widget_TaggedText_instRpcEncodingTaggedText___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { @@ -4019,7 +4461,7 @@ lean_inc(x_6); lean_dec(x_1); lean_inc(x_3); x_7 = lean_apply_3(x_6, lean_box(0), x_3, x_4); -x_8 = l_Lean_Widget_TaggedText_mapM___rarg(x_3, x_7, x_5); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__1___rarg(x_3, x_7, x_5); return x_8; } } @@ -4032,7 +4474,7 @@ lean_inc(x_6); lean_dec(x_1); lean_inc(x_3); x_7 = lean_apply_3(x_6, lean_box(0), x_3, x_4); -x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__1___rarg(x_3, x_7, x_5); +x_8 = l_Lean_Widget_TaggedText_mapM___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__7___rarg(x_3, x_7, x_5); return x_8; } } @@ -4083,6 +4525,30 @@ x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedTe return x_8; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___lambda__1(x_7, x_2, x_3, x_4, x_8, x_6); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Widget_TaggedText_instRpcEncodingTaggedText___spec__8___rarg(x_1, x_2, x_6, x_7, x_5); +return x_8; +} +} static lean_object* _init_l___private_Lean_Widget_TaggedText_0__Lean_Widget_TaggedText_TaggedState_out___default() { _start: { diff --git a/stage0/stdlib/Std/Data/PersistentArray.c b/stage0/stdlib/Std/Data/PersistentArray.c index cd8e5abb7175..5199e1a2b12d 100644 --- a/stage0/stdlib/Std/Data/PersistentArray.c +++ b/stage0/stdlib/Std/Data/PersistentArray.c @@ -973,7 +973,7 @@ static lean_object* _init_l_Std_PersistentArray_getAux___rarg___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Std_PersistentArray_getAux___rarg___closed__1; x_2 = l_Std_PersistentArray_getAux___rarg___closed__2; -x_3 = lean_unsigned_to_nat(62u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(36u); x_5 = l_Std_PersistentArray_getAux___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/tests/elabissues/issues8.lean b/tests/elabissues/issues8.lean index fea4289061c2..73bd4e19302b 100644 --- a/tests/elabissues/issues8.lean +++ b/tests/elabissues/issues8.lean @@ -7,6 +7,7 @@ The following example works, but it adds a coercion at `forceInt i`. The elaborated term is ``` fun (n i : Nat) => if n == i then forceNat n else forceInt (coe i) +``` -/ fun n i => if n == i then forceNat n else forceInt i -- works diff --git a/tests/lean/1298.lean b/tests/lean/1298.lean new file mode 100644 index 000000000000..26c885dc496a --- /dev/null +++ b/tests/lean/1298.lean @@ -0,0 +1,15 @@ +class Semiring (R : Type u) extends Add R, HPow R Nat R, Mul R where + zero : R + +instance [Semiring R] : OfNat R n where + ofNat := Semiring.zero + +def Nat.cast [Semiring R] (n : Nat) : R := let _ := n = n; Semiring.zero + +@[defaultInstance high] instance [Semiring R] : HPow R Nat R := inferInstance + +instance [Semiring R] : CoeTail Nat R where + coe n := n.cast + +variable (R) [Semiring R] +#check (8 + 2 ^ 2 * 3 : R) = 20 diff --git a/tests/lean/1298.lean.expected.out b/tests/lean/1298.lean.expected.out new file mode 100644 index 000000000000..e7576b1e745e --- /dev/null +++ b/tests/lean/1298.lean.expected.out @@ -0,0 +1 @@ +8 + 2 ^ 2 * 3 = 20 : Prop diff --git a/tests/lean/1301.lean b/tests/lean/1301.lean new file mode 100644 index 000000000000..ba57c1a0948b --- /dev/null +++ b/tests/lean/1301.lean @@ -0,0 +1,10 @@ +syntax "tac" : tactic +theorem a : True := by tac +#check a -- should be declared + +theorem a' : True ∧ True := ⟨by tac, by tac⟩ +#check a' -- should be declared + +syntax "term" : term +def b (n : Nat) : Nat := term +#print b -- should be declared diff --git a/tests/lean/1301.lean.expected.out b/tests/lean/1301.lean.expected.out new file mode 100644 index 000000000000..964b6e3b2df8 --- /dev/null +++ b/tests/lean/1301.lean.expected.out @@ -0,0 +1,8 @@ +1301.lean:2:23-2:26: error: tactic 'tacticTac' has not been implemented +a : True +1301.lean:5:32-5:35: error: tactic 'tacticTac' has not been implemented +a' : True ∧ True +1301.lean:9:25-9:29: error: elaboration function for 'termTerm' has not been implemented + term +def b : Nat → Nat := +sorryAx (Nat → Nat) true diff --git a/tests/lean/1321.lean b/tests/lean/1321.lean new file mode 100644 index 000000000000..e2434ee03ad4 --- /dev/null +++ b/tests/lean/1321.lean @@ -0,0 +1,11 @@ + +@[reducible] +syntax (name := fooParser) "foo" term : term + +#print fooParser + +macro_rules + | `(foo $x) => `($x + 1) + +#check foo 5 + diff --git a/tests/lean/1321.lean.expected.out b/tests/lean/1321.lean.expected.out new file mode 100644 index 000000000000..2b81ffa6ba3d --- /dev/null +++ b/tests/lean/1321.lean.expected.out @@ -0,0 +1,4 @@ +@[reducible] def fooParser : Lean.ParserDescr := +Lean.ParserDescr.node `fooParser 1022 + (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol "foo") (Lean.ParserDescr.cat `term 0)) +5 + 1 : Nat diff --git a/tests/lean/1358.lean b/tests/lean/1358.lean new file mode 100644 index 000000000000..0da37df27c99 --- /dev/null +++ b/tests/lean/1358.lean @@ -0,0 +1,10 @@ +import Lean.Elab.Tactic + +open Lean Elab Tactic in +elab "print!" : tactic => do + logInfo "foo" + throwError "error" + +example : True := by + print! + admit diff --git a/tests/lean/1358.lean.expected.out b/tests/lean/1358.lean.expected.out new file mode 100644 index 000000000000..7bee343402be --- /dev/null +++ b/tests/lean/1358.lean.expected.out @@ -0,0 +1,2 @@ +foo +1358.lean:9:2-9:8: error: error diff --git a/tests/lean/248.lean.expected.out b/tests/lean/248.lean.expected.out index 5c9ae74696b3..2444eeee1aa5 100644 --- a/tests/lean/248.lean.expected.out +++ b/tests/lean/248.lean.expected.out @@ -1 +1 @@ -248.lean:1:28-1:31: error: invalid 'implementedBy' argument 'foo', function cannot be implemented by itself +248.lean:1:2-1:19: error: invalid 'implementedBy' argument 'foo', function cannot be implemented by itself diff --git a/tests/lean/343.lean.expected.out b/tests/lean/343.lean.expected.out index dfab8285760b..b6c0daaf99b7 100644 --- a/tests/lean/343.lean.expected.out +++ b/tests/lean/343.lean.expected.out @@ -5,3 +5,9 @@ while trying to unify Catish.Obj Catish.Obj with CatIsh.{max ?u ?u, max (?u + 1) (?u + 1)} +343.lean:30:0-30:54: error: failed to solve universe constraint + max (?u+1) (?u+1) =?= max (?u+1) (?u+1) +while trying to unify + Catish.Obj : Type (max ((max (u_1 + 1) (u_2 + 1)) + 1) ((max u_3 u_4) + 1)) +with + CatIsh : Type (max ((max u_4 u_3) + 1) ((max (u_4 + 1) (u_3 + 1)) + 1)) diff --git a/tests/lean/423.lean.expected.out b/tests/lean/423.lean.expected.out index b5b3f9697067..2b54a56ed9ea 100644 --- a/tests/lean/423.lean.expected.out +++ b/tests/lean/423.lean.expected.out @@ -1,9 +1,11 @@ -423.lean:3:39-3:40: error: type mismatch - 0 +423.lean:3:35-3:40: error: application type mismatch + HAdd.hAdd a +argument + a has type - Nat : Type -but is expected to have type T : Sort u +but is expected to have type + Nat : Type 423.lean:5:37-5:38: error: application type mismatch Add T argument @@ -20,9 +22,11 @@ has type Sort u : Type u but is expected to have type Type ?u : Type (?u + 1) -423.lean:5:59-5:60: error: type mismatch - 0 +423.lean:5:55-5:60: error: application type mismatch + HAdd.hAdd a +argument + a has type - Nat : Type -but is expected to have type T : Sort u +but is expected to have type + Nat : Type diff --git a/tests/lean/625.lean b/tests/lean/625.lean index 1880ef48219e..b40c72c61389 100644 --- a/tests/lean/625.lean +++ b/tests/lean/625.lean @@ -1,8 +1,8 @@ import Lean open Lean Lean.PrettyPrinter -def pfoo : PUnit → PUnit := id -def px : PUnit := () +def foo : PUnit → PUnit := id +def x : PUnit := () @[appUnexpander foo] def unexpandFoo : Unexpander := fun _ => `(sorry) diff --git a/tests/lean/625.lean.expected.out b/tests/lean/625.lean.expected.out index 5f485bdf9d44..897acac56c0c 100644 --- a/tests/lean/625.lean.expected.out +++ b/tests/lean/625.lean.expected.out @@ -1,3 +1,2 @@ -625.lean:7:25-7:36: error: unknown constant 'foo' -foo x +sorry foo.{1} x diff --git a/tests/lean/973.lean.expected.out b/tests/lean/973.lean.expected.out index 4daf61c04584..a56dc3b7b150 100644 --- a/tests/lean/973.lean.expected.out +++ b/tests/lean/973.lean.expected.out @@ -1,2 +1,2 @@ -973.lean:5:8-5:22: error: invalid `simp` theorem, equation is equivalent to +973.lean:4:2-4:6: error: invalid `simp` theorem, equation is equivalent to x = x diff --git a/tests/lean/autoImplicitForbidden.lean b/tests/lean/autoImplicitForbidden.lean index 54b54dca3167..9cc11570aebe 100644 --- a/tests/lean/autoImplicitForbidden.lean +++ b/tests/lean/autoImplicitForbidden.lean @@ -21,3 +21,10 @@ mutual inductive Ex2 : Type end + + +structure Bar := + (x : Na) + (y : Nat := foobar) -- Error at `foobar` + +#print Bar.mk diff --git a/tests/lean/autoImplicitForbidden.lean.expected.out b/tests/lean/autoImplicitForbidden.lean.expected.out index 33c9afc6852d..dc281130195d 100644 --- a/tests/lean/autoImplicitForbidden.lean.expected.out +++ b/tests/lean/autoImplicitForbidden.lean.expected.out @@ -3,3 +3,5 @@ autoImplicitForbidden.lean:6:10-6:11: error: unknown identifier 'h' autoImplicitForbidden.lean:13:24-13:27: error: unknown identifier 'Bla' autoImplicitForbidden.lean:16:21-16:24: error: unknown identifier 'Foo' autoImplicitForbidden.lean:20:18-20:21: error: unknown identifier 'Ex2' +autoImplicitForbidden.lean:28:14-28:20: error: unknown identifier 'foobar' +constructor Bar.mk.{u_1} : ({Na : Sort u_1} → Na) → Nat → Bar diff --git a/tests/lean/class_def_must_fail.lean.expected.out b/tests/lean/class_def_must_fail.lean.expected.out index 0d7b98fa8929..ef5d4e31b64c 100644 --- a/tests/lean/class_def_must_fail.lean.expected.out +++ b/tests/lean/class_def_must_fail.lean.expected.out @@ -1,2 +1,2 @@ -class_def_must_fail.lean:2:13-2:16: error: invalid 'class', declaration 'Foo' must be inductive datatype, structure, or constant -class_def_must_fail.lean:7:18-7:21: error: invalid 'class', declaration 'Bla' must be inductive datatype, structure, or constant +class_def_must_fail.lean:2:2-2:7: error: invalid 'class', declaration 'Foo' must be inductive datatype, structure, or constant +class_def_must_fail.lean:7:11-7:16: error: invalid 'class', declaration 'Bla' must be inductive datatype, structure, or constant diff --git a/tests/lean/csimpAttr.lean.expected.out b/tests/lean/csimpAttr.lean.expected.out index 6cbefeae02cf..d69d1215be26 100644 --- a/tests/lean/csimpAttr.lean.expected.out +++ b/tests/lean/csimpAttr.lean.expected.out @@ -3,4 +3,4 @@ def f (x_1 : obj) : obj := let x_2 : obj := Nat.add x_1 x_1; let x_3 : obj := Nat.add x_2 x_2; - ret x_3csimpAttr.lean:7:17-7:28: error: invalid 'csimp' theorem, only constant replacement theorems (e.g., `@f = @g`) are currently supported. + ret x_3csimpAttr.lean:7:2-7:7: error: invalid 'csimp' theorem, only constant replacement theorems (e.g., `@f = @g`) are currently supported. diff --git a/tests/lean/derivingRpcEncoding.lean b/tests/lean/derivingRpcEncoding.lean new file mode 100644 index 000000000000..4608ebbf6f8d --- /dev/null +++ b/tests/lean/derivingRpcEncoding.lean @@ -0,0 +1,109 @@ +import Lean.Server.Rpc.Basic + +open Lean Server + +abbrev M := StateM (Array (Name × NonScalar)) + +instance : MonadRpcSession M where + rpcStoreRef typeName obj := + (return ⟨(← get).size.toUSize⟩) <* modify (·.push (typeName, obj)) + rpcGetRef r := return (← get)[r.p]? + rpcReleaseRef _ := return false + +def M.run (x : ExceptT String M α) : Except String α := x.run' #[] + +def test (α : Type) [RpcEncoding α β] [FromJson β] [ToJson β] (a : α) := M.run do + let json := toJson (← rpcEncode a) + let packet ← ofExcept (fromJson? (α := β) json) + let _ ← rpcDecode (α := α) packet + return json + +@[reducible] +def rpcPacketFor (α : Type) {β : outParam Type} [RpcEncoding α β] := β + +structure FooRef where + a : Array Nat + deriving Inhabited, RpcEncoding with { withRef := true } + +#check instRpcEncodingWithRpcRefFooRefRpcRef +#eval test (WithRpcRef FooRef) default + +structure FooJson where + s : String + deriving FromJson, ToJson, Inhabited + +structure Bar where + fooRef : WithRpcRef FooRef + fooJson : FooJson + deriving RpcEncoding, Inhabited + +#check instRpcEncodingBar +#eval test Bar default + +structure BarTrans where + bar : Bar + deriving RpcEncoding, Inhabited + +#check instRpcEncodingBarTrans +#eval test BarTrans default + +structure Baz where + arr : Array String -- non-constant field + deriving RpcEncoding, Inhabited + +#check instRpcEncodingBaz +#eval test Baz default + +structure FooGeneric (α : Type) where + a : α + b? : Option α + deriving RpcEncoding, Inhabited + +#check instRpcEncodingFooGeneric +#eval test (FooGeneric Nat) default +#eval test (FooGeneric Nat) { a := 3, b? := some 42 } + +inductive BazInductive + | baz (arr : Array Bar) + deriving RpcEncoding, Inhabited + +#check instRpcEncodingBazInductive +#eval test BazInductive ⟨#[default, default]⟩ + +inductive FooInductive (α : Type) where + | a : α → WithRpcRef FooRef → FooInductive α + | b : (n : Nat) → (a : α) → (m : Nat) → FooInductive α + deriving RpcEncoding, Inhabited + +#check instRpcEncodingFooInductive +#eval test (FooInductive BazInductive) (.a default default) +#eval test (FooInductive BazInductive) (.b 42 default default) + +inductive FooNested (α : Type) where + | a : α → Array (FooNested α) → FooNested α + deriving RpcEncoding, Inhabited + +#eval test (FooNested BazInductive) (.a default #[default]) + +inductive FooParam (n : Nat) where + | a : Nat → FooParam n + deriving RpcEncoding, Inhabited + +#check instRpcEncodingFooParam +#eval test (FooParam 10) (.a 42) + +inductive Unused (α : Type) | a + deriving RpcEncoding, Inhabited + +#check instRpcEncodingUnused +structure NoRpcEncoding +#eval test (Unused NoRpcEncoding) default + +structure UnusedStruct (α : Type) + deriving RpcEncoding, Inhabited + +#check instRpcEncodingUnusedStruct +#eval test (UnusedStruct NoRpcEncoding) default + +deriving instance Repr, RpcEncoding for Empty +#eval M.run do rpcDecode (α := Empty) (← fromJson? .null) diff --git a/tests/lean/derivingRpcEncoding.lean.expected.out b/tests/lean/derivingRpcEncoding.lean.expected.out new file mode 100644 index 000000000000..281522e27fed --- /dev/null +++ b/tests/lean/derivingRpcEncoding.lean.expected.out @@ -0,0 +1,29 @@ +instRpcEncodingWithRpcRefFooRefRpcRef : RpcEncoding (WithRpcRef FooRef) Lsp.RpcRef +ok: {"p": "0"} +instRpcEncodingBar : RpcEncoding Bar RpcEncodingPacket✝ +ok: {"fooRef": {"p": "0"}, "fooJson": {"s": ""}} +instRpcEncodingBarTrans : RpcEncoding BarTrans RpcEncodingPacket✝ +ok: {"bar": {"fooRef": {"p": "0"}, "fooJson": {"s": ""}}} +instRpcEncodingBaz : RpcEncoding Baz RpcEncodingPacket✝ +ok: {"arr": []} +instRpcEncodingFooGeneric : (α αPacket : Type) → + [inst : RpcEncoding α αPacket] → RpcEncoding (FooGeneric α) (RpcEncodingPacket✝ αPacket) +ok: {"a": 0} +ok: {"b": 42, "a": 3} +instRpcEncodingBazInductive : RpcEncoding BazInductive RpcEncodingPacket✝ +ok: {"baz": + {"arr": + [{"fooRef": {"p": "0"}, "fooJson": {"s": ""}}, + {"fooRef": {"p": "1"}, "fooJson": {"s": ""}}]}} +instRpcEncodingFooInductive : (α αPacket : Type) → + [inst : RpcEncoding α αPacket] → RpcEncoding (FooInductive α) (RpcEncodingPacket✝ αPacket) +ok: {"a": [{"baz": {"arr": []}}, {"p": "0"}]} +ok: {"b": {"n": 42, "m": 0, "a": {"baz": {"arr": []}}}} +ok: {"a": [{"baz": {"arr": []}}, [{"a": [{"baz": {"arr": []}}, []]}]]} +instRpcEncodingFooParam : (n : Nat) → RpcEncoding (FooParam n) RpcEncodingPacket✝ +ok: {"a": 42} +instRpcEncodingUnused : (α : Type) → RpcEncoding (Unused α) RpcEncodingPacket✝ +ok: "a" +instRpcEncodingUnusedStruct : (α : Type) → RpcEncoding (UnusedStruct α) RpcEncodingPacket✝ +ok: {} +Except.error "no inductive constructor matched" diff --git a/tests/lean/docStr.lean.expected.out b/tests/lean/docStr.lean.expected.out index 680c7cb4038e..832ed0796958 100644 --- a/tests/lean/docStr.lean.expected.out +++ b/tests/lean/docStr.lean.expected.out @@ -17,7 +17,7 @@ doc string for 'g' is not available "let rec documentation at g " "Gadget for optional parameter support. " "Auxiliary Declaration used to implement the named patterns `x@h:p` " -"Similar to `forallTelescope`, but given `type` of the form `forall xs, A`,\n it reduces `A` and continues bulding the telescope if it is a `forall`. " +"Similar to `forallTelescope`, but given `type` of the form `forall xs, A`,\nit reduces `A` and continues bulding the telescope if it is a `forall`. " Foo := { range := { pos := { line := 4, column := 0 }, charUtf16 := 0, diff --git a/tests/lean/heapSort.lean.expected.out b/tests/lean/heapSort.lean.expected.out index 08d16eb1737a..6d8ef35cd963 100644 --- a/tests/lean/heapSort.lean.expected.out +++ b/tests/lean/heapSort.lean.expected.out @@ -11,4 +11,4 @@ heapSort.lean:102:4-102:13: warning: declaration uses 'sorry' | some x => let_fun this := (_ : BinaryHeap.size (BinaryHeap.popMax a) < BinaryHeap.size a); Array.heapSort.loop lt (BinaryHeap.popMax a) (Array.push out x) -heapSort.lean:178:17-178:39: warning: declaration uses 'sorry' +heapSort.lean:178:11-178:15: warning: declaration uses 'sorry' diff --git a/tests/lean/holes.lean.expected.out b/tests/lean/holes.lean.expected.out index 53d15a5fbaa2..d7b937828804 100644 --- a/tests/lean/holes.lean.expected.out +++ b/tests/lean/holes.lean.expected.out @@ -22,12 +22,12 @@ x : Nat ⊢ Type holes.lean:13:10-13:11: error: failed to infer binder type holes.lean:15:16-15:17: error: failed to infer binder type -holes.lean:18:9-18:10: error: failed to infer binder type holes.lean:19:0-19:3: error: don't know how to synthesize implicit argument @f Nat (?m a) a context: a : Nat f : {α : Type} → {β : ?m a} → α → α := fun {α} {β} a => a ⊢ ?m a +holes.lean:18:9-18:10: error: failed to infer binder type holes.lean:21:25-22:4: error: failed to infer definition type holes.lean:25:8-25:11: error: failed to infer 'let rec' declaration type diff --git a/tests/lean/implementedByIssue.lean.expected.out b/tests/lean/implementedByIssue.lean.expected.out index ff83f54145ab..060227cb8c71 100644 --- a/tests/lean/implementedByIssue.lean.expected.out +++ b/tests/lean/implementedByIssue.lean.expected.out @@ -1,5 +1,5 @@ -implementedByIssue.lean:15:32-15:42: error: invalid 'implementedBy' argument 'Hidden.get_2', 'Hidden.get_2' has 0 universe level parameter(s), but 'Hidden.Array.data' has 1 -implementedByIssue.lean:19:32-19:42: error: invalid 'implementedBy' argument 'Hidden.get_3', 'Hidden.get_3' has type +implementedByIssue.lean:15:11-15:30: error: invalid 'implementedBy' argument 'Hidden.get_2', 'Hidden.get_2' has 0 universe level parameter(s), but 'Hidden.Array.data' has 1 +implementedByIssue.lean:19:11-19:30: error: invalid 'implementedBy' argument 'Hidden.get_3', 'Hidden.get_3' has type {α : Type u} → {n : Nat} → Fin n → Array α n → α but 'Hidden.Array.data' has type {α : Type u} → {n : Nat} → Array α n → Fin n → α diff --git a/tests/lean/inductive1.lean.expected.out b/tests/lean/inductive1.lean.expected.out index 82dfbce113b4..8d1507874e81 100644 --- a/tests/lean/inductive1.lean.expected.out +++ b/tests/lean/inductive1.lean.expected.out @@ -18,7 +18,7 @@ inductive1.lean:69:2-69:5: error: 'Boo.T1.bla' has already been declared inductive1.lean:73:10-73:12: error: 'Boo.T1' has already been declared inductive1.lean:80:0-80:27: error: invalid use of 'partial' in inductive declaration inductive1.lean:81:0-81:33: error: invalid use of 'noncomputable' in inductive declaration -inductive1.lean:82:10-82:30: error: declaration is not a definition 'T1'' +inductive1.lean:82:2-82:8: error: declaration is not a definition 'T1'' inductive1.lean:85:0-85:17: error: invalid 'private' constructor in a 'private' inductive datatype inductive1.lean:93:7-93:26: error: invalid inductive type, cannot mix unsafe and safe declarations in a mutually inductive datatypes inductive1.lean:100:0-100:4: error: constructor resulting type must be specified in inductive family declaration diff --git a/tests/lean/infoTree.lean.expected.out b/tests/lean/infoTree.lean.expected.out index 91f0045e59ea..4bcbf427f760 100644 --- a/tests/lean/infoTree.lean.expected.out +++ b/tests/lean/infoTree.lean.expected.out @@ -116,20 +116,20 @@ [Elab.info] command @ ⟨21, 0⟩-⟨25, 10⟩ @ Lean.Elab.Command.elabDeclaration Nat → Nat → Bool → Nat : Type @ ⟨21, 9⟩-⟨21, 39⟩ @ Lean.Elab.Term.elabDepArrow Nat : Type @ ⟨21, 16⟩-⟨21, 19⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.549} @ ⟨21, 16⟩-⟨21, 19⟩ + [.] `Nat : some Sort.{?_uniq.562} @ ⟨21, 16⟩-⟨21, 19⟩ Nat : Type @ ⟨21, 16⟩-⟨21, 19⟩ x (isBinder := true) : Nat @ ⟨21, 10⟩-⟨21, 11⟩ Nat : Type @ ⟨21, 16⟩-⟨21, 19⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.551} @ ⟨21, 16⟩-⟨21, 19⟩ + [.] `Nat : some Sort.{?_uniq.564} @ ⟨21, 16⟩-⟨21, 19⟩ Nat : Type @ ⟨21, 16⟩-⟨21, 19⟩ y (isBinder := true) : Nat @ ⟨21, 12⟩-⟨21, 13⟩ Bool → Nat : Type @ ⟨21, 23⟩-⟨21, 39⟩ @ Lean.Elab.Term.elabDepArrow Bool : Type @ ⟨21, 28⟩-⟨21, 32⟩ @ Lean.Elab.Term.elabIdent - [.] `Bool : some Sort.{?_uniq.554} @ ⟨21, 28⟩-⟨21, 32⟩ + [.] `Bool : some Sort.{?_uniq.567} @ ⟨21, 28⟩-⟨21, 32⟩ Bool : Type @ ⟨21, 28⟩-⟨21, 32⟩ b (isBinder := true) : Bool @ ⟨21, 24⟩-⟨21, 25⟩ Nat : Type @ ⟨21, 36⟩-⟨21, 39⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.556} @ ⟨21, 36⟩-⟨21, 39⟩ + [.] `Nat : some Sort.{?_uniq.569} @ ⟨21, 36⟩-⟨21, 39⟩ Nat : Type @ ⟨21, 36⟩-⟨21, 39⟩ f2 (isBinder := true) : Nat → Nat → Bool → Nat @ ⟨21, 4⟩-⟨21, 6⟩ fun x y b => @@ -186,7 +186,7 @@ ===> Prod.mk✝ (x + y) (x - y) (x + y, x - y) : Nat × Nat @ ⟨23, 18⟩†-⟨23, 31⟩ @ Lean.Elab.Term.elabApp - [.] `Prod.mk._@.infoTree._hyg.88 : some ?_uniq.568 @ ⟨23, 18⟩†-⟨23, 32⟩† + [.] `Prod.mk._@.infoTree._hyg.88 : some ?_uniq.581 @ ⟨23, 18⟩†-⟨23, 32⟩† @Prod.mk : {α β : Type} → α → β → α × β @ ⟨23, 18⟩†-⟨23, 32⟩† x + y : Nat @ ⟨23, 19⟩-⟨23, 24⟩ @ «_aux_Init_Notation___macroRules_term_+__2» Macro expansion @@ -224,8 +224,8 @@ [.] `z : none @ ⟨23, 9⟩-⟨23, 10⟩ [.] `w : none @ ⟨23, 12⟩-⟨23, 13⟩ [.] `Prod.mk._@.infoTree._hyg.102 : some Prod.{0 0} Nat Nat @ ⟨23, 4⟩†-⟨25, 10⟩† - [.] `z : some [mdata _patWithRef: ?_uniq.636] @ ⟨23, 9⟩-⟨23, 10⟩ - [.] `w : some [mdata _patWithRef: ?_uniq.637] @ ⟨23, 12⟩-⟨23, 13⟩ + [.] `z : some [mdata _patWithRef: ?_uniq.675] @ ⟨23, 9⟩-⟨23, 10⟩ + [.] `w : some [mdata _patWithRef: ?_uniq.676] @ ⟨23, 12⟩-⟨23, 13⟩ (z, w) : Nat × Nat @ ⟨23, 4⟩†-⟨23, 13⟩ Nat : Type @ ⟨23, 4⟩†-⟨23, 13⟩† Nat : Type @ ⟨23, 4⟩†-⟨23, 13⟩† @@ -269,13 +269,13 @@ ===> Prod✝ Nat (Array (Array Nat)) Nat × Array (Array Nat) : Type @ ⟨27, 12⟩†-⟨27, 35⟩ @ Lean.Elab.Term.elabApp - [.] `Prod._@.infoTree._hyg.127 : some Sort.{?_uniq.764} @ ⟨27, 12⟩†-⟨27, 35⟩† + [.] `Prod._@.infoTree._hyg.127 : some Sort.{?_uniq.809} @ ⟨27, 12⟩†-⟨27, 35⟩† Prod : Type → Type → Type @ ⟨27, 12⟩†-⟨27, 35⟩† Nat : Type @ ⟨27, 12⟩-⟨27, 15⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Type.{?_uniq.766} @ ⟨27, 12⟩-⟨27, 15⟩ + [.] `Nat : some Type.{?_uniq.811} @ ⟨27, 12⟩-⟨27, 15⟩ Nat : Type @ ⟨27, 12⟩-⟨27, 15⟩ Array (Array Nat) : Type @ ⟨27, 18⟩-⟨27, 35⟩ @ Lean.Elab.Term.elabApp - [.] `Array : some Type.{?_uniq.765} @ ⟨27, 18⟩-⟨27, 23⟩ + [.] `Array : some Type.{?_uniq.810} @ ⟨27, 18⟩-⟨27, 23⟩ Array : Type → Type @ ⟨27, 18⟩-⟨27, 23⟩ Array Nat : Type @ ⟨27, 24⟩-⟨27, 35⟩ @ Lean.Elab.Term.expandParen Macro expansion @@ -283,17 +283,17 @@ ===> Array Nat Array Nat : Type @ ⟨27, 25⟩-⟨27, 34⟩ @ Lean.Elab.Term.elabApp - [.] `Array : some Type.{?_uniq.767} @ ⟨27, 25⟩-⟨27, 30⟩ + [.] `Array : some Type.{?_uniq.812} @ ⟨27, 25⟩-⟨27, 30⟩ Array : Type → Type @ ⟨27, 25⟩-⟨27, 30⟩ Nat : Type @ ⟨27, 31⟩-⟨27, 34⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Type.{?_uniq.768} @ ⟨27, 31⟩-⟨27, 34⟩ + [.] `Nat : some Type.{?_uniq.813} @ ⟨27, 31⟩-⟨27, 34⟩ Nat : Type @ ⟨27, 31⟩-⟨27, 34⟩ s (isBinder := true) : Nat × Array (Array Nat) @ ⟨27, 8⟩-⟨27, 9⟩ Array Nat : Type @ ⟨27, 39⟩-⟨27, 48⟩ @ Lean.Elab.Term.elabApp - [.] `Array : some Sort.{?_uniq.770} @ ⟨27, 39⟩-⟨27, 44⟩ + [.] `Array : some Sort.{?_uniq.815} @ ⟨27, 39⟩-⟨27, 44⟩ Array : Type → Type @ ⟨27, 39⟩-⟨27, 44⟩ Nat : Type @ ⟨27, 45⟩-⟨27, 48⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Type.{?_uniq.771} @ ⟨27, 45⟩-⟨27, 48⟩ + [.] `Nat : some Type.{?_uniq.816} @ ⟨27, 45⟩-⟨27, 48⟩ Nat : Type @ ⟨27, 45⟩-⟨27, 48⟩ f3 (isBinder := true) : Nat × Array (Array Nat) → Array Nat @ ⟨27, 4⟩-⟨27, 6⟩ s (isBinder := true) : Nat × Array (Array Nat) @ ⟨27, 8⟩-⟨27, 9⟩ @@ -311,24 +311,24 @@ [inst : Inhabited Elem] → (xs : Cont) → (i : Idx) → [inst : Decidable (Dom xs i)] → Elem @ ⟨28, 2⟩†-⟨28, 9⟩† s.snd : Array (Array Nat) @ ⟨28, 2⟩-⟨28, 5⟩ @ Lean.Elab.Term.elabProj - [.] `s : some ?_uniq.777 @ ⟨28, 2⟩-⟨28, 3⟩ + [.] `s : some ?_uniq.822 @ ⟨28, 2⟩-⟨28, 3⟩ s : Nat × Array (Array Nat) @ ⟨28, 2⟩-⟨28, 3⟩ @Prod.snd : {α β : Type} → α × β → β @ ⟨28, 4⟩-⟨28, 5⟩ 1 : Nat @ ⟨28, 6⟩-⟨28, 7⟩ @ Lean.Elab.Term.elabNumLit [.] s.snd[1]! : Array Nat @ ⟨28, 2⟩-⟨28, 9⟩ : some Array.{0} Nat @Array.push : {α : Type} → Array α → α → Array α @ ⟨28, 10⟩-⟨28, 14⟩ s.fst : Nat @ ⟨28, 15⟩-⟨28, 18⟩ @ Lean.Elab.Term.elabProj - [.] `s : some ?_uniq.1071 @ ⟨28, 15⟩-⟨28, 16⟩ + [.] `s : some ?_uniq.1116 @ ⟨28, 15⟩-⟨28, 16⟩ s : Nat × Array (Array Nat) @ ⟨28, 15⟩-⟨28, 16⟩ @Prod.fst : {α β : Type} → α × β → α @ ⟨28, 17⟩-⟨28, 18⟩ f3 (isBinder := true) : Nat × Array (Array Nat) → Array Nat @ ⟨27, 4⟩-⟨27, 6⟩ [Elab.info] command @ ⟨30, 0⟩-⟨31, 20⟩ @ Lean.Elab.Command.elabDeclaration B : Type @ ⟨30, 14⟩-⟨30, 15⟩ @ Lean.Elab.Term.elabIdent - [.] `B : some Sort.{?_uniq.1083} @ ⟨30, 14⟩-⟨30, 15⟩ + [.] `B : some Sort.{?_uniq.1128} @ ⟨30, 14⟩-⟨30, 15⟩ B : Type @ ⟨30, 14⟩-⟨30, 15⟩ arg (isBinder := true) : B @ ⟨30, 8⟩-⟨30, 11⟩ Nat : Type @ ⟨30, 19⟩-⟨30, 22⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.1085} @ ⟨30, 19⟩-⟨30, 22⟩ + [.] `Nat : some Sort.{?_uniq.1130} @ ⟨30, 19⟩-⟨30, 22⟩ Nat : Type @ ⟨30, 19⟩-⟨30, 22⟩ f4 (isBinder := true) : B → Nat @ ⟨30, 4⟩-⟨30, 6⟩ arg (isBinder := true) : B @ ⟨30, 8⟩-⟨30, 11⟩ @@ -345,11 +345,11 @@ f4 (isBinder := true) : B → Nat @ ⟨30, 4⟩-⟨30, 6⟩ [Elab.info] command @ ⟨33, 0⟩-⟨35, 1⟩ @ Lean.Elab.Command.elabDeclaration Nat : Type @ ⟨33, 12⟩-⟨33, 15⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.1105} @ ⟨33, 12⟩-⟨33, 15⟩ + [.] `Nat : some Sort.{?_uniq.1150} @ ⟨33, 12⟩-⟨33, 15⟩ Nat : Type @ ⟨33, 12⟩-⟨33, 15⟩ x (isBinder := true) : Nat @ ⟨33, 8⟩-⟨33, 9⟩ B : Type @ ⟨33, 19⟩-⟨33, 20⟩ @ Lean.Elab.Term.elabIdent - [.] `B : some Sort.{?_uniq.1107} @ ⟨33, 19⟩-⟨33, 20⟩ + [.] `B : some Sort.{?_uniq.1152} @ ⟨33, 19⟩-⟨33, 20⟩ B : Type @ ⟨33, 19⟩-⟨33, 20⟩ f5 (isBinder := true) : Nat → B @ ⟨33, 4⟩-⟨33, 6⟩ x (isBinder := true) : Nat @ ⟨33, 8⟩-⟨33, 9⟩ @@ -388,94 +388,102 @@ bitwise bne xor : Nat → Nat → Nat @ ⟨38, 7⟩-⟨38, 10⟩ command @ ⟨37, 0⟩†-⟨38, 10⟩† @ Lean.Elab.Command.elabEnd infoTree.lean:41:0: error: expected identifier or term -[Elab.info] command @ ⟨39, 0⟩-⟨39, 30⟩ @ no_elab +[Elab.info] command @ ⟨39, 0⟩-⟨39, 30⟩ @ Lean.Elab.Command.elabDeclaration + Inhabited Nat : Type @ ⟨39, 11⟩-⟨39, 24⟩ @ Lean.Elab.Term.elabApp + [.] `Inhabited : some Sort.{?_uniq.1173} @ ⟨39, 11⟩-⟨39, 20⟩ + Inhabited : Type → Type @ ⟨39, 11⟩-⟨39, 20⟩ + Nat : Type @ ⟨39, 21⟩-⟨39, 24⟩ @ Lean.Elab.Term.elabIdent + [.] `Nat : some Sort.{?_uniq.1174} @ ⟨39, 21⟩-⟨39, 24⟩ + Nat : Type @ ⟨39, 21⟩-⟨39, 24⟩ + instInhabitedNat_1 (isBinder := true) : Inhabited Nat @ ⟨39, 0⟩†-⟨39, 30⟩† + instInhabitedNat_1 (isBinder := true) : Inhabited Nat @ ⟨39, 0⟩-⟨39, 8⟩ infoTree.lean:44:0: error: expected stx [Elab.info] command @ ⟨41, 0⟩-⟨41, 5⟩ @ no_elab [Elab.info] command @ ⟨44, 0⟩-⟨44, 22⟩ @ Lean.Elab.Command.elabSetOption [.] (Command.set_option "set_option" `pp.raw) @ ⟨44, 0⟩-⟨44, 17⟩ [Elab.info] command @ ⟨45, 0⟩-⟨47, 8⟩ @ Lean.Elab.Command.elabDeclaration Nat : Type @ ⟨45, 14⟩-⟨45, 17⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.1128} @ ⟨45, 14⟩-⟨45, 17⟩ + [.] `Nat : some Sort.{?_uniq.1177} @ ⟨45, 14⟩-⟨45, 17⟩ Nat : Type @ ⟨45, 14⟩-⟨45, 17⟩ - _uniq.1129 (isBinder := true) : Nat @ ⟨45, 8⟩-⟨45, 9⟩ + _uniq.1178 (isBinder := true) : Nat @ ⟨45, 8⟩-⟨45, 9⟩ Nat : Type @ ⟨45, 14⟩-⟨45, 17⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.1130} @ ⟨45, 14⟩-⟨45, 17⟩ + [.] `Nat : some Sort.{?_uniq.1179} @ ⟨45, 14⟩-⟨45, 17⟩ Nat : Type @ ⟨45, 14⟩-⟨45, 17⟩ - _uniq.1131 (isBinder := true) : Nat @ ⟨45, 10⟩-⟨45, 11⟩ - Eq.{1} Nat _uniq.1129 _uniq.1129 : Prop @ ⟨45, 21⟩-⟨45, 26⟩ @ «_aux_Init_Notation___macroRules_term_=__2» + _uniq.1180 (isBinder := true) : Nat @ ⟨45, 10⟩-⟨45, 11⟩ + Eq.{1} Nat _uniq.1178 _uniq.1178 : Prop @ ⟨45, 21⟩-⟨45, 26⟩ @ «_aux_Init_Notation___macroRules_term_=__2» Macro expansion («term_=_» `x "=" `x) ===> - (Term.binrel "binrel%" `Eq._@.infoTree._hyg.180 `x `x) - Eq.{1} Nat _uniq.1129 _uniq.1129 : Prop @ ⟨45, 21⟩†-⟨45, 26⟩ @ Lean.Elab.Term.BinOp.elabBinRel - [.] `Eq._@.infoTree._hyg.180 : none @ ⟨45, 21⟩†-⟨45, 26⟩† - _uniq.1129 : Nat @ ⟨45, 21⟩-⟨45, 22⟩ @ Lean.Elab.Term.elabIdent + (Term.binrel "binrel%" `Eq._@.infoTree._hyg.182 `x `x) + Eq.{1} Nat _uniq.1178 _uniq.1178 : Prop @ ⟨45, 21⟩†-⟨45, 26⟩ @ Lean.Elab.Term.BinOp.elabBinRel + [.] `Eq._@.infoTree._hyg.182 : none @ ⟨45, 21⟩†-⟨45, 26⟩† + _uniq.1178 : Nat @ ⟨45, 21⟩-⟨45, 22⟩ @ Lean.Elab.Term.elabIdent [.] `x : none @ ⟨45, 21⟩-⟨45, 22⟩ - _uniq.1129 : Nat @ ⟨45, 21⟩-⟨45, 22⟩ - _uniq.1129 : Nat @ ⟨45, 25⟩-⟨45, 26⟩ @ Lean.Elab.Term.elabIdent + _uniq.1178 : Nat @ ⟨45, 21⟩-⟨45, 22⟩ + _uniq.1178 : Nat @ ⟨45, 25⟩-⟨45, 26⟩ @ Lean.Elab.Term.elabIdent [.] `x : none @ ⟨45, 25⟩-⟨45, 26⟩ - _uniq.1129 : Nat @ ⟨45, 25⟩-⟨45, 26⟩ - _uniq.1135 (isBinder := true) : forall (x : Nat), Nat -> (Eq.{1} Nat x x) @ ⟨45, 4⟩-⟨45, 6⟩ - _uniq.1136 (isBinder := true) : Nat @ ⟨45, 8⟩-⟨45, 9⟩ - _uniq.1137 (isBinder := true) : Nat @ ⟨45, 10⟩-⟨45, 11⟩ - (fun (f7 : forall (x : Nat), Nat -> (Eq.{1} Nat x x)) => [mdata _recApp: f7 _uniq.1136 _uniq.1137]) f6.f7 : Eq.{1} Nat _uniq.1136 _uniq.1136 @ ⟨46, 2⟩-⟨47, 8⟩ @ Lean.Elab.Term.elabLetRec + _uniq.1178 : Nat @ ⟨45, 25⟩-⟨45, 26⟩ + _uniq.1184 (isBinder := true) : forall (x : Nat), Nat -> (Eq.{1} Nat x x) @ ⟨45, 4⟩-⟨45, 6⟩ + _uniq.1185 (isBinder := true) : Nat @ ⟨45, 8⟩-⟨45, 9⟩ + _uniq.1186 (isBinder := true) : Nat @ ⟨45, 10⟩-⟨45, 11⟩ + (fun (f7 : forall (x : Nat), Nat -> (Eq.{1} Nat x x)) => [mdata _recApp: f7 _uniq.1185 _uniq.1186]) f6.f7 : Eq.{1} Nat _uniq.1185 _uniq.1185 @ ⟨46, 2⟩-⟨47, 8⟩ @ Lean.Elab.Term.elabLetRec Nat : Type @ ⟨46, 20⟩-⟨46, 23⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.1138} @ ⟨46, 20⟩-⟨46, 23⟩ + [.] `Nat : some Sort.{?_uniq.1187} @ ⟨46, 20⟩-⟨46, 23⟩ Nat : Type @ ⟨46, 20⟩-⟨46, 23⟩ - _uniq.1139 (isBinder := true) : Nat @ ⟨46, 14⟩-⟨46, 15⟩ + _uniq.1188 (isBinder := true) : Nat @ ⟨46, 14⟩-⟨46, 15⟩ Nat : Type @ ⟨46, 20⟩-⟨46, 23⟩ @ Lean.Elab.Term.elabIdent - [.] `Nat : some Sort.{?_uniq.1140} @ ⟨46, 20⟩-⟨46, 23⟩ + [.] `Nat : some Sort.{?_uniq.1189} @ ⟨46, 20⟩-⟨46, 23⟩ Nat : Type @ ⟨46, 20⟩-⟨46, 23⟩ - _uniq.1141 (isBinder := true) : Nat @ ⟨46, 16⟩-⟨46, 17⟩ - Eq.{1} Nat _uniq.1139 _uniq.1139 : Prop @ ⟨46, 27⟩-⟨46, 32⟩ @ «_aux_Init_Notation___macroRules_term_=__2» + _uniq.1190 (isBinder := true) : Nat @ ⟨46, 16⟩-⟨46, 17⟩ + Eq.{1} Nat _uniq.1188 _uniq.1188 : Prop @ ⟨46, 27⟩-⟨46, 32⟩ @ «_aux_Init_Notation___macroRules_term_=__2» Macro expansion («term_=_» `x "=" `x) ===> - (Term.binrel "binrel%" `Eq._@.infoTree._hyg.188 `x `x) - Eq.{1} Nat _uniq.1139 _uniq.1139 : Prop @ ⟨46, 27⟩†-⟨46, 32⟩ @ Lean.Elab.Term.BinOp.elabBinRel - [.] `Eq._@.infoTree._hyg.188 : none @ ⟨46, 27⟩†-⟨46, 32⟩† - _uniq.1139 : Nat @ ⟨46, 27⟩-⟨46, 28⟩ @ Lean.Elab.Term.elabIdent + (Term.binrel "binrel%" `Eq._@.infoTree._hyg.190 `x `x) + Eq.{1} Nat _uniq.1188 _uniq.1188 : Prop @ ⟨46, 27⟩†-⟨46, 32⟩ @ Lean.Elab.Term.BinOp.elabBinRel + [.] `Eq._@.infoTree._hyg.190 : none @ ⟨46, 27⟩†-⟨46, 32⟩† + _uniq.1188 : Nat @ ⟨46, 27⟩-⟨46, 28⟩ @ Lean.Elab.Term.elabIdent [.] `x : none @ ⟨46, 27⟩-⟨46, 28⟩ - _uniq.1139 : Nat @ ⟨46, 27⟩-⟨46, 28⟩ - _uniq.1139 : Nat @ ⟨46, 31⟩-⟨46, 32⟩ @ Lean.Elab.Term.elabIdent + _uniq.1188 : Nat @ ⟨46, 27⟩-⟨46, 28⟩ + _uniq.1188 : Nat @ ⟨46, 31⟩-⟨46, 32⟩ @ Lean.Elab.Term.elabIdent [.] `x : none @ ⟨46, 31⟩-⟨46, 32⟩ - _uniq.1139 : Nat @ ⟨46, 31⟩-⟨46, 32⟩ - _uniq.1146 (isBinder := true) : forall (x : Nat), Nat -> (Eq.{1} Nat x x) @ ⟨46, 10⟩-⟨46, 12⟩ - _uniq.1147 (isBinder := true) : Nat @ ⟨46, 14⟩-⟨46, 15⟩ - _uniq.1148 (isBinder := true) : Nat @ ⟨46, 16⟩-⟨46, 17⟩ - Eq.refl.{1} Nat _uniq.1147 : Eq.{1} Nat _uniq.1147 _uniq.1147 @ ⟨46, 36⟩-⟨46, 45⟩ @ Lean.Elab.Term.elabApp - [.] `Eq.refl : some Eq.{?_uniq.1143} Nat _uniq.1147 _uniq.1147 @ ⟨46, 36⟩-⟨46, 43⟩ + _uniq.1188 : Nat @ ⟨46, 31⟩-⟨46, 32⟩ + _uniq.1195 (isBinder := true) : forall (x : Nat), Nat -> (Eq.{1} Nat x x) @ ⟨46, 10⟩-⟨46, 12⟩ + _uniq.1196 (isBinder := true) : Nat @ ⟨46, 14⟩-⟨46, 15⟩ + _uniq.1197 (isBinder := true) : Nat @ ⟨46, 16⟩-⟨46, 17⟩ + Eq.refl.{1} Nat _uniq.1196 : Eq.{1} Nat _uniq.1196 _uniq.1196 @ ⟨46, 36⟩-⟨46, 45⟩ @ Lean.Elab.Term.elabApp + [.] `Eq.refl : some Eq.{?_uniq.1192} Nat _uniq.1196 _uniq.1196 @ ⟨46, 36⟩-⟨46, 43⟩ Eq.refl.{1} : forall {α : Type} (a : α), Eq.{1} α a a @ ⟨46, 36⟩-⟨46, 43⟩ - _uniq.1147 : Nat @ ⟨46, 44⟩-⟨46, 45⟩ @ Lean.Elab.Term.elabIdent - [.] `x : some ?_uniq.1150 @ ⟨46, 44⟩-⟨46, 45⟩ - _uniq.1147 : Nat @ ⟨46, 44⟩-⟨46, 45⟩ - [mdata _recApp: _uniq.1146 _uniq.1136 _uniq.1137] : Eq.{1} Nat _uniq.1136 _uniq.1136 @ ⟨47, 2⟩-⟨47, 8⟩ @ Lean.Elab.Term.elabApp - [.] `f7 : some Eq.{1} Nat _uniq.1136 _uniq.1136 @ ⟨47, 2⟩-⟨47, 4⟩ - _uniq.1146 : forall (x : Nat), Nat -> (Eq.{1} Nat x x) @ ⟨47, 2⟩-⟨47, 4⟩ - _uniq.1136 : Nat @ ⟨47, 5⟩-⟨47, 6⟩ @ Lean.Elab.Term.elabIdent + _uniq.1196 : Nat @ ⟨46, 44⟩-⟨46, 45⟩ @ Lean.Elab.Term.elabIdent + [.] `x : some ?_uniq.1199 @ ⟨46, 44⟩-⟨46, 45⟩ + _uniq.1196 : Nat @ ⟨46, 44⟩-⟨46, 45⟩ + [mdata _recApp: _uniq.1195 _uniq.1185 _uniq.1186] : Eq.{1} Nat _uniq.1185 _uniq.1185 @ ⟨47, 2⟩-⟨47, 8⟩ @ Lean.Elab.Term.elabApp + [.] `f7 : some Eq.{1} Nat _uniq.1185 _uniq.1185 @ ⟨47, 2⟩-⟨47, 4⟩ + _uniq.1195 : forall (x : Nat), Nat -> (Eq.{1} Nat x x) @ ⟨47, 2⟩-⟨47, 4⟩ + _uniq.1185 : Nat @ ⟨47, 5⟩-⟨47, 6⟩ @ Lean.Elab.Term.elabIdent [.] `x : some Nat @ ⟨47, 5⟩-⟨47, 6⟩ - _uniq.1136 : Nat @ ⟨47, 5⟩-⟨47, 6⟩ - _uniq.1137 : Nat @ ⟨47, 7⟩-⟨47, 8⟩ @ Lean.Elab.Term.elabIdent + _uniq.1185 : Nat @ ⟨47, 5⟩-⟨47, 6⟩ + _uniq.1186 : Nat @ ⟨47, 7⟩-⟨47, 8⟩ @ Lean.Elab.Term.elabIdent [.] `y : some Nat @ ⟨47, 7⟩-⟨47, 8⟩ - _uniq.1137 : Nat @ ⟨47, 7⟩-⟨47, 8⟩ + _uniq.1186 : Nat @ ⟨47, 7⟩-⟨47, 8⟩ f6.f7 (isBinder := true) : forall (x : Nat), Nat -> (Eq.{1} Nat x x) @ ⟨46, 10⟩-⟨46, 12⟩ f6 (isBinder := true) : forall (x : Nat), Nat -> (Eq.{1} Nat x x) @ ⟨45, 4⟩-⟨45, 6⟩ [Elab.info] command @ ⟨50, 0⟩-⟨50, 32⟩ @ Lean.Elab.Command.elabDeclaration B : Type @ ⟨50, 12⟩-⟨50, 13⟩ @ Lean.Elab.Term.elabIdent - [.] `B : some Sort.{?_uniq.1170} @ ⟨50, 12⟩-⟨50, 13⟩ + [.] `B : some Sort.{?_uniq.1219} @ ⟨50, 12⟩-⟨50, 13⟩ B : Type @ ⟨50, 12⟩-⟨50, 13⟩ - _uniq.1171 (isBinder := true) : B @ ⟨50, 8⟩-⟨50, 9⟩ + _uniq.1220 (isBinder := true) : B @ ⟨50, 8⟩-⟨50, 9⟩ B : Type @ ⟨50, 17⟩-⟨50, 18⟩ @ Lean.Elab.Term.elabIdent - [.] `B : some Sort.{?_uniq.1172} @ ⟨50, 17⟩-⟨50, 18⟩ + [.] `B : some Sort.{?_uniq.1221} @ ⟨50, 17⟩-⟨50, 18⟩ B : Type @ ⟨50, 17⟩-⟨50, 18⟩ - _uniq.1173 (isBinder := true) : B -> B @ ⟨50, 4⟩-⟨50, 6⟩ - _uniq.1174 (isBinder := true) : B @ ⟨50, 8⟩-⟨50, 9⟩ - B.mk (B.pair _uniq.1174) : B @ ⟨50, 22⟩-⟨50, 32⟩ @ Lean.Elab.Term.StructInst.elabStructInst - _uniq.1174 : B @ ⟨50, 24⟩-⟨50, 25⟩ - B.pair _uniq.1174 : Prod.{0 0} A A @ ⟨50, 24⟩-⟨50, 25⟩† @ Lean.Elab.Term.elabProj + _uniq.1222 (isBinder := true) : B -> B @ ⟨50, 4⟩-⟨50, 6⟩ + _uniq.1223 (isBinder := true) : B @ ⟨50, 8⟩-⟨50, 9⟩ + B.mk (B.pair _uniq.1223) : B @ ⟨50, 22⟩-⟨50, 32⟩ @ Lean.Elab.Term.StructInst.elabStructInst + _uniq.1223 : B @ ⟨50, 24⟩-⟨50, 25⟩ + B.pair _uniq.1223 : Prod.{0 0} A A @ ⟨50, 24⟩-⟨50, 25⟩† @ Lean.Elab.Term.elabProj [.] `b : some Prod.{0 0} A A @ ⟨50, 24⟩-⟨50, 25⟩ - _uniq.1174 : B @ ⟨50, 24⟩-⟨50, 25⟩ - [.] _uniq.1174 : B @ ⟨50, 24⟩-⟨50, 25⟩ : some Prod.{0 0} A A + _uniq.1223 : B @ ⟨50, 24⟩-⟨50, 25⟩ + [.] _uniq.1223 : B @ ⟨50, 24⟩-⟨50, 25⟩ : some Prod.{0 0} A A B.pair : B -> (Prod.{0 0} A A) @ ⟨50, 24⟩†-⟨50, 25⟩† - pair : Prod.{0 0} A A := B.pair _uniq.1174 @ ⟨50, 22⟩†-⟨50, 32⟩ + pair : Prod.{0 0} A A := B.pair _uniq.1223 @ ⟨50, 22⟩†-⟨50, 32⟩ f7 (isBinder := true) : B -> B @ ⟨50, 4⟩-⟨50, 6⟩ diff --git a/tests/lean/interactive/533.lean.expected.out b/tests/lean/interactive/533.lean.expected.out index 9df0a8c39401..1307149e12ff 100644 --- a/tests/lean/interactive/533.lean.expected.out +++ b/tests/lean/interactive/533.lean.expected.out @@ -2,7 +2,13 @@ "position": {"line": 2, "character": 10}} {"items": [{"label": "False", "kind": 22, "detail": "Prop"}, - {"label": "Fin", "kind": 22, "detail": "Nat → Type"}, + {"label": "Fin", + "kind": 22, + "documentation": + {"value": + "`Fin n` is a natural number `i` with the constraint that `0 ≤ i < n`. ", + "kind": "markdown"}, + "detail": "Nat → Type"}, {"label": "Float", "kind": 22, "detail": "Type"}, {"label": "FloatArray", "kind": 22, "detail": "Type"}, {"label": "FloatSpec", "kind": 22, "detail": "Type 1"}, @@ -15,9 +21,18 @@ "kind": 7, "detail": "(Type u₁ → Type u₂) →\n (ρ : Type u) → (α : outParam (Type v)) → outParam (Membership α ρ) → Type (max (max (max u (u₁ + 1)) u₂) v)"}, - {"label": "ForInStep", "kind": 22, "detail": "Type u → Type u"}, + {"label": "ForInStep", + "kind": 22, + "documentation": + {"value": "Auxiliary type used to compile `for x in xs` notation. ", + "kind": "markdown"}, + "detail": "Type u → Type u"}, {"label": "ForM", "kind": 7, + "documentation": + {"value": + "Typeclass for the polymorphic `forM` operation described in the \"do unchained\" paper.\nRemark:\n- `γ` is a \"container\" type of elements of type `α`.\n- `α` is treated as an output parameter by the typeclass resolution procedure.\n That is, it tries to find an instance using only `m` and `γ`.\n", + "kind": "markdown"}, "detail": "(Type u → Type v) → Type w₁ → outParam (Type w₂) → Type (max (max (max (u + 1) v) w₁) w₂)"}, {"label": "Function", "kind": 9, "detail": "namespace"}, diff --git a/tests/lean/interactive/completionAtPrint.lean.expected.out b/tests/lean/interactive/completionAtPrint.lean.expected.out index edf3bd6a25a1..48577fdddf38 100644 --- a/tests/lean/interactive/completionAtPrint.lean.expected.out +++ b/tests/lean/interactive/completionAtPrint.lean.expected.out @@ -8,7 +8,7 @@ "kind": 3, "documentation": {"value": - "Free compacted regions of imports. No live references to imported objects may exist at the time of invocation; in\n particular, `env` should be the last reference to any `Environment` derived from these imports. ", + "Free compacted regions of imports. No live references to imported objects may exist at the time of invocation; in\nparticular, `env` should be the last reference to any `Environment` derived from these imports. ", "kind": "markdown"}, "detail": "Lean.Environment → IO Unit"}], "isIncomplete": true} diff --git a/tests/lean/interactive/completionDocString.lean.expected.out b/tests/lean/interactive/completionDocString.lean.expected.out index 02fa3fdd2235..0514fc48fb41 100644 --- a/tests/lean/interactive/completionDocString.lean.expected.out +++ b/tests/lean/interactive/completionDocString.lean.expected.out @@ -4,7 +4,7 @@ [{"label": "insertAt", "kind": 3, "documentation": - {"value": "Insert element `a` at position `i`.\n Pre: `i < as.size` ", + {"value": "Insert element `a` at position `i`.\nPre: `i < as.size` ", "kind": "markdown"}, "detail": "Array α → Nat → α → Array α"}, {"label": "insertAtAux", diff --git a/tests/lean/interactive/highlight.lean.expected.out b/tests/lean/interactive/highlight.lean.expected.out index 10c86ad5a6c6..8feb7444c434 100644 --- a/tests/lean/interactive/highlight.lean.expected.out +++ b/tests/lean/interactive/highlight.lean.expected.out @@ -82,9 +82,6 @@ {"textDocument": {"uri": "file://highlight.lean"}, "position": {"line": 41, "character": 7}} [{"range": - {"start": {"line": 38, "character": 4}, "end": {"line": 38, "character": 5}}, - "kind": 1}, - {"range": {"start": {"line": 34, "character": 10}, "end": {"line": 34, "character": 11}}, "kind": 1}, @@ -94,6 +91,9 @@ {"range": {"start": {"line": 36, "character": 9}, "end": {"line": 36, "character": 10}}, "kind": 1}, + {"range": + {"start": {"line": 38, "character": 4}, "end": {"line": 38, "character": 5}}, + "kind": 1}, {"range": {"start": {"line": 38, "character": 9}, "end": {"line": 38, "character": 10}}, "kind": 1}, @@ -107,12 +107,12 @@ {"textDocument": {"uri": "file://highlight.lean"}, "position": {"line": 48, "character": 9}} [{"range": - {"start": {"line": 47, "character": 4}, "end": {"line": 47, "character": 5}}, - "kind": 1}, - {"range": {"start": {"line": 45, "character": 10}, "end": {"line": 45, "character": 11}}, "kind": 1}, + {"range": + {"start": {"line": 47, "character": 4}, "end": {"line": 47, "character": 5}}, + "kind": 1}, {"range": {"start": {"line": 48, "character": 9}, "end": {"line": 48, "character": 10}}, "kind": 1}] diff --git a/tests/lean/interactive/hover.lean b/tests/lean/interactive/hover.lean index 6e7f2b0c7d89..876fcb994b9f 100644 --- a/tests/lean/interactive/hover.lean +++ b/tests/lean/interactive/hover.lean @@ -26,7 +26,7 @@ example : True := by /-- My way better tactic -/ macro_rules - | `(tactic| mytac $[only]? $e) => `(apply $e) + | `(tactic| mytac $[only]? $e) => `(tactic| apply $e) example : True := by mytac only True.intro diff --git a/tests/lean/interactive/hover.lean.expected.out b/tests/lean/interactive/hover.lean.expected.out index 2d57d64fb0eb..0a9bd247418c 100644 --- a/tests/lean/interactive/hover.lean.expected.out +++ b/tests/lean/interactive/hover.lean.expected.out @@ -37,7 +37,7 @@ "position": {"line": 39, "character": 2}} {"range": {"start": {"line": 39, "character": 2}, "end": {"line": 39, "character": 23}}, - "contents": {"value": "My ultimate tactic ", "kind": "markdown"}} + "contents": {"value": "My way better tactic ", "kind": "markdown"}} {"textDocument": {"uri": "file://hover.lean"}, "position": {"line": 46, "character": 7}} {"range": diff --git a/tests/lean/linterUnusedVariables.lean b/tests/lean/linterUnusedVariables.lean index 794397d86e16..cd1575cf140e 100644 --- a/tests/lean/linterUnusedVariables.lean +++ b/tests/lean/linterUnusedVariables.lean @@ -205,6 +205,17 @@ opaque externConst (x : Nat) : Nat := let y := 3 5 + +macro "useArg " name:declId arg:ident : command => `(def $name ($arg : α) : α := $arg) +useArg usedMacroVariable a + +macro "doNotUseArg " name:declId arg:ident : command => `(def $name ($arg : α) : Nat := 3) +doNotUseArg unusedMacroVariable b + +macro "ignoreArg " id:declId sig:declSig : command => `(opaque $id $sig) +ignoreArg ignoredMacroVariable (x : UInt32) : UInt32 + + theorem not_eq_zero_of_lt (h : b < a) : a ≠ 0 := by -- *not* unused cases a exact absurd h (Nat.not_lt_zero _) diff --git a/tests/lean/linterUnusedVariables.lean.expected.out b/tests/lean/linterUnusedVariables.lean.expected.out index eedb04f23625..996a5be7b07a 100644 --- a/tests/lean/linterUnusedVariables.lean.expected.out +++ b/tests/lean/linterUnusedVariables.lean.expected.out @@ -12,8 +12,8 @@ linterUnusedVariables.lean:50:11-50:12: warning: unused variable `z` linterUnusedVariables.lean:55:14-55:15: warning: unused variable `y` linterUnusedVariables.lean:61:20-61:21: warning: unused variable `y` linterUnusedVariables.lean:66:34-66:38: warning: unused variable `inst` -linterUnusedVariables.lean:107:25-107:26: warning: unused variable `x` linterUnusedVariables.lean:108:6-108:7: warning: unused variable `y` +linterUnusedVariables.lean:107:25-107:26: warning: unused variable `x` linterUnusedVariables.lean:114:6-114:7: warning: unused variable `a` linterUnusedVariables.lean:124:26-124:27: warning: unused variable `z` linterUnusedVariables.lean:132:9-132:10: warning: unused variable `h` @@ -26,7 +26,8 @@ linterUnusedVariables.lean:191:19-191:20: warning: unused variable `x` linterUnusedVariables.lean:195:6-195:7: warning: unused variable `y` linterUnusedVariables.lean:200:6-200:7: warning: unused variable `y` linterUnusedVariables.lean:205:6-205:7: warning: unused variable `y` -linterUnusedVariables.lean:214:27-214:28: error: don't know how to synthesize placeholder +linterUnusedVariables.lean:213:32-213:33: warning: unused variable `b` +linterUnusedVariables.lean:225:27-225:28: error: don't know how to synthesize placeholder context: bar : ?m bar' : Nat → Nat @@ -35,10 +36,10 @@ bar' : Nat → Nat inst : ToString α a : Nat ⊢ Nat -linterUnusedVariables.lean:215:0-215:7: warning: declaration uses 'sorry' -linterUnusedVariables.lean:216:0-216:7: warning: declaration uses 'sorry' -linterUnusedVariables.lean:219:0: error: expected '{' or tactic -linterUnusedVariables.lean:217:27-217:29: error: unsolved goals +linterUnusedVariables.lean:226:0-226:7: warning: declaration uses 'sorry' +linterUnusedVariables.lean:227:0-227:7: warning: declaration uses 'sorry' +linterUnusedVariables.lean:230:0: error: expected '{' or tactic +linterUnusedVariables.lean:228:27-228:29: error: unsolved goals bar : ?m bar' : Nat → Nat α : Type ?u diff --git a/tests/lean/macroElabRulesIssue1.lean b/tests/lean/macroElabRulesIssue1.lean new file mode 100644 index 000000000000..f511da52e6fd --- /dev/null +++ b/tests/lean/macroElabRulesIssue1.lean @@ -0,0 +1,16 @@ +import Lean + +open Lean Elab Tactic + +syntax "Foo" (ident <|> num) : tactic + +elab_rules : tactic + | `(tactic| Foo $x:num) => + logInfo "num" + +macro_rules + | `(tactic| Foo $x:ident) => `(tactic| trace "ident") + +example : True := by + Foo x -- should not fail + trivial diff --git a/tests/lean/macroElabRulesIssue1.lean.expected.out b/tests/lean/macroElabRulesIssue1.lean.expected.out new file mode 100644 index 000000000000..08a89d1260b4 --- /dev/null +++ b/tests/lean/macroElabRulesIssue1.lean.expected.out @@ -0,0 +1 @@ +ident diff --git a/tests/lean/macroElabRulesIssue2.lean b/tests/lean/macroElabRulesIssue2.lean new file mode 100644 index 000000000000..640f98cda832 --- /dev/null +++ b/tests/lean/macroElabRulesIssue2.lean @@ -0,0 +1,22 @@ +import Lean +open Lean Elab + +declare_syntax_cat fixDecl +syntax ident : fixDecl +syntax ident "<" term : fixDecl + +syntax "Fix₁ " fixDecl : tactic + +elab_rules : tactic + | `(tactic| Fix₁ $x:ident) => logInfo "simple" + +elab_rules : tactic + | `(tactic| Fix₁ $x:ident < $bound:term) => + throwError "Failed at elab_rules" + +macro_rules +| `(ℕ) => `(Nat) + +example : ∀ b : ℕ, ∀ a : Nat, a ≥ 2 → a / a = 1 := by + Fix₁ b + Fix₁ a < 2 -- should produce `Failed at elab_rules` diff --git a/tests/lean/macroElabRulesIssue2.lean.expected.out b/tests/lean/macroElabRulesIssue2.lean.expected.out new file mode 100644 index 000000000000..aea0f1d1ca13 --- /dev/null +++ b/tests/lean/macroElabRulesIssue2.lean.expected.out @@ -0,0 +1,2 @@ +simple +macroElabRulesIssue2.lean:22:2-22:12: error: Failed at elab_rules diff --git a/tests/lean/nonfatalattrs.lean b/tests/lean/nonfatalattrs.lean new file mode 100644 index 000000000000..d5d2838f4fe7 --- /dev/null +++ b/tests/lean/nonfatalattrs.lean @@ -0,0 +1,13 @@ +-- Even if there are errors in the attributes, +-- the definition should still be declared. + +-- Attributes without implementation +syntax "unimplementedattr" : attr +@[unimplementedattr] def foo := 42 +#check foo + +-- Attributes that fail during application +def bar := + let rec @[class] bar : Nat := 42 + bar +#check bar diff --git a/tests/lean/nonfatalattrs.lean.expected.out b/tests/lean/nonfatalattrs.lean.expected.out new file mode 100644 index 000000000000..e30fbc8b60a6 --- /dev/null +++ b/tests/lean/nonfatalattrs.lean.expected.out @@ -0,0 +1,4 @@ +nonfatalattrs.lean:6:2-6:19: error: unknown attribute [attrUnimplementedattr] +foo : Nat +nonfatalattrs.lean:11:12-11:17: error: invalid 'class', declaration 'bar.bar' must be inductive datatype, structure, or constant +bar : Nat diff --git a/tests/lean/rewrite.lean b/tests/lean/rewrite.lean index d49f2b4bec34..446dae0ad429 100644 --- a/tests/lean/rewrite.lean +++ b/tests/lean/rewrite.lean @@ -14,7 +14,7 @@ done axiom zeroAdd (x : Nat) : 0 + x = x -theorem ex2 (x y z) (h₁ : 0 + x = y) (h₂ : 0 + y = z) : x = z := by +theorem ex2a (x y z) (h₁ : 0 + x = y) (h₂ : 0 + y = z) : x = z := by rewrite [zeroAdd] at h₁ h₂; trace_state; subst x; diff --git a/tests/lean/run/1200.lean b/tests/lean/run/1200.lean index ab113ce2bd7c..e04343c04850 100644 --- a/tests/lean/run/1200.lean +++ b/tests/lean/run/1200.lean @@ -1,5 +1,5 @@ example -(h: match .none (α:=α) with +(h: match none (α:=α) with | some _ => True | _ => True): True := by diff --git a/tests/lean/run/1299.lean b/tests/lean/run/1299.lean new file mode 100644 index 000000000000..ba37cc78a000 --- /dev/null +++ b/tests/lean/run/1299.lean @@ -0,0 +1,8 @@ +@[simp] theorem getElem_fin [GetElem Cont Nat Elem Dom] (a : Cont) (i : Fin n) (h : Dom a i) : + a[i] = a[i.1] := rfl + +example (a : Array α) (i : Fin a.size) : a[i] = a[i.1] := by + simp + +example (a : Array α) (i : Fin a.size) : a[i] = a[i.1] := by + rw [getElem_fin] diff --git a/tests/lean/run/1300.lean b/tests/lean/run/1300.lean new file mode 100644 index 000000000000..2072c6e8aa1c --- /dev/null +++ b/tests/lean/run/1300.lean @@ -0,0 +1,6 @@ +set_option trace.Meta.debug true + +example (hv : v < n) (ih: ∀ v : Fin n, ∃ v', v' ≤ v): + True := by + have ⟨w, hw⟩ := ih ⟨v, ‹_›⟩ + trivial diff --git a/tests/lean/run/1308.lean b/tests/lean/run/1308.lean new file mode 100644 index 000000000000..86f28e6f1850 --- /dev/null +++ b/tests/lean/run/1308.lean @@ -0,0 +1,2 @@ +@[defaultInstance high] instance : HPow R Nat R where hPow a _ := a +example (x y : Nat) : (x + y) ^ 3 = x ^ 3 + y ^ 3 + 3 * (x * y ^ 2 + x ^ 2 * y) := sorry diff --git a/tests/lean/run/1337.lean b/tests/lean/run/1337.lean new file mode 100644 index 000000000000..aa914ff820d5 --- /dev/null +++ b/tests/lean/run/1337.lean @@ -0,0 +1,14 @@ +theorem n_minus_one_le_n {n : Nat} : n > 0 → n - 1 < n := by + cases n with + | zero => simp [] + | succ n => + intros + rw [Nat.succ_eq_add_one, Nat.add_sub_cancel] + apply Nat.le.refl + +partial def foo : Array Int → Int + | arr => Id.run do + let mut r : Int := 1 + while h : arr.size > 0 do + r := r * arr[arr.size - 1]'(by apply n_minus_one_le_n h) + return r diff --git a/tests/lean/run/bigop.lean b/tests/lean/run/bigop.lean index 0ee92ab6f575..a317ff915f0c 100644 --- a/tests/lean/run/bigop.lean +++ b/tests/lean/run/bigop.lean @@ -1,18 +1,17 @@ -def Sequence (α : Type) := List α +abbrev Sequence (α : Type) := List α -def BigBody (β α) := α × (β → β → β) × Bool × β +def bigop (init : β) (seq : Sequence α) (op : β → β → β) (f : α → Bool × β) : β := Id.run do + let mut result := init + for a in seq do + let (ok, b) := f a + if ok then + result := op result b + return result -def applyBig {α β : Type} (body : BigBody β α) (x : β) : β := - let (_, op, b, v) := body; - if b then op v x else x +#eval bigop 0 [1, 2, 4] Add.add fun elem => (elem % 2 == 0, elem * 2) -def reducebig {α β : Type} (idx : β) (r : Sequence α) (body : α → BigBody β α) : β := - r.foldr (applyBig ∘ body) idx - -def bigop := @reducebig - -partial def iota : Nat → Nat → List Nat - | m, 0 => [] +def iota : Nat → Nat → List Nat + | _, 0 => [] | m, n+1 => m :: iota (m+1) n def index_iota (m n : Nat) := iota m (n - m) @@ -23,18 +22,20 @@ class Enumerable (α : Type) where instance : Enumerable Bool where elems := [false, true] --- instance {α β} [Enumerable α] [Enumerable β]: Enumerable (α × β) := --- { elems := do let a ← Enumerable.elems α; let b ← Enumerable.elems β; pure (a, b) } - -partial def finElemsAux (n : Nat) : (i : Nat) → i < n → List (Fin n) - | 0, h => [⟨0, h⟩] - | i+1, h => ⟨i+1, h⟩ :: finElemsAux n i (Nat.lt_of_succ_lt h) +instance {α β} [Enumerable α] [Enumerable β]: Enumerable (α × β) where + elems := Enumerable.elems.bind fun (a : α) => Enumerable.elems.bind fun (b : β) => [(a, b)] -partial def finElems : (n : Nat) → List (Fin n) - | 0 => [] - | (n+1) => finElemsAux (n+1) n (Nat.lt_succ_self n) +def finElems (n : Nat) : List (Fin n) := + match n with + | 0 => [] + | n+1 => go (n+1) n (by simp_arith) +where + go (n : Nat) (i : Nat) (h : i < n) : List (Fin n) := + match i with + | 0 => [⟨0, h⟩] + | i+1 => ⟨i+1, h⟩ :: go n i (Nat.lt_of_succ_lt h) -instance {n} : Enumerable (Fin n) where +instance : Enumerable (Fin n) where elems := (finElems n).reverse instance : OfNat (Fin (Nat.succ n)) m := @@ -49,30 +50,30 @@ syntax ident "<-" term "|" term : index -- Primitive notation for big operators syntax "_big" "[" term "," term "]" "(" index ")" term : term --- We define how to expand `_bigop` with the different kinds of index +-- We define how to expand `_big` with the different kinds of index macro_rules -| `(_big [$op, $idx] ($i:ident <- $r | $p) $F) => `(bigop $idx $r (fun $i:ident => ($i:ident, $op, $p, $F))) -| `(_big [$op, $idx] ($i:ident <- $r) $F) => `(bigop $idx $r (fun $i:ident => ($i:ident, $op, true, $F))) -| `(_big [$op, $idx] ($lower:term ≤ $i:ident < $upper) $F) => `(bigop $idx (index_iota $lower $upper) (fun $i:ident => ($i:ident, $op, true, $F))) -| `(_big [$op, $idx] ($lower:term ≤ $i:ident < $upper | $p) $F) => `(bigop $idx (index_iota $lower $upper) (fun $i:ident => ($i:ident, $op, $p, $F))) +| `(_big [$op, $idx] ($i:ident <- $r | $p) $F) => `(bigop $idx $r $op (fun $i:ident => ($p, $F))) +| `(_big [$op, $idx] ($i:ident <- $r) $F) => `(bigop $idx $r $op (fun $i:ident => (true, $F))) +| `(_big [$op, $idx] ($lower:term ≤ $i:ident < $upper) $F) => `(bigop $idx (index_iota $lower $upper) $op (fun $i:ident => (true, $F))) +| `(_big [$op, $idx] ($lower:term ≤ $i:ident < $upper | $p) $F) => `(bigop $idx (index_iota $lower $upper) $op (fun $i:ident => ($p, $F))) --- Define `Sum` -syntax "Sum" "(" index ")" term : term -macro_rules | `(Sum ($idx) $F) => `(_big [Add.add, 0] ($idx) $F) +-- Define `∑ ` +syntax "∑ " "(" index ")" term : term +macro_rules | `(∑ ($idx) $F) => `(_big [Add.add, 0] ($idx) $F) -- We can already use `Sum` with the different kinds of index. -#check Sum (i <- [0, 2, 4] | i != 2) i -#check Sum (10 ≤ i < 20 | i != 5) i+1 -#check Sum (10 ≤ i < 20) i+1 +#check ∑ (i <- [0, 2, 4] | i != 2) i +#check ∑ (10 ≤ i < 20 | i != 5) i+1 +#check ∑ (10 ≤ i < 20) i+1 --- Define `Prod` -syntax "Prod" "(" index ")" term : term -macro_rules | `(Prod ($idx) $F) => `(_big [Mul.mul, 1] ($idx) $F) +-- Define `∏` +syntax "∏" "(" index ")" term : term +macro_rules | `(∏ ($idx) $F) => `(_big [Mul.mul, 1] ($idx) $F) -- The examples above now also work for `Prod` -#check Prod (i <- [0, 2, 4] | i != 2) i -#check Prod (10 ≤ i < 20 | i != 5) i+1 -#check Prod (10 ≤ i < 20) i+1 +#check ∏ (i <- [0, 2, 4] | i != 2) i +#check ∏ (10 ≤ i < 20 | i != 5) i+1 +#check ∏ (10 ≤ i < 20) i+1 -- We can extend our grammar for the syntax category `index`. syntax ident "|" term : index @@ -80,24 +81,24 @@ syntax ident ":" term : index syntax ident ":" term "|" term : index -- And new rules macro_rules -| `(_big [$op, $idx] ($i:ident : $type) $F) => `(bigop $idx (Enumerable.elems (α := $type)) (fun $i:ident => ($i:ident, $op, true, $F))) -| `(_big [$op, $idx] ($i:ident : $type | $p) $F) => `(bigop $idx (Enumerable.elems (α := $type)) (fun $i:ident => ($i:ident, $op, $p, $F))) -| `(_big [$op, $idx] ($i:ident | $p) $F) => `(bigop $idx (Enumerable.elems) (fun $i:ident => ($i:ident, $op, $p, $F))) +| `(_big [$op, $idx] ($i:ident : $type) $F) => `(bigop $idx (Enumerable.elems (α := $type)) $op (fun $i:ident => (true, $F))) +| `(_big [$op, $idx] ($i:ident : $type | $p) $F) => `(bigop $idx (Enumerable.elems (α := $type)) $op (fun $i:ident => ($p, $F))) +| `(_big [$op, $idx] ($i:ident | $p) $F) => `(bigop $idx (Enumerable.elems) $op (fun $i:ident => ($p, $F))) -- The new syntax is immediately available for all big operators that we have defined def myPred (x : Fin 10) : Bool := true -#check Sum (i : Fin 10) i+1 -#check Sum (i : Fin 10 | i != 2) i+1 -#check Sum (i | myPred i) i+i -#check Prod (i : Fin 10) i+1 -#check Prod (i : Fin 10 | i != 2) i+1 -#check Prod (i | myPred i) i+i +#check ∑ (i : Fin 10) i+1 +#check ∑ (i : Fin 10 | i != 2) i+1 +#check ∑ (i | myPred i) i+i +#check ∏ (i : Fin 10) i+1 +#check ∏ (i : Fin 10 | i != 2) i+1 +#check ∏ (i | myPred i) i+i -- We can easily create alternative syntax for any big operator. -syntax "Σ" index "=>" term : term -macro_rules | `(Σ $idx => $F) => `(Prod ($idx) $F) +syntax "Summation" index "=>" term : term +macro_rules | `(Summation $idx => $F) => `(∑ ($idx) $F) -#check Σ 10 ≤ i < 20 => i+1 +#check Summation 10 ≤ i < 20 => i+1 -- Now, we create command for automating the generation of big operators. syntax "def_bigop" str term:max term:max : command diff --git a/tests/lean/run/derivingRpcEncoding.lean b/tests/lean/run/derivingRpcEncoding.lean deleted file mode 100644 index 7708b1347fba..000000000000 --- a/tests/lean/run/derivingRpcEncoding.lean +++ /dev/null @@ -1,55 +0,0 @@ -import Lean.Server.Rpc.Basic - -open Lean Server - -@[reducible] -def rpcPacketFor (α : Type) {β : outParam Type} [RpcEncoding α β] := β - -structure FooRef where - a : Array Nat - deriving RpcEncoding with { withRef := true } - -#synth FromJson (rpcPacketFor (WithRpcRef FooRef)) -#synth ToJson (rpcPacketFor (WithRpcRef FooRef)) - -structure FooJson where - s : String - deriving FromJson, ToJson - -structure Bar where - fooRef : WithRpcRef FooRef - fooJson : FooJson - deriving RpcEncoding - -#synth FromJson (rpcPacketFor Bar) -#synth ToJson (rpcPacketFor Bar) - -structure BarTrans where - bar : Bar - deriving RpcEncoding - -#synth FromJson (rpcPacketFor BarTrans) -#synth ToJson (rpcPacketFor BarTrans) - -structure Baz where - arr : Array String -- non-constant field - deriving RpcEncoding - -#synth FromJson (rpcPacketFor Baz) -#synth ToJson (rpcPacketFor Baz) - -structure FooGeneric (α : Type) where - a : α - b? : Option α - deriving RpcEncoding - -#synth FromJson (rpcPacketFor <| FooGeneric Nat) -#synth ToJson (rpcPacketFor <| FooGeneric Nat) - -inductive FooInductive (α : Type) where - | a : α → Bar → FooInductive α - | b : (n : Nat) → (a : α) → Nat → FooInductive α - deriving RpcEncoding - -#synth FromJson (rpcPacketFor <| FooInductive Nat) -#synth ToJson (rpcPacketFor <| FooInductive Nat) diff --git a/tests/lean/run/foApprox.lean b/tests/lean/run/foApprox.lean new file mode 100644 index 000000000000..475d409be270 --- /dev/null +++ b/tests/lean/run/foApprox.lean @@ -0,0 +1,12 @@ +def f : Prop → Prop := id + +class Foo (foo : Prop → Prop) where + l : x → foo x + +instance : Foo f where + l := by simp_all [f] + +theorem test' (h : x = True) : f x := by + have _ := True + apply Foo.l -- `?foo ?x =?= [mdata noImplicitLambda:1 f x]` + simp [h] diff --git a/tests/lean/run/parserQuot.lean b/tests/lean/run/parserQuot.lean new file mode 100644 index 000000000000..aec5306fdf4c --- /dev/null +++ b/tests/lean/run/parserQuot.lean @@ -0,0 +1,6 @@ +syntax blockingConsts := "blocking" "[" ident,* "]" +macro "specialize_def" i:ident "[" ts:term,* "]" block:blockingConsts : tactic => do + /- expected 'blocking' -/ + if let `(blockingConsts|blocking [ $is:ident,* ]) := block then + sorry + sorry diff --git a/tests/lean/run/unifhint1.lean b/tests/lean/run/unifhint1.lean index 5cad7fcd436f..9e0c05917e0e 100644 --- a/tests/lean/run/unifhint1.lean +++ b/tests/lean/run/unifhint1.lean @@ -16,6 +16,7 @@ instance : CoeSort Magma.{u} (Type u) where def mul {s : Magma} (a b : s) : s := s.mul a b +/-- hi -/ unif_hint (s : Magma) where s =?= Nat.Magma |- s.α =?= Nat diff --git a/tests/lean/run/unsafeInit.lean b/tests/lean/run/unsafeInit.lean new file mode 100644 index 000000000000..56e8afa9753a --- /dev/null +++ b/tests/lean/run/unsafeInit.lean @@ -0,0 +1 @@ +unsafe initialize no : Nat ← pure lcUnreachable diff --git a/tests/lean/scopedInstanceOutsideNamespace.lean.expected.out b/tests/lean/scopedInstanceOutsideNamespace.lean.expected.out index e57e2296884f..4329447b0f88 100644 --- a/tests/lean/scopedInstanceOutsideNamespace.lean.expected.out +++ b/tests/lean/scopedInstanceOutsideNamespace.lean.expected.out @@ -1,4 +1,4 @@ scopedInstanceOutsideNamespace.lean:1:0-2:38: error: scoped attributes must be used inside namespaces "true" scopedInstanceOutsideNamespace.lean:6:0-6:30: error: scoped attributes must be used inside namespaces -scopedInstanceOutsideNamespace.lean:8:0-10:38: error: scoped attributes must be used inside namespaces +scopedInstanceOutsideNamespace.lean:8:2-8:17: error: scoped attributes must be used inside namespaces diff --git a/tests/lean/scopedMacros.lean.expected.out b/tests/lean/scopedMacros.lean.expected.out index 08d8154d9ed1..fa4f357b33a5 100644 --- a/tests/lean/scopedMacros.lean.expected.out +++ b/tests/lean/scopedMacros.lean.expected.out @@ -1,7 +1,7 @@ 10 + 1 : Nat scopedMacros.lean:11:7-11:11: error: unknown identifier 'foo!' 10 + 1 : Nat -scopedMacros.lean:19:0-19:50: error: scoped attributes must be used inside namespaces +scopedMacros.lean:19:0-19:37: error: scoped attributes must be used inside namespaces scopedMacros.lean:19:7-19:50: error: invalid syntax node kind 'termBla!_' scopedMacros.lean:29:7-29:11: error: unknown identifier 'bla!' scopedMacros.lean:36:0-36:45: error: scoped attributes must be used inside namespaces diff --git a/tests/lean/typeMismatch.lean b/tests/lean/typeMismatch.lean index a8e9bdd5393d..0f34c2031586 100644 --- a/tests/lean/typeMismatch.lean +++ b/tests/lean/typeMismatch.lean @@ -8,5 +8,5 @@ IO.println "" open Lean -def test (x : Expr) : MetaM Unit := +def test2 (x : Expr) : MetaM Unit := Meta.isDefEq x x diff --git a/tests/lean/unifHintAndTC.lean b/tests/lean/unifHintAndTC.lean index 814102cd7dfa..578e3abb6087 100644 --- a/tests/lean/unifHintAndTC.lean +++ b/tests/lean/unifHintAndTC.lean @@ -1,37 +1,38 @@ -structure Magma.{u} where - α : Type u - mul : α → α → α +structure Magma where + carrier : Type u + mul : carrier → carrier → carrier -instance : CoeSort Magma.{u} (Type u) where - coe m := m.α +instance : CoeSort Magma (Type u) where + coe m := m.carrier def mul {s : Magma} (a b : s) : s := s.mul a b -infixl:70 (priority := high) "*" => mul +infixl:70 (priority := high) " * " => mul + +example {S : Magma} (a b c : S) : b = c → a * b = a * c := by + intro h; rw [h] def Nat.Magma : Magma where - α := Nat + carrier := Nat mul a b := Nat.mul a b -def Prod.Magma (m : Magma.{u}) (n : Magma.{v}) : Magma where - α := m.α × n.α - mul a b := (a.1 * b.1, a.2 * b.2) - unif_hint (s : Magma) where - s =?= Nat.Magma |- s.α =?= Nat + s =?= Nat.Magma |- s.carrier =?= Nat + +example (x : Nat) : Nat := + x * x + +def Prod.Magma (m : Magma) (n : Magma) : Magma where + carrier := m.carrier × n.carrier + mul a b := (a.1 * b.1, a.2 * b.2) unif_hint (s : Magma) (m : Magma) (n : Magma) (β : Type u) (δ : Type v) where - m.α =?= β - n.α =?= δ + m.carrier =?= β + n.carrier =?= δ s =?= Prod.Magma m n |- - s.α =?= β × δ - -def f1 (x : Nat) : Nat := - x * x - -#eval f1 10 + s.carrier =?= β × δ def f2 (x y : Nat) : Nat × Nat := (x, y) * (x, y) @@ -44,13 +45,13 @@ def f3 (x y : Nat) : Nat × Nat × Nat := #eval f3 7 24 def magmaOfMul (α : Type u) [Mul α] : Magma where -- Bridge between `Mul α` and `Magma` - α := α + carrier := α mul a b := Mul.mul a b unif_hint (s : Magma) (α : Type u) [Mul α] where s =?= magmaOfMul α |- - s.α =?= α + s.carrier =?= α def g (x y : Int) : Int := x * y -- Note that we don't have a hint connecting Magma's carrier and Int diff --git a/tests/lean/unifHintAndTC.lean.expected.out b/tests/lean/unifHintAndTC.lean.expected.out index 81382ea1dd9e..d52e94aefbfc 100644 --- a/tests/lean/unifHintAndTC.lean.expected.out +++ b/tests/lean/unifHintAndTC.lean.expected.out @@ -1,4 +1,3 @@ -100 (100, 400) (49, 576, 576) def g : Int → Int → Int := diff --git a/tests/lean/updateExprIssue.lean.expected.out b/tests/lean/updateExprIssue.lean.expected.out index c15dbe0275b9..10537d1e321f 100644 --- a/tests/lean/updateExprIssue.lean.expected.out +++ b/tests/lean/updateExprIssue.lean.expected.out @@ -13,9 +13,24 @@ def sefFn (x_1 : obj) (x_2 : obj) : obj := Lean.Expr.const._impl → ret x_1 Lean.Expr.app._impl → - let x_3 : obj := proj[1] x_1; - let x_4 : obj := Lean.Expr.updateApp x_1 x_2 x_3 ◾; - ret x_4 + let x_3 : obj := proj[0] x_1; + let x_4 : obj := proj[1] x_1; + let x_5 : usize := ptrAddrUnsafe ◾ x_3; + let x_6 : usize := ptrAddrUnsafe ◾ x_2; + let x_7 : u8 := USize.decEq x_5 x_6; + case x_7 : obj of + Bool.false → + let x_8 : obj := Lean.Expr.app._override x_2 x_4; + ret x_8 + Bool.true → + let x_9 : usize := ptrAddrUnsafe ◾ x_4; + let x_10 : u8 := USize.decEq x_9 x_9; + case x_10 : obj of + Bool.false → + let x_11 : obj := Lean.Expr.app._override x_2 x_4; + ret x_11 + Bool.true → + ret x_1 Lean.Expr.lam._impl → ret x_1 Lean.Expr.forallE._impl → diff --git a/tests/pkg/user_attr/UserAttr/BlaAttr.lean b/tests/pkg/user_attr/UserAttr/BlaAttr.lean index e6d9b1df4dfa..d4a57f5a60db 100644 --- a/tests/pkg/user_attr/UserAttr/BlaAttr.lean +++ b/tests/pkg/user_attr/UserAttr/BlaAttr.lean @@ -5,3 +5,18 @@ open Lean initialize blaAttr : TagAttribute ← registerTagAttribute `bla "simple user defined attribute" register_simp_attr my_simp "my own simp attribute" + +syntax (name := foo) "foo" num "important"? : attr + +initialize fooAttr : ParametricAttribute (Nat × Bool) ← + registerParametricAttribute { + name := `foo + descr := "parametric attribute containing a priority and flag" + getParam := fun _ stx => + match stx with + | `(attr| foo $prio:num $[important%$imp]?) => + return (prio.getNat, imp.isSome) + | _ => throwError "unexpected foo attribute" + afterSet := fun declName _ => do + IO.println s!"set attribute [foo] at {declName}" + } diff --git a/tests/pkg/user_attr/UserAttr/Tst.lean b/tests/pkg/user_attr/UserAttr/Tst.lean index 1a08e5f33331..cb8ce3849c91 100644 --- a/tests/pkg/user_attr/UserAttr/Tst.lean +++ b/tests/pkg/user_attr/UserAttr/Tst.lean @@ -4,6 +4,24 @@ import UserAttr.BlaAttr @[bla] def f (x : Nat) := x + 2 @[bla] def g (x : Nat) := x + 1 +@[foo 10] def h1 (x : Nat) := 2*x + 1 +@[foo 20 important] def h2 (x : Nat) := 2*x + 1 + +open Lean in +def hasBlaAttr (declName : Name) : CoreM Bool := + return blaAttr.hasTag (← getEnv) declName + +#eval hasBlaAttr ``f +#eval hasBlaAttr ``id + +open Lean in +def getFooAttrInfo? (declName : Name) : CoreM (Option (Nat × Bool)) := + return fooAttr.getParam (← getEnv) declName + +#eval getFooAttrInfo? ``f +#eval getFooAttrInfo? ``h1 +#eval getFooAttrInfo? ``h2 + @[my_simp] theorem f_eq : f x = x + 2 := rfl @[my_simp] theorem g_eq : g x = x + 1 := rfl @@ -23,13 +41,12 @@ macro "my_simp" : tactic => `(simp [my_simp]) example : f x = id (x + 2) := by my_simp - @[simp low, my_simp low] -theorem expand_mul_add (x y z : Nat) : x * (y + z) = x * y + x * y := sorry +axiom expand_mul_add (x y z : Nat) : x * (y + z) = x * y + x * y @[simp high, my_simp high] -theorem expand_add_mul (x y z : Nat) : (x + y) * z = x * z + y * z := sorry +axiom expand_add_mul (x y z : Nat) : (x + y) * z = x * z + y * z @[simp, my_simp] -theorem lassoc_add (x y z : Nat) : x + (y + z) = x + y + z := sorry +axiom lassoc_add (x y z : Nat) : x + (y + z) = x + y + z set_option trace.Meta.Tactic.simp.rewrite true @@ -39,12 +56,22 @@ theorem ex1 (x : Nat) : (x + x) * (x + x) = x * x + x * x + x * x + x * x := by -- Rewrites: expand_add_mul -> expand_mul_add -> lassoc_add theorem ex2 (x : Nat) : (x + x) * (x + x) = x * x + x * x + x * x + x * x := by simp -open Lean -open Lean.Meta +open Lean Meta in def checkProofs : MetaM Unit := do - let ConstantInfo.thmInfo info1 ← getConstInfo `ex1 | throwError "unexpected" - let ConstantInfo.thmInfo info2 ← getConstInfo `ex2 | throwError "unexpected" + let .thmInfo info1 ← getConstInfo `ex1 | throwError "unexpected" + let .thmInfo info2 ← getConstInfo `ex2 | throwError "unexpected" unless info1.value == info2.value do throwError "unexpected values" #eval checkProofs + +open Lean Meta in +def showThmsOf (simpAttrName : Name) : MetaM Unit := do + let some simpExt ← getSimpExtension? simpAttrName + | throwError "`{simpAttrName}` is not a simp attribute" + let thms ← simpExt.getTheorems + let thmNames := thms.lemmaNames.fold (init := #[]) fun acc lemmaName => acc.push lemmaName + for thmName in thmNames do + IO.println thmName + +#eval showThmsOf `my_simp